From 4674f4e3de12c604357c58e41aea85b91f5fde3c Mon Sep 17 00:00:00 2001 From: =?UTF-8?q?Henrik=20B=C3=B6ving?= Date: Wed, 15 Jan 2025 13:44:33 +0100 Subject: [PATCH 1/3] feat: add the int_toBitVec simpset --- src/Lean/Elab/Tactic/BVDecide/Frontend/Attr.lean | 3 +++ 1 file changed, 3 insertions(+) diff --git a/src/Lean/Elab/Tactic/BVDecide/Frontend/Attr.lean b/src/Lean/Elab/Tactic/BVDecide/Frontend/Attr.lean index bfca67675de2..dd88e69d9771 100644 --- a/src/Lean/Elab/Tactic/BVDecide/Frontend/Attr.lean +++ b/src/Lean/Elab/Tactic/BVDecide/Frontend/Attr.lean @@ -38,6 +38,9 @@ declare_config_elab elabBVDecideConfig Lean.Elab.Tactic.BVDecide.Frontend.BVDeci builtin_initialize bvNormalizeExt : Meta.SimpExtension ← Meta.registerSimpAttr `bv_normalize "simp theorems used by bv_normalize" +builtin_initialize intToBitVecExt : Meta.SimpExtension ← + Meta.registerSimpAttr `int_toBitVec "simp theorems used to convert UIntX/IntX statements into BitVec ones" + /-- Builtin `bv_normalize` simprocs. -/ builtin_initialize builtinBVNormalizeSimprocsRef : IO.Ref Meta.Simp.Simprocs ← IO.mkRef {} From 0361f83207de68736de3c1a9d32939df0d9972f6 Mon Sep 17 00:00:00 2001 From: =?UTF-8?q?Henrik=20B=C3=B6ving?= Date: Wed, 15 Jan 2025 13:44:45 +0100 Subject: [PATCH 2/3] chore: update stage0 --- stage0/src/runtime/CMakeLists.txt | 3 +- stage0/src/runtime/init_module.cpp | 2 + stage0/src/runtime/libuv.cpp | 19 +- stage0/src/runtime/libuv.h | 22 +- stage0/src/runtime/object.h | 5 + stage0/src/runtime/uv/event_loop.cpp | 143 + stage0/src/runtime/uv/event_loop.h | 47 + stage0/src/runtime/uv/timer.cpp | 254 + stage0/src/runtime/uv/timer.h | 54 + stage0/src/util/shell.cpp | 14 + stage0/stdlib/Init/Data/Array/Basic.c | 209 +- stage0/stdlib/Init/Data/BitVec/Lemmas.c | 6 +- stage0/stdlib/Init/Data/UInt/Bitwise.c | 2225 +- stage0/stdlib/Init/Data/Vector/Basic.c | 547 +- stage0/stdlib/Init/Data/Vector/Lemmas.c | 6 +- stage0/stdlib/Init/Grind.c | 6 +- stage0/stdlib/Init/Grind/Offset.c | 1318 +- stage0/stdlib/Init/Grind/PP.c | 363 + stage0/stdlib/Lake/Build/Actions.c | 802 +- stage0/stdlib/Lake/Build/Common.c | 1337 +- stage0/stdlib/Lake/Build/Job.c | 425 +- stage0/stdlib/Lake/Build/Module.c | 402 +- stage0/stdlib/Lake/CLI/Build.c | 1539 +- stage0/stdlib/Lake/Load/Lean/Elab.c | 4 +- stage0/stdlib/Lake/Load/Toml.c | 30220 +++++++++------- stage0/stdlib/Lake/Toml/Decode.c | 2187 +- stage0/stdlib/Lean/AddDecl.c | 49 - stage0/stdlib/Lean/BuiltinDocAttr.c | 30 +- stage0/stdlib/Lean/Compiler/IR/Basic.c | 2 +- stage0/stdlib/Lean/Compiler/InitAttr.c | 796 +- stage0/stdlib/Lean/Compiler/LCNF/MonoTypes.c | 18 +- stage0/stdlib/Lean/Compiler/Old.c | 33 - stage0/stdlib/Lean/CoreM.c | 23 +- stage0/stdlib/Lean/Data/AssocList.c | 44 +- stage0/stdlib/Lean/Elab/App.c | 7085 ++-- stage0/stdlib/Lean/Elab/Import.c | 253 +- .../Lean/Elab/Tactic/BVDecide/Frontend/Attr.c | 349 +- .../Elab/Tactic/BVDecide/Frontend/BVCheck.c | 8 +- .../Elab/Tactic/BVDecide/Frontend/BVDecide.c | 6 +- .../Elab/Tactic/BVDecide/Frontend/BVTrace.c | 6 +- .../Elab/Tactic/BVDecide/Frontend/Normalize.c | 19944 +--------- .../Tactic/BVDecide/Frontend/Normalize/AC.c | 548 + .../BVDecide/Frontend/Normalize/AndFlatten.c | 2797 ++ .../BVDecide/Frontend/Normalize/Basic.c | 5175 +++ .../Frontend/Normalize/EmbeddedConstraint.c | 1895 + .../BVDecide/Frontend/Normalize/Rewrite.c | 3691 ++ .../BVDecide/Frontend/Normalize/Simproc.c | 11406 ++++++ stage0/stdlib/Lean/Elab/Tactic/Grind.c | 215 +- stage0/stdlib/Lean/Elab/Tactic/Simproc.c | 4 - stage0/stdlib/Lean/Elab/Term.c | 6 +- stage0/stdlib/Lean/Elab/Util.c | 4 +- stage0/stdlib/Lean/KeyedDeclsAttribute.c | 2 + stage0/stdlib/Lean/Linter/MissingDocs.c | 6 - stage0/stdlib/Lean/Linter/UnusedVariables.c | 12 +- stage0/stdlib/Lean/Meta/AppBuilder.c | 662 +- stage0/stdlib/Lean/Meta/Basic.c | 488 +- stage0/stdlib/Lean/Meta/Tactic/Grind.c | 824 +- stage0/stdlib/Lean/Meta/Tactic/Grind/Arith.c | 41 + .../Meta/Tactic/Grind/Arith/Internalize.c | 39 + .../stdlib/Lean/Meta/Tactic/Grind/Arith/Inv.c | 39 + .../Lean/Meta/Tactic/Grind/Arith/Main.c | 913 + .../Lean/Meta/Tactic/Grind/Arith/Model.c | 1702 + .../Lean/Meta/Tactic/Grind/Arith/Offset.c | 19994 ++++++++++ .../Lean/Meta/Tactic/Grind/Arith/ProofUtil.c | 2733 ++ .../Lean/Meta/Tactic/Grind/Arith/Types.c | 509 + .../Lean/Meta/Tactic/Grind/Arith/Util.c | 1736 + stage0/stdlib/Lean/Meta/Tactic/Grind/Canon.c | 2 +- .../Lean/Meta/Tactic/Grind/Combinators.c | 2 +- stage0/stdlib/Lean/Meta/Tactic/Grind/Core.c | 15134 ++++---- stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c | 3768 +- .../Lean/Meta/Tactic/Grind/EMatchTheorem.c | 1074 +- .../stdlib/Lean/Meta/Tactic/Grind/ENodeKey.c | 138 + .../Lean/Meta/Tactic/Grind/ForallProp.c | 1446 +- .../Lean/Meta/Tactic/Grind/Internalize.c | 10297 +++--- stage0/stdlib/Lean/Meta/Tactic/Grind/Intro.c | 6929 ++-- stage0/stdlib/Lean/Meta/Tactic/Grind/Inv.c | 1466 +- stage0/stdlib/Lean/Meta/Tactic/Grind/Main.c | 1231 +- stage0/stdlib/Lean/Meta/Tactic/Grind/PP.c | 6547 +++- stage0/stdlib/Lean/Meta/Tactic/Grind/Proj.c | 195 +- stage0/stdlib/Lean/Meta/Tactic/Grind/Proof.c | 3340 +- .../stdlib/Lean/Meta/Tactic/Grind/Propagate.c | 964 +- .../Lean/Meta/Tactic/Grind/PropagatorAttr.c | 2 - stage0/stdlib/Lean/Meta/Tactic/Grind/Simp.c | 2190 +- stage0/stdlib/Lean/Meta/Tactic/Grind/Split.c | 6616 ++-- stage0/stdlib/Lean/Meta/Tactic/Grind/Types.c | 9527 +++-- .../Lean/Meta/Tactic/LinearArith/Nat/Simp.c | 1123 +- stage0/stdlib/Lean/Meta/Tactic/Simp/Simproc.c | 30 +- stage0/stdlib/Lean/Parser/Extension.c | 39 +- stage0/stdlib/Lean/ParserCompiler.c | 18355 ++++++---- stage0/stdlib/Lean/Server/CodeActions/Attr.c | 17 - stage0/stdlib/Lean/Server/CodeActions/Basic.c | 16 +- stage0/stdlib/Lean/Server/Completion.c | 2064 +- .../Completion/CompletionInfoSelection.c | 1310 +- .../Lean/Server/FileWorker/RequestHandling.c | 909 +- .../Lean/Server/FileWorker/WidgetRequests.c | 14 +- stage0/stdlib/Lean/Server/Watchdog.c | 1793 +- stage0/stdlib/Lean/Util/Path.c | 139 + stage0/stdlib/Lean/Util/Profiler.c | 1203 +- .../Lean/Widget/InteractiveDiagnostic.c | 932 +- stage0/stdlib/Lean/Widget/UserWidget.c | 21 +- stage0/stdlib/Std/Data/DHashMap/Basic.c | 1250 +- .../Data/DHashMap/Internal/AssocList/Basic.c | 486 + .../Data/DHashMap/Internal/AssocList/Lemmas.c | 112 +- .../stdlib/Std/Data/DHashMap/Internal/Defs.c | 610 + .../Data/DHashMap/Internal/List/Associative.c | 236 + .../stdlib/Std/Data/DHashMap/Internal/Model.c | 1095 +- .../Std/Data/DHashMap/Internal/RawLemmas.c | 10 +- stage0/stdlib/Std/Data/DHashMap/Internal/WF.c | 90 + stage0/stdlib/Std/Data/HashMap/Basic.c | 3282 +- stage0/stdlib/Std/Internal.c | 10 +- stage0/stdlib/Std/Internal/Async.c | 33 + stage0/stdlib/Std/Internal/Async/Basic.c | 704 + stage0/stdlib/Std/Internal/Async/Timer.c | 909 + stage0/stdlib/Std/Internal/UV.c | 108 + .../stdlib/Std/Time/DateTime/PlainDateTime.c | 316 +- stage0/stdlib/Std/Time/DateTime/Timestamp.c | 251 +- stage0/stdlib/Std/Time/Format.c | 138 +- stage0/stdlib/Std/Time/Format/Basic.c | 2011 +- stage0/stdlib/Std/Time/Notation.c | 751 +- stage0/stdlib/Std/Time/Time/PlainTime.c | 1046 +- stage0/stdlib/Std/Time/Zoned/Database/TZdb.c | 218 +- stage0/stdlib/Std/Time/Zoned/DateTime.c | 32 +- stage0/stdlib/Std/Time/Zoned/ZonedDateTime.c | 42 +- 123 files changed, 148877 insertions(+), 89942 deletions(-) create mode 100644 stage0/src/runtime/uv/event_loop.cpp create mode 100644 stage0/src/runtime/uv/event_loop.h create mode 100644 stage0/src/runtime/uv/timer.cpp create mode 100644 stage0/src/runtime/uv/timer.h create mode 100644 stage0/stdlib/Init/Grind/PP.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AC.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AndFlatten.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Basic.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/EmbeddedConstraint.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Rewrite.c create mode 100644 stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Simproc.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Internalize.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Inv.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Main.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Model.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Offset.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/ProofUtil.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Types.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Util.c create mode 100644 stage0/stdlib/Lean/Meta/Tactic/Grind/ENodeKey.c create mode 100644 stage0/stdlib/Std/Internal/Async.c create mode 100644 stage0/stdlib/Std/Internal/Async/Basic.c create mode 100644 stage0/stdlib/Std/Internal/Async/Timer.c create mode 100644 stage0/stdlib/Std/Internal/UV.c diff --git a/stage0/src/runtime/CMakeLists.txt b/stage0/src/runtime/CMakeLists.txt index d6d8b50b395d..fc1e41f41693 100644 --- a/stage0/src/runtime/CMakeLists.txt +++ b/stage0/src/runtime/CMakeLists.txt @@ -2,7 +2,8 @@ set(RUNTIME_OBJS debug.cpp thread.cpp mpz.cpp utf8.cpp object.cpp apply.cpp exception.cpp interrupt.cpp memory.cpp stackinfo.cpp compact.cpp init_module.cpp load_dynlib.cpp io.cpp hash.cpp platform.cpp alloc.cpp allocprof.cpp sharecommon.cpp stack_overflow.cpp -process.cpp object_ref.cpp mpn.cpp mutex.cpp libuv.cpp uv/net_addr.cpp) +process.cpp object_ref.cpp mpn.cpp mutex.cpp libuv.cpp uv/net_addr.cpp uv/event_loop.cpp +uv/timer.cpp) add_library(leanrt_initial-exec STATIC ${RUNTIME_OBJS}) set_target_properties(leanrt_initial-exec PROPERTIES ARCHIVE_OUTPUT_DIRECTORY ${CMAKE_CURRENT_BINARY_DIR}) diff --git a/stage0/src/runtime/init_module.cpp b/stage0/src/runtime/init_module.cpp index 8bf949d8bd5d..9ae9afb76390 100644 --- a/stage0/src/runtime/init_module.cpp +++ b/stage0/src/runtime/init_module.cpp @@ -13,6 +13,7 @@ Author: Leonardo de Moura #include "runtime/process.h" #include "runtime/mutex.h" #include "runtime/init_module.h" +#include "runtime/libuv.h" namespace lean { extern "C" LEAN_EXPORT void lean_initialize_runtime_module() { @@ -24,6 +25,7 @@ extern "C" LEAN_EXPORT void lean_initialize_runtime_module() { initialize_mutex(); initialize_process(); initialize_stack_overflow(); + initialize_libuv(); } void initialize_runtime_module() { lean_initialize_runtime_module(); diff --git a/stage0/src/runtime/libuv.cpp b/stage0/src/runtime/libuv.cpp index 627eb848d3ef..f625c115950f 100644 --- a/stage0/src/runtime/libuv.cpp +++ b/stage0/src/runtime/libuv.cpp @@ -2,21 +2,36 @@ Copyright (c) 2024 Lean FRO, LLC. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. -Author: Markus Himmel -*/ +Author: Markus Himmel, Sofia Rodrigues + */ +#include #include "runtime/libuv.h" +#include "runtime/object.h" + +namespace lean { #ifndef LEAN_EMSCRIPTEN #include +extern "C" void initialize_libuv() { + initialize_libuv_timer(); + initialize_libuv_loop(); + + lthread([]() { event_loop_run_loop(&global_ev); }); +} + +/* Lean.libUVVersionFn : Unit → Nat */ extern "C" LEAN_EXPORT lean_obj_res lean_libuv_version(lean_obj_arg o) { return lean_unsigned_to_nat(uv_version()); } #else +extern "C" void initialize_libuv() {} + extern "C" LEAN_EXPORT lean_obj_res lean_libuv_version(lean_obj_arg o) { return lean_box(0); } #endif +} \ No newline at end of file diff --git a/stage0/src/runtime/libuv.h b/stage0/src/runtime/libuv.h index 4c53786a59d6..94afa55aa2b0 100644 --- a/stage0/src/runtime/libuv.h +++ b/stage0/src/runtime/libuv.h @@ -2,9 +2,29 @@ Copyright (c) 2024 Lean FRO, LLC. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. -Author: Markus Himmel +Author: Markus Himmel, Sofia Rodrigues */ #pragma once #include +#include "runtime/uv/event_loop.h" + #include "runtime/uv/timer.h" +#include "runtime/alloc.h" +#include "runtime/io.h" +#include "runtime/utf8.h" +#include "runtime/object.h" +#include "runtime/thread.h" +#include "runtime/allocprof.h" +#include "runtime/object.h" +namespace lean { +#ifndef LEAN_EMSCRIPTEN +#include +#endif + +extern "C" void initialize_libuv(); + +// ======================================= +// General LibUV functions. extern "C" LEAN_EXPORT lean_obj_res lean_libuv_version(lean_obj_arg); + +} \ No newline at end of file diff --git a/stage0/src/runtime/object.h b/stage0/src/runtime/object.h index f94b32e95482..4f7fcc782a7c 100644 --- a/stage0/src/runtime/object.h +++ b/stage0/src/runtime/object.h @@ -467,6 +467,11 @@ inline obj_res st_ref_set(b_obj_arg r, obj_arg v, obj_arg w) { return lean_st_re inline obj_res st_ref_reset(b_obj_arg r, obj_arg w) { return lean_st_ref_reset(r, w); } inline obj_res st_ref_swap(b_obj_arg r, obj_arg v, obj_arg w) { return lean_st_ref_swap(r, v, w); } + +extern "C" LEAN_EXPORT obj_res lean_io_promise_new(obj_arg); +extern "C" LEAN_EXPORT obj_res lean_io_promise_resolve(obj_arg value, b_obj_arg promise, obj_arg); +extern "C" LEAN_EXPORT obj_res lean_io_promise_result(obj_arg promise); + // ======================================= // Module initialization/finalization void initialize_object(); diff --git a/stage0/src/runtime/uv/event_loop.cpp b/stage0/src/runtime/uv/event_loop.cpp new file mode 100644 index 000000000000..0afd59534ee4 --- /dev/null +++ b/stage0/src/runtime/uv/event_loop.cpp @@ -0,0 +1,143 @@ +/* +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Sofia Rodrigues, Henrik Böving +*/ +#include "runtime/uv/event_loop.h" + + +/* +This file builds a thread safe event loop on top of the thread unsafe libuv event loop. +We achieve this by always having a `uv_async_t` associated with the libuv event loop. +As `uv_async_t` are a thread safe primitive it is safe to send a notification to it from another +thread. Once this notification arrives the event loop suspends its own execution and unlocks a mutex +that protects it. This mutex can then be taken by another thread that wants to work with the event +loop. After that work is done it signals a condition variable that the event loop is waiting on +to continue its execution. +*/ + +namespace lean { +#ifndef LEAN_EMSCRIPTEN +using namespace std; + +event_loop_t global_ev; + +// Utility function for error checking. This function is only used inside the +// initializition of the event loop. +static void check_uv(int result, const char * msg) { + if (result != 0) { + std::string err_message = std::string(msg) + ": " + uv_strerror(result); + lean_internal_panic(err_message.c_str()); + } +} + +// The callback that stops the loop when it's called. +void async_callback(uv_async_t * handle) { + uv_stop(handle->loop); +} + +// Interrupts the event loop and stops it so it can receive future requests. +void event_loop_interrupt(event_loop_t * event_loop) { + int result = uv_async_send(&event_loop->async); + (void)result; + lean_assert(result == 0); +} + +// Initializes the event loop +void event_loop_init(event_loop_t * event_loop) { + event_loop->loop = uv_default_loop(); + check_uv(uv_mutex_init_recursive(&event_loop->mutex), "Failed to initialize mutex"); + check_uv(uv_cond_init(&event_loop->cond_var), "Failed to initialize condition variable"); + check_uv(uv_async_init(event_loop->loop, &event_loop->async, NULL), "Failed to initialize async"); + event_loop->n_waiters = 0; +} + +// Locks the event loop for the side of the requesters. +void event_loop_lock(event_loop_t * event_loop) { + if (uv_mutex_trylock(&event_loop->mutex) != 0) { + event_loop->n_waiters++; + event_loop_interrupt(event_loop); + uv_mutex_lock(&event_loop->mutex); + event_loop->n_waiters--; + } +} + +// Unlock event loop +void event_loop_unlock(event_loop_t * event_loop) { + if (event_loop->n_waiters == 0) { + uv_cond_signal(&event_loop->cond_var); + } + uv_mutex_unlock(&event_loop->mutex); +} + +// Runs the loop and stops when it needs to register new requests. +void event_loop_run_loop(event_loop_t * event_loop) { + while (uv_loop_alive(event_loop->loop)) { + uv_mutex_lock(&event_loop->mutex); + + while (event_loop->n_waiters != 0) { + uv_cond_wait(&event_loop->cond_var, &event_loop->mutex); + } + + uv_run(event_loop->loop, UV_RUN_ONCE); + /* + * We leave `uv_run` only when `uv_stop` is called as there is always the `uv_async_t` so + * we can never run out of things to wait on. `uv_stop` is only called from `async_callback` + * when another thread wants to work with the event loop so we need to give up the mutex. + */ + + uv_mutex_unlock(&event_loop->mutex); + } +} + +/* Std.Internal.UV.Loop.configure (options : Loop.Options) : BaseIO Unit */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_configure(b_obj_arg options, obj_arg /* w */ ) { + bool accum = lean_ctor_get_uint8(options, 0); + bool block = lean_ctor_get_uint8(options, 1); + + event_loop_lock(&global_ev); + + if (accum && uv_loop_configure(global_ev.loop, UV_METRICS_IDLE_TIME) != 0) { + return io_result_mk_error("failed to configure global_ev.loop with UV_METRICS_IDLE_TIME"); + } + + #if!defined(WIN32) && !defined(_WIN32) + if (block && uv_loop_configure(global_ev.loop, UV_LOOP_BLOCK_SIGNAL, SIGPROF) != 0) { + return io_result_mk_error("failed to configure global_ev.loop with UV_LOOP_BLOCK_SIGNAL"); + } + #endif + + event_loop_unlock(&global_ev); + + return lean_io_result_mk_ok(lean_box(0)); +} + +/* Std.Internal.UV.Loop.alive : BaseIO UInt64 */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_alive(obj_arg /* w */ ) { + event_loop_lock(&global_ev); + int is_alive = uv_loop_alive(global_ev.loop); + event_loop_unlock(&global_ev); + + return lean_io_result_mk_ok(lean_box(is_alive)); +} + +void initialize_libuv_loop() { + event_loop_init(&global_ev); +} + +#else + +/* Std.Internal.UV.Loop.configure (options : Loop.Options) : BaseIO Unit */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_configure(b_obj_arg options, obj_arg /* w */ ) { + return io_result_mk_error("lean_uv_event_loop_configure is not supported"); +} + +/* Std.Internal.UV.Loop.alive : BaseIO UInt64 */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_alive(obj_arg /* w */ ) { + return io_result_mk_error("lean_uv_event_loop_alive is not supported"); +} + +#endif + +} \ No newline at end of file diff --git a/stage0/src/runtime/uv/event_loop.h b/stage0/src/runtime/uv/event_loop.h new file mode 100644 index 000000000000..42dba397e3fa --- /dev/null +++ b/stage0/src/runtime/uv/event_loop.h @@ -0,0 +1,47 @@ +/* +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Sofia Rodrigues +*/ +#pragma once +#include +#include "runtime/io.h" +#include "runtime/object.h" + +namespace lean { + +void initialize_libuv_loop(); + +#ifndef LEAN_EMSCRIPTEN +using namespace std; +#include + +// Event loop structure for managing asynchronous events and synchronization across multiple threads. +typedef struct { + uv_loop_t * loop; // The libuv event loop. + uv_mutex_t mutex; // Mutex for protecting `loop`. + uv_cond_t cond_var; // Condition variable for signaling that `loop` is free. + uv_async_t async; // Async handle to interrupt `loop`. + _Atomic(int) n_waiters; // Atomic counter for managing waiters for `loop`. +} event_loop_t; + +// The multithreaded event loop object for all tasks in the task manager. +extern event_loop_t global_ev; + +// ======================================= +// Event loop manipulation functions. +void event_loop_init(event_loop_t *event_loop); +void event_loop_cleanup(event_loop_t *event_loop); +void event_loop_lock(event_loop_t *event_loop); +void event_loop_unlock(event_loop_t *event_loop); +void event_loop_run_loop(event_loop_t *event_loop); + +#endif + +// ======================================= +// Global event loop manipulation functions +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_configure(b_obj_arg options, obj_arg /* w */ ); +extern "C" LEAN_EXPORT lean_obj_res lean_uv_event_loop_alive(obj_arg /* w */ ); + +} diff --git a/stage0/src/runtime/uv/timer.cpp b/stage0/src/runtime/uv/timer.cpp new file mode 100644 index 000000000000..c34443c08b94 --- /dev/null +++ b/stage0/src/runtime/uv/timer.cpp @@ -0,0 +1,254 @@ +/* +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Sofia Rodrigues, Henrik Böving +*/ +#include "runtime/uv/timer.h" + +namespace lean { +#ifndef LEAN_EMSCRIPTEN + +using namespace std; + +// The finalizer of the `Timer`. +void lean_uv_timer_finalizer(void* ptr) { + lean_uv_timer_object * timer = (lean_uv_timer_object*) ptr; + + if (timer->m_promise != NULL) { + lean_dec(timer->m_promise); + } + + event_loop_lock(&global_ev); + + uv_close((uv_handle_t*)timer->m_uv_timer, [](uv_handle_t* handle) { + free(handle); + }); + + event_loop_unlock(&global_ev); + + free(timer); +} + +void initialize_libuv_timer() { + g_uv_timer_external_class = lean_register_external_class(lean_uv_timer_finalizer, [](void* obj, lean_object* f) { + if (((lean_uv_timer_object*)obj)->m_promise != NULL) { + lean_inc(f); + lean_apply_1(f, ((lean_uv_timer_object*)obj)->m_promise); + } + }); +} + +void handle_timer_event(uv_timer_t* handle) { + lean_object * obj = (lean_object*)handle->data; + lean_uv_timer_object * timer = lean_to_uv_timer(obj); + // handle_timer_event may only be called while the timer is running, this means the promise must + // not be NULL. + lean_assert(timer->m_state == TIMER_STATE_RUNNING); + lean_assert(timer->m_promise != NULL); + + if (timer->m_repeating) { + if (lean_io_get_task_state_core(timer->m_promise) != 2) { + lean_object* res = lean_io_promise_resolve(lean_box(0), timer->m_promise, lean_io_mk_world()); + lean_dec(res); + } + } else { + lean_assert(lean_io_get_task_state_core(timer->m_promise) != 2); + uv_timer_stop(timer->m_uv_timer); + timer->m_state = TIMER_STATE_FINISHED; + + lean_object* res = lean_io_promise_resolve(lean_box(0), timer->m_promise, lean_io_mk_world()); + lean_dec(res); + + // The loop does not need to keep the timer alive anymore. + lean_dec(obj); + } +} + +/* Std.Internal.UV.Timer.mk (timeout : UInt64) (repeating : Bool) : IO Timer */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_mk(uint64_t timeout, uint8_t repeating, obj_arg /* w */) { + lean_uv_timer_object * timer = (lean_uv_timer_object*)malloc(sizeof(lean_uv_timer_object)); + timer->m_timeout = timeout; + timer->m_repeating = repeating; + timer->m_state = TIMER_STATE_INITIAL; + timer->m_promise = NULL; + + uv_timer_t * uv_timer = (uv_timer_t*)malloc(sizeof(uv_timer_t)); + + event_loop_lock(&global_ev); + int result = uv_timer_init(global_ev.loop, uv_timer); + event_loop_unlock(&global_ev); + + if (result != 0) { + free(uv_timer); + free(timer); + std::string err = std::string("failed to initialize timer: ") + uv_strerror(result); + return io_result_mk_error(err.c_str()); + } + + timer->m_uv_timer = uv_timer; + + lean_object * obj = lean_uv_timer_new(timer); + lean_mark_mt(obj); + timer->m_uv_timer->data = obj; + + return lean_io_result_mk_ok(obj); +} + +/* Std.Internal.UV.Timer.next (timer : @& Timer) : IO (IO.Promise Unit) */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_next(b_obj_arg obj, obj_arg /* w */ ) { + lean_uv_timer_object * timer = lean_to_uv_timer(obj); + + auto create_promise = []() { + lean_object * prom_res = lean_io_promise_new(lean_io_mk_world()); + lean_object * promise = lean_ctor_get(prom_res, 0); + lean_inc(promise); + lean_dec(prom_res); + + return promise; + }; + + auto setup_timer = [create_promise, obj, timer]() { + lean_assert(timer->m_promise == NULL); + timer->m_promise = create_promise(); + timer->m_state = TIMER_STATE_RUNNING; + + // The event loop must keep the timer alive for the duration of the run time. + lean_inc(obj); + + event_loop_lock(&global_ev); + + int result = uv_timer_start( + timer->m_uv_timer, + handle_timer_event, + timer->m_repeating ? 0 : timer->m_timeout, + timer->m_repeating ? timer->m_timeout : 0 + ); + + event_loop_unlock(&global_ev); + + if (result != 0) { + lean_dec(obj); + std::string err = std::string("failed to initialize timer: ") + uv_strerror(result); + return io_result_mk_error(err.c_str()); + } else { + lean_inc(timer->m_promise); + return lean_io_result_mk_ok(timer->m_promise); + } + }; + + if (timer->m_repeating) { + switch (timer->m_state) { + case TIMER_STATE_INITIAL: + { + return setup_timer(); + } + case TIMER_STATE_RUNNING: + { + lean_assert(timer->m_promise != NULL); + // 2 indicates finished + if (lean_io_get_task_state_core(timer->m_promise) == 2) { + lean_dec(timer->m_promise); + timer->m_promise = create_promise(); + lean_inc(timer->m_promise); + return lean_io_result_mk_ok(timer->m_promise); + } else { + lean_inc(timer->m_promise); + return lean_io_result_mk_ok(timer->m_promise); + } + } + case TIMER_STATE_FINISHED: + { + lean_assert(timer->m_promise != NULL); + lean_inc(timer->m_promise); + return lean_io_result_mk_ok(timer->m_promise); + } + } + } else { + if (timer->m_state == TIMER_STATE_INITIAL) { + return setup_timer(); + } else { + lean_assert(timer->m_promise != NULL); + + lean_inc(timer->m_promise); + return lean_io_result_mk_ok(timer->m_promise); + } + } +} + +/* Std.Internal.UV.Timer.reset (timer : @& Timer) : IO Unit */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_reset(b_obj_arg obj, obj_arg /* w */ ) { + lean_uv_timer_object * timer = lean_to_uv_timer(obj); + + if (timer->m_state == TIMER_STATE_RUNNING) { + lean_assert(timer->m_promise != NULL); + + event_loop_lock(&global_ev); + + uv_timer_stop(timer->m_uv_timer); + + int result = uv_timer_start( + timer->m_uv_timer, + handle_timer_event, + timer->m_timeout, + timer->m_repeating ? timer->m_timeout : 0 + ); + + event_loop_unlock(&global_ev); + + if (result != 0) { + return io_result_mk_error("failed to restart uv_timer"); + } else { + return lean_io_result_mk_ok(lean_box(0)); + } + } else { + return lean_io_result_mk_ok(lean_box(0)); + } +} + +/* Std.Internal.UV.Timer.stop (timer : @& Timer) : IO Unit */ +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_stop(b_obj_arg obj, obj_arg /* w */) { + lean_uv_timer_object * timer = lean_to_uv_timer(obj); + + if (timer->m_state == TIMER_STATE_RUNNING) { + lean_assert(timer->m_promise != NULL); + + event_loop_lock(&global_ev); + + uv_timer_stop(timer->m_uv_timer); + + event_loop_unlock(&global_ev); + + timer->m_state = TIMER_STATE_FINISHED; + + // The loop does not need to keep the timer alive anymore. + lean_dec(obj); + + return lean_io_result_mk_ok(lean_box(0)); + } else { + return lean_io_result_mk_ok(lean_box(0)); + } +} + +#else + +void lean_uv_timer_finalizer(void* ptr); + +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_mk(uint64_t timeout, uint8_t repeating, obj_arg /* w */) { + return io_result_mk_error("lean_uv_timer_mk is not supported"); +} + +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_next(b_obj_arg timer, obj_arg /* w */ ) { + return io_result_mk_error("lean_uv_timer_next is not supported"); +} + +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_reset(b_obj_arg timer, obj_arg /* w */ ) { + return io_result_mk_error("lean_uv_timer_reset is not supported"); +} + +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_stop(b_obj_arg timer, obj_arg /* w */ ) { + return io_result_mk_error("lean_uv_timer_stop is not supported"); +} + +#endif +} diff --git a/stage0/src/runtime/uv/timer.h b/stage0/src/runtime/uv/timer.h new file mode 100644 index 000000000000..cda80d34fc70 --- /dev/null +++ b/stage0/src/runtime/uv/timer.h @@ -0,0 +1,54 @@ +/* +Copyright (c) 2024 Lean FRO, LLC. All rights reserved. +Released under Apache 2.0 license as described in the file LICENSE. + +Author: Sofia Rodrigues, Henrik Böving +*/ +#pragma once +#include +#include "runtime/uv/event_loop.h" + +namespace lean { + +static lean_external_class * g_uv_timer_external_class = NULL; +void initialize_libuv_timer(); + +#ifndef LEAN_EMSCRIPTEN +using namespace std; +#include + +enum uv_timer_state { + TIMER_STATE_INITIAL, + TIMER_STATE_RUNNING, + TIMER_STATE_FINISHED, +}; + +// Structure for managing a single UV timer object, including promise handling, timeout, and +// repeating behavior. +typedef struct { + uv_timer_t * m_uv_timer; // LibUV timer handle. + lean_object * m_promise; // The associated promise for asynchronous results. + uint64_t m_timeout; // Timeout duration in milliseconds. + bool m_repeating; // Flag indicating if the timer is repeating. + uv_timer_state m_state; // The state of the timer. Beyond the API description on the Lean + // side this state has the invariant: + // `m_state != TIMER_STATE_INITIAL` -> `m_promise != NULL` +} lean_uv_timer_object; + +// ======================================= +// Timer object manipulation functions. +static inline lean_object* lean_uv_timer_new(lean_uv_timer_object * s) { return lean_alloc_external(g_uv_timer_external_class, s); } +static inline lean_uv_timer_object* lean_to_uv_timer(lean_object * o) { return (lean_uv_timer_object*)(lean_get_external_data(o)); } + +#else + +// ======================================= +// Timer manipulation functions +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_mk(uint64_t timeout, uint8_t repeating, obj_arg /* w */); +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_next(b_obj_arg timer, obj_arg /* w */); +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_reset(b_obj_arg timer, obj_arg /* w */); +extern "C" LEAN_EXPORT lean_obj_res lean_uv_timer_stop(b_obj_arg timer, obj_arg /* w */); + +#endif + +} diff --git a/stage0/src/util/shell.cpp b/stage0/src/util/shell.cpp index a39ca0b6586c..a3c4a5452cca 100644 --- a/stage0/src/util/shell.cpp +++ b/stage0/src/util/shell.cpp @@ -225,6 +225,7 @@ static void display_help(std::ostream & out) { std::cout << " --json report Lean output (e.g., messages) as JSON (one per line)\n"; std::cout << " -E --error=kind report Lean messages of kind as errors\n"; std::cout << " --deps just print dependencies of a Lean input\n"; + std::cout << " --src-deps just print dependency sources of a Lean input\n"; std::cout << " --print-prefix print the installation prefix for Lean and exit\n"; std::cout << " --print-libdir print the installation directory for Lean's built-in libraries and exit\n"; std::cout << " --profile display elaboration/type checking time for each definition/theorem\n"; @@ -235,6 +236,7 @@ static void display_help(std::ostream & out) { std::cout << " -D name=value set a configuration option (see set_option command)\n"; } +static int only_src_deps = 0; static int print_prefix = 0; static int print_libdir = 0; static int json_output = 0; @@ -255,6 +257,7 @@ static struct option g_long_options[] = { {"stats", no_argument, 0, 'a'}, {"quiet", no_argument, 0, 'q'}, {"deps", no_argument, 0, 'd'}, + {"src-deps", no_argument, &only_src_deps, 1}, {"deps-json", no_argument, 0, 'J'}, {"timeout", optional_argument, 0, 'T'}, {"c", optional_argument, 0, 'c'}, @@ -399,6 +402,12 @@ void print_imports(std::string const & input, std::string const & fname) { consume_io_result(lean_print_imports(mk_string(input), mk_option_some(mk_string(fname)), io_mk_world())); } +/* def printImportSrcs (input : String) (fileName : Option String := none) : IO Unit */ +extern "C" object* lean_print_import_srcs(object* input, object* file_name, object* w); +void print_import_srcs(std::string const & input, std::string const & fname) { + consume_io_result(lean_print_import_srcs(mk_string(input), mk_option_some(mk_string(fname)), io_mk_world())); +} + /* def printImportsJson (fileNames : Array String) : IO Unit */ extern "C" object* lean_print_imports_json(object * file_names, object * w); void print_imports_json(array_ref const & fnames) { @@ -697,6 +706,11 @@ extern "C" LEAN_EXPORT int lean_main(int argc, char ** argv) { return 0; } + if (only_src_deps) { + print_import_srcs(contents, mod_fn); + return 0; + } + // Quick and dirty `#lang` support // TODO: make it extensible, and add `lean4md` if (contents.compare(0, 5, "#lang") == 0) { diff --git a/stage0/stdlib/Init/Data/Array/Basic.c b/stage0/stdlib/Init/Data/Array/Basic.c index 407555c9bae0..7a3973379174 100644 --- a/stage0/stdlib/Init/Data/Array/Basic.c +++ b/stage0/stdlib/Init/Data/Array/Basic.c @@ -67,7 +67,6 @@ LEAN_EXPORT lean_object* l_Array_findFinIdx_x3f_loop(lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithAll___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_ofFn_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findM_x3f___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_10766_; LEAN_EXPORT lean_object* l_Array_eraseP(lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__List_toArrayAux_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__3; @@ -142,6 +141,7 @@ LEAN_EXPORT lean_object* l_Array_elem___rarg___boxed(lean_object*, lean_object*, LEAN_EXPORT lean_object* l_Array_indexOf_x3f___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_1588____closed__4; static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__4; +LEAN_EXPORT lean_object* l_Array_sum(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Array_contains___spec__1___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t); static lean_object* l_Array_instRepr___rarg___closed__8; LEAN_EXPORT lean_object* l_Array_findIdx_x3f_loop___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -157,6 +157,7 @@ LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___at_Array_findRev_x3f___ LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_all___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListAppend___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_unzip(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Array_reduceOption___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findIdx_x3f_loop(lean_object*); @@ -169,6 +170,7 @@ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEqv___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_List_toString___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWith___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM(lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__4; LEAN_EXPORT lean_object* l_Array_back(lean_object*); @@ -250,7 +252,6 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findIdxM_x3f___ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_toListImpl___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_append___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_2619_; LEAN_EXPORT lean_object* l_Array_mapMUnsafe(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_instToString(lean_object*); LEAN_EXPORT lean_object* l_Array_reverse___rarg(lean_object*); @@ -385,7 +386,6 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_1596_; LEAN_EXPORT lean_object* l_panic___at_Array_eraseIdx_x21___spec__1___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___rarg___lambda__1(size_t, lean_object*, lean_object*, lean_object*, size_t, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_11146_; LEAN_EXPORT lean_object* l_Array_modify___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -442,6 +442,7 @@ LEAN_EXPORT lean_object* l_Array_back_x21___rarg___boxed(lean_object*, lean_obje LEAN_EXPORT lean_object* l_Array_filterMapM___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSome_x3f(lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_1588____closed__15; +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_eraseIdx_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_instInhabited(lean_object*); LEAN_EXPORT lean_object* l_Array_getEvenElems___rarg___boxed(lean_object*); @@ -449,6 +450,7 @@ LEAN_EXPORT lean_object* l_List_foldl___at_Array_appendList___spec__1(lean_objec LEAN_EXPORT lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Array_findSome_x21___rarg___closed__1; static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__14; +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_2624_; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_find_x3f___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instRepr___rarg___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findSomeM_x3f___spec__1(lean_object*, lean_object*, lean_object*); @@ -473,6 +475,7 @@ static lean_object* l_Array_instRepr___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_reduceOption___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_modify___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__11; +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_11179_; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Array_allM___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t); @@ -481,6 +484,7 @@ LEAN_EXPORT lean_object* l_Array_isEmpty___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_append___rarg___boxed(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__16; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_forM___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_foldr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_split___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_take_loop___rarg(lean_object*, lean_object*); @@ -515,6 +519,7 @@ LEAN_EXPORT uint8_t l_Array_contains___rarg(lean_object*, lean_object*, lean_obj LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_eraseReps___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_sum___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filter___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Array_filterM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Array_Basic_0__Array_allDiffAux___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -628,6 +633,7 @@ size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_flatMapM(lean_object*, lean_object*, lean_object*); static lean_object* l_term_x23_x5b___x2c_x5d___closed__6; +LEAN_EXPORT lean_object* l_Array_sum___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_instRepr___rarg___closed__4; LEAN_EXPORT lean_object* l_Array_ofFn_go___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithAll_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -644,6 +650,7 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findIdxM_x3f___ static lean_object* l___aux__Init__Data__Array__Basic______macroRules__term_x23_x5b___x2c_x5d__1___closed__15; LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_zipWithIndex___spec__1(lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWithIndex___rarg___boxed(lean_object*); @@ -677,6 +684,7 @@ LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdx___spec__1(lean LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_zipWith(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at_Array_mapIdxM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrM_fold___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findIdxM_x3f___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_allM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -734,6 +742,7 @@ static lean_object* l_Array_getEvenElems___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_findM_x3f___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_insertAt___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_findSomeRevM_x3f_find___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Array_Basic___hyg_10799_; LEAN_EXPORT lean_object* l_Array_modifyMUnsafe___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapM_map___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_isEmpty___rarg(lean_object*); @@ -1887,10 +1896,13 @@ return x_2; LEAN_EXPORT lean_object* l_Array_singleton___rarg(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; -x_2 = lean_unsigned_to_nat(1u); -x_3 = lean_mk_array(x_2, x_1); -return x_3; +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = lean_box(0); +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +x_4 = lean_array_mk(x_3); +return x_4; } } LEAN_EXPORT lean_object* l_Array_singleton(lean_object* x_1) { @@ -2054,7 +2066,7 @@ lean_dec(x_1); return x_2; } } -static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_2619_() { +static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_2624_() { _start: { lean_object* x_1; @@ -2160,7 +2172,7 @@ x_9 = l_Array_swapAt_x21___rarg___closed__2; x_10 = lean_string_append(x_8, x_9); x_11 = l_Array_swapAt_x21___rarg___closed__3; x_12 = l_Array_swapAt_x21___rarg___closed__4; -x_13 = lean_unsigned_to_nat(272u); +x_13 = lean_unsigned_to_nat(271u); x_14 = lean_unsigned_to_nat(4u); x_15 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_11, x_12, x_13, x_14, x_10); lean_dec(x_10); @@ -6008,6 +6020,163 @@ lean_dec(x_3); return x_6; } } +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_eq(x_3, x_4); +if (x_6 == 0) +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_sub(x_3, x_7); +x_9 = lean_array_uget(x_2, x_8); +lean_inc(x_1); +x_10 = lean_apply_2(x_1, x_9, x_5); +x_3 = x_8; +x_5 = x_10; +goto _start; +} +else +{ +lean_dec(x_1); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = lean_usize_dec_eq(x_3, x_4); +if (x_6 == 0) +{ +size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_7 = 1; +x_8 = lean_usize_sub(x_3, x_7); +x_9 = lean_array_uget(x_2, x_8); +lean_inc(x_1); +x_10 = lean_apply_2(x_1, x_9, x_5); +x_3 = x_8; +x_5 = x_10; +goto _start; +} +else +{ +lean_dec(x_1); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg___boxed), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_sum___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_array_get_size(x_3); +x_5 = lean_nat_dec_le(x_4, x_4); +if (x_5 == 0) +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_lt(x_6, x_4); +if (x_7 == 0) +{ +lean_dec(x_4); +lean_dec(x_1); +return x_2; +} +else +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_usize_of_nat(x_4); +lean_dec(x_4); +x_9 = 0; +x_10 = l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg(x_1, x_3, x_8, x_9, x_2); +return x_10; +} +} +else +{ +lean_object* x_11; uint8_t x_12; +x_11 = lean_unsigned_to_nat(0u); +x_12 = lean_nat_dec_lt(x_11, x_4); +if (x_12 == 0) +{ +lean_dec(x_4); +lean_dec(x_1); +return x_2; +} +else +{ +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_usize_of_nat(x_4); +lean_dec(x_4); +x_14 = 0; +x_15 = l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg(x_1, x_3, x_13, x_14, x_2); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_sum(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_sum___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_foldrMUnsafe_fold___at_Array_sum___spec__1___rarg(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_foldrMUnsafe_fold___at_Array_sum___spec__2___rarg(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Array_sum___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Array_sum___rarg(x_1, x_2, x_3); +lean_dec(x_3); +return x_4; +} +} LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Array_map___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { @@ -6701,7 +6870,7 @@ static lean_object* _init_l_Array_findSome_x21___rarg___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_swapAt_x21___rarg___closed__3; x_2 = l_Array_findSome_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(613u); +x_3 = lean_unsigned_to_nat(618u); x_4 = lean_unsigned_to_nat(14u); x_5 = l_Array_findSome_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -9947,7 +10116,7 @@ lean_dec(x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_10766_() { +static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_10799_() { _start: { lean_object* x_1; @@ -10059,7 +10228,7 @@ static lean_object* _init_l_Array_eraseIdx_x21___rarg___closed__3() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_swapAt_x21___rarg___closed__3; x_2 = l_Array_eraseIdx_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(841u); +x_3 = lean_unsigned_to_nat(846u); x_4 = lean_unsigned_to_nat(45u); x_5 = l_Array_eraseIdx_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10156,7 +10325,7 @@ x_2 = lean_alloc_closure((void*)(l_Array_eraseP___rarg), 2, 0); return x_2; } } -static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_11146_() { +static lean_object* _init_l___auto____x40_Init_Data_Array_Basic___hyg_11179_() { _start: { lean_object* x_1; @@ -10289,7 +10458,7 @@ static lean_object* _init_l_Array_insertIdx_x21___rarg___closed__2() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Array_swapAt_x21___rarg___closed__3; x_2 = l_Array_insertIdx_x21___rarg___closed__1; -x_3 = lean_unsigned_to_nat(875u); +x_3 = lean_unsigned_to_nat(880u); x_4 = lean_unsigned_to_nat(7u); x_5 = l_Array_eraseIdx_x21___rarg___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -12270,8 +12439,8 @@ l_Array_instGetElemUSizeLtNatToNatSize___closed__1 = _init_l_Array_instGetElemUS lean_mark_persistent(l_Array_instGetElemUSizeLtNatToNatSize___closed__1); l_Array_range___closed__1 = _init_l_Array_range___closed__1(); lean_mark_persistent(l_Array_range___closed__1); -l___auto____x40_Init_Data_Array_Basic___hyg_2619_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_2619_(); -lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_2619_); +l___auto____x40_Init_Data_Array_Basic___hyg_2624_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_2624_(); +lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_2624_); l_Array_swapAt_x21___rarg___closed__1 = _init_l_Array_swapAt_x21___rarg___closed__1(); lean_mark_persistent(l_Array_swapAt_x21___rarg___closed__1); l_Array_swapAt_x21___rarg___closed__2 = _init_l_Array_swapAt_x21___rarg___closed__2(); @@ -12302,16 +12471,16 @@ l_Array_filter___rarg___closed__1 = _init_l_Array_filter___rarg___closed__1(); lean_mark_persistent(l_Array_filter___rarg___closed__1); l_Array_partition___rarg___closed__1 = _init_l_Array_partition___rarg___closed__1(); lean_mark_persistent(l_Array_partition___rarg___closed__1); -l___auto____x40_Init_Data_Array_Basic___hyg_10766_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_10766_(); -lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_10766_); +l___auto____x40_Init_Data_Array_Basic___hyg_10799_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_10799_(); +lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_10799_); l_Array_eraseIdx_x21___rarg___closed__1 = _init_l_Array_eraseIdx_x21___rarg___closed__1(); lean_mark_persistent(l_Array_eraseIdx_x21___rarg___closed__1); l_Array_eraseIdx_x21___rarg___closed__2 = _init_l_Array_eraseIdx_x21___rarg___closed__2(); lean_mark_persistent(l_Array_eraseIdx_x21___rarg___closed__2); l_Array_eraseIdx_x21___rarg___closed__3 = _init_l_Array_eraseIdx_x21___rarg___closed__3(); lean_mark_persistent(l_Array_eraseIdx_x21___rarg___closed__3); -l___auto____x40_Init_Data_Array_Basic___hyg_11146_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_11146_(); -lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_11146_); +l___auto____x40_Init_Data_Array_Basic___hyg_11179_ = _init_l___auto____x40_Init_Data_Array_Basic___hyg_11179_(); +lean_mark_persistent(l___auto____x40_Init_Data_Array_Basic___hyg_11179_); l_Array_insertIdx_x21___rarg___closed__1 = _init_l_Array_insertIdx_x21___rarg___closed__1(); lean_mark_persistent(l_Array_insertIdx_x21___rarg___closed__1); l_Array_insertIdx_x21___rarg___closed__2 = _init_l_Array_insertIdx_x21___rarg___closed__2(); diff --git a/stage0/stdlib/Init/Data/BitVec/Lemmas.c b/stage0/stdlib/Init/Data/BitVec/Lemmas.c index 325daedf3fa2..0ffb3f9fb200 100644 --- a/stage0/stdlib/Init/Data/BitVec/Lemmas.c +++ b/stage0/stdlib/Init/Data/BitVec/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.BitVec.Lemmas -// Imports: Init.Data.Bool Init.Data.BitVec.Basic Init.Data.Fin.Lemmas Init.Data.Nat.Lemmas Init.Data.Nat.Div.Lemmas Init.Data.Nat.Mod Init.Data.Int.Bitwise.Lemmas Init.Data.Int.Pow +// Imports: Init.Data.Bool Init.Data.BitVec.Basic Init.Data.Fin.Lemmas Init.Data.Nat.Lemmas Init.Data.Nat.Div.Lemmas Init.Data.Nat.Mod Init.Data.Nat.Div.Lemmas Init.Data.Int.Bitwise.Lemmas Init.Data.Int.Pow #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -623,6 +623,7 @@ lean_object* initialize_Init_Data_Fin_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Nat_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Nat_Div_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Nat_Mod(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Nat_Div_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Int_Bitwise_Lemmas(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Int_Pow(uint8_t builtin, lean_object*); static bool _G_initialized = false; @@ -648,6 +649,9 @@ lean_dec_ref(res); res = initialize_Init_Data_Nat_Mod(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Nat_Div_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Init_Data_Int_Bitwise_Lemmas(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Init/Data/UInt/Bitwise.c b/stage0/stdlib/Init/Data/UInt/Bitwise.c index 5ee540dfd83a..2bdf88e86737 100644 --- a/stage0/stdlib/Init/Data/UInt/Bitwise.c +++ b/stage0/stdlib/Init/Data/UInt/Bitwise.c @@ -14,11 +14,13 @@ extern "C" { #endif static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__114; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__70; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__16; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__48; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98; lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__13; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__8; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161; @@ -26,11 +28,14 @@ static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__11; LEAN_EXPORT lean_object* l_commandDeclare__bitwise__uint__theorems____; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__65; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__46; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__57; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__163; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__169; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__52; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__103; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__82; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__7; @@ -57,9 +62,11 @@ uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__25; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__144; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__77; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__18; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__64; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__54; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__33; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__36; @@ -70,6 +77,7 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__156; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__29; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__111; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__126; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__1; @@ -81,9 +89,11 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__150; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__138; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__50; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180; lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__41; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__172; @@ -106,6 +116,7 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__75; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__9; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__162; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__132; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__47; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__1; @@ -127,6 +138,7 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__160; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86; @@ -140,9 +152,13 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__10; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__14; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__69; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__26; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__53; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__3; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__152; @@ -152,14 +168,18 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__11; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__109; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__12; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__60; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__2; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__164; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__135; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__116; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__39; @@ -171,9 +191,14 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__38; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__66; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__148; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__56; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__15; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__94; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__8; @@ -181,7 +206,9 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__5; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__43; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__129; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__153; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__140; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78; @@ -201,18 +228,27 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__79; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__125; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206; LEAN_EXPORT lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1(lean_object*, lean_object*, lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__93; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__91; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__139; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__32; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__88; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__76; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__87; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__170; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209; static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__6; lean_object* l_String_toSubstring_x27(lean_object*); static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104; @@ -220,6 +256,7 @@ static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandD static lean_object* l_commandDeclare__bitwise__uint__theorems_______closed__15; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92; static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__20; +static lean_object* l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210; static lean_object* _init_l_commandDeclare__bitwise__uint__theorems_______closed__1() { _start: { @@ -669,7 +706,7 @@ static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__co _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("toBitVec_and", 12, 12); +x_1 = lean_mk_string_unchecked("toBitVec_add", 12, 12); return x_1; } } @@ -716,7 +753,7 @@ static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__co _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("explicitBinder", 14, 14); +x_1 = lean_mk_string_unchecked("implicitBinder", 14, 14); return x_1; } } @@ -736,7 +773,7 @@ static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__co _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("(", 1, 1); +x_1 = lean_mk_string_unchecked("{", 1, 1); return x_1; } } @@ -806,7 +843,7 @@ static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__co _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked(")", 1, 1); +x_1 = lean_mk_string_unchecked("}", 1, 1); return x_1; } } @@ -892,29 +929,45 @@ static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__co _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_&&&_", 9, 9); +x_1 = lean_mk_string_unchecked("(", 1, 1); return x_1; } } static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__56() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_+_", 7, 7); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__57() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__55; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__56; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__57() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__58() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("&&&", 3, 3); +x_1 = lean_mk_string_unchecked("+", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__58() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(")", 1, 1); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__60() { _start: { lean_object* x_1; @@ -922,7 +975,7 @@ x_1 = lean_mk_string_unchecked(".", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61() { _start: { lean_object* x_1; @@ -930,26 +983,26 @@ x_1 = lean_mk_string_unchecked("toBitVec", 8, 8); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__60() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__62() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__63() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__62() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__64() { _start: { lean_object* x_1; @@ -957,7 +1010,7 @@ x_1 = lean_mk_string_unchecked("=", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__63() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__65() { _start: { lean_object* x_1; @@ -965,26 +1018,26 @@ x_1 = lean_mk_string_unchecked("a.toBitVec", 10, 10); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__64() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__66() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__63; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__65; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__65() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__67() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__39; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__66() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__68() { _start: { lean_object* x_1; @@ -992,26 +1045,26 @@ x_1 = lean_mk_string_unchecked("b.toBitVec", 10, 10); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__67() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__69() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__66; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__68; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__68() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__70() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__42; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__69() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__71() { _start: { lean_object* x_1; @@ -1019,19 +1072,19 @@ x_1 = lean_mk_string_unchecked("declValSimple", 13, 13); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__70() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__5; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__69; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__71; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__71() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__73() { _start: { lean_object* x_1; @@ -1039,7 +1092,7 @@ x_1 = lean_mk_string_unchecked(":=", 2, 2); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74() { _start: { lean_object* x_1; @@ -1047,26 +1100,26 @@ x_1 = lean_mk_string_unchecked("rfl", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__73() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__75() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__76() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__75() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__77() { _start: { lean_object* x_1; @@ -1074,7 +1127,7 @@ x_1 = lean_mk_string_unchecked("Termination", 11, 11); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__76() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78() { _start: { lean_object* x_1; @@ -1082,178 +1135,205 @@ x_1 = lean_mk_string_unchecked("suffix", 6, 6); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__77() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__79() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__75; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__76; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__77; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("toBitVec_or", 11, 11); +x_1 = lean_mk_string_unchecked("toBitVec_sub", 12, 12); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__79() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__81() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__82() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__78; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__81() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__83() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_|||_", 9, 9); +x_1 = lean_mk_string_unchecked("term_-_", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__82() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__84() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__81; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__83; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__83() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__85() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("|||", 3, 3); +x_1 = lean_mk_string_unchecked("-", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__84() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("toBitVec_xor", 12, 12); +x_1 = lean_mk_string_unchecked("toBitVec_mul", 12, 12); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__85() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__87() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__84; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__88() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__84; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__87() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__89() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_^^^_", 9, 9); +x_1 = lean_mk_string_unchecked("term_*_", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__88() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__90() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__87; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__89; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__89() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__91() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("^^^", 3, 3); +x_1 = lean_mk_string_unchecked("*", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__90() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("toBitVec_shiftLeft", 18, 18); +x_1 = lean_mk_string_unchecked("toBitVec_div", 12, 12); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__91() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__93() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__90; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__94() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__90; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__93() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__95() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("term_<<<_", 9, 9); +x_1 = lean_mk_string_unchecked("term_/_", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__94() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__96() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__93; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__95; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__95() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__97() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("<<<", 3, 3); +x_1 = lean_mk_string_unchecked("/", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__96() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_mod", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__100() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__101() { _start: { lean_object* x_1; @@ -1261,17 +1341,17 @@ x_1 = lean_mk_string_unchecked("term_%_", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__97() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__102() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__96; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__101; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__103() { _start: { lean_object* x_1; @@ -1279,7 +1359,292 @@ x_1 = lean_mk_string_unchecked("%", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_not", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__106() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__107() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term~~~_", 8, 8); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__107; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__109() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("~~~", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__110() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_and", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__111() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__110; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__112() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__110; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__113() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("explicitBinder", 14, 14); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__114() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__13; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__113; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__115() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_&&&_", 9, 9); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__116() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__115; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__117() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("&&&", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__118() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_or", 11, 11); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__119() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__118; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__118; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__121() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_|||_", 9, 9); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__122() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__121; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__123() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("|||", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_xor", 12, 12); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__125() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__126() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__127() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_^^^_", 9, 9); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__128() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__127; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__129() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("^^^", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__130() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("toBitVec_shiftLeft", 18, 18); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__130; +x_2 = l_String_toSubstring_x27(x_1); +return x_2; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__132() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__130; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__133() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term_<<<_", 9, 9); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__133; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__135() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("<<<", 3, 3); +return x_1; +} +} +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__136() { _start: { lean_object* x_1; @@ -1287,26 +1652,26 @@ x_1 = lean_mk_string_unchecked("toBitVec_shiftRight", 19, 19); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__100() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__137() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__136; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__101() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__138() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__136; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__102() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__139() { _start: { lean_object* x_1; @@ -1314,17 +1679,17 @@ x_1 = lean_mk_string_unchecked("term_>>>_", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__103() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__140() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__102; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__139; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__141() { _start: { lean_object* x_1; @@ -1332,7 +1697,7 @@ x_1 = lean_mk_string_unchecked(">>>", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142() { _start: { lean_object* x_1; @@ -1340,26 +1705,26 @@ x_1 = lean_mk_string_unchecked("toNat_and", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__106() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__143() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__107() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__144() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145() { _start: { lean_object* x_1; @@ -1367,26 +1732,26 @@ x_1 = lean_mk_string_unchecked("toNat", 5, 5); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__109() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__110() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__147() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__111() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__148() { _start: { lean_object* x_1; @@ -1394,26 +1759,26 @@ x_1 = lean_mk_string_unchecked("a.toNat", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__112() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__111; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__148; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__113() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__150() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__39; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__114() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__151() { _start: { lean_object* x_1; @@ -1421,26 +1786,26 @@ x_1 = lean_mk_string_unchecked("b.toNat", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__115() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__152() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__114; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__151; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__116() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__153() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__42; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__117() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__154() { _start: { lean_object* x_1; @@ -1448,19 +1813,19 @@ x_1 = lean_mk_string_unchecked("byTactic", 8, 8); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__118() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__13; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__117; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__154; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__119() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__156() { _start: { lean_object* x_1; @@ -1468,7 +1833,7 @@ x_1 = lean_mk_string_unchecked("by", 2, 2); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157() { _start: { lean_object* x_1; @@ -1476,7 +1841,7 @@ x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__121() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__158() { _start: { lean_object* x_1; @@ -1484,19 +1849,19 @@ x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__122() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__159() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__121; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__158; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__123() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__160() { _start: { lean_object* x_1; @@ -1504,31 +1869,31 @@ x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__123; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__160; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__125() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__162() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__22; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__126() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__163() { _start: { lean_object* x_1; @@ -1536,19 +1901,19 @@ x_1 = lean_mk_string_unchecked("optConfig", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__127() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__164() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__126; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__163; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__128() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__165() { _start: { lean_object* x_1; @@ -1556,7 +1921,7 @@ x_1 = lean_mk_string_unchecked("[", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__129() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__166() { _start: { lean_object* x_1; @@ -1564,19 +1929,19 @@ x_1 = lean_mk_string_unchecked("simpLemma", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__130() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__167() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; -x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__129; +x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__166; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__168() { _start: { lean_object* x_1; @@ -1584,26 +1949,26 @@ x_1 = lean_mk_string_unchecked("toNat_or", 8, 8); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__132() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__169() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__168; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__133() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__170() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__168; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171() { _start: { lean_object* x_1; @@ -1611,26 +1976,26 @@ x_1 = lean_mk_string_unchecked("toNat_xor", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__135() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__172() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__136() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__137() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174() { _start: { lean_object* x_1; @@ -1638,26 +2003,26 @@ x_1 = lean_mk_string_unchecked("toNat_shiftLeft", 15, 15); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__138() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__137; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__139() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__137; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__140() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177() { _start: { lean_object* x_1; @@ -1665,17 +2030,17 @@ x_1 = lean_mk_string_unchecked("term_^_", 7, 7); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__141() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__140; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179() { _start: { lean_object* x_1; @@ -1683,17 +2048,17 @@ x_1 = lean_mk_string_unchecked("num", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__143() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__144() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181() { _start: { lean_object* x_1; @@ -1701,7 +2066,7 @@ x_1 = lean_mk_string_unchecked("2", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182() { _start: { lean_object* x_1; @@ -1709,7 +2074,7 @@ x_1 = lean_mk_string_unchecked("^", 1, 1); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183() { _start: { lean_object* x_1; @@ -1717,26 +2082,26 @@ x_1 = lean_mk_string_unchecked("toNat_shiftRight", 16, 16); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__147() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__148() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186() { _start: { lean_object* x_1; @@ -1744,19 +2109,19 @@ x_1 = lean_mk_string_unchecked("in", 2, 2); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__150() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__5; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__151() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188() { _start: { lean_object* x_1; @@ -1764,19 +2129,19 @@ x_1 = lean_mk_string_unchecked("open", 4, 4); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__152() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__5; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__151; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__153() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190() { _start: { lean_object* x_1; @@ -1784,19 +2149,19 @@ x_1 = lean_mk_string_unchecked("openOnly", 8, 8); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__154() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__5; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__153; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192() { _start: { lean_object* x_1; @@ -1804,17 +2169,17 @@ x_1 = lean_mk_string_unchecked("deprecated", 10, 10); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__156() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194() { _start: { lean_object* x_1; @@ -1822,7 +2187,7 @@ x_1 = lean_mk_string_unchecked("since", 5, 5); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__158() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195() { _start: { lean_object* x_1; @@ -1830,17 +2195,17 @@ x_1 = lean_mk_string_unchecked("str", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__159() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__158; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__160() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197() { _start: { lean_object* x_1; @@ -1848,7 +2213,7 @@ x_1 = lean_mk_string_unchecked("\"2024-11-28\"", 12, 12); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198() { _start: { lean_object* x_1; @@ -1856,26 +2221,26 @@ x_1 = lean_mk_string_unchecked("and_toNat", 9, 9); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__162() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__163() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__164() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201() { _start: { lean_object* x_1; @@ -1883,19 +2248,19 @@ x_1 = lean_mk_string_unchecked("app", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__165() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__13; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__164; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__166() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203() { _start: { lean_object* x_1; @@ -1903,16 +2268,16 @@ x_1 = lean_mk_string_unchecked("BitVec.toNat_and", 16, 16); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__167() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__166; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203; x_2 = l_String_toSubstring_x27(x_1); return x_2; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__168() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205() { _start: { lean_object* x_1; @@ -1920,17 +2285,17 @@ x_1 = lean_mk_string_unchecked("BitVec", 6, 6); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__169() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__168; -x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105; +x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205; +x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__142; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__170() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207() { _start: { lean_object* x_1; @@ -1938,19 +2303,19 @@ x_1 = lean_mk_string_unchecked("ellipsis", 8, 8); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__13; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__170; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__172() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209() { _start: { lean_object* x_1; @@ -1958,7 +2323,7 @@ x_1 = lean_mk_string_unchecked("..", 2, 2); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210() { _start: { lean_object* x_1; @@ -1966,14 +2331,14 @@ x_1 = lean_mk_string_unchecked("end", 3, 3); return x_1; } } -static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174() { +static lean_object* _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__3; x_2 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__4; x_3 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__5; -x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173; +x_4 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -1997,7 +2362,7 @@ return x_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; x_8 = lean_unsigned_to_nat(1u); x_9 = l_Lean_Syntax_getArg(x_1, x_8); x_10 = lean_unsigned_to_nat(2u); @@ -2133,752 +2498,1088 @@ lean_ctor_set(x_66, 0, x_14); lean_ctor_set(x_66, 1, x_65); x_67 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__37; lean_inc(x_66); -lean_inc(x_21); +lean_inc(x_64); +lean_inc(x_61); lean_inc(x_54); lean_inc(x_14); -x_68 = l_Lean_Syntax_node5(x_14, x_67, x_54, x_61, x_64, x_21, x_66); +x_68 = l_Lean_Syntax_node4(x_14, x_67, x_54, x_61, x_64, x_66); lean_inc(x_14); x_69 = l_Lean_Syntax_node1(x_14, x_19, x_68); -x_70 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__57; +x_70 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__55; lean_inc(x_14); x_71 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_71, 0, x_14); lean_ctor_set(x_71, 1, x_70); -x_72 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__56; +x_72 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__58; +lean_inc(x_14); +x_73 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_73, 0, x_14); +lean_ctor_set(x_73, 1, x_72); +x_74 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__57; lean_inc(x_60); -lean_inc(x_71); +lean_inc(x_73); lean_inc(x_57); lean_inc(x_14); -x_73 = l_Lean_Syntax_node3(x_14, x_72, x_57, x_71, x_60); -x_74 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__54; -lean_inc(x_66); -lean_inc(x_54); -lean_inc(x_14); -x_75 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_73, x_66); -x_76 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__58; +x_75 = l_Lean_Syntax_node3(x_14, x_74, x_57, x_73, x_60); +x_76 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__59; lean_inc(x_14); x_77 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_77, 0, x_14); lean_ctor_set(x_77, 1, x_76); -x_78 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__60; -x_79 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__61; -lean_inc(x_14); -x_80 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_80, 0, x_14); -lean_ctor_set(x_80, 1, x_78); -lean_ctor_set(x_80, 2, x_79); -lean_ctor_set(x_80, 3, x_47); -x_81 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__52; -lean_inc(x_80); +x_78 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__54; lean_inc(x_77); -lean_inc(x_75); +lean_inc(x_71); lean_inc(x_14); -x_82 = l_Lean_Syntax_node3(x_14, x_81, x_75, x_77, x_80); -x_83 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__62; +x_79 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_75, x_77); +x_80 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__60; lean_inc(x_14); -x_84 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_84, 0, x_14); -lean_ctor_set(x_84, 1, x_83); -x_85 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__64; -x_86 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__65; -lean_inc(x_14); -x_87 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_87, 0, x_14); -lean_ctor_set(x_87, 1, x_85); -lean_ctor_set(x_87, 2, x_86); -lean_ctor_set(x_87, 3, x_47); -x_88 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__67; -x_89 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__68; -lean_inc(x_14); -x_90 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_90, 0, x_14); -lean_ctor_set(x_90, 1, x_88); -lean_ctor_set(x_90, 2, x_89); -lean_ctor_set(x_90, 3, x_47); -lean_inc(x_90); -lean_inc(x_71); -lean_inc(x_87); +x_81 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_81, 0, x_14); +lean_ctor_set(x_81, 1, x_80); +x_82 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__62; +x_83 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__63; lean_inc(x_14); -x_91 = l_Lean_Syntax_node3(x_14, x_72, x_87, x_71, x_90); -x_92 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__50; +x_84 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_84, 0, x_14); +lean_ctor_set(x_84, 1, x_82); +lean_ctor_set(x_84, 2, x_83); +lean_ctor_set(x_84, 3, x_47); +x_85 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__52; lean_inc(x_84); -lean_inc(x_14); -x_93 = l_Lean_Syntax_node3(x_14, x_92, x_82, x_84, x_91); -x_94 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__48; +lean_inc(x_81); +lean_inc(x_14); +x_86 = l_Lean_Syntax_node3(x_14, x_85, x_79, x_81, x_84); +x_87 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__64; +lean_inc(x_14); +x_88 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_88, 0, x_14); +lean_ctor_set(x_88, 1, x_87); +x_89 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__66; +x_90 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__67; +lean_inc(x_14); +x_91 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_91, 0, x_14); +lean_ctor_set(x_91, 1, x_89); +lean_ctor_set(x_91, 2, x_90); +lean_ctor_set(x_91, 3, x_47); +x_92 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__69; +x_93 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__70; +lean_inc(x_14); +x_94 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_94, 0, x_14); +lean_ctor_set(x_94, 1, x_92); +lean_ctor_set(x_94, 2, x_93); +lean_ctor_set(x_94, 3, x_47); +lean_inc(x_94); +lean_inc(x_91); +lean_inc(x_14); +x_95 = l_Lean_Syntax_node3(x_14, x_74, x_91, x_73, x_94); +x_96 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__50; +lean_inc(x_88); +lean_inc(x_14); +x_97 = l_Lean_Syntax_node3(x_14, x_96, x_86, x_88, x_95); +x_98 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__48; lean_inc(x_63); lean_inc(x_14); -x_95 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_93); -x_96 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__35; +x_99 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_97); +x_100 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__35; lean_inc(x_69); lean_inc(x_14); -x_97 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_95); -x_98 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__71; -lean_inc(x_14); -x_99 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_99, 0, x_14); -lean_ctor_set(x_99, 1, x_98); -x_100 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__73; -x_101 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__74; -lean_inc(x_14); -x_102 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_102, 0, x_14); -lean_ctor_set(x_102, 1, x_100); -lean_ctor_set(x_102, 2, x_101); -lean_ctor_set(x_102, 3, x_47); -x_103 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__77; +x_101 = l_Lean_Syntax_node2(x_14, x_100, x_69, x_99); +x_102 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__73; +lean_inc(x_14); +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_14); +lean_ctor_set(x_103, 1, x_102); +x_104 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__75; +x_105 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__76; +lean_inc(x_14); +x_106 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_106, 0, x_14); +lean_ctor_set(x_106, 1, x_104); +lean_ctor_set(x_106, 2, x_105); +lean_ctor_set(x_106, 3, x_47); +x_107 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__79; lean_inc_n(x_21, 2); lean_inc(x_14); -x_104 = l_Lean_Syntax_node2(x_14, x_103, x_21, x_21); -x_105 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__70; +x_108 = l_Lean_Syntax_node2(x_14, x_107, x_21, x_21); +x_109 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__72; lean_inc(x_21); -lean_inc(x_104); -lean_inc(x_99); +lean_inc(x_108); +lean_inc(x_103); lean_inc(x_14); -x_106 = l_Lean_Syntax_node4(x_14, x_105, x_99, x_102, x_104, x_21); -x_107 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__28; -lean_inc(x_106); +x_110 = l_Lean_Syntax_node4(x_14, x_109, x_103, x_106, x_108, x_21); +x_111 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__28; +lean_inc(x_110); lean_inc(x_46); lean_inc(x_14); -x_108 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_52, x_97, x_106); -x_109 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__9; +x_112 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_52, x_101, x_110); +x_113 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__9; lean_inc(x_44); lean_inc(x_14); -x_110 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_108); -x_111 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__79; -x_112 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__80; +x_114 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_112); +x_115 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__81; +x_116 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__82; lean_inc(x_14); -x_113 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_113, 0, x_14); -lean_ctor_set(x_113, 1, x_111); -lean_ctor_set(x_113, 2, x_112); -lean_ctor_set(x_113, 3, x_47); +x_117 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_117, 0, x_14); +lean_ctor_set(x_117, 1, x_115); +lean_ctor_set(x_117, 2, x_116); +lean_ctor_set(x_117, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_114 = l_Lean_Syntax_node2(x_14, x_51, x_113, x_21); -x_115 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__83; +x_118 = l_Lean_Syntax_node2(x_14, x_51, x_117, x_21); +x_119 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__85; lean_inc(x_14); -x_116 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_116, 0, x_14); -lean_ctor_set(x_116, 1, x_115); -x_117 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__82; +x_120 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_120, 0, x_14); +lean_ctor_set(x_120, 1, x_119); +x_121 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__84; lean_inc(x_60); -lean_inc(x_116); +lean_inc(x_120); lean_inc(x_57); lean_inc(x_14); -x_118 = l_Lean_Syntax_node3(x_14, x_117, x_57, x_116, x_60); -lean_inc(x_66); -lean_inc(x_54); -lean_inc(x_14); -x_119 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_118, x_66); -lean_inc(x_80); +x_122 = l_Lean_Syntax_node3(x_14, x_121, x_57, x_120, x_60); lean_inc(x_77); -lean_inc(x_119); -lean_inc(x_14); -x_120 = l_Lean_Syntax_node3(x_14, x_81, x_119, x_77, x_80); -lean_inc(x_90); -lean_inc(x_116); -lean_inc(x_87); +lean_inc(x_71); lean_inc(x_14); -x_121 = l_Lean_Syntax_node3(x_14, x_117, x_87, x_116, x_90); +x_123 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_122, x_77); lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_14); +x_124 = l_Lean_Syntax_node3(x_14, x_85, x_123, x_81, x_84); +lean_inc(x_94); +lean_inc(x_91); lean_inc(x_14); -x_122 = l_Lean_Syntax_node3(x_14, x_92, x_120, x_84, x_121); +x_125 = l_Lean_Syntax_node3(x_14, x_121, x_91, x_120, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_126 = l_Lean_Syntax_node3(x_14, x_96, x_124, x_88, x_125); lean_inc(x_63); lean_inc(x_14); -x_123 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_122); +x_127 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_126); lean_inc(x_69); lean_inc(x_14); -x_124 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_123); -lean_inc(x_106); +x_128 = l_Lean_Syntax_node2(x_14, x_100, x_69, x_127); +lean_inc(x_110); lean_inc(x_46); lean_inc(x_14); -x_125 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_114, x_124, x_106); +x_129 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_118, x_128, x_110); lean_inc(x_44); lean_inc(x_14); -x_126 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_125); -x_127 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__85; -x_128 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__86; +x_130 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_129); +x_131 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__87; +x_132 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__88; lean_inc(x_14); -x_129 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_129, 0, x_14); -lean_ctor_set(x_129, 1, x_127); -lean_ctor_set(x_129, 2, x_128); -lean_ctor_set(x_129, 3, x_47); +x_133 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_133, 0, x_14); +lean_ctor_set(x_133, 1, x_131); +lean_ctor_set(x_133, 2, x_132); +lean_ctor_set(x_133, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_130 = l_Lean_Syntax_node2(x_14, x_51, x_129, x_21); -x_131 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__89; +x_134 = l_Lean_Syntax_node2(x_14, x_51, x_133, x_21); +x_135 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__91; lean_inc(x_14); -x_132 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_132, 0, x_14); -lean_ctor_set(x_132, 1, x_131); -x_133 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__88; +x_136 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_136, 0, x_14); +lean_ctor_set(x_136, 1, x_135); +x_137 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__90; lean_inc(x_60); -lean_inc(x_132); +lean_inc(x_136); lean_inc(x_57); lean_inc(x_14); -x_134 = l_Lean_Syntax_node3(x_14, x_133, x_57, x_132, x_60); -lean_inc(x_66); -lean_inc(x_54); -lean_inc(x_14); -x_135 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_134, x_66); -lean_inc(x_80); +x_138 = l_Lean_Syntax_node3(x_14, x_137, x_57, x_136, x_60); lean_inc(x_77); -lean_inc(x_135); -lean_inc(x_14); -x_136 = l_Lean_Syntax_node3(x_14, x_81, x_135, x_77, x_80); -lean_inc(x_90); -lean_inc(x_132); -lean_inc(x_87); +lean_inc(x_71); lean_inc(x_14); -x_137 = l_Lean_Syntax_node3(x_14, x_133, x_87, x_132, x_90); +x_139 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_138, x_77); lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_14); +x_140 = l_Lean_Syntax_node3(x_14, x_85, x_139, x_81, x_84); +lean_inc(x_94); +lean_inc(x_91); +lean_inc(x_14); +x_141 = l_Lean_Syntax_node3(x_14, x_137, x_91, x_136, x_94); +lean_inc(x_88); lean_inc(x_14); -x_138 = l_Lean_Syntax_node3(x_14, x_92, x_136, x_84, x_137); +x_142 = l_Lean_Syntax_node3(x_14, x_96, x_140, x_88, x_141); lean_inc(x_63); lean_inc(x_14); -x_139 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_138); +x_143 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_142); lean_inc(x_69); lean_inc(x_14); -x_140 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_139); -lean_inc(x_106); +x_144 = l_Lean_Syntax_node2(x_14, x_100, x_69, x_143); +lean_inc(x_110); lean_inc(x_46); lean_inc(x_14); -x_141 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_130, x_140, x_106); +x_145 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_134, x_144, x_110); lean_inc(x_44); lean_inc(x_14); -x_142 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_141); -x_143 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__91; -x_144 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__92; +x_146 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_145); +x_147 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__93; +x_148 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__94; lean_inc(x_14); -x_145 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_145, 0, x_14); -lean_ctor_set(x_145, 1, x_143); -lean_ctor_set(x_145, 2, x_144); -lean_ctor_set(x_145, 3, x_47); +x_149 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_149, 0, x_14); +lean_ctor_set(x_149, 1, x_147); +lean_ctor_set(x_149, 2, x_148); +lean_ctor_set(x_149, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_146 = l_Lean_Syntax_node2(x_14, x_51, x_145, x_21); -x_147 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__95; +x_150 = l_Lean_Syntax_node2(x_14, x_51, x_149, x_21); +x_151 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__97; lean_inc(x_14); -x_148 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_148, 0, x_14); -lean_ctor_set(x_148, 1, x_147); -x_149 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__94; +x_152 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_152, 0, x_14); +lean_ctor_set(x_152, 1, x_151); +x_153 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__96; lean_inc(x_60); -lean_inc(x_148); +lean_inc(x_152); lean_inc(x_57); lean_inc(x_14); -x_150 = l_Lean_Syntax_node3(x_14, x_149, x_57, x_148, x_60); -lean_inc(x_66); -lean_inc(x_54); +x_154 = l_Lean_Syntax_node3(x_14, x_153, x_57, x_152, x_60); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_155 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_154, x_77); +lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_14); +x_156 = l_Lean_Syntax_node3(x_14, x_85, x_155, x_81, x_84); +lean_inc(x_94); +lean_inc(x_91); +lean_inc(x_14); +x_157 = l_Lean_Syntax_node3(x_14, x_153, x_91, x_152, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_158 = l_Lean_Syntax_node3(x_14, x_96, x_156, x_88, x_157); +lean_inc(x_63); +lean_inc(x_14); +x_159 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_158); +lean_inc(x_69); +lean_inc(x_14); +x_160 = l_Lean_Syntax_node2(x_14, x_100, x_69, x_159); +lean_inc(x_110); +lean_inc(x_46); +lean_inc(x_14); +x_161 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_150, x_160, x_110); +lean_inc(x_44); +lean_inc(x_14); +x_162 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_161); +x_163 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__99; +x_164 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__100; +lean_inc(x_14); +x_165 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_165, 0, x_14); +lean_ctor_set(x_165, 1, x_163); +lean_ctor_set(x_165, 2, x_164); +lean_ctor_set(x_165, 3, x_47); +lean_inc(x_21); lean_inc(x_14); -x_151 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_150, x_66); -lean_inc(x_80); +x_166 = l_Lean_Syntax_node2(x_14, x_51, x_165, x_21); +x_167 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__103; +lean_inc(x_14); +x_168 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_168, 0, x_14); +lean_ctor_set(x_168, 1, x_167); +x_169 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__102; +lean_inc(x_60); +lean_inc(x_168); +lean_inc(x_57); +lean_inc(x_14); +x_170 = l_Lean_Syntax_node3(x_14, x_169, x_57, x_168, x_60); lean_inc(x_77); -lean_inc(x_151); +lean_inc(x_71); lean_inc(x_14); -x_152 = l_Lean_Syntax_node3(x_14, x_81, x_151, x_77, x_80); -x_153 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__98; +x_171 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_170, x_77); +lean_inc(x_84); +lean_inc(x_81); lean_inc(x_14); -x_154 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_154, 0, x_14); -lean_ctor_set(x_154, 1, x_153); -x_155 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__97; -lean_inc(x_11); -lean_inc(x_154); +x_172 = l_Lean_Syntax_node3(x_14, x_85, x_171, x_81, x_84); +lean_inc(x_94); +lean_inc(x_168); +lean_inc(x_91); lean_inc(x_14); -x_156 = l_Lean_Syntax_node3(x_14, x_155, x_90, x_154, x_11); -lean_inc(x_66); -lean_inc(x_54); +x_173 = l_Lean_Syntax_node3(x_14, x_169, x_91, x_168, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_174 = l_Lean_Syntax_node3(x_14, x_96, x_172, x_88, x_173); +lean_inc(x_63); +lean_inc(x_14); +x_175 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_174); +lean_inc(x_14); +x_176 = l_Lean_Syntax_node2(x_14, x_100, x_69, x_175); +lean_inc(x_110); +lean_inc(x_46); +lean_inc(x_14); +x_177 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_166, x_176, x_110); +lean_inc(x_44); lean_inc(x_14); -x_157 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_156, x_66); -lean_inc(x_157); -lean_inc(x_148); -lean_inc(x_87); +x_178 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_177); +x_179 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__105; +x_180 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__106; +lean_inc(x_14); +x_181 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_181, 0, x_14); +lean_ctor_set(x_181, 1, x_179); +lean_ctor_set(x_181, 2, x_180); +lean_ctor_set(x_181, 3, x_47); +lean_inc(x_21); +lean_inc(x_14); +x_182 = l_Lean_Syntax_node2(x_14, x_51, x_181, x_21); +lean_inc(x_57); +lean_inc(x_14); +x_183 = l_Lean_Syntax_node1(x_14, x_19, x_57); +lean_inc(x_64); +lean_inc(x_14); +x_184 = l_Lean_Syntax_node4(x_14, x_67, x_54, x_183, x_64, x_66); +lean_inc(x_14); +x_185 = l_Lean_Syntax_node1(x_14, x_19, x_184); +x_186 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__109; lean_inc(x_14); -x_158 = l_Lean_Syntax_node3(x_14, x_149, x_87, x_148, x_157); +x_187 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_187, 0, x_14); +lean_ctor_set(x_187, 1, x_186); +x_188 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__108; +lean_inc(x_57); +lean_inc(x_187); +lean_inc(x_14); +x_189 = l_Lean_Syntax_node2(x_14, x_188, x_187, x_57); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_190 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_189, x_77); lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_14); +x_191 = l_Lean_Syntax_node3(x_14, x_85, x_190, x_81, x_84); +lean_inc(x_91); lean_inc(x_14); -x_159 = l_Lean_Syntax_node3(x_14, x_92, x_152, x_84, x_158); +x_192 = l_Lean_Syntax_node2(x_14, x_188, x_187, x_91); +lean_inc(x_88); +lean_inc(x_14); +x_193 = l_Lean_Syntax_node3(x_14, x_96, x_191, x_88, x_192); lean_inc(x_63); lean_inc(x_14); -x_160 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_159); -lean_inc(x_69); +x_194 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_193); lean_inc(x_14); -x_161 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_160); -lean_inc(x_106); +x_195 = l_Lean_Syntax_node2(x_14, x_100, x_185, x_194); +lean_inc(x_110); lean_inc(x_46); lean_inc(x_14); -x_162 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_146, x_161, x_106); +x_196 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_182, x_195, x_110); lean_inc(x_44); lean_inc(x_14); -x_163 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_162); -x_164 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__100; -x_165 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__101; +x_197 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_196); +x_198 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__111; +x_199 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__112; +lean_inc(x_14); +x_200 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_200, 0, x_14); +lean_ctor_set(x_200, 1, x_198); +lean_ctor_set(x_200, 2, x_199); +lean_ctor_set(x_200, 3, x_47); +lean_inc(x_21); lean_inc(x_14); -x_166 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_166, 0, x_14); -lean_ctor_set(x_166, 1, x_164); -lean_ctor_set(x_166, 2, x_165); -lean_ctor_set(x_166, 3, x_47); +x_201 = l_Lean_Syntax_node2(x_14, x_51, x_200, x_21); +x_202 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__114; +lean_inc(x_77); lean_inc(x_21); +lean_inc(x_71); lean_inc(x_14); -x_167 = l_Lean_Syntax_node2(x_14, x_51, x_166, x_21); -x_168 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__104; +x_203 = l_Lean_Syntax_node5(x_14, x_202, x_71, x_61, x_64, x_21, x_77); lean_inc(x_14); -x_169 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_169, 0, x_14); -lean_ctor_set(x_169, 1, x_168); -x_170 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__103; -lean_inc(x_169); +x_204 = l_Lean_Syntax_node1(x_14, x_19, x_203); +x_205 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__117; lean_inc(x_14); -x_171 = l_Lean_Syntax_node3(x_14, x_170, x_57, x_169, x_60); -lean_inc(x_66); -lean_inc(x_54); +x_206 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_206, 0, x_14); +lean_ctor_set(x_206, 1, x_205); +x_207 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__116; +lean_inc(x_60); +lean_inc(x_206); +lean_inc(x_57); lean_inc(x_14); -x_172 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_171, x_66); +x_208 = l_Lean_Syntax_node3(x_14, x_207, x_57, x_206, x_60); lean_inc(x_77); -lean_inc(x_172); +lean_inc(x_71); +lean_inc(x_14); +x_209 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_208, x_77); +lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_209); +lean_inc(x_14); +x_210 = l_Lean_Syntax_node3(x_14, x_85, x_209, x_81, x_84); +lean_inc(x_94); +lean_inc(x_206); +lean_inc(x_91); +lean_inc(x_14); +x_211 = l_Lean_Syntax_node3(x_14, x_207, x_91, x_206, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_212 = l_Lean_Syntax_node3(x_14, x_96, x_210, x_88, x_211); +lean_inc(x_63); lean_inc(x_14); -x_173 = l_Lean_Syntax_node3(x_14, x_81, x_172, x_77, x_80); -lean_inc(x_169); +x_213 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_212); +lean_inc(x_204); lean_inc(x_14); -x_174 = l_Lean_Syntax_node3(x_14, x_170, x_87, x_169, x_157); +x_214 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_213); +lean_inc(x_110); +lean_inc(x_46); +lean_inc(x_14); +x_215 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_201, x_214, x_110); +lean_inc(x_44); +lean_inc(x_14); +x_216 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_215); +x_217 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__119; +x_218 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__120; +lean_inc(x_14); +x_219 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_219, 0, x_14); +lean_ctor_set(x_219, 1, x_217); +lean_ctor_set(x_219, 2, x_218); +lean_ctor_set(x_219, 3, x_47); +lean_inc(x_21); +lean_inc(x_14); +x_220 = l_Lean_Syntax_node2(x_14, x_51, x_219, x_21); +x_221 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__123; +lean_inc(x_14); +x_222 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_222, 0, x_14); +lean_ctor_set(x_222, 1, x_221); +x_223 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__122; +lean_inc(x_60); +lean_inc(x_222); +lean_inc(x_57); +lean_inc(x_14); +x_224 = l_Lean_Syntax_node3(x_14, x_223, x_57, x_222, x_60); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_225 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_224, x_77); lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_225); +lean_inc(x_14); +x_226 = l_Lean_Syntax_node3(x_14, x_85, x_225, x_81, x_84); +lean_inc(x_94); +lean_inc(x_222); +lean_inc(x_91); lean_inc(x_14); -x_175 = l_Lean_Syntax_node3(x_14, x_92, x_173, x_84, x_174); +x_227 = l_Lean_Syntax_node3(x_14, x_223, x_91, x_222, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_228 = l_Lean_Syntax_node3(x_14, x_96, x_226, x_88, x_227); lean_inc(x_63); lean_inc(x_14); -x_176 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_175); -lean_inc(x_69); +x_229 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_228); +lean_inc(x_204); lean_inc(x_14); -x_177 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_176); +x_230 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_229); +lean_inc(x_110); lean_inc(x_46); lean_inc(x_14); -x_178 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_167, x_177, x_106); +x_231 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_220, x_230, x_110); lean_inc(x_44); lean_inc(x_14); -x_179 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_178); -x_180 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__106; -x_181 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__107; +x_232 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_231); +x_233 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__125; +x_234 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__126; lean_inc(x_14); -x_182 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_182, 0, x_14); -lean_ctor_set(x_182, 1, x_180); -lean_ctor_set(x_182, 2, x_181); -lean_ctor_set(x_182, 3, x_47); +x_235 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_235, 0, x_14); +lean_ctor_set(x_235, 1, x_233); +lean_ctor_set(x_235, 2, x_234); +lean_ctor_set(x_235, 3, x_47); lean_inc(x_21); -lean_inc(x_182); -lean_inc(x_14); -x_183 = l_Lean_Syntax_node2(x_14, x_51, x_182, x_21); -x_184 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__109; -x_185 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__110; -lean_inc(x_14); -x_186 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_186, 0, x_14); -lean_ctor_set(x_186, 1, x_184); -lean_ctor_set(x_186, 2, x_185); -lean_ctor_set(x_186, 3, x_47); -lean_inc(x_186); +lean_inc(x_14); +x_236 = l_Lean_Syntax_node2(x_14, x_51, x_235, x_21); +x_237 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__129; +lean_inc(x_14); +x_238 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_238, 0, x_14); +lean_ctor_set(x_238, 1, x_237); +x_239 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__128; +lean_inc(x_60); +lean_inc(x_238); +lean_inc(x_57); +lean_inc(x_14); +x_240 = l_Lean_Syntax_node3(x_14, x_239, x_57, x_238, x_60); lean_inc(x_77); +lean_inc(x_71); lean_inc(x_14); -x_187 = l_Lean_Syntax_node3(x_14, x_81, x_75, x_77, x_186); -x_188 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__112; -x_189 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__113; -lean_inc(x_14); -x_190 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_190, 0, x_14); -lean_ctor_set(x_190, 1, x_188); -lean_ctor_set(x_190, 2, x_189); -lean_ctor_set(x_190, 3, x_47); -x_191 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__115; -x_192 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__116; -lean_inc(x_14); -x_193 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_193, 0, x_14); -lean_ctor_set(x_193, 1, x_191); -lean_ctor_set(x_193, 2, x_192); -lean_ctor_set(x_193, 3, x_47); -lean_inc(x_193); -lean_inc(x_190); -lean_inc(x_14); -x_194 = l_Lean_Syntax_node3(x_14, x_72, x_190, x_71, x_193); +x_241 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_240, x_77); lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_241); +lean_inc(x_14); +x_242 = l_Lean_Syntax_node3(x_14, x_85, x_241, x_81, x_84); +lean_inc(x_94); +lean_inc(x_238); +lean_inc(x_91); lean_inc(x_14); -x_195 = l_Lean_Syntax_node3(x_14, x_92, x_187, x_84, x_194); +x_243 = l_Lean_Syntax_node3(x_14, x_239, x_91, x_238, x_94); +lean_inc(x_88); +lean_inc(x_14); +x_244 = l_Lean_Syntax_node3(x_14, x_96, x_242, x_88, x_243); lean_inc(x_63); lean_inc(x_14); -x_196 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_195); -lean_inc(x_69); +x_245 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_244); +lean_inc(x_204); +lean_inc(x_14); +x_246 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_245); +lean_inc(x_110); +lean_inc(x_46); +lean_inc(x_14); +x_247 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_236, x_246, x_110); +lean_inc(x_44); +lean_inc(x_14); +x_248 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_247); +x_249 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__131; +x_250 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__132; +lean_inc(x_14); +x_251 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_251, 0, x_14); +lean_ctor_set(x_251, 1, x_249); +lean_ctor_set(x_251, 2, x_250); +lean_ctor_set(x_251, 3, x_47); +lean_inc(x_21); +lean_inc(x_14); +x_252 = l_Lean_Syntax_node2(x_14, x_51, x_251, x_21); +x_253 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__135; +lean_inc(x_14); +x_254 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_254, 0, x_14); +lean_ctor_set(x_254, 1, x_253); +x_255 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__134; +lean_inc(x_60); +lean_inc(x_254); +lean_inc(x_57); +lean_inc(x_14); +x_256 = l_Lean_Syntax_node3(x_14, x_255, x_57, x_254, x_60); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_257 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_256, x_77); +lean_inc(x_84); +lean_inc(x_81); +lean_inc(x_257); +lean_inc(x_14); +x_258 = l_Lean_Syntax_node3(x_14, x_85, x_257, x_81, x_84); +lean_inc(x_11); +lean_inc(x_168); +lean_inc(x_14); +x_259 = l_Lean_Syntax_node3(x_14, x_169, x_94, x_168, x_11); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_260 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_259, x_77); +lean_inc(x_260); +lean_inc(x_254); +lean_inc(x_91); +lean_inc(x_14); +x_261 = l_Lean_Syntax_node3(x_14, x_255, x_91, x_254, x_260); +lean_inc(x_88); +lean_inc(x_14); +x_262 = l_Lean_Syntax_node3(x_14, x_96, x_258, x_88, x_261); +lean_inc(x_63); +lean_inc(x_14); +x_263 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_262); +lean_inc(x_204); +lean_inc(x_14); +x_264 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_263); +lean_inc(x_110); +lean_inc(x_46); +lean_inc(x_14); +x_265 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_252, x_264, x_110); +lean_inc(x_44); +lean_inc(x_14); +x_266 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_265); +x_267 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__137; +x_268 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__138; +lean_inc(x_14); +x_269 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_269, 0, x_14); +lean_ctor_set(x_269, 1, x_267); +lean_ctor_set(x_269, 2, x_268); +lean_ctor_set(x_269, 3, x_47); +lean_inc(x_21); +lean_inc(x_14); +x_270 = l_Lean_Syntax_node2(x_14, x_51, x_269, x_21); +x_271 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__141; +lean_inc(x_14); +x_272 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_272, 0, x_14); +lean_ctor_set(x_272, 1, x_271); +x_273 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__140; +lean_inc(x_272); +lean_inc(x_14); +x_274 = l_Lean_Syntax_node3(x_14, x_273, x_57, x_272, x_60); +lean_inc(x_77); +lean_inc(x_71); +lean_inc(x_14); +x_275 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_274, x_77); +lean_inc(x_81); +lean_inc(x_275); +lean_inc(x_14); +x_276 = l_Lean_Syntax_node3(x_14, x_85, x_275, x_81, x_84); +lean_inc(x_272); +lean_inc(x_14); +x_277 = l_Lean_Syntax_node3(x_14, x_273, x_91, x_272, x_260); +lean_inc(x_88); +lean_inc(x_14); +x_278 = l_Lean_Syntax_node3(x_14, x_96, x_276, x_88, x_277); +lean_inc(x_63); +lean_inc(x_14); +x_279 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_278); +lean_inc(x_204); +lean_inc(x_14); +x_280 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_279); +lean_inc(x_46); +lean_inc(x_14); +x_281 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_270, x_280, x_110); +lean_inc(x_44); +lean_inc(x_14); +x_282 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_281); +x_283 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__143; +x_284 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__144; +lean_inc(x_14); +x_285 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_285, 0, x_14); +lean_ctor_set(x_285, 1, x_283); +lean_ctor_set(x_285, 2, x_284); +lean_ctor_set(x_285, 3, x_47); +lean_inc(x_21); +lean_inc(x_285); +lean_inc(x_14); +x_286 = l_Lean_Syntax_node2(x_14, x_51, x_285, x_21); +x_287 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__146; +x_288 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__147; +lean_inc(x_14); +x_289 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_289, 0, x_14); +lean_ctor_set(x_289, 1, x_287); +lean_ctor_set(x_289, 2, x_288); +lean_ctor_set(x_289, 3, x_47); +lean_inc(x_289); +lean_inc(x_81); +lean_inc(x_14); +x_290 = l_Lean_Syntax_node3(x_14, x_85, x_209, x_81, x_289); +x_291 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149; +x_292 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__150; +lean_inc(x_14); +x_293 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_293, 0, x_14); +lean_ctor_set(x_293, 1, x_291); +lean_ctor_set(x_293, 2, x_292); +lean_ctor_set(x_293, 3, x_47); +x_294 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__152; +x_295 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__153; +lean_inc(x_14); +x_296 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_296, 0, x_14); +lean_ctor_set(x_296, 1, x_294); +lean_ctor_set(x_296, 2, x_295); +lean_ctor_set(x_296, 3, x_47); +lean_inc(x_296); +lean_inc(x_293); +lean_inc(x_14); +x_297 = l_Lean_Syntax_node3(x_14, x_207, x_293, x_206, x_296); +lean_inc(x_88); +lean_inc(x_14); +x_298 = l_Lean_Syntax_node3(x_14, x_96, x_290, x_88, x_297); +lean_inc(x_63); +lean_inc(x_14); +x_299 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_298); +lean_inc(x_204); lean_inc(x_14); -x_197 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_196); -x_198 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__119; +x_300 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_299); +x_301 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__156; lean_inc(x_14); -x_199 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_199, 0, x_14); -lean_ctor_set(x_199, 1, x_198); -x_200 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__127; +x_302 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_302, 0, x_14); +lean_ctor_set(x_302, 1, x_301); +x_303 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__164; lean_inc(x_21); lean_inc(x_14); -x_201 = l_Lean_Syntax_node1(x_14, x_200, x_21); -x_202 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__128; +x_304 = l_Lean_Syntax_node1(x_14, x_303, x_21); +x_305 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__165; lean_inc(x_14); -x_203 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_203, 0, x_14); -lean_ctor_set(x_203, 1, x_202); -x_204 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__130; -lean_inc(x_186); +x_306 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_306, 0, x_14); +lean_ctor_set(x_306, 1, x_305); +x_307 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__167; +lean_inc(x_289); lean_inc_n(x_21, 2); lean_inc(x_14); -x_205 = l_Lean_Syntax_node3(x_14, x_204, x_21, x_21, x_186); +x_308 = l_Lean_Syntax_node3(x_14, x_307, x_21, x_21, x_289); lean_inc(x_14); -x_206 = l_Lean_Syntax_node1(x_14, x_19, x_205); +x_309 = l_Lean_Syntax_node1(x_14, x_19, x_308); lean_inc(x_34); lean_inc(x_14); -x_207 = l_Lean_Syntax_node3(x_14, x_19, x_203, x_206, x_34); -x_208 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__125; +x_310 = l_Lean_Syntax_node3(x_14, x_19, x_306, x_309, x_34); +x_311 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__162; lean_inc_n(x_21, 3); lean_inc(x_14); -x_209 = l_Lean_Syntax_node6(x_14, x_208, x_27, x_201, x_21, x_21, x_207, x_21); +x_312 = l_Lean_Syntax_node6(x_14, x_311, x_27, x_304, x_21, x_21, x_310, x_21); lean_inc(x_14); -x_210 = l_Lean_Syntax_node1(x_14, x_19, x_209); -x_211 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__124; +x_313 = l_Lean_Syntax_node1(x_14, x_19, x_312); +x_314 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__161; lean_inc(x_14); -x_212 = l_Lean_Syntax_node1(x_14, x_211, x_210); -x_213 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__122; +x_315 = l_Lean_Syntax_node1(x_14, x_314, x_313); +x_316 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__159; lean_inc(x_14); -x_214 = l_Lean_Syntax_node1(x_14, x_213, x_212); -x_215 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__118; +x_317 = l_Lean_Syntax_node1(x_14, x_316, x_315); +x_318 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155; lean_inc(x_14); -x_216 = l_Lean_Syntax_node2(x_14, x_215, x_199, x_214); +x_319 = l_Lean_Syntax_node2(x_14, x_318, x_302, x_317); lean_inc(x_21); -lean_inc(x_104); -lean_inc(x_99); +lean_inc(x_108); +lean_inc(x_103); lean_inc(x_14); -x_217 = l_Lean_Syntax_node4(x_14, x_105, x_99, x_216, x_104, x_21); -lean_inc(x_217); -lean_inc(x_197); +x_320 = l_Lean_Syntax_node4(x_14, x_109, x_103, x_319, x_108, x_21); +lean_inc(x_320); +lean_inc(x_300); lean_inc(x_46); lean_inc(x_14); -x_218 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_183, x_197, x_217); +x_321 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_286, x_300, x_320); lean_inc(x_44); lean_inc(x_14); -x_219 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_218); -x_220 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__132; -x_221 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__133; +x_322 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_321); +x_323 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__169; +x_324 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__170; lean_inc(x_14); -x_222 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_222, 0, x_14); -lean_ctor_set(x_222, 1, x_220); -lean_ctor_set(x_222, 2, x_221); -lean_ctor_set(x_222, 3, x_47); +x_325 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_325, 0, x_14); +lean_ctor_set(x_325, 1, x_323); +lean_ctor_set(x_325, 2, x_324); +lean_ctor_set(x_325, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_223 = l_Lean_Syntax_node2(x_14, x_51, x_222, x_21); -lean_inc(x_186); -lean_inc(x_77); +x_326 = l_Lean_Syntax_node2(x_14, x_51, x_325, x_21); +lean_inc(x_289); +lean_inc(x_81); lean_inc(x_14); -x_224 = l_Lean_Syntax_node3(x_14, x_81, x_119, x_77, x_186); -lean_inc(x_193); -lean_inc(x_190); +x_327 = l_Lean_Syntax_node3(x_14, x_85, x_225, x_81, x_289); +lean_inc(x_296); +lean_inc(x_293); lean_inc(x_14); -x_225 = l_Lean_Syntax_node3(x_14, x_117, x_190, x_116, x_193); -lean_inc(x_84); +x_328 = l_Lean_Syntax_node3(x_14, x_223, x_293, x_222, x_296); +lean_inc(x_88); lean_inc(x_14); -x_226 = l_Lean_Syntax_node3(x_14, x_92, x_224, x_84, x_225); +x_329 = l_Lean_Syntax_node3(x_14, x_96, x_327, x_88, x_328); lean_inc(x_63); lean_inc(x_14); -x_227 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_226); -lean_inc(x_69); +x_330 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_329); +lean_inc(x_204); lean_inc(x_14); -x_228 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_227); -lean_inc(x_217); +x_331 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_330); +lean_inc(x_320); lean_inc(x_46); lean_inc(x_14); -x_229 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_223, x_228, x_217); +x_332 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_326, x_331, x_320); lean_inc(x_44); lean_inc(x_14); -x_230 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_229); -x_231 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__135; -x_232 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__136; +x_333 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_332); +x_334 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__172; +x_335 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173; lean_inc(x_14); -x_233 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_233, 0, x_14); -lean_ctor_set(x_233, 1, x_231); -lean_ctor_set(x_233, 2, x_232); -lean_ctor_set(x_233, 3, x_47); +x_336 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_336, 0, x_14); +lean_ctor_set(x_336, 1, x_334); +lean_ctor_set(x_336, 2, x_335); +lean_ctor_set(x_336, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_234 = l_Lean_Syntax_node2(x_14, x_51, x_233, x_21); -lean_inc(x_186); -lean_inc(x_77); +x_337 = l_Lean_Syntax_node2(x_14, x_51, x_336, x_21); +lean_inc(x_289); +lean_inc(x_81); lean_inc(x_14); -x_235 = l_Lean_Syntax_node3(x_14, x_81, x_135, x_77, x_186); -lean_inc(x_193); -lean_inc(x_190); +x_338 = l_Lean_Syntax_node3(x_14, x_85, x_241, x_81, x_289); +lean_inc(x_296); +lean_inc(x_293); lean_inc(x_14); -x_236 = l_Lean_Syntax_node3(x_14, x_133, x_190, x_132, x_193); -lean_inc(x_84); +x_339 = l_Lean_Syntax_node3(x_14, x_239, x_293, x_238, x_296); +lean_inc(x_88); lean_inc(x_14); -x_237 = l_Lean_Syntax_node3(x_14, x_92, x_235, x_84, x_236); +x_340 = l_Lean_Syntax_node3(x_14, x_96, x_338, x_88, x_339); lean_inc(x_63); lean_inc(x_14); -x_238 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_237); -lean_inc(x_69); +x_341 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_340); +lean_inc(x_204); lean_inc(x_14); -x_239 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_238); -lean_inc(x_217); +x_342 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_341); +lean_inc(x_320); lean_inc(x_46); lean_inc(x_14); -x_240 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_234, x_239, x_217); +x_343 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_337, x_342, x_320); lean_inc(x_44); lean_inc(x_14); -x_241 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_240); -x_242 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__138; -x_243 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__139; +x_344 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_343); +x_345 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175; +x_346 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176; lean_inc(x_14); -x_244 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_244, 0, x_14); -lean_ctor_set(x_244, 1, x_242); -lean_ctor_set(x_244, 2, x_243); -lean_ctor_set(x_244, 3, x_47); +x_347 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_347, 0, x_14); +lean_ctor_set(x_347, 1, x_345); +lean_ctor_set(x_347, 2, x_346); +lean_ctor_set(x_347, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_245 = l_Lean_Syntax_node2(x_14, x_51, x_244, x_21); -lean_inc(x_186); -lean_inc(x_77); +x_348 = l_Lean_Syntax_node2(x_14, x_51, x_347, x_21); +lean_inc(x_289); +lean_inc(x_81); lean_inc(x_14); -x_246 = l_Lean_Syntax_node3(x_14, x_81, x_151, x_77, x_186); +x_349 = l_Lean_Syntax_node3(x_14, x_85, x_257, x_81, x_289); lean_inc(x_11); -lean_inc(x_154); +lean_inc(x_168); lean_inc(x_14); -x_247 = l_Lean_Syntax_node3(x_14, x_155, x_193, x_154, x_11); -lean_inc(x_66); -lean_inc(x_54); +x_350 = l_Lean_Syntax_node3(x_14, x_169, x_296, x_168, x_11); +lean_inc(x_77); +lean_inc(x_71); lean_inc(x_14); -x_248 = l_Lean_Syntax_node3(x_14, x_74, x_54, x_247, x_66); -lean_inc(x_248); -lean_inc(x_190); +x_351 = l_Lean_Syntax_node3(x_14, x_78, x_71, x_350, x_77); +lean_inc(x_351); +lean_inc(x_293); lean_inc(x_14); -x_249 = l_Lean_Syntax_node3(x_14, x_149, x_190, x_148, x_248); -x_250 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__144; +x_352 = l_Lean_Syntax_node3(x_14, x_255, x_293, x_254, x_351); +x_353 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181; lean_inc(x_14); -x_251 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_251, 0, x_14); -lean_ctor_set(x_251, 1, x_250); -x_252 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__143; +x_354 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_354, 0, x_14); +lean_ctor_set(x_354, 1, x_353); +x_355 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180; lean_inc(x_14); -x_253 = l_Lean_Syntax_node1(x_14, x_252, x_251); -x_254 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__145; +x_356 = l_Lean_Syntax_node1(x_14, x_355, x_354); +x_357 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182; lean_inc(x_14); -x_255 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_255, 0, x_14); -lean_ctor_set(x_255, 1, x_254); -x_256 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__141; +x_358 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_358, 0, x_14); +lean_ctor_set(x_358, 1, x_357); +x_359 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178; lean_inc(x_14); -x_257 = l_Lean_Syntax_node3(x_14, x_256, x_253, x_255, x_11); +x_360 = l_Lean_Syntax_node3(x_14, x_359, x_356, x_358, x_11); lean_inc(x_14); -x_258 = l_Lean_Syntax_node3(x_14, x_155, x_249, x_154, x_257); -lean_inc(x_84); +x_361 = l_Lean_Syntax_node3(x_14, x_169, x_352, x_168, x_360); +lean_inc(x_88); lean_inc(x_14); -x_259 = l_Lean_Syntax_node3(x_14, x_92, x_246, x_84, x_258); +x_362 = l_Lean_Syntax_node3(x_14, x_96, x_349, x_88, x_361); lean_inc(x_63); lean_inc(x_14); -x_260 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_259); -lean_inc(x_69); +x_363 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_362); +lean_inc(x_204); lean_inc(x_14); -x_261 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_260); -lean_inc(x_217); +x_364 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_363); +lean_inc(x_320); lean_inc(x_46); lean_inc(x_14); -x_262 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_245, x_261, x_217); +x_365 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_348, x_364, x_320); lean_inc(x_44); lean_inc(x_14); -x_263 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_262); -x_264 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__147; -x_265 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__148; +x_366 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_365); +x_367 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184; +x_368 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185; lean_inc(x_14); -x_266 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_266, 0, x_14); -lean_ctor_set(x_266, 1, x_264); -lean_ctor_set(x_266, 2, x_265); -lean_ctor_set(x_266, 3, x_47); +x_369 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_369, 0, x_14); +lean_ctor_set(x_369, 1, x_367); +lean_ctor_set(x_369, 2, x_368); +lean_ctor_set(x_369, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_267 = l_Lean_Syntax_node2(x_14, x_51, x_266, x_21); +x_370 = l_Lean_Syntax_node2(x_14, x_51, x_369, x_21); lean_inc(x_14); -x_268 = l_Lean_Syntax_node3(x_14, x_81, x_172, x_77, x_186); +x_371 = l_Lean_Syntax_node3(x_14, x_85, x_275, x_81, x_289); lean_inc(x_14); -x_269 = l_Lean_Syntax_node3(x_14, x_170, x_190, x_169, x_248); +x_372 = l_Lean_Syntax_node3(x_14, x_273, x_293, x_272, x_351); lean_inc(x_14); -x_270 = l_Lean_Syntax_node3(x_14, x_92, x_268, x_84, x_269); +x_373 = l_Lean_Syntax_node3(x_14, x_96, x_371, x_88, x_372); lean_inc(x_14); -x_271 = l_Lean_Syntax_node2(x_14, x_94, x_63, x_270); +x_374 = l_Lean_Syntax_node2(x_14, x_98, x_63, x_373); lean_inc(x_14); -x_272 = l_Lean_Syntax_node2(x_14, x_96, x_69, x_271); +x_375 = l_Lean_Syntax_node2(x_14, x_100, x_204, x_374); lean_inc(x_46); lean_inc(x_14); -x_273 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_267, x_272, x_217); +x_376 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_370, x_375, x_320); lean_inc(x_14); -x_274 = l_Lean_Syntax_node2(x_14, x_109, x_44, x_273); -x_275 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__151; +x_377 = l_Lean_Syntax_node2(x_14, x_113, x_44, x_376); +x_378 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188; lean_inc(x_14); -x_276 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_276, 0, x_14); -lean_ctor_set(x_276, 1, x_275); +x_379 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_379, 0, x_14); +lean_ctor_set(x_379, 1, x_378); lean_inc(x_14); -x_277 = l_Lean_Syntax_node1(x_14, x_19, x_182); -x_278 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__154; -lean_inc(x_66); -lean_inc(x_277); -lean_inc(x_54); +x_380 = l_Lean_Syntax_node1(x_14, x_19, x_285); +x_381 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191; +lean_inc(x_77); +lean_inc(x_380); +lean_inc(x_71); lean_inc(x_9); lean_inc(x_14); -x_279 = l_Lean_Syntax_node4(x_14, x_278, x_9, x_54, x_277, x_66); -x_280 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__152; +x_382 = l_Lean_Syntax_node4(x_14, x_381, x_9, x_71, x_380, x_77); +x_383 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189; lean_inc(x_14); -x_281 = l_Lean_Syntax_node2(x_14, x_280, x_276, x_279); -x_282 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__149; +x_384 = l_Lean_Syntax_node2(x_14, x_383, x_379, x_382); +x_385 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186; lean_inc(x_14); -x_283 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_283, 0, x_14); -lean_ctor_set(x_283, 1, x_282); -x_284 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__155; +x_386 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_386, 0, x_14); +lean_ctor_set(x_386, 1, x_385); +x_387 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192; lean_inc(x_14); -x_285 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_285, 0, x_14); -lean_ctor_set(x_285, 1, x_284); -x_286 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__157; +x_388 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_388, 0, x_14); +lean_ctor_set(x_388, 1, x_387); +x_389 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194; lean_inc(x_14); -x_287 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_287, 0, x_14); -lean_ctor_set(x_287, 1, x_286); -x_288 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__160; +x_390 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_390, 0, x_14); +lean_ctor_set(x_390, 1, x_389); +x_391 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197; lean_inc(x_14); -x_289 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_289, 0, x_14); -lean_ctor_set(x_289, 1, x_288); -x_290 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__159; +x_392 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_392, 0, x_14); +lean_ctor_set(x_392, 1, x_391); +x_393 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196; lean_inc(x_14); -x_291 = l_Lean_Syntax_node1(x_14, x_290, x_289); -lean_inc(x_99); +x_394 = l_Lean_Syntax_node1(x_14, x_393, x_392); +lean_inc(x_103); lean_inc(x_14); -x_292 = l_Lean_Syntax_node5(x_14, x_19, x_54, x_287, x_99, x_291, x_66); -x_293 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__156; +x_395 = l_Lean_Syntax_node5(x_14, x_19, x_71, x_390, x_103, x_394, x_77); +x_396 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193; lean_inc(x_21); lean_inc(x_14); -x_294 = l_Lean_Syntax_node4(x_14, x_293, x_285, x_277, x_21, x_292); +x_397 = l_Lean_Syntax_node4(x_14, x_396, x_388, x_380, x_21, x_395); lean_inc(x_14); -x_295 = l_Lean_Syntax_node2(x_14, x_30, x_25, x_294); +x_398 = l_Lean_Syntax_node2(x_14, x_30, x_25, x_397); lean_inc(x_14); -x_296 = l_Lean_Syntax_node1(x_14, x_19, x_295); +x_399 = l_Lean_Syntax_node1(x_14, x_19, x_398); lean_inc(x_14); -x_297 = l_Lean_Syntax_node3(x_14, x_35, x_23, x_296, x_34); +x_400 = l_Lean_Syntax_node3(x_14, x_35, x_23, x_399, x_34); lean_inc(x_14); -x_298 = l_Lean_Syntax_node1(x_14, x_19, x_297); +x_401 = l_Lean_Syntax_node1(x_14, x_19, x_400); lean_inc_n(x_21, 4); lean_inc(x_14); -x_299 = l_Lean_Syntax_node6(x_14, x_43, x_21, x_298, x_42, x_21, x_21, x_21); -x_300 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__162; -x_301 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__163; +x_402 = l_Lean_Syntax_node6(x_14, x_43, x_21, x_401, x_42, x_21, x_21, x_21); +x_403 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199; +x_404 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200; lean_inc(x_14); -x_302 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_302, 0, x_14); -lean_ctor_set(x_302, 1, x_300); -lean_ctor_set(x_302, 2, x_301); -lean_ctor_set(x_302, 3, x_47); +x_405 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_405, 0, x_14); +lean_ctor_set(x_405, 1, x_403); +lean_ctor_set(x_405, 2, x_404); +lean_ctor_set(x_405, 3, x_47); lean_inc(x_21); lean_inc(x_14); -x_303 = l_Lean_Syntax_node2(x_14, x_51, x_302, x_21); -x_304 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__167; -x_305 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__169; -lean_inc(x_14); -x_306 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_306, 0, x_14); -lean_ctor_set(x_306, 1, x_304); -lean_ctor_set(x_306, 2, x_305); -lean_ctor_set(x_306, 3, x_47); -x_307 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__172; -lean_inc(x_14); -x_308 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_308, 0, x_14); -lean_ctor_set(x_308, 1, x_307); -x_309 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__171; -lean_inc(x_14); -x_310 = l_Lean_Syntax_node1(x_14, x_309, x_308); -lean_inc(x_14); -x_311 = l_Lean_Syntax_node1(x_14, x_19, x_310); -x_312 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__165; -lean_inc(x_14); -x_313 = l_Lean_Syntax_node2(x_14, x_312, x_306, x_311); -lean_inc(x_14); -x_314 = l_Lean_Syntax_node4(x_14, x_105, x_99, x_313, x_104, x_21); -lean_inc(x_14); -x_315 = l_Lean_Syntax_node4(x_14, x_107, x_46, x_303, x_197, x_314); -lean_inc(x_14); -x_316 = l_Lean_Syntax_node2(x_14, x_109, x_299, x_315); -x_317 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__150; -lean_inc(x_14); -x_318 = l_Lean_Syntax_node3(x_14, x_317, x_281, x_283, x_316); -x_319 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173; -lean_inc(x_14); -x_320 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_320, 0, x_14); -lean_ctor_set(x_320, 1, x_319); -lean_inc(x_14); -x_321 = l_Lean_Syntax_node1(x_14, x_19, x_9); -x_322 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174; -lean_inc(x_14); -x_323 = l_Lean_Syntax_node2(x_14, x_322, x_320, x_321); -x_324 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_324, 0, x_323); -lean_ctor_set(x_324, 1, x_47); -x_325 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_325, 0, x_318); -lean_ctor_set(x_325, 1, x_324); -x_326 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_326, 0, x_274); -lean_ctor_set(x_326, 1, x_325); -x_327 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_327, 0, x_263); -lean_ctor_set(x_327, 1, x_326); -x_328 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_328, 0, x_241); -lean_ctor_set(x_328, 1, x_327); -x_329 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_329, 0, x_230); -lean_ctor_set(x_329, 1, x_328); -x_330 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_330, 0, x_219); -lean_ctor_set(x_330, 1, x_329); -x_331 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_331, 0, x_179); -lean_ctor_set(x_331, 1, x_330); -x_332 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_332, 0, x_163); -lean_ctor_set(x_332, 1, x_331); -x_333 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_333, 0, x_142); -lean_ctor_set(x_333, 1, x_332); -x_334 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_334, 0, x_126); -lean_ctor_set(x_334, 1, x_333); -x_335 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_335, 0, x_110); -lean_ctor_set(x_335, 1, x_334); -x_336 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_336, 0, x_18); -lean_ctor_set(x_336, 1, x_335); -x_337 = lean_array_mk(x_336); -x_338 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_338, 0, x_14); -lean_ctor_set(x_338, 1, x_19); -lean_ctor_set(x_338, 2, x_337); -x_339 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_339, 0, x_338); -lean_ctor_set(x_339, 1, x_3); -return x_339; +x_406 = l_Lean_Syntax_node2(x_14, x_51, x_405, x_21); +x_407 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204; +x_408 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206; +lean_inc(x_14); +x_409 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_409, 0, x_14); +lean_ctor_set(x_409, 1, x_407); +lean_ctor_set(x_409, 2, x_408); +lean_ctor_set(x_409, 3, x_47); +x_410 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209; +lean_inc(x_14); +x_411 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_411, 0, x_14); +lean_ctor_set(x_411, 1, x_410); +x_412 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208; +lean_inc(x_14); +x_413 = l_Lean_Syntax_node1(x_14, x_412, x_411); +lean_inc(x_14); +x_414 = l_Lean_Syntax_node1(x_14, x_19, x_413); +x_415 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202; +lean_inc(x_14); +x_416 = l_Lean_Syntax_node2(x_14, x_415, x_409, x_414); +lean_inc(x_14); +x_417 = l_Lean_Syntax_node4(x_14, x_109, x_103, x_416, x_108, x_21); +lean_inc(x_14); +x_418 = l_Lean_Syntax_node4(x_14, x_111, x_46, x_406, x_300, x_417); +lean_inc(x_14); +x_419 = l_Lean_Syntax_node2(x_14, x_113, x_402, x_418); +x_420 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187; +lean_inc(x_14); +x_421 = l_Lean_Syntax_node3(x_14, x_420, x_384, x_386, x_419); +x_422 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210; +lean_inc(x_14); +x_423 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_423, 0, x_14); +lean_ctor_set(x_423, 1, x_422); +lean_inc(x_14); +x_424 = l_Lean_Syntax_node1(x_14, x_19, x_9); +x_425 = l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211; +lean_inc(x_14); +x_426 = l_Lean_Syntax_node2(x_14, x_425, x_423, x_424); +x_427 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_427, 0, x_426); +lean_ctor_set(x_427, 1, x_47); +x_428 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_428, 0, x_421); +lean_ctor_set(x_428, 1, x_427); +x_429 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_429, 0, x_377); +lean_ctor_set(x_429, 1, x_428); +x_430 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_430, 0, x_366); +lean_ctor_set(x_430, 1, x_429); +x_431 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_431, 0, x_344); +lean_ctor_set(x_431, 1, x_430); +x_432 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_432, 0, x_333); +lean_ctor_set(x_432, 1, x_431); +x_433 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_433, 0, x_322); +lean_ctor_set(x_433, 1, x_432); +x_434 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_434, 0, x_282); +lean_ctor_set(x_434, 1, x_433); +x_435 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_435, 0, x_266); +lean_ctor_set(x_435, 1, x_434); +x_436 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_436, 0, x_248); +lean_ctor_set(x_436, 1, x_435); +x_437 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_437, 0, x_232); +lean_ctor_set(x_437, 1, x_436); +x_438 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_438, 0, x_216); +lean_ctor_set(x_438, 1, x_437); +x_439 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_439, 0, x_197); +lean_ctor_set(x_439, 1, x_438); +x_440 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_440, 0, x_178); +lean_ctor_set(x_440, 1, x_439); +x_441 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_441, 0, x_162); +lean_ctor_set(x_441, 1, x_440); +x_442 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_442, 0, x_146); +lean_ctor_set(x_442, 1, x_441); +x_443 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_443, 0, x_130); +lean_ctor_set(x_443, 1, x_442); +x_444 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_444, 0, x_114); +lean_ctor_set(x_444, 1, x_443); +x_445 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_445, 0, x_18); +lean_ctor_set(x_445, 1, x_444); +x_446 = lean_array_mk(x_445); +x_447 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_447, 0, x_14); +lean_ctor_set(x_447, 1, x_19); +lean_ctor_set(x_447, 2, x_446); +x_448 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_448, 0, x_447); +lean_ctor_set(x_448, 1, x_3); +return x_448; } } } @@ -3288,6 +3989,80 @@ l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uin lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__173); l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174(); lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__174); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__175); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__176); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__177); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__178); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__179); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__180); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__181); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__182); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__183); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__184); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__185); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__186); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__187); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__188); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__189); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__190); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__191); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__192); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__193); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__194); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__195); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__196); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__197); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__198); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__199); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__200); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__201); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__202); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__203); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__204); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__205); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__206); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__207); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__208); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__209); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__210); +l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211 = _init_l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211(); +lean_mark_persistent(l___aux__Init__Data__UInt__Bitwise______macroRules__commandDeclare__bitwise__uint__theorems______1___closed__211); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Data/Vector/Basic.c b/stage0/stdlib/Init/Data/Vector/Basic.c index d9cb8ca75d85..8118e368c23e 100644 --- a/stage0/stdlib/Init/Data/Vector/Basic.c +++ b/stage0/stdlib/Init/Data/Vector/Basic.c @@ -16,37 +16,40 @@ extern "C" { LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_map___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__2; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__28; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28; LEAN_EXPORT lean_object* l_Vector_instMembership(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_singleton(lean_object*); static lean_object* l_Vector_lex___rarg___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_uget___rarg(lean_object*, size_t, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__2; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27; LEAN_EXPORT lean_object* l_Vector_drop___boxed(lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__2; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__28; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__20; lean_object* l_Array_take___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Vector_instBEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__36; uint8_t l_Array_isEqvAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1(lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__20; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__19; lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__31; LEAN_EXPORT lean_object* l_Vector_map___rarg(lean_object*, lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__9; LEAN_EXPORT lean_object* l_Vector_isEqv(lean_object*); LEAN_EXPORT lean_object* l_Vector_back_x21___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_mkVector___rarg(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26; LEAN_EXPORT lean_object* l_Vector_back_x3f___rarg___boxed(lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__17; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__22; LEAN_EXPORT lean_object* l_Vector_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_any___spec__1(lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__30; LEAN_EXPORT lean_object* l_Vector_range___boxed(lean_object*); LEAN_EXPORT uint8_t l_Vector_any___rarg(lean_object*, lean_object*); @@ -58,7 +61,6 @@ static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init LEAN_EXPORT lean_object* l_Vector_foldl(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__10; LEAN_EXPORT lean_object* l_Vector_set_x21___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24; LEAN_EXPORT lean_object* l_Array_toVector___rarg(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Vector_foldr___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_lex___rarg___closed__2; @@ -70,6 +72,7 @@ static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__V LEAN_EXPORT lean_object* l_instReprVector___rarg(lean_object*); lean_object* lean_array_fswap(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_instReprVector___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__24; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__2; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__1; @@ -81,21 +84,19 @@ lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_back_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Vector_foldr___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_toVector(lean_object*); +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1980_; LEAN_EXPORT lean_object* l_Vector_get(lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__14; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__25; LEAN_EXPORT lean_object* l_Vector_swap___boxed(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21; LEAN_EXPORT lean_object* l_Vector_swap___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__19; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__8; LEAN_EXPORT lean_object* l_Vector_reverse___boxed(lean_object*, lean_object*); lean_object* l_Lean_Syntax_getArgs(lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1599_; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__13; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19; LEAN_EXPORT lean_object* l_Vector_foldrM___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_swap(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__7; @@ -111,12 +112,12 @@ LEAN_EXPORT uint8_t l_Array_isEqvAux___at_Vector_instBEq___spec__1___rarg(lean_o LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_any___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__4; lean_object* l_Lean_Syntax_TSepArray_getElems___rarg(lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__25; LEAN_EXPORT uint8_t l_Vector_contains___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instGetElemNatLt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_all(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33; LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__decEqVector____x40_Init_Data_Vector_Basic___hyg_98____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__40; @@ -125,18 +126,16 @@ LEAN_EXPORT lean_object* l_Vector_instLE___boxed(lean_object*, lean_object*, lea LEAN_EXPORT lean_object* l_Vector_foldrM(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__16; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_eraseIdx(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1650_; lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_uget___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20; LEAN_EXPORT lean_object* l_Vector_singleton___rarg(lean_object*); LEAN_EXPORT lean_object* l_Vector_contains(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__13; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Vector_foldr___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3; LEAN_EXPORT lean_object* l_Vector_all___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Vector_instBEq___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Vector_instLT___boxed(lean_object*, lean_object*, lean_object*); @@ -144,10 +143,8 @@ LEAN_EXPORT lean_object* l_Vector_instGetElemNatLt___boxed(lean_object*, lean_ob static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__14; LEAN_EXPORT lean_object* l_Vector_any___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_indexOf_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1929_; LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_anyM___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5; LEAN_EXPORT lean_object* l_Vector_extract(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_tail___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_setIfInBounds(lean_object*, lean_object*); @@ -157,36 +154,38 @@ static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__V static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__32; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__11; LEAN_EXPORT lean_object* l_Vector_cast___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1724_; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_all___spec__1(lean_object*); LEAN_EXPORT uint8_t l_Vector_isPrefixOf___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_foldl___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_mkEmpty___rarg(lean_object*); LEAN_EXPORT lean_object* l_Vector_elimAsArray___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__decEqVector____x40_Init_Data_Vector_Basic___hyg_98_(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8; LEAN_EXPORT lean_object* l_Vector_instHAppendHAddNat___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_head___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_range___lambda__1___boxed(lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_allM___spec__1___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swapAt(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Vector_any___spec__1___rarg(lean_object*, lean_object*, size_t, size_t); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24; LEAN_EXPORT lean_object* l_Vector_map___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swapIfInBounds___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__8; static lean_object* l_Vector_swapAt_x21___rarg___closed__3; LEAN_EXPORT lean_object* l_instReprVector(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9; LEAN_EXPORT lean_object* l_Vector_foldr(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_back(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__8; lean_object* l_Array_reverse___rarg(lean_object*); LEAN_EXPORT lean_object* l_Vector_getD___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__7; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9; LEAN_EXPORT lean_object* l_Vector_pop(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_uget___boxed(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29; LEAN_EXPORT lean_object* l_Vector_extract___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13; LEAN_EXPORT lean_object* l_Vector_allM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_foldl___rarg(lean_object*, lean_object*, lean_object*); @@ -205,6 +204,9 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_map___spec__1___rarg LEAN_EXPORT lean_object* l_Vector_contains___boxed(lean_object*, lean_object*); lean_object* l_Array_ofFn___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_all___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__4; LEAN_EXPORT lean_object* l_Vector_cast___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Vector_extract___boxed(lean_object*, lean_object*); @@ -212,6 +214,7 @@ static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed_ LEAN_EXPORT lean_object* l_Vector_set___boxed(lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__10; LEAN_EXPORT lean_object* l_Vector_elimAsArray(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403_; LEAN_EXPORT lean_object* l_Vector_contains___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____spec__2(lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__5; @@ -221,27 +224,25 @@ LEAN_EXPORT lean_object* l_Vector_isPrefixOf___rarg___boxed(lean_object*, lean_o LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Vector_foldr___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swap___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__10; +LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1642_; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_foldl___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Array_back_x3f___rarg(lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30; LEAN_EXPORT lean_object* l_panic___at_Vector_swapAt_x21___spec__1___boxed(lean_object*, lean_object*); lean_object* lean_array_pop(lean_object*); LEAN_EXPORT lean_object* l_Vector_reverse(lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__1; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__27; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13; LEAN_EXPORT lean_object* l_Vector_zipWith___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__9; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__16; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_map(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_allM___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_take___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_getD(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__8; LEAN_EXPORT lean_object* l_Vector_anyM___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_set_x21(lean_object*, lean_object*); @@ -262,20 +263,20 @@ static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init LEAN_EXPORT uint8_t l_Vector_lex___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Vector_ofFn___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__24; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_eraseIdx_x21___rarg___closed__4; LEAN_EXPORT lean_object* l_Vector_elimAsList___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instInhabited___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_get___rarg___boxed(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10; LEAN_EXPORT lean_object* l_Vector_foldl___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_foldr___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_swapAt_x21___rarg___closed__1; LEAN_EXPORT lean_object* l_Vector_drop___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352_; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__13; LEAN_EXPORT lean_object* l_Vector_elimAsArray___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_lex___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -284,24 +285,24 @@ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_eraseIdx_x21(lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_lex___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12; static lean_object* l_Vector_swapAt_x21___rarg___closed__4; LEAN_EXPORT lean_object* l_Vector_back_x3f___rarg(lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__26; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__5; LEAN_EXPORT lean_object* l_Vector_swapAt_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23; static lean_object* l_Vector_eraseIdx_x21___rarg___closed__2; LEAN_EXPORT lean_object* l_Vector_set___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__17; lean_object* l_Array_indexOfAux___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1591_; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__7; LEAN_EXPORT lean_object* l_Vector_back_x21___rarg___boxed(lean_object*, lean_object*); lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_take___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_any(lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__3; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Vector_indexOf_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_foldlM___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_head___rarg(lean_object*); @@ -322,11 +323,11 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Vector_foldr___spec__2__ LEAN_EXPORT lean_object* l_Vector_instLE(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__3; LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__decEqVector____x40_Init_Data_Vector_Basic___hyg_98____rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__3; lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_allM___spec__1___rarg___lambda__1(lean_object*, uint8_t); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__39; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_allM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Vector_extract___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_foldl___boxed(lean_object*, lean_object*, lean_object*); @@ -334,7 +335,6 @@ LEAN_EXPORT lean_object* l_Vector_lex___rarg___lambda__1___boxed(lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__2; LEAN_EXPORT lean_object* l_Vector_getD___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instGetElemNatLt___rarg___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11; LEAN_EXPORT lean_object* l_Vector_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instBEq___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_push___boxed(lean_object*, lean_object*); @@ -342,9 +342,9 @@ LEAN_EXPORT uint8_t l_instDecidableEqVector___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_panic___at_Vector_eraseIdx_x21___spec__1___boxed(lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__3; static lean_object* l_Vector_eraseIdx_x21___rarg___closed__3; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16; static lean_object* l_Vector_swapAt_x21___rarg___closed__2; static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__31; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2; LEAN_EXPORT lean_object* l_Array_isEqvAux___at_Vector_instBEq___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_any___rarg___boxed(lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__22; @@ -356,15 +356,16 @@ lean_object* lean_string_length(lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__21; LEAN_EXPORT lean_object* l_Vector_allM___rarg(lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29; uint8_t l_Array_contains___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__23; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Vector_instHAppendHAddNat___closed__1; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__33; -LEAN_EXPORT lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1673_; LEAN_EXPORT lean_object* l_Vector_isPrefixOf(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swapIfInBounds(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1; LEAN_EXPORT lean_object* l_Vector_foldlM(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__10; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__6; @@ -374,21 +375,21 @@ static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__V LEAN_EXPORT lean_object* l_Array_toVector___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Vector_cast(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__17; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swapAt___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__21; lean_object* lean_panic_fn(lean_object*, lean_object*); uint8_t l_Array_instDecidableEq___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6; static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__4; lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_isEqv___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__11; +LEAN_EXPORT lean_object* l_Vector_flatten___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_back_x21___rarg(lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__38; static lean_object* l_Vector_range___closed__1; LEAN_EXPORT lean_object* l_Vector_append___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__7; LEAN_EXPORT lean_object* l_Vector_tail___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__5; @@ -398,6 +399,8 @@ LEAN_EXPORT lean_object* l_Vector_mkEmpty___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Vector_set___rarg(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__15; LEAN_EXPORT lean_object* l_panic___at_Vector_eraseIdx_x21___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_setIfInBounds___boxed(lean_object*, lean_object*); @@ -410,12 +413,12 @@ LEAN_EXPORT lean_object* l_Vector_allM___boxed(lean_object*, lean_object*, lean_ static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__35; LEAN_EXPORT lean_object* l_instDecidableEqVector(lean_object*, lean_object*); lean_object* l_Array_foldrMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23; LEAN_EXPORT lean_object* l_Vector_back___rarg___boxed(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__27; LEAN_EXPORT lean_object* l_Vector_reverse___rarg(lean_object*); size_t lean_array_size(lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18; lean_object* l_Array_foldlMUnsafe_fold___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_instDecidableEqVector___boxed(lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__11; @@ -435,35 +438,39 @@ LEAN_EXPORT lean_object* l_Vector_zipWith___rarg___boxed(lean_object*, lean_obje static lean_object* l_Vector_eraseIdx_x21___rarg___closed__1; LEAN_EXPORT lean_object* l_Vector_instMembership___boxed(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25; LEAN_EXPORT lean_object* l_Vector_indexOf_x3f___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_append___rarg___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Vector_flatten(lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__5; LEAN_EXPORT lean_object* l_Vector_set(lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_swap(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instGetElemNatLt___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15; uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Vector_ofFn(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__1; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__3; static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__15; static lean_object* l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__4; -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2(lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17; LEAN_EXPORT lean_object* l_Vector_setIfInBounds___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__18; LEAN_EXPORT lean_object* l_Std_Format_joinSep___at___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_zipWith(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__12; LEAN_EXPORT lean_object* l_Vector_range(lean_object*); -static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17; +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5; static lean_object* l_Vector_term_x23v_x5b___x2c_x5d___closed__17; LEAN_EXPORT lean_object* l_Vector_mkEmpty(lean_object*); LEAN_EXPORT lean_object* l_Vector_eraseIdx_x21___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_push___rarg(lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20; LEAN_EXPORT lean_object* l_Vector_back_x21___rarg(lean_object*, lean_object*); lean_object* l_String_toSubstring_x27(lean_object*); LEAN_EXPORT lean_object* l_Vector_back___rarg(lean_object*); @@ -473,8 +480,10 @@ lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); LEAN_EXPORT lean_object* l_Vector_anyM(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Init_Data_Vector_Basic_0__reprVector____x40_Init_Data_Vector_Basic___hyg_32____rarg___closed__13; LEAN_EXPORT lean_object* l_Vector_elimAsList(lean_object*, lean_object*, lean_object*); +static lean_object* l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4; LEAN_EXPORT lean_object* l_Vector_mkVector(lean_object*); LEAN_EXPORT lean_object* l_Vector_append___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Vector_flatten___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Vector_allM___spec__1___rarg___lambda__2(size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, uint8_t); LEAN_EXPORT lean_object* l_Vector_drop___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Vector_instLT(lean_object*, lean_object*, lean_object*); @@ -3300,6 +3309,156 @@ lean_dec(x_3); return x_4; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = 1; +x_10 = lean_usize_add(x_3, x_9); +x_11 = lean_array_uset(x_8, x_3, x_6); +x_3 = x_10; +x_4 = x_11; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; +x_6 = lean_array_uget(x_1, x_2); +x_7 = l_Array_append___rarg(x_4, x_6); +lean_dec(x_6); +x_8 = 1; +x_9 = lean_usize_add(x_2, x_8); +x_2 = x_9; +x_4 = x_7; +goto _start; +} +else +{ +return x_4; +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Vector_flatten___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_4 = lean_array_size(x_3); +x_5 = 0; +x_6 = l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg(x_1, x_4, x_5, x_3); +x_7 = lean_array_get_size(x_6); +x_8 = lean_unsigned_to_nat(0u); +x_9 = lean_nat_dec_lt(x_8, x_7); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +x_10 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; +return x_10; +} +else +{ +uint8_t x_11; +x_11 = lean_nat_dec_le(x_7, x_7); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_7); +lean_dec(x_6); +x_12 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; +return x_12; +} +else +{ +size_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_usize_of_nat(x_7); +lean_dec(x_7); +x_14 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; +x_15 = l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg(x_6, x_5, x_13, x_14); +lean_dec(x_6); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Vector_flatten(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Vector_flatten___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at_Vector_flatten___spec__1___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Vector_flatten___spec__2___rarg(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Vector_flatten___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Vector_flatten___rarg(x_1, x_2, x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +} static lean_object* _init_l_Vector_zipWith___rarg___closed__1() { _start: { @@ -3363,7 +3522,7 @@ lean_dec(x_1); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1591_() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1642_() { _start: { lean_object* x_1; @@ -3371,7 +3530,7 @@ x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__17; return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1599_() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1650_() { _start: { lean_object* x_1; @@ -3449,7 +3608,7 @@ lean_dec(x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1673_() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1724_() { _start: { lean_object* x_1; @@ -3564,7 +3723,7 @@ x_10 = l_Vector_swapAt_x21___rarg___closed__2; x_11 = lean_string_append(x_9, x_10); x_12 = l_Vector_swapAt_x21___rarg___closed__3; x_13 = l_Vector_swapAt_x21___rarg___closed__4; -x_14 = lean_unsigned_to_nat(272u); +x_14 = lean_unsigned_to_nat(271u); x_15 = lean_unsigned_to_nat(4u); x_16 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_12, x_13, x_14, x_15, x_11); lean_dec(x_11); @@ -3869,7 +4028,7 @@ lean_dec(x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1929_() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1980_() { _start: { lean_object* x_1; @@ -3949,7 +4108,7 @@ static lean_object* _init_l_Vector_eraseIdx_x21___rarg___closed__4() { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Vector_eraseIdx_x21___rarg___closed__1; x_2 = l_Vector_eraseIdx_x21___rarg___closed__2; -x_3 = lean_unsigned_to_nat(261u); +x_3 = lean_unsigned_to_nat(265u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Vector_eraseIdx_x21___rarg___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4675,7 +4834,7 @@ lean_dec(x_2); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1() { _start: { lean_object* x_1; @@ -4683,41 +4842,41 @@ x_1 = lean_mk_string_unchecked("exact", 5, 5); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__1; x_2 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__2; x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__1; -x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1; +x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1; x_3 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5() { _start: { lean_object* x_1; @@ -4725,19 +4884,19 @@ x_1 = lean_mk_string_unchecked("paren", 5, 5); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__1; x_2 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__2; x_3 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__3; -x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5; +x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -4749,17 +4908,17 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9() { _start: { lean_object* x_1; @@ -4767,17 +4926,17 @@ x_1 = lean_mk_string_unchecked("term_<_", 7, 7); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11() { _start: { lean_object* x_1; @@ -4785,19 +4944,19 @@ x_1 = lean_mk_string_unchecked("cdot", 4, 4); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__1; x_2 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__2; x_3 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__3; -x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11; +x_4 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13() { _start: { lean_object* x_1; @@ -4805,35 +4964,35 @@ x_1 = lean_mk_string_unchecked("·", 2, 1); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13; x_3 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -4841,17 +5000,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18() { _start: { lean_object* x_1; @@ -4859,45 +5018,45 @@ x_1 = lean_mk_string_unchecked("<", 1, 1); return x_1; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18; x_3 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -4905,17 +5064,17 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -4927,23 +5086,23 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -4951,23 +5110,23 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -4975,23 +5134,23 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); x_2 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__15; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -4999,23 +5158,23 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__5; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -5023,23 +5182,23 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Vector___aux__Init__Data__Vector__Basic______macroRules__Vector__term_x23v_x5b___x2c_x5d__1___closed__26; -x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32; +x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32; x_3 = lean_array_push(x_1, x_2); return x_3; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = lean_box(2); x_2 = l___auto____x40_Init_Data_Vector_Basic___hyg_1091____closed__3; -x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33; +x_3 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33; x_4 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -5047,11 +5206,11 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352_() { +static lean_object* _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403_() { _start: { lean_object* x_1; -x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34; +x_1 = l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34; return x_1; } } @@ -5535,12 +5694,12 @@ l_Vector_instHAppendHAddNat___closed__1 = _init_l_Vector_instHAppendHAddNat___cl lean_mark_persistent(l_Vector_instHAppendHAddNat___closed__1); l_Vector_zipWith___rarg___closed__1 = _init_l_Vector_zipWith___rarg___closed__1(); lean_mark_persistent(l_Vector_zipWith___rarg___closed__1); -l___auto____x40_Init_Data_Vector_Basic___hyg_1591_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1591_(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1591_); -l___auto____x40_Init_Data_Vector_Basic___hyg_1599_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1599_(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1599_); -l___auto____x40_Init_Data_Vector_Basic___hyg_1673_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1673_(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1673_); +l___auto____x40_Init_Data_Vector_Basic___hyg_1642_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1642_(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1642_); +l___auto____x40_Init_Data_Vector_Basic___hyg_1650_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1650_(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1650_); +l___auto____x40_Init_Data_Vector_Basic___hyg_1724_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1724_(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1724_); l_Vector_swapAt_x21___rarg___closed__1 = _init_l_Vector_swapAt_x21___rarg___closed__1(); lean_mark_persistent(l_Vector_swapAt_x21___rarg___closed__1); l_Vector_swapAt_x21___rarg___closed__2 = _init_l_Vector_swapAt_x21___rarg___closed__2(); @@ -5551,8 +5710,8 @@ l_Vector_swapAt_x21___rarg___closed__4 = _init_l_Vector_swapAt_x21___rarg___clos lean_mark_persistent(l_Vector_swapAt_x21___rarg___closed__4); l_Vector_range___closed__1 = _init_l_Vector_range___closed__1(); lean_mark_persistent(l_Vector_range___closed__1); -l___auto____x40_Init_Data_Vector_Basic___hyg_1929_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1929_(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1929_); +l___auto____x40_Init_Data_Vector_Basic___hyg_1980_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_1980_(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_1980_); l_Vector_eraseIdx_x21___rarg___closed__1 = _init_l_Vector_eraseIdx_x21___rarg___closed__1(); lean_mark_persistent(l_Vector_eraseIdx_x21___rarg___closed__1); l_Vector_eraseIdx_x21___rarg___closed__2 = _init_l_Vector_eraseIdx_x21___rarg___closed__2(); @@ -5561,76 +5720,76 @@ l_Vector_eraseIdx_x21___rarg___closed__3 = _init_l_Vector_eraseIdx_x21___rarg___ lean_mark_persistent(l_Vector_eraseIdx_x21___rarg___closed__3); l_Vector_eraseIdx_x21___rarg___closed__4 = _init_l_Vector_eraseIdx_x21___rarg___closed__4(); lean_mark_persistent(l_Vector_eraseIdx_x21___rarg___closed__4); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__1); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__2); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__3); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__4); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__5); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__6); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__7); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__8); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__9); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__10); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__11); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__12); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__13); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__14); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__15); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__16); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__17); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__18); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__19); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__20); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__21); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__22); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__23); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__24); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__25); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__26); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__27); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__28); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__29); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__30); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__31); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__32); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__33); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352____closed__34); -l___auto____x40_Init_Data_Vector_Basic___hyg_2352_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2352_(); -lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2352_); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__1); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__2); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__3); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__4); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__5); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__6); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__7); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__8); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__9); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__10); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__11); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__12); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__13); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__14); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__15); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__16); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__17); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__18); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__19); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__20); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__21); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__22); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__23); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__24); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__25); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__26); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__27); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__28); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__29); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__30); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__31); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__32); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__33); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34 = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403____closed__34); +l___auto____x40_Init_Data_Vector_Basic___hyg_2403_ = _init_l___auto____x40_Init_Data_Vector_Basic___hyg_2403_(); +lean_mark_persistent(l___auto____x40_Init_Data_Vector_Basic___hyg_2403_); l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__1 = _init_l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__1(); lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__1); l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__2 = _init_l_Std_Range_forIn_x27_loop___at_Vector_lex___spec__1___rarg___closed__2(); diff --git a/stage0/stdlib/Init/Data/Vector/Lemmas.c b/stage0/stdlib/Init/Data/Vector/Lemmas.c index cc18c411afa8..27ab46a19777 100644 --- a/stage0/stdlib/Init/Data/Vector/Lemmas.c +++ b/stage0/stdlib/Init/Data/Vector/Lemmas.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Data.Vector.Lemmas -// Imports: Init.Data.Vector.Basic +// Imports: Init.Data.Vector.Basic Init.Data.Array.Attach #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -278,6 +278,7 @@ return x_4; } } lean_object* initialize_Init_Data_Vector_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Data_Array_Attach(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Data_Vector_Lemmas(uint8_t builtin, lean_object* w) { lean_object * res; @@ -286,6 +287,9 @@ _G_initialized = true; res = initialize_Init_Data_Vector_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Data_Array_Attach(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Grind.c b/stage0/stdlib/Init/Grind.c index 883821f27a08..7fa16948ddaa 100644 --- a/stage0/stdlib/Init/Grind.c +++ b/stage0/stdlib/Init/Grind.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Init.Grind -// Imports: Init.Grind.Norm Init.Grind.Tactics Init.Grind.Lemmas Init.Grind.Cases Init.Grind.Propagator Init.Grind.Util Init.Grind.Offset +// Imports: Init.Grind.Norm Init.Grind.Tactics Init.Grind.Lemmas Init.Grind.Cases Init.Grind.Propagator Init.Grind.Util Init.Grind.Offset Init.Grind.PP #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -20,6 +20,7 @@ lean_object* initialize_Init_Grind_Cases(uint8_t builtin, lean_object*); lean_object* initialize_Init_Grind_Propagator(uint8_t builtin, lean_object*); lean_object* initialize_Init_Grind_Util(uint8_t builtin, lean_object*); lean_object* initialize_Init_Grind_Offset(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Grind_PP(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Init_Grind(uint8_t builtin, lean_object* w) { lean_object * res; @@ -46,6 +47,9 @@ lean_dec_ref(res); res = initialize_Init_Grind_Offset(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Grind_PP(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Grind/Offset.c b/stage0/stdlib/Init/Grind/Offset.c index 755f50a70b76..f3b9a067be89 100644 --- a/stage0/stdlib/Init/Grind/Offset.c +++ b/stage0/stdlib/Init/Grind/Offset.c @@ -13,1264 +13,46 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16; -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isImpliedBy(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_instDecidableEqCnstr(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_instInhabitedCnstr; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Var_denote___boxed(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstrs_isFalse(lean_object*); -lean_object* l_Lean_RArray_getImpl___rarg(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isImpliedBy___boxed(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_trans(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_instReprCnstr; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isFalse___boxed(lean_object*); -lean_object* lean_nat_to_int(lean_object*); -static lean_object* l_Lean_Grind_Offset_instInhabitedCnstr___closed__1; -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isTrivial(lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_instDecidableEqCnstr___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Grind_Offset_instReprCnstr___closed__1; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isTrivial___boxed(lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__2_splitter(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Var_denote(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75_(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_trans(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isFalse(lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173____boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Grind_Offset_trivialCnstr___closed__1; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_trivialCnstr; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26; -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_trans___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); -lean_object* lean_string_length(lean_object*); -uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173_(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_isLt___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Grind_isLt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_isLE___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19; -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12; -lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_fixedVar; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter(lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__2_splitter___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_trans_x27(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_isFalse___boxed(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter(lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27; -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____boxed(lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9; -lean_object* lean_nat_add(lean_object*, lean_object*); -lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24; -static lean_object* _init_l_Lean_Grind_Offset_fixedVar() { +LEAN_EXPORT uint8_t l_Lean_Grind_isLE(lean_object*, lean_object*); +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Grind_isLt(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_1; -x_1 = lean_unsigned_to_nat(100000000u); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Var_denote(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = l_Lean_Grind_Offset_fixedVar; -x_4 = lean_nat_dec_eq(x_2, x_3); -if (x_4 == 0) -{ -lean_object* x_5; -x_5 = l_Lean_RArray_getImpl___rarg(x_1, x_2); -return x_5; -} -else -{ -lean_object* x_6; -x_6 = lean_unsigned_to_nat(1u); -return x_6; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Var_denote___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Grind_Offset_Var_denote(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("x", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2; -x_3 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" := ", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3; -x_2 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5; -x_3 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(5u); -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(",", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("y", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("k", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("l", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("{ ", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16; -x_2 = lean_string_length(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17; -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" }", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7; -x_2 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23; -x_3 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24; -x_2 = 0; -x_3 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7; -x_2 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27; -x_3 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28; -x_2 = 0; -x_3 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = l___private_Init_Data_Repr_0__Nat_reprFast(x_3); -x_5 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_5, 0, x_4); -x_6 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7; -x_7 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_5); -x_8 = 0; -x_9 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_9, 0, x_7); -lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_8); -x_10 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6; -x_11 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -x_12 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9; -x_13 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -x_14 = lean_box(1); -x_15 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -x_16 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11; -x_17 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_17, 0, x_15); -lean_ctor_set(x_17, 1, x_16); -x_18 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5; -x_19 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); -x_22 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_22, 0, x_21); -x_23 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_23, 0, x_6); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*1, x_8); -x_25 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_25, 0, x_19); -lean_ctor_set(x_25, 1, x_24); -x_26 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_12); -x_27 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_14); -x_28 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13; -x_29 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -x_30 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_18); -x_31 = lean_ctor_get(x_1, 2); -lean_inc(x_31); -x_32 = l___private_Init_Data_Repr_0__Nat_reprFast(x_31); -x_33 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_33, 0, x_32); -x_34 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_34, 0, x_6); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set_uint8(x_35, sizeof(void*)*1, x_8); -x_36 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_36, 0, x_30); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_12); -x_38 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_14); -x_39 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15; -x_40 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -x_41 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_18); -x_42 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); -lean_dec(x_1); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_43 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25; -x_44 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_44, 0, x_41); -lean_ctor_set(x_44, 1, x_43); -x_45 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19; -x_46 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -x_47 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21; -x_48 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -x_49 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18; -x_50 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -x_51 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set_uint8(x_51, sizeof(void*)*1, x_8); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_52 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29; -x_53 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_53, 0, x_41); -lean_ctor_set(x_53, 1, x_52); -x_54 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19; -x_55 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_53); -x_56 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21; -x_57 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -x_58 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18; -x_59 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_57); -x_60 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set_uint8(x_60, sizeof(void*)*1, x_8); -return x_60; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75_(x_1, x_2); -lean_dec(x_2); +uint8_t x_3; +x_3 = lean_nat_dec_lt(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Grind_Offset_instReprCnstr___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____boxed), 2, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Grind_Offset_instReprCnstr() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Grind_Offset_instReprCnstr___closed__1; -return x_1; -} -} -LEAN_EXPORT uint8_t l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173_(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; -x_3 = lean_ctor_get(x_1, 0); -x_4 = lean_ctor_get(x_1, 1); -x_5 = lean_ctor_get(x_1, 2); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); -x_7 = lean_ctor_get(x_2, 0); -x_8 = lean_ctor_get(x_2, 1); -x_9 = lean_ctor_get(x_2, 2); -x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); -x_11 = lean_nat_dec_eq(x_3, x_7); -if (x_11 == 0) -{ -uint8_t x_12; -x_12 = 0; -return x_12; -} -else -{ -uint8_t x_13; -x_13 = lean_nat_dec_eq(x_4, x_8); -if (x_13 == 0) -{ -uint8_t x_14; -x_14 = 0; -return x_14; -} -else -{ -uint8_t x_15; -x_15 = lean_nat_dec_eq(x_5, x_9); -if (x_15 == 0) -{ -uint8_t x_16; -x_16 = 0; -return x_16; -} -else -{ -if (x_6 == 0) -{ -if (x_10 == 0) -{ -uint8_t x_17; -x_17 = 1; -return x_17; -} -else -{ -uint8_t x_18; -x_18 = 0; -return x_18; -} -} -else -{ -return x_10; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Grind_isLt___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173_(x_1, x_2); +x_3 = l_Lean_Grind_isLt(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_instDecidableEqCnstr(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Lean_Grind_isLE(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; -x_3 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173_(x_1, x_2); +x_3 = lean_nat_dec_le(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_instDecidableEqCnstr___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Grind_isLE___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Grind_Offset_instDecidableEqCnstr(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Grind_Offset_instInhabitedCnstr___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = 0; -x_3 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_1); -lean_ctor_set(x_3, 2, x_1); -lean_ctor_set_uint8(x_3, sizeof(void*)*3, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Grind_Offset_instInhabitedCnstr() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Grind_Offset_instInhabitedCnstr___closed__1; -return x_1; -} -} -static lean_object* _init_l_Lean_Grind_Offset_trivialCnstr___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = 1; -x_3 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_1); -lean_ctor_set(x_3, 2, x_1); -lean_ctor_set_uint8(x_3, sizeof(void*)*3, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Grind_Offset_trivialCnstr() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Grind_Offset_trivialCnstr___closed__1; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_trans(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_ctor_get(x_1, 1); -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_nat_dec_eq(x_3, x_4); -lean_dec(x_4); -if (x_5 == 0) -{ -lean_object* x_6; -lean_dec(x_2); -x_6 = l_Lean_Grind_Offset_trivialCnstr; -return x_6; -} -else -{ -uint8_t x_7; -x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); -if (x_7 == 0) -{ -uint8_t x_8; -x_8 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); -if (x_8 == 0) -{ -uint8_t x_9; -x_9 = !lean_is_exclusive(x_2); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_10 = lean_ctor_get(x_1, 0); -x_11 = lean_ctor_get(x_1, 2); -x_12 = lean_ctor_get(x_2, 2); -x_13 = lean_ctor_get(x_2, 0); -lean_dec(x_13); -x_14 = lean_nat_add(x_11, x_12); -lean_dec(x_12); -x_15 = 0; -lean_inc(x_10); -lean_ctor_set(x_2, 2, x_14); -lean_ctor_set(x_2, 0, x_10); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_15); -return x_2; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_16 = lean_ctor_get(x_1, 0); -x_17 = lean_ctor_get(x_1, 2); -x_18 = lean_ctor_get(x_2, 1); -x_19 = lean_ctor_get(x_2, 2); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_2); -x_20 = lean_nat_add(x_17, x_19); -lean_dec(x_19); -x_21 = 0; -lean_inc(x_16); -x_22 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_22, 0, x_16); -lean_ctor_set(x_22, 1, x_18); -lean_ctor_set(x_22, 2, x_20); -lean_ctor_set_uint8(x_22, sizeof(void*)*3, x_21); -return x_22; -} -} -else -{ -uint8_t x_23; -x_23 = !lean_is_exclusive(x_2); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_24 = lean_ctor_get(x_1, 0); -x_25 = lean_ctor_get(x_1, 2); -x_26 = lean_ctor_get(x_2, 2); -x_27 = lean_ctor_get(x_2, 0); -lean_dec(x_27); -x_28 = lean_nat_dec_lt(x_25, x_26); -if (x_28 == 0) -{ -lean_object* x_29; uint8_t x_30; -x_29 = lean_nat_sub(x_25, x_26); -lean_dec(x_26); -x_30 = 0; -lean_inc(x_24); -lean_ctor_set(x_2, 2, x_29); -lean_ctor_set(x_2, 0, x_24); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_30); -return x_2; -} -else -{ -lean_object* x_31; uint8_t x_32; -x_31 = lean_nat_sub(x_26, x_25); -lean_dec(x_26); -x_32 = 1; -lean_inc(x_24); -lean_ctor_set(x_2, 2, x_31); -lean_ctor_set(x_2, 0, x_24); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_32); -return x_2; -} -} -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_33 = lean_ctor_get(x_1, 0); -x_34 = lean_ctor_get(x_1, 2); -x_35 = lean_ctor_get(x_2, 1); -x_36 = lean_ctor_get(x_2, 2); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_2); -x_37 = lean_nat_dec_lt(x_34, x_36); -if (x_37 == 0) -{ -lean_object* x_38; uint8_t x_39; lean_object* x_40; -x_38 = lean_nat_sub(x_34, x_36); -lean_dec(x_36); -x_39 = 0; -lean_inc(x_33); -x_40 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_40, 0, x_33); -lean_ctor_set(x_40, 1, x_35); -lean_ctor_set(x_40, 2, x_38); -lean_ctor_set_uint8(x_40, sizeof(void*)*3, x_39); -return x_40; -} -else -{ -lean_object* x_41; uint8_t x_42; lean_object* x_43; -x_41 = lean_nat_sub(x_36, x_34); -lean_dec(x_36); -x_42 = 1; -lean_inc(x_33); -x_43 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_43, 0, x_33); -lean_ctor_set(x_43, 1, x_35); -lean_ctor_set(x_43, 2, x_41); -lean_ctor_set_uint8(x_43, sizeof(void*)*3, x_42); -return x_43; -} -} -} -} -else -{ -uint8_t x_44; -x_44 = lean_ctor_get_uint8(x_2, sizeof(void*)*3); -if (x_44 == 0) -{ -uint8_t x_45; -x_45 = !lean_is_exclusive(x_2); -if (x_45 == 0) -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_46 = lean_ctor_get(x_1, 0); -x_47 = lean_ctor_get(x_1, 2); -x_48 = lean_ctor_get(x_2, 2); -x_49 = lean_ctor_get(x_2, 0); -lean_dec(x_49); -x_50 = lean_nat_dec_lt(x_47, x_48); -if (x_50 == 0) -{ -lean_object* x_51; uint8_t x_52; -x_51 = lean_nat_sub(x_47, x_48); -lean_dec(x_48); -x_52 = 1; -lean_inc(x_46); -lean_ctor_set(x_2, 2, x_51); -lean_ctor_set(x_2, 0, x_46); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_52); -return x_2; -} -else -{ -lean_object* x_53; uint8_t x_54; -x_53 = lean_nat_sub(x_48, x_47); -lean_dec(x_48); -x_54 = 0; -lean_inc(x_46); -lean_ctor_set(x_2, 2, x_53); -lean_ctor_set(x_2, 0, x_46); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_54); -return x_2; -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_55 = lean_ctor_get(x_1, 0); -x_56 = lean_ctor_get(x_1, 2); -x_57 = lean_ctor_get(x_2, 1); -x_58 = lean_ctor_get(x_2, 2); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_2); -x_59 = lean_nat_dec_lt(x_56, x_58); -if (x_59 == 0) -{ -lean_object* x_60; uint8_t x_61; lean_object* x_62; -x_60 = lean_nat_sub(x_56, x_58); -lean_dec(x_58); -x_61 = 1; -lean_inc(x_55); -x_62 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_62, 0, x_55); -lean_ctor_set(x_62, 1, x_57); -lean_ctor_set(x_62, 2, x_60); -lean_ctor_set_uint8(x_62, sizeof(void*)*3, x_61); -return x_62; -} -else -{ -lean_object* x_63; uint8_t x_64; lean_object* x_65; -x_63 = lean_nat_sub(x_58, x_56); -lean_dec(x_58); -x_64 = 0; -lean_inc(x_55); -x_65 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_65, 0, x_55); -lean_ctor_set(x_65, 1, x_57); -lean_ctor_set(x_65, 2, x_63); -lean_ctor_set_uint8(x_65, sizeof(void*)*3, x_64); -return x_65; -} -} -} -else -{ -uint8_t x_66; -x_66 = !lean_is_exclusive(x_2); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -x_67 = lean_ctor_get(x_1, 0); -x_68 = lean_ctor_get(x_1, 2); -x_69 = lean_ctor_get(x_2, 2); -x_70 = lean_ctor_get(x_2, 0); -lean_dec(x_70); -x_71 = lean_nat_add(x_68, x_69); -lean_dec(x_69); -x_72 = 1; -lean_inc(x_67); -lean_ctor_set(x_2, 2, x_71); -lean_ctor_set(x_2, 0, x_67); -lean_ctor_set_uint8(x_2, sizeof(void*)*3, x_72); -return x_2; -} -else -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; lean_object* x_79; -x_73 = lean_ctor_get(x_1, 0); -x_74 = lean_ctor_get(x_1, 2); -x_75 = lean_ctor_get(x_2, 1); -x_76 = lean_ctor_get(x_2, 2); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_2); -x_77 = lean_nat_add(x_74, x_76); -lean_dec(x_76); -x_78 = 1; -lean_inc(x_73); -x_79 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_79, 0, x_73); -lean_ctor_set(x_79, 1, x_75); -lean_ctor_set(x_79, 2, x_77); -lean_ctor_set_uint8(x_79, sizeof(void*)*3, x_78); -return x_79; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_trans___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Grind_Offset_Cnstr_trans(x_1, x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 2); -lean_inc(x_5); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); -lean_dec(x_1); -x_7 = lean_box(x_6); -x_8 = lean_apply_4(x_2, x_3, x_4, x_5, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__2_splitter(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__2_splitter___rarg), 2, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -if (x_1 == 0) -{ -if (x_2 == 0) -{ -lean_inc(x_3); -return x_3; -} -else -{ -lean_inc(x_4); -return x_4; -} -} -else -{ -if (x_2 == 0) -{ -lean_inc(x_5); -return x_5; -} -else -{ -lean_inc(x_6); -return x_6; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg___boxed), 6, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -uint8_t x_7; uint8_t x_8; lean_object* x_9; -x_7 = lean_unbox(x_1); -lean_dec(x_1); -x_8 = lean_unbox(x_2); +x_3 = l_Lean_Grind_isLE(x_1, x_2); lean_dec(x_2); -x_9 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstr_trans_match__1_splitter___rarg(x_7, x_8, x_3, x_4, x_5, x_6); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_9; -} -} -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isTrivial(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; -x_2 = lean_ctor_get(x_1, 0); -x_3 = lean_ctor_get(x_1, 1); -x_4 = lean_nat_dec_eq(x_2, x_3); -if (x_4 == 0) -{ -uint8_t x_5; -x_5 = 0; -return x_5; -} -else -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_ctor_get(x_1, 2); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_eq(x_6, x_7); -return x_8; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isTrivial___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Grind_Offset_Cnstr_isTrivial(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isFalse(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; -x_2 = lean_ctor_get(x_1, 0); -x_3 = lean_ctor_get(x_1, 1); -x_4 = lean_nat_dec_eq(x_2, x_3); -if (x_4 == 0) -{ -uint8_t x_5; -x_5 = 0; -return x_5; -} -else -{ -lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_6 = lean_ctor_get(x_1, 2); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_eq(x_6, x_7); -if (x_8 == 0) -{ -uint8_t x_9; -x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*3); -return x_9; -} -else -{ -uint8_t x_10; -x_10 = 0; -return x_10; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isFalse___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Grind_Offset_Cnstr_isFalse(x_1); lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_dec(x_3); -lean_inc(x_2); -return x_2; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_1, 1); -lean_inc(x_5); -lean_dec(x_1); -x_6 = lean_apply_2(x_3, x_4, x_5); -return x_6; -} -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg___boxed), 3, 0); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_Cnstrs_denoteAnd_x27_match__1_splitter___rarg(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_trans_x27(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -return x_1; -} -else -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_2, 0); -lean_inc(x_3); -x_4 = lean_ctor_get(x_2, 1); -lean_inc(x_4); -lean_dec(x_2); -x_5 = l_Lean_Grind_Offset_Cnstr_trans(x_1, x_3); -lean_dec(x_1); -x_1 = x_5; -x_2 = x_4; -goto _start; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_trans(lean_object* x_1) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_2; -x_2 = l_Lean_Grind_Offset_trivialCnstr; -return x_2; -} -else -{ -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -lean_dec(x_1); -x_5 = l_Lean_Grind_Offset_Cnstrs_trans_x27(x_3, x_4); -return x_5; -} -} -} -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstrs_isFalse(lean_object* x_1) { -_start: -{ -lean_object* x_2; uint8_t x_3; -x_2 = l_Lean_Grind_Offset_Cnstrs_trans(x_1); -x_3 = l_Lean_Grind_Offset_Cnstr_isFalse(x_2); -lean_dec(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstrs_isFalse___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_Lean_Grind_Offset_Cnstrs_isFalse(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT uint8_t l_Lean_Grind_Offset_Cnstr_isImpliedBy(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; uint8_t x_4; -x_3 = l_Lean_Grind_Offset_Cnstrs_trans(x_1); -x_4 = l___private_Init_Grind_Offset_0__Lean_Grind_Offset_decEqCnstr____x40_Init_Grind_Offset___hyg_173_(x_3, x_2); -lean_dec(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Grind_Offset_Cnstr_isImpliedBy___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Grind_Offset_Cnstr_isImpliedBy(x_1, x_2); -lean_dec(x_2); x_4 = lean_box(x_3); return x_4; } @@ -1288,78 +70,6 @@ lean_dec_ref(res); res = initialize_Init_Omega(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Grind_Offset_fixedVar = _init_l_Lean_Grind_Offset_fixedVar(); -lean_mark_persistent(l_Lean_Grind_Offset_fixedVar); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__1); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__2); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__3); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__4); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__5); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__6); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__7); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__8); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__9); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__10); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__11); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__12); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__13); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__14); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__15); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__16); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__17); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__18); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__19); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__20); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__21); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__22); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__23); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__24); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__25); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__26); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__27); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__28); -l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29 = _init_l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29(); -lean_mark_persistent(l___private_Init_Grind_Offset_0__Lean_Grind_Offset_reprCnstr____x40_Init_Grind_Offset___hyg_75____closed__29); -l_Lean_Grind_Offset_instReprCnstr___closed__1 = _init_l_Lean_Grind_Offset_instReprCnstr___closed__1(); -lean_mark_persistent(l_Lean_Grind_Offset_instReprCnstr___closed__1); -l_Lean_Grind_Offset_instReprCnstr = _init_l_Lean_Grind_Offset_instReprCnstr(); -lean_mark_persistent(l_Lean_Grind_Offset_instReprCnstr); -l_Lean_Grind_Offset_instInhabitedCnstr___closed__1 = _init_l_Lean_Grind_Offset_instInhabitedCnstr___closed__1(); -lean_mark_persistent(l_Lean_Grind_Offset_instInhabitedCnstr___closed__1); -l_Lean_Grind_Offset_instInhabitedCnstr = _init_l_Lean_Grind_Offset_instInhabitedCnstr(); -lean_mark_persistent(l_Lean_Grind_Offset_instInhabitedCnstr); -l_Lean_Grind_Offset_trivialCnstr___closed__1 = _init_l_Lean_Grind_Offset_trivialCnstr___closed__1(); -lean_mark_persistent(l_Lean_Grind_Offset_trivialCnstr___closed__1); -l_Lean_Grind_Offset_trivialCnstr = _init_l_Lean_Grind_Offset_trivialCnstr(); -lean_mark_persistent(l_Lean_Grind_Offset_trivialCnstr); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Init/Grind/PP.c b/stage0/stdlib/Init/Grind/PP.c new file mode 100644 index 000000000000..f8100343c45a --- /dev/null +++ b/stage0/stdlib/Init/Grind/PP.c @@ -0,0 +1,363 @@ +// Lean compiler output +// Module: Init.Grind.PP +// Imports: Init.NotationExtra +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_nodeDefUnexpander(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__1; +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__7; +static lean_object* l_Lean_Grind_NodeDefUnexpander___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__8; +uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__4; +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__3; +LEAN_EXPORT lean_object* l_Lean_Grind_node__def(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__5; +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__6; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___rarg___boxed(lean_object*); +uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); +lean_object* lean_mk_syntax_ident(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_toCtorIdx(lean_object*); +static lean_object* l_Lean_Grind_NodeDefUnexpander___rarg___closed__1; +static lean_object* l_Lean_Grind_nodeDefUnexpander___closed__2; +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander(lean_object*, lean_object*); +lean_object* l_Lean_TSyntax_getNat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_nodeDefUnexpander___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_toCtorIdx___boxed(lean_object*); +static lean_object* l_Lean_Grind_NodeDefUnexpander___rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander___rarg(lean_object*); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_string_append(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_node__def___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_toCtorIdx(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_unsigned_to_nat(0u); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_toCtorIdx___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Grind_NodeDef_toCtorIdx(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___rarg(lean_object* x_1) { +_start: +{ +lean_inc(x_1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l_Lean_Grind_NodeDef_noConfusion___rarg___boxed), 1, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___rarg___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Grind_NodeDef_noConfusion___rarg(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDef_noConfusion___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Grind_NodeDef_noConfusion(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_node__def(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_box(0); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_node__def___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Grind_node__def(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Parser", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("app", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Grind_nodeDefUnexpander___closed__1; +x_2 = l_Lean_Grind_nodeDefUnexpander___closed__2; +x_3 = l_Lean_Grind_nodeDefUnexpander___closed__3; +x_4 = l_Lean_Grind_nodeDefUnexpander___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("num", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Grind_nodeDefUnexpander___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Grind_nodeDefUnexpander___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("#", 1, 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_nodeDefUnexpander(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint8_t x_5; +x_4 = l_Lean_Grind_nodeDefUnexpander___closed__5; +lean_inc(x_1); +x_5 = l_Lean_Syntax_isOfKind(x_1, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_3); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_8 = lean_unsigned_to_nat(1u); +x_9 = l_Lean_Syntax_getArg(x_1, x_8); +lean_dec(x_1); +lean_inc(x_9); +x_10 = l_Lean_Syntax_matchesNull(x_9, x_8); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +lean_dec(x_9); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_3); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_unsigned_to_nat(0u); +x_14 = l_Lean_Syntax_getArg(x_9, x_13); +lean_dec(x_9); +x_15 = l_Lean_Grind_nodeDefUnexpander___closed__7; +lean_inc(x_14); +x_16 = l_Lean_Syntax_isOfKind(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_14); +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_3); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_19 = l_Lean_TSyntax_getNat(x_14); +lean_dec(x_14); +x_20 = l___private_Init_Data_Repr_0__Nat_reprFast(x_19); +x_21 = l_Lean_Grind_nodeDefUnexpander___closed__8; +x_22 = lean_string_append(x_21, x_20); +lean_dec(x_20); +x_23 = lean_box(0); +x_24 = l_Lean_Name_str___override(x_23, x_22); +x_25 = lean_mk_syntax_ident(x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_3); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_nodeDefUnexpander___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Grind_nodeDefUnexpander(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("NodeDef", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Grind_NodeDefUnexpander___rarg___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Grind_NodeDefUnexpander___rarg___closed__2; +x_2 = lean_mk_syntax_ident(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Grind_NodeDefUnexpander___rarg___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Grind_NodeDefUnexpander___rarg), 1, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Grind_NodeDefUnexpander___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Grind_NodeDefUnexpander(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +lean_object* initialize_Init_NotationExtra(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Init_Grind_PP(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_NotationExtra(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Grind_nodeDefUnexpander___closed__1 = _init_l_Lean_Grind_nodeDefUnexpander___closed__1(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__1); +l_Lean_Grind_nodeDefUnexpander___closed__2 = _init_l_Lean_Grind_nodeDefUnexpander___closed__2(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__2); +l_Lean_Grind_nodeDefUnexpander___closed__3 = _init_l_Lean_Grind_nodeDefUnexpander___closed__3(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__3); +l_Lean_Grind_nodeDefUnexpander___closed__4 = _init_l_Lean_Grind_nodeDefUnexpander___closed__4(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__4); +l_Lean_Grind_nodeDefUnexpander___closed__5 = _init_l_Lean_Grind_nodeDefUnexpander___closed__5(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__5); +l_Lean_Grind_nodeDefUnexpander___closed__6 = _init_l_Lean_Grind_nodeDefUnexpander___closed__6(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__6); +l_Lean_Grind_nodeDefUnexpander___closed__7 = _init_l_Lean_Grind_nodeDefUnexpander___closed__7(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__7); +l_Lean_Grind_nodeDefUnexpander___closed__8 = _init_l_Lean_Grind_nodeDefUnexpander___closed__8(); +lean_mark_persistent(l_Lean_Grind_nodeDefUnexpander___closed__8); +l_Lean_Grind_NodeDefUnexpander___rarg___closed__1 = _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__1(); +lean_mark_persistent(l_Lean_Grind_NodeDefUnexpander___rarg___closed__1); +l_Lean_Grind_NodeDefUnexpander___rarg___closed__2 = _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__2(); +lean_mark_persistent(l_Lean_Grind_NodeDefUnexpander___rarg___closed__2); +l_Lean_Grind_NodeDefUnexpander___rarg___closed__3 = _init_l_Lean_Grind_NodeDefUnexpander___rarg___closed__3(); +lean_mark_persistent(l_Lean_Grind_NodeDefUnexpander___rarg___closed__3); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lake/Build/Actions.c b/stage0/stdlib/Lake/Build/Actions.c index 5fec66b9f717..c028b5802e81 100644 --- a/stage0/stdlib/Lake/Build/Actions.c +++ b/stage0/stdlib/Lake/Build/Actions.c @@ -31,7 +31,6 @@ static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lake_compileLeanModule___s LEAN_EXPORT lean_object* l_Lake_compileSharedLib(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_compileLeanModule___lambda__4___closed__1; -static lean_object* l_Lake_compileExe___closed__5; extern uint8_t l_System_Platform_isOSX; lean_object* lean_array_push(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -58,7 +57,7 @@ lean_object* lean_string_push(lean_object*, uint32_t); LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_compileExe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_IO_FS_createDirAll(lean_object*, lean_object*); -static lean_object* l_Lake_compileExe___closed__1; +LEAN_EXPORT lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv(lean_object*); LEAN_EXPORT lean_object* l_Lake_logSerialMessage___at_Lake_compileLeanModule___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); @@ -75,6 +74,7 @@ LEAN_EXPORT lean_object* l_Lake_tar___lambda__1(lean_object*, lean_object*, lean LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_download___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lake_mkCmdLog(lean_object*); +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6; LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Message_0__Lean_fromJsonSerialMessage____x40_Lean_Message___hyg_3357_(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lake_tar___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,13 +92,13 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spe LEAN_EXPORT lean_object* l_Lake_untar(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); lean_object* l_Lake_getSearchPath(lean_object*, lean_object*); -static lean_object* l_Lake_compileExe___closed__6; LEAN_EXPORT lean_object* l_Lake_download___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_tar___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_untar___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lake_tar___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4; LEAN_EXPORT lean_object* l_Lake_compileO___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_compileStaticLib___closed__1; LEAN_EXPORT lean_object* l_Lake_download___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -107,6 +107,7 @@ static lean_object* l_Lake_compileO___closed__1; lean_object* l_Std_Internal_Parsec_String_Parser_run___rarg(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_System_SearchPath_toString(lean_object*); +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(lean_object*, lean_object*, lean_object*); @@ -119,9 +120,9 @@ LEAN_EXPORT lean_object* l_Lake_compileExe___boxed(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Lake_tar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_download___spec__1(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_List_foldlM___at_Lake_compileLeanModule___spec__3___closed__2; +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2; lean_object* l_Lean_Json_Parser_any(lean_object*); extern lean_object* l_Lake_sharedLibPathEnvVar; -static lean_object* l_Lake_compileExe___closed__2; lean_object* l_Lake_proc(lean_object*, uint8_t, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); size_t lean_usize_add(size_t, size_t); @@ -147,12 +148,12 @@ LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__5___boxed(lean_objec LEAN_EXPORT lean_object* l_Lake_compileLeanModule___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_compileLeanModule___lambda__2___closed__1; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -static lean_object* l_Lake_compileExe___closed__4; lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); -static lean_object* l_Lake_compileExe___closed__3; +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1; static lean_object* l_Lake_untar___closed__1; static lean_object* l_Lake_tar___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lake_compileLeanModule___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3; static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lake_compileLeanModule___spec__1___closed__1() { _start: { @@ -2629,113 +2630,7 @@ x_6 = l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spec__1(x_4, x_5, x_3) return x_6; } } -static lean_object* _init_l_Lake_compileSharedLib___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("-shared", 7, 7); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lake_compileSharedLib(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lake_createParentDirs(x_1, x_5); -if (lean_obj_tag(x_6) == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_7 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_dec(x_6); -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_1); -lean_ctor_set(x_9, 1, x_8); -x_10 = l_Lake_compileLeanModule___closed__2; -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -x_12 = l_Lake_compileSharedLib___closed__1; -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -x_14 = lean_array_mk(x_13); -x_15 = l_Array_append___rarg(x_14, x_2); -x_16 = lean_box(0); -x_17 = l_Lake_compileLeanModule___lambda__4___closed__2; -x_18 = l_Lake_compileO___closed__1; -x_19 = 0; -x_20 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_20, 0, x_17); -lean_ctor_set(x_20, 1, x_3); -lean_ctor_set(x_20, 2, x_15); -lean_ctor_set(x_20, 3, x_16); -lean_ctor_set(x_20, 4, x_18); -lean_ctor_set_uint8(x_20, sizeof(void*)*5, x_19); -x_21 = l_Lake_proc(x_20, x_19, x_4, x_7); -return x_21; -} -else -{ -uint8_t x_22; -lean_dec(x_3); -lean_dec(x_1); -x_22 = !lean_is_exclusive(x_6); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_23 = lean_ctor_get(x_6, 0); -x_24 = lean_io_error_to_string(x_23); -x_25 = 3; -x_26 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set_uint8(x_26, sizeof(void*)*1, x_25); -x_27 = lean_array_get_size(x_4); -x_28 = lean_array_push(x_4, x_26); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 0, x_29); -return x_6; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_30 = lean_ctor_get(x_6, 0); -x_31 = lean_ctor_get(x_6, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_6); -x_32 = lean_io_error_to_string(x_30); -x_33 = 3; -x_34 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set_uint8(x_34, sizeof(void*)*1, x_33); -x_35 = lean_array_get_size(x_4); -x_36 = lean_array_push(x_4, x_34); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_31); -return x_38; -} -} -} -} -LEAN_EXPORT lean_object* l_Lake_compileSharedLib___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lake_compileSharedLib(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_2); -return x_6; -} -} -static lean_object* _init_l_Lake_compileExe___closed__1() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1() { _start: { lean_object* x_1; @@ -2743,7 +2638,7 @@ x_1 = lean_mk_string_unchecked("MACOSX_DEPLOYMENT_TARGET", 24, 24); return x_1; } } -static lean_object* _init_l_Lake_compileExe___closed__2() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2() { _start: { lean_object* x_1; @@ -2751,408 +2646,473 @@ x_1 = lean_mk_string_unchecked("99.0", 4, 4); return x_1; } } -static lean_object* _init_l_Lake_compileExe___closed__3() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lake_compileExe___closed__2; +x_1 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lake_compileExe___closed__4() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lake_compileExe___closed__1; -x_2 = l_Lake_compileExe___closed__3; +x_1 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1; +x_2 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lake_compileExe___closed__5() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lake_compileExe___closed__4; +x_2 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4; x_3 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_3, 0, x_2); lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lake_compileExe___closed__6() { +static lean_object* _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lake_compileExe___closed__5; +x_1 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5; x_2 = lean_array_mk(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lake_compileExe(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv(lean_object* x_1) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_44; lean_object* x_45; lean_object* x_86; -x_86 = l_Lake_createParentDirs(x_1, x_6); -if (lean_obj_tag(x_86) == 0) +uint8_t x_2; +x_2 = l_System_Platform_isOSX; +if (x_2 == 0) +{ +lean_object* x_3; lean_object* x_4; +x_3 = l_Lake_compileO___closed__1; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_3); +lean_ctor_set(x_4, 1, x_1); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; +x_5 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1; +x_6 = lean_io_getenv(x_5, x_1); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +if (lean_obj_tag(x_7) == 0) { -uint8_t x_87; -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_6); +if (x_8 == 0) { -lean_object* x_88; -x_88 = lean_ctor_get(x_86, 1); -lean_ctor_set(x_86, 1, x_5); -x_44 = x_86; -x_45 = x_88; -goto block_85; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_6, 0); +lean_dec(x_9); +x_10 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6; +lean_ctor_set(x_6, 0, x_10); +return x_6; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_86, 0); -x_90 = lean_ctor_get(x_86, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_86); -x_91 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_5); -x_44 = x_91; -x_45 = x_90; -goto block_85; +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); +lean_dec(x_6); +x_12 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } } else { -uint8_t x_92; -x_92 = !lean_is_exclusive(x_86); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_93 = lean_ctor_get(x_86, 0); -x_94 = lean_ctor_get(x_86, 1); -x_95 = lean_io_error_to_string(x_93); -x_96 = 3; -x_97 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set_uint8(x_97, sizeof(void*)*1, x_96); -x_98 = lean_array_get_size(x_5); -x_99 = lean_array_push(x_5, x_97); -lean_ctor_set(x_86, 1, x_99); -lean_ctor_set(x_86, 0, x_98); -x_44 = x_86; -x_45 = x_94; -goto block_85; +uint8_t x_14; +lean_dec(x_7); +x_14 = !lean_is_exclusive(x_6); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_6, 0); +lean_dec(x_15); +x_16 = l_Lake_compileO___closed__1; +lean_ctor_set(x_6, 0, x_16); +return x_6; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_100 = lean_ctor_get(x_86, 0); -x_101 = lean_ctor_get(x_86, 1); -lean_inc(x_101); -lean_inc(x_100); -lean_dec(x_86); -x_102 = lean_io_error_to_string(x_100); -x_103 = 3; -x_104 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set_uint8(x_104, sizeof(void*)*1, x_103); -x_105 = lean_array_get_size(x_5); -x_106 = lean_array_push(x_5, x_104); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -x_44 = x_107; -x_45 = x_101; -goto block_85; -} -} -block_43: +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_6, 1); +lean_inc(x_17); +lean_dec(x_6); +x_18 = l_Lake_compileO___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; +} +} +} +else { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_7); -if (x_9 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_6); +if (x_20 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_10 = lean_ctor_get(x_7, 0); -x_11 = lean_ctor_get(x_7, 1); -x_12 = lean_box(0); -lean_ctor_set_tag(x_7, 1); -lean_ctor_set(x_7, 1, x_12); -lean_ctor_set(x_7, 0, x_1); -x_13 = l_Lake_compileLeanModule___closed__2; -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_7); -x_15 = lean_array_mk(x_14); -x_16 = lean_array_size(x_2); -x_17 = 0; -x_18 = l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spec__1(x_16, x_17, x_2); -x_19 = l_Array_append___rarg(x_15, x_18); -lean_dec(x_18); -x_20 = l_Array_append___rarg(x_19, x_3); -x_21 = lean_box(0); -x_22 = l_Lake_compileLeanModule___lambda__4___closed__2; -x_23 = 0; -x_24 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_4); -lean_ctor_set(x_24, 2, x_20); -lean_ctor_set(x_24, 3, x_21); -lean_ctor_set(x_24, 4, x_10); -lean_ctor_set_uint8(x_24, sizeof(void*)*5, x_23); -x_25 = l_Lake_proc(x_24, x_23, x_11, x_8); -return x_25; +return x_6; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; -x_26 = lean_ctor_get(x_7, 0); -x_27 = lean_ctor_get(x_7, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_7); -x_28 = lean_box(0); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_1); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lake_compileLeanModule___closed__2; -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -x_32 = lean_array_mk(x_31); -x_33 = lean_array_size(x_2); -x_34 = 0; -x_35 = l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spec__1(x_33, x_34, x_2); -x_36 = l_Array_append___rarg(x_32, x_35); -lean_dec(x_35); -x_37 = l_Array_append___rarg(x_36, x_3); -x_38 = lean_box(0); -x_39 = l_Lake_compileLeanModule___lambda__4___closed__2; -x_40 = 0; -x_41 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_4); -lean_ctor_set(x_41, 2, x_37); -lean_ctor_set(x_41, 3, x_38); -lean_ctor_set(x_41, 4, x_26); -lean_ctor_set_uint8(x_41, sizeof(void*)*5, x_40); -x_42 = l_Lake_proc(x_41, x_40, x_27, x_8); -return x_42; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_6, 0); +x_22 = lean_ctor_get(x_6, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_6); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} } } -block_85: +} +static lean_object* _init_l_Lake_compileSharedLib___closed__1() { +_start: { -if (lean_obj_tag(x_44) == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("-shared", 7, 7); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lake_compileSharedLib(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -uint8_t x_46; -x_46 = !lean_is_exclusive(x_44); -if (x_46 == 0) +lean_object* x_6; +x_6 = l_Lake_createParentDirs(x_1, x_5); +if (lean_obj_tag(x_6) == 0) { -lean_object* x_47; lean_object* x_48; uint8_t x_49; -x_47 = lean_ctor_get(x_44, 1); -x_48 = lean_ctor_get(x_44, 0); -lean_dec(x_48); -x_49 = l_System_Platform_isOSX; -if (x_49 == 0) +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +x_8 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv(x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_50; -x_50 = l_Lake_compileO___closed__1; -lean_ctor_set(x_44, 0, x_50); -x_7 = x_44; -x_8 = x_45; -goto block_43; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); +x_13 = l_Lake_compileLeanModule___closed__2; +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +x_15 = l_Lake_compileSharedLib___closed__1; +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = lean_array_mk(x_16); +x_18 = l_Array_append___rarg(x_17, x_2); +x_19 = lean_box(0); +x_20 = l_Lake_compileLeanModule___lambda__4___closed__2; +x_21 = 0; +x_22 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_3); +lean_ctor_set(x_22, 2, x_18); +lean_ctor_set(x_22, 3, x_19); +lean_ctor_set(x_22, 4, x_9); +lean_ctor_set_uint8(x_22, sizeof(void*)*5, x_21); +x_23 = l_Lake_proc(x_22, x_21, x_4, x_10); +return x_23; } else { -lean_object* x_51; lean_object* x_52; -x_51 = l_Lake_compileExe___closed__1; -x_52 = lean_io_getenv(x_51, x_45); -if (lean_obj_tag(x_52) == 0) -{ -lean_object* x_53; -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -if (lean_obj_tag(x_53) == 0) +uint8_t x_24; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_8); +if (x_24 == 0) { -lean_object* x_54; lean_object* x_55; -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = l_Lake_compileExe___closed__6; -lean_ctor_set(x_44, 0, x_55); -x_7 = x_44; -x_8 = x_54; -goto block_43; +return x_8; } else { -lean_object* x_56; lean_object* x_57; -lean_dec(x_53); -x_56 = lean_ctor_get(x_52, 1); -lean_inc(x_56); -lean_dec(x_52); -x_57 = l_Lake_compileO___closed__1; -lean_ctor_set(x_44, 0, x_57); -x_7 = x_44; -x_8 = x_56; -goto block_43; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_8, 0); +x_26 = lean_ctor_get(x_8, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_8); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} } } else { -uint8_t x_58; -lean_free_object(x_44); -lean_dec(x_47); -lean_dec(x_4); -lean_dec(x_2); +uint8_t x_28; +lean_dec(x_3); lean_dec(x_1); -x_58 = !lean_is_exclusive(x_52); -if (x_58 == 0) +x_28 = !lean_is_exclusive(x_6); +if (x_28 == 0) { -return x_52; +lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_29 = lean_ctor_get(x_6, 0); +x_30 = lean_io_error_to_string(x_29); +x_31 = 3; +x_32 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set_uint8(x_32, sizeof(void*)*1, x_31); +x_33 = lean_array_get_size(x_4); +x_34 = lean_array_push(x_4, x_32); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +lean_ctor_set_tag(x_6, 0); +lean_ctor_set(x_6, 0, x_35); +return x_6; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_52, 0); -x_60 = lean_ctor_get(x_52, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_52); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_36 = lean_ctor_get(x_6, 0); +x_37 = lean_ctor_get(x_6, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_6); +x_38 = lean_io_error_to_string(x_36); +x_39 = 3; +x_40 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set_uint8(x_40, sizeof(void*)*1, x_39); +x_41 = lean_array_get_size(x_4); +x_42 = lean_array_push(x_4, x_40); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_37); +return x_44; } } } } -else +LEAN_EXPORT lean_object* l_Lake_compileSharedLib___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_62; uint8_t x_63; -x_62 = lean_ctor_get(x_44, 1); -lean_inc(x_62); -lean_dec(x_44); -x_63 = l_System_Platform_isOSX; -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; -x_64 = l_Lake_compileO___closed__1; -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -x_7 = x_65; -x_8 = x_45; -goto block_43; +lean_object* x_6; +x_6 = l_Lake_compileSharedLib(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_2); +return x_6; } -else +} +LEAN_EXPORT lean_object* l_Lake_compileExe(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_66; lean_object* x_67; -x_66 = l_Lake_compileExe___closed__1; -x_67 = lean_io_getenv(x_66, x_45); -if (lean_obj_tag(x_67) == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_39; +x_39 = l_Lake_createParentDirs(x_1, x_6); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_68; -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -if (lean_obj_tag(x_68) == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -lean_dec(x_67); -x_70 = l_Lake_compileExe___closed__6; -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_62); -x_7 = x_71; -x_8 = x_69; -goto block_43; +lean_object* x_41; +x_41 = lean_ctor_get(x_39, 1); +lean_ctor_set(x_39, 1, x_5); +x_7 = x_39; +x_8 = x_41; +goto block_38; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -lean_dec(x_68); -x_72 = lean_ctor_get(x_67, 1); -lean_inc(x_72); -lean_dec(x_67); -x_73 = l_Lake_compileO___closed__1; -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_62); -x_7 = x_74; -x_8 = x_72; -goto block_43; +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_39, 0); +x_43 = lean_ctor_get(x_39, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_39); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_5); +x_7 = x_44; +x_8 = x_43; +goto block_38; +} +} +else +{ +uint8_t x_45; +x_45 = !lean_is_exclusive(x_39); +if (x_45 == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_46 = lean_ctor_get(x_39, 0); +x_47 = lean_ctor_get(x_39, 1); +x_48 = lean_io_error_to_string(x_46); +x_49 = 3; +x_50 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*1, x_49); +x_51 = lean_array_get_size(x_5); +x_52 = lean_array_push(x_5, x_50); +lean_ctor_set(x_39, 1, x_52); +lean_ctor_set(x_39, 0, x_51); +x_7 = x_39; +x_8 = x_47; +goto block_38; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_53 = lean_ctor_get(x_39, 0); +x_54 = lean_ctor_get(x_39, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_39); +x_55 = lean_io_error_to_string(x_53); +x_56 = 3; +x_57 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set_uint8(x_57, sizeof(void*)*1, x_56); +x_58 = lean_array_get_size(x_5); +x_59 = lean_array_push(x_5, x_57); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +x_7 = x_60; +x_8 = x_54; +goto block_38; } } +block_38: +{ +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv(x_8); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_1); +lean_ctor_set(x_14, 1, x_13); +x_15 = l_Lake_compileLeanModule___closed__2; +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = lean_array_mk(x_16); +x_18 = lean_array_size(x_2); +x_19 = 0; +x_20 = l_Array_mapMUnsafe_map___at_Lake_compileStaticLib___spec__1(x_18, x_19, x_2); +x_21 = l_Array_append___rarg(x_17, x_20); +lean_dec(x_20); +x_22 = l_Array_append___rarg(x_21, x_3); +x_23 = lean_box(0); +x_24 = l_Lake_compileLeanModule___lambda__4___closed__2; +x_25 = 0; +x_26 = lean_alloc_ctor(0, 5, 1); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_4); +lean_ctor_set(x_26, 2, x_22); +lean_ctor_set(x_26, 3, x_23); +lean_ctor_set(x_26, 4, x_11); +lean_ctor_set_uint8(x_26, sizeof(void*)*5, x_25); +x_27 = l_Lake_proc(x_26, x_25, x_9, x_12); +return x_27; +} else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -lean_dec(x_62); +uint8_t x_28; +lean_dec(x_9); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_75 = lean_ctor_get(x_67, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_67, 1); -lean_inc(x_76); -if (lean_is_exclusive(x_67)) { - lean_ctor_release(x_67, 0); - lean_ctor_release(x_67, 1); - x_77 = x_67; -} else { - lean_dec_ref(x_67); - x_77 = lean_box(0); -} -if (lean_is_scalar(x_77)) { - x_78 = lean_alloc_ctor(1, 2, 0); -} else { - x_78 = x_77; -} -lean_ctor_set(x_78, 0, x_75); -lean_ctor_set(x_78, 1, x_76); -return x_78; +x_28 = !lean_is_exclusive(x_10); +if (x_28 == 0) +{ +return x_10; } +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_10, 0); +x_30 = lean_ctor_get(x_10, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_10); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } } else { -uint8_t x_79; +uint8_t x_32; lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_79 = !lean_is_exclusive(x_44); -if (x_79 == 0) +x_32 = !lean_is_exclusive(x_7); +if (x_32 == 0) { -lean_object* x_80; -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_44); -lean_ctor_set(x_80, 1, x_45); -return x_80; +lean_object* x_33; +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_7); +lean_ctor_set(x_33, 1, x_8); +return x_33; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_81 = lean_ctor_get(x_44, 0); -x_82 = lean_ctor_get(x_44, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_44); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -x_84 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_84, 0, x_83); -lean_ctor_set(x_84, 1, x_45); -return x_84; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_7, 0); +x_35 = lean_ctor_get(x_7, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_7); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_8); +return x_37; } } } @@ -4508,20 +4468,20 @@ l_Lake_compileO___closed__1 = _init_l_Lake_compileO___closed__1(); lean_mark_persistent(l_Lake_compileO___closed__1); l_Lake_compileStaticLib___closed__1 = _init_l_Lake_compileStaticLib___closed__1(); lean_mark_persistent(l_Lake_compileStaticLib___closed__1); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__1); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__2); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__3); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__4); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__5); +l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6 = _init_l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6(); +lean_mark_persistent(l___private_Lake_Build_Actions_0__Lake_getMacOSXDeploymentEnv___closed__6); l_Lake_compileSharedLib___closed__1 = _init_l_Lake_compileSharedLib___closed__1(); lean_mark_persistent(l_Lake_compileSharedLib___closed__1); -l_Lake_compileExe___closed__1 = _init_l_Lake_compileExe___closed__1(); -lean_mark_persistent(l_Lake_compileExe___closed__1); -l_Lake_compileExe___closed__2 = _init_l_Lake_compileExe___closed__2(); -lean_mark_persistent(l_Lake_compileExe___closed__2); -l_Lake_compileExe___closed__3 = _init_l_Lake_compileExe___closed__3(); -lean_mark_persistent(l_Lake_compileExe___closed__3); -l_Lake_compileExe___closed__4 = _init_l_Lake_compileExe___closed__4(); -lean_mark_persistent(l_Lake_compileExe___closed__4); -l_Lake_compileExe___closed__5 = _init_l_Lake_compileExe___closed__5(); -lean_mark_persistent(l_Lake_compileExe___closed__5); -l_Lake_compileExe___closed__6 = _init_l_Lake_compileExe___closed__6(); -lean_mark_persistent(l_Lake_compileExe___closed__6); l_Array_foldlMUnsafe_fold___at_Lake_download___spec__1___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lake_download___spec__1___closed__1(); lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lake_download___spec__1___closed__1); l_Lake_download___lambda__1___closed__1 = _init_l_Lake_download___lambda__1___closed__1(); diff --git a/stage0/stdlib/Lake/Build/Common.c b/stage0/stdlib/Lake/Build/Common.c index b53952b6aa6b..02e7127dff60 100644 --- a/stage0/stdlib/Lake/Build/Common.c +++ b/stage0/stdlib/Lake/Build/Common.c @@ -17425,245 +17425,303 @@ if (x_17 == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; x_18 = lean_ctor_get(x_7, 0); -x_19 = l_Lake_compileSharedLib(x_4, x_15, x_16, x_18, x_8); +x_19 = lean_ctor_get(x_7, 1); +x_20 = l_Lake_compileSharedLib(x_4, x_15, x_16, x_18, x_8); lean_dec(x_15); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); if (lean_obj_tag(x_20) == 0) { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = !lean_is_exclusive(x_20); -if (x_23 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_20); +if (x_22 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_20, 1); -lean_ctor_set(x_7, 0, x_24); -lean_ctor_set(x_20, 1, x_7); -return x_19; +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_20, 0); +lean_dec(x_23); +x_24 = !lean_is_exclusive(x_21); +if (x_24 == 0) +{ +lean_object* x_25; +x_25 = lean_ctor_get(x_21, 1); +lean_ctor_set(x_7, 0, x_25); +lean_ctor_set(x_21, 1, x_7); +return x_20; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_20, 0); -x_26 = lean_ctor_get(x_20, 1); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 0); +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_20); -lean_ctor_set(x_7, 0, x_26); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_7); -lean_ctor_set(x_19, 0, x_27); -return x_19; +lean_dec(x_21); +lean_ctor_set(x_7, 0, x_27); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_7); +lean_ctor_set(x_20, 0, x_28); +return x_20; } } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_28 = lean_ctor_get(x_19, 1); -lean_inc(x_28); -lean_dec(x_19); -x_29 = lean_ctor_get(x_20, 0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_20, 1); lean_inc(x_29); -x_30 = lean_ctor_get(x_20, 1); +lean_dec(x_20); +x_30 = lean_ctor_get(x_21, 0); lean_inc(x_30); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - lean_ctor_release(x_20, 1); - x_31 = x_20; +x_31 = lean_ctor_get(x_21, 1); +lean_inc(x_31); +if (lean_is_exclusive(x_21)) { + lean_ctor_release(x_21, 0); + lean_ctor_release(x_21, 1); + x_32 = x_21; } else { - lean_dec_ref(x_20); - x_31 = lean_box(0); + lean_dec_ref(x_21); + x_32 = lean_box(0); } -lean_ctor_set(x_7, 0, x_30); -if (lean_is_scalar(x_31)) { - x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_31); +if (lean_is_scalar(x_32)) { + x_33 = lean_alloc_ctor(0, 2, 0); } else { - x_32 = x_31; + x_33 = x_32; } -lean_ctor_set(x_32, 0, x_29); -lean_ctor_set(x_32, 1, x_7); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_28); -return x_33; +lean_ctor_set(x_33, 0, x_30); +lean_ctor_set(x_33, 1, x_7); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_29); +return x_34; } } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_19); -if (x_34 == 0) +uint8_t x_35; +x_35 = !lean_is_exclusive(x_20); +if (x_35 == 0) { -lean_object* x_35; uint8_t x_36; -x_35 = lean_ctor_get(x_19, 0); -lean_dec(x_35); -x_36 = !lean_is_exclusive(x_20); -if (x_36 == 0) +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_20, 0); +lean_dec(x_36); +x_37 = !lean_is_exclusive(x_21); +if (x_37 == 0) { -lean_object* x_37; -x_37 = lean_ctor_get(x_20, 1); -lean_ctor_set(x_7, 0, x_37); -lean_ctor_set(x_20, 1, x_7); -return x_19; +lean_object* x_38; +x_38 = lean_ctor_get(x_21, 1); +lean_ctor_set(x_7, 0, x_38); +lean_ctor_set(x_21, 1, x_7); +return x_20; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_20, 0); -x_39 = lean_ctor_get(x_20, 1); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_21, 0); +x_40 = lean_ctor_get(x_21, 1); +lean_inc(x_40); lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_20); -lean_ctor_set(x_7, 0, x_39); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_7); -lean_ctor_set(x_19, 0, x_40); -return x_19; +lean_dec(x_21); +lean_ctor_set(x_7, 0, x_40); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_7); +lean_ctor_set(x_20, 0, x_41); +return x_20; } } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_41 = lean_ctor_get(x_19, 1); -lean_inc(x_41); -lean_dec(x_19); -x_42 = lean_ctor_get(x_20, 0); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_42 = lean_ctor_get(x_20, 1); lean_inc(x_42); -x_43 = lean_ctor_get(x_20, 1); +lean_dec(x_20); +x_43 = lean_ctor_get(x_21, 0); lean_inc(x_43); -if (lean_is_exclusive(x_20)) { - lean_ctor_release(x_20, 0); - lean_ctor_release(x_20, 1); - x_44 = x_20; +x_44 = lean_ctor_get(x_21, 1); +lean_inc(x_44); +if (lean_is_exclusive(x_21)) { + lean_ctor_release(x_21, 0); + lean_ctor_release(x_21, 1); + x_45 = x_21; } else { - lean_dec_ref(x_20); - x_44 = lean_box(0); + lean_dec_ref(x_21); + x_45 = lean_box(0); } -lean_ctor_set(x_7, 0, x_43); -if (lean_is_scalar(x_44)) { - x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_44); +if (lean_is_scalar(x_45)) { + x_46 = lean_alloc_ctor(1, 2, 0); } else { - x_45 = x_44; + x_46 = x_45; } -lean_ctor_set(x_45, 0, x_42); -lean_ctor_set(x_45, 1, x_7); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_41); -return x_46; +lean_ctor_set(x_46, 0, x_43); +lean_ctor_set(x_46, 1, x_7); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_42); +return x_47; } } } else { -lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_47 = lean_ctor_get(x_7, 0); -x_48 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); -x_49 = lean_ctor_get(x_7, 1); +uint8_t x_48; +lean_free_object(x_7); +lean_dec(x_19); +x_48 = !lean_is_exclusive(x_20); +if (x_48 == 0) +{ +return x_20; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_20, 0); +x_50 = lean_ctor_get(x_20, 1); +lean_inc(x_50); lean_inc(x_49); -lean_inc(x_47); +lean_dec(x_20); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; +x_52 = lean_ctor_get(x_7, 0); +x_53 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); +x_54 = lean_ctor_get(x_7, 1); +lean_inc(x_54); +lean_inc(x_52); lean_dec(x_7); -x_50 = l_Lake_compileSharedLib(x_4, x_15, x_16, x_47, x_8); +x_55 = l_Lake_compileSharedLib(x_4, x_15, x_16, x_52, x_8); lean_dec(x_15); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -if (lean_obj_tag(x_51) == 0) +if (lean_obj_tag(x_55) == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_53 = x_50; +lean_object* x_56; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +if (lean_obj_tag(x_56) == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_58 = x_55; } else { - lean_dec_ref(x_50); - x_53 = lean_box(0); + lean_dec_ref(x_55); + x_58 = lean_box(0); } -x_54 = lean_ctor_get(x_51, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_51, 1); -lean_inc(x_55); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_56 = x_51; +x_59 = lean_ctor_get(x_56, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_56, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_61 = x_56; } else { - lean_dec_ref(x_51); - x_56 = lean_box(0); + lean_dec_ref(x_56); + x_61 = lean_box(0); } -x_57 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_49); -lean_ctor_set_uint8(x_57, sizeof(void*)*2, x_48); -if (lean_is_scalar(x_56)) { - x_58 = lean_alloc_ctor(0, 2, 0); +x_62 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_54); +lean_ctor_set_uint8(x_62, sizeof(void*)*2, x_53); +if (lean_is_scalar(x_61)) { + x_63 = lean_alloc_ctor(0, 2, 0); } else { - x_58 = x_56; + x_63 = x_61; } -lean_ctor_set(x_58, 0, x_54); -lean_ctor_set(x_58, 1, x_57); -if (lean_is_scalar(x_53)) { - x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_59); +lean_ctor_set(x_63, 1, x_62); +if (lean_is_scalar(x_58)) { + x_64 = lean_alloc_ctor(0, 2, 0); } else { - x_59 = x_53; + x_64 = x_58; } -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_52); -return x_59; +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_57); +return x_64; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_ctor_get(x_50, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_61 = x_50; +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_65 = lean_ctor_get(x_55, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_66 = x_55; } else { - lean_dec_ref(x_50); - x_61 = lean_box(0); + lean_dec_ref(x_55); + x_66 = lean_box(0); } -x_62 = lean_ctor_get(x_51, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_51, 1); -lean_inc(x_63); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_64 = x_51; +x_67 = lean_ctor_get(x_56, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_56, 1); +lean_inc(x_68); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_69 = x_56; } else { - lean_dec_ref(x_51); - x_64 = lean_box(0); + lean_dec_ref(x_56); + x_69 = lean_box(0); } -x_65 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_49); -lean_ctor_set_uint8(x_65, sizeof(void*)*2, x_48); -if (lean_is_scalar(x_64)) { - x_66 = lean_alloc_ctor(1, 2, 0); +x_70 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_54); +lean_ctor_set_uint8(x_70, sizeof(void*)*2, x_53); +if (lean_is_scalar(x_69)) { + x_71 = lean_alloc_ctor(1, 2, 0); } else { - x_66 = x_64; + x_71 = x_69; } -lean_ctor_set(x_66, 0, x_62); -lean_ctor_set(x_66, 1, x_65); -if (lean_is_scalar(x_61)) { - x_67 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_67); +lean_ctor_set(x_71, 1, x_70); +if (lean_is_scalar(x_66)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_61; + x_72 = x_66; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_60); -return x_67; +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_65); +return x_72; +} +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_dec(x_54); +x_73 = lean_ctor_get(x_55, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_55, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_75 = x_55; +} else { + lean_dec_ref(x_55); + x_75 = lean_box(0); +} +if (lean_is_scalar(x_75)) { + x_76 = lean_alloc_ctor(1, 2, 0); +} else { + x_76 = x_75; +} +lean_ctor_set(x_76, 0, x_73); +lean_ctor_set(x_76, 1, x_74); +return x_76; } } } @@ -18608,548 +18666,663 @@ lean_dec(x_5); x_11 = !lean_is_exclusive(x_7); if (x_11 == 0) { -lean_object* x_12; uint8_t x_13; +lean_object* x_12; lean_object* x_13; uint8_t x_14; x_12 = lean_ctor_get(x_7, 0); -x_13 = l_System_Platform_isOSX; -if (x_13 == 0) +x_13 = lean_ctor_get(x_7, 1); +x_14 = l_System_Platform_isOSX; +if (x_14 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_14 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__2; -x_15 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_15, 0, x_1); -lean_ctor_set(x_15, 1, x_14); -x_16 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__3; -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = lean_array_mk(x_17); -x_19 = l_Array_append___rarg(x_18, x_2); -x_20 = l_Array_append___rarg(x_19, x_3); -x_21 = l_Array_append___rarg(x_20, x_9); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_15 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__2; +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_1); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__3; +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +x_19 = lean_array_mk(x_18); +x_20 = l_Array_append___rarg(x_19, x_2); +x_21 = l_Array_append___rarg(x_20, x_3); +x_22 = l_Array_append___rarg(x_21, x_9); lean_dec(x_9); -x_22 = l_Lake_compileSharedLib(x_4, x_21, x_10, x_12, x_8); -lean_dec(x_21); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); +x_23 = l_Lake_compileSharedLib(x_4, x_22, x_10, x_12, x_8); +lean_dec(x_22); if (lean_obj_tag(x_23) == 0) { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_22); -if (x_24 == 0) +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_25; uint8_t x_26; -x_25 = lean_ctor_get(x_22, 0); -lean_dec(x_25); -x_26 = !lean_is_exclusive(x_23); -if (x_26 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_23); +if (x_25 == 0) { -lean_object* x_27; -x_27 = lean_ctor_get(x_23, 1); -lean_ctor_set(x_7, 0, x_27); -lean_ctor_set(x_23, 1, x_7); -return x_22; +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) +{ +lean_object* x_28; +x_28 = lean_ctor_get(x_24, 1); +lean_ctor_set(x_7, 0, x_28); +lean_ctor_set(x_24, 1, x_7); +return x_23; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 0); -x_29 = lean_ctor_get(x_23, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_23); -lean_ctor_set(x_7, 0, x_29); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_7); -lean_ctor_set(x_22, 0, x_30); -return x_22; +lean_dec(x_24); +lean_ctor_set(x_7, 0, x_30); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_7); +lean_ctor_set(x_23, 0, x_31); +return x_23; } } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_31 = lean_ctor_get(x_22, 1); -lean_inc(x_31); -lean_dec(x_22); -x_32 = lean_ctor_get(x_23, 0); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_32 = lean_ctor_get(x_23, 1); lean_inc(x_32); -x_33 = lean_ctor_get(x_23, 1); +lean_dec(x_23); +x_33 = lean_ctor_get(x_24, 0); lean_inc(x_33); -if (lean_is_exclusive(x_23)) { - lean_ctor_release(x_23, 0); - lean_ctor_release(x_23, 1); - x_34 = x_23; +x_34 = lean_ctor_get(x_24, 1); +lean_inc(x_34); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_35 = x_24; } else { - lean_dec_ref(x_23); - x_34 = lean_box(0); + lean_dec_ref(x_24); + x_35 = lean_box(0); } -lean_ctor_set(x_7, 0, x_33); -if (lean_is_scalar(x_34)) { - x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_34); +if (lean_is_scalar(x_35)) { + x_36 = lean_alloc_ctor(0, 2, 0); } else { - x_35 = x_34; + x_36 = x_35; } -lean_ctor_set(x_35, 0, x_32); -lean_ctor_set(x_35, 1, x_7); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_31); -return x_36; +lean_ctor_set(x_36, 0, x_33); +lean_ctor_set(x_36, 1, x_7); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_32); +return x_37; } } else { -uint8_t x_37; -x_37 = !lean_is_exclusive(x_22); -if (x_37 == 0) +uint8_t x_38; +x_38 = !lean_is_exclusive(x_23); +if (x_38 == 0) { -lean_object* x_38; uint8_t x_39; -x_38 = lean_ctor_get(x_22, 0); -lean_dec(x_38); -x_39 = !lean_is_exclusive(x_23); -if (x_39 == 0) +lean_object* x_39; uint8_t x_40; +x_39 = lean_ctor_get(x_23, 0); +lean_dec(x_39); +x_40 = !lean_is_exclusive(x_24); +if (x_40 == 0) { -lean_object* x_40; -x_40 = lean_ctor_get(x_23, 1); -lean_ctor_set(x_7, 0, x_40); -lean_ctor_set(x_23, 1, x_7); -return x_22; +lean_object* x_41; +x_41 = lean_ctor_get(x_24, 1); +lean_ctor_set(x_7, 0, x_41); +lean_ctor_set(x_24, 1, x_7); +return x_23; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_23, 0); -x_42 = lean_ctor_get(x_23, 1); +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_24, 0); +x_43 = lean_ctor_get(x_24, 1); +lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_23); -lean_ctor_set(x_7, 0, x_42); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_7); -lean_ctor_set(x_22, 0, x_43); -return x_22; +lean_dec(x_24); +lean_ctor_set(x_7, 0, x_43); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_7); +lean_ctor_set(x_23, 0, x_44); +return x_23; } } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_44 = lean_ctor_get(x_22, 1); -lean_inc(x_44); -lean_dec(x_22); -x_45 = lean_ctor_get(x_23, 0); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_23, 1); lean_inc(x_45); -x_46 = lean_ctor_get(x_23, 1); +lean_dec(x_23); +x_46 = lean_ctor_get(x_24, 0); lean_inc(x_46); -if (lean_is_exclusive(x_23)) { - lean_ctor_release(x_23, 0); - lean_ctor_release(x_23, 1); - x_47 = x_23; +x_47 = lean_ctor_get(x_24, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_48 = x_24; } else { - lean_dec_ref(x_23); - x_47 = lean_box(0); + lean_dec_ref(x_24); + x_48 = lean_box(0); } -lean_ctor_set(x_7, 0, x_46); -if (lean_is_scalar(x_47)) { - x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_47); +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(1, 2, 0); } else { - x_48 = x_47; + x_49 = x_48; } -lean_ctor_set(x_48, 0, x_45); -lean_ctor_set(x_48, 1, x_7); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_44); -return x_49; +lean_ctor_set(x_49, 0, x_46); +lean_ctor_set(x_49, 1, x_7); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_45); +return x_50; } } } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_50 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__4; -x_51 = lean_string_append(x_50, x_1); +uint8_t x_51; +lean_free_object(x_7); +lean_dec(x_13); +x_51 = !lean_is_exclusive(x_23); +if (x_51 == 0) +{ +return x_23; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_23, 0); +x_53 = lean_ctor_get(x_23, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_23); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_55 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__4; +x_56 = lean_string_append(x_55, x_1); lean_dec(x_1); -x_52 = l_Lake_BuildMetadata_fromJson_x3f___closed__1; -x_53 = lean_string_append(x_51, x_52); -x_54 = lean_box(0); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_array_mk(x_55); -x_57 = l_Array_append___rarg(x_56, x_2); -x_58 = l_Array_append___rarg(x_57, x_3); -x_59 = l_Array_append___rarg(x_58, x_9); +x_57 = l_Lake_BuildMetadata_fromJson_x3f___closed__1; +x_58 = lean_string_append(x_56, x_57); +x_59 = lean_box(0); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +x_61 = lean_array_mk(x_60); +x_62 = l_Array_append___rarg(x_61, x_2); +x_63 = l_Array_append___rarg(x_62, x_3); +x_64 = l_Array_append___rarg(x_63, x_9); lean_dec(x_9); -x_60 = l_Lake_compileSharedLib(x_4, x_59, x_10, x_12, x_8); -lean_dec(x_59); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -if (lean_obj_tag(x_61) == 0) +x_65 = l_Lake_compileSharedLib(x_4, x_64, x_10, x_12, x_8); +lean_dec(x_64); +if (lean_obj_tag(x_65) == 0) { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_60); -if (x_62 == 0) +lean_object* x_66; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +if (lean_obj_tag(x_66) == 0) { -lean_object* x_63; uint8_t x_64; -x_63 = lean_ctor_get(x_60, 0); -lean_dec(x_63); -x_64 = !lean_is_exclusive(x_61); -if (x_64 == 0) +uint8_t x_67; +x_67 = !lean_is_exclusive(x_65); +if (x_67 == 0) { -lean_object* x_65; -x_65 = lean_ctor_get(x_61, 1); -lean_ctor_set(x_7, 0, x_65); -lean_ctor_set(x_61, 1, x_7); -return x_60; +lean_object* x_68; uint8_t x_69; +x_68 = lean_ctor_get(x_65, 0); +lean_dec(x_68); +x_69 = !lean_is_exclusive(x_66); +if (x_69 == 0) +{ +lean_object* x_70; +x_70 = lean_ctor_get(x_66, 1); +lean_ctor_set(x_7, 0, x_70); +lean_ctor_set(x_66, 1, x_7); +return x_65; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_61, 0); -x_67 = lean_ctor_get(x_61, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_61); -lean_ctor_set(x_7, 0, x_67); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_7); -lean_ctor_set(x_60, 0, x_68); -return x_60; +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_66, 0); +x_72 = lean_ctor_get(x_66, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_66); +lean_ctor_set(x_7, 0, x_72); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_7); +lean_ctor_set(x_65, 0, x_73); +return x_65; } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_69 = lean_ctor_get(x_60, 1); -lean_inc(x_69); -lean_dec(x_60); -x_70 = lean_ctor_get(x_61, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_61, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_72 = x_61; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_74 = lean_ctor_get(x_65, 1); +lean_inc(x_74); +lean_dec(x_65); +x_75 = lean_ctor_get(x_66, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_66, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_77 = x_66; } else { - lean_dec_ref(x_61); - x_72 = lean_box(0); + lean_dec_ref(x_66); + x_77 = lean_box(0); } -lean_ctor_set(x_7, 0, x_71); -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_76); +if (lean_is_scalar(x_77)) { + x_78 = lean_alloc_ctor(0, 2, 0); } else { - x_73 = x_72; + x_78 = x_77; } -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_7); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_69); -return x_74; +lean_ctor_set(x_78, 0, x_75); +lean_ctor_set(x_78, 1, x_7); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_74); +return x_79; } } else { -uint8_t x_75; -x_75 = !lean_is_exclusive(x_60); -if (x_75 == 0) +uint8_t x_80; +x_80 = !lean_is_exclusive(x_65); +if (x_80 == 0) { -lean_object* x_76; uint8_t x_77; -x_76 = lean_ctor_get(x_60, 0); -lean_dec(x_76); -x_77 = !lean_is_exclusive(x_61); -if (x_77 == 0) +lean_object* x_81; uint8_t x_82; +x_81 = lean_ctor_get(x_65, 0); +lean_dec(x_81); +x_82 = !lean_is_exclusive(x_66); +if (x_82 == 0) { -lean_object* x_78; -x_78 = lean_ctor_get(x_61, 1); -lean_ctor_set(x_7, 0, x_78); -lean_ctor_set(x_61, 1, x_7); -return x_60; +lean_object* x_83; +x_83 = lean_ctor_get(x_66, 1); +lean_ctor_set(x_7, 0, x_83); +lean_ctor_set(x_66, 1, x_7); +return x_65; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_61, 0); -x_80 = lean_ctor_get(x_61, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_61); -lean_ctor_set(x_7, 0, x_80); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_7); -lean_ctor_set(x_60, 0, x_81); -return x_60; +lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_84 = lean_ctor_get(x_66, 0); +x_85 = lean_ctor_get(x_66, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_66); +lean_ctor_set(x_7, 0, x_85); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_7); +lean_ctor_set(x_65, 0, x_86); +return x_65; } } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_82 = lean_ctor_get(x_60, 1); -lean_inc(x_82); -lean_dec(x_60); -x_83 = lean_ctor_get(x_61, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_61, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_85 = x_61; +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_87 = lean_ctor_get(x_65, 1); +lean_inc(x_87); +lean_dec(x_65); +x_88 = lean_ctor_get(x_66, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_66, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_90 = x_66; } else { - lean_dec_ref(x_61); - x_85 = lean_box(0); + lean_dec_ref(x_66); + x_90 = lean_box(0); } -lean_ctor_set(x_7, 0, x_84); -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_89); +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); } else { - x_86 = x_85; + x_91 = x_90; } -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_7); -x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_82); -return x_87; +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_7); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_87); +return x_92; } } } +else +{ +uint8_t x_93; +lean_free_object(x_7); +lean_dec(x_13); +x_93 = !lean_is_exclusive(x_65); +if (x_93 == 0) +{ +return x_65; } else { -lean_object* x_88; uint8_t x_89; lean_object* x_90; uint8_t x_91; -x_88 = lean_ctor_get(x_7, 0); -x_89 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); -x_90 = lean_ctor_get(x_7, 1); -lean_inc(x_90); -lean_inc(x_88); +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_65, 0); +x_95 = lean_ctor_get(x_65, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_65); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +return x_96; +} +} +} +} +else +{ +lean_object* x_97; uint8_t x_98; lean_object* x_99; uint8_t x_100; +x_97 = lean_ctor_get(x_7, 0); +x_98 = lean_ctor_get_uint8(x_7, sizeof(void*)*2); +x_99 = lean_ctor_get(x_7, 1); +lean_inc(x_99); +lean_inc(x_97); lean_dec(x_7); -x_91 = l_System_Platform_isOSX; -if (x_91 == 0) +x_100 = l_System_Platform_isOSX; +if (x_100 == 0) { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_92 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__2; -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_1); -lean_ctor_set(x_93, 1, x_92); -x_94 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__3; -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_93); -x_96 = lean_array_mk(x_95); -x_97 = l_Array_append___rarg(x_96, x_2); -x_98 = l_Array_append___rarg(x_97, x_3); -x_99 = l_Array_append___rarg(x_98, x_9); +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_101 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__2; +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_1); +lean_ctor_set(x_102, 1, x_101); +x_103 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__3; +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_102); +x_105 = lean_array_mk(x_104); +x_106 = l_Array_append___rarg(x_105, x_2); +x_107 = l_Array_append___rarg(x_106, x_3); +x_108 = l_Array_append___rarg(x_107, x_9); lean_dec(x_9); -x_100 = l_Lake_compileSharedLib(x_4, x_99, x_10, x_88, x_8); -lean_dec(x_99); -x_101 = lean_ctor_get(x_100, 0); -lean_inc(x_101); -if (lean_obj_tag(x_101) == 0) +x_109 = l_Lake_compileSharedLib(x_4, x_108, x_10, x_97, x_8); +lean_dec(x_108); +if (lean_obj_tag(x_109) == 0) { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_102 = lean_ctor_get(x_100, 1); -lean_inc(x_102); -if (lean_is_exclusive(x_100)) { - lean_ctor_release(x_100, 0); - lean_ctor_release(x_100, 1); - x_103 = x_100; +lean_object* x_110; +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +if (lean_obj_tag(x_110) == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_112 = x_109; } else { - lean_dec_ref(x_100); - x_103 = lean_box(0); + lean_dec_ref(x_109); + x_112 = lean_box(0); } -x_104 = lean_ctor_get(x_101, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_101, 1); -lean_inc(x_105); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_106 = x_101; +x_113 = lean_ctor_get(x_110, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_110, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_115 = x_110; } else { - lean_dec_ref(x_101); - x_106 = lean_box(0); + lean_dec_ref(x_110); + x_115 = lean_box(0); } -x_107 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_90); -lean_ctor_set_uint8(x_107, sizeof(void*)*2, x_89); -if (lean_is_scalar(x_106)) { - x_108 = lean_alloc_ctor(0, 2, 0); +x_116 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_99); +lean_ctor_set_uint8(x_116, sizeof(void*)*2, x_98); +if (lean_is_scalar(x_115)) { + x_117 = lean_alloc_ctor(0, 2, 0); } else { - x_108 = x_106; + x_117 = x_115; } -lean_ctor_set(x_108, 0, x_104); -lean_ctor_set(x_108, 1, x_107); -if (lean_is_scalar(x_103)) { - x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_113); +lean_ctor_set(x_117, 1, x_116); +if (lean_is_scalar(x_112)) { + x_118 = lean_alloc_ctor(0, 2, 0); } else { - x_109 = x_103; + x_118 = x_112; } -lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_102); -return x_109; +lean_ctor_set(x_118, 0, x_117); +lean_ctor_set(x_118, 1, x_111); +return x_118; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_110 = lean_ctor_get(x_100, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_100)) { - lean_ctor_release(x_100, 0); - lean_ctor_release(x_100, 1); - x_111 = x_100; +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_119 = lean_ctor_get(x_109, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_120 = x_109; } else { - lean_dec_ref(x_100); - x_111 = lean_box(0); + lean_dec_ref(x_109); + x_120 = lean_box(0); } -x_112 = lean_ctor_get(x_101, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_101, 1); -lean_inc(x_113); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_114 = x_101; +x_121 = lean_ctor_get(x_110, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_110, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_110)) { + lean_ctor_release(x_110, 0); + lean_ctor_release(x_110, 1); + x_123 = x_110; } else { - lean_dec_ref(x_101); - x_114 = lean_box(0); + lean_dec_ref(x_110); + x_123 = lean_box(0); } -x_115 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_90); -lean_ctor_set_uint8(x_115, sizeof(void*)*2, x_89); -if (lean_is_scalar(x_114)) { - x_116 = lean_alloc_ctor(1, 2, 0); +x_124 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_99); +lean_ctor_set_uint8(x_124, sizeof(void*)*2, x_98); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(1, 2, 0); } else { - x_116 = x_114; + x_125 = x_123; } -lean_ctor_set(x_116, 0, x_112); -lean_ctor_set(x_116, 1, x_115); -if (lean_is_scalar(x_111)) { - x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_121); +lean_ctor_set(x_125, 1, x_124); +if (lean_is_scalar(x_120)) { + x_126 = lean_alloc_ctor(0, 2, 0); } else { - x_117 = x_111; + x_126 = x_120; } -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_117, 1, x_110); -return x_117; +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_119); +return x_126; } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_118 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__4; -x_119 = lean_string_append(x_118, x_1); +lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_dec(x_99); +x_127 = lean_ctor_get(x_109, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_109, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_129 = x_109; +} else { + lean_dec_ref(x_109); + x_129 = lean_box(0); +} +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); +} else { + x_130 = x_129; +} +lean_ctor_set(x_130, 0, x_127); +lean_ctor_set(x_130, 1, x_128); +return x_130; +} +} +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_131 = l_Lake_buildLeanSharedLibOfStatic___lambda__1___closed__4; +x_132 = lean_string_append(x_131, x_1); lean_dec(x_1); -x_120 = l_Lake_BuildMetadata_fromJson_x3f___closed__1; -x_121 = lean_string_append(x_119, x_120); -x_122 = lean_box(0); -x_123 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); -x_124 = lean_array_mk(x_123); -x_125 = l_Array_append___rarg(x_124, x_2); -x_126 = l_Array_append___rarg(x_125, x_3); -x_127 = l_Array_append___rarg(x_126, x_9); +x_133 = l_Lake_BuildMetadata_fromJson_x3f___closed__1; +x_134 = lean_string_append(x_132, x_133); +x_135 = lean_box(0); +x_136 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +x_137 = lean_array_mk(x_136); +x_138 = l_Array_append___rarg(x_137, x_2); +x_139 = l_Array_append___rarg(x_138, x_3); +x_140 = l_Array_append___rarg(x_139, x_9); lean_dec(x_9); -x_128 = l_Lake_compileSharedLib(x_4, x_127, x_10, x_88, x_8); -lean_dec(x_127); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -if (lean_obj_tag(x_129) == 0) +x_141 = l_Lake_compileSharedLib(x_4, x_140, x_10, x_97, x_8); +lean_dec(x_140); +if (lean_obj_tag(x_141) == 0) { -lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_128)) { - lean_ctor_release(x_128, 0); - lean_ctor_release(x_128, 1); - x_131 = x_128; -} else { - lean_dec_ref(x_128); - x_131 = lean_box(0); -} -x_132 = lean_ctor_get(x_129, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_129, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_129)) { - lean_ctor_release(x_129, 0); - lean_ctor_release(x_129, 1); - x_134 = x_129; +lean_object* x_142; +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +if (lean_obj_tag(x_142) == 0) +{ +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_144 = x_141; } else { - lean_dec_ref(x_129); - x_134 = lean_box(0); + lean_dec_ref(x_141); + x_144 = lean_box(0); } -x_135 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_90); -lean_ctor_set_uint8(x_135, sizeof(void*)*2, x_89); -if (lean_is_scalar(x_134)) { - x_136 = lean_alloc_ctor(0, 2, 0); +x_145 = lean_ctor_get(x_142, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_142, 1); +lean_inc(x_146); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + lean_ctor_release(x_142, 1); + x_147 = x_142; +} else { + lean_dec_ref(x_142); + x_147 = lean_box(0); +} +x_148 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_148, 0, x_146); +lean_ctor_set(x_148, 1, x_99); +lean_ctor_set_uint8(x_148, sizeof(void*)*2, x_98); +if (lean_is_scalar(x_147)) { + x_149 = lean_alloc_ctor(0, 2, 0); } else { - x_136 = x_134; + x_149 = x_147; } -lean_ctor_set(x_136, 0, x_132); -lean_ctor_set(x_136, 1, x_135); -if (lean_is_scalar(x_131)) { - x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_145); +lean_ctor_set(x_149, 1, x_148); +if (lean_is_scalar(x_144)) { + x_150 = lean_alloc_ctor(0, 2, 0); } else { - x_137 = x_131; + x_150 = x_144; } -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_130); -return x_137; +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_143); +return x_150; } else { -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_138 = lean_ctor_get(x_128, 1); -lean_inc(x_138); -if (lean_is_exclusive(x_128)) { - lean_ctor_release(x_128, 0); - lean_ctor_release(x_128, 1); - x_139 = x_128; +lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_151 = lean_ctor_get(x_141, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_152 = x_141; } else { - lean_dec_ref(x_128); - x_139 = lean_box(0); + lean_dec_ref(x_141); + x_152 = lean_box(0); } -x_140 = lean_ctor_get(x_129, 0); -lean_inc(x_140); -x_141 = lean_ctor_get(x_129, 1); -lean_inc(x_141); -if (lean_is_exclusive(x_129)) { - lean_ctor_release(x_129, 0); - lean_ctor_release(x_129, 1); - x_142 = x_129; +x_153 = lean_ctor_get(x_142, 0); +lean_inc(x_153); +x_154 = lean_ctor_get(x_142, 1); +lean_inc(x_154); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + lean_ctor_release(x_142, 1); + x_155 = x_142; } else { - lean_dec_ref(x_129); - x_142 = lean_box(0); + lean_dec_ref(x_142); + x_155 = lean_box(0); } -x_143 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_143, 0, x_141); -lean_ctor_set(x_143, 1, x_90); -lean_ctor_set_uint8(x_143, sizeof(void*)*2, x_89); -if (lean_is_scalar(x_142)) { - x_144 = lean_alloc_ctor(1, 2, 0); +x_156 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_156, 0, x_154); +lean_ctor_set(x_156, 1, x_99); +lean_ctor_set_uint8(x_156, sizeof(void*)*2, x_98); +if (lean_is_scalar(x_155)) { + x_157 = lean_alloc_ctor(1, 2, 0); } else { - x_144 = x_142; + x_157 = x_155; } -lean_ctor_set(x_144, 0, x_140); -lean_ctor_set(x_144, 1, x_143); -if (lean_is_scalar(x_139)) { - x_145 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_157, 0, x_153); +lean_ctor_set(x_157, 1, x_156); +if (lean_is_scalar(x_152)) { + x_158 = lean_alloc_ctor(0, 2, 0); } else { - x_145 = x_139; + x_158 = x_152; } -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_138); -return x_145; +lean_ctor_set(x_158, 0, x_157); +lean_ctor_set(x_158, 1, x_151); +return x_158; +} +} +else +{ +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +lean_dec(x_99); +x_159 = lean_ctor_get(x_141, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_141, 1); +lean_inc(x_160); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_161 = x_141; +} else { + lean_dec_ref(x_141); + x_161 = lean_box(0); +} +if (lean_is_scalar(x_161)) { + x_162 = lean_alloc_ctor(1, 2, 0); +} else { + x_162 = x_161; +} +lean_ctor_set(x_162, 0, x_159); +lean_ctor_set(x_162, 1, x_160); +return x_162; } } } diff --git a/stage0/stdlib/Lake/Build/Job.c b/stage0/stdlib/Lake/Build/Job.c index fe3e53f49b9b..218127d0f93a 100644 --- a/stage0/stdlib/Lake/Build/Job.c +++ b/stage0/stdlib/Lake/Build/Job.c @@ -23114,270 +23114,321 @@ lean_dec(x_1); x_5 = !lean_is_exclusive(x_2); if (x_5 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; x_6 = lean_ctor_get(x_2, 1); x_7 = lean_ctor_get(x_2, 0); lean_dec(x_7); +lean_inc(x_4); x_8 = l_Lake_JobState_merge(x_4, x_6); -lean_ctor_set(x_2, 1, x_8); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get_uint8(x_8, sizeof(void*)*2); +lean_dec(x_8); +x_11 = !lean_is_exclusive(x_4); +if (x_11 == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_4, 0); +lean_dec(x_12); +lean_ctor_set(x_4, 0, x_9); +lean_ctor_set_uint8(x_4, sizeof(void*)*2, x_10); +lean_ctor_set(x_2, 1, x_4); lean_ctor_set(x_2, 0, x_3); return x_2; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -lean_dec(x_2); -x_10 = l_Lake_JobState_merge(x_4, x_9); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_3); -lean_ctor_set(x_11, 1, x_10); -return x_11; +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_4, 1); +lean_inc(x_13); +lean_dec(x_4); +x_14 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_14, 0, x_9); +lean_ctor_set(x_14, 1, x_13); +lean_ctor_set_uint8(x_14, sizeof(void*)*2, x_10); +lean_ctor_set(x_2, 1, x_14); +lean_ctor_set(x_2, 0, x_3); +return x_2; } } else { -lean_object* x_12; uint8_t x_13; -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_2); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; -x_14 = lean_ctor_get(x_2, 1); -x_15 = lean_ctor_get(x_2, 0); -lean_dec(x_15); -lean_inc(x_12); -x_16 = l_Lake_JobState_merge(x_12, x_14); +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +lean_dec(x_2); +lean_inc(x_4); +x_16 = l_Lake_JobState_merge(x_4, x_15); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); lean_dec(x_16); -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) +x_19 = lean_ctor_get(x_4, 1); +lean_inc(x_19); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + lean_ctor_release(x_4, 1); + x_20 = x_4; +} else { + lean_dec_ref(x_4); + x_20 = lean_box(0); +} +if (lean_is_scalar(x_20)) { + x_21 = lean_alloc_ctor(0, 2, 1); +} else { + x_21 = x_20; +} +lean_ctor_set(x_21, 0, x_17); +lean_ctor_set(x_21, 1, x_19); +lean_ctor_set_uint8(x_21, sizeof(void*)*2, x_18); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_3); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_12, 0); -lean_dec(x_20); -lean_ctor_set(x_12, 0, x_17); -lean_ctor_set_uint8(x_12, sizeof(void*)*2, x_18); -x_21 = lean_unsigned_to_nat(0u); -lean_ctor_set(x_2, 1, x_12); -lean_ctor_set(x_2, 0, x_21); +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_2); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; uint8_t x_30; +x_25 = lean_ctor_get(x_2, 1); +x_26 = lean_ctor_get(x_2, 0); +lean_dec(x_26); +lean_inc(x_23); +x_27 = l_Lake_JobState_merge(x_23, x_25); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get_uint8(x_27, sizeof(void*)*2); +lean_dec(x_27); +x_30 = !lean_is_exclusive(x_23); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_23, 0); +lean_dec(x_31); +lean_ctor_set(x_23, 0, x_28); +lean_ctor_set_uint8(x_23, sizeof(void*)*2, x_29); +x_32 = lean_unsigned_to_nat(0u); +lean_ctor_set(x_2, 1, x_23); +lean_ctor_set(x_2, 0, x_32); return x_2; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); -lean_dec(x_12); -x_23 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_23, 0, x_17); -lean_ctor_set(x_23, 1, x_22); -lean_ctor_set_uint8(x_23, sizeof(void*)*2, x_18); -x_24 = lean_unsigned_to_nat(0u); -lean_ctor_set(x_2, 1, x_23); -lean_ctor_set(x_2, 0, x_24); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_23, 1); +lean_inc(x_33); +lean_dec(x_23); +x_34 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_34, 0, x_28); +lean_ctor_set(x_34, 1, x_33); +lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_29); +x_35 = lean_unsigned_to_nat(0u); +lean_ctor_set(x_2, 1, x_34); +lean_ctor_set(x_2, 0, x_35); return x_2; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_25 = lean_ctor_get(x_2, 1); -lean_inc(x_25); +lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_36 = lean_ctor_get(x_2, 1); +lean_inc(x_36); lean_dec(x_2); -lean_inc(x_12); -x_26 = l_Lake_JobState_merge(x_12, x_25); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get_uint8(x_26, sizeof(void*)*2); -lean_dec(x_26); -x_29 = lean_ctor_get(x_12, 1); -lean_inc(x_29); -if (lean_is_exclusive(x_12)) { - lean_ctor_release(x_12, 0); - lean_ctor_release(x_12, 1); - x_30 = x_12; +lean_inc(x_23); +x_37 = l_Lake_JobState_merge(x_23, x_36); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get_uint8(x_37, sizeof(void*)*2); +lean_dec(x_37); +x_40 = lean_ctor_get(x_23, 1); +lean_inc(x_40); +if (lean_is_exclusive(x_23)) { + lean_ctor_release(x_23, 0); + lean_ctor_release(x_23, 1); + x_41 = x_23; } else { - lean_dec_ref(x_12); - x_30 = lean_box(0); + lean_dec_ref(x_23); + x_41 = lean_box(0); } -if (lean_is_scalar(x_30)) { - x_31 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_41)) { + x_42 = lean_alloc_ctor(0, 2, 1); } else { - x_31 = x_30; + x_42 = x_41; } -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2, x_28); -x_32 = lean_unsigned_to_nat(0u); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -return x_33; +lean_ctor_set(x_42, 0, x_38); +lean_ctor_set(x_42, 1, x_40); +lean_ctor_set_uint8(x_42, sizeof(void*)*2, x_39); +x_43 = lean_unsigned_to_nat(0u); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_42); +return x_44; } } } else { -lean_object* x_34; -x_34 = lean_ctor_get(x_1, 1); -lean_inc(x_34); +lean_object* x_45; +x_45 = lean_ctor_get(x_1, 1); +lean_inc(x_45); lean_dec(x_1); if (lean_obj_tag(x_2) == 0) { -lean_object* x_35; uint8_t x_36; -x_35 = lean_ctor_get(x_34, 1); -lean_inc(x_35); -x_36 = !lean_is_exclusive(x_2); -if (x_36 == 0) +lean_object* x_46; uint8_t x_47; +x_46 = lean_ctor_get(x_45, 1); +lean_inc(x_46); +x_47 = !lean_is_exclusive(x_2); +if (x_47 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_37 = lean_ctor_get(x_2, 1); -x_38 = lean_ctor_get(x_2, 0); -lean_dec(x_38); -x_39 = l_Lake_JobState_merge(x_34, x_37); -x_40 = !lean_is_exclusive(x_39); -if (x_40 == 0) +lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; +x_48 = lean_ctor_get(x_2, 1); +x_49 = lean_ctor_get(x_2, 0); +lean_dec(x_49); +x_50 = l_Lake_JobState_merge(x_45, x_48); +x_51 = !lean_is_exclusive(x_50); +if (x_51 == 0) { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_39, 1); -lean_dec(x_41); -lean_ctor_set(x_39, 1, x_35); -x_42 = lean_unsigned_to_nat(0u); +lean_object* x_52; lean_object* x_53; +x_52 = lean_ctor_get(x_50, 1); +lean_dec(x_52); +lean_ctor_set(x_50, 1, x_46); +x_53 = lean_unsigned_to_nat(0u); lean_ctor_set_tag(x_2, 1); -lean_ctor_set(x_2, 1, x_39); -lean_ctor_set(x_2, 0, x_42); +lean_ctor_set(x_2, 1, x_50); +lean_ctor_set(x_2, 0, x_53); return x_2; } else { -lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_39, 0); -x_44 = lean_ctor_get_uint8(x_39, sizeof(void*)*2); -lean_inc(x_43); -lean_dec(x_39); -x_45 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_35); -lean_ctor_set_uint8(x_45, sizeof(void*)*2, x_44); -x_46 = lean_unsigned_to_nat(0u); +lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_50, 0); +x_55 = lean_ctor_get_uint8(x_50, sizeof(void*)*2); +lean_inc(x_54); +lean_dec(x_50); +x_56 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_46); +lean_ctor_set_uint8(x_56, sizeof(void*)*2, x_55); +x_57 = lean_unsigned_to_nat(0u); lean_ctor_set_tag(x_2, 1); -lean_ctor_set(x_2, 1, x_45); -lean_ctor_set(x_2, 0, x_46); +lean_ctor_set(x_2, 1, x_56); +lean_ctor_set(x_2, 0, x_57); return x_2; } } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_47 = lean_ctor_get(x_2, 1); -lean_inc(x_47); +lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_58 = lean_ctor_get(x_2, 1); +lean_inc(x_58); lean_dec(x_2); -x_48 = l_Lake_JobState_merge(x_34, x_47); -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get_uint8(x_48, sizeof(void*)*2); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_51 = x_48; +x_59 = l_Lake_JobState_merge(x_45, x_58); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get_uint8(x_59, sizeof(void*)*2); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_62 = x_59; } else { - lean_dec_ref(x_48); - x_51 = lean_box(0); + lean_dec_ref(x_59); + x_62 = lean_box(0); } -if (lean_is_scalar(x_51)) { - x_52 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_62)) { + x_63 = lean_alloc_ctor(0, 2, 1); } else { - x_52 = x_51; + x_63 = x_62; } -lean_ctor_set(x_52, 0, x_49); -lean_ctor_set(x_52, 1, x_35); -lean_ctor_set_uint8(x_52, sizeof(void*)*2, x_50); -x_53 = lean_unsigned_to_nat(0u); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); -return x_54; +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_46); +lean_ctor_set_uint8(x_63, sizeof(void*)*2, x_61); +x_64 = lean_unsigned_to_nat(0u); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } else { -lean_object* x_55; uint8_t x_56; -x_55 = lean_ctor_get(x_34, 1); -lean_inc(x_55); -x_56 = !lean_is_exclusive(x_2); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; -x_57 = lean_ctor_get(x_2, 1); -x_58 = lean_ctor_get(x_2, 0); -lean_dec(x_58); -x_59 = l_Lake_JobState_merge(x_34, x_57); -x_60 = !lean_is_exclusive(x_59); -if (x_60 == 0) +lean_object* x_66; uint8_t x_67; +x_66 = lean_ctor_get(x_45, 1); +lean_inc(x_66); +x_67 = !lean_is_exclusive(x_2); +if (x_67 == 0) { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_59, 1); -lean_dec(x_61); -lean_ctor_set(x_59, 1, x_55); -x_62 = lean_unsigned_to_nat(0u); -lean_ctor_set(x_2, 1, x_59); -lean_ctor_set(x_2, 0, x_62); +lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; +x_68 = lean_ctor_get(x_2, 1); +x_69 = lean_ctor_get(x_2, 0); +lean_dec(x_69); +x_70 = l_Lake_JobState_merge(x_45, x_68); +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) +{ +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_70, 1); +lean_dec(x_72); +lean_ctor_set(x_70, 1, x_66); +x_73 = lean_unsigned_to_nat(0u); +lean_ctor_set(x_2, 1, x_70); +lean_ctor_set(x_2, 0, x_73); return x_2; } else { -lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; -x_63 = lean_ctor_get(x_59, 0); -x_64 = lean_ctor_get_uint8(x_59, sizeof(void*)*2); -lean_inc(x_63); -lean_dec(x_59); -x_65 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_55); -lean_ctor_set_uint8(x_65, sizeof(void*)*2, x_64); -x_66 = lean_unsigned_to_nat(0u); -lean_ctor_set(x_2, 1, x_65); -lean_ctor_set(x_2, 0, x_66); +lean_object* x_74; uint8_t x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_70, 0); +x_75 = lean_ctor_get_uint8(x_70, sizeof(void*)*2); +lean_inc(x_74); +lean_dec(x_70); +x_76 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_66); +lean_ctor_set_uint8(x_76, sizeof(void*)*2, x_75); +x_77 = lean_unsigned_to_nat(0u); +lean_ctor_set(x_2, 1, x_76); +lean_ctor_set(x_2, 0, x_77); return x_2; } } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_67 = lean_ctor_get(x_2, 1); -lean_inc(x_67); +lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_78 = lean_ctor_get(x_2, 1); +lean_inc(x_78); lean_dec(x_2); -x_68 = l_Lake_JobState_merge(x_34, x_67); -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get_uint8(x_68, sizeof(void*)*2); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_71 = x_68; +x_79 = l_Lake_JobState_merge(x_45, x_78); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get_uint8(x_79, sizeof(void*)*2); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_82 = x_79; } else { - lean_dec_ref(x_68); - x_71 = lean_box(0); + lean_dec_ref(x_79); + x_82 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(0, 2, 1); } else { - x_72 = x_71; + x_83 = x_82; } -lean_ctor_set(x_72, 0, x_69); -lean_ctor_set(x_72, 1, x_55); -lean_ctor_set_uint8(x_72, sizeof(void*)*2, x_70); -x_73 = lean_unsigned_to_nat(0u); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_72); -return x_74; +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_66); +lean_ctor_set_uint8(x_83, sizeof(void*)*2, x_81); +x_84 = lean_unsigned_to_nat(0u); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_83); +return x_85; } } } diff --git a/stage0/stdlib/Lake/Build/Module.c b/stage0/stdlib/Lake/Build/Module.c index 955494e28323..8c570743f4e8 100644 --- a/stage0/stdlib/Lake/Build/Module.c +++ b/stage0/stdlib/Lake/Build/Module.c @@ -24560,245 +24560,303 @@ if (x_39 == 0) { lean_object* x_40; lean_object* x_41; lean_object* x_42; x_40 = lean_ctor_get(x_12, 0); -x_41 = l_Lake_compileSharedLib(x_9, x_37, x_38, x_40, x_13); +x_41 = lean_ctor_get(x_12, 1); +x_42 = l_Lake_compileSharedLib(x_9, x_37, x_38, x_40, x_13); lean_dec(x_37); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); if (lean_obj_tag(x_42) == 0) { -uint8_t x_43; -x_43 = !lean_is_exclusive(x_41); -if (x_43 == 0) +lean_object* x_43; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_44; uint8_t x_45; -x_44 = lean_ctor_get(x_41, 0); -lean_dec(x_44); -x_45 = !lean_is_exclusive(x_42); -if (x_45 == 0) +uint8_t x_44; +x_44 = !lean_is_exclusive(x_42); +if (x_44 == 0) { -lean_object* x_46; -x_46 = lean_ctor_get(x_42, 1); -lean_ctor_set(x_12, 0, x_46); -lean_ctor_set(x_42, 1, x_12); -return x_41; +lean_object* x_45; uint8_t x_46; +x_45 = lean_ctor_get(x_42, 0); +lean_dec(x_45); +x_46 = !lean_is_exclusive(x_43); +if (x_46 == 0) +{ +lean_object* x_47; +x_47 = lean_ctor_get(x_43, 1); +lean_ctor_set(x_12, 0, x_47); +lean_ctor_set(x_43, 1, x_12); +return x_42; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_42, 0); -x_48 = lean_ctor_get(x_42, 1); +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_43, 0); +x_49 = lean_ctor_get(x_43, 1); +lean_inc(x_49); lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_42); -lean_ctor_set(x_12, 0, x_48); -x_49 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_12); -lean_ctor_set(x_41, 0, x_49); -return x_41; +lean_dec(x_43); +lean_ctor_set(x_12, 0, x_49); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_12); +lean_ctor_set(x_42, 0, x_50); +return x_42; } } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_50 = lean_ctor_get(x_41, 1); -lean_inc(x_50); -lean_dec(x_41); -x_51 = lean_ctor_get(x_42, 0); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_51 = lean_ctor_get(x_42, 1); lean_inc(x_51); -x_52 = lean_ctor_get(x_42, 1); +lean_dec(x_42); +x_52 = lean_ctor_get(x_43, 0); lean_inc(x_52); -if (lean_is_exclusive(x_42)) { - lean_ctor_release(x_42, 0); - lean_ctor_release(x_42, 1); - x_53 = x_42; +x_53 = lean_ctor_get(x_43, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_54 = x_43; } else { - lean_dec_ref(x_42); - x_53 = lean_box(0); + lean_dec_ref(x_43); + x_54 = lean_box(0); } -lean_ctor_set(x_12, 0, x_52); -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_53); +if (lean_is_scalar(x_54)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_54 = x_53; + x_55 = x_54; } -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_12); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_50); -return x_55; +lean_ctor_set(x_55, 0, x_52); +lean_ctor_set(x_55, 1, x_12); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_51); +return x_56; } } else { -uint8_t x_56; -x_56 = !lean_is_exclusive(x_41); -if (x_56 == 0) +uint8_t x_57; +x_57 = !lean_is_exclusive(x_42); +if (x_57 == 0) { -lean_object* x_57; uint8_t x_58; -x_57 = lean_ctor_get(x_41, 0); -lean_dec(x_57); -x_58 = !lean_is_exclusive(x_42); -if (x_58 == 0) +lean_object* x_58; uint8_t x_59; +x_58 = lean_ctor_get(x_42, 0); +lean_dec(x_58); +x_59 = !lean_is_exclusive(x_43); +if (x_59 == 0) { -lean_object* x_59; -x_59 = lean_ctor_get(x_42, 1); -lean_ctor_set(x_12, 0, x_59); -lean_ctor_set(x_42, 1, x_12); -return x_41; +lean_object* x_60; +x_60 = lean_ctor_get(x_43, 1); +lean_ctor_set(x_12, 0, x_60); +lean_ctor_set(x_43, 1, x_12); +return x_42; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_42, 0); -x_61 = lean_ctor_get(x_42, 1); +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_43, 0); +x_62 = lean_ctor_get(x_43, 1); +lean_inc(x_62); lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_42); -lean_ctor_set(x_12, 0, x_61); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_12); -lean_ctor_set(x_41, 0, x_62); -return x_41; +lean_dec(x_43); +lean_ctor_set(x_12, 0, x_62); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_12); +lean_ctor_set(x_42, 0, x_63); +return x_42; } } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_63 = lean_ctor_get(x_41, 1); -lean_inc(x_63); -lean_dec(x_41); -x_64 = lean_ctor_get(x_42, 0); +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_64 = lean_ctor_get(x_42, 1); lean_inc(x_64); -x_65 = lean_ctor_get(x_42, 1); +lean_dec(x_42); +x_65 = lean_ctor_get(x_43, 0); lean_inc(x_65); -if (lean_is_exclusive(x_42)) { - lean_ctor_release(x_42, 0); - lean_ctor_release(x_42, 1); - x_66 = x_42; +x_66 = lean_ctor_get(x_43, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_67 = x_43; } else { - lean_dec_ref(x_42); - x_66 = lean_box(0); + lean_dec_ref(x_43); + x_67 = lean_box(0); } -lean_ctor_set(x_12, 0, x_65); -if (lean_is_scalar(x_66)) { - x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_66); +if (lean_is_scalar(x_67)) { + x_68 = lean_alloc_ctor(1, 2, 0); } else { - x_67 = x_66; + x_68 = x_67; } -lean_ctor_set(x_67, 0, x_64); -lean_ctor_set(x_67, 1, x_12); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_63); -return x_68; +lean_ctor_set(x_68, 0, x_65); +lean_ctor_set(x_68, 1, x_12); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_64); +return x_69; } } } else { -lean_object* x_69; uint8_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_69 = lean_ctor_get(x_12, 0); -x_70 = lean_ctor_get_uint8(x_12, sizeof(void*)*2); -x_71 = lean_ctor_get(x_12, 1); +uint8_t x_70; +lean_free_object(x_12); +lean_dec(x_41); +x_70 = !lean_is_exclusive(x_42); +if (x_70 == 0) +{ +return x_42; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_42, 0); +x_72 = lean_ctor_get(x_42, 1); +lean_inc(x_72); lean_inc(x_71); -lean_inc(x_69); +lean_dec(x_42); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} +} +else +{ +lean_object* x_74; uint8_t x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_12, 0); +x_75 = lean_ctor_get_uint8(x_12, sizeof(void*)*2); +x_76 = lean_ctor_get(x_12, 1); +lean_inc(x_76); +lean_inc(x_74); lean_dec(x_12); -x_72 = l_Lake_compileSharedLib(x_9, x_37, x_38, x_69, x_13); +x_77 = l_Lake_compileSharedLib(x_9, x_37, x_38, x_74, x_13); lean_dec(x_37); -x_73 = lean_ctor_get(x_72, 0); -lean_inc(x_73); -if (lean_obj_tag(x_73) == 0) +if (lean_obj_tag(x_77) == 0) { -lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_74 = lean_ctor_get(x_72, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_75 = x_72; +lean_object* x_78; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +if (lean_obj_tag(x_78) == 0) +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_80 = x_77; } else { - lean_dec_ref(x_72); - x_75 = lean_box(0); + lean_dec_ref(x_77); + x_80 = lean_box(0); } -x_76 = lean_ctor_get(x_73, 0); -lean_inc(x_76); -x_77 = lean_ctor_get(x_73, 1); -lean_inc(x_77); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_78 = x_73; +x_81 = lean_ctor_get(x_78, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_78, 1); +lean_inc(x_82); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_83 = x_78; } else { - lean_dec_ref(x_73); - x_78 = lean_box(0); + lean_dec_ref(x_78); + x_83 = lean_box(0); } -x_79 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_71); -lean_ctor_set_uint8(x_79, sizeof(void*)*2, x_70); -if (lean_is_scalar(x_78)) { - x_80 = lean_alloc_ctor(0, 2, 0); +x_84 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_76); +lean_ctor_set_uint8(x_84, sizeof(void*)*2, x_75); +if (lean_is_scalar(x_83)) { + x_85 = lean_alloc_ctor(0, 2, 0); } else { - x_80 = x_78; + x_85 = x_83; } -lean_ctor_set(x_80, 0, x_76); -lean_ctor_set(x_80, 1, x_79); -if (lean_is_scalar(x_75)) { - x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_81); +lean_ctor_set(x_85, 1, x_84); +if (lean_is_scalar(x_80)) { + x_86 = lean_alloc_ctor(0, 2, 0); } else { - x_81 = x_75; + x_86 = x_80; } -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_74); -return x_81; +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_79); +return x_86; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_82 = lean_ctor_get(x_72, 1); -lean_inc(x_82); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_83 = x_72; +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_87 = lean_ctor_get(x_77, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_88 = x_77; } else { - lean_dec_ref(x_72); - x_83 = lean_box(0); + lean_dec_ref(x_77); + x_88 = lean_box(0); } -x_84 = lean_ctor_get(x_73, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_73, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_86 = x_73; +x_89 = lean_ctor_get(x_78, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_78, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_91 = x_78; +} else { + lean_dec_ref(x_78); + x_91 = lean_box(0); +} +x_92 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_76); +lean_ctor_set_uint8(x_92, sizeof(void*)*2, x_75); +if (lean_is_scalar(x_91)) { + x_93 = lean_alloc_ctor(1, 2, 0); } else { - lean_dec_ref(x_73); - x_86 = lean_box(0); + x_93 = x_91; } -x_87 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_71); -lean_ctor_set_uint8(x_87, sizeof(void*)*2, x_70); -if (lean_is_scalar(x_86)) { - x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_89); +lean_ctor_set(x_93, 1, x_92); +if (lean_is_scalar(x_88)) { + x_94 = lean_alloc_ctor(0, 2, 0); } else { - x_88 = x_86; + x_94 = x_88; } -lean_ctor_set(x_88, 0, x_84); -lean_ctor_set(x_88, 1, x_87); -if (lean_is_scalar(x_83)) { - x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_93); +lean_ctor_set(x_94, 1, x_87); +return x_94; +} +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_76); +x_95 = lean_ctor_get(x_77, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_77, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_97 = x_77; +} else { + lean_dec_ref(x_77); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); } else { - x_89 = x_83; + x_98 = x_97; } -lean_ctor_set(x_89, 0, x_88); -lean_ctor_set(x_89, 1, x_82); -return x_89; +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; } } } diff --git a/stage0/stdlib/Lake/CLI/Build.c b/stage0/stdlib/Lake/CLI/Build.c index b75e35aeb4a8..c24aa954a11a 100644 --- a/stage0/stdlib/Lake/CLI/Build.c +++ b/stage0/stdlib/Lake/CLI/Build.c @@ -28,7 +28,6 @@ lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); lean_object* l_Lake_BuildInfo_key(lean_object*); static lean_object* l_Lake_resolveExternLibTarget___closed__3; LEAN_EXPORT lean_object* l_Lake_parseTargetSpecs(lean_object*, lean_object*); -lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); uint8_t l_Lean_Name_isAnonymous(lean_object*); static lean_object* l_Lake_resolveExeTarget___closed__2; @@ -2024,40 +2023,46 @@ uint8_t x_9; x_9 = !lean_is_exclusive(x_5); if (x_9 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_10 = lean_ctor_get(x_5, 0); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -lean_ctor_set(x_5, 0, x_12); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_11); +x_13 = lean_array_mk(x_12); +lean_ctor_set(x_5, 0, x_13); return x_5; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_5, 0); -lean_inc(x_13); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_14 = lean_ctor_get(x_5, 0); +lean_inc(x_14); lean_dec(x_5); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_13); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_15); -return x_16; +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = lean_array_mk(x_16); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; } } } else { -lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_dec(x_3); -x_17 = lean_ctor_get(x_2, 1); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 7); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_array_size(x_18); -x_20 = 0; -x_21 = l_Array_mapMUnsafe_map___at_Lake_resolveLibTarget___spec__1(x_1, x_2, x_19, x_20, x_18); -return x_21; +x_19 = lean_ctor_get(x_2, 1); +lean_inc(x_19); +x_20 = lean_ctor_get(x_19, 7); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_array_size(x_20); +x_22 = 0; +x_23 = l_Array_mapMUnsafe_map___at_Lake_resolveLibTarget___spec__1(x_1, x_2, x_21, x_22, x_20); +return x_23; } } } @@ -2478,208 +2483,232 @@ uint8_t x_27; x_27 = !lean_is_exclusive(x_23); if (x_27 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; x_28 = lean_ctor_get(x_23, 0); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_mk_array(x_29, x_28); -lean_ctor_set(x_23, 0, x_30); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_array_mk(x_30); +lean_ctor_set(x_23, 0, x_31); return x_23; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_31 = lean_ctor_get(x_23, 0); -lean_inc(x_31); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_32 = lean_ctor_get(x_23, 0); +lean_inc(x_32); lean_dec(x_23); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_31); -x_34 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_array_mk(x_34); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_35); +return x_36; } } } } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_dec(x_3); -x_35 = lean_ctor_get(x_13, 0); -lean_inc(x_35); +x_37 = lean_ctor_get(x_13, 0); +lean_inc(x_37); lean_dec(x_13); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_2); -lean_ctor_set(x_36, 1, x_35); -x_37 = l_Lake_resolveLibTarget(x_1, x_36, x_4); -return x_37; +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_2); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lake_resolveLibTarget(x_1, x_38, x_4); +return x_39; } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_10, 0); -lean_inc(x_38); +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_10, 0); +lean_inc(x_40); lean_dec(x_10); -x_39 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_39, 0, x_2); -lean_ctor_set(x_39, 1, x_3); -lean_ctor_set(x_39, 2, x_38); -x_40 = l_Lake_resolveExternLibTarget(x_39, x_4); -if (lean_obj_tag(x_40) == 0) -{ -uint8_t x_41; -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +x_41 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_41, 0, x_2); +lean_ctor_set(x_41, 1, x_3); +lean_ctor_set(x_41, 2, x_40); +x_42 = l_Lake_resolveExternLibTarget(x_41, x_4); +if (lean_obj_tag(x_42) == 0) +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) { -return x_40; +return x_42; } else { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_40, 0); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_43, 0, x_42); -return x_43; +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_42, 0); +lean_inc(x_44); +lean_dec(x_42); +x_45 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_45, 0, x_44); +return x_45; } } else { -uint8_t x_44; -x_44 = !lean_is_exclusive(x_40); -if (x_44 == 0) +uint8_t x_46; +x_46 = !lean_is_exclusive(x_42); +if (x_46 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_40, 0); -x_46 = lean_unsigned_to_nat(1u); -x_47 = lean_mk_array(x_46, x_45); -lean_ctor_set(x_40, 0, x_47); -return x_40; +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_42, 0); +x_48 = lean_box(0); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_array_mk(x_49); +lean_ctor_set(x_42, 0, x_50); +return x_42; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_40, 0); -lean_inc(x_48); -lean_dec(x_40); -x_49 = lean_unsigned_to_nat(1u); -x_50 = lean_mk_array(x_49, x_48); -x_51 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_51, 0, x_50); -return x_51; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_51 = lean_ctor_get(x_42, 0); +lean_inc(x_51); +lean_dec(x_42); +x_52 = lean_box(0); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_54 = lean_array_mk(x_53); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_54); +return x_55; } } } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_dec(x_3); -x_52 = lean_ctor_get(x_8, 0); -lean_inc(x_52); +x_56 = lean_ctor_get(x_8, 0); +lean_inc(x_56); lean_dec(x_8); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_2); -lean_ctor_set(x_53, 1, x_52); -x_54 = l_Lake_resolveExeTarget(x_53, x_4); -if (lean_obj_tag(x_54) == 0) +x_57 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_2); +lean_ctor_set(x_57, 1, x_56); +x_58 = l_Lake_resolveExeTarget(x_57, x_4); +if (lean_obj_tag(x_58) == 0) { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +uint8_t x_59; +x_59 = !lean_is_exclusive(x_58); +if (x_59 == 0) { -return x_54; +return x_58; } else { -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_54, 0); -lean_inc(x_56); -lean_dec(x_54); -x_57 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_57, 0, x_56); -return x_57; +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_58, 0); +lean_inc(x_60); +lean_dec(x_58); +x_61 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_61, 0, x_60); +return x_61; } } else { -uint8_t x_58; -x_58 = !lean_is_exclusive(x_54); -if (x_58 == 0) +uint8_t x_62; +x_62 = !lean_is_exclusive(x_58); +if (x_62 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_54, 0); -x_60 = lean_unsigned_to_nat(1u); -x_61 = lean_mk_array(x_60, x_59); -lean_ctor_set(x_54, 0, x_61); -return x_54; +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_63 = lean_ctor_get(x_58, 0); +x_64 = lean_box(0); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +x_66 = lean_array_mk(x_65); +lean_ctor_set(x_58, 0, x_66); +return x_58; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_54, 0); -lean_inc(x_62); -lean_dec(x_54); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_mk_array(x_63, x_62); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_64); -return x_65; +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_67 = lean_ctor_get(x_58, 0); +lean_inc(x_67); +lean_dec(x_58); +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +x_70 = lean_array_mk(x_69); +x_71 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_71, 0, x_70); +return x_71; } } } } else { -lean_object* x_66; lean_object* x_67; -x_66 = lean_ctor_get(x_5, 0); -lean_inc(x_66); +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_5, 0); +lean_inc(x_72); lean_dec(x_5); -x_67 = l_Lake_resolveCustomTarget(x_2, x_3, x_4, x_66); -if (lean_obj_tag(x_67) == 0) +x_73 = l_Lake_resolveCustomTarget(x_2, x_3, x_4, x_72); +if (lean_obj_tag(x_73) == 0) { -uint8_t x_68; -x_68 = !lean_is_exclusive(x_67); -if (x_68 == 0) +uint8_t x_74; +x_74 = !lean_is_exclusive(x_73); +if (x_74 == 0) { -return x_67; +return x_73; } else { -lean_object* x_69; lean_object* x_70; -x_69 = lean_ctor_get(x_67, 0); -lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_70, 0, x_69); -return x_70; +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_73, 0); +lean_inc(x_75); +lean_dec(x_73); +x_76 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_76, 0, x_75); +return x_76; } } else { -uint8_t x_71; -x_71 = !lean_is_exclusive(x_67); -if (x_71 == 0) +uint8_t x_77; +x_77 = !lean_is_exclusive(x_73); +if (x_77 == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_67, 0); -x_73 = lean_unsigned_to_nat(1u); -x_74 = lean_mk_array(x_73, x_72); -lean_ctor_set(x_67, 0, x_74); -return x_67; +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_73, 0); +x_79 = lean_box(0); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_array_mk(x_80); +lean_ctor_set(x_73, 0, x_81); +return x_73; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_75 = lean_ctor_get(x_67, 0); -lean_inc(x_75); -lean_dec(x_67); -x_76 = lean_unsigned_to_nat(1u); -x_77 = lean_mk_array(x_76, x_75); -x_78 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_78, 0, x_77); -return x_78; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_82 = lean_ctor_get(x_73, 0); +lean_inc(x_82); +lean_dec(x_73); +x_83 = lean_box(0); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = lean_array_mk(x_84); +x_86 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_86, 0, x_85); +return x_86; } } } @@ -2919,7 +2948,7 @@ lean_free_object(x_5); x_14 = !lean_is_exclusive(x_11); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_15 = lean_ctor_get(x_11, 0); x_16 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_16, 0, x_2); @@ -2927,89 +2956,98 @@ lean_ctor_set(x_16, 1, x_3); x_17 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_17, 0, x_16); lean_ctor_set(x_17, 1, x_15); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_mk_array(x_18, x_17); -lean_ctor_set(x_11, 0, x_19); +x_18 = lean_box(0); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_array_mk(x_19); +lean_ctor_set(x_11, 0, x_20); return x_11; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_11, 0); -lean_inc(x_20); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_21 = lean_ctor_get(x_11, 0); +lean_inc(x_21); lean_dec(x_11); -x_21 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_21, 0, x_2); -lean_ctor_set(x_21, 1, x_3); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_2); +lean_ctor_set(x_22, 1, x_3); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = lean_array_mk(x_25); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_26); +return x_27; } } } else { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_5, 0); -lean_inc(x_26); +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_5, 0); +lean_inc(x_28); lean_dec(x_5); -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -if (lean_obj_tag(x_27) == 0) +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_dec(x_2); -x_28 = l_Lake_resolvePackageTarget___closed__1; -x_29 = lean_alloc_ctor(17, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_3); -x_30 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_30, 0, x_29); -return x_30; +x_30 = l_Lake_resolvePackageTarget___closed__1; +x_31 = lean_alloc_ctor(17, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_3); +x_32 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_32, 0, x_31); +return x_32; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_31 = lean_ctor_get(x_27, 0); -lean_inc(x_31); -if (lean_is_exclusive(x_27)) { - lean_ctor_release(x_27, 0); - x_32 = x_27; +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_33 = lean_ctor_get(x_29, 0); +lean_inc(x_33); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + x_34 = x_29; } else { - lean_dec_ref(x_27); - x_32 = lean_box(0); + lean_dec_ref(x_29); + x_34 = lean_box(0); } -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_2); -lean_ctor_set(x_33, 1, x_3); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_31); -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_mk_array(x_35, x_34); -if (lean_is_scalar(x_32)) { - x_37 = lean_alloc_ctor(1, 1, 0); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_2); +lean_ctor_set(x_35, 1, x_3); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_33); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_array_mk(x_38); +if (lean_is_scalar(x_34)) { + x_40 = lean_alloc_ctor(1, 1, 0); } else { - x_37 = x_32; + x_40 = x_34; } -lean_ctor_set(x_37, 0, x_36); -return x_37; +lean_ctor_set(x_40, 0, x_39); +return x_40; } } } } else { -lean_object* x_38; +lean_object* x_41; lean_dec(x_3); -x_38 = l_Lake_resolveDefaultPackageTarget(x_1, x_2); -return x_38; +x_41 = l_Lake_resolveDefaultPackageTarget(x_1, x_2); +return x_41; } } } @@ -3093,215 +3131,297 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_14); if (x_18 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_19 = lean_ctor_get(x_14, 0); -x_20 = lean_unsigned_to_nat(1u); -x_21 = lean_mk_array(x_20, x_19); -lean_ctor_set(x_14, 0, x_21); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = lean_array_mk(x_21); +lean_ctor_set(x_14, 0, x_22); return x_14; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_14, 0); -lean_inc(x_22); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_14, 0); +lean_inc(x_23); lean_dec(x_14); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_26 = lean_array_mk(x_25); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_26); +return x_27; } } } } else { -lean_object* x_26; lean_object* x_27; +lean_object* x_28; lean_object* x_29; lean_dec(x_2); -x_26 = lean_ctor_get(x_9, 0); -lean_inc(x_26); +x_28 = lean_ctor_get(x_9, 0); +lean_inc(x_28); lean_dec(x_9); -x_27 = l_Lake_resolvePackageTarget(x_1, x_26, x_3); -return x_27; +x_29 = l_Lake_resolvePackageTarget(x_1, x_28, x_3); +return x_29; } } else { -lean_object* x_28; lean_object* x_29; +lean_object* x_30; lean_object* x_31; lean_dec(x_2); -x_28 = lean_ctor_get(x_7, 0); -lean_inc(x_28); +x_30 = lean_ctor_get(x_7, 0); +lean_inc(x_30); lean_dec(x_7); -x_29 = l_Lake_resolveLibTarget(x_1, x_28, x_3); -return x_29; +x_31 = l_Lake_resolveLibTarget(x_1, x_30, x_3); +return x_31; } } else { -lean_object* x_30; lean_object* x_31; +lean_object* x_32; lean_object* x_33; lean_dec(x_2); -x_30 = lean_ctor_get(x_6, 0); -lean_inc(x_30); +x_32 = lean_ctor_get(x_6, 0); +lean_inc(x_32); lean_dec(x_6); -x_31 = l_Lake_resolveExternLibTarget(x_30, x_3); -if (lean_obj_tag(x_31) == 0) +x_33 = l_Lake_resolveExternLibTarget(x_32, x_3); +if (lean_obj_tag(x_33) == 0) { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) { -return x_31; +return x_33; } else { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_31, 0); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_36, 0, x_35); +return x_36; } } else { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_31); -if (x_35 == 0) +uint8_t x_37; +x_37 = !lean_is_exclusive(x_33); +if (x_37 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_31, 0); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -lean_ctor_set(x_31, 0, x_38); -return x_31; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_33, 0); +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_array_mk(x_40); +lean_ctor_set(x_33, 0, x_41); +return x_33; } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_31, 0); -lean_inc(x_39); -lean_dec(x_31); -x_40 = lean_unsigned_to_nat(1u); -x_41 = lean_mk_array(x_40, x_39); -x_42 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_42, 0, x_41); -return x_42; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_ctor_get(x_33, 0); +lean_inc(x_42); +lean_dec(x_33); +x_43 = lean_box(0); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_array_mk(x_44); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +return x_46; } } } } else { -lean_object* x_43; lean_object* x_44; +lean_object* x_47; lean_object* x_48; lean_dec(x_2); -x_43 = lean_ctor_get(x_5, 0); -lean_inc(x_43); +x_47 = lean_ctor_get(x_5, 0); +lean_inc(x_47); lean_dec(x_5); -x_44 = l_Lake_resolveExeTarget(x_43, x_3); -if (lean_obj_tag(x_44) == 0) +x_48 = l_Lake_resolveExeTarget(x_47, x_3); +if (lean_obj_tag(x_48) == 0) { -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) +uint8_t x_49; +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) { -return x_44; +return x_48; } else { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_44, 0); -lean_inc(x_46); -lean_dec(x_44); -x_47 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_47, 0, x_46); -return x_47; +lean_object* x_50; lean_object* x_51; +x_50 = lean_ctor_get(x_48, 0); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_51, 0, x_50); +return x_51; } } else { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_44); -if (x_48 == 0) +uint8_t x_52; +x_52 = !lean_is_exclusive(x_48); +if (x_52 == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_44, 0); -x_50 = lean_unsigned_to_nat(1u); -x_51 = lean_mk_array(x_50, x_49); -lean_ctor_set(x_44, 0, x_51); -return x_44; +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_48, 0); +x_54 = lean_box(0); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +x_56 = lean_array_mk(x_55); +lean_ctor_set(x_48, 0, x_56); +return x_48; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_44, 0); -lean_inc(x_52); -lean_dec(x_44); -x_53 = lean_unsigned_to_nat(1u); -x_54 = lean_mk_array(x_53, x_52); -x_55 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_55, 0, x_54); -return x_55; +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_57 = lean_ctor_get(x_48, 0); +lean_inc(x_57); +lean_dec(x_48); +x_58 = lean_box(0); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +x_60 = lean_array_mk(x_59); +x_61 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_61, 0, x_60); +return x_61; } } } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_56 = lean_ctor_get(x_4, 0); -lean_inc(x_56); +lean_object* x_62; uint8_t x_63; +x_62 = lean_ctor_get(x_4, 0); +lean_inc(x_62); lean_dec(x_4); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = l_Lake_resolveCustomTarget(x_57, x_2, x_3, x_58); -if (lean_obj_tag(x_59) == 0) +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_62, 0); +x_65 = lean_ctor_get(x_62, 1); +x_66 = l_Lake_resolveCustomTarget(x_64, x_2, x_3, x_65); +if (lean_obj_tag(x_66) == 0) { -uint8_t x_60; -x_60 = !lean_is_exclusive(x_59); -if (x_60 == 0) +uint8_t x_67; +lean_free_object(x_62); +x_67 = !lean_is_exclusive(x_66); +if (x_67 == 0) { -return x_59; +return x_66; } else { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_59, 0); -lean_inc(x_61); -lean_dec(x_59); -x_62 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_62, 0, x_61); -return x_62; +lean_object* x_68; lean_object* x_69; +x_68 = lean_ctor_get(x_66, 0); +lean_inc(x_68); +lean_dec(x_66); +x_69 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_69, 0, x_68); +return x_69; } } else { -uint8_t x_63; -x_63 = !lean_is_exclusive(x_59); -if (x_63 == 0) +uint8_t x_70; +x_70 = !lean_is_exclusive(x_66); +if (x_70 == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_59, 0); -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_mk_array(x_65, x_64); -lean_ctor_set(x_59, 0, x_66); -return x_59; +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_66, 0); +x_72 = lean_box(0); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_72); +lean_ctor_set(x_62, 0, x_71); +x_73 = lean_array_mk(x_62); +lean_ctor_set(x_66, 0, x_73); +return x_66; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_67 = lean_ctor_get(x_59, 0); -lean_inc(x_67); -lean_dec(x_59); -x_68 = lean_unsigned_to_nat(1u); -x_69 = lean_mk_array(x_68, x_67); -x_70 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_70, 0, x_69); -return x_70; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_66, 0); +lean_inc(x_74); +lean_dec(x_66); +x_75 = lean_box(0); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_75); +lean_ctor_set(x_62, 0, x_74); +x_76 = lean_array_mk(x_62); +x_77 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_77, 0, x_76); +return x_77; +} +} +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_62, 0); +x_79 = lean_ctor_get(x_62, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_62); +x_80 = l_Lake_resolveCustomTarget(x_78, x_2, x_3, x_79); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_82 = x_80; +} else { + lean_dec_ref(x_80); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(0, 1, 0); +} else { + x_83 = x_82; +} +lean_ctor_set(x_83, 0, x_81); +return x_83; +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_84 = lean_ctor_get(x_80, 0); +lean_inc(x_84); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_85 = x_80; +} else { + lean_dec_ref(x_80); + x_85 = lean_box(0); +} +x_86 = lean_box(0); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_86); +x_88 = lean_array_mk(x_87); +if (lean_is_scalar(x_85)) { + x_89 = lean_alloc_ctor(1, 1, 0); +} else { + x_89 = x_85; +} +lean_ctor_set(x_89, 0, x_88); +return x_89; } } } @@ -3434,51 +3554,51 @@ return x_2; LEAN_EXPORT lean_object* l_Lake_resolveTargetBaseSpec(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; uint8_t x_149; -x_149 = l_Lake_resolveTargetBaseSpec___closed__11; -if (x_149 == 0) +lean_object* x_4; lean_object* x_5; uint8_t x_160; +x_160 = l_Lake_resolveTargetBaseSpec___closed__11; +if (x_160 == 0) { -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; -x_150 = lean_box(0); -x_151 = l_Lake_resolveTargetBaseSpec___closed__9; -x_152 = lean_unsigned_to_nat(0u); -x_153 = l_String_splitOnAux(x_2, x_151, x_152, x_152, x_152, x_150); -if (lean_obj_tag(x_153) == 0) +lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_161 = lean_box(0); +x_162 = l_Lake_resolveTargetBaseSpec___closed__9; +x_163 = lean_unsigned_to_nat(0u); +x_164 = l_String_splitOnAux(x_2, x_162, x_163, x_163, x_163, x_161); +if (lean_obj_tag(x_164) == 0) { -lean_object* x_154; lean_object* x_155; lean_object* x_156; +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_3); lean_dec(x_1); -x_154 = l_Lake_resolveTargetBaseSpec___boxed__const__1; -x_155 = lean_alloc_ctor(18, 2, 0); -lean_ctor_set(x_155, 0, x_2); -lean_ctor_set(x_155, 1, x_154); -x_156 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_156, 0, x_155); -return x_156; +x_165 = l_Lake_resolveTargetBaseSpec___boxed__const__1; +x_166 = lean_alloc_ctor(18, 2, 0); +lean_ctor_set(x_166, 0, x_2); +lean_ctor_set(x_166, 1, x_165); +x_167 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_167, 0, x_166); +return x_167; } else { -lean_object* x_157; lean_object* x_158; -x_157 = lean_ctor_get(x_153, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_153, 1); -lean_inc(x_158); -lean_dec(x_153); -x_4 = x_157; -x_5 = x_158; -goto block_148; +lean_object* x_168; lean_object* x_169; +x_168 = lean_ctor_get(x_164, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_164, 1); +lean_inc(x_169); +lean_dec(x_164); +x_4 = x_168; +x_5 = x_169; +goto block_159; } } else { -lean_object* x_159; -x_159 = lean_box(0); +lean_object* x_170; +x_170 = lean_box(0); lean_inc(x_2); x_4 = x_2; -x_5 = x_159; -goto block_148; +x_5 = x_170; +goto block_159; } -block_148: +block_159: { if (lean_obj_tag(x_5) == 0) { @@ -3591,22 +3711,30 @@ uint8_t x_37; x_37 = !lean_is_exclusive(x_33); if (x_37 == 0) { -lean_object* x_38; lean_object* x_39; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; x_38 = lean_ctor_get(x_33, 0); -x_39 = lean_mk_array(x_24, x_38); -lean_ctor_set(x_33, 0, x_39); +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_array_mk(x_40); +lean_ctor_set(x_33, 0, x_41); return x_33; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_33, 0); -lean_inc(x_40); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_42 = lean_ctor_get(x_33, 0); +lean_inc(x_42); lean_dec(x_33); -x_41 = lean_mk_array(x_24, x_40); -x_42 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_42, 0, x_41); -return x_42; +x_43 = lean_box(0); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_array_mk(x_44); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +return x_46; } } } @@ -3614,297 +3742,325 @@ return x_42; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_43 = lean_unsigned_to_nat(1u); -x_44 = l_Substring_nextn(x_9, x_43, x_7); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_unsigned_to_nat(1u); +x_48 = l_Substring_nextn(x_9, x_47, x_7); lean_dec(x_9); -x_45 = lean_nat_add(x_7, x_44); -lean_dec(x_44); -x_46 = lean_string_utf8_extract(x_4, x_45, x_6); +x_49 = lean_nat_add(x_7, x_48); +lean_dec(x_48); +x_50 = lean_string_utf8_extract(x_4, x_49, x_6); lean_dec(x_6); -lean_dec(x_45); +lean_dec(x_49); lean_dec(x_4); -x_47 = l_Lake_parsePackageSpec(x_1, x_46); -if (lean_obj_tag(x_47) == 0) +x_51 = l_Lake_parsePackageSpec(x_1, x_50); +if (lean_obj_tag(x_51) == 0) { -uint8_t x_48; +uint8_t x_52; lean_dec(x_3); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) +x_52 = !lean_is_exclusive(x_51); +if (x_52 == 0) { -return x_47; +return x_51; } else { -lean_object* x_49; lean_object* x_50; -x_49 = lean_ctor_get(x_47, 0); -lean_inc(x_49); -lean_dec(x_47); -x_50 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_50, 0, x_49); -return x_50; +lean_object* x_53; lean_object* x_54; +x_53 = lean_ctor_get(x_51, 0); +lean_inc(x_53); +lean_dec(x_51); +x_54 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_54, 0, x_53); +return x_54; } } else { -lean_object* x_51; lean_object* x_52; -x_51 = lean_ctor_get(x_47, 0); -lean_inc(x_51); -lean_dec(x_47); -x_52 = l_Lake_resolvePackageTarget(x_1, x_51, x_3); +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_51, 0); +lean_inc(x_55); +lean_dec(x_51); +x_56 = l_Lake_resolvePackageTarget(x_1, x_55, x_3); lean_dec(x_1); -return x_52; +return x_56; } } } else { -lean_object* x_53; lean_object* x_54; +lean_object* x_57; lean_object* x_58; lean_dec(x_6); lean_dec(x_4); -x_53 = lean_ctor_get(x_1, 0); -lean_inc(x_53); -x_54 = l_Lake_resolvePackageTarget(x_1, x_53, x_3); +x_57 = lean_ctor_get(x_1, 0); +lean_inc(x_57); +x_58 = l_Lake_resolvePackageTarget(x_1, x_57, x_3); lean_dec(x_1); -return x_54; +return x_58; } } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_5, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_5, 1); -lean_inc(x_56); -lean_dec(x_5); -if (lean_obj_tag(x_56) == 0) +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_5, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_5, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_5)) { + lean_ctor_release(x_5, 0); + lean_ctor_release(x_5, 1); + x_61 = x_5; +} else { + lean_dec_ref(x_5); + x_61 = lean_box(0); +} +if (lean_obj_tag(x_60) == 0) { -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; uint8_t x_146; lean_dec(x_2); -x_127 = lean_string_utf8_byte_size(x_4); -x_128 = lean_unsigned_to_nat(0u); -lean_inc(x_127); +x_138 = lean_string_utf8_byte_size(x_4); +x_139 = lean_unsigned_to_nat(0u); +lean_inc(x_138); lean_inc(x_4); -x_129 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_129, 0, x_4); -lean_ctor_set(x_129, 1, x_128); -lean_ctor_set(x_129, 2, x_127); -x_130 = l_Lake_resolveTargetBaseSpec___closed__2; -x_131 = l_Substring_nextn(x_129, x_130, x_128); -x_132 = lean_nat_add(x_128, x_131); -lean_dec(x_131); +x_140 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_140, 0, x_4); +lean_ctor_set(x_140, 1, x_139); +lean_ctor_set(x_140, 2, x_138); +x_141 = l_Lake_resolveTargetBaseSpec___closed__2; +x_142 = l_Substring_nextn(x_140, x_141, x_139); +x_143 = lean_nat_add(x_139, x_142); +lean_dec(x_142); lean_inc(x_4); -x_133 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_133, 0, x_4); -lean_ctor_set(x_133, 1, x_128); -lean_ctor_set(x_133, 2, x_132); -x_134 = l_Lake_resolveTargetBaseSpec___closed__4; -x_135 = l_Substring_beq(x_133, x_134); -if (x_135 == 0) -{ -lean_dec(x_129); -lean_dec(x_127); -x_57 = x_4; -goto block_126; -} -else -{ -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_136 = lean_unsigned_to_nat(1u); -x_137 = l_Substring_nextn(x_129, x_136, x_128); -lean_dec(x_129); -x_138 = lean_nat_add(x_128, x_137); -lean_dec(x_137); -x_139 = lean_string_utf8_extract(x_4, x_138, x_127); -lean_dec(x_127); +x_144 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_144, 0, x_4); +lean_ctor_set(x_144, 1, x_139); +lean_ctor_set(x_144, 2, x_143); +x_145 = l_Lake_resolveTargetBaseSpec___closed__4; +x_146 = l_Substring_beq(x_144, x_145); +if (x_146 == 0) +{ +lean_dec(x_140); lean_dec(x_138); +x_62 = x_4; +goto block_137; +} +else +{ +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_147 = lean_unsigned_to_nat(1u); +x_148 = l_Substring_nextn(x_140, x_147, x_139); +lean_dec(x_140); +x_149 = lean_nat_add(x_139, x_148); +lean_dec(x_148); +x_150 = lean_string_utf8_extract(x_4, x_149, x_138); +lean_dec(x_138); +lean_dec(x_149); lean_dec(x_4); -x_57 = x_139; -goto block_126; +x_62 = x_150; +goto block_137; } } else { -uint8_t x_140; -lean_dec(x_55); +uint8_t x_151; +lean_dec(x_61); +lean_dec(x_59); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_140 = !lean_is_exclusive(x_56); -if (x_140 == 0) +x_151 = !lean_is_exclusive(x_60); +if (x_151 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_141 = lean_ctor_get(x_56, 1); -lean_dec(x_141); -x_142 = lean_ctor_get(x_56, 0); -lean_dec(x_142); -x_143 = l_Lake_resolveTargetBaseSpec___boxed__const__1; -lean_ctor_set_tag(x_56, 18); -lean_ctor_set(x_56, 1, x_143); -lean_ctor_set(x_56, 0, x_2); -x_144 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_144, 0, x_56); -return x_144; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_152 = lean_ctor_get(x_60, 1); +lean_dec(x_152); +x_153 = lean_ctor_get(x_60, 0); +lean_dec(x_153); +x_154 = l_Lake_resolveTargetBaseSpec___boxed__const__1; +lean_ctor_set_tag(x_60, 18); +lean_ctor_set(x_60, 1, x_154); +lean_ctor_set(x_60, 0, x_2); +x_155 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_155, 0, x_60); +return x_155; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; -lean_dec(x_56); -x_145 = l_Lake_resolveTargetBaseSpec___boxed__const__1; -x_146 = lean_alloc_ctor(18, 2, 0); -lean_ctor_set(x_146, 0, x_2); -lean_ctor_set(x_146, 1, x_145); -x_147 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_147, 0, x_146); -return x_147; +lean_object* x_156; lean_object* x_157; lean_object* x_158; +lean_dec(x_60); +x_156 = l_Lake_resolveTargetBaseSpec___boxed__const__1; +x_157 = lean_alloc_ctor(18, 2, 0); +lean_ctor_set(x_157, 0, x_2); +lean_ctor_set(x_157, 1, x_156); +x_158 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_158, 0, x_157); +return x_158; } } -block_126: +block_137: { -lean_object* x_58; -x_58 = l_Lake_parsePackageSpec(x_1, x_57); -if (lean_obj_tag(x_58) == 0) +lean_object* x_63; +x_63 = l_Lake_parsePackageSpec(x_1, x_62); +if (lean_obj_tag(x_63) == 0) { -uint8_t x_59; -lean_dec(x_55); +uint8_t x_64; +lean_dec(x_61); +lean_dec(x_59); lean_dec(x_3); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_58); -if (x_59 == 0) +x_64 = !lean_is_exclusive(x_63); +if (x_64 == 0) { -return x_58; +return x_63; } else { -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_58, 0); -lean_inc(x_60); -lean_dec(x_58); -x_61 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_61, 0, x_60); -return x_61; +lean_object* x_65; lean_object* x_66; +x_65 = lean_ctor_get(x_63, 0); +lean_inc(x_65); +lean_dec(x_63); +x_66 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_66, 0, x_65); +return x_66; } } else { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_58); -if (x_62 == 0) +uint8_t x_67; +x_67 = !lean_is_exclusive(x_63); +if (x_67 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_63 = lean_ctor_get(x_58, 0); -x_64 = lean_string_utf8_byte_size(x_55); -x_65 = lean_unsigned_to_nat(0u); -x_66 = lean_nat_dec_eq(x_64, x_65); -if (x_66 == 0) +lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; +x_68 = lean_ctor_get(x_63, 0); +x_69 = lean_string_utf8_byte_size(x_59); +x_70 = lean_unsigned_to_nat(0u); +x_71 = lean_nat_dec_eq(x_69, x_70); +if (x_71 == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -lean_inc(x_64); -lean_inc(x_55); -x_67 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_67, 0, x_55); -lean_ctor_set(x_67, 1, x_65); -lean_ctor_set(x_67, 2, x_64); -x_68 = l_Lake_resolveTargetBaseSpec___closed__6; -x_69 = l_Substring_nextn(x_67, x_68, x_65); -x_70 = lean_nat_add(x_65, x_69); +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; +lean_inc(x_69); +lean_inc(x_59); +x_72 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_72, 0, x_59); +lean_ctor_set(x_72, 1, x_70); +lean_ctor_set(x_72, 2, x_69); +x_73 = l_Lake_resolveTargetBaseSpec___closed__6; +x_74 = l_Substring_nextn(x_72, x_73, x_70); +x_75 = lean_nat_add(x_70, x_74); +lean_dec(x_74); +lean_inc(x_59); +x_76 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_76, 0, x_59); +lean_ctor_set(x_76, 1, x_70); +lean_ctor_set(x_76, 2, x_75); +x_77 = l_Lake_resolveTargetBaseSpec___closed__8; +x_78 = l_Substring_beq(x_76, x_77); +if (x_78 == 0) +{ +lean_object* x_79; lean_object* x_80; +lean_dec(x_72); lean_dec(x_69); -lean_inc(x_55); -x_71 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_71, 0, x_55); -lean_ctor_set(x_71, 1, x_65); -lean_ctor_set(x_71, 2, x_70); -x_72 = l_Lake_resolveTargetBaseSpec___closed__8; -x_73 = l_Substring_beq(x_71, x_72); -if (x_73 == 0) -{ -lean_object* x_74; lean_object* x_75; -lean_dec(x_67); -lean_dec(x_64); -lean_free_object(x_58); -x_74 = l_Lake_stringToLegalOrSimpleName(x_55); -x_75 = l_Lake_resolveTargetInPackage(x_1, x_63, x_74, x_3); +lean_free_object(x_63); +lean_dec(x_61); +x_79 = l_Lake_stringToLegalOrSimpleName(x_59); +x_80 = l_Lake_resolveTargetInPackage(x_1, x_68, x_79, x_3); lean_dec(x_1); -return x_75; +return x_80; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_76 = lean_unsigned_to_nat(1u); -x_77 = l_Substring_nextn(x_67, x_76, x_65); -lean_dec(x_67); -x_78 = lean_nat_add(x_65, x_77); -lean_dec(x_77); -x_79 = lean_string_utf8_extract(x_55, x_78, x_64); -lean_dec(x_64); -lean_dec(x_78); -lean_dec(x_55); -x_80 = l_String_toName(x_79); -lean_inc(x_80); -x_81 = l_Lake_Package_findTargetModule_x3f(x_80, x_63); -if (lean_obj_tag(x_81) == 0) +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_81 = lean_unsigned_to_nat(1u); +x_82 = l_Substring_nextn(x_72, x_81, x_70); +lean_dec(x_72); +x_83 = lean_nat_add(x_70, x_82); +lean_dec(x_82); +x_84 = lean_string_utf8_extract(x_59, x_83, x_69); +lean_dec(x_69); +lean_dec(x_83); +lean_dec(x_59); +x_85 = l_String_toName(x_84); +lean_inc(x_85); +x_86 = l_Lake_Package_findTargetModule_x3f(x_85, x_68); +if (lean_obj_tag(x_86) == 0) { -lean_object* x_82; +lean_object* x_87; +lean_dec(x_61); lean_dec(x_3); lean_dec(x_1); -x_82 = lean_alloc_ctor(10, 1, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set_tag(x_58, 0); -lean_ctor_set(x_58, 0, x_82); -return x_58; +x_87 = lean_alloc_ctor(10, 1, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set_tag(x_63, 0); +lean_ctor_set(x_63, 0, x_87); +return x_63; } else { -lean_object* x_83; lean_object* x_84; -lean_dec(x_80); -lean_free_object(x_58); -x_83 = lean_ctor_get(x_81, 0); -lean_inc(x_83); -lean_dec(x_81); -x_84 = l_Lake_resolveModuleTarget(x_1, x_83, x_3); +lean_object* x_88; lean_object* x_89; +lean_dec(x_85); +lean_free_object(x_63); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +lean_dec(x_86); +x_89 = l_Lake_resolveModuleTarget(x_1, x_88, x_3); lean_dec(x_1); -if (lean_obj_tag(x_84) == 0) +if (lean_obj_tag(x_89) == 0) { -uint8_t x_85; -x_85 = !lean_is_exclusive(x_84); -if (x_85 == 0) +uint8_t x_90; +lean_dec(x_61); +x_90 = !lean_is_exclusive(x_89); +if (x_90 == 0) { -return x_84; +return x_89; } else { -lean_object* x_86; lean_object* x_87; -x_86 = lean_ctor_get(x_84, 0); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_87, 0, x_86); -return x_87; +lean_object* x_91; lean_object* x_92; +x_91 = lean_ctor_get(x_89, 0); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_92, 0, x_91); +return x_92; } } else { -uint8_t x_88; -x_88 = !lean_is_exclusive(x_84); -if (x_88 == 0) +uint8_t x_93; +x_93 = !lean_is_exclusive(x_89); +if (x_93 == 0) { -lean_object* x_89; lean_object* x_90; -x_89 = lean_ctor_get(x_84, 0); -x_90 = lean_mk_array(x_76, x_89); -lean_ctor_set(x_84, 0, x_90); -return x_84; +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_94 = lean_ctor_get(x_89, 0); +x_95 = lean_box(0); +if (lean_is_scalar(x_61)) { + x_96 = lean_alloc_ctor(1, 2, 0); +} else { + x_96 = x_61; +} +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_array_mk(x_96); +lean_ctor_set(x_89, 0, x_97); +return x_89; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_84, 0); -lean_inc(x_91); -lean_dec(x_84); -x_92 = lean_mk_array(x_76, x_91); -x_93 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_93, 0, x_92); -return x_93; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_98 = lean_ctor_get(x_89, 0); +lean_inc(x_98); +lean_dec(x_89); +x_99 = lean_box(0); +if (lean_is_scalar(x_61)) { + x_100 = lean_alloc_ctor(1, 2, 0); +} else { + x_100 = x_61; +} +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +x_101 = lean_array_mk(x_100); +x_102 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_102, 0, x_101); +return x_102; } } } @@ -3912,141 +4068,154 @@ return x_93; } else { -lean_object* x_94; -lean_dec(x_64); -lean_free_object(x_58); -lean_dec(x_55); -x_94 = l_Lake_resolvePackageTarget(x_1, x_63, x_3); +lean_object* x_103; +lean_dec(x_69); +lean_free_object(x_63); +lean_dec(x_61); +lean_dec(x_59); +x_103 = l_Lake_resolvePackageTarget(x_1, x_68, x_3); lean_dec(x_1); -return x_94; +return x_103; } } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; -x_95 = lean_ctor_get(x_58, 0); -lean_inc(x_95); -lean_dec(x_58); -x_96 = lean_string_utf8_byte_size(x_55); -x_97 = lean_unsigned_to_nat(0u); -x_98 = lean_nat_dec_eq(x_96, x_97); -if (x_98 == 0) +lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; +x_104 = lean_ctor_get(x_63, 0); +lean_inc(x_104); +lean_dec(x_63); +x_105 = lean_string_utf8_byte_size(x_59); +x_106 = lean_unsigned_to_nat(0u); +x_107 = lean_nat_dec_eq(x_105, x_106); +if (x_107 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; -lean_inc(x_96); -lean_inc(x_55); -x_99 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_99, 0, x_55); -lean_ctor_set(x_99, 1, x_97); -lean_ctor_set(x_99, 2, x_96); -x_100 = l_Lake_resolveTargetBaseSpec___closed__6; -x_101 = l_Substring_nextn(x_99, x_100, x_97); -x_102 = lean_nat_add(x_97, x_101); -lean_dec(x_101); -lean_inc(x_55); -x_103 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_103, 0, x_55); -lean_ctor_set(x_103, 1, x_97); -lean_ctor_set(x_103, 2, x_102); -x_104 = l_Lake_resolveTargetBaseSpec___closed__8; -x_105 = l_Substring_beq(x_103, x_104); -if (x_105 == 0) -{ -lean_object* x_106; lean_object* x_107; -lean_dec(x_99); -lean_dec(x_96); -x_106 = l_Lake_stringToLegalOrSimpleName(x_55); -x_107 = l_Lake_resolveTargetInPackage(x_1, x_95, x_106, x_3); +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; +lean_inc(x_105); +lean_inc(x_59); +x_108 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_108, 0, x_59); +lean_ctor_set(x_108, 1, x_106); +lean_ctor_set(x_108, 2, x_105); +x_109 = l_Lake_resolveTargetBaseSpec___closed__6; +x_110 = l_Substring_nextn(x_108, x_109, x_106); +x_111 = lean_nat_add(x_106, x_110); +lean_dec(x_110); +lean_inc(x_59); +x_112 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_112, 0, x_59); +lean_ctor_set(x_112, 1, x_106); +lean_ctor_set(x_112, 2, x_111); +x_113 = l_Lake_resolveTargetBaseSpec___closed__8; +x_114 = l_Substring_beq(x_112, x_113); +if (x_114 == 0) +{ +lean_object* x_115; lean_object* x_116; +lean_dec(x_108); +lean_dec(x_105); +lean_dec(x_61); +x_115 = l_Lake_stringToLegalOrSimpleName(x_59); +x_116 = l_Lake_resolveTargetInPackage(x_1, x_104, x_115, x_3); lean_dec(x_1); -return x_107; +return x_116; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_108 = lean_unsigned_to_nat(1u); -x_109 = l_Substring_nextn(x_99, x_108, x_97); -lean_dec(x_99); -x_110 = lean_nat_add(x_97, x_109); -lean_dec(x_109); -x_111 = lean_string_utf8_extract(x_55, x_110, x_96); -lean_dec(x_96); -lean_dec(x_110); -lean_dec(x_55); -x_112 = l_String_toName(x_111); -lean_inc(x_112); -x_113 = l_Lake_Package_findTargetModule_x3f(x_112, x_95); -if (lean_obj_tag(x_113) == 0) +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_117 = lean_unsigned_to_nat(1u); +x_118 = l_Substring_nextn(x_108, x_117, x_106); +lean_dec(x_108); +x_119 = lean_nat_add(x_106, x_118); +lean_dec(x_118); +x_120 = lean_string_utf8_extract(x_59, x_119, x_105); +lean_dec(x_105); +lean_dec(x_119); +lean_dec(x_59); +x_121 = l_String_toName(x_120); +lean_inc(x_121); +x_122 = l_Lake_Package_findTargetModule_x3f(x_121, x_104); +if (lean_obj_tag(x_122) == 0) { -lean_object* x_114; lean_object* x_115; +lean_object* x_123; lean_object* x_124; +lean_dec(x_61); lean_dec(x_3); lean_dec(x_1); -x_114 = lean_alloc_ctor(10, 1, 0); -lean_ctor_set(x_114, 0, x_112); -x_115 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_115, 0, x_114); -return x_115; +x_123 = lean_alloc_ctor(10, 1, 0); +lean_ctor_set(x_123, 0, x_121); +x_124 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_124, 0, x_123); +return x_124; } else { -lean_object* x_116; lean_object* x_117; -lean_dec(x_112); -x_116 = lean_ctor_get(x_113, 0); -lean_inc(x_116); -lean_dec(x_113); -x_117 = l_Lake_resolveModuleTarget(x_1, x_116, x_3); +lean_object* x_125; lean_object* x_126; +lean_dec(x_121); +x_125 = lean_ctor_get(x_122, 0); +lean_inc(x_125); +lean_dec(x_122); +x_126 = l_Lake_resolveModuleTarget(x_1, x_125, x_3); lean_dec(x_1); -if (lean_obj_tag(x_117) == 0) +if (lean_obj_tag(x_126) == 0) { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -if (lean_is_exclusive(x_117)) { - lean_ctor_release(x_117, 0); - x_119 = x_117; +lean_object* x_127; lean_object* x_128; lean_object* x_129; +lean_dec(x_61); +x_127 = lean_ctor_get(x_126, 0); +lean_inc(x_127); +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + x_128 = x_126; } else { - lean_dec_ref(x_117); - x_119 = lean_box(0); + lean_dec_ref(x_126); + x_128 = lean_box(0); } -if (lean_is_scalar(x_119)) { - x_120 = lean_alloc_ctor(0, 1, 0); +if (lean_is_scalar(x_128)) { + x_129 = lean_alloc_ctor(0, 1, 0); } else { - x_120 = x_119; + x_129 = x_128; } -lean_ctor_set(x_120, 0, x_118); -return x_120; +lean_ctor_set(x_129, 0, x_127); +return x_129; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_121 = lean_ctor_get(x_117, 0); -lean_inc(x_121); -if (lean_is_exclusive(x_117)) { - lean_ctor_release(x_117, 0); - x_122 = x_117; +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_130 = lean_ctor_get(x_126, 0); +lean_inc(x_130); +if (lean_is_exclusive(x_126)) { + lean_ctor_release(x_126, 0); + x_131 = x_126; } else { - lean_dec_ref(x_117); - x_122 = lean_box(0); + lean_dec_ref(x_126); + x_131 = lean_box(0); } -x_123 = lean_mk_array(x_108, x_121); -if (lean_is_scalar(x_122)) { - x_124 = lean_alloc_ctor(1, 1, 0); +x_132 = lean_box(0); +if (lean_is_scalar(x_61)) { + x_133 = lean_alloc_ctor(1, 2, 0); } else { - x_124 = x_122; + x_133 = x_61; } -lean_ctor_set(x_124, 0, x_123); -return x_124; +lean_ctor_set(x_133, 0, x_130); +lean_ctor_set(x_133, 1, x_132); +x_134 = lean_array_mk(x_133); +if (lean_is_scalar(x_131)) { + x_135 = lean_alloc_ctor(1, 1, 0); +} else { + x_135 = x_131; +} +lean_ctor_set(x_135, 0, x_134); +return x_135; } } } } else { -lean_object* x_125; -lean_dec(x_96); -lean_dec(x_55); -x_125 = l_Lake_resolvePackageTarget(x_1, x_95, x_3); +lean_object* x_136; +lean_dec(x_105); +lean_dec(x_61); +lean_dec(x_59); +x_136 = l_Lake_resolvePackageTarget(x_1, x_104, x_3); lean_dec(x_1); -return x_125; +return x_136; } } } diff --git a/stage0/stdlib/Lake/Load/Lean/Elab.c b/stage0/stdlib/Lake/Load/Lean/Elab.c index 6426e614fb52..327082b965eb 100644 --- a/stage0/stdlib/Lake/Load/Lean/Elab.c +++ b/stage0/stdlib/Lake/Load/Lean/Elab.c @@ -175,6 +175,7 @@ lean_object* l_IO_FS_readFile(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_importModulesUsingCache___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lake_Load_Lean_Elab_0__Lake_fromJsonConfigTrace____x40_Lake_Load_Lean_Elab___hyg_1110____closed__3; static lean_object* l_Array_foldlMUnsafe_fold___at_Lake_importConfigFileCore___spec__3___closed__1; +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__47; static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__25; static lean_object* l_Lake_elabConfigFile___closed__1; @@ -284,7 +285,6 @@ static lean_object* l___private_Lake_Load_Lean_Elab_0__Lake_fromJsonConfigTrace_ lean_object* lean_environment_add(lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); static lean_object* l_Lake_importConfigFileCore_lakeExts___closed__28; -lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonPosition____x40_Lean_Data_Lsp_Basic___hyg_221____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lake_Load_Lean_Elab_0__Lake_addToEnv___boxed(lean_object*, lean_object*); lean_object* l_Lean_MessageLog_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lake_importModulesUsingCache___spec__3(lean_object*); @@ -4643,7 +4643,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_10); lean_ctor_set(x_30, 1, x_29); x_31 = l___private_Lake_Load_Lean_Elab_0__Lake_toJsonConfigTrace____x40_Lake_Load_Lean_Elab___hyg_1030____closed__4; -x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonPosition____x40_Lean_Data_Lsp_Basic___hyg_221____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } diff --git a/stage0/stdlib/Lake/Load/Toml.c b/stage0/stdlib/Lake/Load/Toml.c index 89f4a16021e9..7ce1353f7282 100644 --- a/stage0/stdlib/Lake/Load/Toml.c +++ b/stage0/stdlib/Lake/Load/Toml.c @@ -32,6 +32,7 @@ static lean_object* l_Lake_LeanExeConfig_decodeToml___closed__2; LEAN_EXPORT lean_object* l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_LeanOption_decodeToml___closed__4; static lean_object* l_Lake_decodeLeanOptions___closed__2; +static lean_object* l_Lake_instDecodeTomlLeanExeConfig___closed__1; static lean_object* l_Lake_PackageConfig_decodeToml___closed__60; LEAN_EXPORT lean_object* l_Lake_LeanLibConfig_decodeToml(lean_object*, lean_object*); lean_object* l_System_FilePath_join(lean_object*, lean_object*); @@ -43,6 +44,7 @@ extern lean_object* l_Lake_defaultBuildDir; static lean_object* l_Lake_PackageConfig_decodeToml___closed__33; static uint8_t l_Lake_PackageConfig_decodeToml___closed__37; static lean_object* l_Lake_PackageConfig_decodeToml___closed__17; +static lean_object* l_Lake_instDecodeTomlDependencySrc___closed__1; lean_object* l_Array_push___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__58; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_loadTomlConfig___spec__8(size_t, size_t, lean_object*); @@ -55,12 +57,13 @@ static lean_object* l_Lake_LeanOption_decodeToml___closed__2; static lean_object* l_Lake_StrPat_decodeToml___closed__8; static lean_object* l_Lake_LeanConfig_decodeToml___closed__6; LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanOptionValue(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanConfig___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DependencySrc_decodeToml___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_LeanConfig_decodeToml___closed__1; lean_object* l_Lake_Toml_ppKey(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval___at_Lake_StrPat_decodeToml___spec__4(lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependency(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependency; LEAN_EXPORT lean_object* l_Lean_PersistentArray_forMAux___at_Lake_loadTomlConfig___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DependencySrc_decodeToml___closed__15; LEAN_EXPORT lean_object* l_Lake_StrPat_decodeToml(lean_object*, lean_object*); @@ -69,10 +72,11 @@ static lean_object* l_Lake_PackageConfig_decodeToml___closed__11; lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__62; LEAN_EXPORT lean_object* l_Lake_instDecodeTomlStdVer(lean_object*); +static lean_object* l_Lake_WorkspaceConfig_decodeToml___closed__3; static lean_object* l_Lake_DependencySrc_decodeToml___closed__1; lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2___lambda__1(lean_object*, lean_object*, lean_object*); -lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lake_defaultPackagesDir; uint8_t lean_usize_dec_eq(size_t, size_t); @@ -129,6 +133,7 @@ static lean_object* l_Lake_LeanConfig_decodeToml___closed__8; static lean_object* l_Lake_PackageConfig_decodeToml___closed__21; LEAN_EXPORT lean_object* l_Lake_Glob_ofString_x3f(lean_object*); static lean_object* l_Lake_LeanOptionValue_decodeToml___closed__1; +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependency___lambda__1(lean_object*); static lean_object* l_Lake_takeNamePart___closed__1; lean_object* l_Lake_RBArray_mkEmpty___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_StdVer_decodeToml(lean_object*); @@ -141,7 +146,7 @@ static lean_object* l_Lake_PackageConfig_decodeToml___closed__12; static lean_object* l_Lake_LeanConfig_decodeToml___closed__21; static lean_object* l_Lake_LeanConfig_decodeToml___closed__15; LEAN_EXPORT lean_object* l_Lake_Glob_ofString_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlPackageConfig(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlPackageConfig; static lean_object* l_Lake_LeanOption_decodeToml___closed__1; static lean_object* l_Lake_LeanConfig_decodeToml___closed__23; static lean_object* l_Lake_LeanOption_decodeToml___closed__8; @@ -162,17 +167,19 @@ static lean_object* l_Lake_LeanConfig_decodeToml___closed__5; uint8_t l_instDecidableNot___rarg(uint8_t); static lean_object* l_Lake_StrPat_decodeToml___closed__2; static lean_object* l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlWorkspaceConfig___lambda__1(lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__18; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__1___boxed(lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__8; static lean_object* l_Lake_PackageConfig_decodeToml___closed__50; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanExeConfig(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanExeConfig; static lean_object* l_Lake_Toml_Table_decode_x3f___at_Lake_StrPat_decodeToml___spec__3___closed__1; static lean_object* l_Lake_Dependency_decodeToml___closed__9; static lean_object* l_Lake_takeNamePart___closed__4; static lean_object* l_Lake_PackageConfig_decodeToml___closed__26; uint8_t lean_uint32_dec_le(uint32_t, uint32_t); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlPackageConfig___lambda__1(lean_object*); lean_object* lean_nat_to_int(lean_object*); static lean_object* l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__4; static lean_object* l_Lake_PackageConfig_decodeToml___closed__40; @@ -194,15 +201,17 @@ static lean_object* l_Lake_LeanConfig_decodeToml___closed__10; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__13(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__61; LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanConfig(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanConfig; static lean_object* l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_LeanLibConfig_decodeToml___spec__2(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__19; LEAN_EXPORT lean_object* l_Lake_Dependency_decodeToml(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanLibConfig___lambda__1(lean_object*); static lean_object* l_Lake_LeanLibConfig_decodeToml___closed__6; lean_object* l_Lean_Parser_mkInputContext(lean_object*, lean_object*, uint8_t); static lean_object* l_Lake_Dependency_decodeToml___closed__4; +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanExeConfig___lambda__1(lean_object*); static lean_object* l_Lake_LeanConfig_decodeToml___closed__17; lean_object* l_Substring_takeWhileAux___at___private_Init_Meta_0__Lean_Syntax_splitNameLitAux___spec__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_LeanConfig_decodeToml___closed__16; @@ -219,7 +228,7 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_StrPat_decodeToml___sp static lean_object* l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__2; static lean_object* l_Lake_StrPat_decodeToml___closed__4; static lean_object* l_Lake_PackageConfig_decodeToml___closed__22; -static uint8_t l_Lake_LeanOption_decodeToml___closed__7; +static lean_object* l_Lake_LeanOption_decodeToml___closed__7; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_StrPat_decodeToml___closed__5; static lean_object* l_Lake_PackageConfig_decodeToml___closed__31; @@ -239,13 +248,14 @@ LEAN_EXPORT lean_object* l_Lean_PersistentArray_forM___at_Lake_loadTomlConfig___ static lean_object* l_Lake_BuildType_decodeToml___closed__5; static lean_object* l_Lake_PackageConfig_decodeToml___closed__39; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlWorkspaceConfig(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlWorkspaceConfig; static lean_object* l_Lake_LeanConfig_decodeToml___closed__18; uint32_t lean_string_utf8_get_fast(lean_object*, lean_object*); lean_object* l_Lean_Syntax_decodeNatLitVal_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__9(lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__15; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lake_instDecodeTomlLeanConfig___closed__1; static lean_object* l_Lake_DependencySrc_decodeToml___closed__17; static lean_object* l_Lake_PackageConfig_decodeToml___closed__55; static lean_object* l_Lake_loadTomlConfig___closed__6; @@ -258,6 +268,7 @@ static lean_object* l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___s static lean_object* l_Lake_Dependency_decodeToml___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_LeanLibConfig_decodeToml___spec__5(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lake_Glob_ofString_x3f___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lake_instDecodeTomlPackageConfig___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_LeanOption_decodeToml___closed__9; LEAN_EXPORT lean_object* l_Lean_MessageLog_forM___at_Lake_loadTomlConfig___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -277,7 +288,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___sp static lean_object* l_Lake_LeanConfig_decodeToml___closed__20; lean_object* l_IO_FS_readFile(lean_object*, lean_object*); uint8_t l_Lean_isLetterLike(uint32_t); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanLibConfig(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanLibConfig; static lean_object* l_Lake_PackageConfig_decodeToml___closed__2; lean_object* l_Substring_nextn(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DependencySrc_decodeToml___closed__19; @@ -289,6 +300,7 @@ static lean_object* l_Lake_LeanOption_decodeToml___closed__11; static lean_object* l_Lake_PackageConfig_decodeToml___closed__45; static lean_object* l_Lake_PackageConfig_decodeToml___closed__44; static lean_object* l_Lake_DependencySrc_decodeToml___closed__6; +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependencySrc___lambda__1(lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__32; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern uint32_t l_Lean_idEndEscape; @@ -300,6 +312,7 @@ lean_object* l_Lake_StdVer_parse(lean_object*); lean_object* l_Lake_mergeErrors___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_LeanConfig_decodeToml___closed__24; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_StrPat_decodeToml___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lake_DependencySrc_decodeToml___closed__20; LEAN_EXPORT uint8_t l_Lake_StrPat_decodeToml___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__5(lean_object*, lean_object*); static lean_object* l_Lake_BuildType_decodeToml___closed__1; @@ -321,12 +334,14 @@ uint8_t lean_uint32_dec_eq(uint32_t, uint32_t); LEAN_EXPORT lean_object* l_Lake_decodeLeanOptionsAux___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__14; LEAN_EXPORT lean_object* l_Lake_instDecodeTomlGlob(lean_object*); +static lean_object* l_Lake_instDecodeTomlLeanLibConfig___closed__1; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lake_PackageConfig_decodeToml___closed__43; LEAN_EXPORT lean_object* l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_DependencySrc_decodeToml___closed__11; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_PackageConfig_decodeToml___spec__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__12(lean_object*); +static lean_object* l_Lake_instDecodeTomlDependency___closed__1; LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanOption; lean_object* l_String_toName(lean_object*); static lean_object* l_Lake_DependencySrc_decodeToml___closed__16; @@ -345,7 +360,7 @@ LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeTom static lean_object* l_Lake_DependencySrc_decodeToml___closed__4; static lean_object* l_Lake_DependencySrc_decodeToml___closed__7; LEAN_EXPORT lean_object* l_Lake_StrPat_decodeToml___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependencySrc(lean_object*); +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependencySrc; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___at_Lake_PackageConfig_decodeToml___spec__1(lean_object*); static lean_object* l_Lake_loadTomlConfig___closed__11; extern lean_object* l_Lake_defaultVersionTags; @@ -358,9 +373,10 @@ static lean_object* l_Lake_PackageConfig_decodeToml___closed__49; static lean_object* l_Lake_LeanConfig_decodeToml___closed__11; static lean_object* l_Lake_Dependency_decodeToml___closed__7; LEAN_EXPORT lean_object* l_Lake_LeanLibConfig_decodeToml___lambda__1(lean_object*, uint8_t); +static lean_object* l_Lake_WorkspaceConfig_decodeToml___closed__4; static lean_object* l_Lake_takeNamePart___closed__3; lean_object* lean_array_mk(lean_object*); -static lean_object* l_Lake_LeanOption_decodeToml___closed__5; +static uint8_t l_Lake_LeanOption_decodeToml___closed__5; static lean_object* l_Lake_Backend_decodeToml___closed__3; static lean_object* l_Lake_DependencySrc_decodeToml___closed__2; LEAN_EXPORT lean_object* l_Lake_Glob_decodeToml(lean_object*); @@ -1559,43 +1575,49 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_4); -lean_ctor_set(x_2, 0, x_6); +x_5 = lean_box(0); +x_6 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_array_mk(x_6); +lean_ctor_set(x_2, 0, x_7); return x_2; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); lean_dec(x_2); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_mk_array(x_8, x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) { return x_2; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } } @@ -1775,43 +1797,49 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_4); -lean_ctor_set(x_2, 0, x_6); +x_5 = lean_box(0); +x_6 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_array_mk(x_6); +lean_ctor_set(x_2, 0, x_7); return x_2; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); lean_dec(x_2); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_mk_array(x_8, x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) { return x_2; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } } @@ -1912,138 +1940,131 @@ lean_object* x_3; switch (lean_obj_tag(x_2)) { case 0: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_2); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -x_12 = l_String_toName(x_11); -if (lean_obj_tag(x_12) == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_2); +if (x_12 == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -lean_ctor_set(x_2, 1, x_13); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_2); -x_3 = x_15; -goto block_8; +x_13 = lean_ctor_get(x_2, 0); +x_14 = lean_ctor_get(x_2, 1); +x_15 = l_String_toName(x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; +x_16 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +lean_ctor_set(x_2, 1, x_16); +x_3 = x_2; +goto block_11; } else { -lean_object* x_16; +lean_object* x_17; lean_free_object(x_2); -lean_dec(x_10); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_12); -return x_16; +lean_dec(x_13); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_15); +return x_17; } } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_2, 0); -x_18 = lean_ctor_get(x_2, 1); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_2, 0); +x_19 = lean_ctor_get(x_2, 1); +lean_inc(x_19); lean_inc(x_18); -lean_inc(x_17); lean_dec(x_2); -x_19 = l_String_toName(x_18); -if (lean_obj_tag(x_19) == 0) +x_20 = l_String_toName(x_19); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_17); -lean_ctor_set(x_21, 1, x_20); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_mk_array(x_22, x_21); -x_3 = x_23; -goto block_8; +lean_object* x_21; lean_object* x_22; +x_21 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_18); +lean_ctor_set(x_22, 1, x_21); +x_3 = x_22; +goto block_11; } else { -lean_object* x_24; -lean_dec(x_17); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_19); -return x_24; +lean_object* x_23; +lean_dec(x_18); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_20); +return x_23; } } } case 2: { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_2, 0); -lean_inc(x_25); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_2, 0); +lean_inc(x_24); lean_dec(x_2); -x_26 = l_Lake_Glob_decodeToml___closed__2; -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -x_28 = lean_unsigned_to_nat(1u); -x_29 = lean_mk_array(x_28, x_27); -x_3 = x_29; -goto block_8; +x_25 = l_Lake_Glob_decodeToml___closed__2; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_3 = x_26; +goto block_11; } case 3: { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_2, 0); -lean_inc(x_30); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_2, 0); +lean_inc(x_27); lean_dec(x_2); -x_31 = l_Lake_Glob_decodeToml___closed__2; -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_mk_array(x_33, x_32); -x_3 = x_34; -goto block_8; +x_28 = l_Lake_Glob_decodeToml___closed__2; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +x_3 = x_29; +goto block_11; } default: { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_2); -if (x_35 == 0) +uint8_t x_30; +x_30 = !lean_is_exclusive(x_2); +if (x_30 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_2, 1); -lean_dec(x_36); -x_37 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_2, 1); +lean_dec(x_31); +x_32 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_37); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_2); -x_3 = x_39; -goto block_8; +lean_ctor_set(x_2, 1, x_32); +x_3 = x_2; +goto block_11; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_40 = lean_ctor_get(x_2, 0); -lean_inc(x_40); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_2, 0); +lean_inc(x_33); lean_dec(x_2); -x_41 = l_Lake_Glob_decodeToml___closed__2; -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_unsigned_to_nat(1u); -x_44 = lean_mk_array(x_43, x_42); -x_3 = x_44; -goto block_8; +x_34 = l_Lake_Glob_decodeToml___closed__2; +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_3 = x_35; +goto block_11; } } } -block_8: +block_11: { -size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_array_size(x_3); -x_5 = 0; -x_6 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__3(x_1, x_4, x_5, x_3); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +x_7 = lean_array_size(x_6); +x_8 = 0; +x_9 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__3(x_1, x_7, x_8, x_6); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; } } } @@ -2080,7 +2101,7 @@ lean_inc(x_2); x_5 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_4, x_2, x_1); if (lean_obj_tag(x_5) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_6 = l_Lake_Toml_ppKey(x_2); lean_dec(x_2); x_7 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__2; @@ -2091,25 +2112,28 @@ x_10 = lean_string_append(x_8, x_9); x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_3); lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_3); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_ctor_get(x_15, 1); +x_16 = lean_ctor_get(x_5, 0); lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2(x_2, x_16); +lean_dec(x_5); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2(x_2, x_17); lean_dec(x_2); -return x_17; +return x_18; } } } @@ -2189,49 +2213,55 @@ uint8_t x_4; x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; lean_object* x_10; +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; x_5 = lean_ctor_get(x_3, 0); -x_6 = lean_unsigned_to_nat(1u); -x_7 = lean_mk_array(x_6, x_5); -x_8 = lean_array_size(x_7); -x_9 = 0; -x_10 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__6(x_1, x_8, x_9, x_7); -lean_ctor_set(x_3, 0, x_10); +x_6 = lean_box(0); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_5); +lean_ctor_set(x_7, 1, x_6); +x_8 = lean_array_mk(x_7); +x_9 = lean_array_size(x_8); +x_10 = 0; +x_11 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__6(x_1, x_9, x_10, x_8); +lean_ctor_set(x_3, 0, x_11); return x_3; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; -x_11 = lean_ctor_get(x_3, 0); -lean_inc(x_11); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; +x_12 = lean_ctor_get(x_3, 0); +lean_inc(x_12); lean_dec(x_3); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_array_size(x_13); -x_15 = 0; -x_16 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__6(x_1, x_14, x_15, x_13); -x_17 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_17, 0, x_16); -return x_17; +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_array_mk(x_14); +x_16 = lean_array_size(x_15); +x_17 = 0; +x_18 = l_Array_mapMUnsafe_map___at_Lake_LeanOption_decodeToml___spec__6(x_1, x_16, x_17, x_15); +x_19 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_19, 0, x_18); +return x_19; } } else { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_3); -if (x_18 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_3); +if (x_20 == 0) { return x_3; } else { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_3, 0); -lean_inc(x_19); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_3, 0); +lean_inc(x_21); lean_dec(x_3); -x_20 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +return x_22; } } } @@ -2245,7 +2275,7 @@ lean_inc(x_2); x_5 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_4, x_2, x_1); if (lean_obj_tag(x_5) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_6 = l_Lake_Toml_ppKey(x_2); lean_dec(x_2); x_7 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__2; @@ -2256,25 +2286,28 @@ x_10 = lean_string_append(x_8, x_9); x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_3); lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_3); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_ctor_get(x_15, 1); +x_16 = lean_ctor_get(x_5, 0); lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__5(x_2, x_16); +lean_dec(x_5); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__5(x_2, x_17); lean_dec(x_2); -return x_17; +return x_18; } } } @@ -2313,43 +2346,43 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lake_LeanOption_decodeToml___closed__5() { +static uint8_t _init_l_Lake_LeanOption_decodeToml___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_LeanOption_decodeToml___closed__4; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; uint8_t x_2; +x_1 = l_Lake_LeanOption_decodeToml___closed__3; +x_2 = l_Array_isEmpty___rarg(x_1); +return x_2; } } static lean_object* _init_l_Lake_LeanOption_decodeToml___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lake_LeanOption_decodeToml___closed__5; -x_2 = lean_alloc_ctor(1, 1, 0); +x_1 = l_Lake_LeanOption_decodeToml___closed__3; +x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static uint8_t _init_l_Lake_LeanOption_decodeToml___closed__7() { +static lean_object* _init_l_Lake_LeanOption_decodeToml___closed__7() { _start: { -lean_object* x_1; uint8_t x_2; -x_1 = l_Lake_LeanOption_decodeToml___closed__3; -x_2 = l_Array_isEmpty___rarg(x_1); -return x_2; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_LeanOption_decodeToml___closed__4; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; } } static lean_object* _init_l_Lake_LeanOption_decodeToml___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lake_LeanOption_decodeToml___closed__3; -x_2 = lean_alloc_ctor(0, 1, 0); +x_1 = l_Lake_LeanOption_decodeToml___closed__7; +x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } @@ -2515,88 +2548,70 @@ return x_41; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_74; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_80; lean_dec(x_30); x_42 = lean_unsigned_to_nat(0u); x_43 = lean_array_fget(x_31, x_42); switch (lean_obj_tag(x_43)) { case 0: { -uint8_t x_106; -x_106 = !lean_is_exclusive(x_43); -if (x_106 == 0) +uint8_t x_115; +x_115 = !lean_is_exclusive(x_43); +if (x_115 == 0) { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_43, 0); -x_108 = lean_ctor_get(x_43, 1); -x_109 = l_String_toName(x_108); -if (lean_obj_tag(x_109) == 0) +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_43, 0); +x_117 = lean_ctor_get(x_43, 1); +x_118 = l_String_toName(x_117); +if (lean_obj_tag(x_118) == 0) { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -lean_ctor_set(x_43, 1, x_110); -x_111 = lean_unsigned_to_nat(1u); -x_112 = lean_mk_array(x_111, x_43); -x_44 = x_112; -goto block_73; +lean_object* x_119; +lean_dec(x_32); +x_119 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +lean_ctor_set(x_43, 1, x_119); +x_80 = x_43; +goto block_114; } else { lean_free_object(x_43); -lean_dec(x_107); -lean_dec(x_32); -x_74 = x_109; -goto block_105; +lean_dec(x_116); +x_44 = x_118; +goto block_79; } } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_43, 0); -x_114 = lean_ctor_get(x_43, 1); -lean_inc(x_114); -lean_inc(x_113); +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_ctor_get(x_43, 0); +x_121 = lean_ctor_get(x_43, 1); +lean_inc(x_121); +lean_inc(x_120); lean_dec(x_43); -x_115 = l_String_toName(x_114); -if (lean_obj_tag(x_115) == 0) +x_122 = l_String_toName(x_121); +if (lean_obj_tag(x_122) == 0) { -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_116 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_113); -lean_ctor_set(x_117, 1, x_116); -x_118 = lean_unsigned_to_nat(1u); -x_119 = lean_mk_array(x_118, x_117); -x_44 = x_119; -goto block_73; +lean_object* x_123; lean_object* x_124; +lean_dec(x_32); +x_123 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_120); +lean_ctor_set(x_124, 1, x_123); +x_80 = x_124; +goto block_114; } else { -lean_dec(x_113); -lean_dec(x_32); -x_74 = x_115; -goto block_105; +lean_dec(x_120); +x_44 = x_122; +goto block_79; } } } case 2: { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_120 = lean_ctor_get(x_43, 0); -lean_inc(x_120); -lean_dec(x_43); -x_121 = l_Lake_Glob_decodeToml___closed__2; -x_122 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_122, 0, x_120); -lean_ctor_set(x_122, 1, x_121); -x_123 = lean_unsigned_to_nat(1u); -x_124 = lean_mk_array(x_123, x_122); -x_44 = x_124; -goto block_73; -} -case 3: -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_32); x_125 = lean_ctor_get(x_43, 0); lean_inc(x_125); lean_dec(x_43); @@ -2604,298 +2619,337 @@ x_126 = l_Lake_Glob_decodeToml___closed__2; x_127 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_127, 0, x_125); lean_ctor_set(x_127, 1, x_126); -x_128 = lean_unsigned_to_nat(1u); -x_129 = lean_mk_array(x_128, x_127); -x_44 = x_129; -goto block_73; +x_80 = x_127; +goto block_114; +} +case 3: +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_dec(x_32); +x_128 = lean_ctor_get(x_43, 0); +lean_inc(x_128); +lean_dec(x_43); +x_129 = l_Lake_Glob_decodeToml___closed__2; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +x_80 = x_130; +goto block_114; } default: { -uint8_t x_130; -x_130 = !lean_is_exclusive(x_43); -if (x_130 == 0) +uint8_t x_131; +lean_dec(x_32); +x_131 = !lean_is_exclusive(x_43); +if (x_131 == 0) { -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_131 = lean_ctor_get(x_43, 1); -lean_dec(x_131); -x_132 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_132; lean_object* x_133; +x_132 = lean_ctor_get(x_43, 1); +lean_dec(x_132); +x_133 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_43, 0); -lean_ctor_set(x_43, 1, x_132); -x_133 = lean_unsigned_to_nat(1u); -x_134 = lean_mk_array(x_133, x_43); -x_44 = x_134; -goto block_73; +lean_ctor_set(x_43, 1, x_133); +x_80 = x_43; +goto block_114; } else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_135 = lean_ctor_get(x_43, 0); -lean_inc(x_135); +lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_134 = lean_ctor_get(x_43, 0); +lean_inc(x_134); lean_dec(x_43); -x_136 = l_Lake_Glob_decodeToml___closed__2; -x_137 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_137, 0, x_135); -lean_ctor_set(x_137, 1, x_136); -x_138 = lean_unsigned_to_nat(1u); -x_139 = lean_mk_array(x_138, x_137); -x_44 = x_139; -goto block_73; +x_135 = l_Lake_Glob_decodeToml___closed__2; +x_136 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +x_80 = x_136; +goto block_114; } } } -block_73: +block_79: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = l_Lake_LeanOption_decodeToml___closed__3; -x_46 = l_Array_append___rarg(x_45, x_44); -lean_dec(x_44); -x_47 = lean_unsigned_to_nat(1u); -x_48 = lean_array_fget(x_31, x_47); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_unsigned_to_nat(1u); +x_46 = lean_array_fget(x_31, x_45); lean_dec(x_31); -x_49 = l_Lake_LeanOptionValue_decodeToml(x_48); -if (lean_obj_tag(x_49) == 0) +x_47 = l_Lake_LeanOptionValue_decodeToml(x_46); +if (lean_obj_tag(x_47) == 0) { -uint8_t x_50; -lean_dec(x_32); -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) +uint8_t x_48; +x_48 = !lean_is_exclusive(x_47); +if (x_48 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_51 = lean_ctor_get(x_49, 0); -x_52 = lean_mk_array(x_47, x_51); -x_53 = l_Array_append___rarg(x_46, x_52); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; +x_49 = lean_ctor_get(x_47, 0); +x_50 = lean_box(0); +if (lean_is_scalar(x_32)) { + x_51 = lean_alloc_ctor(1, 2, 0); +} else { + x_51 = x_32; + lean_ctor_set_tag(x_51, 1); +} +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_array_mk(x_51); +x_53 = l_Lake_LeanOption_decodeToml___closed__3; +x_54 = l_Array_append___rarg(x_53, x_52); lean_dec(x_52); -x_54 = l_Array_isEmpty___rarg(x_53); -if (x_54 == 0) +x_55 = l_Lake_LeanOption_decodeToml___closed__4; +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_44); +lean_ctor_set(x_56, 1, x_55); +x_57 = l_Array_isEmpty___rarg(x_54); +if (x_57 == 0) { -lean_ctor_set(x_49, 0, x_53); -return x_49; +lean_dec(x_56); +lean_ctor_set(x_47, 0, x_54); +return x_47; } else { -lean_object* x_55; -lean_dec(x_53); -lean_free_object(x_49); -x_55 = l_Lake_LeanOption_decodeToml___closed__6; -return x_55; +lean_dec(x_54); +lean_ctor_set_tag(x_47, 1); +lean_ctor_set(x_47, 0, x_56); +return x_47; } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_56 = lean_ctor_get(x_49, 0); -lean_inc(x_56); -lean_dec(x_49); -x_57 = lean_mk_array(x_47, x_56); -x_58 = l_Array_append___rarg(x_46, x_57); -lean_dec(x_57); -x_59 = l_Array_isEmpty___rarg(x_58); -if (x_59 == 0) -{ -lean_object* x_60; -x_60 = lean_alloc_ctor(0, 1, 0); +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_58 = lean_ctor_get(x_47, 0); +lean_inc(x_58); +lean_dec(x_47); +x_59 = lean_box(0); +if (lean_is_scalar(x_32)) { + x_60 = lean_alloc_ctor(1, 2, 0); +} else { + x_60 = x_32; + lean_ctor_set_tag(x_60, 1); +} lean_ctor_set(x_60, 0, x_58); -return x_60; +lean_ctor_set(x_60, 1, x_59); +x_61 = lean_array_mk(x_60); +x_62 = l_Lake_LeanOption_decodeToml___closed__3; +x_63 = l_Array_append___rarg(x_62, x_61); +lean_dec(x_61); +x_64 = l_Lake_LeanOption_decodeToml___closed__4; +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_44); +lean_ctor_set(x_65, 1, x_64); +x_66 = l_Array_isEmpty___rarg(x_63); +if (x_66 == 0) +{ +lean_object* x_67; +lean_dec(x_65); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_63); +return x_67; } else { -lean_object* x_61; -lean_dec(x_58); -x_61 = l_Lake_LeanOption_decodeToml___closed__6; -return x_61; +lean_object* x_68; +lean_dec(x_63); +x_68 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_68, 0, x_65); +return x_68; } } } else { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_49); -if (x_62 == 0) +uint8_t x_69; +x_69 = !lean_is_exclusive(x_47); +if (x_69 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_63 = lean_ctor_get(x_49, 0); -x_64 = lean_box(0); -if (lean_is_scalar(x_32)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_32; - lean_ctor_set_tag(x_65, 0); -} -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_63); -x_66 = l_Array_isEmpty___rarg(x_46); -if (x_66 == 0) +lean_object* x_70; uint8_t x_71; +x_70 = lean_ctor_get(x_47, 0); +x_71 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_71 == 0) { -lean_dec(x_65); -lean_ctor_set_tag(x_49, 0); -lean_ctor_set(x_49, 0, x_46); -return x_49; +lean_object* x_72; +lean_free_object(x_47); +lean_dec(x_70); +lean_dec(x_44); +lean_dec(x_32); +x_72 = l_Lake_LeanOption_decodeToml___closed__6; +return x_72; } else { -lean_dec(x_46); -lean_ctor_set(x_49, 0, x_65); -return x_49; +lean_object* x_73; +if (lean_is_scalar(x_32)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_32; + lean_ctor_set_tag(x_73, 0); +} +lean_ctor_set(x_73, 0, x_44); +lean_ctor_set(x_73, 1, x_70); +lean_ctor_set(x_47, 0, x_73); +return x_47; } } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_67 = lean_ctor_get(x_49, 0); -lean_inc(x_67); -lean_dec(x_49); -x_68 = lean_box(0); -if (lean_is_scalar(x_32)) { - x_69 = lean_alloc_ctor(0, 2, 0); -} else { - x_69 = x_32; - lean_ctor_set_tag(x_69, 0); -} -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_67); -x_70 = l_Array_isEmpty___rarg(x_46); -if (x_70 == 0) +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_47, 0); +lean_inc(x_74); +lean_dec(x_47); +x_75 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_75 == 0) { -lean_object* x_71; -lean_dec(x_69); -x_71 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_71, 0, x_46); -return x_71; +lean_object* x_76; +lean_dec(x_74); +lean_dec(x_44); +lean_dec(x_32); +x_76 = l_Lake_LeanOption_decodeToml___closed__6; +return x_76; } else { -lean_object* x_72; -lean_dec(x_46); -x_72 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_72, 0, x_69); -return x_72; +lean_object* x_77; lean_object* x_78; +if (lean_is_scalar(x_32)) { + x_77 = lean_alloc_ctor(0, 2, 0); +} else { + x_77 = x_32; + lean_ctor_set_tag(x_77, 0); +} +lean_ctor_set(x_77, 0, x_44); +lean_ctor_set(x_77, 1, x_74); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_77); +return x_78; } } } } -block_105: +block_114: { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_unsigned_to_nat(1u); -x_76 = lean_array_fget(x_31, x_75); +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_81 = lean_box(0); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_array_mk(x_82); +x_84 = l_Lake_LeanOption_decodeToml___closed__3; +x_85 = l_Array_append___rarg(x_84, x_83); +lean_dec(x_83); +x_86 = lean_unsigned_to_nat(1u); +x_87 = lean_array_fget(x_31, x_86); lean_dec(x_31); -x_77 = l_Lake_LeanOptionValue_decodeToml(x_76); -if (lean_obj_tag(x_77) == 0) +x_88 = l_Lake_LeanOptionValue_decodeToml(x_87); +if (lean_obj_tag(x_88) == 0) { -uint8_t x_78; -x_78 = !lean_is_exclusive(x_77); -if (x_78 == 0) +uint8_t x_89; +x_89 = !lean_is_exclusive(x_88); +if (x_89 == 0) { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; -x_79 = lean_ctor_get(x_77, 0); -x_80 = lean_mk_array(x_75, x_79); -x_81 = l_Lake_LeanOption_decodeToml___closed__3; -x_82 = l_Array_append___rarg(x_81, x_80); -lean_dec(x_80); -x_83 = l_Lake_LeanOption_decodeToml___closed__4; -x_84 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_84, 0, x_74); -lean_ctor_set(x_84, 1, x_83); -x_85 = l_Array_isEmpty___rarg(x_82); -if (x_85 == 0) +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; +x_90 = lean_ctor_get(x_88, 0); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_81); +x_92 = lean_array_mk(x_91); +x_93 = l_Array_append___rarg(x_85, x_92); +lean_dec(x_92); +x_94 = l_Array_isEmpty___rarg(x_93); +if (x_94 == 0) { -lean_dec(x_84); -lean_ctor_set(x_77, 0, x_82); -return x_77; +lean_ctor_set(x_88, 0, x_93); +return x_88; } else { -lean_dec(x_82); -lean_ctor_set_tag(x_77, 1); -lean_ctor_set(x_77, 0, x_84); -return x_77; +lean_object* x_95; +lean_dec(x_93); +lean_free_object(x_88); +x_95 = l_Lake_LeanOption_decodeToml___closed__8; +return x_95; } } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; -x_86 = lean_ctor_get(x_77, 0); -lean_inc(x_86); -lean_dec(x_77); -x_87 = lean_mk_array(x_75, x_86); -x_88 = l_Lake_LeanOption_decodeToml___closed__3; -x_89 = l_Array_append___rarg(x_88, x_87); -lean_dec(x_87); -x_90 = l_Lake_LeanOption_decodeToml___closed__4; -x_91 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_91, 0, x_74); -lean_ctor_set(x_91, 1, x_90); -x_92 = l_Array_isEmpty___rarg(x_89); -if (x_92 == 0) +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_96 = lean_ctor_get(x_88, 0); +lean_inc(x_96); +lean_dec(x_88); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_81); +x_98 = lean_array_mk(x_97); +x_99 = l_Array_append___rarg(x_85, x_98); +lean_dec(x_98); +x_100 = l_Array_isEmpty___rarg(x_99); +if (x_100 == 0) { -lean_object* x_93; -lean_dec(x_91); -x_93 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_93, 0, x_89); -return x_93; +lean_object* x_101; +x_101 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_101, 0, x_99); +return x_101; } else { -lean_object* x_94; -lean_dec(x_89); -x_94 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_94, 0, x_91); -return x_94; +lean_object* x_102; +lean_dec(x_99); +x_102 = l_Lake_LeanOption_decodeToml___closed__8; +return x_102; } } } else { -uint8_t x_95; -x_95 = !lean_is_exclusive(x_77); -if (x_95 == 0) +uint8_t x_103; +x_103 = !lean_is_exclusive(x_88); +if (x_103 == 0) { -lean_object* x_96; uint8_t x_97; -x_96 = lean_ctor_get(x_77, 0); -x_97 = l_Lake_LeanOption_decodeToml___closed__7; -if (x_97 == 0) +lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; +x_104 = lean_ctor_get(x_88, 0); +x_105 = lean_box(0); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_104); +x_107 = l_Array_isEmpty___rarg(x_85); +if (x_107 == 0) { -lean_object* x_98; -lean_free_object(x_77); -lean_dec(x_96); -lean_dec(x_74); -x_98 = l_Lake_LeanOption_decodeToml___closed__8; -return x_98; +lean_dec(x_106); +lean_ctor_set_tag(x_88, 0); +lean_ctor_set(x_88, 0, x_85); +return x_88; } else { -lean_object* x_99; -x_99 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_99, 0, x_74); -lean_ctor_set(x_99, 1, x_96); -lean_ctor_set(x_77, 0, x_99); -return x_77; +lean_dec(x_85); +lean_ctor_set(x_88, 0, x_106); +return x_88; } } else { -lean_object* x_100; uint8_t x_101; -x_100 = lean_ctor_get(x_77, 0); -lean_inc(x_100); -lean_dec(x_77); -x_101 = l_Lake_LeanOption_decodeToml___closed__7; -if (x_101 == 0) +lean_object* x_108; lean_object* x_109; lean_object* x_110; uint8_t x_111; +x_108 = lean_ctor_get(x_88, 0); +lean_inc(x_108); +lean_dec(x_88); +x_109 = lean_box(0); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_108); +x_111 = l_Array_isEmpty___rarg(x_85); +if (x_111 == 0) { -lean_object* x_102; -lean_dec(x_100); -lean_dec(x_74); -x_102 = l_Lake_LeanOption_decodeToml___closed__8; -return x_102; +lean_object* x_112; +lean_dec(x_110); +x_112 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_112, 0, x_85); +return x_112; } else { -lean_object* x_103; lean_object* x_104; -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_74); -lean_ctor_set(x_103, 1, x_100); -x_104 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_104, 0, x_103); -return x_104; +lean_object* x_113; +lean_dec(x_85); +x_113 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_113, 0, x_110); +return x_113; } } } @@ -2904,259 +2958,259 @@ return x_104; } case 6: { -uint8_t x_140; -x_140 = !lean_is_exclusive(x_1); -if (x_140 == 0) +uint8_t x_137; +x_137 = !lean_is_exclusive(x_1); +if (x_137 == 0) { -lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_141 = lean_ctor_get(x_1, 0); -x_142 = lean_ctor_get(x_1, 1); -x_143 = l_Lake_LeanOption_decodeToml___closed__10; -lean_inc(x_141); +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_138 = lean_ctor_get(x_1, 0); +x_139 = lean_ctor_get(x_1, 1); +x_140 = l_Lake_LeanOption_decodeToml___closed__10; +lean_inc(x_138); +lean_inc(x_139); +x_141 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_139, x_140, x_138); +if (lean_obj_tag(x_141) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_142 = lean_ctor_get(x_141, 0); lean_inc(x_142); -x_144 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_142, x_143, x_141); -if (lean_obj_tag(x_144) == 0) +lean_dec(x_141); +x_143 = l_Lake_LeanOption_decodeToml___closed__3; +x_144 = l_Array_append___rarg(x_143, x_142); +lean_dec(x_142); +x_145 = l_Lake_LeanOption_decodeToml___closed__12; +x_146 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_139, x_145, x_138); +if (lean_obj_tag(x_146) == 0) { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_145 = lean_ctor_get(x_144, 0); -lean_inc(x_145); -lean_dec(x_144); -x_146 = l_Lake_LeanOption_decodeToml___closed__3; -x_147 = l_Array_append___rarg(x_146, x_145); -lean_dec(x_145); -x_148 = l_Lake_LeanOption_decodeToml___closed__12; -x_149 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_142, x_148, x_141); -if (lean_obj_tag(x_149) == 0) -{ -uint8_t x_150; +uint8_t x_147; lean_free_object(x_1); -x_150 = !lean_is_exclusive(x_149); -if (x_150 == 0) +x_147 = !lean_is_exclusive(x_146); +if (x_147 == 0) { -lean_object* x_151; lean_object* x_152; uint8_t x_153; -x_151 = lean_ctor_get(x_149, 0); -x_152 = l_Array_append___rarg(x_147, x_151); -lean_dec(x_151); -x_153 = l_Array_isEmpty___rarg(x_152); -if (x_153 == 0) +lean_object* x_148; lean_object* x_149; uint8_t x_150; +x_148 = lean_ctor_get(x_146, 0); +x_149 = l_Array_append___rarg(x_144, x_148); +lean_dec(x_148); +x_150 = l_Array_isEmpty___rarg(x_149); +if (x_150 == 0) { -lean_ctor_set(x_149, 0, x_152); -return x_149; +lean_ctor_set(x_146, 0, x_149); +return x_146; } else { -lean_object* x_154; -lean_dec(x_152); -lean_free_object(x_149); -x_154 = l_Lake_LeanOption_decodeToml___closed__6; -return x_154; +lean_object* x_151; +lean_dec(x_149); +lean_free_object(x_146); +x_151 = l_Lake_LeanOption_decodeToml___closed__8; +return x_151; } } else { -lean_object* x_155; lean_object* x_156; uint8_t x_157; -x_155 = lean_ctor_get(x_149, 0); -lean_inc(x_155); -lean_dec(x_149); -x_156 = l_Array_append___rarg(x_147, x_155); -lean_dec(x_155); -x_157 = l_Array_isEmpty___rarg(x_156); -if (x_157 == 0) +lean_object* x_152; lean_object* x_153; uint8_t x_154; +x_152 = lean_ctor_get(x_146, 0); +lean_inc(x_152); +lean_dec(x_146); +x_153 = l_Array_append___rarg(x_144, x_152); +lean_dec(x_152); +x_154 = l_Array_isEmpty___rarg(x_153); +if (x_154 == 0) { -lean_object* x_158; -x_158 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_158, 0, x_156); -return x_158; +lean_object* x_155; +x_155 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_155, 0, x_153); +return x_155; } else { -lean_object* x_159; -lean_dec(x_156); -x_159 = l_Lake_LeanOption_decodeToml___closed__6; -return x_159; +lean_object* x_156; +lean_dec(x_153); +x_156 = l_Lake_LeanOption_decodeToml___closed__8; +return x_156; } } } else { -uint8_t x_160; -x_160 = !lean_is_exclusive(x_149); +uint8_t x_157; +x_157 = !lean_is_exclusive(x_146); +if (x_157 == 0) +{ +lean_object* x_158; lean_object* x_159; uint8_t x_160; +x_158 = lean_ctor_get(x_146, 0); +x_159 = lean_box(0); +lean_ctor_set_tag(x_1, 0); +lean_ctor_set(x_1, 1, x_158); +lean_ctor_set(x_1, 0, x_159); +x_160 = l_Array_isEmpty___rarg(x_144); if (x_160 == 0) { +lean_dec(x_1); +lean_ctor_set_tag(x_146, 0); +lean_ctor_set(x_146, 0, x_144); +return x_146; +} +else +{ +lean_dec(x_144); +lean_ctor_set(x_146, 0, x_1); +return x_146; +} +} +else +{ lean_object* x_161; lean_object* x_162; uint8_t x_163; -x_161 = lean_ctor_get(x_149, 0); +x_161 = lean_ctor_get(x_146, 0); +lean_inc(x_161); +lean_dec(x_146); x_162 = lean_box(0); lean_ctor_set_tag(x_1, 0); lean_ctor_set(x_1, 1, x_161); lean_ctor_set(x_1, 0, x_162); -x_163 = l_Array_isEmpty___rarg(x_147); +x_163 = l_Array_isEmpty___rarg(x_144); if (x_163 == 0) { +lean_object* x_164; lean_dec(x_1); -lean_ctor_set_tag(x_149, 0); -lean_ctor_set(x_149, 0, x_147); -return x_149; +x_164 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_164, 0, x_144); +return x_164; } else { -lean_dec(x_147); -lean_ctor_set(x_149, 0, x_1); -return x_149; +lean_object* x_165; +lean_dec(x_144); +x_165 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_165, 0, x_1); +return x_165; +} +} } } else { -lean_object* x_164; lean_object* x_165; uint8_t x_166; -x_164 = lean_ctor_get(x_149, 0); -lean_inc(x_164); -lean_dec(x_149); -x_165 = lean_box(0); +lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_166 = lean_ctor_get(x_141, 0); +lean_inc(x_166); +lean_dec(x_141); +x_167 = l_Lake_LeanOption_decodeToml___closed__12; +x_168 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_139, x_167, x_138); +if (lean_obj_tag(x_168) == 0) +{ +uint8_t x_169; +x_169 = !lean_is_exclusive(x_168); +if (x_169 == 0) +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; +x_170 = lean_ctor_get(x_168, 0); +x_171 = l_Lake_LeanOption_decodeToml___closed__3; +x_172 = l_Array_append___rarg(x_171, x_170); +lean_dec(x_170); +x_173 = l_Lake_LeanOption_decodeToml___closed__4; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_164); -lean_ctor_set(x_1, 0, x_165); -x_166 = l_Array_isEmpty___rarg(x_147); -if (x_166 == 0) +lean_ctor_set(x_1, 1, x_173); +lean_ctor_set(x_1, 0, x_166); +x_174 = l_Array_isEmpty___rarg(x_172); +if (x_174 == 0) { -lean_object* x_167; lean_dec(x_1); -x_167 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_167, 0, x_147); -return x_167; +lean_ctor_set(x_168, 0, x_172); +return x_168; } else { -lean_object* x_168; -lean_dec(x_147); -x_168 = lean_alloc_ctor(1, 1, 0); +lean_dec(x_172); +lean_ctor_set_tag(x_168, 1); lean_ctor_set(x_168, 0, x_1); return x_168; } } -} -} else { -lean_object* x_169; lean_object* x_170; lean_object* x_171; -x_169 = lean_ctor_get(x_144, 0); -lean_inc(x_169); -lean_dec(x_144); -x_170 = l_Lake_LeanOption_decodeToml___closed__12; -x_171 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_142, x_170, x_141); -if (lean_obj_tag(x_171) == 0) -{ -uint8_t x_172; -x_172 = !lean_is_exclusive(x_171); -if (x_172 == 0) -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; uint8_t x_177; -x_173 = lean_ctor_get(x_171, 0); -x_174 = l_Lake_LeanOption_decodeToml___closed__3; -x_175 = l_Array_append___rarg(x_174, x_173); -lean_dec(x_173); -x_176 = l_Lake_LeanOption_decodeToml___closed__4; +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_175 = lean_ctor_get(x_168, 0); +lean_inc(x_175); +lean_dec(x_168); +x_176 = l_Lake_LeanOption_decodeToml___closed__3; +x_177 = l_Array_append___rarg(x_176, x_175); +lean_dec(x_175); +x_178 = l_Lake_LeanOption_decodeToml___closed__4; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_176); -lean_ctor_set(x_1, 0, x_169); -x_177 = l_Array_isEmpty___rarg(x_175); -if (x_177 == 0) +lean_ctor_set(x_1, 1, x_178); +lean_ctor_set(x_1, 0, x_166); +x_179 = l_Array_isEmpty___rarg(x_177); +if (x_179 == 0) { +lean_object* x_180; lean_dec(x_1); -lean_ctor_set(x_171, 0, x_175); -return x_171; +x_180 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_180, 0, x_177); +return x_180; } else { -lean_dec(x_175); -lean_ctor_set_tag(x_171, 1); -lean_ctor_set(x_171, 0, x_1); -return x_171; +lean_object* x_181; +lean_dec(x_177); +x_181 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_181, 0, x_1); +return x_181; +} } } else { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; uint8_t x_182; -x_178 = lean_ctor_get(x_171, 0); -lean_inc(x_178); -lean_dec(x_171); -x_179 = l_Lake_LeanOption_decodeToml___closed__3; -x_180 = l_Array_append___rarg(x_179, x_178); -lean_dec(x_178); -x_181 = l_Lake_LeanOption_decodeToml___closed__4; -lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_181); -lean_ctor_set(x_1, 0, x_169); -x_182 = l_Array_isEmpty___rarg(x_180); +uint8_t x_182; +x_182 = !lean_is_exclusive(x_168); if (x_182 == 0) { -lean_object* x_183; -lean_dec(x_1); -x_183 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_183, 0, x_180); -return x_183; +lean_object* x_183; uint8_t x_184; +x_183 = lean_ctor_get(x_168, 0); +x_184 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_184 == 0) +{ +lean_object* x_185; +lean_free_object(x_168); +lean_dec(x_183); +lean_dec(x_166); +lean_free_object(x_1); +x_185 = l_Lake_LeanOption_decodeToml___closed__6; +return x_185; } else { -lean_object* x_184; -lean_dec(x_180); -x_184 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_184, 0, x_1); -return x_184; -} +lean_ctor_set_tag(x_1, 0); +lean_ctor_set(x_1, 1, x_183); +lean_ctor_set(x_1, 0, x_166); +lean_ctor_set(x_168, 0, x_1); +return x_168; } } else { -uint8_t x_185; -x_185 = !lean_is_exclusive(x_171); -if (x_185 == 0) -{ lean_object* x_186; uint8_t x_187; -x_186 = lean_ctor_get(x_171, 0); -x_187 = l_Lake_LeanOption_decodeToml___closed__7; +x_186 = lean_ctor_get(x_168, 0); +lean_inc(x_186); +lean_dec(x_168); +x_187 = l_Lake_LeanOption_decodeToml___closed__5; if (x_187 == 0) { lean_object* x_188; -lean_free_object(x_171); lean_dec(x_186); -lean_dec(x_169); +lean_dec(x_166); lean_free_object(x_1); -x_188 = l_Lake_LeanOption_decodeToml___closed__8; +x_188 = l_Lake_LeanOption_decodeToml___closed__6; return x_188; } else { +lean_object* x_189; lean_ctor_set_tag(x_1, 0); lean_ctor_set(x_1, 1, x_186); -lean_ctor_set(x_1, 0, x_169); -lean_ctor_set(x_171, 0, x_1); -return x_171; -} -} -else -{ -lean_object* x_189; uint8_t x_190; -x_189 = lean_ctor_get(x_171, 0); -lean_inc(x_189); -lean_dec(x_171); -x_190 = l_Lake_LeanOption_decodeToml___closed__7; -if (x_190 == 0) -{ -lean_object* x_191; -lean_dec(x_189); -lean_dec(x_169); -lean_free_object(x_1); -x_191 = l_Lake_LeanOption_decodeToml___closed__8; -return x_191; -} -else -{ -lean_object* x_192; -lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_189); -lean_ctor_set(x_1, 0, x_169); -x_192 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_192, 0, x_1); -return x_192; +lean_ctor_set(x_1, 0, x_166); +x_189 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_189, 0, x_1); +return x_189; } } } @@ -3164,195 +3218,195 @@ return x_192; } else { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; -x_193 = lean_ctor_get(x_1, 0); -x_194 = lean_ctor_get(x_1, 1); -lean_inc(x_194); -lean_inc(x_193); +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; +x_190 = lean_ctor_get(x_1, 0); +x_191 = lean_ctor_get(x_1, 1); +lean_inc(x_191); +lean_inc(x_190); lean_dec(x_1); -x_195 = l_Lake_LeanOption_decodeToml___closed__10; -lean_inc(x_193); -lean_inc(x_194); -x_196 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_194, x_195, x_193); -if (lean_obj_tag(x_196) == 0) +x_192 = l_Lake_LeanOption_decodeToml___closed__10; +lean_inc(x_190); +lean_inc(x_191); +x_193 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_191, x_192, x_190); +if (lean_obj_tag(x_193) == 0) { -lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -x_197 = lean_ctor_get(x_196, 0); -lean_inc(x_197); -lean_dec(x_196); -x_198 = l_Lake_LeanOption_decodeToml___closed__3; -x_199 = l_Array_append___rarg(x_198, x_197); -lean_dec(x_197); -x_200 = l_Lake_LeanOption_decodeToml___closed__12; -x_201 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_194, x_200, x_193); -if (lean_obj_tag(x_201) == 0) +lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; +x_194 = lean_ctor_get(x_193, 0); +lean_inc(x_194); +lean_dec(x_193); +x_195 = l_Lake_LeanOption_decodeToml___closed__3; +x_196 = l_Array_append___rarg(x_195, x_194); +lean_dec(x_194); +x_197 = l_Lake_LeanOption_decodeToml___closed__12; +x_198 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_191, x_197, x_190); +if (lean_obj_tag(x_198) == 0) { -lean_object* x_202; lean_object* x_203; lean_object* x_204; uint8_t x_205; -x_202 = lean_ctor_get(x_201, 0); -lean_inc(x_202); -if (lean_is_exclusive(x_201)) { - lean_ctor_release(x_201, 0); - x_203 = x_201; +lean_object* x_199; lean_object* x_200; lean_object* x_201; uint8_t x_202; +x_199 = lean_ctor_get(x_198, 0); +lean_inc(x_199); +if (lean_is_exclusive(x_198)) { + lean_ctor_release(x_198, 0); + x_200 = x_198; } else { - lean_dec_ref(x_201); - x_203 = lean_box(0); + lean_dec_ref(x_198); + x_200 = lean_box(0); } -x_204 = l_Array_append___rarg(x_199, x_202); -lean_dec(x_202); -x_205 = l_Array_isEmpty___rarg(x_204); -if (x_205 == 0) +x_201 = l_Array_append___rarg(x_196, x_199); +lean_dec(x_199); +x_202 = l_Array_isEmpty___rarg(x_201); +if (x_202 == 0) { -lean_object* x_206; -if (lean_is_scalar(x_203)) { - x_206 = lean_alloc_ctor(0, 1, 0); +lean_object* x_203; +if (lean_is_scalar(x_200)) { + x_203 = lean_alloc_ctor(0, 1, 0); } else { - x_206 = x_203; + x_203 = x_200; } -lean_ctor_set(x_206, 0, x_204); -return x_206; +lean_ctor_set(x_203, 0, x_201); +return x_203; } else { -lean_object* x_207; -lean_dec(x_204); -lean_dec(x_203); -x_207 = l_Lake_LeanOption_decodeToml___closed__6; -return x_207; +lean_object* x_204; +lean_dec(x_201); +lean_dec(x_200); +x_204 = l_Lake_LeanOption_decodeToml___closed__8; +return x_204; } } else { -lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; uint8_t x_212; -x_208 = lean_ctor_get(x_201, 0); -lean_inc(x_208); -if (lean_is_exclusive(x_201)) { - lean_ctor_release(x_201, 0); - x_209 = x_201; +lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; uint8_t x_209; +x_205 = lean_ctor_get(x_198, 0); +lean_inc(x_205); +if (lean_is_exclusive(x_198)) { + lean_ctor_release(x_198, 0); + x_206 = x_198; } else { - lean_dec_ref(x_201); - x_209 = lean_box(0); + lean_dec_ref(x_198); + x_206 = lean_box(0); } -x_210 = lean_box(0); -x_211 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_211, 0, x_210); -lean_ctor_set(x_211, 1, x_208); -x_212 = l_Array_isEmpty___rarg(x_199); -if (x_212 == 0) -{ -lean_object* x_213; -lean_dec(x_211); -if (lean_is_scalar(x_209)) { - x_213 = lean_alloc_ctor(0, 1, 0); +x_207 = lean_box(0); +x_208 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_208, 0, x_207); +lean_ctor_set(x_208, 1, x_205); +x_209 = l_Array_isEmpty___rarg(x_196); +if (x_209 == 0) +{ +lean_object* x_210; +lean_dec(x_208); +if (lean_is_scalar(x_206)) { + x_210 = lean_alloc_ctor(0, 1, 0); } else { - x_213 = x_209; - lean_ctor_set_tag(x_213, 0); + x_210 = x_206; + lean_ctor_set_tag(x_210, 0); } -lean_ctor_set(x_213, 0, x_199); -return x_213; +lean_ctor_set(x_210, 0, x_196); +return x_210; } else { -lean_object* x_214; -lean_dec(x_199); -if (lean_is_scalar(x_209)) { - x_214 = lean_alloc_ctor(1, 1, 0); +lean_object* x_211; +lean_dec(x_196); +if (lean_is_scalar(x_206)) { + x_211 = lean_alloc_ctor(1, 1, 0); } else { - x_214 = x_209; + x_211 = x_206; } -lean_ctor_set(x_214, 0, x_211); -return x_214; +lean_ctor_set(x_211, 0, x_208); +return x_211; } } } else { -lean_object* x_215; lean_object* x_216; lean_object* x_217; -x_215 = lean_ctor_get(x_196, 0); -lean_inc(x_215); -lean_dec(x_196); -x_216 = l_Lake_LeanOption_decodeToml___closed__12; -x_217 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_194, x_216, x_193); -if (lean_obj_tag(x_217) == 0) +lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_212 = lean_ctor_get(x_193, 0); +lean_inc(x_212); +lean_dec(x_193); +x_213 = l_Lake_LeanOption_decodeToml___closed__12; +x_214 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__4(x_191, x_213, x_190); +if (lean_obj_tag(x_214) == 0) { -lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; -x_218 = lean_ctor_get(x_217, 0); -lean_inc(x_218); -if (lean_is_exclusive(x_217)) { - lean_ctor_release(x_217, 0); - x_219 = x_217; +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; uint8_t x_221; +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + x_216 = x_214; } else { - lean_dec_ref(x_217); - x_219 = lean_box(0); + lean_dec_ref(x_214); + x_216 = lean_box(0); } -x_220 = l_Lake_LeanOption_decodeToml___closed__3; -x_221 = l_Array_append___rarg(x_220, x_218); -lean_dec(x_218); -x_222 = l_Lake_LeanOption_decodeToml___closed__4; -x_223 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_223, 0, x_215); -lean_ctor_set(x_223, 1, x_222); -x_224 = l_Array_isEmpty___rarg(x_221); -if (x_224 == 0) -{ -lean_object* x_225; -lean_dec(x_223); -if (lean_is_scalar(x_219)) { - x_225 = lean_alloc_ctor(0, 1, 0); +x_217 = l_Lake_LeanOption_decodeToml___closed__3; +x_218 = l_Array_append___rarg(x_217, x_215); +lean_dec(x_215); +x_219 = l_Lake_LeanOption_decodeToml___closed__4; +x_220 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_220, 0, x_212); +lean_ctor_set(x_220, 1, x_219); +x_221 = l_Array_isEmpty___rarg(x_218); +if (x_221 == 0) +{ +lean_object* x_222; +lean_dec(x_220); +if (lean_is_scalar(x_216)) { + x_222 = lean_alloc_ctor(0, 1, 0); } else { - x_225 = x_219; + x_222 = x_216; } -lean_ctor_set(x_225, 0, x_221); -return x_225; +lean_ctor_set(x_222, 0, x_218); +return x_222; } else { -lean_object* x_226; -lean_dec(x_221); -if (lean_is_scalar(x_219)) { - x_226 = lean_alloc_ctor(1, 1, 0); +lean_object* x_223; +lean_dec(x_218); +if (lean_is_scalar(x_216)) { + x_223 = lean_alloc_ctor(1, 1, 0); } else { - x_226 = x_219; - lean_ctor_set_tag(x_226, 1); + x_223 = x_216; + lean_ctor_set_tag(x_223, 1); } -lean_ctor_set(x_226, 0, x_223); -return x_226; +lean_ctor_set(x_223, 0, x_220); +return x_223; } } else { -lean_object* x_227; lean_object* x_228; uint8_t x_229; -x_227 = lean_ctor_get(x_217, 0); -lean_inc(x_227); -if (lean_is_exclusive(x_217)) { - lean_ctor_release(x_217, 0); - x_228 = x_217; +lean_object* x_224; lean_object* x_225; uint8_t x_226; +x_224 = lean_ctor_get(x_214, 0); +lean_inc(x_224); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + x_225 = x_214; } else { - lean_dec_ref(x_217); - x_228 = lean_box(0); + lean_dec_ref(x_214); + x_225 = lean_box(0); } -x_229 = l_Lake_LeanOption_decodeToml___closed__7; -if (x_229 == 0) +x_226 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_226 == 0) { -lean_object* x_230; -lean_dec(x_228); -lean_dec(x_227); -lean_dec(x_215); -x_230 = l_Lake_LeanOption_decodeToml___closed__8; -return x_230; +lean_object* x_227; +lean_dec(x_225); +lean_dec(x_224); +lean_dec(x_212); +x_227 = l_Lake_LeanOption_decodeToml___closed__6; +return x_227; } else { -lean_object* x_231; lean_object* x_232; -x_231 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_231, 0, x_215); -lean_ctor_set(x_231, 1, x_227); -if (lean_is_scalar(x_228)) { - x_232 = lean_alloc_ctor(1, 1, 0); +lean_object* x_228; lean_object* x_229; +x_228 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_228, 0, x_212); +lean_ctor_set(x_228, 1, x_224); +if (lean_is_scalar(x_225)) { + x_229 = lean_alloc_ctor(1, 1, 0); } else { - x_232 = x_228; + x_229 = x_225; } -lean_ctor_set(x_232, 0, x_231); -return x_232; +lean_ctor_set(x_229, 0, x_228); +return x_229; } } } @@ -3360,43 +3414,43 @@ return x_232; } default: { -uint8_t x_233; -x_233 = !lean_is_exclusive(x_1); -if (x_233 == 0) +uint8_t x_230; +x_230 = !lean_is_exclusive(x_1); +if (x_230 == 0) { -lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_234 = lean_ctor_get(x_1, 1); -lean_dec(x_234); -x_235 = l_Lake_LeanOption_decodeToml___closed__1; +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_231 = lean_ctor_get(x_1, 1); +lean_dec(x_231); +x_232 = l_Lake_LeanOption_decodeToml___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_235); -x_236 = lean_box(0); -x_237 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_237, 0, x_1); -lean_ctor_set(x_237, 1, x_236); -x_238 = lean_array_mk(x_237); -x_239 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_239, 0, x_238); -return x_239; +lean_ctor_set(x_1, 1, x_232); +x_233 = lean_box(0); +x_234 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_234, 0, x_1); +lean_ctor_set(x_234, 1, x_233); +x_235 = lean_array_mk(x_234); +x_236 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_236, 0, x_235); +return x_236; } else { -lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_240 = lean_ctor_get(x_1, 0); -lean_inc(x_240); +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; +x_237 = lean_ctor_get(x_1, 0); +lean_inc(x_237); lean_dec(x_1); -x_241 = l_Lake_LeanOption_decodeToml___closed__1; -x_242 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_242, 0, x_240); -lean_ctor_set(x_242, 1, x_241); -x_243 = lean_box(0); -x_244 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_244, 0, x_242); -lean_ctor_set(x_244, 1, x_243); -x_245 = lean_array_mk(x_244); -x_246 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_246, 0, x_245); -return x_246; +x_238 = l_Lake_LeanOption_decodeToml___closed__1; +x_239 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_239, 0, x_237); +lean_ctor_set(x_239, 1, x_238); +x_240 = lean_box(0); +x_241 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_241, 0, x_239); +lean_ctor_set(x_241, 1, x_240); +x_242 = lean_array_mk(x_241); +x_243 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_243, 0, x_242); +return x_243; } } } @@ -3771,43 +3825,49 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_4); -lean_ctor_set(x_2, 0, x_6); +x_5 = lean_box(0); +x_6 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_array_mk(x_6); +lean_ctor_set(x_2, 0, x_7); return x_2; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); lean_dec(x_2); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_mk_array(x_8, x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) { return x_2; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } } @@ -4073,43 +4133,49 @@ uint8_t x_3; x_3 = !lean_is_exclusive(x_2); if (x_3 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_4); -lean_ctor_set(x_2, 0, x_6); +x_5 = lean_box(0); +x_6 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_6, 0, x_4); +lean_ctor_set(x_6, 1, x_5); +x_7 = lean_array_mk(x_6); +lean_ctor_set(x_2, 0, x_7); return x_2; } else { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_2, 0); -lean_inc(x_7); +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); lean_dec(x_2); -x_8 = lean_unsigned_to_nat(1u); -x_9 = lean_mk_array(x_8, x_7); -x_10 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_9 = lean_box(0); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +return x_12; } } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_2); -if (x_11 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_2); +if (x_13 == 0) { return x_2; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } } } @@ -4158,122 +4224,447 @@ return x_5; LEAN_EXPORT lean_object* l_Lake_decodeLeanOptionsAux(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -if (lean_obj_tag(x_1) == 6) +switch (lean_obj_tag(x_1)) { +case 1: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_4 = lean_ctor_get(x_1, 1); -lean_inc(x_4); -lean_dec(x_1); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -lean_dec(x_4); -x_6 = lean_array_get_size(x_5); -x_7 = lean_unsigned_to_nat(0u); -x_8 = lean_nat_dec_lt(x_7, x_6); -if (x_8 == 0) +lean_object* x_4; uint8_t x_5; +lean_inc(x_1); +x_4 = l_Lake_LeanOptionValue_decodeToml(x_1); +x_5 = !lean_is_exclusive(x_1); +if (x_5 == 0) { +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_1, 1); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -return x_3; -} -else +x_7 = lean_ctor_get(x_1, 0); +lean_dec(x_7); +x_8 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_8, 0, x_2); +if (lean_obj_tag(x_4) == 0) { uint8_t x_9; -x_9 = lean_nat_dec_le(x_6, x_6); +x_9 = !lean_is_exclusive(x_4); if (x_9 == 0) { -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -return x_3; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_4, 0); +x_11 = lean_box(0); +lean_ctor_set(x_1, 1, x_11); +lean_ctor_set(x_1, 0, x_10); +x_12 = lean_array_mk(x_1); +lean_ctor_set(x_4, 0, x_12); +x_13 = l_Lake_mergeErrors___rarg(x_3, x_4, x_8); +return x_13; } else { -size_t x_10; size_t x_11; lean_object* x_12; -x_10 = 0; -x_11 = lean_usize_of_nat(x_6); -lean_dec(x_6); -x_12 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1(x_2, x_5, x_10, x_11, x_3); -lean_dec(x_5); -return x_12; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_14 = lean_ctor_get(x_4, 0); +lean_inc(x_14); +lean_dec(x_4); +x_15 = lean_box(0); +lean_ctor_set(x_1, 1, x_15); +lean_ctor_set(x_1, 0, x_14); +x_16 = lean_array_mk(x_1); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_16); +x_18 = l_Lake_mergeErrors___rarg(x_3, x_17, x_8); +return x_18; } } else { -lean_object* x_13; lean_object* x_14; -x_13 = l_Lake_LeanOptionValue_decodeToml(x_1); -x_14 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); -lean_closure_set(x_14, 0, x_2); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_13); -if (x_15 == 0) +uint8_t x_19; +lean_free_object(x_1); +x_19 = !lean_is_exclusive(x_4); +if (x_19 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_13, 0); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -lean_ctor_set(x_13, 0, x_18); -x_19 = l_Lake_mergeErrors___rarg(x_3, x_13, x_14); -return x_19; +lean_object* x_20; +x_20 = l_Lake_mergeErrors___rarg(x_3, x_4, x_8); +return x_20; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_20 = lean_ctor_get(x_13, 0); -lean_inc(x_20); -lean_dec(x_13); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_mk_array(x_21, x_20); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = l_Lake_mergeErrors___rarg(x_3, x_23, x_14); -return x_24; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_4, 0); +lean_inc(x_21); +lean_dec(x_4); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lake_mergeErrors___rarg(x_3, x_22, x_8); +return x_23; +} } } else { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_13); -if (x_25 == 0) +lean_object* x_24; +lean_dec(x_1); +x_24 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_24, 0, x_2); +if (lean_obj_tag(x_4) == 0) { -lean_object* x_26; -x_26 = l_Lake_mergeErrors___rarg(x_3, x_13, x_14); -return x_26; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_25 = lean_ctor_get(x_4, 0); +lean_inc(x_25); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + x_26 = x_4; +} else { + lean_dec_ref(x_4); + x_26 = lean_box(0); +} +x_27 = lean_box(0); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_25); +lean_ctor_set(x_28, 1, x_27); +x_29 = lean_array_mk(x_28); +if (lean_is_scalar(x_26)) { + x_30 = lean_alloc_ctor(0, 1, 0); +} else { + x_30 = x_26; +} +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lake_mergeErrors___rarg(x_3, x_30, x_24); +return x_31; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_13, 0); -lean_inc(x_27); -lean_dec(x_13); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = l_Lake_mergeErrors___rarg(x_3, x_28, x_14); -return x_29; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_4, 0); +lean_inc(x_32); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + x_33 = x_4; +} else { + lean_dec_ref(x_4); + x_33 = lean_box(0); } +if (lean_is_scalar(x_33)) { + x_34 = lean_alloc_ctor(1, 1, 0); +} else { + x_34 = x_33; } +lean_ctor_set(x_34, 0, x_32); +x_35 = l_Lake_mergeErrors___rarg(x_3, x_34, x_24); +return x_35; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +case 2: { -size_t x_6; size_t x_7; lean_object* x_8; -x_6 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_7 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_8 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1(x_1, x_2, x_6, x_7, x_5); -lean_dec(x_2); -return x_8; -} -} -static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1() { -_start: +lean_object* x_36; lean_object* x_37; +x_36 = l_Lake_LeanOptionValue_decodeToml(x_1); +x_37 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_37, 0, x_2); +if (lean_obj_tag(x_36) == 0) +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_36); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_39 = lean_ctor_get(x_36, 0); +x_40 = lean_box(0); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_array_mk(x_41); +lean_ctor_set(x_36, 0, x_42); +x_43 = l_Lake_mergeErrors___rarg(x_3, x_36, x_37); +return x_43; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_44 = lean_ctor_get(x_36, 0); +lean_inc(x_44); +lean_dec(x_36); +x_45 = lean_box(0); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +x_47 = lean_array_mk(x_46); +x_48 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_48, 0, x_47); +x_49 = l_Lake_mergeErrors___rarg(x_3, x_48, x_37); +return x_49; +} +} +else +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_36); +if (x_50 == 0) +{ +lean_object* x_51; +x_51 = l_Lake_mergeErrors___rarg(x_3, x_36, x_37); +return x_51; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_36, 0); +lean_inc(x_52); +lean_dec(x_36); +x_53 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_53, 0, x_52); +x_54 = l_Lake_mergeErrors___rarg(x_3, x_53, x_37); +return x_54; +} +} +} +case 3: +{ +lean_object* x_55; lean_object* x_56; +x_55 = l_Lake_LeanOptionValue_decodeToml(x_1); +x_56 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_56, 0, x_2); +if (lean_obj_tag(x_55) == 0) +{ +uint8_t x_57; +x_57 = !lean_is_exclusive(x_55); +if (x_57 == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_58 = lean_ctor_get(x_55, 0); +x_59 = lean_box(0); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +x_61 = lean_array_mk(x_60); +lean_ctor_set(x_55, 0, x_61); +x_62 = l_Lake_mergeErrors___rarg(x_3, x_55, x_56); +return x_62; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_63 = lean_ctor_get(x_55, 0); +lean_inc(x_63); +lean_dec(x_55); +x_64 = lean_box(0); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +x_66 = lean_array_mk(x_65); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +x_68 = l_Lake_mergeErrors___rarg(x_3, x_67, x_56); +return x_68; +} +} +else +{ +uint8_t x_69; +x_69 = !lean_is_exclusive(x_55); +if (x_69 == 0) +{ +lean_object* x_70; +x_70 = l_Lake_mergeErrors___rarg(x_3, x_55, x_56); +return x_70; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_55, 0); +lean_inc(x_71); +lean_dec(x_55); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_71); +x_73 = l_Lake_mergeErrors___rarg(x_3, x_72, x_56); +return x_73; +} +} +} +case 6: +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; +x_74 = lean_ctor_get(x_1, 1); +lean_inc(x_74); +lean_dec(x_1); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_array_get_size(x_75); +x_77 = lean_unsigned_to_nat(0u); +x_78 = lean_nat_dec_lt(x_77, x_76); +if (x_78 == 0) +{ +lean_dec(x_76); +lean_dec(x_75); +lean_dec(x_2); +return x_3; +} +else +{ +uint8_t x_79; +x_79 = lean_nat_dec_le(x_76, x_76); +if (x_79 == 0) +{ +lean_dec(x_76); +lean_dec(x_75); +lean_dec(x_2); +return x_3; +} +else +{ +size_t x_80; size_t x_81; lean_object* x_82; +x_80 = 0; +x_81 = lean_usize_of_nat(x_76); +lean_dec(x_76); +x_82 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1(x_2, x_75, x_80, x_81, x_3); +lean_dec(x_75); +return x_82; +} +} +} +default: +{ +lean_object* x_83; uint8_t x_84; +lean_inc(x_1); +x_83 = l_Lake_LeanOptionValue_decodeToml(x_1); +x_84 = !lean_is_exclusive(x_1); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_1, 1); +lean_dec(x_85); +x_86 = lean_ctor_get(x_1, 0); +lean_dec(x_86); +x_87 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_87, 0, x_2); +if (lean_obj_tag(x_83) == 0) +{ +uint8_t x_88; +x_88 = !lean_is_exclusive(x_83); +if (x_88 == 0) +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_89 = lean_ctor_get(x_83, 0); +x_90 = lean_box(0); +lean_ctor_set_tag(x_1, 1); +lean_ctor_set(x_1, 1, x_90); +lean_ctor_set(x_1, 0, x_89); +x_91 = lean_array_mk(x_1); +lean_ctor_set(x_83, 0, x_91); +x_92 = l_Lake_mergeErrors___rarg(x_3, x_83, x_87); +return x_92; +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_83, 0); +lean_inc(x_93); +lean_dec(x_83); +x_94 = lean_box(0); +lean_ctor_set_tag(x_1, 1); +lean_ctor_set(x_1, 1, x_94); +lean_ctor_set(x_1, 0, x_93); +x_95 = lean_array_mk(x_1); +x_96 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_96, 0, x_95); +x_97 = l_Lake_mergeErrors___rarg(x_3, x_96, x_87); +return x_97; +} +} +else +{ +uint8_t x_98; +lean_free_object(x_1); +x_98 = !lean_is_exclusive(x_83); +if (x_98 == 0) +{ +lean_object* x_99; +x_99 = l_Lake_mergeErrors___rarg(x_3, x_83, x_87); +return x_99; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_83, 0); +lean_inc(x_100); +lean_dec(x_83); +x_101 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_101, 0, x_100); +x_102 = l_Lake_mergeErrors___rarg(x_3, x_101, x_87); +return x_102; +} +} +} +else +{ +lean_object* x_103; +lean_dec(x_1); +x_103 = lean_alloc_closure((void*)(l_Lake_decodeLeanOptionsAux___lambda__1), 3, 1); +lean_closure_set(x_103, 0, x_2); +if (lean_obj_tag(x_83) == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_104 = lean_ctor_get(x_83, 0); +lean_inc(x_104); +if (lean_is_exclusive(x_83)) { + lean_ctor_release(x_83, 0); + x_105 = x_83; +} else { + lean_dec_ref(x_83); + x_105 = lean_box(0); +} +x_106 = lean_box(0); +x_107 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_107, 0, x_104); +lean_ctor_set(x_107, 1, x_106); +x_108 = lean_array_mk(x_107); +if (lean_is_scalar(x_105)) { + x_109 = lean_alloc_ctor(0, 1, 0); +} else { + x_109 = x_105; +} +lean_ctor_set(x_109, 0, x_108); +x_110 = l_Lake_mergeErrors___rarg(x_3, x_109, x_103); +return x_110; +} +else +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_111 = lean_ctor_get(x_83, 0); +lean_inc(x_111); +if (lean_is_exclusive(x_83)) { + lean_ctor_release(x_83, 0); + x_112 = x_83; +} else { + lean_dec_ref(x_83); + x_112 = lean_box(0); +} +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(1, 1, 0); +} else { + x_113 = x_112; +} +lean_ctor_set(x_113, 0, x_111); +x_114 = l_Lake_mergeErrors___rarg(x_3, x_113, x_103); +return x_114; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_8 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptionsAux___spec__1(x_1, x_2, x_6, x_7, x_5); +lean_dec(x_2); +return x_8; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1() { +_start: { lean_object* x_1; x_1 = lean_alloc_closure((void*)(l_Array_push___boxed), 3, 1); @@ -4606,154 +4997,139 @@ return x_7; LEAN_EXPORT lean_object* l_Lake_StdVer_decodeToml(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -x_4 = lean_ctor_get(x_1, 1); -x_5 = l_Lake_StdVer_parse(x_4); -lean_dec(x_4); -if (lean_obj_tag(x_5) == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +x_11 = l_Lake_StdVer_parse(x_10); +lean_dec(x_10); +if (lean_obj_tag(x_11) == 0) { -uint8_t x_6; -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_box(0); -lean_ctor_set(x_1, 1, x_7); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_1); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_array_mk(x_9); -lean_ctor_set(x_5, 0, x_10); -return x_5; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_box(0); +lean_ctor_set(x_1, 1, x_13); +x_15 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_15, 0, x_1); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_array_mk(x_15); +lean_ctor_set(x_11, 0, x_16); +return x_11; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_5, 0); -lean_inc(x_11); -lean_dec(x_5); -x_12 = lean_box(0); -lean_ctor_set(x_1, 1, x_11); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_12); -x_14 = lean_array_mk(x_13); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_11, 0); +lean_inc(x_17); +lean_dec(x_11); +x_18 = lean_box(0); +lean_ctor_set(x_1, 1, x_17); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_array_mk(x_19); +x_21 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_21, 0, x_20); +return x_21; } } else { -uint8_t x_16; +uint8_t x_22; lean_free_object(x_1); -lean_dec(x_3); -x_16 = !lean_is_exclusive(x_5); -if (x_16 == 0) +lean_dec(x_9); +x_22 = !lean_is_exclusive(x_11); +if (x_22 == 0) { -return x_5; +return x_11; } else { -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_5, 0); -lean_inc(x_17); -lean_dec(x_5); -x_18 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_18, 0, x_17); -return x_18; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_11, 0); +lean_inc(x_23); +lean_dec(x_11); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_23); +return x_24; } } } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_1, 0); -x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -lean_inc(x_19); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +x_26 = lean_ctor_get(x_1, 1); +lean_inc(x_26); +lean_inc(x_25); lean_dec(x_1); -x_21 = l_Lake_StdVer_parse(x_20); -lean_dec(x_20); -if (lean_obj_tag(x_21) == 0) +x_27 = l_Lake_StdVer_parse(x_26); +lean_dec(x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - x_23 = x_21; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +if (lean_is_exclusive(x_27)) { + lean_ctor_release(x_27, 0); + x_29 = x_27; } else { - lean_dec_ref(x_21); - x_23 = lean_box(0); + lean_dec_ref(x_27); + x_29 = lean_box(0); } -x_24 = lean_box(0); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_19); -lean_ctor_set(x_25, 1, x_22); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -x_27 = lean_array_mk(x_26); -if (lean_is_scalar(x_23)) { - x_28 = lean_alloc_ctor(0, 1, 0); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_25); +lean_ctor_set(x_31, 1, x_28); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +x_33 = lean_array_mk(x_32); +if (lean_is_scalar(x_29)) { + x_34 = lean_alloc_ctor(0, 1, 0); } else { - x_28 = x_23; + x_34 = x_29; } -lean_ctor_set(x_28, 0, x_27); -return x_28; +lean_ctor_set(x_34, 0, x_33); +return x_34; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_dec(x_19); -x_29 = lean_ctor_get(x_21, 0); -lean_inc(x_29); -if (lean_is_exclusive(x_21)) { - lean_ctor_release(x_21, 0); - x_30 = x_21; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_25); +x_35 = lean_ctor_get(x_27, 0); +lean_inc(x_35); +if (lean_is_exclusive(x_27)) { + lean_ctor_release(x_27, 0); + x_36 = x_27; } else { - lean_dec_ref(x_21); - x_30 = lean_box(0); + lean_dec_ref(x_27); + x_36 = lean_box(0); } -if (lean_is_scalar(x_30)) { - x_31 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 1, 0); } else { - x_31 = x_30; + x_37 = x_36; } -lean_ctor_set(x_31, 0, x_29); -return x_31; +lean_ctor_set(x_37, 0, x_35); +return x_37; } } } case 2: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_32 = lean_ctor_get(x_1, 0); -lean_inc(x_32); -lean_dec(x_1); -x_33 = l_Lake_Glob_decodeToml___closed__2; -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_mk_array(x_35, x_34); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -return x_37; -} -case 3: -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_38; lean_object* x_39; lean_object* x_40; x_38 = lean_ctor_get(x_1, 0); lean_inc(x_38); lean_dec(x_1); @@ -4761,11 +5137,21 @@ x_39 = l_Lake_Glob_decodeToml___closed__2; x_40 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_40, 0, x_38); lean_ctor_set(x_40, 1, x_39); -x_41 = lean_unsigned_to_nat(1u); -x_42 = lean_mk_array(x_41, x_40); -x_43 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_43, 0, x_42); -return x_43; +x_2 = x_40; +goto block_7; +} +case 3: +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_1, 0); +lean_inc(x_41); +lean_dec(x_1); +x_42 = l_Lake_Glob_decodeToml___closed__2; +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_2 = x_43; +goto block_7; } default: { @@ -4773,36 +5159,42 @@ uint8_t x_44; x_44 = !lean_is_exclusive(x_1); if (x_44 == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_object* x_45; lean_object* x_46; x_45 = lean_ctor_get(x_1, 1); lean_dec(x_45); x_46 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_1, 0); lean_ctor_set(x_1, 1, x_46); -x_47 = lean_unsigned_to_nat(1u); -x_48 = lean_mk_array(x_47, x_1); -x_49 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_49, 0, x_48); -return x_49; +x_2 = x_1; +goto block_7; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_50 = lean_ctor_get(x_1, 0); -lean_inc(x_50); +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_1, 0); +lean_inc(x_47); lean_dec(x_1); -x_51 = l_Lake_Glob_decodeToml___closed__2; -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -x_53 = lean_unsigned_to_nat(1u); -x_54 = lean_mk_array(x_53, x_52); -x_55 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_55, 0, x_54); -return x_55; +x_48 = l_Lake_Glob_decodeToml___closed__2; +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_2 = x_49; +goto block_7; } } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } LEAN_EXPORT lean_object* l_Lake_instDecodeTomlStdVer(lean_object* x_1) { @@ -4820,38 +5212,18 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -x_11 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_12 = l_Lake_mergeErrors___rarg(x_4, x_10, x_11); -x_2 = x_8; -x_4 = x_12; -goto _start; -} -case 2: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_14 = lean_ctor_get(x_6, 0); -lean_inc(x_14); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); lean_dec(x_6); -x_15 = l_Lake_Glob_decodeToml___closed__2; -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); +x_19 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_19, 0, x_18); x_20 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; x_21 = l_Lake_mergeErrors___rarg(x_4, x_19, x_20); @@ -4859,9 +5231,9 @@ x_2 = x_8; x_4 = x_21; goto _start; } -case 3: +case 2: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_object* x_23; lean_object* x_24; lean_object* x_25; x_23 = lean_ctor_get(x_6, 0); lean_inc(x_23); lean_dec(x_6); @@ -4869,60 +5241,68 @@ x_24 = l_Lake_Glob_decodeToml___closed__2; x_25 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_25); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_30 = l_Lake_mergeErrors___rarg(x_4, x_28, x_29); -x_2 = x_8; -x_4 = x_30; -goto _start; +x_9 = x_25; +goto block_17; +} +case 3: +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_6, 0); +lean_inc(x_26); +lean_dec(x_6); +x_27 = l_Lake_Glob_decodeToml___closed__2; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_9 = x_28; +goto block_17; } default: { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_6); -if (x_32 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_6); +if (x_29 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_33 = lean_ctor_get(x_6, 1); -lean_dec(x_33); -x_34 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_6, 1); +lean_dec(x_30); +x_31 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_34); -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_mk_array(x_35, x_6); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -x_38 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_39 = l_Lake_mergeErrors___rarg(x_4, x_37, x_38); -x_2 = x_8; -x_4 = x_39; -goto _start; +lean_ctor_set(x_6, 1, x_31); +x_9 = x_6; +goto block_17; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_41 = lean_ctor_get(x_6, 0); -lean_inc(x_41); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_6, 0); +lean_inc(x_32); lean_dec(x_6); -x_42 = l_Lake_Glob_decodeToml___closed__2; -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_unsigned_to_nat(1u); -x_45 = lean_mk_array(x_44, x_43); -x_46 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_47 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_48 = l_Lake_mergeErrors___rarg(x_4, x_46, x_47); -x_2 = x_8; -x_4 = x_48; -goto _start; +x_33 = l_Lake_Glob_decodeToml___closed__2; +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_9 = x_34; +goto block_17; } } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; +} } else { @@ -5038,87 +5418,84 @@ lean_object* x_3; switch (lean_obj_tag(x_2)) { case 0: { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); lean_dec(x_2); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +return x_13; } case 2: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_12 = l_Lake_Glob_decodeToml___closed__2; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_13); -x_3 = x_15; -goto block_8; +x_15 = l_Lake_Glob_decodeToml___closed__2; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_3 = x_16; +goto block_11; } case 3: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_2, 0); -lean_inc(x_16); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_2, 0); +lean_inc(x_17); lean_dec(x_2); -x_17 = l_Lake_Glob_decodeToml___closed__2; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_18); -x_3 = x_20; -goto block_8; +x_18 = l_Lake_Glob_decodeToml___closed__2; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_3 = x_19; +goto block_11; } default: { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_2); -if (x_21 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_2); +if (x_20 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_2, 1); -lean_dec(x_22); -x_23 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_2, 1); +lean_dec(x_21); +x_22 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_23); -x_24 = lean_unsigned_to_nat(1u); -x_25 = lean_mk_array(x_24, x_2); -x_3 = x_25; -goto block_8; +lean_ctor_set(x_2, 1, x_22); +x_3 = x_2; +goto block_11; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_26 = lean_ctor_get(x_2, 0); -lean_inc(x_26); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_2, 0); +lean_inc(x_23); lean_dec(x_2); -x_27 = l_Lake_Glob_decodeToml___closed__2; -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_mk_array(x_29, x_28); -x_3 = x_30; -goto block_8; +x_24 = l_Lake_Glob_decodeToml___closed__2; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_3 = x_25; +goto block_11; } } } -block_8: +block_11: { -size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_array_size(x_3); -x_5 = 0; -x_6 = l_Array_mapMUnsafe_map___at_Lake_StrPat_decodeToml___spec__5(x_1, x_4, x_5, x_3); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +x_7 = lean_array_size(x_6); +x_8 = 0; +x_9 = l_Array_mapMUnsafe_map___at_Lake_StrPat_decodeToml___spec__5(x_1, x_7, x_8, x_6); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; } } } @@ -6302,152 +6679,257 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_WorkspaceConfig_decodeToml(lean_object* x_1) { +static lean_object* _init_l_Lake_WorkspaceConfig_decodeToml___closed__3() { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_8; lean_object* x_9; lean_object* x_10; -x_8 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_9 = l_Lake_WorkspaceConfig_decodeToml___closed__2; -x_10 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_8, x_9, x_1); -if (lean_obj_tag(x_10) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Lake_defaultPackagesDir; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lake_WorkspaceConfig_decodeToml___closed__4() { +_start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lake_defaultPackagesDir; -x_12 = l_Lake_LeanOption_decodeToml___closed__3; -x_2 = x_11; -x_3 = x_12; -goto block_7; +uint8_t x_1; +x_1 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_1 == 0) +{ +lean_object* x_2; +x_2 = l_Lake_LeanOption_decodeToml___closed__6; +return x_2; } else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_10, 0); -lean_inc(x_13); -lean_dec(x_10); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -switch (lean_obj_tag(x_14)) { -case 0: -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = l_Lake_LeanOption_decodeToml___closed__3; -x_2 = x_15; -x_3 = x_16; -goto block_7; +lean_object* x_3; +x_3 = l_Lake_WorkspaceConfig_decodeToml___closed__3; +return x_3; } -case 2: +} +} +LEAN_EXPORT lean_object* l_Lake_WorkspaceConfig_decodeToml(lean_object* x_1) { +_start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_17 = lean_ctor_get(x_14, 0); -lean_inc(x_17); -lean_dec(x_14); -x_18 = l_Lake_Glob_decodeToml___closed__2; -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_unsigned_to_nat(1u); -x_21 = lean_mk_array(x_20, x_19); -x_22 = l_Lake_LeanOption_decodeToml___closed__3; -x_23 = l_Array_append___rarg(x_22, x_21); -lean_dec(x_21); -x_24 = l_Lake_defaultPackagesDir; +lean_object* x_2; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_13 = l_Lake_WorkspaceConfig_decodeToml___closed__2; +x_14 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_12, x_13, x_1); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; +x_15 = l_Lake_WorkspaceConfig_decodeToml___closed__4; +return x_15; +} +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_14); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_14, 0); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +switch (lean_obj_tag(x_18)) { +case 0: +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_20 == 0) +{ +lean_object* x_21; +lean_dec(x_19); +lean_free_object(x_14); +x_21 = l_Lake_LeanOption_decodeToml___closed__6; +return x_21; +} +else +{ +lean_ctor_set(x_14, 0, x_19); +return x_14; +} +} +case 2: +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_free_object(x_14); +x_22 = lean_ctor_get(x_18, 0); +lean_inc(x_22); +lean_dec(x_18); +x_23 = l_Lake_Glob_decodeToml___closed__2; +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); x_2 = x_24; -x_3 = x_23; -goto block_7; +goto block_11; } case 3: { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_25 = lean_ctor_get(x_14, 0); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_free_object(x_14); +x_25 = lean_ctor_get(x_18, 0); lean_inc(x_25); -lean_dec(x_14); +lean_dec(x_18); x_26 = l_Lake_Glob_decodeToml___closed__2; x_27 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_27, 0, x_25); lean_ctor_set(x_27, 1, x_26); -x_28 = lean_unsigned_to_nat(1u); -x_29 = lean_mk_array(x_28, x_27); -x_30 = l_Lake_LeanOption_decodeToml___closed__3; -x_31 = l_Array_append___rarg(x_30, x_29); -lean_dec(x_29); -x_32 = l_Lake_defaultPackagesDir; -x_2 = x_32; -x_3 = x_31; -goto block_7; +x_2 = x_27; +goto block_11; } default: { -uint8_t x_33; -x_33 = !lean_is_exclusive(x_14); -if (x_33 == 0) +uint8_t x_28; +lean_free_object(x_14); +x_28 = !lean_is_exclusive(x_18); +if (x_28 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_34 = lean_ctor_get(x_14, 1); -lean_dec(x_34); -x_35 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_14, 0); -lean_ctor_set(x_14, 1, x_35); -x_36 = lean_unsigned_to_nat(1u); -x_37 = lean_mk_array(x_36, x_14); -x_38 = l_Lake_LeanOption_decodeToml___closed__3; -x_39 = l_Array_append___rarg(x_38, x_37); -lean_dec(x_37); -x_40 = l_Lake_defaultPackagesDir; -x_2 = x_40; -x_3 = x_39; -goto block_7; +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_18, 1); +lean_dec(x_29); +x_30 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_18, 0); +lean_ctor_set(x_18, 1, x_30); +x_2 = x_18; +goto block_11; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_41 = lean_ctor_get(x_14, 0); -lean_inc(x_41); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_18, 0); +lean_inc(x_31); +lean_dec(x_18); +x_32 = l_Lake_Glob_decodeToml___closed__2; +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +x_2 = x_33; +goto block_11; +} +} +} +} +else +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_14, 0); +lean_inc(x_34); lean_dec(x_14); -x_42 = l_Lake_Glob_decodeToml___closed__2; -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_unsigned_to_nat(1u); -x_45 = lean_mk_array(x_44, x_43); -x_46 = l_Lake_LeanOption_decodeToml___closed__3; -x_47 = l_Array_append___rarg(x_46, x_45); -lean_dec(x_45); -x_48 = l_Lake_defaultPackagesDir; -x_2 = x_48; -x_3 = x_47; -goto block_7; +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +lean_dec(x_34); +switch (lean_obj_tag(x_35)) { +case 0: +{ +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_37 = l_Lake_LeanOption_decodeToml___closed__5; +if (x_37 == 0) +{ +lean_object* x_38; +lean_dec(x_36); +x_38 = l_Lake_LeanOption_decodeToml___closed__6; +return x_38; } +else +{ +lean_object* x_39; +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_36); +return x_39; } } +case 2: +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_35, 0); +lean_inc(x_40); +lean_dec(x_35); +x_41 = l_Lake_Glob_decodeToml___closed__2; +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_2 = x_42; +goto block_11; } -block_7: +case 3: { -uint8_t x_4; -x_4 = l_Array_isEmpty___rarg(x_3); -if (x_4 == 0) +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_35, 0); +lean_inc(x_43); +lean_dec(x_35); +x_44 = l_Lake_Glob_decodeToml___closed__2; +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +x_2 = x_45; +goto block_11; +} +default: { -lean_object* x_5; -lean_dec(x_2); -x_5 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_5, 0, x_3); -return x_5; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_35, 0); +lean_inc(x_46); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_47 = x_35; +} else { + lean_dec_ref(x_35); + x_47 = lean_box(0); +} +x_48 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_47)) { + x_49 = lean_alloc_ctor(0, 2, 0); +} else { + x_49 = x_47; + lean_ctor_set_tag(x_49, 0); +} +lean_ctor_set(x_49, 0, x_46); +lean_ctor_set(x_49, 1, x_48); +x_2 = x_49; +goto block_11; +} +} +} +} +block_11: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = l_Lake_LeanOption_decodeToml___closed__3; +x_7 = l_Array_append___rarg(x_6, x_5); +lean_dec(x_5); +x_8 = l_Array_isEmpty___rarg(x_7); +if (x_8 == 0) +{ +lean_object* x_9; +x_9 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_9, 0, x_7); +return x_9; } else { -lean_object* x_6; -lean_dec(x_3); -x_6 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_6, 0, x_2); -return x_6; +lean_object* x_10; +lean_dec(x_7); +x_10 = l_Lake_WorkspaceConfig_decodeToml___closed__3; +return x_10; } } } } -static lean_object* _init_l_Lake_instDecodeTomlWorkspaceConfig___closed__1() { +static lean_object* _init_l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -6455,121 +6937,132 @@ x_1 = lean_mk_string_unchecked("expected table", 14, 14); return x_1; } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlWorkspaceConfig(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlWorkspaceConfig___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_1, 1); -lean_inc(x_26); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); lean_dec(x_1); -x_27 = l_Lake_WorkspaceConfig_decodeToml(x_26); -return x_27; +x_21 = l_Lake_WorkspaceConfig_decodeToml(x_20); +return x_21; } default: { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_1); -if (x_28 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_1, 1); -lean_dec(x_29); -x_30 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_mk_array(x_31, x_1); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +lean_ctor_set(x_1, 1, x_24); +x_2 = x_1; +goto block_7; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); lean_dec(x_1); -x_35 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_39, 0, x_38); -return x_39; +x_26 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_2 = x_27; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } } +static lean_object* _init_l_Lake_instDecodeTomlWorkspaceConfig___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlWorkspaceConfig___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_instDecodeTomlWorkspaceConfig() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +return x_1; } } static lean_object* _init_l_Lake_LeanConfig_decodeToml___closed__1() { @@ -6789,58 +7282,61 @@ return x_3; LEAN_EXPORT lean_object* l_Lake_LeanConfig_decodeToml(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; uint8_t x_8; lean_object* x_9; lean_object* x_471; lean_object* x_472; lean_object* x_473; -x_471 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_472 = l_Lake_LeanConfig_decodeToml___closed__24; +lean_object* x_2; lean_object* x_3; uint8_t x_8; lean_object* x_9; lean_object* x_342; lean_object* x_343; lean_object* x_344; +x_342 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_343 = l_Lake_LeanConfig_decodeToml___closed__24; lean_inc(x_1); -x_473 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_471, x_472, x_1); -if (lean_obj_tag(x_473) == 0) -{ -uint8_t x_474; lean_object* x_475; -x_474 = 3; -x_475 = l_Lake_LeanOption_decodeToml___closed__3; -x_8 = x_474; -x_9 = x_475; -goto block_470; +x_344 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_342, x_343, x_1); +if (lean_obj_tag(x_344) == 0) +{ +uint8_t x_345; lean_object* x_346; +x_345 = 3; +x_346 = l_Lake_LeanOption_decodeToml___closed__3; +x_8 = x_345; +x_9 = x_346; +goto block_341; } else { -lean_object* x_476; lean_object* x_477; lean_object* x_478; -x_476 = lean_ctor_get(x_473, 0); -lean_inc(x_476); -lean_dec(x_473); -x_477 = lean_ctor_get(x_476, 1); -lean_inc(x_477); -lean_dec(x_476); -x_478 = l_Lake_BuildType_decodeToml(x_477); -if (lean_obj_tag(x_478) == 0) -{ -lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; uint8_t x_484; -x_479 = lean_ctor_get(x_478, 0); -lean_inc(x_479); -lean_dec(x_478); -x_480 = lean_unsigned_to_nat(1u); -x_481 = lean_mk_array(x_480, x_479); -x_482 = l_Lake_LeanOption_decodeToml___closed__3; -x_483 = l_Array_append___rarg(x_482, x_481); -lean_dec(x_481); -x_484 = 3; -x_8 = x_484; -x_9 = x_483; -goto block_470; +lean_object* x_347; lean_object* x_348; lean_object* x_349; +x_347 = lean_ctor_get(x_344, 0); +lean_inc(x_347); +lean_dec(x_344); +x_348 = lean_ctor_get(x_347, 1); +lean_inc(x_348); +lean_dec(x_347); +x_349 = l_Lake_BuildType_decodeToml(x_348); +if (lean_obj_tag(x_349) == 0) +{ +lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; uint8_t x_356; +x_350 = lean_ctor_get(x_349, 0); +lean_inc(x_350); +lean_dec(x_349); +x_351 = lean_box(0); +x_352 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_352, 0, x_350); +lean_ctor_set(x_352, 1, x_351); +x_353 = lean_array_mk(x_352); +x_354 = l_Lake_LeanOption_decodeToml___closed__3; +x_355 = l_Array_append___rarg(x_354, x_353); +lean_dec(x_353); +x_356 = 3; +x_8 = x_356; +x_9 = x_355; +goto block_341; } else { -lean_object* x_485; lean_object* x_486; uint8_t x_487; -x_485 = lean_ctor_get(x_478, 0); -lean_inc(x_485); -lean_dec(x_478); -x_486 = l_Lake_LeanOption_decodeToml___closed__3; -x_487 = lean_unbox(x_485); -lean_dec(x_485); -x_8 = x_487; -x_9 = x_486; -goto block_470; +lean_object* x_357; lean_object* x_358; uint8_t x_359; +x_357 = lean_ctor_get(x_349, 0); +lean_inc(x_357); +lean_dec(x_349); +x_358 = l_Lake_LeanOption_decodeToml___closed__3; +x_359 = lean_unbox(x_357); +lean_dec(x_357); +x_8 = x_359; +x_9 = x_358; +goto block_341; } } block_7: @@ -6864,1698 +7360,1495 @@ lean_ctor_set(x_6, 0, x_2); return x_6; } } -block_470: +block_341: { -uint8_t x_10; lean_object* x_11; lean_object* x_456; lean_object* x_457; lean_object* x_458; -x_456 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_457 = l_Lake_LeanConfig_decodeToml___closed__22; +uint8_t x_10; lean_object* x_11; lean_object* x_326; lean_object* x_327; lean_object* x_328; +x_326 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_327 = l_Lake_LeanConfig_decodeToml___closed__22; lean_inc(x_1); -x_458 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_456, x_457, x_1); -if (lean_obj_tag(x_458) == 0) +x_328 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_326, x_327, x_1); +if (lean_obj_tag(x_328) == 0) { -uint8_t x_459; -x_459 = 2; -x_10 = x_459; +uint8_t x_329; +x_329 = 2; +x_10 = x_329; x_11 = x_9; -goto block_455; +goto block_325; } else { -lean_object* x_460; lean_object* x_461; lean_object* x_462; -x_460 = lean_ctor_get(x_458, 0); -lean_inc(x_460); -lean_dec(x_458); -x_461 = lean_ctor_get(x_460, 1); -lean_inc(x_461); -lean_dec(x_460); -x_462 = l_Lake_Backend_decodeToml(x_461); -if (lean_obj_tag(x_462) == 0) -{ -lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; uint8_t x_467; -x_463 = lean_ctor_get(x_462, 0); -lean_inc(x_463); -lean_dec(x_462); -x_464 = lean_unsigned_to_nat(1u); -x_465 = lean_mk_array(x_464, x_463); -x_466 = l_Array_append___rarg(x_9, x_465); -lean_dec(x_465); -x_467 = 2; -x_10 = x_467; -x_11 = x_466; -goto block_455; +lean_object* x_330; lean_object* x_331; lean_object* x_332; +x_330 = lean_ctor_get(x_328, 0); +lean_inc(x_330); +lean_dec(x_328); +x_331 = lean_ctor_get(x_330, 1); +lean_inc(x_331); +lean_dec(x_330); +x_332 = l_Lake_Backend_decodeToml(x_331); +if (lean_obj_tag(x_332) == 0) +{ +lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; uint8_t x_338; +x_333 = lean_ctor_get(x_332, 0); +lean_inc(x_333); +lean_dec(x_332); +x_334 = lean_box(0); +x_335 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_335, 0, x_333); +lean_ctor_set(x_335, 1, x_334); +x_336 = lean_array_mk(x_335); +x_337 = l_Array_append___rarg(x_9, x_336); +lean_dec(x_336); +x_338 = 2; +x_10 = x_338; +x_11 = x_337; +goto block_325; } else { -lean_object* x_468; uint8_t x_469; -x_468 = lean_ctor_get(x_462, 0); -lean_inc(x_468); -lean_dec(x_462); -x_469 = lean_unbox(x_468); -lean_dec(x_468); -x_10 = x_469; +lean_object* x_339; uint8_t x_340; +x_339 = lean_ctor_get(x_332, 0); +lean_inc(x_339); +lean_dec(x_332); +x_340 = lean_unbox(x_339); +lean_dec(x_339); +x_10 = x_340; x_11 = x_9; -goto block_455; +goto block_325; } } -block_455: +block_325: { -lean_object* x_12; lean_object* x_13; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; -x_391 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_392 = l_Lake_LeanConfig_decodeToml___closed__19; +lean_object* x_12; lean_object* x_13; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; +x_279 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_280 = l_Lake_LeanConfig_decodeToml___closed__19; lean_inc(x_1); -x_393 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_391, x_392, x_1); -x_394 = lean_box(0); -if (lean_obj_tag(x_393) == 0) +x_281 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_279, x_280, x_1); +x_282 = lean_box(0); +if (lean_obj_tag(x_281) == 0) { -x_12 = x_394; +x_12 = x_282; x_13 = x_11; -goto block_390; +goto block_278; } else { -uint8_t x_395; -x_395 = !lean_is_exclusive(x_393); -if (x_395 == 0) +uint8_t x_289; +x_289 = !lean_is_exclusive(x_281); +if (x_289 == 0) { -lean_object* x_396; lean_object* x_397; -x_396 = lean_ctor_get(x_393, 0); -x_397 = lean_ctor_get(x_396, 1); -lean_inc(x_397); -lean_dec(x_396); -switch (lean_obj_tag(x_397)) { +lean_object* x_290; lean_object* x_291; +x_290 = lean_ctor_get(x_281, 0); +x_291 = lean_ctor_get(x_290, 1); +lean_inc(x_291); +lean_dec(x_290); +switch (lean_obj_tag(x_291)) { case 0: { -uint8_t x_398; -lean_free_object(x_393); -x_398 = !lean_is_exclusive(x_397); -if (x_398 == 0) -{ -lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; -x_399 = lean_ctor_get(x_397, 1); -lean_dec(x_399); -x_400 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_397, 1, x_400); -x_401 = lean_unsigned_to_nat(1u); -x_402 = lean_mk_array(x_401, x_397); -x_403 = l_Array_append___rarg(x_11, x_402); -lean_dec(x_402); -x_12 = x_394; -x_13 = x_403; -goto block_390; +uint8_t x_292; +lean_free_object(x_281); +x_292 = !lean_is_exclusive(x_291); +if (x_292 == 0) +{ +lean_object* x_293; lean_object* x_294; +x_293 = lean_ctor_get(x_291, 1); +lean_dec(x_293); +x_294 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_291, 1, x_294); +x_283 = x_291; +goto block_288; } else { -lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; -x_404 = lean_ctor_get(x_397, 0); -lean_inc(x_404); -lean_dec(x_397); -x_405 = l_Lake_LeanConfig_decodeToml___closed__20; -x_406 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_406, 0, x_404); -lean_ctor_set(x_406, 1, x_405); -x_407 = lean_unsigned_to_nat(1u); -x_408 = lean_mk_array(x_407, x_406); -x_409 = l_Array_append___rarg(x_11, x_408); -lean_dec(x_408); -x_12 = x_394; -x_13 = x_409; -goto block_390; +lean_object* x_295; lean_object* x_296; lean_object* x_297; +x_295 = lean_ctor_get(x_291, 0); +lean_inc(x_295); +lean_dec(x_291); +x_296 = l_Lake_LeanConfig_decodeToml___closed__20; +x_297 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_297, 0, x_295); +lean_ctor_set(x_297, 1, x_296); +x_283 = x_297; +goto block_288; } } case 2: { -lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; -lean_free_object(x_393); -x_410 = lean_ctor_get(x_397, 0); -lean_inc(x_410); -lean_dec(x_397); -x_411 = l_Lake_LeanConfig_decodeToml___closed__20; -x_412 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_412, 0, x_410); -lean_ctor_set(x_412, 1, x_411); -x_413 = lean_unsigned_to_nat(1u); -x_414 = lean_mk_array(x_413, x_412); -x_415 = l_Array_append___rarg(x_11, x_414); -lean_dec(x_414); -x_12 = x_394; -x_13 = x_415; -goto block_390; +lean_object* x_298; lean_object* x_299; lean_object* x_300; +lean_free_object(x_281); +x_298 = lean_ctor_get(x_291, 0); +lean_inc(x_298); +lean_dec(x_291); +x_299 = l_Lake_LeanConfig_decodeToml___closed__20; +x_300 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_300, 0, x_298); +lean_ctor_set(x_300, 1, x_299); +x_283 = x_300; +goto block_288; } case 3: { -uint8_t x_416; lean_object* x_417; -x_416 = lean_ctor_get_uint8(x_397, sizeof(void*)*1); -lean_dec(x_397); -x_417 = lean_box(x_416); -lean_ctor_set(x_393, 0, x_417); -x_12 = x_393; +uint8_t x_301; lean_object* x_302; +x_301 = lean_ctor_get_uint8(x_291, sizeof(void*)*1); +lean_dec(x_291); +x_302 = lean_box(x_301); +lean_ctor_set(x_281, 0, x_302); +x_12 = x_281; x_13 = x_11; -goto block_390; +goto block_278; } default: { -uint8_t x_418; -lean_free_object(x_393); -x_418 = !lean_is_exclusive(x_397); -if (x_418 == 0) -{ -lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; -x_419 = lean_ctor_get(x_397, 1); -lean_dec(x_419); -x_420 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_397, 0); -lean_ctor_set(x_397, 1, x_420); -x_421 = lean_unsigned_to_nat(1u); -x_422 = lean_mk_array(x_421, x_397); -x_423 = l_Array_append___rarg(x_11, x_422); -lean_dec(x_422); -x_12 = x_394; -x_13 = x_423; -goto block_390; +uint8_t x_303; +lean_free_object(x_281); +x_303 = !lean_is_exclusive(x_291); +if (x_303 == 0) +{ +lean_object* x_304; lean_object* x_305; +x_304 = lean_ctor_get(x_291, 1); +lean_dec(x_304); +x_305 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_291, 0); +lean_ctor_set(x_291, 1, x_305); +x_283 = x_291; +goto block_288; } else { -lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; -x_424 = lean_ctor_get(x_397, 0); -lean_inc(x_424); -lean_dec(x_397); -x_425 = l_Lake_LeanConfig_decodeToml___closed__20; -x_426 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_426, 0, x_424); -lean_ctor_set(x_426, 1, x_425); -x_427 = lean_unsigned_to_nat(1u); -x_428 = lean_mk_array(x_427, x_426); -x_429 = l_Array_append___rarg(x_11, x_428); -lean_dec(x_428); -x_12 = x_394; -x_13 = x_429; -goto block_390; +lean_object* x_306; lean_object* x_307; lean_object* x_308; +x_306 = lean_ctor_get(x_291, 0); +lean_inc(x_306); +lean_dec(x_291); +x_307 = l_Lake_LeanConfig_decodeToml___closed__20; +x_308 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_308, 0, x_306); +lean_ctor_set(x_308, 1, x_307); +x_283 = x_308; +goto block_288; } } } } else { -lean_object* x_430; lean_object* x_431; -x_430 = lean_ctor_get(x_393, 0); -lean_inc(x_430); -lean_dec(x_393); -x_431 = lean_ctor_get(x_430, 1); -lean_inc(x_431); -lean_dec(x_430); -switch (lean_obj_tag(x_431)) { +lean_object* x_309; lean_object* x_310; +x_309 = lean_ctor_get(x_281, 0); +lean_inc(x_309); +lean_dec(x_281); +x_310 = lean_ctor_get(x_309, 1); +lean_inc(x_310); +lean_dec(x_309); +switch (lean_obj_tag(x_310)) { case 0: { -lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; -x_432 = lean_ctor_get(x_431, 0); -lean_inc(x_432); -if (lean_is_exclusive(x_431)) { - lean_ctor_release(x_431, 0); - lean_ctor_release(x_431, 1); - x_433 = x_431; +lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_311 = lean_ctor_get(x_310, 0); +lean_inc(x_311); +if (lean_is_exclusive(x_310)) { + lean_ctor_release(x_310, 0); + lean_ctor_release(x_310, 1); + x_312 = x_310; } else { - lean_dec_ref(x_431); - x_433 = lean_box(0); + lean_dec_ref(x_310); + x_312 = lean_box(0); } -x_434 = l_Lake_LeanConfig_decodeToml___closed__20; -if (lean_is_scalar(x_433)) { - x_435 = lean_alloc_ctor(0, 2, 0); +x_313 = l_Lake_LeanConfig_decodeToml___closed__20; +if (lean_is_scalar(x_312)) { + x_314 = lean_alloc_ctor(0, 2, 0); } else { - x_435 = x_433; + x_314 = x_312; } -lean_ctor_set(x_435, 0, x_432); -lean_ctor_set(x_435, 1, x_434); -x_436 = lean_unsigned_to_nat(1u); -x_437 = lean_mk_array(x_436, x_435); -x_438 = l_Array_append___rarg(x_11, x_437); -lean_dec(x_437); -x_12 = x_394; -x_13 = x_438; -goto block_390; +lean_ctor_set(x_314, 0, x_311); +lean_ctor_set(x_314, 1, x_313); +x_283 = x_314; +goto block_288; } case 2: { -lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; -x_439 = lean_ctor_get(x_431, 0); -lean_inc(x_439); -lean_dec(x_431); -x_440 = l_Lake_LeanConfig_decodeToml___closed__20; -x_441 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_441, 0, x_439); -lean_ctor_set(x_441, 1, x_440); -x_442 = lean_unsigned_to_nat(1u); -x_443 = lean_mk_array(x_442, x_441); -x_444 = l_Array_append___rarg(x_11, x_443); -lean_dec(x_443); -x_12 = x_394; -x_13 = x_444; -goto block_390; +lean_object* x_315; lean_object* x_316; lean_object* x_317; +x_315 = lean_ctor_get(x_310, 0); +lean_inc(x_315); +lean_dec(x_310); +x_316 = l_Lake_LeanConfig_decodeToml___closed__20; +x_317 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_317, 0, x_315); +lean_ctor_set(x_317, 1, x_316); +x_283 = x_317; +goto block_288; } case 3: { -uint8_t x_445; lean_object* x_446; lean_object* x_447; -x_445 = lean_ctor_get_uint8(x_431, sizeof(void*)*1); -lean_dec(x_431); -x_446 = lean_box(x_445); -x_447 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_447, 0, x_446); -x_12 = x_447; +uint8_t x_318; lean_object* x_319; lean_object* x_320; +x_318 = lean_ctor_get_uint8(x_310, sizeof(void*)*1); +lean_dec(x_310); +x_319 = lean_box(x_318); +x_320 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_320, 0, x_319); +x_12 = x_320; x_13 = x_11; -goto block_390; +goto block_278; } default: { -lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; -x_448 = lean_ctor_get(x_431, 0); -lean_inc(x_448); -if (lean_is_exclusive(x_431)) { - lean_ctor_release(x_431, 0); - lean_ctor_release(x_431, 1); - x_449 = x_431; +lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; +x_321 = lean_ctor_get(x_310, 0); +lean_inc(x_321); +if (lean_is_exclusive(x_310)) { + lean_ctor_release(x_310, 0); + lean_ctor_release(x_310, 1); + x_322 = x_310; } else { - lean_dec_ref(x_431); - x_449 = lean_box(0); + lean_dec_ref(x_310); + x_322 = lean_box(0); } -x_450 = l_Lake_LeanConfig_decodeToml___closed__20; -if (lean_is_scalar(x_449)) { - x_451 = lean_alloc_ctor(0, 2, 0); +x_323 = l_Lake_LeanConfig_decodeToml___closed__20; +if (lean_is_scalar(x_322)) { + x_324 = lean_alloc_ctor(0, 2, 0); } else { - x_451 = x_449; - lean_ctor_set_tag(x_451, 0); -} -lean_ctor_set(x_451, 0, x_448); -lean_ctor_set(x_451, 1, x_450); -x_452 = lean_unsigned_to_nat(1u); -x_453 = lean_mk_array(x_452, x_451); -x_454 = l_Array_append___rarg(x_11, x_453); -lean_dec(x_453); -x_12 = x_394; -x_13 = x_454; -goto block_390; + x_324 = x_322; + lean_ctor_set_tag(x_324, 0); } +lean_ctor_set(x_324, 0, x_321); +lean_ctor_set(x_324, 1, x_323); +x_283 = x_324; +goto block_288; } } } -block_390: +} +block_278: { -lean_object* x_14; lean_object* x_15; lean_object* x_379; lean_object* x_380; lean_object* x_381; -x_379 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_380 = l_Lake_LeanConfig_decodeToml___closed__17; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_267; lean_object* x_268; lean_object* x_269; +x_14 = lean_box(0); +x_267 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_268 = l_Lake_LeanConfig_decodeToml___closed__17; lean_inc(x_1); -x_381 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_379, x_380, x_1); -if (lean_obj_tag(x_381) == 0) +x_269 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_267, x_268, x_1); +if (lean_obj_tag(x_269) == 0) { -lean_object* x_382; -x_382 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_382; -x_15 = x_13; -goto block_378; +lean_object* x_270; +x_270 = l_Lake_decodeLeanOptions___closed__1; +x_15 = x_270; +x_16 = x_13; +goto block_266; } else { -lean_object* x_383; lean_object* x_384; lean_object* x_385; -x_383 = lean_ctor_get(x_381, 0); -lean_inc(x_383); -lean_dec(x_381); -x_384 = lean_ctor_get(x_383, 1); -lean_inc(x_384); -lean_dec(x_383); -x_385 = l_Lake_decodeLeanOptions(x_384); -if (lean_obj_tag(x_385) == 0) +lean_object* x_271; lean_object* x_272; lean_object* x_273; +x_271 = lean_ctor_get(x_269, 0); +lean_inc(x_271); +lean_dec(x_269); +x_272 = lean_ctor_get(x_271, 1); +lean_inc(x_272); +lean_dec(x_271); +x_273 = l_Lake_decodeLeanOptions(x_272); +if (lean_obj_tag(x_273) == 0) { -lean_object* x_386; lean_object* x_387; lean_object* x_388; -x_386 = lean_ctor_get(x_385, 0); -lean_inc(x_386); -lean_dec(x_385); -x_387 = l_Array_append___rarg(x_13, x_386); -lean_dec(x_386); -x_388 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_388; -x_15 = x_387; -goto block_378; +lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_274 = lean_ctor_get(x_273, 0); +lean_inc(x_274); +lean_dec(x_273); +x_275 = l_Array_append___rarg(x_13, x_274); +lean_dec(x_274); +x_276 = l_Lake_decodeLeanOptions___closed__1; +x_15 = x_276; +x_16 = x_275; +goto block_266; } else { -lean_object* x_389; -x_389 = lean_ctor_get(x_385, 0); -lean_inc(x_389); -lean_dec(x_385); -x_14 = x_389; -x_15 = x_13; -goto block_378; +lean_object* x_277; +x_277 = lean_ctor_get(x_273, 0); +lean_inc(x_277); +lean_dec(x_273); +x_15 = x_277; +x_16 = x_13; +goto block_266; } } -block_378: +block_266: { -lean_object* x_16; lean_object* x_17; lean_object* x_367; lean_object* x_368; lean_object* x_369; -x_367 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_368 = l_Lake_LeanConfig_decodeToml___closed__15; +lean_object* x_17; lean_object* x_18; lean_object* x_255; lean_object* x_256; lean_object* x_257; +x_255 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_256 = l_Lake_LeanConfig_decodeToml___closed__15; lean_inc(x_1); -x_369 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_367, x_368, x_1); -if (lean_obj_tag(x_369) == 0) +x_257 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_255, x_256, x_1); +if (lean_obj_tag(x_257) == 0) { -lean_object* x_370; -x_370 = l_Lake_decodeLeanOptions___closed__1; -x_16 = x_370; -x_17 = x_15; -goto block_366; +lean_object* x_258; +x_258 = l_Lake_decodeLeanOptions___closed__1; +x_17 = x_258; +x_18 = x_16; +goto block_254; } else { -lean_object* x_371; lean_object* x_372; lean_object* x_373; -x_371 = lean_ctor_get(x_369, 0); -lean_inc(x_371); -lean_dec(x_369); -x_372 = lean_ctor_get(x_371, 1); -lean_inc(x_372); -lean_dec(x_371); -x_373 = l_Lake_decodeLeanOptions(x_372); -if (lean_obj_tag(x_373) == 0) +lean_object* x_259; lean_object* x_260; lean_object* x_261; +x_259 = lean_ctor_get(x_257, 0); +lean_inc(x_259); +lean_dec(x_257); +x_260 = lean_ctor_get(x_259, 1); +lean_inc(x_260); +lean_dec(x_259); +x_261 = l_Lake_decodeLeanOptions(x_260); +if (lean_obj_tag(x_261) == 0) { -lean_object* x_374; lean_object* x_375; lean_object* x_376; -x_374 = lean_ctor_get(x_373, 0); -lean_inc(x_374); -lean_dec(x_373); -x_375 = l_Array_append___rarg(x_15, x_374); -lean_dec(x_374); -x_376 = l_Lake_decodeLeanOptions___closed__1; -x_16 = x_376; -x_17 = x_375; -goto block_366; +lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_262 = lean_ctor_get(x_261, 0); +lean_inc(x_262); +lean_dec(x_261); +x_263 = l_Array_append___rarg(x_16, x_262); +lean_dec(x_262); +x_264 = l_Lake_decodeLeanOptions___closed__1; +x_17 = x_264; +x_18 = x_263; +goto block_254; } else { -lean_object* x_377; -x_377 = lean_ctor_get(x_373, 0); -lean_inc(x_377); -lean_dec(x_373); -x_16 = x_377; -x_17 = x_15; -goto block_366; +lean_object* x_265; +x_265 = lean_ctor_get(x_261, 0); +lean_inc(x_265); +lean_dec(x_261); +x_17 = x_265; +x_18 = x_16; +goto block_254; } } -block_366: +block_254: { -lean_object* x_18; lean_object* x_19; lean_object* x_312; lean_object* x_313; lean_object* x_314; -x_312 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_313 = l_Lake_LeanConfig_decodeToml___closed__2; +lean_object* x_19; lean_object* x_20; lean_object* x_218; lean_object* x_224; lean_object* x_225; lean_object* x_226; +x_224 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_225 = l_Lake_LeanConfig_decodeToml___closed__2; lean_inc(x_1); -x_314 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_312, x_313, x_1); -if (lean_obj_tag(x_314) == 0) +x_226 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_224, x_225, x_1); +if (lean_obj_tag(x_226) == 0) { -lean_object* x_315; -x_315 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_315; -x_19 = x_17; -goto block_311; +lean_object* x_227; +x_227 = l_Lake_decodeLeanOptions___closed__1; +x_19 = x_227; +x_20 = x_18; +goto block_217; } else { -lean_object* x_316; lean_object* x_317; -x_316 = lean_ctor_get(x_314, 0); -lean_inc(x_316); -lean_dec(x_314); -x_317 = lean_ctor_get(x_316, 1); -lean_inc(x_317); -lean_dec(x_316); -switch (lean_obj_tag(x_317)) { +lean_object* x_228; lean_object* x_229; +x_228 = lean_ctor_get(x_226, 0); +lean_inc(x_228); +lean_dec(x_226); +x_229 = lean_ctor_get(x_228, 1); +lean_inc(x_229); +lean_dec(x_228); +switch (lean_obj_tag(x_229)) { case 0: { -uint8_t x_318; -x_318 = !lean_is_exclusive(x_317); -if (x_318 == 0) +uint8_t x_230; +x_230 = !lean_is_exclusive(x_229); +if (x_230 == 0) { -lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; -x_319 = lean_ctor_get(x_317, 1); -lean_dec(x_319); -x_320 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_317, 1, x_320); -x_321 = lean_unsigned_to_nat(1u); -x_322 = lean_mk_array(x_321, x_317); -x_323 = l_Array_append___rarg(x_17, x_322); -lean_dec(x_322); -x_324 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_324; -x_19 = x_323; -goto block_311; +lean_object* x_231; lean_object* x_232; +x_231 = lean_ctor_get(x_229, 1); +lean_dec(x_231); +x_232 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_229, 1, x_232); +x_218 = x_229; +goto block_223; } else { -lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; -x_325 = lean_ctor_get(x_317, 0); -lean_inc(x_325); -lean_dec(x_317); -x_326 = l_Lake_LeanConfig_decodeToml___closed__5; -x_327 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_327, 0, x_325); -lean_ctor_set(x_327, 1, x_326); -x_328 = lean_unsigned_to_nat(1u); -x_329 = lean_mk_array(x_328, x_327); -x_330 = l_Array_append___rarg(x_17, x_329); -lean_dec(x_329); -x_331 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_331; -x_19 = x_330; -goto block_311; +lean_object* x_233; lean_object* x_234; lean_object* x_235; +x_233 = lean_ctor_get(x_229, 0); +lean_inc(x_233); +lean_dec(x_229); +x_234 = l_Lake_LeanConfig_decodeToml___closed__5; +x_235 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_235, 0, x_233); +lean_ctor_set(x_235, 1, x_234); +x_218 = x_235; +goto block_223; } } case 2: { -lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; -x_332 = lean_ctor_get(x_317, 0); -lean_inc(x_332); -lean_dec(x_317); -x_333 = l_Lake_LeanConfig_decodeToml___closed__5; -x_334 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_334, 0, x_332); -lean_ctor_set(x_334, 1, x_333); -x_335 = lean_unsigned_to_nat(1u); -x_336 = lean_mk_array(x_335, x_334); -x_337 = l_Array_append___rarg(x_17, x_336); -lean_dec(x_336); -x_338 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_338; -x_19 = x_337; -goto block_311; +lean_object* x_236; lean_object* x_237; lean_object* x_238; +x_236 = lean_ctor_get(x_229, 0); +lean_inc(x_236); +lean_dec(x_229); +x_237 = l_Lake_LeanConfig_decodeToml___closed__5; +x_238 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_238, 0, x_236); +lean_ctor_set(x_238, 1, x_237); +x_218 = x_238; +goto block_223; } case 3: { -lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; -x_339 = lean_ctor_get(x_317, 0); -lean_inc(x_339); -lean_dec(x_317); -x_340 = l_Lake_LeanConfig_decodeToml___closed__5; -x_341 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_341, 0, x_339); -lean_ctor_set(x_341, 1, x_340); -x_342 = lean_unsigned_to_nat(1u); -x_343 = lean_mk_array(x_342, x_341); -x_344 = l_Array_append___rarg(x_17, x_343); -lean_dec(x_343); -x_345 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_345; -x_19 = x_344; -goto block_311; +lean_object* x_239; lean_object* x_240; lean_object* x_241; +x_239 = lean_ctor_get(x_229, 0); +lean_inc(x_239); +lean_dec(x_229); +x_240 = l_Lake_LeanConfig_decodeToml___closed__5; +x_241 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_241, 0, x_239); +lean_ctor_set(x_241, 1, x_240); +x_218 = x_241; +goto block_223; } case 5: { -lean_object* x_346; lean_object* x_347; -x_346 = lean_ctor_get(x_317, 1); -lean_inc(x_346); -lean_dec(x_317); -x_347 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_346); -lean_dec(x_346); -if (lean_obj_tag(x_347) == 0) +lean_object* x_242; lean_object* x_243; +x_242 = lean_ctor_get(x_229, 1); +lean_inc(x_242); +lean_dec(x_229); +x_243 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_242); +lean_dec(x_242); +if (lean_obj_tag(x_243) == 0) { -lean_object* x_348; lean_object* x_349; lean_object* x_350; -x_348 = lean_ctor_get(x_347, 0); -lean_inc(x_348); -lean_dec(x_347); -x_349 = l_Array_append___rarg(x_17, x_348); -lean_dec(x_348); -x_350 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_350; -x_19 = x_349; -goto block_311; +lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_244 = lean_ctor_get(x_243, 0); +lean_inc(x_244); +lean_dec(x_243); +x_245 = l_Array_append___rarg(x_18, x_244); +lean_dec(x_244); +x_246 = l_Lake_decodeLeanOptions___closed__1; +x_19 = x_246; +x_20 = x_245; +goto block_217; } else { -lean_object* x_351; -x_351 = lean_ctor_get(x_347, 0); -lean_inc(x_351); -lean_dec(x_347); -x_18 = x_351; -x_19 = x_17; -goto block_311; +lean_object* x_247; +x_247 = lean_ctor_get(x_243, 0); +lean_inc(x_247); +lean_dec(x_243); +x_19 = x_247; +x_20 = x_18; +goto block_217; } } default: { -uint8_t x_352; -x_352 = !lean_is_exclusive(x_317); -if (x_352 == 0) +uint8_t x_248; +x_248 = !lean_is_exclusive(x_229); +if (x_248 == 0) { -lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; -x_353 = lean_ctor_get(x_317, 1); -lean_dec(x_353); -x_354 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_317, 0); -lean_ctor_set(x_317, 1, x_354); -x_355 = lean_unsigned_to_nat(1u); -x_356 = lean_mk_array(x_355, x_317); -x_357 = l_Array_append___rarg(x_17, x_356); -lean_dec(x_356); -x_358 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_358; -x_19 = x_357; -goto block_311; +lean_object* x_249; lean_object* x_250; +x_249 = lean_ctor_get(x_229, 1); +lean_dec(x_249); +x_250 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_229, 0); +lean_ctor_set(x_229, 1, x_250); +x_218 = x_229; +goto block_223; } else { -lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; lean_object* x_365; -x_359 = lean_ctor_get(x_317, 0); -lean_inc(x_359); -lean_dec(x_317); -x_360 = l_Lake_LeanConfig_decodeToml___closed__5; -x_361 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_361, 0, x_359); -lean_ctor_set(x_361, 1, x_360); -x_362 = lean_unsigned_to_nat(1u); -x_363 = lean_mk_array(x_362, x_361); -x_364 = l_Array_append___rarg(x_17, x_363); -lean_dec(x_363); -x_365 = l_Lake_decodeLeanOptions___closed__1; -x_18 = x_365; -x_19 = x_364; -goto block_311; +lean_object* x_251; lean_object* x_252; lean_object* x_253; +x_251 = lean_ctor_get(x_229, 0); +lean_inc(x_251); +lean_dec(x_229); +x_252 = l_Lake_LeanConfig_decodeToml___closed__5; +x_253 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_253, 0, x_251); +lean_ctor_set(x_253, 1, x_252); +x_218 = x_253; +goto block_223; } } } } -block_311: +block_217: { -lean_object* x_20; lean_object* x_21; lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_257 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_258 = l_Lake_LeanConfig_decodeToml___closed__13; +lean_object* x_21; lean_object* x_22; lean_object* x_181; lean_object* x_187; lean_object* x_188; lean_object* x_189; +x_187 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_188 = l_Lake_LeanConfig_decodeToml___closed__13; lean_inc(x_1); -x_259 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_257, x_258, x_1); -if (lean_obj_tag(x_259) == 0) +x_189 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_187, x_188, x_1); +if (lean_obj_tag(x_189) == 0) { -lean_object* x_260; -x_260 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_260; -x_21 = x_19; -goto block_256; +lean_object* x_190; +x_190 = l_Lake_decodeLeanOptions___closed__1; +x_21 = x_190; +x_22 = x_20; +goto block_180; } else { -lean_object* x_261; lean_object* x_262; -x_261 = lean_ctor_get(x_259, 0); -lean_inc(x_261); -lean_dec(x_259); -x_262 = lean_ctor_get(x_261, 1); -lean_inc(x_262); -lean_dec(x_261); -switch (lean_obj_tag(x_262)) { +lean_object* x_191; lean_object* x_192; +x_191 = lean_ctor_get(x_189, 0); +lean_inc(x_191); +lean_dec(x_189); +x_192 = lean_ctor_get(x_191, 1); +lean_inc(x_192); +lean_dec(x_191); +switch (lean_obj_tag(x_192)) { case 0: { -uint8_t x_263; -x_263 = !lean_is_exclusive(x_262); -if (x_263 == 0) +uint8_t x_193; +x_193 = !lean_is_exclusive(x_192); +if (x_193 == 0) { -lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; -x_264 = lean_ctor_get(x_262, 1); -lean_dec(x_264); -x_265 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_262, 1, x_265); -x_266 = lean_unsigned_to_nat(1u); -x_267 = lean_mk_array(x_266, x_262); -x_268 = l_Array_append___rarg(x_19, x_267); -lean_dec(x_267); -x_269 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_269; -x_21 = x_268; -goto block_256; +lean_object* x_194; lean_object* x_195; +x_194 = lean_ctor_get(x_192, 1); +lean_dec(x_194); +x_195 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_192, 1, x_195); +x_181 = x_192; +goto block_186; } else { -lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; -x_270 = lean_ctor_get(x_262, 0); -lean_inc(x_270); -lean_dec(x_262); -x_271 = l_Lake_LeanConfig_decodeToml___closed__5; -x_272 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_272, 0, x_270); -lean_ctor_set(x_272, 1, x_271); -x_273 = lean_unsigned_to_nat(1u); -x_274 = lean_mk_array(x_273, x_272); -x_275 = l_Array_append___rarg(x_19, x_274); -lean_dec(x_274); -x_276 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_276; -x_21 = x_275; -goto block_256; +lean_object* x_196; lean_object* x_197; lean_object* x_198; +x_196 = lean_ctor_get(x_192, 0); +lean_inc(x_196); +lean_dec(x_192); +x_197 = l_Lake_LeanConfig_decodeToml___closed__5; +x_198 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_197); +x_181 = x_198; +goto block_186; } } case 2: { -lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; -x_277 = lean_ctor_get(x_262, 0); -lean_inc(x_277); -lean_dec(x_262); -x_278 = l_Lake_LeanConfig_decodeToml___closed__5; -x_279 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_279, 0, x_277); -lean_ctor_set(x_279, 1, x_278); -x_280 = lean_unsigned_to_nat(1u); -x_281 = lean_mk_array(x_280, x_279); -x_282 = l_Array_append___rarg(x_19, x_281); -lean_dec(x_281); -x_283 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_283; -x_21 = x_282; -goto block_256; +lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_199 = lean_ctor_get(x_192, 0); +lean_inc(x_199); +lean_dec(x_192); +x_200 = l_Lake_LeanConfig_decodeToml___closed__5; +x_201 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_201, 0, x_199); +lean_ctor_set(x_201, 1, x_200); +x_181 = x_201; +goto block_186; } case 3: { -lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; -x_284 = lean_ctor_get(x_262, 0); -lean_inc(x_284); -lean_dec(x_262); -x_285 = l_Lake_LeanConfig_decodeToml___closed__5; -x_286 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_286, 0, x_284); -lean_ctor_set(x_286, 1, x_285); -x_287 = lean_unsigned_to_nat(1u); -x_288 = lean_mk_array(x_287, x_286); -x_289 = l_Array_append___rarg(x_19, x_288); -lean_dec(x_288); -x_290 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_290; -x_21 = x_289; -goto block_256; +lean_object* x_202; lean_object* x_203; lean_object* x_204; +x_202 = lean_ctor_get(x_192, 0); +lean_inc(x_202); +lean_dec(x_192); +x_203 = l_Lake_LeanConfig_decodeToml___closed__5; +x_204 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_204, 0, x_202); +lean_ctor_set(x_204, 1, x_203); +x_181 = x_204; +goto block_186; } case 5: { -lean_object* x_291; lean_object* x_292; -x_291 = lean_ctor_get(x_262, 1); -lean_inc(x_291); -lean_dec(x_262); -x_292 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_291); -lean_dec(x_291); -if (lean_obj_tag(x_292) == 0) +lean_object* x_205; lean_object* x_206; +x_205 = lean_ctor_get(x_192, 1); +lean_inc(x_205); +lean_dec(x_192); +x_206 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_205); +lean_dec(x_205); +if (lean_obj_tag(x_206) == 0) { -lean_object* x_293; lean_object* x_294; lean_object* x_295; -x_293 = lean_ctor_get(x_292, 0); -lean_inc(x_293); -lean_dec(x_292); -x_294 = l_Array_append___rarg(x_19, x_293); -lean_dec(x_293); -x_295 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_295; -x_21 = x_294; -goto block_256; +lean_object* x_207; lean_object* x_208; lean_object* x_209; +x_207 = lean_ctor_get(x_206, 0); +lean_inc(x_207); +lean_dec(x_206); +x_208 = l_Array_append___rarg(x_20, x_207); +lean_dec(x_207); +x_209 = l_Lake_decodeLeanOptions___closed__1; +x_21 = x_209; +x_22 = x_208; +goto block_180; } else { -lean_object* x_296; -x_296 = lean_ctor_get(x_292, 0); -lean_inc(x_296); -lean_dec(x_292); -x_20 = x_296; -x_21 = x_19; -goto block_256; +lean_object* x_210; +x_210 = lean_ctor_get(x_206, 0); +lean_inc(x_210); +lean_dec(x_206); +x_21 = x_210; +x_22 = x_20; +goto block_180; } } default: { -uint8_t x_297; -x_297 = !lean_is_exclusive(x_262); -if (x_297 == 0) -{ -lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; -x_298 = lean_ctor_get(x_262, 1); -lean_dec(x_298); -x_299 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_262, 0); -lean_ctor_set(x_262, 1, x_299); -x_300 = lean_unsigned_to_nat(1u); -x_301 = lean_mk_array(x_300, x_262); -x_302 = l_Array_append___rarg(x_19, x_301); -lean_dec(x_301); -x_303 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_303; -x_21 = x_302; -goto block_256; +uint8_t x_211; +x_211 = !lean_is_exclusive(x_192); +if (x_211 == 0) +{ +lean_object* x_212; lean_object* x_213; +x_212 = lean_ctor_get(x_192, 1); +lean_dec(x_212); +x_213 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_192, 0); +lean_ctor_set(x_192, 1, x_213); +x_181 = x_192; +goto block_186; } else { -lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; -x_304 = lean_ctor_get(x_262, 0); -lean_inc(x_304); -lean_dec(x_262); -x_305 = l_Lake_LeanConfig_decodeToml___closed__5; -x_306 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_306, 0, x_304); -lean_ctor_set(x_306, 1, x_305); -x_307 = lean_unsigned_to_nat(1u); -x_308 = lean_mk_array(x_307, x_306); -x_309 = l_Array_append___rarg(x_19, x_308); -lean_dec(x_308); -x_310 = l_Lake_decodeLeanOptions___closed__1; -x_20 = x_310; -x_21 = x_309; -goto block_256; +lean_object* x_214; lean_object* x_215; lean_object* x_216; +x_214 = lean_ctor_get(x_192, 0); +lean_inc(x_214); +lean_dec(x_192); +x_215 = l_Lake_LeanConfig_decodeToml___closed__5; +x_216 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_216, 0, x_214); +lean_ctor_set(x_216, 1, x_215); +x_181 = x_216; +goto block_186; } } } } -block_256: +block_180: { -lean_object* x_22; lean_object* x_23; lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_202 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_203 = l_Lake_LeanConfig_decodeToml___closed__11; +lean_object* x_23; lean_object* x_24; lean_object* x_144; lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_150 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_151 = l_Lake_LeanConfig_decodeToml___closed__11; lean_inc(x_1); -x_204 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_202, x_203, x_1); -if (lean_obj_tag(x_204) == 0) +x_152 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_150, x_151, x_1); +if (lean_obj_tag(x_152) == 0) { -lean_object* x_205; -x_205 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_205; -x_23 = x_21; -goto block_201; +lean_object* x_153; +x_153 = l_Lake_decodeLeanOptions___closed__1; +x_23 = x_153; +x_24 = x_22; +goto block_143; } else { -lean_object* x_206; lean_object* x_207; -x_206 = lean_ctor_get(x_204, 0); -lean_inc(x_206); -lean_dec(x_204); -x_207 = lean_ctor_get(x_206, 1); -lean_inc(x_207); -lean_dec(x_206); -switch (lean_obj_tag(x_207)) { +lean_object* x_154; lean_object* x_155; +x_154 = lean_ctor_get(x_152, 0); +lean_inc(x_154); +lean_dec(x_152); +x_155 = lean_ctor_get(x_154, 1); +lean_inc(x_155); +lean_dec(x_154); +switch (lean_obj_tag(x_155)) { case 0: { -uint8_t x_208; -x_208 = !lean_is_exclusive(x_207); -if (x_208 == 0) +uint8_t x_156; +x_156 = !lean_is_exclusive(x_155); +if (x_156 == 0) { -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -x_209 = lean_ctor_get(x_207, 1); -lean_dec(x_209); -x_210 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_207, 1, x_210); -x_211 = lean_unsigned_to_nat(1u); -x_212 = lean_mk_array(x_211, x_207); -x_213 = l_Array_append___rarg(x_21, x_212); -lean_dec(x_212); -x_214 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_214; -x_23 = x_213; -goto block_201; +lean_object* x_157; lean_object* x_158; +x_157 = lean_ctor_get(x_155, 1); +lean_dec(x_157); +x_158 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_155, 1, x_158); +x_144 = x_155; +goto block_149; } else { -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; -x_215 = lean_ctor_get(x_207, 0); -lean_inc(x_215); -lean_dec(x_207); -x_216 = l_Lake_LeanConfig_decodeToml___closed__5; -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_215); -lean_ctor_set(x_217, 1, x_216); -x_218 = lean_unsigned_to_nat(1u); -x_219 = lean_mk_array(x_218, x_217); -x_220 = l_Array_append___rarg(x_21, x_219); -lean_dec(x_219); -x_221 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_221; -x_23 = x_220; -goto block_201; +lean_object* x_159; lean_object* x_160; lean_object* x_161; +x_159 = lean_ctor_get(x_155, 0); +lean_inc(x_159); +lean_dec(x_155); +x_160 = l_Lake_LeanConfig_decodeToml___closed__5; +x_161 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_161, 0, x_159); +lean_ctor_set(x_161, 1, x_160); +x_144 = x_161; +goto block_149; } } case 2: { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; -x_222 = lean_ctor_get(x_207, 0); -lean_inc(x_222); -lean_dec(x_207); -x_223 = l_Lake_LeanConfig_decodeToml___closed__5; -x_224 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_224, 0, x_222); -lean_ctor_set(x_224, 1, x_223); -x_225 = lean_unsigned_to_nat(1u); -x_226 = lean_mk_array(x_225, x_224); -x_227 = l_Array_append___rarg(x_21, x_226); -lean_dec(x_226); -x_228 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_228; -x_23 = x_227; -goto block_201; +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_155, 0); +lean_inc(x_162); +lean_dec(x_155); +x_163 = l_Lake_LeanConfig_decodeToml___closed__5; +x_164 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_164, 0, x_162); +lean_ctor_set(x_164, 1, x_163); +x_144 = x_164; +goto block_149; } case 3: { -lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; -x_229 = lean_ctor_get(x_207, 0); -lean_inc(x_229); -lean_dec(x_207); -x_230 = l_Lake_LeanConfig_decodeToml___closed__5; -x_231 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_231, 0, x_229); -lean_ctor_set(x_231, 1, x_230); -x_232 = lean_unsigned_to_nat(1u); -x_233 = lean_mk_array(x_232, x_231); -x_234 = l_Array_append___rarg(x_21, x_233); -lean_dec(x_233); -x_235 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_235; -x_23 = x_234; -goto block_201; +lean_object* x_165; lean_object* x_166; lean_object* x_167; +x_165 = lean_ctor_get(x_155, 0); +lean_inc(x_165); +lean_dec(x_155); +x_166 = l_Lake_LeanConfig_decodeToml___closed__5; +x_167 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_165); +lean_ctor_set(x_167, 1, x_166); +x_144 = x_167; +goto block_149; } case 5: { -lean_object* x_236; lean_object* x_237; -x_236 = lean_ctor_get(x_207, 1); -lean_inc(x_236); -lean_dec(x_207); -x_237 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_236); -lean_dec(x_236); -if (lean_obj_tag(x_237) == 0) +lean_object* x_168; lean_object* x_169; +x_168 = lean_ctor_get(x_155, 1); +lean_inc(x_168); +lean_dec(x_155); +x_169 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_168); +lean_dec(x_168); +if (lean_obj_tag(x_169) == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; -x_238 = lean_ctor_get(x_237, 0); -lean_inc(x_238); -lean_dec(x_237); -x_239 = l_Array_append___rarg(x_21, x_238); -lean_dec(x_238); -x_240 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_240; -x_23 = x_239; -goto block_201; +lean_object* x_170; lean_object* x_171; lean_object* x_172; +x_170 = lean_ctor_get(x_169, 0); +lean_inc(x_170); +lean_dec(x_169); +x_171 = l_Array_append___rarg(x_22, x_170); +lean_dec(x_170); +x_172 = l_Lake_decodeLeanOptions___closed__1; +x_23 = x_172; +x_24 = x_171; +goto block_143; } else { -lean_object* x_241; -x_241 = lean_ctor_get(x_237, 0); -lean_inc(x_241); -lean_dec(x_237); -x_22 = x_241; -x_23 = x_21; -goto block_201; +lean_object* x_173; +x_173 = lean_ctor_get(x_169, 0); +lean_inc(x_173); +lean_dec(x_169); +x_23 = x_173; +x_24 = x_22; +goto block_143; } } default: { -uint8_t x_242; -x_242 = !lean_is_exclusive(x_207); -if (x_242 == 0) +uint8_t x_174; +x_174 = !lean_is_exclusive(x_155); +if (x_174 == 0) { -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; -x_243 = lean_ctor_get(x_207, 1); -lean_dec(x_243); -x_244 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_207, 0); -lean_ctor_set(x_207, 1, x_244); -x_245 = lean_unsigned_to_nat(1u); -x_246 = lean_mk_array(x_245, x_207); -x_247 = l_Array_append___rarg(x_21, x_246); -lean_dec(x_246); -x_248 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_248; -x_23 = x_247; -goto block_201; -} -else -{ -lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -x_249 = lean_ctor_get(x_207, 0); -lean_inc(x_249); -lean_dec(x_207); -x_250 = l_Lake_LeanConfig_decodeToml___closed__5; -x_251 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_251, 0, x_249); -lean_ctor_set(x_251, 1, x_250); -x_252 = lean_unsigned_to_nat(1u); -x_253 = lean_mk_array(x_252, x_251); -x_254 = l_Array_append___rarg(x_21, x_253); -lean_dec(x_253); -x_255 = l_Lake_decodeLeanOptions___closed__1; -x_22 = x_255; -x_23 = x_254; -goto block_201; +lean_object* x_175; lean_object* x_176; +x_175 = lean_ctor_get(x_155, 1); +lean_dec(x_175); +x_176 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_155, 0); +lean_ctor_set(x_155, 1, x_176); +x_144 = x_155; +goto block_149; +} +else +{ +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_155, 0); +lean_inc(x_177); +lean_dec(x_155); +x_178 = l_Lake_LeanConfig_decodeToml___closed__5; +x_179 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +x_144 = x_179; +goto block_149; } } } } -block_201: +block_143: { -lean_object* x_24; lean_object* x_25; lean_object* x_147; lean_object* x_148; lean_object* x_149; -x_147 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_148 = l_Lake_LeanConfig_decodeToml___closed__9; +lean_object* x_25; lean_object* x_26; lean_object* x_107; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_114 = l_Lake_LeanConfig_decodeToml___closed__9; lean_inc(x_1); -x_149 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_147, x_148, x_1); -if (lean_obj_tag(x_149) == 0) +x_115 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_113, x_114, x_1); +if (lean_obj_tag(x_115) == 0) { -lean_object* x_150; -x_150 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_150; -x_25 = x_23; -goto block_146; +lean_object* x_116; +x_116 = l_Lake_decodeLeanOptions___closed__1; +x_25 = x_116; +x_26 = x_24; +goto block_106; } else { -lean_object* x_151; lean_object* x_152; -x_151 = lean_ctor_get(x_149, 0); -lean_inc(x_151); -lean_dec(x_149); -x_152 = lean_ctor_get(x_151, 1); -lean_inc(x_152); -lean_dec(x_151); -switch (lean_obj_tag(x_152)) { +lean_object* x_117; lean_object* x_118; +x_117 = lean_ctor_get(x_115, 0); +lean_inc(x_117); +lean_dec(x_115); +x_118 = lean_ctor_get(x_117, 1); +lean_inc(x_118); +lean_dec(x_117); +switch (lean_obj_tag(x_118)) { case 0: { -uint8_t x_153; -x_153 = !lean_is_exclusive(x_152); -if (x_153 == 0) +uint8_t x_119; +x_119 = !lean_is_exclusive(x_118); +if (x_119 == 0) { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_154 = lean_ctor_get(x_152, 1); -lean_dec(x_154); -x_155 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_152, 1, x_155); -x_156 = lean_unsigned_to_nat(1u); -x_157 = lean_mk_array(x_156, x_152); -x_158 = l_Array_append___rarg(x_23, x_157); -lean_dec(x_157); -x_159 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_159; -x_25 = x_158; -goto block_146; +lean_object* x_120; lean_object* x_121; +x_120 = lean_ctor_get(x_118, 1); +lean_dec(x_120); +x_121 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_118, 1, x_121); +x_107 = x_118; +goto block_112; } else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_160 = lean_ctor_get(x_152, 0); -lean_inc(x_160); -lean_dec(x_152); -x_161 = l_Lake_LeanConfig_decodeToml___closed__5; -x_162 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_162, 0, x_160); -lean_ctor_set(x_162, 1, x_161); -x_163 = lean_unsigned_to_nat(1u); -x_164 = lean_mk_array(x_163, x_162); -x_165 = l_Array_append___rarg(x_23, x_164); -lean_dec(x_164); -x_166 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_166; -x_25 = x_165; -goto block_146; +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_118, 0); +lean_inc(x_122); +lean_dec(x_118); +x_123 = l_Lake_LeanConfig_decodeToml___closed__5; +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +x_107 = x_124; +goto block_112; } } case 2: { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_167 = lean_ctor_get(x_152, 0); -lean_inc(x_167); -lean_dec(x_152); -x_168 = l_Lake_LeanConfig_decodeToml___closed__5; -x_169 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_169, 0, x_167); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_unsigned_to_nat(1u); -x_171 = lean_mk_array(x_170, x_169); -x_172 = l_Array_append___rarg(x_23, x_171); -lean_dec(x_171); -x_173 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_173; -x_25 = x_172; -goto block_146; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_118, 0); +lean_inc(x_125); +lean_dec(x_118); +x_126 = l_Lake_LeanConfig_decodeToml___closed__5; +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +x_107 = x_127; +goto block_112; } case 3: { -lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; -x_174 = lean_ctor_get(x_152, 0); -lean_inc(x_174); -lean_dec(x_152); -x_175 = l_Lake_LeanConfig_decodeToml___closed__5; -x_176 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_176, 0, x_174); -lean_ctor_set(x_176, 1, x_175); -x_177 = lean_unsigned_to_nat(1u); -x_178 = lean_mk_array(x_177, x_176); -x_179 = l_Array_append___rarg(x_23, x_178); -lean_dec(x_178); -x_180 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_180; -x_25 = x_179; -goto block_146; +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_118, 0); +lean_inc(x_128); +lean_dec(x_118); +x_129 = l_Lake_LeanConfig_decodeToml___closed__5; +x_130 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +x_107 = x_130; +goto block_112; } case 5: { -lean_object* x_181; lean_object* x_182; -x_181 = lean_ctor_get(x_152, 1); -lean_inc(x_181); -lean_dec(x_152); -x_182 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_181); -lean_dec(x_181); -if (lean_obj_tag(x_182) == 0) +lean_object* x_131; lean_object* x_132; +x_131 = lean_ctor_get(x_118, 1); +lean_inc(x_131); +lean_dec(x_118); +x_132 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_131); +lean_dec(x_131); +if (lean_obj_tag(x_132) == 0) { -lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_183 = lean_ctor_get(x_182, 0); -lean_inc(x_183); -lean_dec(x_182); -x_184 = l_Array_append___rarg(x_23, x_183); -lean_dec(x_183); -x_185 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_185; -x_25 = x_184; -goto block_146; +lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_133 = lean_ctor_get(x_132, 0); +lean_inc(x_133); +lean_dec(x_132); +x_134 = l_Array_append___rarg(x_24, x_133); +lean_dec(x_133); +x_135 = l_Lake_decodeLeanOptions___closed__1; +x_25 = x_135; +x_26 = x_134; +goto block_106; } else { -lean_object* x_186; -x_186 = lean_ctor_get(x_182, 0); -lean_inc(x_186); -lean_dec(x_182); -x_24 = x_186; -x_25 = x_23; -goto block_146; +lean_object* x_136; +x_136 = lean_ctor_get(x_132, 0); +lean_inc(x_136); +lean_dec(x_132); +x_25 = x_136; +x_26 = x_24; +goto block_106; } } default: { -uint8_t x_187; -x_187 = !lean_is_exclusive(x_152); -if (x_187 == 0) +uint8_t x_137; +x_137 = !lean_is_exclusive(x_118); +if (x_137 == 0) { -lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; -x_188 = lean_ctor_get(x_152, 1); -lean_dec(x_188); -x_189 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_152, 0); -lean_ctor_set(x_152, 1, x_189); -x_190 = lean_unsigned_to_nat(1u); -x_191 = lean_mk_array(x_190, x_152); -x_192 = l_Array_append___rarg(x_23, x_191); -lean_dec(x_191); -x_193 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_193; -x_25 = x_192; -goto block_146; +lean_object* x_138; lean_object* x_139; +x_138 = lean_ctor_get(x_118, 1); +lean_dec(x_138); +x_139 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_118, 0); +lean_ctor_set(x_118, 1, x_139); +x_107 = x_118; +goto block_112; } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_194 = lean_ctor_get(x_152, 0); -lean_inc(x_194); -lean_dec(x_152); -x_195 = l_Lake_LeanConfig_decodeToml___closed__5; -x_196 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_196, 0, x_194); -lean_ctor_set(x_196, 1, x_195); -x_197 = lean_unsigned_to_nat(1u); -x_198 = lean_mk_array(x_197, x_196); -x_199 = l_Array_append___rarg(x_23, x_198); -lean_dec(x_198); -x_200 = l_Lake_decodeLeanOptions___closed__1; -x_24 = x_200; -x_25 = x_199; -goto block_146; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_118, 0); +lean_inc(x_140); +lean_dec(x_118); +x_141 = l_Lake_LeanConfig_decodeToml___closed__5; +x_142 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +x_107 = x_142; +goto block_112; } } } } -block_146: +block_106: { -lean_object* x_26; lean_object* x_27; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_92 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_93 = l_Lake_LeanConfig_decodeToml___closed__7; +lean_object* x_27; lean_object* x_28; lean_object* x_70; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_77 = l_Lake_LeanConfig_decodeToml___closed__7; lean_inc(x_1); -x_94 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_92, x_93, x_1); -if (lean_obj_tag(x_94) == 0) +x_78 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_76, x_77, x_1); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_95; -x_95 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_95; -x_27 = x_25; -goto block_91; +lean_object* x_79; +x_79 = l_Lake_decodeLeanOptions___closed__1; +x_27 = x_79; +x_28 = x_26; +goto block_69; } else { -lean_object* x_96; lean_object* x_97; -x_96 = lean_ctor_get(x_94, 0); -lean_inc(x_96); -lean_dec(x_94); -x_97 = lean_ctor_get(x_96, 1); -lean_inc(x_97); -lean_dec(x_96); -switch (lean_obj_tag(x_97)) { +lean_object* x_80; lean_object* x_81; +x_80 = lean_ctor_get(x_78, 0); +lean_inc(x_80); +lean_dec(x_78); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +lean_dec(x_80); +switch (lean_obj_tag(x_81)) { case 0: { -uint8_t x_98; -x_98 = !lean_is_exclusive(x_97); -if (x_98 == 0) +uint8_t x_82; +x_82 = !lean_is_exclusive(x_81); +if (x_82 == 0) { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_99 = lean_ctor_get(x_97, 1); -lean_dec(x_99); -x_100 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_97, 1, x_100); -x_101 = lean_unsigned_to_nat(1u); -x_102 = lean_mk_array(x_101, x_97); -x_103 = l_Array_append___rarg(x_25, x_102); -lean_dec(x_102); -x_104 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_104; -x_27 = x_103; -goto block_91; +lean_object* x_83; lean_object* x_84; +x_83 = lean_ctor_get(x_81, 1); +lean_dec(x_83); +x_84 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_81, 1, x_84); +x_70 = x_81; +goto block_75; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_105 = lean_ctor_get(x_97, 0); -lean_inc(x_105); -lean_dec(x_97); -x_106 = l_Lake_LeanConfig_decodeToml___closed__5; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -x_108 = lean_unsigned_to_nat(1u); -x_109 = lean_mk_array(x_108, x_107); -x_110 = l_Array_append___rarg(x_25, x_109); -lean_dec(x_109); -x_111 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_111; -x_27 = x_110; -goto block_91; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_81, 0); +lean_inc(x_85); +lean_dec(x_81); +x_86 = l_Lake_LeanConfig_decodeToml___closed__5; +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +x_70 = x_87; +goto block_75; } } case 2: { -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_112 = lean_ctor_get(x_97, 0); -lean_inc(x_112); -lean_dec(x_97); -x_113 = l_Lake_LeanConfig_decodeToml___closed__5; -x_114 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_114, 0, x_112); -lean_ctor_set(x_114, 1, x_113); -x_115 = lean_unsigned_to_nat(1u); -x_116 = lean_mk_array(x_115, x_114); -x_117 = l_Array_append___rarg(x_25, x_116); -lean_dec(x_116); -x_118 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_118; -x_27 = x_117; -goto block_91; +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_81, 0); +lean_inc(x_88); +lean_dec(x_81); +x_89 = l_Lake_LeanConfig_decodeToml___closed__5; +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_70 = x_90; +goto block_75; } case 3: { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_119 = lean_ctor_get(x_97, 0); -lean_inc(x_119); -lean_dec(x_97); -x_120 = l_Lake_LeanConfig_decodeToml___closed__5; -x_121 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_121, 0, x_119); -lean_ctor_set(x_121, 1, x_120); -x_122 = lean_unsigned_to_nat(1u); -x_123 = lean_mk_array(x_122, x_121); -x_124 = l_Array_append___rarg(x_25, x_123); -lean_dec(x_123); -x_125 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_125; -x_27 = x_124; -goto block_91; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_81, 0); +lean_inc(x_91); +lean_dec(x_81); +x_92 = l_Lake_LeanConfig_decodeToml___closed__5; +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_70 = x_93; +goto block_75; } case 5: { -lean_object* x_126; lean_object* x_127; -x_126 = lean_ctor_get(x_97, 1); -lean_inc(x_126); -lean_dec(x_97); -x_127 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_126); -lean_dec(x_126); -if (lean_obj_tag(x_127) == 0) +lean_object* x_94; lean_object* x_95; +x_94 = lean_ctor_get(x_81, 1); +lean_inc(x_94); +lean_dec(x_81); +x_95 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_94); +lean_dec(x_94); +if (lean_obj_tag(x_95) == 0) { -lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_128 = lean_ctor_get(x_127, 0); -lean_inc(x_128); -lean_dec(x_127); -x_129 = l_Array_append___rarg(x_25, x_128); -lean_dec(x_128); -x_130 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_130; -x_27 = x_129; -goto block_91; +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_95, 0); +lean_inc(x_96); +lean_dec(x_95); +x_97 = l_Array_append___rarg(x_26, x_96); +lean_dec(x_96); +x_98 = l_Lake_decodeLeanOptions___closed__1; +x_27 = x_98; +x_28 = x_97; +goto block_69; } else { -lean_object* x_131; -x_131 = lean_ctor_get(x_127, 0); -lean_inc(x_131); -lean_dec(x_127); -x_26 = x_131; -x_27 = x_25; -goto block_91; +lean_object* x_99; +x_99 = lean_ctor_get(x_95, 0); +lean_inc(x_99); +lean_dec(x_95); +x_27 = x_99; +x_28 = x_26; +goto block_69; } } default: { -uint8_t x_132; -x_132 = !lean_is_exclusive(x_97); -if (x_132 == 0) +uint8_t x_100; +x_100 = !lean_is_exclusive(x_81); +if (x_100 == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; -x_133 = lean_ctor_get(x_97, 1); -lean_dec(x_133); -x_134 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_97, 0); -lean_ctor_set(x_97, 1, x_134); -x_135 = lean_unsigned_to_nat(1u); -x_136 = lean_mk_array(x_135, x_97); -x_137 = l_Array_append___rarg(x_25, x_136); -lean_dec(x_136); -x_138 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_138; -x_27 = x_137; -goto block_91; +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_81, 1); +lean_dec(x_101); +x_102 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_81, 0); +lean_ctor_set(x_81, 1, x_102); +x_70 = x_81; +goto block_75; } else { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_139 = lean_ctor_get(x_97, 0); -lean_inc(x_139); -lean_dec(x_97); -x_140 = l_Lake_LeanConfig_decodeToml___closed__5; -x_141 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -x_142 = lean_unsigned_to_nat(1u); -x_143 = lean_mk_array(x_142, x_141); -x_144 = l_Array_append___rarg(x_25, x_143); -lean_dec(x_143); -x_145 = l_Lake_decodeLeanOptions___closed__1; -x_26 = x_145; -x_27 = x_144; -goto block_91; +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_81, 0); +lean_inc(x_103); +lean_dec(x_81); +x_104 = l_Lake_LeanConfig_decodeToml___closed__5; +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +x_70 = x_105; +goto block_75; } } } } -block_91: +block_69: { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_29 = l_Lake_LeanConfig_decodeToml___closed__4; -x_30 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_28, x_29, x_1); -if (lean_obj_tag(x_30) == 0) +lean_object* x_29; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_37 = l_Lake_LeanConfig_decodeToml___closed__4; +x_38 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_36, x_37, x_1); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_31; lean_object* x_32; -x_31 = l_Lake_decodeLeanOptions___closed__1; -x_32 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_32, 0, x_14); -lean_ctor_set(x_32, 1, x_18); -lean_ctor_set(x_32, 2, x_20); -lean_ctor_set(x_32, 3, x_22); -lean_ctor_set(x_32, 4, x_16); -lean_ctor_set(x_32, 5, x_24); -lean_ctor_set(x_32, 6, x_26); -lean_ctor_set(x_32, 7, x_31); -lean_ctor_set(x_32, 8, x_12); -lean_ctor_set_uint8(x_32, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_32, sizeof(void*)*9 + 1, x_10); -x_2 = x_32; -x_3 = x_27; +lean_object* x_39; lean_object* x_40; +x_39 = l_Lake_decodeLeanOptions___closed__1; +x_40 = lean_alloc_ctor(0, 9, 2); +lean_ctor_set(x_40, 0, x_15); +lean_ctor_set(x_40, 1, x_19); +lean_ctor_set(x_40, 2, x_21); +lean_ctor_set(x_40, 3, x_23); +lean_ctor_set(x_40, 4, x_17); +lean_ctor_set(x_40, 5, x_25); +lean_ctor_set(x_40, 6, x_27); +lean_ctor_set(x_40, 7, x_39); +lean_ctor_set(x_40, 8, x_12); +lean_ctor_set_uint8(x_40, sizeof(void*)*9, x_8); +lean_ctor_set_uint8(x_40, sizeof(void*)*9 + 1, x_10); +x_2 = x_40; +x_3 = x_28; goto block_7; } else { -lean_object* x_33; lean_object* x_34; -x_33 = lean_ctor_get(x_30, 0); -lean_inc(x_33); -lean_dec(x_30); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -switch (lean_obj_tag(x_34)) { +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_38, 0); +lean_inc(x_41); +lean_dec(x_38); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +switch (lean_obj_tag(x_42)) { case 0: { -uint8_t x_35; -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_36 = lean_ctor_get(x_34, 1); -lean_dec(x_36); -x_37 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_34, 1, x_37); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_34); -x_40 = l_Array_append___rarg(x_27, x_39); -lean_dec(x_39); -x_41 = l_Lake_decodeLeanOptions___closed__1; -x_42 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_42, 0, x_14); -lean_ctor_set(x_42, 1, x_18); -lean_ctor_set(x_42, 2, x_20); -lean_ctor_set(x_42, 3, x_22); -lean_ctor_set(x_42, 4, x_16); -lean_ctor_set(x_42, 5, x_24); -lean_ctor_set(x_42, 6, x_26); -lean_ctor_set(x_42, 7, x_41); -lean_ctor_set(x_42, 8, x_12); -lean_ctor_set_uint8(x_42, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_42, sizeof(void*)*9 + 1, x_10); -x_2 = x_42; -x_3 = x_40; -goto block_7; +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_42, 1); +lean_dec(x_44); +x_45 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_42, 1, x_45); +x_29 = x_42; +goto block_35; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_43 = lean_ctor_get(x_34, 0); -lean_inc(x_43); -lean_dec(x_34); -x_44 = l_Lake_LeanConfig_decodeToml___closed__5; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_unsigned_to_nat(1u); -x_47 = lean_mk_array(x_46, x_45); -x_48 = l_Array_append___rarg(x_27, x_47); -lean_dec(x_47); -x_49 = l_Lake_decodeLeanOptions___closed__1; -x_50 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_50, 0, x_14); -lean_ctor_set(x_50, 1, x_18); -lean_ctor_set(x_50, 2, x_20); -lean_ctor_set(x_50, 3, x_22); -lean_ctor_set(x_50, 4, x_16); -lean_ctor_set(x_50, 5, x_24); -lean_ctor_set(x_50, 6, x_26); -lean_ctor_set(x_50, 7, x_49); -lean_ctor_set(x_50, 8, x_12); -lean_ctor_set_uint8(x_50, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_50, sizeof(void*)*9 + 1, x_10); -x_2 = x_50; -x_3 = x_48; -goto block_7; +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_42, 0); +lean_inc(x_46); +lean_dec(x_42); +x_47 = l_Lake_LeanConfig_decodeToml___closed__5; +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +x_29 = x_48; +goto block_35; } } case 2: { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_51 = lean_ctor_get(x_34, 0); -lean_inc(x_51); -lean_dec(x_34); -x_52 = l_Lake_LeanConfig_decodeToml___closed__5; -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_mk_array(x_54, x_53); -x_56 = l_Array_append___rarg(x_27, x_55); -lean_dec(x_55); -x_57 = l_Lake_decodeLeanOptions___closed__1; -x_58 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_58, 0, x_14); -lean_ctor_set(x_58, 1, x_18); -lean_ctor_set(x_58, 2, x_20); -lean_ctor_set(x_58, 3, x_22); -lean_ctor_set(x_58, 4, x_16); -lean_ctor_set(x_58, 5, x_24); -lean_ctor_set(x_58, 6, x_26); -lean_ctor_set(x_58, 7, x_57); -lean_ctor_set(x_58, 8, x_12); -lean_ctor_set_uint8(x_58, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_58, sizeof(void*)*9 + 1, x_10); -x_2 = x_58; -x_3 = x_56; -goto block_7; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_42, 0); +lean_inc(x_49); +lean_dec(x_42); +x_50 = l_Lake_LeanConfig_decodeToml___closed__5; +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +x_29 = x_51; +goto block_35; } case 3: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_59 = lean_ctor_get(x_34, 0); -lean_inc(x_59); -lean_dec(x_34); -x_60 = l_Lake_LeanConfig_decodeToml___closed__5; -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -x_62 = lean_unsigned_to_nat(1u); -x_63 = lean_mk_array(x_62, x_61); -x_64 = l_Array_append___rarg(x_27, x_63); -lean_dec(x_63); -x_65 = l_Lake_decodeLeanOptions___closed__1; -x_66 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_66, 0, x_14); -lean_ctor_set(x_66, 1, x_18); -lean_ctor_set(x_66, 2, x_20); -lean_ctor_set(x_66, 3, x_22); -lean_ctor_set(x_66, 4, x_16); -lean_ctor_set(x_66, 5, x_24); -lean_ctor_set(x_66, 6, x_26); -lean_ctor_set(x_66, 7, x_65); -lean_ctor_set(x_66, 8, x_12); -lean_ctor_set_uint8(x_66, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_66, sizeof(void*)*9 + 1, x_10); -x_2 = x_66; -x_3 = x_64; -goto block_7; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_42, 0); +lean_inc(x_52); +lean_dec(x_42); +x_53 = l_Lake_LeanConfig_decodeToml___closed__5; +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +x_29 = x_54; +goto block_35; } case 5: { -lean_object* x_67; lean_object* x_68; -x_67 = lean_ctor_get(x_34, 1); -lean_inc(x_67); -lean_dec(x_34); -x_68 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_67); -lean_dec(x_67); -if (lean_obj_tag(x_68) == 0) +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_42, 1); +lean_inc(x_55); +lean_dec(x_42); +x_56 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_55); +lean_dec(x_55); +if (lean_obj_tag(x_56) == 0) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -lean_dec(x_68); -x_70 = l_Array_append___rarg(x_27, x_69); -lean_dec(x_69); -x_71 = l_Lake_decodeLeanOptions___closed__1; -x_72 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_72, 0, x_14); -lean_ctor_set(x_72, 1, x_18); -lean_ctor_set(x_72, 2, x_20); -lean_ctor_set(x_72, 3, x_22); -lean_ctor_set(x_72, 4, x_16); -lean_ctor_set(x_72, 5, x_24); -lean_ctor_set(x_72, 6, x_26); -lean_ctor_set(x_72, 7, x_71); -lean_ctor_set(x_72, 8, x_12); -lean_ctor_set_uint8(x_72, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_72, sizeof(void*)*9 + 1, x_10); -x_2 = x_72; -x_3 = x_70; +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +lean_dec(x_56); +x_58 = l_Array_append___rarg(x_28, x_57); +lean_dec(x_57); +x_59 = l_Lake_decodeLeanOptions___closed__1; +x_60 = lean_alloc_ctor(0, 9, 2); +lean_ctor_set(x_60, 0, x_15); +lean_ctor_set(x_60, 1, x_19); +lean_ctor_set(x_60, 2, x_21); +lean_ctor_set(x_60, 3, x_23); +lean_ctor_set(x_60, 4, x_17); +lean_ctor_set(x_60, 5, x_25); +lean_ctor_set(x_60, 6, x_27); +lean_ctor_set(x_60, 7, x_59); +lean_ctor_set(x_60, 8, x_12); +lean_ctor_set_uint8(x_60, sizeof(void*)*9, x_8); +lean_ctor_set_uint8(x_60, sizeof(void*)*9 + 1, x_10); +x_2 = x_60; +x_3 = x_58; goto block_7; } else { -lean_object* x_73; lean_object* x_74; -x_73 = lean_ctor_get(x_68, 0); -lean_inc(x_73); -lean_dec(x_68); -x_74 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_74, 0, x_14); -lean_ctor_set(x_74, 1, x_18); -lean_ctor_set(x_74, 2, x_20); -lean_ctor_set(x_74, 3, x_22); -lean_ctor_set(x_74, 4, x_16); -lean_ctor_set(x_74, 5, x_24); -lean_ctor_set(x_74, 6, x_26); -lean_ctor_set(x_74, 7, x_73); -lean_ctor_set(x_74, 8, x_12); -lean_ctor_set_uint8(x_74, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_74, sizeof(void*)*9 + 1, x_10); -x_2 = x_74; -x_3 = x_27; +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_56, 0); +lean_inc(x_61); +lean_dec(x_56); +x_62 = lean_alloc_ctor(0, 9, 2); +lean_ctor_set(x_62, 0, x_15); +lean_ctor_set(x_62, 1, x_19); +lean_ctor_set(x_62, 2, x_21); +lean_ctor_set(x_62, 3, x_23); +lean_ctor_set(x_62, 4, x_17); +lean_ctor_set(x_62, 5, x_25); +lean_ctor_set(x_62, 6, x_27); +lean_ctor_set(x_62, 7, x_61); +lean_ctor_set(x_62, 8, x_12); +lean_ctor_set_uint8(x_62, sizeof(void*)*9, x_8); +lean_ctor_set_uint8(x_62, sizeof(void*)*9 + 1, x_10); +x_2 = x_62; +x_3 = x_28; goto block_7; } } default: { -uint8_t x_75; -x_75 = !lean_is_exclusive(x_34); -if (x_75 == 0) +uint8_t x_63; +x_63 = !lean_is_exclusive(x_42); +if (x_63 == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_76 = lean_ctor_get(x_34, 1); -lean_dec(x_76); -x_77 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_34, 0); -lean_ctor_set(x_34, 1, x_77); -x_78 = lean_unsigned_to_nat(1u); -x_79 = lean_mk_array(x_78, x_34); -x_80 = l_Array_append___rarg(x_27, x_79); -lean_dec(x_79); -x_81 = l_Lake_decodeLeanOptions___closed__1; -x_82 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_82, 0, x_14); -lean_ctor_set(x_82, 1, x_18); -lean_ctor_set(x_82, 2, x_20); -lean_ctor_set(x_82, 3, x_22); -lean_ctor_set(x_82, 4, x_16); -lean_ctor_set(x_82, 5, x_24); -lean_ctor_set(x_82, 6, x_26); -lean_ctor_set(x_82, 7, x_81); -lean_ctor_set(x_82, 8, x_12); -lean_ctor_set_uint8(x_82, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_82, sizeof(void*)*9 + 1, x_10); -x_2 = x_82; -x_3 = x_80; -goto block_7; +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_42, 1); +lean_dec(x_64); +x_65 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_42, 0); +lean_ctor_set(x_42, 1, x_65); +x_29 = x_42; +goto block_35; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_83 = lean_ctor_get(x_34, 0); -lean_inc(x_83); -lean_dec(x_34); -x_84 = l_Lake_LeanConfig_decodeToml___closed__5; -x_85 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -x_86 = lean_unsigned_to_nat(1u); -x_87 = lean_mk_array(x_86, x_85); -x_88 = l_Array_append___rarg(x_27, x_87); -lean_dec(x_87); -x_89 = l_Lake_decodeLeanOptions___closed__1; -x_90 = lean_alloc_ctor(0, 9, 2); -lean_ctor_set(x_90, 0, x_14); -lean_ctor_set(x_90, 1, x_18); -lean_ctor_set(x_90, 2, x_20); -lean_ctor_set(x_90, 3, x_22); -lean_ctor_set(x_90, 4, x_16); -lean_ctor_set(x_90, 5, x_24); -lean_ctor_set(x_90, 6, x_26); -lean_ctor_set(x_90, 7, x_89); -lean_ctor_set(x_90, 8, x_12); -lean_ctor_set_uint8(x_90, sizeof(void*)*9, x_8); -lean_ctor_set_uint8(x_90, sizeof(void*)*9 + 1, x_10); -x_2 = x_90; -x_3 = x_88; +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_42, 0); +lean_inc(x_66); +lean_dec(x_42); +x_67 = l_Lake_LeanConfig_decodeToml___closed__5; +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +x_29 = x_68; +goto block_35; +} +} +} +} +block_35: +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_14); +x_31 = lean_array_mk(x_30); +x_32 = l_Array_append___rarg(x_28, x_31); +lean_dec(x_31); +x_33 = l_Lake_decodeLeanOptions___closed__1; +x_34 = lean_alloc_ctor(0, 9, 2); +lean_ctor_set(x_34, 0, x_15); +lean_ctor_set(x_34, 1, x_19); +lean_ctor_set(x_34, 2, x_21); +lean_ctor_set(x_34, 3, x_23); +lean_ctor_set(x_34, 4, x_17); +lean_ctor_set(x_34, 5, x_25); +lean_ctor_set(x_34, 6, x_27); +lean_ctor_set(x_34, 7, x_33); +lean_ctor_set(x_34, 8, x_12); +lean_ctor_set_uint8(x_34, sizeof(void*)*9, x_8); +lean_ctor_set_uint8(x_34, sizeof(void*)*9 + 1, x_10); +x_2 = x_34; +x_3 = x_32; goto block_7; } } +block_75: +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_14); +x_72 = lean_array_mk(x_71); +x_73 = l_Array_append___rarg(x_26, x_72); +lean_dec(x_72); +x_74 = l_Lake_decodeLeanOptions___closed__1; +x_27 = x_74; +x_28 = x_73; +goto block_69; +} +} +block_112: +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_107); +lean_ctor_set(x_108, 1, x_14); +x_109 = lean_array_mk(x_108); +x_110 = l_Array_append___rarg(x_24, x_109); +lean_dec(x_109); +x_111 = l_Lake_decodeLeanOptions___closed__1; +x_25 = x_111; +x_26 = x_110; +goto block_106; +} } +block_149: +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_145 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_145, 0, x_144); +lean_ctor_set(x_145, 1, x_14); +x_146 = lean_array_mk(x_145); +x_147 = l_Array_append___rarg(x_22, x_146); +lean_dec(x_146); +x_148 = l_Lake_decodeLeanOptions___closed__1; +x_23 = x_148; +x_24 = x_147; +goto block_143; } } +block_186: +{ +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_182 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_14); +x_183 = lean_array_mk(x_182); +x_184 = l_Array_append___rarg(x_20, x_183); +lean_dec(x_183); +x_185 = l_Lake_decodeLeanOptions___closed__1; +x_21 = x_185; +x_22 = x_184; +goto block_180; } } +block_223: +{ +lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; +x_219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_219, 0, x_218); +lean_ctor_set(x_219, 1, x_14); +x_220 = lean_array_mk(x_219); +x_221 = l_Array_append___rarg(x_18, x_220); +lean_dec(x_220); +x_222 = l_Lake_decodeLeanOptions___closed__1; +x_19 = x_222; +x_20 = x_221; +goto block_217; } } } } +block_288: +{ +lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; +x_284 = lean_box(0); +x_285 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_285, 0, x_283); +lean_ctor_set(x_285, 1, x_284); +x_286 = lean_array_mk(x_285); +x_287 = l_Array_append___rarg(x_11, x_286); +lean_dec(x_286); +x_12 = x_282; +x_13 = x_287; +goto block_278; } } } } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanConfig(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanConfig___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_1, 1); -lean_inc(x_26); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); lean_dec(x_1); -x_27 = l_Lake_LeanConfig_decodeToml(x_26); -return x_27; +x_21 = l_Lake_LeanConfig_decodeToml(x_20); +return x_21; } default: { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_1); -if (x_28 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_1, 1); -lean_dec(x_29); -x_30 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_mk_array(x_31, x_1); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +lean_ctor_set(x_1, 1, x_24); +x_2 = x_1; +goto block_7; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); lean_dec(x_1); -x_35 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_39, 0, x_38); -return x_39; +x_26 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_2 = x_27; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } } +static lean_object* _init_l_Lake_instDecodeTomlLeanConfig___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlLeanConfig___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_instDecodeTomlLeanConfig() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlLeanConfig___closed__1; +return x_1; } } LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_PackageConfig_decodeToml___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { @@ -8565,38 +8858,18 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_6, 1); -lean_inc(x_9); -lean_dec(x_6); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -x_11 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_12 = l_Lake_mergeErrors___rarg(x_4, x_10, x_11); -x_2 = x_8; -x_4 = x_12; -goto _start; -} -case 2: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_14 = lean_ctor_get(x_6, 0); -lean_inc(x_14); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_6, 1); +lean_inc(x_18); lean_dec(x_6); -x_15 = l_Lake_Glob_decodeToml___closed__2; -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); +x_19 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_19, 0, x_18); x_20 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; x_21 = l_Lake_mergeErrors___rarg(x_4, x_19, x_20); @@ -8604,9 +8877,9 @@ x_2 = x_8; x_4 = x_21; goto _start; } -case 3: +case 2: { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +lean_object* x_23; lean_object* x_24; lean_object* x_25; x_23 = lean_ctor_get(x_6, 0); lean_inc(x_23); lean_dec(x_6); @@ -8614,60 +8887,68 @@ x_24 = l_Lake_Glob_decodeToml___closed__2; x_25 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_25, 0, x_23); lean_ctor_set(x_25, 1, x_24); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_25); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_30 = l_Lake_mergeErrors___rarg(x_4, x_28, x_29); -x_2 = x_8; -x_4 = x_30; -goto _start; +x_9 = x_25; +goto block_17; +} +case 3: +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_6, 0); +lean_inc(x_26); +lean_dec(x_6); +x_27 = l_Lake_Glob_decodeToml___closed__2; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_9 = x_28; +goto block_17; } default: { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_6); -if (x_32 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_6); +if (x_29 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_33 = lean_ctor_get(x_6, 1); -lean_dec(x_33); -x_34 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_6, 1); +lean_dec(x_30); +x_31 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_34); -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_mk_array(x_35, x_6); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -x_38 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_39 = l_Lake_mergeErrors___rarg(x_4, x_37, x_38); -x_2 = x_8; -x_4 = x_39; -goto _start; +lean_ctor_set(x_6, 1, x_31); +x_9 = x_6; +goto block_17; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_41 = lean_ctor_get(x_6, 0); -lean_inc(x_41); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_6, 0); +lean_inc(x_32); lean_dec(x_6); -x_42 = l_Lake_Glob_decodeToml___closed__2; -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_unsigned_to_nat(1u); -x_45 = lean_mk_array(x_44, x_43); -x_46 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_47 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_48 = l_Lake_mergeErrors___rarg(x_4, x_46, x_47); -x_2 = x_8; -x_4 = x_48; -goto _start; +x_33 = l_Lake_Glob_decodeToml___closed__2; +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_9 = x_34; +goto block_17; } } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; +} } else { @@ -8720,7 +9001,7 @@ lean_inc(x_2); x_5 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_4, x_2, x_1); if (lean_obj_tag(x_5) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_6 = l_Lake_Toml_ppKey(x_2); lean_dec(x_2); x_7 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__2; @@ -8731,25 +9012,28 @@ x_10 = lean_string_append(x_8, x_9); x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_3); lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_3); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_ctor_get(x_15, 1); +x_16 = lean_ctor_get(x_5, 0); lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lake_Toml_decodeKeyval___at_Lake_StrPat_decodeToml___spec__4(x_2, x_16); +lean_dec(x_5); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lake_Toml_decodeKeyval___at_Lake_StrPat_decodeToml___spec__4(x_2, x_17); lean_dec(x_2); -return x_17; +return x_18; } } } @@ -8850,33 +9134,33 @@ static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__10() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("readmeFile", 10, 10); +x_1 = lean_mk_string_unchecked("README.md", 9, 9); return x_1; } } static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__11() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("readmeFile", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__12() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lake_PackageConfig_decodeToml___closed__10; +x_2 = l_Lake_PackageConfig_decodeToml___closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__12() { +static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__13() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("README.md", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("licenseFiles", 12, 12); +x_1 = lean_mk_string_unchecked("licenseFiles", 12, 12); return x_1; } } @@ -9289,26 +9573,26 @@ static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__58() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("srcDir", 6, 6); +x_1 = lean_mk_string_unchecked(".", 1, 1); return x_1; } } static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__59() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_PackageConfig_decodeToml___closed__58; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("srcDir", 6, 6); +return x_1; } } static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__60() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(".", 1, 1); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_PackageConfig_decodeToml___closed__59; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } static lean_object* _init_l_Lake_PackageConfig_decodeToml___closed__61() { @@ -9332,34 +9616,34 @@ return x_3; LEAN_EXPORT lean_object* l_Lake_PackageConfig_decodeToml(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_1119; lean_object* x_1120; -x_1119 = l_Lake_LeanOption_decodeToml___closed__10; +lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_827; lean_object* x_828; +x_827 = l_Lake_LeanOption_decodeToml___closed__10; lean_inc(x_1); -x_1120 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_1119, x_2); -if (lean_obj_tag(x_1120) == 0) +x_828 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_827, x_2); +if (lean_obj_tag(x_828) == 0) { -lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; lean_object* x_1124; -x_1121 = lean_ctor_get(x_1120, 0); -lean_inc(x_1121); -lean_dec(x_1120); -x_1122 = l_Lake_LeanOption_decodeToml___closed__3; -x_1123 = l_Array_append___rarg(x_1122, x_1121); -lean_dec(x_1121); -x_1124 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_1124; -x_10 = x_1123; -goto block_1118; -} -else -{ -lean_object* x_1125; lean_object* x_1126; -x_1125 = lean_ctor_get(x_1120, 0); -lean_inc(x_1125); -lean_dec(x_1120); -x_1126 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_1125; -x_10 = x_1126; -goto block_1118; +lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; +x_829 = lean_ctor_get(x_828, 0); +lean_inc(x_829); +lean_dec(x_828); +x_830 = l_Lake_LeanOption_decodeToml___closed__3; +x_831 = l_Array_append___rarg(x_830, x_829); +lean_dec(x_829); +x_832 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_832; +x_10 = x_831; +goto block_826; +} +else +{ +lean_object* x_833; lean_object* x_834; +x_833 = lean_ctor_get(x_828, 0); +lean_inc(x_833); +lean_dec(x_828); +x_834 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_833; +x_10 = x_834; +goto block_826; } block_8: { @@ -9382,3655 +9666,3325 @@ lean_ctor_set(x_7, 0, x_3); return x_7; } } -block_1118: +block_826: { -lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_1076; lean_object* x_1077; lean_object* x_1078; +lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_797; lean_object* x_804; lean_object* x_805; lean_object* x_806; x_11 = l_Lake_stringToLegalOrSimpleName(x_9); -x_1076 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_1077 = l_Lake_PackageConfig_decodeToml___closed__62; +x_804 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_805 = l_Lake_PackageConfig_decodeToml___closed__62; lean_inc(x_1); -x_1078 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1076, x_1077, x_1); -if (lean_obj_tag(x_1078) == 0) +x_806 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_804, x_805, x_1); +if (lean_obj_tag(x_806) == 0) { -uint8_t x_1079; -x_1079 = 0; -x_12 = x_1079; +uint8_t x_807; +x_807 = 0; +x_12 = x_807; x_13 = x_10; -goto block_1075; +goto block_796; } else { -lean_object* x_1080; lean_object* x_1081; -x_1080 = lean_ctor_get(x_1078, 0); -lean_inc(x_1080); -lean_dec(x_1078); -x_1081 = lean_ctor_get(x_1080, 1); -lean_inc(x_1081); -lean_dec(x_1080); -switch (lean_obj_tag(x_1081)) { +lean_object* x_808; lean_object* x_809; +x_808 = lean_ctor_get(x_806, 0); +lean_inc(x_808); +lean_dec(x_806); +x_809 = lean_ctor_get(x_808, 1); +lean_inc(x_809); +lean_dec(x_808); +switch (lean_obj_tag(x_809)) { case 0: { -uint8_t x_1082; -x_1082 = !lean_is_exclusive(x_1081); -if (x_1082 == 0) -{ -lean_object* x_1083; lean_object* x_1084; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; uint8_t x_1088; -x_1083 = lean_ctor_get(x_1081, 1); -lean_dec(x_1083); -x_1084 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_1081, 1, x_1084); -x_1085 = lean_unsigned_to_nat(1u); -x_1086 = lean_mk_array(x_1085, x_1081); -x_1087 = l_Array_append___rarg(x_10, x_1086); -lean_dec(x_1086); -x_1088 = 0; -x_12 = x_1088; -x_13 = x_1087; -goto block_1075; -} -else -{ -lean_object* x_1089; lean_object* x_1090; lean_object* x_1091; lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; uint8_t x_1095; -x_1089 = lean_ctor_get(x_1081, 0); -lean_inc(x_1089); -lean_dec(x_1081); -x_1090 = l_Lake_LeanConfig_decodeToml___closed__20; -x_1091 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1091, 0, x_1089); -lean_ctor_set(x_1091, 1, x_1090); -x_1092 = lean_unsigned_to_nat(1u); -x_1093 = lean_mk_array(x_1092, x_1091); -x_1094 = l_Array_append___rarg(x_10, x_1093); -lean_dec(x_1093); -x_1095 = 0; -x_12 = x_1095; -x_13 = x_1094; -goto block_1075; +uint8_t x_810; +x_810 = !lean_is_exclusive(x_809); +if (x_810 == 0) +{ +lean_object* x_811; lean_object* x_812; +x_811 = lean_ctor_get(x_809, 1); +lean_dec(x_811); +x_812 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_809, 1, x_812); +x_797 = x_809; +goto block_803; +} +else +{ +lean_object* x_813; lean_object* x_814; lean_object* x_815; +x_813 = lean_ctor_get(x_809, 0); +lean_inc(x_813); +lean_dec(x_809); +x_814 = l_Lake_LeanConfig_decodeToml___closed__20; +x_815 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_815, 0, x_813); +lean_ctor_set(x_815, 1, x_814); +x_797 = x_815; +goto block_803; } } case 2: { -lean_object* x_1096; lean_object* x_1097; lean_object* x_1098; lean_object* x_1099; lean_object* x_1100; lean_object* x_1101; uint8_t x_1102; -x_1096 = lean_ctor_get(x_1081, 0); -lean_inc(x_1096); -lean_dec(x_1081); -x_1097 = l_Lake_LeanConfig_decodeToml___closed__20; -x_1098 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1098, 0, x_1096); -lean_ctor_set(x_1098, 1, x_1097); -x_1099 = lean_unsigned_to_nat(1u); -x_1100 = lean_mk_array(x_1099, x_1098); -x_1101 = l_Array_append___rarg(x_10, x_1100); -lean_dec(x_1100); -x_1102 = 0; -x_12 = x_1102; -x_13 = x_1101; -goto block_1075; +lean_object* x_816; lean_object* x_817; lean_object* x_818; +x_816 = lean_ctor_get(x_809, 0); +lean_inc(x_816); +lean_dec(x_809); +x_817 = l_Lake_LeanConfig_decodeToml___closed__20; +x_818 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_818, 0, x_816); +lean_ctor_set(x_818, 1, x_817); +x_797 = x_818; +goto block_803; } case 3: { -uint8_t x_1103; -x_1103 = lean_ctor_get_uint8(x_1081, sizeof(void*)*1); -lean_dec(x_1081); -x_12 = x_1103; +uint8_t x_819; +x_819 = lean_ctor_get_uint8(x_809, sizeof(void*)*1); +lean_dec(x_809); +x_12 = x_819; x_13 = x_10; -goto block_1075; +goto block_796; } default: { -uint8_t x_1104; -x_1104 = !lean_is_exclusive(x_1081); -if (x_1104 == 0) -{ -lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; lean_object* x_1109; uint8_t x_1110; -x_1105 = lean_ctor_get(x_1081, 1); -lean_dec(x_1105); -x_1106 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_1081, 0); -lean_ctor_set(x_1081, 1, x_1106); -x_1107 = lean_unsigned_to_nat(1u); -x_1108 = lean_mk_array(x_1107, x_1081); -x_1109 = l_Array_append___rarg(x_10, x_1108); -lean_dec(x_1108); -x_1110 = 0; -x_12 = x_1110; -x_13 = x_1109; -goto block_1075; -} -else -{ -lean_object* x_1111; lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; lean_object* x_1115; lean_object* x_1116; uint8_t x_1117; -x_1111 = lean_ctor_get(x_1081, 0); -lean_inc(x_1111); -lean_dec(x_1081); -x_1112 = l_Lake_LeanConfig_decodeToml___closed__20; -x_1113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1113, 0, x_1111); -lean_ctor_set(x_1113, 1, x_1112); -x_1114 = lean_unsigned_to_nat(1u); -x_1115 = lean_mk_array(x_1114, x_1113); -x_1116 = l_Array_append___rarg(x_10, x_1115); -lean_dec(x_1115); -x_1117 = 0; -x_12 = x_1117; -x_13 = x_1116; -goto block_1075; +uint8_t x_820; +x_820 = !lean_is_exclusive(x_809); +if (x_820 == 0) +{ +lean_object* x_821; lean_object* x_822; +x_821 = lean_ctor_get(x_809, 1); +lean_dec(x_821); +x_822 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_809, 0); +lean_ctor_set(x_809, 1, x_822); +x_797 = x_809; +goto block_803; +} +else +{ +lean_object* x_823; lean_object* x_824; lean_object* x_825; +x_823 = lean_ctor_get(x_809, 0); +lean_inc(x_823); +lean_dec(x_809); +x_824 = l_Lake_LeanConfig_decodeToml___closed__20; +x_825 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_825, 0, x_823); +lean_ctor_set(x_825, 1, x_824); +x_797 = x_825; +goto block_803; } } } } -block_1075: +block_796: { -lean_object* x_14; lean_object* x_15; lean_object* x_1021; lean_object* x_1022; lean_object* x_1023; -x_1021 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_1022 = l_Lake_PackageConfig_decodeToml___closed__2; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_760; lean_object* x_766; lean_object* x_767; lean_object* x_768; +x_14 = lean_box(0); +x_766 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_767 = l_Lake_PackageConfig_decodeToml___closed__2; lean_inc(x_1); -x_1023 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1021, x_1022, x_1); -if (lean_obj_tag(x_1023) == 0) +x_768 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_766, x_767, x_1); +if (lean_obj_tag(x_768) == 0) { -lean_object* x_1024; -x_1024 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1024; -x_15 = x_13; -goto block_1020; +lean_object* x_769; +x_769 = l_Lake_decodeLeanOptions___closed__1; +x_15 = x_769; +x_16 = x_13; +goto block_759; } else { -lean_object* x_1025; lean_object* x_1026; -x_1025 = lean_ctor_get(x_1023, 0); -lean_inc(x_1025); -lean_dec(x_1023); -x_1026 = lean_ctor_get(x_1025, 1); -lean_inc(x_1026); -lean_dec(x_1025); -switch (lean_obj_tag(x_1026)) { +lean_object* x_770; lean_object* x_771; +x_770 = lean_ctor_get(x_768, 0); +lean_inc(x_770); +lean_dec(x_768); +x_771 = lean_ctor_get(x_770, 1); +lean_inc(x_771); +lean_dec(x_770); +switch (lean_obj_tag(x_771)) { case 0: { -uint8_t x_1027; -x_1027 = !lean_is_exclusive(x_1026); -if (x_1027 == 0) -{ -lean_object* x_1028; lean_object* x_1029; lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; lean_object* x_1033; -x_1028 = lean_ctor_get(x_1026, 1); -lean_dec(x_1028); -x_1029 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_1026, 1, x_1029); -x_1030 = lean_unsigned_to_nat(1u); -x_1031 = lean_mk_array(x_1030, x_1026); -x_1032 = l_Array_append___rarg(x_13, x_1031); -lean_dec(x_1031); -x_1033 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1033; -x_15 = x_1032; -goto block_1020; -} -else -{ -lean_object* x_1034; lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; -x_1034 = lean_ctor_get(x_1026, 0); -lean_inc(x_1034); -lean_dec(x_1026); -x_1035 = l_Lake_LeanConfig_decodeToml___closed__5; -x_1036 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1036, 0, x_1034); -lean_ctor_set(x_1036, 1, x_1035); -x_1037 = lean_unsigned_to_nat(1u); -x_1038 = lean_mk_array(x_1037, x_1036); -x_1039 = l_Array_append___rarg(x_13, x_1038); -lean_dec(x_1038); -x_1040 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1040; -x_15 = x_1039; -goto block_1020; +uint8_t x_772; +x_772 = !lean_is_exclusive(x_771); +if (x_772 == 0) +{ +lean_object* x_773; lean_object* x_774; +x_773 = lean_ctor_get(x_771, 1); +lean_dec(x_773); +x_774 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_771, 1, x_774); +x_760 = x_771; +goto block_765; +} +else +{ +lean_object* x_775; lean_object* x_776; lean_object* x_777; +x_775 = lean_ctor_get(x_771, 0); +lean_inc(x_775); +lean_dec(x_771); +x_776 = l_Lake_LeanConfig_decodeToml___closed__5; +x_777 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_777, 0, x_775); +lean_ctor_set(x_777, 1, x_776); +x_760 = x_777; +goto block_765; } } case 2: { -lean_object* x_1041; lean_object* x_1042; lean_object* x_1043; lean_object* x_1044; lean_object* x_1045; lean_object* x_1046; lean_object* x_1047; -x_1041 = lean_ctor_get(x_1026, 0); -lean_inc(x_1041); -lean_dec(x_1026); -x_1042 = l_Lake_LeanConfig_decodeToml___closed__5; -x_1043 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1043, 0, x_1041); -lean_ctor_set(x_1043, 1, x_1042); -x_1044 = lean_unsigned_to_nat(1u); -x_1045 = lean_mk_array(x_1044, x_1043); -x_1046 = l_Array_append___rarg(x_13, x_1045); -lean_dec(x_1045); -x_1047 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1047; -x_15 = x_1046; -goto block_1020; +lean_object* x_778; lean_object* x_779; lean_object* x_780; +x_778 = lean_ctor_get(x_771, 0); +lean_inc(x_778); +lean_dec(x_771); +x_779 = l_Lake_LeanConfig_decodeToml___closed__5; +x_780 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_780, 0, x_778); +lean_ctor_set(x_780, 1, x_779); +x_760 = x_780; +goto block_765; } case 3: { -lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; lean_object* x_1051; lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; -x_1048 = lean_ctor_get(x_1026, 0); -lean_inc(x_1048); -lean_dec(x_1026); -x_1049 = l_Lake_LeanConfig_decodeToml___closed__5; -x_1050 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1050, 0, x_1048); -lean_ctor_set(x_1050, 1, x_1049); -x_1051 = lean_unsigned_to_nat(1u); -x_1052 = lean_mk_array(x_1051, x_1050); -x_1053 = l_Array_append___rarg(x_13, x_1052); -lean_dec(x_1052); -x_1054 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1054; -x_15 = x_1053; -goto block_1020; +lean_object* x_781; lean_object* x_782; lean_object* x_783; +x_781 = lean_ctor_get(x_771, 0); +lean_inc(x_781); +lean_dec(x_771); +x_782 = l_Lake_LeanConfig_decodeToml___closed__5; +x_783 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_783, 0, x_781); +lean_ctor_set(x_783, 1, x_782); +x_760 = x_783; +goto block_765; } case 5: { -lean_object* x_1055; lean_object* x_1056; -x_1055 = lean_ctor_get(x_1026, 1); -lean_inc(x_1055); -lean_dec(x_1026); -x_1056 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_1055); -lean_dec(x_1055); -if (lean_obj_tag(x_1056) == 0) -{ -lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; -x_1057 = lean_ctor_get(x_1056, 0); -lean_inc(x_1057); -lean_dec(x_1056); -x_1058 = l_Array_append___rarg(x_13, x_1057); -lean_dec(x_1057); -x_1059 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1059; -x_15 = x_1058; -goto block_1020; -} -else -{ -lean_object* x_1060; -x_1060 = lean_ctor_get(x_1056, 0); -lean_inc(x_1060); -lean_dec(x_1056); -x_14 = x_1060; -x_15 = x_13; -goto block_1020; +lean_object* x_784; lean_object* x_785; +x_784 = lean_ctor_get(x_771, 1); +lean_inc(x_784); +lean_dec(x_771); +x_785 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_784); +lean_dec(x_784); +if (lean_obj_tag(x_785) == 0) +{ +lean_object* x_786; lean_object* x_787; lean_object* x_788; +x_786 = lean_ctor_get(x_785, 0); +lean_inc(x_786); +lean_dec(x_785); +x_787 = l_Array_append___rarg(x_13, x_786); +lean_dec(x_786); +x_788 = l_Lake_decodeLeanOptions___closed__1; +x_15 = x_788; +x_16 = x_787; +goto block_759; +} +else +{ +lean_object* x_789; +x_789 = lean_ctor_get(x_785, 0); +lean_inc(x_789); +lean_dec(x_785); +x_15 = x_789; +x_16 = x_13; +goto block_759; } } default: { -uint8_t x_1061; -x_1061 = !lean_is_exclusive(x_1026); -if (x_1061 == 0) +uint8_t x_790; +x_790 = !lean_is_exclusive(x_771); +if (x_790 == 0) { -lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; lean_object* x_1065; lean_object* x_1066; lean_object* x_1067; -x_1062 = lean_ctor_get(x_1026, 1); -lean_dec(x_1062); -x_1063 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_1026, 0); -lean_ctor_set(x_1026, 1, x_1063); -x_1064 = lean_unsigned_to_nat(1u); -x_1065 = lean_mk_array(x_1064, x_1026); -x_1066 = l_Array_append___rarg(x_13, x_1065); -lean_dec(x_1065); -x_1067 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1067; -x_15 = x_1066; -goto block_1020; -} -else -{ -lean_object* x_1068; lean_object* x_1069; lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; lean_object* x_1073; lean_object* x_1074; -x_1068 = lean_ctor_get(x_1026, 0); -lean_inc(x_1068); -lean_dec(x_1026); -x_1069 = l_Lake_LeanConfig_decodeToml___closed__5; -x_1070 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1070, 0, x_1068); -lean_ctor_set(x_1070, 1, x_1069); -x_1071 = lean_unsigned_to_nat(1u); -x_1072 = lean_mk_array(x_1071, x_1070); -x_1073 = l_Array_append___rarg(x_13, x_1072); -lean_dec(x_1072); -x_1074 = l_Lake_decodeLeanOptions___closed__1; -x_14 = x_1074; -x_15 = x_1073; -goto block_1020; -} -} -} -} -block_1020: -{ -lean_object* x_16; lean_object* x_17; lean_object* x_985; lean_object* x_986; lean_object* x_987; -x_985 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_986 = l_Lake_PackageConfig_decodeToml___closed__59; +lean_object* x_791; lean_object* x_792; +x_791 = lean_ctor_get(x_771, 1); +lean_dec(x_791); +x_792 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_771, 0); +lean_ctor_set(x_771, 1, x_792); +x_760 = x_771; +goto block_765; +} +else +{ +lean_object* x_793; lean_object* x_794; lean_object* x_795; +x_793 = lean_ctor_get(x_771, 0); +lean_inc(x_793); +lean_dec(x_771); +x_794 = l_Lake_LeanConfig_decodeToml___closed__5; +x_795 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_795, 0, x_793); +lean_ctor_set(x_795, 1, x_794); +x_760 = x_795; +goto block_765; +} +} +} +} +block_759: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_734; lean_object* x_740; lean_object* x_741; lean_object* x_742; +x_740 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_741 = l_Lake_PackageConfig_decodeToml___closed__60; lean_inc(x_1); -x_987 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_985, x_986, x_1); -if (lean_obj_tag(x_987) == 0) +x_742 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_740, x_741, x_1); +if (lean_obj_tag(x_742) == 0) { -lean_object* x_988; -x_988 = l_Lake_PackageConfig_decodeToml___closed__60; -x_16 = x_988; -x_17 = x_15; -goto block_984; +lean_object* x_743; +x_743 = l_Lake_PackageConfig_decodeToml___closed__58; +x_17 = x_743; +x_18 = x_16; +goto block_733; } else { -lean_object* x_989; lean_object* x_990; -x_989 = lean_ctor_get(x_987, 0); -lean_inc(x_989); -lean_dec(x_987); -x_990 = lean_ctor_get(x_989, 1); -lean_inc(x_990); -lean_dec(x_989); -switch (lean_obj_tag(x_990)) { +lean_object* x_744; lean_object* x_745; +x_744 = lean_ctor_get(x_742, 0); +lean_inc(x_744); +lean_dec(x_742); +x_745 = lean_ctor_get(x_744, 1); +lean_inc(x_745); +lean_dec(x_744); +switch (lean_obj_tag(x_745)) { case 0: { -lean_object* x_991; -x_991 = lean_ctor_get(x_990, 1); -lean_inc(x_991); -lean_dec(x_990); -x_16 = x_991; -x_17 = x_15; -goto block_984; +lean_object* x_746; +x_746 = lean_ctor_get(x_745, 1); +lean_inc(x_746); +lean_dec(x_745); +x_17 = x_746; +x_18 = x_16; +goto block_733; } case 2: { -lean_object* x_992; lean_object* x_993; lean_object* x_994; lean_object* x_995; lean_object* x_996; lean_object* x_997; lean_object* x_998; -x_992 = lean_ctor_get(x_990, 0); -lean_inc(x_992); -lean_dec(x_990); -x_993 = l_Lake_Glob_decodeToml___closed__2; -x_994 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_994, 0, x_992); -lean_ctor_set(x_994, 1, x_993); -x_995 = lean_unsigned_to_nat(1u); -x_996 = lean_mk_array(x_995, x_994); -x_997 = l_Array_append___rarg(x_15, x_996); -lean_dec(x_996); -x_998 = l_Lake_PackageConfig_decodeToml___closed__60; -x_16 = x_998; -x_17 = x_997; -goto block_984; +lean_object* x_747; lean_object* x_748; lean_object* x_749; +x_747 = lean_ctor_get(x_745, 0); +lean_inc(x_747); +lean_dec(x_745); +x_748 = l_Lake_Glob_decodeToml___closed__2; +x_749 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_749, 0, x_747); +lean_ctor_set(x_749, 1, x_748); +x_734 = x_749; +goto block_739; } case 3: { -lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; lean_object* x_1005; -x_999 = lean_ctor_get(x_990, 0); -lean_inc(x_999); -lean_dec(x_990); -x_1000 = l_Lake_Glob_decodeToml___closed__2; -x_1001 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1001, 0, x_999); -lean_ctor_set(x_1001, 1, x_1000); -x_1002 = lean_unsigned_to_nat(1u); -x_1003 = lean_mk_array(x_1002, x_1001); -x_1004 = l_Array_append___rarg(x_15, x_1003); -lean_dec(x_1003); -x_1005 = l_Lake_PackageConfig_decodeToml___closed__60; -x_16 = x_1005; -x_17 = x_1004; -goto block_984; +lean_object* x_750; lean_object* x_751; lean_object* x_752; +x_750 = lean_ctor_get(x_745, 0); +lean_inc(x_750); +lean_dec(x_745); +x_751 = l_Lake_Glob_decodeToml___closed__2; +x_752 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_752, 0, x_750); +lean_ctor_set(x_752, 1, x_751); +x_734 = x_752; +goto block_739; } default: { -uint8_t x_1006; -x_1006 = !lean_is_exclusive(x_990); -if (x_1006 == 0) -{ -lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; lean_object* x_1011; lean_object* x_1012; -x_1007 = lean_ctor_get(x_990, 1); -lean_dec(x_1007); -x_1008 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_990, 0); -lean_ctor_set(x_990, 1, x_1008); -x_1009 = lean_unsigned_to_nat(1u); -x_1010 = lean_mk_array(x_1009, x_990); -x_1011 = l_Array_append___rarg(x_15, x_1010); -lean_dec(x_1010); -x_1012 = l_Lake_PackageConfig_decodeToml___closed__60; -x_16 = x_1012; -x_17 = x_1011; -goto block_984; -} -else -{ -lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; -x_1013 = lean_ctor_get(x_990, 0); -lean_inc(x_1013); -lean_dec(x_990); -x_1014 = l_Lake_Glob_decodeToml___closed__2; -x_1015 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1015, 0, x_1013); -lean_ctor_set(x_1015, 1, x_1014); -x_1016 = lean_unsigned_to_nat(1u); -x_1017 = lean_mk_array(x_1016, x_1015); -x_1018 = l_Array_append___rarg(x_15, x_1017); -lean_dec(x_1017); -x_1019 = l_Lake_PackageConfig_decodeToml___closed__60; -x_16 = x_1019; -x_17 = x_1018; -goto block_984; -} -} -} -} -block_984: -{ -lean_object* x_18; lean_object* x_19; lean_object* x_949; lean_object* x_950; lean_object* x_951; -x_949 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_950 = l_Lake_PackageConfig_decodeToml___closed__57; +uint8_t x_753; +x_753 = !lean_is_exclusive(x_745); +if (x_753 == 0) +{ +lean_object* x_754; lean_object* x_755; +x_754 = lean_ctor_get(x_745, 1); +lean_dec(x_754); +x_755 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_745, 0); +lean_ctor_set(x_745, 1, x_755); +x_734 = x_745; +goto block_739; +} +else +{ +lean_object* x_756; lean_object* x_757; lean_object* x_758; +x_756 = lean_ctor_get(x_745, 0); +lean_inc(x_756); +lean_dec(x_745); +x_757 = l_Lake_Glob_decodeToml___closed__2; +x_758 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_758, 0, x_756); +lean_ctor_set(x_758, 1, x_757); +x_734 = x_758; +goto block_739; +} +} +} +} +block_733: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_708; lean_object* x_714; lean_object* x_715; lean_object* x_716; +x_714 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_715 = l_Lake_PackageConfig_decodeToml___closed__57; lean_inc(x_1); -x_951 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_949, x_950, x_1); -if (lean_obj_tag(x_951) == 0) +x_716 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_714, x_715, x_1); +if (lean_obj_tag(x_716) == 0) { -lean_object* x_952; -x_952 = l_Lake_defaultBuildDir; -x_18 = x_952; -x_19 = x_17; -goto block_948; +lean_object* x_717; +x_717 = l_Lake_defaultBuildDir; +x_19 = x_717; +x_20 = x_18; +goto block_707; } else { -lean_object* x_953; lean_object* x_954; -x_953 = lean_ctor_get(x_951, 0); -lean_inc(x_953); -lean_dec(x_951); -x_954 = lean_ctor_get(x_953, 1); -lean_inc(x_954); -lean_dec(x_953); -switch (lean_obj_tag(x_954)) { +lean_object* x_718; lean_object* x_719; +x_718 = lean_ctor_get(x_716, 0); +lean_inc(x_718); +lean_dec(x_716); +x_719 = lean_ctor_get(x_718, 1); +lean_inc(x_719); +lean_dec(x_718); +switch (lean_obj_tag(x_719)) { case 0: { -lean_object* x_955; -x_955 = lean_ctor_get(x_954, 1); -lean_inc(x_955); -lean_dec(x_954); -x_18 = x_955; -x_19 = x_17; -goto block_948; +lean_object* x_720; +x_720 = lean_ctor_get(x_719, 1); +lean_inc(x_720); +lean_dec(x_719); +x_19 = x_720; +x_20 = x_18; +goto block_707; } case 2: { -lean_object* x_956; lean_object* x_957; lean_object* x_958; lean_object* x_959; lean_object* x_960; lean_object* x_961; lean_object* x_962; -x_956 = lean_ctor_get(x_954, 0); -lean_inc(x_956); -lean_dec(x_954); -x_957 = l_Lake_Glob_decodeToml___closed__2; -x_958 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_958, 0, x_956); -lean_ctor_set(x_958, 1, x_957); -x_959 = lean_unsigned_to_nat(1u); -x_960 = lean_mk_array(x_959, x_958); -x_961 = l_Array_append___rarg(x_17, x_960); -lean_dec(x_960); -x_962 = l_Lake_defaultBuildDir; -x_18 = x_962; -x_19 = x_961; -goto block_948; +lean_object* x_721; lean_object* x_722; lean_object* x_723; +x_721 = lean_ctor_get(x_719, 0); +lean_inc(x_721); +lean_dec(x_719); +x_722 = l_Lake_Glob_decodeToml___closed__2; +x_723 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_723, 0, x_721); +lean_ctor_set(x_723, 1, x_722); +x_708 = x_723; +goto block_713; } case 3: { -lean_object* x_963; lean_object* x_964; lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; -x_963 = lean_ctor_get(x_954, 0); -lean_inc(x_963); -lean_dec(x_954); -x_964 = l_Lake_Glob_decodeToml___closed__2; -x_965 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_965, 0, x_963); -lean_ctor_set(x_965, 1, x_964); -x_966 = lean_unsigned_to_nat(1u); -x_967 = lean_mk_array(x_966, x_965); -x_968 = l_Array_append___rarg(x_17, x_967); -lean_dec(x_967); -x_969 = l_Lake_defaultBuildDir; -x_18 = x_969; -x_19 = x_968; -goto block_948; +lean_object* x_724; lean_object* x_725; lean_object* x_726; +x_724 = lean_ctor_get(x_719, 0); +lean_inc(x_724); +lean_dec(x_719); +x_725 = l_Lake_Glob_decodeToml___closed__2; +x_726 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_726, 0, x_724); +lean_ctor_set(x_726, 1, x_725); +x_708 = x_726; +goto block_713; } default: { -uint8_t x_970; -x_970 = !lean_is_exclusive(x_954); -if (x_970 == 0) -{ -lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; -x_971 = lean_ctor_get(x_954, 1); -lean_dec(x_971); -x_972 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_954, 0); -lean_ctor_set(x_954, 1, x_972); -x_973 = lean_unsigned_to_nat(1u); -x_974 = lean_mk_array(x_973, x_954); -x_975 = l_Array_append___rarg(x_17, x_974); -lean_dec(x_974); -x_976 = l_Lake_defaultBuildDir; -x_18 = x_976; -x_19 = x_975; -goto block_948; +uint8_t x_727; +x_727 = !lean_is_exclusive(x_719); +if (x_727 == 0) +{ +lean_object* x_728; lean_object* x_729; +x_728 = lean_ctor_get(x_719, 1); +lean_dec(x_728); +x_729 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_719, 0); +lean_ctor_set(x_719, 1, x_729); +x_708 = x_719; +goto block_713; } else { -lean_object* x_977; lean_object* x_978; lean_object* x_979; lean_object* x_980; lean_object* x_981; lean_object* x_982; lean_object* x_983; -x_977 = lean_ctor_get(x_954, 0); -lean_inc(x_977); -lean_dec(x_954); -x_978 = l_Lake_Glob_decodeToml___closed__2; -x_979 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_979, 0, x_977); -lean_ctor_set(x_979, 1, x_978); -x_980 = lean_unsigned_to_nat(1u); -x_981 = lean_mk_array(x_980, x_979); -x_982 = l_Array_append___rarg(x_17, x_981); -lean_dec(x_981); -x_983 = l_Lake_defaultBuildDir; -x_18 = x_983; -x_19 = x_982; -goto block_948; +lean_object* x_730; lean_object* x_731; lean_object* x_732; +x_730 = lean_ctor_get(x_719, 0); +lean_inc(x_730); +lean_dec(x_719); +x_731 = l_Lake_Glob_decodeToml___closed__2; +x_732 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_732, 0, x_730); +lean_ctor_set(x_732, 1, x_731); +x_708 = x_732; +goto block_713; } } } } -block_948: +block_707: { -lean_object* x_20; lean_object* x_21; lean_object* x_913; lean_object* x_914; lean_object* x_915; -x_913 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_914 = l_Lake_PackageConfig_decodeToml___closed__55; +lean_object* x_21; lean_object* x_22; lean_object* x_682; lean_object* x_688; lean_object* x_689; lean_object* x_690; +x_688 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_689 = l_Lake_PackageConfig_decodeToml___closed__55; lean_inc(x_1); -x_915 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_913, x_914, x_1); -if (lean_obj_tag(x_915) == 0) +x_690 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_688, x_689, x_1); +if (lean_obj_tag(x_690) == 0) { -lean_object* x_916; -x_916 = l_Lake_defaultLeanLibDir; -x_20 = x_916; -x_21 = x_19; -goto block_912; +lean_object* x_691; +x_691 = l_Lake_defaultLeanLibDir; +x_21 = x_691; +x_22 = x_20; +goto block_681; } else { -lean_object* x_917; lean_object* x_918; -x_917 = lean_ctor_get(x_915, 0); -lean_inc(x_917); -lean_dec(x_915); -x_918 = lean_ctor_get(x_917, 1); -lean_inc(x_918); -lean_dec(x_917); -switch (lean_obj_tag(x_918)) { +lean_object* x_692; lean_object* x_693; +x_692 = lean_ctor_get(x_690, 0); +lean_inc(x_692); +lean_dec(x_690); +x_693 = lean_ctor_get(x_692, 1); +lean_inc(x_693); +lean_dec(x_692); +switch (lean_obj_tag(x_693)) { case 0: { -lean_object* x_919; -x_919 = lean_ctor_get(x_918, 1); -lean_inc(x_919); -lean_dec(x_918); -x_20 = x_919; -x_21 = x_19; -goto block_912; +lean_object* x_694; +x_694 = lean_ctor_get(x_693, 1); +lean_inc(x_694); +lean_dec(x_693); +x_21 = x_694; +x_22 = x_20; +goto block_681; } case 2: { -lean_object* x_920; lean_object* x_921; lean_object* x_922; lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; -x_920 = lean_ctor_get(x_918, 0); -lean_inc(x_920); -lean_dec(x_918); -x_921 = l_Lake_Glob_decodeToml___closed__2; -x_922 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_922, 0, x_920); -lean_ctor_set(x_922, 1, x_921); -x_923 = lean_unsigned_to_nat(1u); -x_924 = lean_mk_array(x_923, x_922); -x_925 = l_Array_append___rarg(x_19, x_924); -lean_dec(x_924); -x_926 = l_Lake_defaultLeanLibDir; -x_20 = x_926; -x_21 = x_925; -goto block_912; +lean_object* x_695; lean_object* x_696; lean_object* x_697; +x_695 = lean_ctor_get(x_693, 0); +lean_inc(x_695); +lean_dec(x_693); +x_696 = l_Lake_Glob_decodeToml___closed__2; +x_697 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_697, 0, x_695); +lean_ctor_set(x_697, 1, x_696); +x_682 = x_697; +goto block_687; } case 3: { -lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; lean_object* x_932; lean_object* x_933; -x_927 = lean_ctor_get(x_918, 0); -lean_inc(x_927); -lean_dec(x_918); -x_928 = l_Lake_Glob_decodeToml___closed__2; -x_929 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_929, 0, x_927); -lean_ctor_set(x_929, 1, x_928); -x_930 = lean_unsigned_to_nat(1u); -x_931 = lean_mk_array(x_930, x_929); -x_932 = l_Array_append___rarg(x_19, x_931); -lean_dec(x_931); -x_933 = l_Lake_defaultLeanLibDir; -x_20 = x_933; -x_21 = x_932; -goto block_912; +lean_object* x_698; lean_object* x_699; lean_object* x_700; +x_698 = lean_ctor_get(x_693, 0); +lean_inc(x_698); +lean_dec(x_693); +x_699 = l_Lake_Glob_decodeToml___closed__2; +x_700 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_700, 0, x_698); +lean_ctor_set(x_700, 1, x_699); +x_682 = x_700; +goto block_687; } default: { -uint8_t x_934; -x_934 = !lean_is_exclusive(x_918); -if (x_934 == 0) +uint8_t x_701; +x_701 = !lean_is_exclusive(x_693); +if (x_701 == 0) { -lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; lean_object* x_940; -x_935 = lean_ctor_get(x_918, 1); -lean_dec(x_935); -x_936 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_918, 0); -lean_ctor_set(x_918, 1, x_936); -x_937 = lean_unsigned_to_nat(1u); -x_938 = lean_mk_array(x_937, x_918); -x_939 = l_Array_append___rarg(x_19, x_938); -lean_dec(x_938); -x_940 = l_Lake_defaultLeanLibDir; -x_20 = x_940; -x_21 = x_939; -goto block_912; -} -else -{ -lean_object* x_941; lean_object* x_942; lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; -x_941 = lean_ctor_get(x_918, 0); -lean_inc(x_941); -lean_dec(x_918); -x_942 = l_Lake_Glob_decodeToml___closed__2; -x_943 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_943, 0, x_941); -lean_ctor_set(x_943, 1, x_942); -x_944 = lean_unsigned_to_nat(1u); -x_945 = lean_mk_array(x_944, x_943); -x_946 = l_Array_append___rarg(x_19, x_945); -lean_dec(x_945); -x_947 = l_Lake_defaultLeanLibDir; -x_20 = x_947; -x_21 = x_946; -goto block_912; -} -} -} -} -block_912: -{ -lean_object* x_22; lean_object* x_23; lean_object* x_877; lean_object* x_878; lean_object* x_879; -x_877 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_878 = l_Lake_PackageConfig_decodeToml___closed__53; +lean_object* x_702; lean_object* x_703; +x_702 = lean_ctor_get(x_693, 1); +lean_dec(x_702); +x_703 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_693, 0); +lean_ctor_set(x_693, 1, x_703); +x_682 = x_693; +goto block_687; +} +else +{ +lean_object* x_704; lean_object* x_705; lean_object* x_706; +x_704 = lean_ctor_get(x_693, 0); +lean_inc(x_704); +lean_dec(x_693); +x_705 = l_Lake_Glob_decodeToml___closed__2; +x_706 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_706, 0, x_704); +lean_ctor_set(x_706, 1, x_705); +x_682 = x_706; +goto block_687; +} +} +} +} +block_681: +{ +lean_object* x_23; lean_object* x_24; lean_object* x_656; lean_object* x_662; lean_object* x_663; lean_object* x_664; +x_662 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_663 = l_Lake_PackageConfig_decodeToml___closed__53; lean_inc(x_1); -x_879 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_877, x_878, x_1); -if (lean_obj_tag(x_879) == 0) +x_664 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_662, x_663, x_1); +if (lean_obj_tag(x_664) == 0) { -lean_object* x_880; -x_880 = l_Lake_defaultNativeLibDir; -x_22 = x_880; -x_23 = x_21; -goto block_876; +lean_object* x_665; +x_665 = l_Lake_defaultNativeLibDir; +x_23 = x_665; +x_24 = x_22; +goto block_655; } else { -lean_object* x_881; lean_object* x_882; -x_881 = lean_ctor_get(x_879, 0); -lean_inc(x_881); -lean_dec(x_879); -x_882 = lean_ctor_get(x_881, 1); -lean_inc(x_882); -lean_dec(x_881); -switch (lean_obj_tag(x_882)) { +lean_object* x_666; lean_object* x_667; +x_666 = lean_ctor_get(x_664, 0); +lean_inc(x_666); +lean_dec(x_664); +x_667 = lean_ctor_get(x_666, 1); +lean_inc(x_667); +lean_dec(x_666); +switch (lean_obj_tag(x_667)) { case 0: { -lean_object* x_883; -x_883 = lean_ctor_get(x_882, 1); -lean_inc(x_883); -lean_dec(x_882); -x_22 = x_883; -x_23 = x_21; -goto block_876; +lean_object* x_668; +x_668 = lean_ctor_get(x_667, 1); +lean_inc(x_668); +lean_dec(x_667); +x_23 = x_668; +x_24 = x_22; +goto block_655; } case 2: { -lean_object* x_884; lean_object* x_885; lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; -x_884 = lean_ctor_get(x_882, 0); -lean_inc(x_884); -lean_dec(x_882); -x_885 = l_Lake_Glob_decodeToml___closed__2; -x_886 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_886, 0, x_884); -lean_ctor_set(x_886, 1, x_885); -x_887 = lean_unsigned_to_nat(1u); -x_888 = lean_mk_array(x_887, x_886); -x_889 = l_Array_append___rarg(x_21, x_888); -lean_dec(x_888); -x_890 = l_Lake_defaultNativeLibDir; -x_22 = x_890; -x_23 = x_889; -goto block_876; +lean_object* x_669; lean_object* x_670; lean_object* x_671; +x_669 = lean_ctor_get(x_667, 0); +lean_inc(x_669); +lean_dec(x_667); +x_670 = l_Lake_Glob_decodeToml___closed__2; +x_671 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_671, 0, x_669); +lean_ctor_set(x_671, 1, x_670); +x_656 = x_671; +goto block_661; } case 3: { -lean_object* x_891; lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; lean_object* x_896; lean_object* x_897; -x_891 = lean_ctor_get(x_882, 0); -lean_inc(x_891); -lean_dec(x_882); -x_892 = l_Lake_Glob_decodeToml___closed__2; -x_893 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_893, 0, x_891); -lean_ctor_set(x_893, 1, x_892); -x_894 = lean_unsigned_to_nat(1u); -x_895 = lean_mk_array(x_894, x_893); -x_896 = l_Array_append___rarg(x_21, x_895); -lean_dec(x_895); -x_897 = l_Lake_defaultNativeLibDir; -x_22 = x_897; -x_23 = x_896; -goto block_876; +lean_object* x_672; lean_object* x_673; lean_object* x_674; +x_672 = lean_ctor_get(x_667, 0); +lean_inc(x_672); +lean_dec(x_667); +x_673 = l_Lake_Glob_decodeToml___closed__2; +x_674 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_674, 0, x_672); +lean_ctor_set(x_674, 1, x_673); +x_656 = x_674; +goto block_661; } default: { -uint8_t x_898; -x_898 = !lean_is_exclusive(x_882); -if (x_898 == 0) -{ -lean_object* x_899; lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; -x_899 = lean_ctor_get(x_882, 1); -lean_dec(x_899); -x_900 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_882, 0); -lean_ctor_set(x_882, 1, x_900); -x_901 = lean_unsigned_to_nat(1u); -x_902 = lean_mk_array(x_901, x_882); -x_903 = l_Array_append___rarg(x_21, x_902); -lean_dec(x_902); -x_904 = l_Lake_defaultNativeLibDir; -x_22 = x_904; -x_23 = x_903; -goto block_876; +uint8_t x_675; +x_675 = !lean_is_exclusive(x_667); +if (x_675 == 0) +{ +lean_object* x_676; lean_object* x_677; +x_676 = lean_ctor_get(x_667, 1); +lean_dec(x_676); +x_677 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_667, 0); +lean_ctor_set(x_667, 1, x_677); +x_656 = x_667; +goto block_661; } else { -lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; -x_905 = lean_ctor_get(x_882, 0); -lean_inc(x_905); -lean_dec(x_882); -x_906 = l_Lake_Glob_decodeToml___closed__2; -x_907 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_907, 0, x_905); -lean_ctor_set(x_907, 1, x_906); -x_908 = lean_unsigned_to_nat(1u); -x_909 = lean_mk_array(x_908, x_907); -x_910 = l_Array_append___rarg(x_21, x_909); -lean_dec(x_909); -x_911 = l_Lake_defaultNativeLibDir; -x_22 = x_911; -x_23 = x_910; -goto block_876; +lean_object* x_678; lean_object* x_679; lean_object* x_680; +x_678 = lean_ctor_get(x_667, 0); +lean_inc(x_678); +lean_dec(x_667); +x_679 = l_Lake_Glob_decodeToml___closed__2; +x_680 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_680, 0, x_678); +lean_ctor_set(x_680, 1, x_679); +x_656 = x_680; +goto block_661; } } } } -block_876: +block_655: { -lean_object* x_24; lean_object* x_25; lean_object* x_841; lean_object* x_842; lean_object* x_843; -x_841 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_842 = l_Lake_PackageConfig_decodeToml___closed__51; +lean_object* x_25; lean_object* x_26; lean_object* x_630; lean_object* x_636; lean_object* x_637; lean_object* x_638; +x_636 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_637 = l_Lake_PackageConfig_decodeToml___closed__51; lean_inc(x_1); -x_843 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_841, x_842, x_1); -if (lean_obj_tag(x_843) == 0) +x_638 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_636, x_637, x_1); +if (lean_obj_tag(x_638) == 0) { -lean_object* x_844; -x_844 = l_Lake_defaultBinDir; -x_24 = x_844; -x_25 = x_23; -goto block_840; +lean_object* x_639; +x_639 = l_Lake_defaultBinDir; +x_25 = x_639; +x_26 = x_24; +goto block_629; } else { -lean_object* x_845; lean_object* x_846; -x_845 = lean_ctor_get(x_843, 0); -lean_inc(x_845); -lean_dec(x_843); -x_846 = lean_ctor_get(x_845, 1); -lean_inc(x_846); -lean_dec(x_845); -switch (lean_obj_tag(x_846)) { +lean_object* x_640; lean_object* x_641; +x_640 = lean_ctor_get(x_638, 0); +lean_inc(x_640); +lean_dec(x_638); +x_641 = lean_ctor_get(x_640, 1); +lean_inc(x_641); +lean_dec(x_640); +switch (lean_obj_tag(x_641)) { case 0: { -lean_object* x_847; -x_847 = lean_ctor_get(x_846, 1); -lean_inc(x_847); -lean_dec(x_846); -x_24 = x_847; -x_25 = x_23; -goto block_840; +lean_object* x_642; +x_642 = lean_ctor_get(x_641, 1); +lean_inc(x_642); +lean_dec(x_641); +x_25 = x_642; +x_26 = x_24; +goto block_629; } case 2: { -lean_object* x_848; lean_object* x_849; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; lean_object* x_854; -x_848 = lean_ctor_get(x_846, 0); -lean_inc(x_848); -lean_dec(x_846); -x_849 = l_Lake_Glob_decodeToml___closed__2; -x_850 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_850, 0, x_848); -lean_ctor_set(x_850, 1, x_849); -x_851 = lean_unsigned_to_nat(1u); -x_852 = lean_mk_array(x_851, x_850); -x_853 = l_Array_append___rarg(x_23, x_852); -lean_dec(x_852); -x_854 = l_Lake_defaultBinDir; -x_24 = x_854; -x_25 = x_853; -goto block_840; +lean_object* x_643; lean_object* x_644; lean_object* x_645; +x_643 = lean_ctor_get(x_641, 0); +lean_inc(x_643); +lean_dec(x_641); +x_644 = l_Lake_Glob_decodeToml___closed__2; +x_645 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_645, 0, x_643); +lean_ctor_set(x_645, 1, x_644); +x_630 = x_645; +goto block_635; } case 3: { -lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; -x_855 = lean_ctor_get(x_846, 0); -lean_inc(x_855); -lean_dec(x_846); -x_856 = l_Lake_Glob_decodeToml___closed__2; -x_857 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_857, 0, x_855); -lean_ctor_set(x_857, 1, x_856); -x_858 = lean_unsigned_to_nat(1u); -x_859 = lean_mk_array(x_858, x_857); -x_860 = l_Array_append___rarg(x_23, x_859); -lean_dec(x_859); -x_861 = l_Lake_defaultBinDir; -x_24 = x_861; -x_25 = x_860; -goto block_840; +lean_object* x_646; lean_object* x_647; lean_object* x_648; +x_646 = lean_ctor_get(x_641, 0); +lean_inc(x_646); +lean_dec(x_641); +x_647 = l_Lake_Glob_decodeToml___closed__2; +x_648 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_648, 0, x_646); +lean_ctor_set(x_648, 1, x_647); +x_630 = x_648; +goto block_635; } default: { -uint8_t x_862; -x_862 = !lean_is_exclusive(x_846); -if (x_862 == 0) -{ -lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; -x_863 = lean_ctor_get(x_846, 1); -lean_dec(x_863); -x_864 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_846, 0); -lean_ctor_set(x_846, 1, x_864); -x_865 = lean_unsigned_to_nat(1u); -x_866 = lean_mk_array(x_865, x_846); -x_867 = l_Array_append___rarg(x_23, x_866); -lean_dec(x_866); -x_868 = l_Lake_defaultBinDir; -x_24 = x_868; -x_25 = x_867; -goto block_840; +uint8_t x_649; +x_649 = !lean_is_exclusive(x_641); +if (x_649 == 0) +{ +lean_object* x_650; lean_object* x_651; +x_650 = lean_ctor_get(x_641, 1); +lean_dec(x_650); +x_651 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_641, 0); +lean_ctor_set(x_641, 1, x_651); +x_630 = x_641; +goto block_635; } else { -lean_object* x_869; lean_object* x_870; lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; -x_869 = lean_ctor_get(x_846, 0); -lean_inc(x_869); -lean_dec(x_846); -x_870 = l_Lake_Glob_decodeToml___closed__2; -x_871 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_871, 0, x_869); -lean_ctor_set(x_871, 1, x_870); -x_872 = lean_unsigned_to_nat(1u); -x_873 = lean_mk_array(x_872, x_871); -x_874 = l_Array_append___rarg(x_23, x_873); -lean_dec(x_873); -x_875 = l_Lake_defaultBinDir; -x_24 = x_875; -x_25 = x_874; -goto block_840; +lean_object* x_652; lean_object* x_653; lean_object* x_654; +x_652 = lean_ctor_get(x_641, 0); +lean_inc(x_652); +lean_dec(x_641); +x_653 = l_Lake_Glob_decodeToml___closed__2; +x_654 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_654, 0, x_652); +lean_ctor_set(x_654, 1, x_653); +x_630 = x_654; +goto block_635; } } } } -block_840: +block_629: { -lean_object* x_26; lean_object* x_27; lean_object* x_805; lean_object* x_806; lean_object* x_807; -x_805 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_806 = l_Lake_PackageConfig_decodeToml___closed__49; +lean_object* x_27; lean_object* x_28; lean_object* x_604; lean_object* x_610; lean_object* x_611; lean_object* x_612; +x_610 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_611 = l_Lake_PackageConfig_decodeToml___closed__49; lean_inc(x_1); -x_807 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_805, x_806, x_1); -if (lean_obj_tag(x_807) == 0) +x_612 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_610, x_611, x_1); +if (lean_obj_tag(x_612) == 0) { -lean_object* x_808; -x_808 = l_Lake_defaultIrDir; -x_26 = x_808; -x_27 = x_25; -goto block_804; +lean_object* x_613; +x_613 = l_Lake_defaultIrDir; +x_27 = x_613; +x_28 = x_26; +goto block_603; } else { -lean_object* x_809; lean_object* x_810; -x_809 = lean_ctor_get(x_807, 0); -lean_inc(x_809); -lean_dec(x_807); -x_810 = lean_ctor_get(x_809, 1); -lean_inc(x_810); -lean_dec(x_809); -switch (lean_obj_tag(x_810)) { +lean_object* x_614; lean_object* x_615; +x_614 = lean_ctor_get(x_612, 0); +lean_inc(x_614); +lean_dec(x_612); +x_615 = lean_ctor_get(x_614, 1); +lean_inc(x_615); +lean_dec(x_614); +switch (lean_obj_tag(x_615)) { case 0: { -lean_object* x_811; -x_811 = lean_ctor_get(x_810, 1); -lean_inc(x_811); -lean_dec(x_810); -x_26 = x_811; -x_27 = x_25; -goto block_804; +lean_object* x_616; +x_616 = lean_ctor_get(x_615, 1); +lean_inc(x_616); +lean_dec(x_615); +x_27 = x_616; +x_28 = x_26; +goto block_603; } case 2: { -lean_object* x_812; lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; -x_812 = lean_ctor_get(x_810, 0); -lean_inc(x_812); -lean_dec(x_810); -x_813 = l_Lake_Glob_decodeToml___closed__2; -x_814 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_814, 0, x_812); -lean_ctor_set(x_814, 1, x_813); -x_815 = lean_unsigned_to_nat(1u); -x_816 = lean_mk_array(x_815, x_814); -x_817 = l_Array_append___rarg(x_25, x_816); -lean_dec(x_816); -x_818 = l_Lake_defaultIrDir; -x_26 = x_818; -x_27 = x_817; -goto block_804; +lean_object* x_617; lean_object* x_618; lean_object* x_619; +x_617 = lean_ctor_get(x_615, 0); +lean_inc(x_617); +lean_dec(x_615); +x_618 = l_Lake_Glob_decodeToml___closed__2; +x_619 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_619, 0, x_617); +lean_ctor_set(x_619, 1, x_618); +x_604 = x_619; +goto block_609; } case 3: { -lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; -x_819 = lean_ctor_get(x_810, 0); -lean_inc(x_819); -lean_dec(x_810); -x_820 = l_Lake_Glob_decodeToml___closed__2; -x_821 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_821, 0, x_819); -lean_ctor_set(x_821, 1, x_820); -x_822 = lean_unsigned_to_nat(1u); -x_823 = lean_mk_array(x_822, x_821); -x_824 = l_Array_append___rarg(x_25, x_823); -lean_dec(x_823); -x_825 = l_Lake_defaultIrDir; -x_26 = x_825; -x_27 = x_824; -goto block_804; +lean_object* x_620; lean_object* x_621; lean_object* x_622; +x_620 = lean_ctor_get(x_615, 0); +lean_inc(x_620); +lean_dec(x_615); +x_621 = l_Lake_Glob_decodeToml___closed__2; +x_622 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_622, 0, x_620); +lean_ctor_set(x_622, 1, x_621); +x_604 = x_622; +goto block_609; } default: { -uint8_t x_826; -x_826 = !lean_is_exclusive(x_810); -if (x_826 == 0) -{ -lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; lean_object* x_831; lean_object* x_832; -x_827 = lean_ctor_get(x_810, 1); -lean_dec(x_827); -x_828 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_810, 0); -lean_ctor_set(x_810, 1, x_828); -x_829 = lean_unsigned_to_nat(1u); -x_830 = lean_mk_array(x_829, x_810); -x_831 = l_Array_append___rarg(x_25, x_830); -lean_dec(x_830); -x_832 = l_Lake_defaultIrDir; -x_26 = x_832; -x_27 = x_831; -goto block_804; -} -else -{ -lean_object* x_833; lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; -x_833 = lean_ctor_get(x_810, 0); -lean_inc(x_833); -lean_dec(x_810); -x_834 = l_Lake_Glob_decodeToml___closed__2; -x_835 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_835, 0, x_833); -lean_ctor_set(x_835, 1, x_834); -x_836 = lean_unsigned_to_nat(1u); -x_837 = lean_mk_array(x_836, x_835); -x_838 = l_Array_append___rarg(x_25, x_837); -lean_dec(x_837); -x_839 = l_Lake_defaultIrDir; -x_26 = x_839; -x_27 = x_838; -goto block_804; +uint8_t x_623; +x_623 = !lean_is_exclusive(x_615); +if (x_623 == 0) +{ +lean_object* x_624; lean_object* x_625; +x_624 = lean_ctor_get(x_615, 1); +lean_dec(x_624); +x_625 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_615, 0); +lean_ctor_set(x_615, 1, x_625); +x_604 = x_615; +goto block_609; +} +else +{ +lean_object* x_626; lean_object* x_627; lean_object* x_628; +x_626 = lean_ctor_get(x_615, 0); +lean_inc(x_626); +lean_dec(x_615); +x_627 = l_Lake_Glob_decodeToml___closed__2; +x_628 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_628, 0, x_626); +lean_ctor_set(x_628, 1, x_627); +x_604 = x_628; +goto block_609; } } } } -block_804: +block_603: { -lean_object* x_28; lean_object* x_29; lean_object* x_749; lean_object* x_750; lean_object* x_751; lean_object* x_752; -x_749 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_750 = l_Lake_PackageConfig_decodeToml___closed__47; +lean_object* x_29; lean_object* x_30; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; +x_564 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_565 = l_Lake_PackageConfig_decodeToml___closed__47; lean_inc(x_1); -x_751 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_749, x_750, x_1); -x_752 = lean_box(0); -if (lean_obj_tag(x_751) == 0) +x_566 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_564, x_565, x_1); +x_567 = lean_box(0); +if (lean_obj_tag(x_566) == 0) { -x_28 = x_752; -x_29 = x_27; -goto block_748; +x_29 = x_567; +x_30 = x_28; +goto block_563; } else { -uint8_t x_753; -x_753 = !lean_is_exclusive(x_751); -if (x_753 == 0) +uint8_t x_573; +x_573 = !lean_is_exclusive(x_566); +if (x_573 == 0) { -lean_object* x_754; lean_object* x_755; -x_754 = lean_ctor_get(x_751, 0); -x_755 = lean_ctor_get(x_754, 1); -lean_inc(x_755); -lean_dec(x_754); -switch (lean_obj_tag(x_755)) { +lean_object* x_574; lean_object* x_575; +x_574 = lean_ctor_get(x_566, 0); +x_575 = lean_ctor_get(x_574, 1); +lean_inc(x_575); +lean_dec(x_574); +switch (lean_obj_tag(x_575)) { case 0: { -lean_object* x_756; -x_756 = lean_ctor_get(x_755, 1); -lean_inc(x_756); -lean_dec(x_755); -lean_ctor_set(x_751, 0, x_756); -x_28 = x_751; -x_29 = x_27; -goto block_748; +lean_object* x_576; +x_576 = lean_ctor_get(x_575, 1); +lean_inc(x_576); +lean_dec(x_575); +lean_ctor_set(x_566, 0, x_576); +x_29 = x_566; +x_30 = x_28; +goto block_563; } case 2: { -lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; -lean_free_object(x_751); -x_757 = lean_ctor_get(x_755, 0); -lean_inc(x_757); -lean_dec(x_755); -x_758 = l_Lake_Glob_decodeToml___closed__2; -x_759 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_759, 0, x_757); -lean_ctor_set(x_759, 1, x_758); -x_760 = lean_unsigned_to_nat(1u); -x_761 = lean_mk_array(x_760, x_759); -x_762 = l_Array_append___rarg(x_27, x_761); -lean_dec(x_761); -x_28 = x_752; -x_29 = x_762; -goto block_748; +lean_object* x_577; lean_object* x_578; lean_object* x_579; +lean_free_object(x_566); +x_577 = lean_ctor_get(x_575, 0); +lean_inc(x_577); +lean_dec(x_575); +x_578 = l_Lake_Glob_decodeToml___closed__2; +x_579 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_579, 0, x_577); +lean_ctor_set(x_579, 1, x_578); +x_568 = x_579; +goto block_572; } case 3: { -lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; -lean_free_object(x_751); -x_763 = lean_ctor_get(x_755, 0); -lean_inc(x_763); -lean_dec(x_755); -x_764 = l_Lake_Glob_decodeToml___closed__2; -x_765 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_765, 0, x_763); -lean_ctor_set(x_765, 1, x_764); -x_766 = lean_unsigned_to_nat(1u); -x_767 = lean_mk_array(x_766, x_765); -x_768 = l_Array_append___rarg(x_27, x_767); -lean_dec(x_767); -x_28 = x_752; -x_29 = x_768; -goto block_748; +lean_object* x_580; lean_object* x_581; lean_object* x_582; +lean_free_object(x_566); +x_580 = lean_ctor_get(x_575, 0); +lean_inc(x_580); +lean_dec(x_575); +x_581 = l_Lake_Glob_decodeToml___closed__2; +x_582 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_582, 0, x_580); +lean_ctor_set(x_582, 1, x_581); +x_568 = x_582; +goto block_572; } default: { -uint8_t x_769; -lean_free_object(x_751); -x_769 = !lean_is_exclusive(x_755); -if (x_769 == 0) +uint8_t x_583; +lean_free_object(x_566); +x_583 = !lean_is_exclusive(x_575); +if (x_583 == 0) { -lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; lean_object* x_774; -x_770 = lean_ctor_get(x_755, 1); -lean_dec(x_770); -x_771 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_755, 0); -lean_ctor_set(x_755, 1, x_771); -x_772 = lean_unsigned_to_nat(1u); -x_773 = lean_mk_array(x_772, x_755); -x_774 = l_Array_append___rarg(x_27, x_773); -lean_dec(x_773); -x_28 = x_752; -x_29 = x_774; -goto block_748; +lean_object* x_584; lean_object* x_585; +x_584 = lean_ctor_get(x_575, 1); +lean_dec(x_584); +x_585 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_575, 0); +lean_ctor_set(x_575, 1, x_585); +x_568 = x_575; +goto block_572; } else { -lean_object* x_775; lean_object* x_776; lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; -x_775 = lean_ctor_get(x_755, 0); -lean_inc(x_775); -lean_dec(x_755); -x_776 = l_Lake_Glob_decodeToml___closed__2; -x_777 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_777, 0, x_775); -lean_ctor_set(x_777, 1, x_776); -x_778 = lean_unsigned_to_nat(1u); -x_779 = lean_mk_array(x_778, x_777); -x_780 = l_Array_append___rarg(x_27, x_779); -lean_dec(x_779); -x_28 = x_752; -x_29 = x_780; -goto block_748; +lean_object* x_586; lean_object* x_587; lean_object* x_588; +x_586 = lean_ctor_get(x_575, 0); +lean_inc(x_586); +lean_dec(x_575); +x_587 = l_Lake_Glob_decodeToml___closed__2; +x_588 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_588, 0, x_586); +lean_ctor_set(x_588, 1, x_587); +x_568 = x_588; +goto block_572; } } } } else { -lean_object* x_781; lean_object* x_782; -x_781 = lean_ctor_get(x_751, 0); -lean_inc(x_781); -lean_dec(x_751); -x_782 = lean_ctor_get(x_781, 1); -lean_inc(x_782); -lean_dec(x_781); -switch (lean_obj_tag(x_782)) { +lean_object* x_589; lean_object* x_590; +x_589 = lean_ctor_get(x_566, 0); +lean_inc(x_589); +lean_dec(x_566); +x_590 = lean_ctor_get(x_589, 1); +lean_inc(x_590); +lean_dec(x_589); +switch (lean_obj_tag(x_590)) { case 0: { -lean_object* x_783; lean_object* x_784; -x_783 = lean_ctor_get(x_782, 1); -lean_inc(x_783); -lean_dec(x_782); -x_784 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_784, 0, x_783); -x_28 = x_784; -x_29 = x_27; -goto block_748; +lean_object* x_591; lean_object* x_592; +x_591 = lean_ctor_get(x_590, 1); +lean_inc(x_591); +lean_dec(x_590); +x_592 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_592, 0, x_591); +x_29 = x_592; +x_30 = x_28; +goto block_563; } case 2: { -lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; -x_785 = lean_ctor_get(x_782, 0); -lean_inc(x_785); -lean_dec(x_782); -x_786 = l_Lake_Glob_decodeToml___closed__2; -x_787 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_787, 0, x_785); -lean_ctor_set(x_787, 1, x_786); -x_788 = lean_unsigned_to_nat(1u); -x_789 = lean_mk_array(x_788, x_787); -x_790 = l_Array_append___rarg(x_27, x_789); -lean_dec(x_789); -x_28 = x_752; -x_29 = x_790; -goto block_748; +lean_object* x_593; lean_object* x_594; lean_object* x_595; +x_593 = lean_ctor_get(x_590, 0); +lean_inc(x_593); +lean_dec(x_590); +x_594 = l_Lake_Glob_decodeToml___closed__2; +x_595 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_595, 0, x_593); +lean_ctor_set(x_595, 1, x_594); +x_568 = x_595; +goto block_572; } case 3: { -lean_object* x_791; lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_796; -x_791 = lean_ctor_get(x_782, 0); -lean_inc(x_791); -lean_dec(x_782); -x_792 = l_Lake_Glob_decodeToml___closed__2; -x_793 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_793, 0, x_791); -lean_ctor_set(x_793, 1, x_792); -x_794 = lean_unsigned_to_nat(1u); -x_795 = lean_mk_array(x_794, x_793); -x_796 = l_Array_append___rarg(x_27, x_795); -lean_dec(x_795); -x_28 = x_752; -x_29 = x_796; -goto block_748; +lean_object* x_596; lean_object* x_597; lean_object* x_598; +x_596 = lean_ctor_get(x_590, 0); +lean_inc(x_596); +lean_dec(x_590); +x_597 = l_Lake_Glob_decodeToml___closed__2; +x_598 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_598, 0, x_596); +lean_ctor_set(x_598, 1, x_597); +x_568 = x_598; +goto block_572; } default: { -lean_object* x_797; lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; -x_797 = lean_ctor_get(x_782, 0); -lean_inc(x_797); -if (lean_is_exclusive(x_782)) { - lean_ctor_release(x_782, 0); - lean_ctor_release(x_782, 1); - x_798 = x_782; +lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; +x_599 = lean_ctor_get(x_590, 0); +lean_inc(x_599); +if (lean_is_exclusive(x_590)) { + lean_ctor_release(x_590, 0); + lean_ctor_release(x_590, 1); + x_600 = x_590; } else { - lean_dec_ref(x_782); - x_798 = lean_box(0); + lean_dec_ref(x_590); + x_600 = lean_box(0); } -x_799 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_798)) { - x_800 = lean_alloc_ctor(0, 2, 0); +x_601 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_600)) { + x_602 = lean_alloc_ctor(0, 2, 0); } else { - x_800 = x_798; - lean_ctor_set_tag(x_800, 0); -} -lean_ctor_set(x_800, 0, x_797); -lean_ctor_set(x_800, 1, x_799); -x_801 = lean_unsigned_to_nat(1u); -x_802 = lean_mk_array(x_801, x_800); -x_803 = l_Array_append___rarg(x_27, x_802); -lean_dec(x_802); -x_28 = x_752; -x_29 = x_803; -goto block_748; + x_602 = x_600; + lean_ctor_set_tag(x_602, 0); } +lean_ctor_set(x_602, 0, x_599); +lean_ctor_set(x_602, 1, x_601); +x_568 = x_602; +goto block_572; } } } -block_748: +} +block_563: { -lean_object* x_30; lean_object* x_31; lean_object* x_693; lean_object* x_694; lean_object* x_695; lean_object* x_696; -x_693 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_694 = l_Lake_PackageConfig_decodeToml___closed__45; +lean_object* x_31; lean_object* x_32; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; +x_524 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_525 = l_Lake_PackageConfig_decodeToml___closed__45; lean_inc(x_1); -x_695 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_693, x_694, x_1); -x_696 = lean_box(0); -if (lean_obj_tag(x_695) == 0) +x_526 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_524, x_525, x_1); +x_527 = lean_box(0); +if (lean_obj_tag(x_526) == 0) { -x_30 = x_696; -x_31 = x_29; -goto block_692; +x_31 = x_527; +x_32 = x_30; +goto block_523; } else { -uint8_t x_697; -x_697 = !lean_is_exclusive(x_695); -if (x_697 == 0) +uint8_t x_533; +x_533 = !lean_is_exclusive(x_526); +if (x_533 == 0) { -lean_object* x_698; lean_object* x_699; -x_698 = lean_ctor_get(x_695, 0); -x_699 = lean_ctor_get(x_698, 1); -lean_inc(x_699); -lean_dec(x_698); -switch (lean_obj_tag(x_699)) { +lean_object* x_534; lean_object* x_535; +x_534 = lean_ctor_get(x_526, 0); +x_535 = lean_ctor_get(x_534, 1); +lean_inc(x_535); +lean_dec(x_534); +switch (lean_obj_tag(x_535)) { case 0: { -lean_object* x_700; -x_700 = lean_ctor_get(x_699, 1); -lean_inc(x_700); -lean_dec(x_699); -lean_ctor_set(x_695, 0, x_700); -x_30 = x_695; -x_31 = x_29; -goto block_692; +lean_object* x_536; +x_536 = lean_ctor_get(x_535, 1); +lean_inc(x_536); +lean_dec(x_535); +lean_ctor_set(x_526, 0, x_536); +x_31 = x_526; +x_32 = x_30; +goto block_523; } case 2: { -lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; -lean_free_object(x_695); -x_701 = lean_ctor_get(x_699, 0); -lean_inc(x_701); -lean_dec(x_699); -x_702 = l_Lake_Glob_decodeToml___closed__2; -x_703 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_703, 0, x_701); -lean_ctor_set(x_703, 1, x_702); -x_704 = lean_unsigned_to_nat(1u); -x_705 = lean_mk_array(x_704, x_703); -x_706 = l_Array_append___rarg(x_29, x_705); -lean_dec(x_705); -x_30 = x_696; -x_31 = x_706; -goto block_692; +lean_object* x_537; lean_object* x_538; lean_object* x_539; +lean_free_object(x_526); +x_537 = lean_ctor_get(x_535, 0); +lean_inc(x_537); +lean_dec(x_535); +x_538 = l_Lake_Glob_decodeToml___closed__2; +x_539 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_539, 0, x_537); +lean_ctor_set(x_539, 1, x_538); +x_528 = x_539; +goto block_532; } case 3: { -lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; -lean_free_object(x_695); -x_707 = lean_ctor_get(x_699, 0); -lean_inc(x_707); -lean_dec(x_699); -x_708 = l_Lake_Glob_decodeToml___closed__2; -x_709 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_709, 0, x_707); -lean_ctor_set(x_709, 1, x_708); -x_710 = lean_unsigned_to_nat(1u); -x_711 = lean_mk_array(x_710, x_709); -x_712 = l_Array_append___rarg(x_29, x_711); -lean_dec(x_711); -x_30 = x_696; -x_31 = x_712; -goto block_692; +lean_object* x_540; lean_object* x_541; lean_object* x_542; +lean_free_object(x_526); +x_540 = lean_ctor_get(x_535, 0); +lean_inc(x_540); +lean_dec(x_535); +x_541 = l_Lake_Glob_decodeToml___closed__2; +x_542 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_542, 0, x_540); +lean_ctor_set(x_542, 1, x_541); +x_528 = x_542; +goto block_532; } default: { -uint8_t x_713; -lean_free_object(x_695); -x_713 = !lean_is_exclusive(x_699); -if (x_713 == 0) -{ -lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; -x_714 = lean_ctor_get(x_699, 1); -lean_dec(x_714); -x_715 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_699, 0); -lean_ctor_set(x_699, 1, x_715); -x_716 = lean_unsigned_to_nat(1u); -x_717 = lean_mk_array(x_716, x_699); -x_718 = l_Array_append___rarg(x_29, x_717); -lean_dec(x_717); -x_30 = x_696; -x_31 = x_718; -goto block_692; -} -else -{ -lean_object* x_719; lean_object* x_720; lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; -x_719 = lean_ctor_get(x_699, 0); -lean_inc(x_719); -lean_dec(x_699); -x_720 = l_Lake_Glob_decodeToml___closed__2; -x_721 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_721, 0, x_719); -lean_ctor_set(x_721, 1, x_720); -x_722 = lean_unsigned_to_nat(1u); -x_723 = lean_mk_array(x_722, x_721); -x_724 = l_Array_append___rarg(x_29, x_723); -lean_dec(x_723); -x_30 = x_696; -x_31 = x_724; -goto block_692; +uint8_t x_543; +lean_free_object(x_526); +x_543 = !lean_is_exclusive(x_535); +if (x_543 == 0) +{ +lean_object* x_544; lean_object* x_545; +x_544 = lean_ctor_get(x_535, 1); +lean_dec(x_544); +x_545 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_535, 0); +lean_ctor_set(x_535, 1, x_545); +x_528 = x_535; +goto block_532; +} +else +{ +lean_object* x_546; lean_object* x_547; lean_object* x_548; +x_546 = lean_ctor_get(x_535, 0); +lean_inc(x_546); +lean_dec(x_535); +x_547 = l_Lake_Glob_decodeToml___closed__2; +x_548 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_548, 0, x_546); +lean_ctor_set(x_548, 1, x_547); +x_528 = x_548; +goto block_532; } } } } else { -lean_object* x_725; lean_object* x_726; -x_725 = lean_ctor_get(x_695, 0); -lean_inc(x_725); -lean_dec(x_695); -x_726 = lean_ctor_get(x_725, 1); -lean_inc(x_726); -lean_dec(x_725); -switch (lean_obj_tag(x_726)) { +lean_object* x_549; lean_object* x_550; +x_549 = lean_ctor_get(x_526, 0); +lean_inc(x_549); +lean_dec(x_526); +x_550 = lean_ctor_get(x_549, 1); +lean_inc(x_550); +lean_dec(x_549); +switch (lean_obj_tag(x_550)) { case 0: { -lean_object* x_727; lean_object* x_728; -x_727 = lean_ctor_get(x_726, 1); -lean_inc(x_727); -lean_dec(x_726); -x_728 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_728, 0, x_727); -x_30 = x_728; -x_31 = x_29; -goto block_692; +lean_object* x_551; lean_object* x_552; +x_551 = lean_ctor_get(x_550, 1); +lean_inc(x_551); +lean_dec(x_550); +x_552 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_552, 0, x_551); +x_31 = x_552; +x_32 = x_30; +goto block_523; } case 2: { -lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; -x_729 = lean_ctor_get(x_726, 0); -lean_inc(x_729); -lean_dec(x_726); -x_730 = l_Lake_Glob_decodeToml___closed__2; -x_731 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_731, 0, x_729); -lean_ctor_set(x_731, 1, x_730); -x_732 = lean_unsigned_to_nat(1u); -x_733 = lean_mk_array(x_732, x_731); -x_734 = l_Array_append___rarg(x_29, x_733); -lean_dec(x_733); -x_30 = x_696; -x_31 = x_734; -goto block_692; +lean_object* x_553; lean_object* x_554; lean_object* x_555; +x_553 = lean_ctor_get(x_550, 0); +lean_inc(x_553); +lean_dec(x_550); +x_554 = l_Lake_Glob_decodeToml___closed__2; +x_555 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_555, 0, x_553); +lean_ctor_set(x_555, 1, x_554); +x_528 = x_555; +goto block_532; } case 3: { -lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; -x_735 = lean_ctor_get(x_726, 0); -lean_inc(x_735); -lean_dec(x_726); -x_736 = l_Lake_Glob_decodeToml___closed__2; -x_737 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_737, 0, x_735); -lean_ctor_set(x_737, 1, x_736); -x_738 = lean_unsigned_to_nat(1u); -x_739 = lean_mk_array(x_738, x_737); -x_740 = l_Array_append___rarg(x_29, x_739); -lean_dec(x_739); -x_30 = x_696; -x_31 = x_740; -goto block_692; +lean_object* x_556; lean_object* x_557; lean_object* x_558; +x_556 = lean_ctor_get(x_550, 0); +lean_inc(x_556); +lean_dec(x_550); +x_557 = l_Lake_Glob_decodeToml___closed__2; +x_558 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_558, 0, x_556); +lean_ctor_set(x_558, 1, x_557); +x_528 = x_558; +goto block_532; } default: { -lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; lean_object* x_747; -x_741 = lean_ctor_get(x_726, 0); -lean_inc(x_741); -if (lean_is_exclusive(x_726)) { - lean_ctor_release(x_726, 0); - lean_ctor_release(x_726, 1); - x_742 = x_726; +lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; +x_559 = lean_ctor_get(x_550, 0); +lean_inc(x_559); +if (lean_is_exclusive(x_550)) { + lean_ctor_release(x_550, 0); + lean_ctor_release(x_550, 1); + x_560 = x_550; } else { - lean_dec_ref(x_726); - x_742 = lean_box(0); + lean_dec_ref(x_550); + x_560 = lean_box(0); } -x_743 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_742)) { - x_744 = lean_alloc_ctor(0, 2, 0); +x_561 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_560)) { + x_562 = lean_alloc_ctor(0, 2, 0); } else { - x_744 = x_742; - lean_ctor_set_tag(x_744, 0); + x_562 = x_560; + lean_ctor_set_tag(x_562, 0); } -lean_ctor_set(x_744, 0, x_741); -lean_ctor_set(x_744, 1, x_743); -x_745 = lean_unsigned_to_nat(1u); -x_746 = lean_mk_array(x_745, x_744); -x_747 = l_Array_append___rarg(x_29, x_746); -lean_dec(x_746); -x_30 = x_696; -x_31 = x_747; -goto block_692; +lean_ctor_set(x_562, 0, x_559); +lean_ctor_set(x_562, 1, x_561); +x_528 = x_562; +goto block_532; } } } } -block_692: +block_523: { -uint8_t x_32; lean_object* x_33; lean_object* x_650; lean_object* x_651; lean_object* x_652; -x_650 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_651 = l_Lake_PackageConfig_decodeToml___closed__43; +uint8_t x_33; lean_object* x_34; lean_object* x_495; lean_object* x_501; lean_object* x_502; lean_object* x_503; +x_501 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_502 = l_Lake_PackageConfig_decodeToml___closed__43; lean_inc(x_1); -x_652 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_650, x_651, x_1); -if (lean_obj_tag(x_652) == 0) +x_503 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_501, x_502, x_1); +if (lean_obj_tag(x_503) == 0) { -uint8_t x_653; -x_653 = 0; -x_32 = x_653; -x_33 = x_31; -goto block_649; +uint8_t x_504; +x_504 = 0; +x_33 = x_504; +x_34 = x_32; +goto block_494; } else { -lean_object* x_654; lean_object* x_655; -x_654 = lean_ctor_get(x_652, 0); -lean_inc(x_654); -lean_dec(x_652); -x_655 = lean_ctor_get(x_654, 1); -lean_inc(x_655); -lean_dec(x_654); -switch (lean_obj_tag(x_655)) { +lean_object* x_505; lean_object* x_506; +x_505 = lean_ctor_get(x_503, 0); +lean_inc(x_505); +lean_dec(x_503); +x_506 = lean_ctor_get(x_505, 1); +lean_inc(x_506); +lean_dec(x_505); +switch (lean_obj_tag(x_506)) { case 0: { -uint8_t x_656; -x_656 = !lean_is_exclusive(x_655); -if (x_656 == 0) -{ -lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; uint8_t x_662; -x_657 = lean_ctor_get(x_655, 1); -lean_dec(x_657); -x_658 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_655, 1, x_658); -x_659 = lean_unsigned_to_nat(1u); -x_660 = lean_mk_array(x_659, x_655); -x_661 = l_Array_append___rarg(x_31, x_660); -lean_dec(x_660); -x_662 = 0; -x_32 = x_662; -x_33 = x_661; -goto block_649; -} -else -{ -lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; uint8_t x_669; -x_663 = lean_ctor_get(x_655, 0); -lean_inc(x_663); -lean_dec(x_655); -x_664 = l_Lake_LeanConfig_decodeToml___closed__20; -x_665 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_665, 0, x_663); -lean_ctor_set(x_665, 1, x_664); -x_666 = lean_unsigned_to_nat(1u); -x_667 = lean_mk_array(x_666, x_665); -x_668 = l_Array_append___rarg(x_31, x_667); -lean_dec(x_667); -x_669 = 0; -x_32 = x_669; -x_33 = x_668; -goto block_649; +uint8_t x_507; +x_507 = !lean_is_exclusive(x_506); +if (x_507 == 0) +{ +lean_object* x_508; lean_object* x_509; +x_508 = lean_ctor_get(x_506, 1); +lean_dec(x_508); +x_509 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_506, 1, x_509); +x_495 = x_506; +goto block_500; +} +else +{ +lean_object* x_510; lean_object* x_511; lean_object* x_512; +x_510 = lean_ctor_get(x_506, 0); +lean_inc(x_510); +lean_dec(x_506); +x_511 = l_Lake_LeanConfig_decodeToml___closed__20; +x_512 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_512, 0, x_510); +lean_ctor_set(x_512, 1, x_511); +x_495 = x_512; +goto block_500; } } case 2: { -lean_object* x_670; lean_object* x_671; lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; uint8_t x_676; -x_670 = lean_ctor_get(x_655, 0); -lean_inc(x_670); -lean_dec(x_655); -x_671 = l_Lake_LeanConfig_decodeToml___closed__20; -x_672 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_672, 0, x_670); -lean_ctor_set(x_672, 1, x_671); -x_673 = lean_unsigned_to_nat(1u); -x_674 = lean_mk_array(x_673, x_672); -x_675 = l_Array_append___rarg(x_31, x_674); -lean_dec(x_674); -x_676 = 0; -x_32 = x_676; -x_33 = x_675; -goto block_649; +lean_object* x_513; lean_object* x_514; lean_object* x_515; +x_513 = lean_ctor_get(x_506, 0); +lean_inc(x_513); +lean_dec(x_506); +x_514 = l_Lake_LeanConfig_decodeToml___closed__20; +x_515 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_515, 0, x_513); +lean_ctor_set(x_515, 1, x_514); +x_495 = x_515; +goto block_500; } case 3: { -uint8_t x_677; -x_677 = lean_ctor_get_uint8(x_655, sizeof(void*)*1); -lean_dec(x_655); -x_32 = x_677; -x_33 = x_31; -goto block_649; +uint8_t x_516; +x_516 = lean_ctor_get_uint8(x_506, sizeof(void*)*1); +lean_dec(x_506); +x_33 = x_516; +x_34 = x_32; +goto block_494; } default: { -uint8_t x_678; -x_678 = !lean_is_exclusive(x_655); -if (x_678 == 0) -{ -lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; uint8_t x_684; -x_679 = lean_ctor_get(x_655, 1); -lean_dec(x_679); -x_680 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_655, 0); -lean_ctor_set(x_655, 1, x_680); -x_681 = lean_unsigned_to_nat(1u); -x_682 = lean_mk_array(x_681, x_655); -x_683 = l_Array_append___rarg(x_31, x_682); -lean_dec(x_682); -x_684 = 0; -x_32 = x_684; -x_33 = x_683; -goto block_649; -} -else -{ -lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; lean_object* x_689; lean_object* x_690; uint8_t x_691; -x_685 = lean_ctor_get(x_655, 0); -lean_inc(x_685); -lean_dec(x_655); -x_686 = l_Lake_LeanConfig_decodeToml___closed__20; -x_687 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_687, 0, x_685); -lean_ctor_set(x_687, 1, x_686); -x_688 = lean_unsigned_to_nat(1u); -x_689 = lean_mk_array(x_688, x_687); -x_690 = l_Array_append___rarg(x_31, x_689); -lean_dec(x_689); -x_691 = 0; -x_32 = x_691; -x_33 = x_690; -goto block_649; -} -} -} -} -block_649: -{ -lean_object* x_34; lean_object* x_35; lean_object* x_614; lean_object* x_615; lean_object* x_616; -x_614 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_615 = l_Lake_PackageConfig_decodeToml___closed__41; +uint8_t x_517; +x_517 = !lean_is_exclusive(x_506); +if (x_517 == 0) +{ +lean_object* x_518; lean_object* x_519; +x_518 = lean_ctor_get(x_506, 1); +lean_dec(x_518); +x_519 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_506, 0); +lean_ctor_set(x_506, 1, x_519); +x_495 = x_506; +goto block_500; +} +else +{ +lean_object* x_520; lean_object* x_521; lean_object* x_522; +x_520 = lean_ctor_get(x_506, 0); +lean_inc(x_520); +lean_dec(x_506); +x_521 = l_Lake_LeanConfig_decodeToml___closed__20; +x_522 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_522, 0, x_520); +lean_ctor_set(x_522, 1, x_521); +x_495 = x_522; +goto block_500; +} +} +} +} +block_494: +{ +lean_object* x_35; lean_object* x_36; lean_object* x_469; lean_object* x_475; lean_object* x_476; lean_object* x_477; +x_475 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_476 = l_Lake_PackageConfig_decodeToml___closed__41; lean_inc(x_1); -x_616 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_614, x_615, x_1); -if (lean_obj_tag(x_616) == 0) +x_477 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_475, x_476, x_1); +if (lean_obj_tag(x_477) == 0) { -lean_object* x_617; -x_617 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_34 = x_617; -x_35 = x_33; -goto block_613; +lean_object* x_478; +x_478 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_35 = x_478; +x_36 = x_34; +goto block_468; } else { -lean_object* x_618; lean_object* x_619; -x_618 = lean_ctor_get(x_616, 0); -lean_inc(x_618); -lean_dec(x_616); -x_619 = lean_ctor_get(x_618, 1); -lean_inc(x_619); -lean_dec(x_618); -switch (lean_obj_tag(x_619)) { +lean_object* x_479; lean_object* x_480; +x_479 = lean_ctor_get(x_477, 0); +lean_inc(x_479); +lean_dec(x_477); +x_480 = lean_ctor_get(x_479, 1); +lean_inc(x_480); +lean_dec(x_479); +switch (lean_obj_tag(x_480)) { case 0: { -lean_object* x_620; -x_620 = lean_ctor_get(x_619, 1); -lean_inc(x_620); -lean_dec(x_619); -x_34 = x_620; -x_35 = x_33; -goto block_613; +lean_object* x_481; +x_481 = lean_ctor_get(x_480, 1); +lean_inc(x_481); +lean_dec(x_480); +x_35 = x_481; +x_36 = x_34; +goto block_468; } case 2: { -lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; -x_621 = lean_ctor_get(x_619, 0); -lean_inc(x_621); -lean_dec(x_619); -x_622 = l_Lake_Glob_decodeToml___closed__2; -x_623 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_623, 0, x_621); -lean_ctor_set(x_623, 1, x_622); -x_624 = lean_unsigned_to_nat(1u); -x_625 = lean_mk_array(x_624, x_623); -x_626 = l_Array_append___rarg(x_33, x_625); -lean_dec(x_625); -x_627 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_34 = x_627; -x_35 = x_626; -goto block_613; +lean_object* x_482; lean_object* x_483; lean_object* x_484; +x_482 = lean_ctor_get(x_480, 0); +lean_inc(x_482); +lean_dec(x_480); +x_483 = l_Lake_Glob_decodeToml___closed__2; +x_484 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_484, 0, x_482); +lean_ctor_set(x_484, 1, x_483); +x_469 = x_484; +goto block_474; } case 3: { -lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; -x_628 = lean_ctor_get(x_619, 0); -lean_inc(x_628); -lean_dec(x_619); -x_629 = l_Lake_Glob_decodeToml___closed__2; -x_630 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_630, 0, x_628); -lean_ctor_set(x_630, 1, x_629); -x_631 = lean_unsigned_to_nat(1u); -x_632 = lean_mk_array(x_631, x_630); -x_633 = l_Array_append___rarg(x_33, x_632); -lean_dec(x_632); -x_634 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_34 = x_634; -x_35 = x_633; -goto block_613; +lean_object* x_485; lean_object* x_486; lean_object* x_487; +x_485 = lean_ctor_get(x_480, 0); +lean_inc(x_485); +lean_dec(x_480); +x_486 = l_Lake_Glob_decodeToml___closed__2; +x_487 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_487, 0, x_485); +lean_ctor_set(x_487, 1, x_486); +x_469 = x_487; +goto block_474; } default: { -uint8_t x_635; -x_635 = !lean_is_exclusive(x_619); -if (x_635 == 0) -{ -lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; -x_636 = lean_ctor_get(x_619, 1); -lean_dec(x_636); -x_637 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_619, 0); -lean_ctor_set(x_619, 1, x_637); -x_638 = lean_unsigned_to_nat(1u); -x_639 = lean_mk_array(x_638, x_619); -x_640 = l_Array_append___rarg(x_33, x_639); -lean_dec(x_639); -x_641 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_34 = x_641; -x_35 = x_640; -goto block_613; -} -else -{ -lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; -x_642 = lean_ctor_get(x_619, 0); -lean_inc(x_642); -lean_dec(x_619); -x_643 = l_Lake_Glob_decodeToml___closed__2; -x_644 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_644, 0, x_642); -lean_ctor_set(x_644, 1, x_643); -x_645 = lean_unsigned_to_nat(1u); -x_646 = lean_mk_array(x_645, x_644); -x_647 = l_Array_append___rarg(x_33, x_646); -lean_dec(x_646); -x_648 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_34 = x_648; -x_35 = x_647; -goto block_613; +uint8_t x_488; +x_488 = !lean_is_exclusive(x_480); +if (x_488 == 0) +{ +lean_object* x_489; lean_object* x_490; +x_489 = lean_ctor_get(x_480, 1); +lean_dec(x_489); +x_490 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_480, 0); +lean_ctor_set(x_480, 1, x_490); +x_469 = x_480; +goto block_474; +} +else +{ +lean_object* x_491; lean_object* x_492; lean_object* x_493; +x_491 = lean_ctor_get(x_480, 0); +lean_inc(x_491); +lean_dec(x_480); +x_492 = l_Lake_Glob_decodeToml___closed__2; +x_493 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_493, 0, x_491); +lean_ctor_set(x_493, 1, x_492); +x_469 = x_493; +goto block_474; } } } } -block_613: +block_468: { -lean_object* x_36; lean_object* x_37; lean_object* x_578; lean_object* x_579; lean_object* x_580; -x_578 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_579 = l_Lake_PackageConfig_decodeToml___closed__39; +lean_object* x_37; lean_object* x_38; lean_object* x_443; lean_object* x_449; lean_object* x_450; lean_object* x_451; +x_449 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_450 = l_Lake_PackageConfig_decodeToml___closed__39; lean_inc(x_1); -x_580 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_578, x_579, x_1); -if (lean_obj_tag(x_580) == 0) +x_451 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_449, x_450, x_1); +if (lean_obj_tag(x_451) == 0) { -lean_object* x_581; -x_581 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_36 = x_581; -x_37 = x_35; -goto block_577; +lean_object* x_452; +x_452 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_37 = x_452; +x_38 = x_36; +goto block_442; } else { -lean_object* x_582; lean_object* x_583; -x_582 = lean_ctor_get(x_580, 0); -lean_inc(x_582); -lean_dec(x_580); -x_583 = lean_ctor_get(x_582, 1); -lean_inc(x_583); -lean_dec(x_582); -switch (lean_obj_tag(x_583)) { +lean_object* x_453; lean_object* x_454; +x_453 = lean_ctor_get(x_451, 0); +lean_inc(x_453); +lean_dec(x_451); +x_454 = lean_ctor_get(x_453, 1); +lean_inc(x_454); +lean_dec(x_453); +switch (lean_obj_tag(x_454)) { case 0: { -lean_object* x_584; -x_584 = lean_ctor_get(x_583, 1); -lean_inc(x_584); -lean_dec(x_583); -x_36 = x_584; -x_37 = x_35; -goto block_577; +lean_object* x_455; +x_455 = lean_ctor_get(x_454, 1); +lean_inc(x_455); +lean_dec(x_454); +x_37 = x_455; +x_38 = x_36; +goto block_442; } case 2: { -lean_object* x_585; lean_object* x_586; lean_object* x_587; lean_object* x_588; lean_object* x_589; lean_object* x_590; lean_object* x_591; -x_585 = lean_ctor_get(x_583, 0); -lean_inc(x_585); -lean_dec(x_583); -x_586 = l_Lake_Glob_decodeToml___closed__2; -x_587 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_587, 0, x_585); -lean_ctor_set(x_587, 1, x_586); -x_588 = lean_unsigned_to_nat(1u); -x_589 = lean_mk_array(x_588, x_587); -x_590 = l_Array_append___rarg(x_35, x_589); -lean_dec(x_589); -x_591 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_36 = x_591; -x_37 = x_590; -goto block_577; +lean_object* x_456; lean_object* x_457; lean_object* x_458; +x_456 = lean_ctor_get(x_454, 0); +lean_inc(x_456); +lean_dec(x_454); +x_457 = l_Lake_Glob_decodeToml___closed__2; +x_458 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_458, 0, x_456); +lean_ctor_set(x_458, 1, x_457); +x_443 = x_458; +goto block_448; } case 3: { -lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; -x_592 = lean_ctor_get(x_583, 0); -lean_inc(x_592); -lean_dec(x_583); -x_593 = l_Lake_Glob_decodeToml___closed__2; -x_594 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_594, 0, x_592); -lean_ctor_set(x_594, 1, x_593); -x_595 = lean_unsigned_to_nat(1u); -x_596 = lean_mk_array(x_595, x_594); -x_597 = l_Array_append___rarg(x_35, x_596); -lean_dec(x_596); -x_598 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_36 = x_598; -x_37 = x_597; -goto block_577; +lean_object* x_459; lean_object* x_460; lean_object* x_461; +x_459 = lean_ctor_get(x_454, 0); +lean_inc(x_459); +lean_dec(x_454); +x_460 = l_Lake_Glob_decodeToml___closed__2; +x_461 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_461, 0, x_459); +lean_ctor_set(x_461, 1, x_460); +x_443 = x_461; +goto block_448; } default: { -uint8_t x_599; -x_599 = !lean_is_exclusive(x_583); -if (x_599 == 0) +uint8_t x_462; +x_462 = !lean_is_exclusive(x_454); +if (x_462 == 0) { -lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; -x_600 = lean_ctor_get(x_583, 1); -lean_dec(x_600); -x_601 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_583, 0); -lean_ctor_set(x_583, 1, x_601); -x_602 = lean_unsigned_to_nat(1u); -x_603 = lean_mk_array(x_602, x_583); -x_604 = l_Array_append___rarg(x_35, x_603); -lean_dec(x_603); -x_605 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_36 = x_605; -x_37 = x_604; -goto block_577; -} -else -{ -lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; lean_object* x_611; lean_object* x_612; -x_606 = lean_ctor_get(x_583, 0); -lean_inc(x_606); -lean_dec(x_583); -x_607 = l_Lake_Glob_decodeToml___closed__2; -x_608 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_608, 0, x_606); -lean_ctor_set(x_608, 1, x_607); -x_609 = lean_unsigned_to_nat(1u); -x_610 = lean_mk_array(x_609, x_608); -x_611 = l_Array_append___rarg(x_35, x_610); -lean_dec(x_610); -x_612 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_36 = x_612; -x_37 = x_611; -goto block_577; -} -} -} -} -block_577: -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_38 = lean_string_utf8_byte_size(x_34); -x_39 = lean_unsigned_to_nat(0u); -x_40 = lean_nat_dec_eq(x_38, x_39); -lean_dec(x_38); -x_41 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_42 = l_Lake_PackageConfig_decodeToml___closed__4; +lean_object* x_463; lean_object* x_464; +x_463 = lean_ctor_get(x_454, 1); +lean_dec(x_463); +x_464 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_454, 0); +lean_ctor_set(x_454, 1, x_464); +x_443 = x_454; +goto block_448; +} +else +{ +lean_object* x_465; lean_object* x_466; lean_object* x_467; +x_465 = lean_ctor_get(x_454, 0); +lean_inc(x_465); +lean_dec(x_454); +x_466 = l_Lake_Glob_decodeToml___closed__2; +x_467 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_467, 0, x_465); +lean_ctor_set(x_467, 1, x_466); +x_443 = x_467; +goto block_448; +} +} +} +} +block_442: +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_39 = lean_string_utf8_byte_size(x_35); +x_40 = lean_unsigned_to_nat(0u); +x_41 = lean_nat_dec_eq(x_39, x_40); +lean_dec(x_39); +x_42 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_43 = l_Lake_PackageConfig_decodeToml___closed__4; lean_inc(x_1); -x_43 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_42, x_1); -if (x_40 == 0) +x_44 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_43, x_1); +if (x_41 == 0) { -uint8_t x_571; -x_571 = l_Lake_PackageConfig_decodeToml___closed__36; -if (x_571 == 0) +uint8_t x_436; +x_436 = l_Lake_PackageConfig_decodeToml___closed__36; +if (x_436 == 0) { -lean_dec(x_34); -x_44 = x_36; -goto block_570; +lean_dec(x_35); +x_45 = x_37; +goto block_435; } else { -lean_object* x_572; uint8_t x_573; -x_572 = lean_string_utf8_byte_size(x_36); -x_573 = lean_nat_dec_eq(x_572, x_39); -lean_dec(x_572); -if (x_573 == 0) +lean_object* x_437; uint8_t x_438; +x_437 = lean_string_utf8_byte_size(x_37); +x_438 = lean_nat_dec_eq(x_437, x_40); +lean_dec(x_437); +if (x_438 == 0) { -lean_dec(x_34); -x_44 = x_36; -goto block_570; +lean_dec(x_35); +x_45 = x_37; +goto block_435; } else { -lean_dec(x_36); -x_44 = x_34; -goto block_570; +lean_dec(x_37); +x_45 = x_35; +goto block_435; } } } else { -uint8_t x_574; -x_574 = l_Lake_PackageConfig_decodeToml___closed__37; -if (x_574 == 0) +uint8_t x_439; +x_439 = l_Lake_PackageConfig_decodeToml___closed__37; +if (x_439 == 0) { -lean_dec(x_34); -x_44 = x_36; -goto block_570; +lean_dec(x_35); +x_45 = x_37; +goto block_435; } else { -lean_object* x_575; uint8_t x_576; -x_575 = lean_string_utf8_byte_size(x_36); -x_576 = lean_nat_dec_eq(x_575, x_39); -lean_dec(x_575); -if (x_576 == 0) +lean_object* x_440; uint8_t x_441; +x_440 = lean_string_utf8_byte_size(x_37); +x_441 = lean_nat_dec_eq(x_440, x_40); +lean_dec(x_440); +if (x_441 == 0) { -lean_dec(x_34); -x_44 = x_36; -goto block_570; +lean_dec(x_35); +x_45 = x_37; +goto block_435; } else { -lean_dec(x_36); -x_44 = x_34; -goto block_570; +lean_dec(x_37); +x_45 = x_35; +goto block_435; } } } -block_570: +block_435: { -lean_object* x_45; lean_object* x_46; -if (lean_obj_tag(x_43) == 0) +lean_object* x_46; lean_object* x_47; lean_object* x_402; +if (lean_obj_tag(x_44) == 0) { -lean_object* x_519; -x_519 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_519; -x_46 = x_37; -goto block_518; +lean_object* x_408; +x_408 = l_Lake_decodeLeanOptions___closed__1; +x_46 = x_408; +x_47 = x_38; +goto block_401; } else { -lean_object* x_520; lean_object* x_521; -x_520 = lean_ctor_get(x_43, 0); -lean_inc(x_520); -lean_dec(x_43); -x_521 = lean_ctor_get(x_520, 1); -lean_inc(x_521); -lean_dec(x_520); -switch (lean_obj_tag(x_521)) { +lean_object* x_409; lean_object* x_410; +x_409 = lean_ctor_get(x_44, 0); +lean_inc(x_409); +lean_dec(x_44); +x_410 = lean_ctor_get(x_409, 1); +lean_inc(x_410); +lean_dec(x_409); +switch (lean_obj_tag(x_410)) { case 0: { -uint8_t x_522; -x_522 = !lean_is_exclusive(x_521); -if (x_522 == 0) +uint8_t x_411; +x_411 = !lean_is_exclusive(x_410); +if (x_411 == 0) { -lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; -x_523 = lean_ctor_get(x_521, 1); -lean_dec(x_523); -x_524 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_521, 1, x_524); -x_525 = lean_unsigned_to_nat(1u); -x_526 = lean_mk_array(x_525, x_521); -x_527 = l_Array_append___rarg(x_37, x_526); -lean_dec(x_526); -x_528 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_528; -x_46 = x_527; -goto block_518; +lean_object* x_412; lean_object* x_413; +x_412 = lean_ctor_get(x_410, 1); +lean_dec(x_412); +x_413 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_410, 1, x_413); +x_402 = x_410; +goto block_407; } else { -lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; -x_529 = lean_ctor_get(x_521, 0); -lean_inc(x_529); -lean_dec(x_521); -x_530 = l_Lake_LeanConfig_decodeToml___closed__5; -x_531 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_531, 0, x_529); -lean_ctor_set(x_531, 1, x_530); -x_532 = lean_unsigned_to_nat(1u); -x_533 = lean_mk_array(x_532, x_531); -x_534 = l_Array_append___rarg(x_37, x_533); -lean_dec(x_533); -x_535 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_535; -x_46 = x_534; -goto block_518; +lean_object* x_414; lean_object* x_415; lean_object* x_416; +x_414 = lean_ctor_get(x_410, 0); +lean_inc(x_414); +lean_dec(x_410); +x_415 = l_Lake_LeanConfig_decodeToml___closed__5; +x_416 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_416, 0, x_414); +lean_ctor_set(x_416, 1, x_415); +x_402 = x_416; +goto block_407; } } case 2: { -lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; -x_536 = lean_ctor_get(x_521, 0); -lean_inc(x_536); -lean_dec(x_521); -x_537 = l_Lake_LeanConfig_decodeToml___closed__5; -x_538 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_538, 0, x_536); -lean_ctor_set(x_538, 1, x_537); -x_539 = lean_unsigned_to_nat(1u); -x_540 = lean_mk_array(x_539, x_538); -x_541 = l_Array_append___rarg(x_37, x_540); -lean_dec(x_540); -x_542 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_542; -x_46 = x_541; -goto block_518; +lean_object* x_417; lean_object* x_418; lean_object* x_419; +x_417 = lean_ctor_get(x_410, 0); +lean_inc(x_417); +lean_dec(x_410); +x_418 = l_Lake_LeanConfig_decodeToml___closed__5; +x_419 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_419, 0, x_417); +lean_ctor_set(x_419, 1, x_418); +x_402 = x_419; +goto block_407; } case 3: { -lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; -x_543 = lean_ctor_get(x_521, 0); -lean_inc(x_543); -lean_dec(x_521); -x_544 = l_Lake_LeanConfig_decodeToml___closed__5; -x_545 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_545, 0, x_543); -lean_ctor_set(x_545, 1, x_544); -x_546 = lean_unsigned_to_nat(1u); -x_547 = lean_mk_array(x_546, x_545); -x_548 = l_Array_append___rarg(x_37, x_547); -lean_dec(x_547); -x_549 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_549; -x_46 = x_548; -goto block_518; +lean_object* x_420; lean_object* x_421; lean_object* x_422; +x_420 = lean_ctor_get(x_410, 0); +lean_inc(x_420); +lean_dec(x_410); +x_421 = l_Lake_LeanConfig_decodeToml___closed__5; +x_422 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_422, 0, x_420); +lean_ctor_set(x_422, 1, x_421); +x_402 = x_422; +goto block_407; } case 5: { -lean_object* x_550; lean_object* x_551; -x_550 = lean_ctor_get(x_521, 1); -lean_inc(x_550); -lean_dec(x_521); -x_551 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_550); -lean_dec(x_550); -if (lean_obj_tag(x_551) == 0) +lean_object* x_423; lean_object* x_424; +x_423 = lean_ctor_get(x_410, 1); +lean_inc(x_423); +lean_dec(x_410); +x_424 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_423); +lean_dec(x_423); +if (lean_obj_tag(x_424) == 0) { -lean_object* x_552; lean_object* x_553; lean_object* x_554; -x_552 = lean_ctor_get(x_551, 0); -lean_inc(x_552); -lean_dec(x_551); -x_553 = l_Array_append___rarg(x_37, x_552); -lean_dec(x_552); -x_554 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_554; -x_46 = x_553; -goto block_518; +lean_object* x_425; lean_object* x_426; lean_object* x_427; +x_425 = lean_ctor_get(x_424, 0); +lean_inc(x_425); +lean_dec(x_424); +x_426 = l_Array_append___rarg(x_38, x_425); +lean_dec(x_425); +x_427 = l_Lake_decodeLeanOptions___closed__1; +x_46 = x_427; +x_47 = x_426; +goto block_401; } else { -lean_object* x_555; -x_555 = lean_ctor_get(x_551, 0); -lean_inc(x_555); -lean_dec(x_551); -x_45 = x_555; -x_46 = x_37; -goto block_518; +lean_object* x_428; +x_428 = lean_ctor_get(x_424, 0); +lean_inc(x_428); +lean_dec(x_424); +x_46 = x_428; +x_47 = x_38; +goto block_401; } } default: { -uint8_t x_556; -x_556 = !lean_is_exclusive(x_521); -if (x_556 == 0) +uint8_t x_429; +x_429 = !lean_is_exclusive(x_410); +if (x_429 == 0) { -lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; lean_object* x_561; lean_object* x_562; -x_557 = lean_ctor_get(x_521, 1); -lean_dec(x_557); -x_558 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_521, 0); -lean_ctor_set(x_521, 1, x_558); -x_559 = lean_unsigned_to_nat(1u); -x_560 = lean_mk_array(x_559, x_521); -x_561 = l_Array_append___rarg(x_37, x_560); -lean_dec(x_560); -x_562 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_562; -x_46 = x_561; -goto block_518; +lean_object* x_430; lean_object* x_431; +x_430 = lean_ctor_get(x_410, 1); +lean_dec(x_430); +x_431 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_410, 0); +lean_ctor_set(x_410, 1, x_431); +x_402 = x_410; +goto block_407; } else { -lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; -x_563 = lean_ctor_get(x_521, 0); -lean_inc(x_563); -lean_dec(x_521); -x_564 = l_Lake_LeanConfig_decodeToml___closed__5; -x_565 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_565, 0, x_563); -lean_ctor_set(x_565, 1, x_564); -x_566 = lean_unsigned_to_nat(1u); -x_567 = lean_mk_array(x_566, x_565); -x_568 = l_Array_append___rarg(x_37, x_567); -lean_dec(x_567); -x_569 = l_Lake_decodeLeanOptions___closed__1; -x_45 = x_569; -x_46 = x_568; -goto block_518; +lean_object* x_432; lean_object* x_433; lean_object* x_434; +x_432 = lean_ctor_get(x_410, 0); +lean_inc(x_432); +lean_dec(x_410); +x_433 = l_Lake_LeanConfig_decodeToml___closed__5; +x_434 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_434, 0, x_432); +lean_ctor_set(x_434, 1, x_433); +x_402 = x_434; +goto block_407; } } } } -block_518: +block_401: { -lean_object* x_47; lean_object* x_48; lean_object* x_484; lean_object* x_485; -x_484 = l_Lake_PackageConfig_decodeToml___closed__35; +lean_object* x_48; lean_object* x_49; lean_object* x_377; lean_object* x_383; lean_object* x_384; +x_383 = l_Lake_PackageConfig_decodeToml___closed__35; lean_inc(x_1); -x_485 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_484, x_1); -if (lean_obj_tag(x_485) == 0) +x_384 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_383, x_1); +if (lean_obj_tag(x_384) == 0) { -lean_object* x_486; -x_486 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_47 = x_486; -x_48 = x_46; -goto block_483; +lean_object* x_385; +x_385 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_48 = x_385; +x_49 = x_47; +goto block_376; } else { -lean_object* x_487; lean_object* x_488; -x_487 = lean_ctor_get(x_485, 0); -lean_inc(x_487); -lean_dec(x_485); -x_488 = lean_ctor_get(x_487, 1); -lean_inc(x_488); -lean_dec(x_487); -switch (lean_obj_tag(x_488)) { +lean_object* x_386; lean_object* x_387; +x_386 = lean_ctor_get(x_384, 0); +lean_inc(x_386); +lean_dec(x_384); +x_387 = lean_ctor_get(x_386, 1); +lean_inc(x_387); +lean_dec(x_386); +switch (lean_obj_tag(x_387)) { case 0: { -lean_object* x_489; -x_489 = lean_ctor_get(x_488, 1); -lean_inc(x_489); -lean_dec(x_488); -x_47 = x_489; -x_48 = x_46; -goto block_483; +lean_object* x_388; +x_388 = lean_ctor_get(x_387, 1); +lean_inc(x_388); +lean_dec(x_387); +x_48 = x_388; +x_49 = x_47; +goto block_376; } case 2: { -lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; -x_490 = lean_ctor_get(x_488, 0); -lean_inc(x_490); -lean_dec(x_488); -x_491 = l_Lake_Glob_decodeToml___closed__2; -x_492 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_492, 0, x_490); -lean_ctor_set(x_492, 1, x_491); -x_493 = lean_unsigned_to_nat(1u); -x_494 = lean_mk_array(x_493, x_492); -x_495 = l_Array_append___rarg(x_46, x_494); -lean_dec(x_494); -x_496 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_47 = x_496; -x_48 = x_495; -goto block_483; +lean_object* x_389; lean_object* x_390; lean_object* x_391; +x_389 = lean_ctor_get(x_387, 0); +lean_inc(x_389); +lean_dec(x_387); +x_390 = l_Lake_Glob_decodeToml___closed__2; +x_391 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_391, 0, x_389); +lean_ctor_set(x_391, 1, x_390); +x_377 = x_391; +goto block_382; } case 3: { -lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; -x_497 = lean_ctor_get(x_488, 0); -lean_inc(x_497); -lean_dec(x_488); -x_498 = l_Lake_Glob_decodeToml___closed__2; -x_499 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_499, 0, x_497); -lean_ctor_set(x_499, 1, x_498); -x_500 = lean_unsigned_to_nat(1u); -x_501 = lean_mk_array(x_500, x_499); -x_502 = l_Array_append___rarg(x_46, x_501); -lean_dec(x_501); -x_503 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_47 = x_503; -x_48 = x_502; -goto block_483; +lean_object* x_392; lean_object* x_393; lean_object* x_394; +x_392 = lean_ctor_get(x_387, 0); +lean_inc(x_392); +lean_dec(x_387); +x_393 = l_Lake_Glob_decodeToml___closed__2; +x_394 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_394, 0, x_392); +lean_ctor_set(x_394, 1, x_393); +x_377 = x_394; +goto block_382; } default: { -uint8_t x_504; -x_504 = !lean_is_exclusive(x_488); -if (x_504 == 0) +uint8_t x_395; +x_395 = !lean_is_exclusive(x_387); +if (x_395 == 0) { -lean_object* x_505; lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; -x_505 = lean_ctor_get(x_488, 1); -lean_dec(x_505); -x_506 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_488, 0); -lean_ctor_set(x_488, 1, x_506); -x_507 = lean_unsigned_to_nat(1u); -x_508 = lean_mk_array(x_507, x_488); -x_509 = l_Array_append___rarg(x_46, x_508); -lean_dec(x_508); -x_510 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_47 = x_510; -x_48 = x_509; -goto block_483; +lean_object* x_396; lean_object* x_397; +x_396 = lean_ctor_get(x_387, 1); +lean_dec(x_396); +x_397 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_387, 0); +lean_ctor_set(x_387, 1, x_397); +x_377 = x_387; +goto block_382; } else { -lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; lean_object* x_517; -x_511 = lean_ctor_get(x_488, 0); -lean_inc(x_511); -lean_dec(x_488); -x_512 = l_Lake_Glob_decodeToml___closed__2; -x_513 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_513, 0, x_511); -lean_ctor_set(x_513, 1, x_512); -x_514 = lean_unsigned_to_nat(1u); -x_515 = lean_mk_array(x_514, x_513); -x_516 = l_Array_append___rarg(x_46, x_515); -lean_dec(x_515); -x_517 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_47 = x_517; -x_48 = x_516; -goto block_483; +lean_object* x_398; lean_object* x_399; lean_object* x_400; +x_398 = lean_ctor_get(x_387, 0); +lean_inc(x_398); +lean_dec(x_387); +x_399 = l_Lake_Glob_decodeToml___closed__2; +x_400 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_400, 0, x_398); +lean_ctor_set(x_400, 1, x_399); +x_377 = x_400; +goto block_382; } } } } -block_483: +block_376: { -lean_object* x_49; lean_object* x_50; lean_object* x_430; lean_object* x_431; -x_430 = l_Lake_PackageConfig_decodeToml___closed__33; +lean_object* x_50; lean_object* x_51; lean_object* x_341; lean_object* x_347; lean_object* x_348; +x_347 = l_Lake_PackageConfig_decodeToml___closed__33; lean_inc(x_1); -x_431 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_430, x_1); -if (lean_obj_tag(x_431) == 0) +x_348 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_347, x_1); +if (lean_obj_tag(x_348) == 0) { -lean_object* x_432; -x_432 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_432; -x_50 = x_48; -goto block_429; +lean_object* x_349; +x_349 = l_Lake_decodeLeanOptions___closed__1; +x_50 = x_349; +x_51 = x_49; +goto block_340; } else { -lean_object* x_433; lean_object* x_434; -x_433 = lean_ctor_get(x_431, 0); -lean_inc(x_433); -lean_dec(x_431); -x_434 = lean_ctor_get(x_433, 1); -lean_inc(x_434); -lean_dec(x_433); -switch (lean_obj_tag(x_434)) { +lean_object* x_350; lean_object* x_351; +x_350 = lean_ctor_get(x_348, 0); +lean_inc(x_350); +lean_dec(x_348); +x_351 = lean_ctor_get(x_350, 1); +lean_inc(x_351); +lean_dec(x_350); +switch (lean_obj_tag(x_351)) { case 0: { -uint8_t x_435; -x_435 = !lean_is_exclusive(x_434); -if (x_435 == 0) +uint8_t x_352; +x_352 = !lean_is_exclusive(x_351); +if (x_352 == 0) { -lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; -x_436 = lean_ctor_get(x_434, 1); -lean_dec(x_436); -x_437 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_434, 1, x_437); -x_438 = lean_unsigned_to_nat(1u); -x_439 = lean_mk_array(x_438, x_434); -x_440 = l_Array_append___rarg(x_48, x_439); -lean_dec(x_439); -x_441 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_441; -x_50 = x_440; -goto block_429; +lean_object* x_353; lean_object* x_354; +x_353 = lean_ctor_get(x_351, 1); +lean_dec(x_353); +x_354 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_351, 1, x_354); +x_341 = x_351; +goto block_346; } else { -lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; -x_442 = lean_ctor_get(x_434, 0); -lean_inc(x_442); -lean_dec(x_434); -x_443 = l_Lake_LeanConfig_decodeToml___closed__5; -x_444 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_444, 0, x_442); -lean_ctor_set(x_444, 1, x_443); -x_445 = lean_unsigned_to_nat(1u); -x_446 = lean_mk_array(x_445, x_444); -x_447 = l_Array_append___rarg(x_48, x_446); -lean_dec(x_446); -x_448 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_448; -x_50 = x_447; -goto block_429; +lean_object* x_355; lean_object* x_356; lean_object* x_357; +x_355 = lean_ctor_get(x_351, 0); +lean_inc(x_355); +lean_dec(x_351); +x_356 = l_Lake_LeanConfig_decodeToml___closed__5; +x_357 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_357, 0, x_355); +lean_ctor_set(x_357, 1, x_356); +x_341 = x_357; +goto block_346; } } case 2: { -lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_455; -x_449 = lean_ctor_get(x_434, 0); -lean_inc(x_449); -lean_dec(x_434); -x_450 = l_Lake_LeanConfig_decodeToml___closed__5; -x_451 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_451, 0, x_449); -lean_ctor_set(x_451, 1, x_450); -x_452 = lean_unsigned_to_nat(1u); -x_453 = lean_mk_array(x_452, x_451); -x_454 = l_Array_append___rarg(x_48, x_453); -lean_dec(x_453); -x_455 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_455; -x_50 = x_454; -goto block_429; +lean_object* x_358; lean_object* x_359; lean_object* x_360; +x_358 = lean_ctor_get(x_351, 0); +lean_inc(x_358); +lean_dec(x_351); +x_359 = l_Lake_LeanConfig_decodeToml___closed__5; +x_360 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_360, 0, x_358); +lean_ctor_set(x_360, 1, x_359); +x_341 = x_360; +goto block_346; } case 3: { -lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; lean_object* x_462; -x_456 = lean_ctor_get(x_434, 0); -lean_inc(x_456); -lean_dec(x_434); -x_457 = l_Lake_LeanConfig_decodeToml___closed__5; -x_458 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_458, 0, x_456); -lean_ctor_set(x_458, 1, x_457); -x_459 = lean_unsigned_to_nat(1u); -x_460 = lean_mk_array(x_459, x_458); -x_461 = l_Array_append___rarg(x_48, x_460); -lean_dec(x_460); -x_462 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_462; -x_50 = x_461; -goto block_429; +lean_object* x_361; lean_object* x_362; lean_object* x_363; +x_361 = lean_ctor_get(x_351, 0); +lean_inc(x_361); +lean_dec(x_351); +x_362 = l_Lake_LeanConfig_decodeToml___closed__5; +x_363 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_363, 0, x_361); +lean_ctor_set(x_363, 1, x_362); +x_341 = x_363; +goto block_346; } case 5: { -lean_object* x_463; lean_object* x_464; -x_463 = lean_ctor_get(x_434, 1); -lean_inc(x_463); -lean_dec(x_434); -x_464 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_463); -lean_dec(x_463); -if (lean_obj_tag(x_464) == 0) +lean_object* x_364; lean_object* x_365; +x_364 = lean_ctor_get(x_351, 1); +lean_inc(x_364); +lean_dec(x_351); +x_365 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_364); +lean_dec(x_364); +if (lean_obj_tag(x_365) == 0) { -lean_object* x_465; lean_object* x_466; lean_object* x_467; -x_465 = lean_ctor_get(x_464, 0); -lean_inc(x_465); -lean_dec(x_464); -x_466 = l_Array_append___rarg(x_48, x_465); -lean_dec(x_465); -x_467 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_467; -x_50 = x_466; -goto block_429; +lean_object* x_366; lean_object* x_367; lean_object* x_368; +x_366 = lean_ctor_get(x_365, 0); +lean_inc(x_366); +lean_dec(x_365); +x_367 = l_Array_append___rarg(x_49, x_366); +lean_dec(x_366); +x_368 = l_Lake_decodeLeanOptions___closed__1; +x_50 = x_368; +x_51 = x_367; +goto block_340; } else { -lean_object* x_468; -x_468 = lean_ctor_get(x_464, 0); -lean_inc(x_468); -lean_dec(x_464); -x_49 = x_468; -x_50 = x_48; -goto block_429; +lean_object* x_369; +x_369 = lean_ctor_get(x_365, 0); +lean_inc(x_369); +lean_dec(x_365); +x_50 = x_369; +x_51 = x_49; +goto block_340; } } default: { -uint8_t x_469; -x_469 = !lean_is_exclusive(x_434); -if (x_469 == 0) +uint8_t x_370; +x_370 = !lean_is_exclusive(x_351); +if (x_370 == 0) { -lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; -x_470 = lean_ctor_get(x_434, 1); -lean_dec(x_470); -x_471 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_434, 0); -lean_ctor_set(x_434, 1, x_471); -x_472 = lean_unsigned_to_nat(1u); -x_473 = lean_mk_array(x_472, x_434); -x_474 = l_Array_append___rarg(x_48, x_473); -lean_dec(x_473); -x_475 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_475; -x_50 = x_474; -goto block_429; -} -else -{ -lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; lean_object* x_482; -x_476 = lean_ctor_get(x_434, 0); -lean_inc(x_476); -lean_dec(x_434); -x_477 = l_Lake_LeanConfig_decodeToml___closed__5; -x_478 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_478, 0, x_476); -lean_ctor_set(x_478, 1, x_477); -x_479 = lean_unsigned_to_nat(1u); -x_480 = lean_mk_array(x_479, x_478); -x_481 = l_Array_append___rarg(x_48, x_480); -lean_dec(x_480); -x_482 = l_Lake_decodeLeanOptions___closed__1; -x_49 = x_482; -x_50 = x_481; -goto block_429; +lean_object* x_371; lean_object* x_372; +x_371 = lean_ctor_get(x_351, 1); +lean_dec(x_371); +x_372 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_351, 0); +lean_ctor_set(x_351, 1, x_372); +x_341 = x_351; +goto block_346; +} +else +{ +lean_object* x_373; lean_object* x_374; lean_object* x_375; +x_373 = lean_ctor_get(x_351, 0); +lean_inc(x_373); +lean_dec(x_351); +x_374 = l_Lake_LeanConfig_decodeToml___closed__5; +x_375 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_375, 0, x_373); +lean_ctor_set(x_375, 1, x_374); +x_341 = x_375; +goto block_346; } } } } -block_429: +block_340: { -lean_object* x_51; lean_object* x_52; lean_object* x_419; lean_object* x_420; -x_419 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_object* x_52; lean_object* x_53; lean_object* x_330; lean_object* x_331; +x_330 = l_Lake_PackageConfig_decodeToml___closed__29; lean_inc(x_1); -x_420 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_419, x_1); -if (lean_obj_tag(x_420) == 0) +x_331 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_330, x_1); +if (lean_obj_tag(x_331) == 0) { -lean_object* x_421; -x_421 = l_Lake_PackageConfig_decodeToml___closed__31; -x_51 = x_421; -x_52 = x_50; -goto block_418; +lean_object* x_332; +x_332 = l_Lake_PackageConfig_decodeToml___closed__31; +x_52 = x_332; +x_53 = x_51; +goto block_329; } else { -lean_object* x_422; lean_object* x_423; lean_object* x_424; -x_422 = lean_ctor_get(x_420, 0); -lean_inc(x_422); -lean_dec(x_420); -x_423 = lean_ctor_get(x_422, 1); -lean_inc(x_423); -lean_dec(x_422); -x_424 = l_Lake_StdVer_decodeToml(x_423); -if (lean_obj_tag(x_424) == 0) +lean_object* x_333; lean_object* x_334; lean_object* x_335; +x_333 = lean_ctor_get(x_331, 0); +lean_inc(x_333); +lean_dec(x_331); +x_334 = lean_ctor_get(x_333, 1); +lean_inc(x_334); +lean_dec(x_333); +x_335 = l_Lake_StdVer_decodeToml(x_334); +if (lean_obj_tag(x_335) == 0) { -lean_object* x_425; lean_object* x_426; lean_object* x_427; -x_425 = lean_ctor_get(x_424, 0); -lean_inc(x_425); -lean_dec(x_424); -x_426 = l_Array_append___rarg(x_50, x_425); -lean_dec(x_425); -x_427 = l_Lake_PackageConfig_decodeToml___closed__31; -x_51 = x_427; -x_52 = x_426; -goto block_418; +lean_object* x_336; lean_object* x_337; lean_object* x_338; +x_336 = lean_ctor_get(x_335, 0); +lean_inc(x_336); +lean_dec(x_335); +x_337 = l_Array_append___rarg(x_51, x_336); +lean_dec(x_336); +x_338 = l_Lake_PackageConfig_decodeToml___closed__31; +x_52 = x_338; +x_53 = x_337; +goto block_329; } else { -lean_object* x_428; -x_428 = lean_ctor_get(x_424, 0); -lean_inc(x_428); -lean_dec(x_424); -x_51 = x_428; -x_52 = x_50; -goto block_418; +lean_object* x_339; +x_339 = lean_ctor_get(x_335, 0); +lean_inc(x_339); +lean_dec(x_335); +x_52 = x_339; +x_53 = x_51; +goto block_329; } } -block_418: +block_329: { -lean_object* x_53; lean_object* x_54; lean_object* x_407; lean_object* x_408; -x_407 = l_Lake_PackageConfig_decodeToml___closed__27; +lean_object* x_54; lean_object* x_55; lean_object* x_318; lean_object* x_319; +x_318 = l_Lake_PackageConfig_decodeToml___closed__27; lean_inc(x_1); -x_408 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_407, x_1); -if (lean_obj_tag(x_408) == 0) +x_319 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_318, x_1); +if (lean_obj_tag(x_319) == 0) { -lean_object* x_409; -x_409 = l_Lake_defaultVersionTags; -x_53 = x_409; -x_54 = x_52; -goto block_406; +lean_object* x_320; +x_320 = l_Lake_defaultVersionTags; +x_54 = x_320; +x_55 = x_53; +goto block_317; } else { -lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; -x_410 = lean_ctor_get(x_408, 0); -lean_inc(x_410); -lean_dec(x_408); -x_411 = lean_ctor_get(x_410, 1); -lean_inc(x_411); -lean_dec(x_410); -x_412 = l_Lake_versionTagPresets; -x_413 = l_Lake_StrPat_decodeToml(x_411, x_412); -if (lean_obj_tag(x_413) == 0) -{ -lean_object* x_414; lean_object* x_415; lean_object* x_416; -x_414 = lean_ctor_get(x_413, 0); -lean_inc(x_414); -lean_dec(x_413); -x_415 = l_Array_append___rarg(x_52, x_414); -lean_dec(x_414); -x_416 = l_Lake_defaultVersionTags; -x_53 = x_416; -x_54 = x_415; -goto block_406; +lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; +x_321 = lean_ctor_get(x_319, 0); +lean_inc(x_321); +lean_dec(x_319); +x_322 = lean_ctor_get(x_321, 1); +lean_inc(x_322); +lean_dec(x_321); +x_323 = l_Lake_versionTagPresets; +x_324 = l_Lake_StrPat_decodeToml(x_322, x_323); +if (lean_obj_tag(x_324) == 0) +{ +lean_object* x_325; lean_object* x_326; lean_object* x_327; +x_325 = lean_ctor_get(x_324, 0); +lean_inc(x_325); +lean_dec(x_324); +x_326 = l_Array_append___rarg(x_53, x_325); +lean_dec(x_325); +x_327 = l_Lake_defaultVersionTags; +x_54 = x_327; +x_55 = x_326; +goto block_317; } else { -lean_object* x_417; -x_417 = lean_ctor_get(x_413, 0); -lean_inc(x_417); -lean_dec(x_413); -x_53 = x_417; -x_54 = x_52; -goto block_406; +lean_object* x_328; +x_328 = lean_ctor_get(x_324, 0); +lean_inc(x_328); +lean_dec(x_324); +x_54 = x_328; +x_55 = x_53; +goto block_317; } } -block_406: +block_317: { -lean_object* x_55; lean_object* x_56; lean_object* x_372; lean_object* x_373; -x_372 = l_Lake_PackageConfig_decodeToml___closed__25; +lean_object* x_56; lean_object* x_57; lean_object* x_293; lean_object* x_299; lean_object* x_300; +x_299 = l_Lake_PackageConfig_decodeToml___closed__25; lean_inc(x_1); -x_373 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_372, x_1); -if (lean_obj_tag(x_373) == 0) +x_300 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_299, x_1); +if (lean_obj_tag(x_300) == 0) { -lean_object* x_374; -x_374 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_55 = x_374; -x_56 = x_54; -goto block_371; +lean_object* x_301; +x_301 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_56 = x_301; +x_57 = x_55; +goto block_292; } else { -lean_object* x_375; lean_object* x_376; -x_375 = lean_ctor_get(x_373, 0); -lean_inc(x_375); -lean_dec(x_373); -x_376 = lean_ctor_get(x_375, 1); -lean_inc(x_376); -lean_dec(x_375); -switch (lean_obj_tag(x_376)) { +lean_object* x_302; lean_object* x_303; +x_302 = lean_ctor_get(x_300, 0); +lean_inc(x_302); +lean_dec(x_300); +x_303 = lean_ctor_get(x_302, 1); +lean_inc(x_303); +lean_dec(x_302); +switch (lean_obj_tag(x_303)) { case 0: { -lean_object* x_377; -x_377 = lean_ctor_get(x_376, 1); -lean_inc(x_377); -lean_dec(x_376); -x_55 = x_377; -x_56 = x_54; -goto block_371; +lean_object* x_304; +x_304 = lean_ctor_get(x_303, 1); +lean_inc(x_304); +lean_dec(x_303); +x_56 = x_304; +x_57 = x_55; +goto block_292; } case 2: { -lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; -x_378 = lean_ctor_get(x_376, 0); -lean_inc(x_378); -lean_dec(x_376); -x_379 = l_Lake_Glob_decodeToml___closed__2; -x_380 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_380, 0, x_378); -lean_ctor_set(x_380, 1, x_379); -x_381 = lean_unsigned_to_nat(1u); -x_382 = lean_mk_array(x_381, x_380); -x_383 = l_Array_append___rarg(x_54, x_382); -lean_dec(x_382); -x_384 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_55 = x_384; -x_56 = x_383; -goto block_371; +lean_object* x_305; lean_object* x_306; lean_object* x_307; +x_305 = lean_ctor_get(x_303, 0); +lean_inc(x_305); +lean_dec(x_303); +x_306 = l_Lake_Glob_decodeToml___closed__2; +x_307 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_307, 0, x_305); +lean_ctor_set(x_307, 1, x_306); +x_293 = x_307; +goto block_298; } case 3: { -lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; -x_385 = lean_ctor_get(x_376, 0); -lean_inc(x_385); -lean_dec(x_376); -x_386 = l_Lake_Glob_decodeToml___closed__2; -x_387 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_387, 0, x_385); -lean_ctor_set(x_387, 1, x_386); -x_388 = lean_unsigned_to_nat(1u); -x_389 = lean_mk_array(x_388, x_387); -x_390 = l_Array_append___rarg(x_54, x_389); -lean_dec(x_389); -x_391 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_55 = x_391; -x_56 = x_390; -goto block_371; +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_303, 0); +lean_inc(x_308); +lean_dec(x_303); +x_309 = l_Lake_Glob_decodeToml___closed__2; +x_310 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +x_293 = x_310; +goto block_298; } default: { -uint8_t x_392; -x_392 = !lean_is_exclusive(x_376); -if (x_392 == 0) -{ -lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; -x_393 = lean_ctor_get(x_376, 1); -lean_dec(x_393); -x_394 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_376, 0); -lean_ctor_set(x_376, 1, x_394); -x_395 = lean_unsigned_to_nat(1u); -x_396 = lean_mk_array(x_395, x_376); -x_397 = l_Array_append___rarg(x_54, x_396); -lean_dec(x_396); -x_398 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_55 = x_398; -x_56 = x_397; -goto block_371; +uint8_t x_311; +x_311 = !lean_is_exclusive(x_303); +if (x_311 == 0) +{ +lean_object* x_312; lean_object* x_313; +x_312 = lean_ctor_get(x_303, 1); +lean_dec(x_312); +x_313 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_303, 0); +lean_ctor_set(x_303, 1, x_313); +x_293 = x_303; +goto block_298; } else { -lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; -x_399 = lean_ctor_get(x_376, 0); -lean_inc(x_399); -lean_dec(x_376); -x_400 = l_Lake_Glob_decodeToml___closed__2; -x_401 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_401, 0, x_399); -lean_ctor_set(x_401, 1, x_400); -x_402 = lean_unsigned_to_nat(1u); -x_403 = lean_mk_array(x_402, x_401); -x_404 = l_Array_append___rarg(x_54, x_403); -lean_dec(x_403); -x_405 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_55 = x_405; -x_56 = x_404; -goto block_371; +lean_object* x_314; lean_object* x_315; lean_object* x_316; +x_314 = lean_ctor_get(x_303, 0); +lean_inc(x_314); +lean_dec(x_303); +x_315 = l_Lake_Glob_decodeToml___closed__2; +x_316 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_316, 0, x_314); +lean_ctor_set(x_316, 1, x_315); +x_293 = x_316; +goto block_298; } } } } -block_371: +block_292: { -lean_object* x_57; lean_object* x_58; lean_object* x_318; lean_object* x_319; -x_318 = l_Lake_PackageConfig_decodeToml___closed__23; +lean_object* x_58; lean_object* x_59; lean_object* x_257; lean_object* x_263; lean_object* x_264; +x_263 = l_Lake_PackageConfig_decodeToml___closed__23; lean_inc(x_1); -x_319 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_318, x_1); -if (lean_obj_tag(x_319) == 0) +x_264 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_263, x_1); +if (lean_obj_tag(x_264) == 0) { -lean_object* x_320; -x_320 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_320; -x_58 = x_56; -goto block_317; +lean_object* x_265; +x_265 = l_Lake_decodeLeanOptions___closed__1; +x_58 = x_265; +x_59 = x_57; +goto block_256; } else { -lean_object* x_321; lean_object* x_322; -x_321 = lean_ctor_get(x_319, 0); -lean_inc(x_321); -lean_dec(x_319); -x_322 = lean_ctor_get(x_321, 1); -lean_inc(x_322); -lean_dec(x_321); -switch (lean_obj_tag(x_322)) { +lean_object* x_266; lean_object* x_267; +x_266 = lean_ctor_get(x_264, 0); +lean_inc(x_266); +lean_dec(x_264); +x_267 = lean_ctor_get(x_266, 1); +lean_inc(x_267); +lean_dec(x_266); +switch (lean_obj_tag(x_267)) { case 0: { -uint8_t x_323; -x_323 = !lean_is_exclusive(x_322); -if (x_323 == 0) +uint8_t x_268; +x_268 = !lean_is_exclusive(x_267); +if (x_268 == 0) { -lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; -x_324 = lean_ctor_get(x_322, 1); -lean_dec(x_324); -x_325 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_322, 1, x_325); -x_326 = lean_unsigned_to_nat(1u); -x_327 = lean_mk_array(x_326, x_322); -x_328 = l_Array_append___rarg(x_56, x_327); -lean_dec(x_327); -x_329 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_329; -x_58 = x_328; -goto block_317; +lean_object* x_269; lean_object* x_270; +x_269 = lean_ctor_get(x_267, 1); +lean_dec(x_269); +x_270 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_267, 1, x_270); +x_257 = x_267; +goto block_262; } else { -lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; -x_330 = lean_ctor_get(x_322, 0); -lean_inc(x_330); -lean_dec(x_322); -x_331 = l_Lake_LeanConfig_decodeToml___closed__5; -x_332 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_332, 0, x_330); -lean_ctor_set(x_332, 1, x_331); -x_333 = lean_unsigned_to_nat(1u); -x_334 = lean_mk_array(x_333, x_332); -x_335 = l_Array_append___rarg(x_56, x_334); -lean_dec(x_334); -x_336 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_336; -x_58 = x_335; -goto block_317; +lean_object* x_271; lean_object* x_272; lean_object* x_273; +x_271 = lean_ctor_get(x_267, 0); +lean_inc(x_271); +lean_dec(x_267); +x_272 = l_Lake_LeanConfig_decodeToml___closed__5; +x_273 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_273, 0, x_271); +lean_ctor_set(x_273, 1, x_272); +x_257 = x_273; +goto block_262; } } case 2: { -lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; -x_337 = lean_ctor_get(x_322, 0); -lean_inc(x_337); -lean_dec(x_322); -x_338 = l_Lake_LeanConfig_decodeToml___closed__5; -x_339 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_339, 0, x_337); -lean_ctor_set(x_339, 1, x_338); -x_340 = lean_unsigned_to_nat(1u); -x_341 = lean_mk_array(x_340, x_339); -x_342 = l_Array_append___rarg(x_56, x_341); -lean_dec(x_341); -x_343 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_343; -x_58 = x_342; -goto block_317; +lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_274 = lean_ctor_get(x_267, 0); +lean_inc(x_274); +lean_dec(x_267); +x_275 = l_Lake_LeanConfig_decodeToml___closed__5; +x_276 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_276, 0, x_274); +lean_ctor_set(x_276, 1, x_275); +x_257 = x_276; +goto block_262; } case 3: { -lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; -x_344 = lean_ctor_get(x_322, 0); -lean_inc(x_344); -lean_dec(x_322); -x_345 = l_Lake_LeanConfig_decodeToml___closed__5; -x_346 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_346, 0, x_344); -lean_ctor_set(x_346, 1, x_345); -x_347 = lean_unsigned_to_nat(1u); -x_348 = lean_mk_array(x_347, x_346); -x_349 = l_Array_append___rarg(x_56, x_348); -lean_dec(x_348); -x_350 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_350; -x_58 = x_349; -goto block_317; +lean_object* x_277; lean_object* x_278; lean_object* x_279; +x_277 = lean_ctor_get(x_267, 0); +lean_inc(x_277); +lean_dec(x_267); +x_278 = l_Lake_LeanConfig_decodeToml___closed__5; +x_279 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_279, 0, x_277); +lean_ctor_set(x_279, 1, x_278); +x_257 = x_279; +goto block_262; } case 5: { -lean_object* x_351; lean_object* x_352; -x_351 = lean_ctor_get(x_322, 1); -lean_inc(x_351); -lean_dec(x_322); -x_352 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_351); -lean_dec(x_351); -if (lean_obj_tag(x_352) == 0) +lean_object* x_280; lean_object* x_281; +x_280 = lean_ctor_get(x_267, 1); +lean_inc(x_280); +lean_dec(x_267); +x_281 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_280); +lean_dec(x_280); +if (lean_obj_tag(x_281) == 0) { -lean_object* x_353; lean_object* x_354; lean_object* x_355; -x_353 = lean_ctor_get(x_352, 0); -lean_inc(x_353); -lean_dec(x_352); -x_354 = l_Array_append___rarg(x_56, x_353); -lean_dec(x_353); -x_355 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_355; -x_58 = x_354; -goto block_317; +lean_object* x_282; lean_object* x_283; lean_object* x_284; +x_282 = lean_ctor_get(x_281, 0); +lean_inc(x_282); +lean_dec(x_281); +x_283 = l_Array_append___rarg(x_57, x_282); +lean_dec(x_282); +x_284 = l_Lake_decodeLeanOptions___closed__1; +x_58 = x_284; +x_59 = x_283; +goto block_256; } else { -lean_object* x_356; -x_356 = lean_ctor_get(x_352, 0); -lean_inc(x_356); -lean_dec(x_352); -x_57 = x_356; -x_58 = x_56; -goto block_317; +lean_object* x_285; +x_285 = lean_ctor_get(x_281, 0); +lean_inc(x_285); +lean_dec(x_281); +x_58 = x_285; +x_59 = x_57; +goto block_256; } } default: { -uint8_t x_357; -x_357 = !lean_is_exclusive(x_322); -if (x_357 == 0) +uint8_t x_286; +x_286 = !lean_is_exclusive(x_267); +if (x_286 == 0) { -lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; -x_358 = lean_ctor_get(x_322, 1); -lean_dec(x_358); -x_359 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_322, 0); -lean_ctor_set(x_322, 1, x_359); -x_360 = lean_unsigned_to_nat(1u); -x_361 = lean_mk_array(x_360, x_322); -x_362 = l_Array_append___rarg(x_56, x_361); -lean_dec(x_361); -x_363 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_363; -x_58 = x_362; -goto block_317; +lean_object* x_287; lean_object* x_288; +x_287 = lean_ctor_get(x_267, 1); +lean_dec(x_287); +x_288 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_267, 0); +lean_ctor_set(x_267, 1, x_288); +x_257 = x_267; +goto block_262; } else { -lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; -x_364 = lean_ctor_get(x_322, 0); -lean_inc(x_364); -lean_dec(x_322); -x_365 = l_Lake_LeanConfig_decodeToml___closed__5; -x_366 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_366, 0, x_364); -lean_ctor_set(x_366, 1, x_365); -x_367 = lean_unsigned_to_nat(1u); -x_368 = lean_mk_array(x_367, x_366); -x_369 = l_Array_append___rarg(x_56, x_368); -lean_dec(x_368); -x_370 = l_Lake_decodeLeanOptions___closed__1; -x_57 = x_370; -x_58 = x_369; -goto block_317; +lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_289 = lean_ctor_get(x_267, 0); +lean_inc(x_289); +lean_dec(x_267); +x_290 = l_Lake_LeanConfig_decodeToml___closed__5; +x_291 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_291, 0, x_289); +lean_ctor_set(x_291, 1, x_290); +x_257 = x_291; +goto block_262; } } } } -block_317: +block_256: { -lean_object* x_59; lean_object* x_60; lean_object* x_283; lean_object* x_284; -x_283 = l_Lake_PackageConfig_decodeToml___closed__21; +lean_object* x_60; lean_object* x_61; lean_object* x_232; lean_object* x_238; lean_object* x_239; +x_238 = l_Lake_PackageConfig_decodeToml___closed__21; lean_inc(x_1); -x_284 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_283, x_1); -if (lean_obj_tag(x_284) == 0) +x_239 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_238, x_1); +if (lean_obj_tag(x_239) == 0) { -lean_object* x_285; -x_285 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_59 = x_285; -x_60 = x_58; -goto block_282; +lean_object* x_240; +x_240 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_60 = x_240; +x_61 = x_59; +goto block_231; } else { -lean_object* x_286; lean_object* x_287; -x_286 = lean_ctor_get(x_284, 0); -lean_inc(x_286); -lean_dec(x_284); -x_287 = lean_ctor_get(x_286, 1); -lean_inc(x_287); -lean_dec(x_286); -switch (lean_obj_tag(x_287)) { +lean_object* x_241; lean_object* x_242; +x_241 = lean_ctor_get(x_239, 0); +lean_inc(x_241); +lean_dec(x_239); +x_242 = lean_ctor_get(x_241, 1); +lean_inc(x_242); +lean_dec(x_241); +switch (lean_obj_tag(x_242)) { case 0: { -lean_object* x_288; -x_288 = lean_ctor_get(x_287, 1); -lean_inc(x_288); -lean_dec(x_287); -x_59 = x_288; -x_60 = x_58; -goto block_282; +lean_object* x_243; +x_243 = lean_ctor_get(x_242, 1); +lean_inc(x_243); +lean_dec(x_242); +x_60 = x_243; +x_61 = x_59; +goto block_231; } case 2: { -lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; -x_289 = lean_ctor_get(x_287, 0); -lean_inc(x_289); -lean_dec(x_287); -x_290 = l_Lake_Glob_decodeToml___closed__2; -x_291 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_291, 0, x_289); -lean_ctor_set(x_291, 1, x_290); -x_292 = lean_unsigned_to_nat(1u); -x_293 = lean_mk_array(x_292, x_291); -x_294 = l_Array_append___rarg(x_58, x_293); -lean_dec(x_293); -x_295 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_59 = x_295; -x_60 = x_294; -goto block_282; +lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_244 = lean_ctor_get(x_242, 0); +lean_inc(x_244); +lean_dec(x_242); +x_245 = l_Lake_Glob_decodeToml___closed__2; +x_246 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_246, 0, x_244); +lean_ctor_set(x_246, 1, x_245); +x_232 = x_246; +goto block_237; } case 3: { -lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; -x_296 = lean_ctor_get(x_287, 0); -lean_inc(x_296); -lean_dec(x_287); -x_297 = l_Lake_Glob_decodeToml___closed__2; -x_298 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_298, 0, x_296); -lean_ctor_set(x_298, 1, x_297); -x_299 = lean_unsigned_to_nat(1u); -x_300 = lean_mk_array(x_299, x_298); -x_301 = l_Array_append___rarg(x_58, x_300); -lean_dec(x_300); -x_302 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_59 = x_302; -x_60 = x_301; -goto block_282; +lean_object* x_247; lean_object* x_248; lean_object* x_249; +x_247 = lean_ctor_get(x_242, 0); +lean_inc(x_247); +lean_dec(x_242); +x_248 = l_Lake_Glob_decodeToml___closed__2; +x_249 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_249, 0, x_247); +lean_ctor_set(x_249, 1, x_248); +x_232 = x_249; +goto block_237; } default: { -uint8_t x_303; -x_303 = !lean_is_exclusive(x_287); -if (x_303 == 0) +uint8_t x_250; +x_250 = !lean_is_exclusive(x_242); +if (x_250 == 0) { -lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; -x_304 = lean_ctor_get(x_287, 1); -lean_dec(x_304); -x_305 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_287, 0); -lean_ctor_set(x_287, 1, x_305); -x_306 = lean_unsigned_to_nat(1u); -x_307 = lean_mk_array(x_306, x_287); -x_308 = l_Array_append___rarg(x_58, x_307); -lean_dec(x_307); -x_309 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_59 = x_309; -x_60 = x_308; -goto block_282; -} -else -{ -lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; -x_310 = lean_ctor_get(x_287, 0); -lean_inc(x_310); -lean_dec(x_287); -x_311 = l_Lake_Glob_decodeToml___closed__2; -x_312 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_312, 0, x_310); -lean_ctor_set(x_312, 1, x_311); -x_313 = lean_unsigned_to_nat(1u); -x_314 = lean_mk_array(x_313, x_312); -x_315 = l_Array_append___rarg(x_58, x_314); -lean_dec(x_314); -x_316 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_59 = x_316; -x_60 = x_315; -goto block_282; +lean_object* x_251; lean_object* x_252; +x_251 = lean_ctor_get(x_242, 1); +lean_dec(x_251); +x_252 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_242, 0); +lean_ctor_set(x_242, 1, x_252); +x_232 = x_242; +goto block_237; +} +else +{ +lean_object* x_253; lean_object* x_254; lean_object* x_255; +x_253 = lean_ctor_get(x_242, 0); +lean_inc(x_253); +lean_dec(x_242); +x_254 = l_Lake_Glob_decodeToml___closed__2; +x_255 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_255, 0, x_253); +lean_ctor_set(x_255, 1, x_254); +x_232 = x_255; +goto block_237; } } } } -block_282: +block_231: { -lean_object* x_61; lean_object* x_62; lean_object* x_248; lean_object* x_249; -x_248 = l_Lake_PackageConfig_decodeToml___closed__19; +lean_object* x_62; lean_object* x_63; lean_object* x_207; lean_object* x_213; lean_object* x_214; +x_213 = l_Lake_PackageConfig_decodeToml___closed__19; lean_inc(x_1); -x_249 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_248, x_1); -if (lean_obj_tag(x_249) == 0) +x_214 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_213, x_1); +if (lean_obj_tag(x_214) == 0) { -lean_object* x_250; -x_250 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_61 = x_250; -x_62 = x_60; -goto block_247; +lean_object* x_215; +x_215 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_62 = x_215; +x_63 = x_61; +goto block_206; } else { -lean_object* x_251; lean_object* x_252; -x_251 = lean_ctor_get(x_249, 0); -lean_inc(x_251); -lean_dec(x_249); -x_252 = lean_ctor_get(x_251, 1); -lean_inc(x_252); -lean_dec(x_251); -switch (lean_obj_tag(x_252)) { +lean_object* x_216; lean_object* x_217; +x_216 = lean_ctor_get(x_214, 0); +lean_inc(x_216); +lean_dec(x_214); +x_217 = lean_ctor_get(x_216, 1); +lean_inc(x_217); +lean_dec(x_216); +switch (lean_obj_tag(x_217)) { case 0: { -lean_object* x_253; -x_253 = lean_ctor_get(x_252, 1); -lean_inc(x_253); -lean_dec(x_252); -x_61 = x_253; -x_62 = x_60; -goto block_247; +lean_object* x_218; +x_218 = lean_ctor_get(x_217, 1); +lean_inc(x_218); +lean_dec(x_217); +x_62 = x_218; +x_63 = x_61; +goto block_206; } case 2: { -lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; -x_254 = lean_ctor_get(x_252, 0); -lean_inc(x_254); -lean_dec(x_252); -x_255 = l_Lake_Glob_decodeToml___closed__2; -x_256 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_256, 0, x_254); -lean_ctor_set(x_256, 1, x_255); -x_257 = lean_unsigned_to_nat(1u); -x_258 = lean_mk_array(x_257, x_256); -x_259 = l_Array_append___rarg(x_60, x_258); -lean_dec(x_258); -x_260 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_61 = x_260; -x_62 = x_259; -goto block_247; +lean_object* x_219; lean_object* x_220; lean_object* x_221; +x_219 = lean_ctor_get(x_217, 0); +lean_inc(x_219); +lean_dec(x_217); +x_220 = l_Lake_Glob_decodeToml___closed__2; +x_221 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_221, 0, x_219); +lean_ctor_set(x_221, 1, x_220); +x_207 = x_221; +goto block_212; } case 3: { -lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; -x_261 = lean_ctor_get(x_252, 0); -lean_inc(x_261); -lean_dec(x_252); -x_262 = l_Lake_Glob_decodeToml___closed__2; -x_263 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_263, 0, x_261); -lean_ctor_set(x_263, 1, x_262); -x_264 = lean_unsigned_to_nat(1u); -x_265 = lean_mk_array(x_264, x_263); -x_266 = l_Array_append___rarg(x_60, x_265); -lean_dec(x_265); -x_267 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_61 = x_267; -x_62 = x_266; -goto block_247; +lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_222 = lean_ctor_get(x_217, 0); +lean_inc(x_222); +lean_dec(x_217); +x_223 = l_Lake_Glob_decodeToml___closed__2; +x_224 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_224, 0, x_222); +lean_ctor_set(x_224, 1, x_223); +x_207 = x_224; +goto block_212; } default: { -uint8_t x_268; -x_268 = !lean_is_exclusive(x_252); -if (x_268 == 0) +uint8_t x_225; +x_225 = !lean_is_exclusive(x_217); +if (x_225 == 0) { -lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; -x_269 = lean_ctor_get(x_252, 1); -lean_dec(x_269); -x_270 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_252, 0); -lean_ctor_set(x_252, 1, x_270); -x_271 = lean_unsigned_to_nat(1u); -x_272 = lean_mk_array(x_271, x_252); -x_273 = l_Array_append___rarg(x_60, x_272); -lean_dec(x_272); -x_274 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_61 = x_274; -x_62 = x_273; -goto block_247; +lean_object* x_226; lean_object* x_227; +x_226 = lean_ctor_get(x_217, 1); +lean_dec(x_226); +x_227 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_217, 0); +lean_ctor_set(x_217, 1, x_227); +x_207 = x_217; +goto block_212; } else { -lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; -x_275 = lean_ctor_get(x_252, 0); -lean_inc(x_275); -lean_dec(x_252); -x_276 = l_Lake_Glob_decodeToml___closed__2; -x_277 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_277, 0, x_275); -lean_ctor_set(x_277, 1, x_276); -x_278 = lean_unsigned_to_nat(1u); -x_279 = lean_mk_array(x_278, x_277); -x_280 = l_Array_append___rarg(x_60, x_279); -lean_dec(x_279); -x_281 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_61 = x_281; -x_62 = x_280; -goto block_247; +lean_object* x_228; lean_object* x_229; lean_object* x_230; +x_228 = lean_ctor_get(x_217, 0); +lean_inc(x_228); +lean_dec(x_217); +x_229 = l_Lake_Glob_decodeToml___closed__2; +x_230 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_230, 0, x_228); +lean_ctor_set(x_230, 1, x_229); +x_207 = x_230; +goto block_212; } } } } -block_247: +block_206: { -lean_object* x_63; lean_object* x_64; lean_object* x_194; lean_object* x_195; -x_194 = l_Lake_PackageConfig_decodeToml___closed__14; +lean_object* x_64; lean_object* x_65; lean_object* x_171; lean_object* x_177; lean_object* x_178; +x_177 = l_Lake_PackageConfig_decodeToml___closed__14; lean_inc(x_1); -x_195 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_194, x_1); -if (lean_obj_tag(x_195) == 0) +x_178 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_177, x_1); +if (lean_obj_tag(x_178) == 0) { -lean_object* x_196; -x_196 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_196; -x_64 = x_62; -goto block_193; +lean_object* x_179; +x_179 = l_Lake_PackageConfig_decodeToml___closed__17; +x_64 = x_179; +x_65 = x_63; +goto block_170; } else { -lean_object* x_197; lean_object* x_198; -x_197 = lean_ctor_get(x_195, 0); -lean_inc(x_197); -lean_dec(x_195); -x_198 = lean_ctor_get(x_197, 1); -lean_inc(x_198); -lean_dec(x_197); -switch (lean_obj_tag(x_198)) { +lean_object* x_180; lean_object* x_181; +x_180 = lean_ctor_get(x_178, 0); +lean_inc(x_180); +lean_dec(x_178); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +lean_dec(x_180); +switch (lean_obj_tag(x_181)) { case 0: { -uint8_t x_199; -x_199 = !lean_is_exclusive(x_198); -if (x_199 == 0) +uint8_t x_182; +x_182 = !lean_is_exclusive(x_181); +if (x_182 == 0) { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; -x_200 = lean_ctor_get(x_198, 1); -lean_dec(x_200); -x_201 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_198, 1, x_201); -x_202 = lean_unsigned_to_nat(1u); -x_203 = lean_mk_array(x_202, x_198); -x_204 = l_Array_append___rarg(x_62, x_203); -lean_dec(x_203); -x_205 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_205; -x_64 = x_204; -goto block_193; +lean_object* x_183; lean_object* x_184; +x_183 = lean_ctor_get(x_181, 1); +lean_dec(x_183); +x_184 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_181, 1, x_184); +x_171 = x_181; +goto block_176; } else { -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_206 = lean_ctor_get(x_198, 0); -lean_inc(x_206); -lean_dec(x_198); -x_207 = l_Lake_LeanConfig_decodeToml___closed__5; -x_208 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_208, 0, x_206); -lean_ctor_set(x_208, 1, x_207); -x_209 = lean_unsigned_to_nat(1u); -x_210 = lean_mk_array(x_209, x_208); -x_211 = l_Array_append___rarg(x_62, x_210); -lean_dec(x_210); -x_212 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_212; -x_64 = x_211; -goto block_193; +lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_185 = lean_ctor_get(x_181, 0); +lean_inc(x_185); +lean_dec(x_181); +x_186 = l_Lake_LeanConfig_decodeToml___closed__5; +x_187 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_187, 0, x_185); +lean_ctor_set(x_187, 1, x_186); +x_171 = x_187; +goto block_176; } } case 2: { -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; -x_213 = lean_ctor_get(x_198, 0); -lean_inc(x_213); -lean_dec(x_198); -x_214 = l_Lake_LeanConfig_decodeToml___closed__5; -x_215 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_215, 0, x_213); -lean_ctor_set(x_215, 1, x_214); -x_216 = lean_unsigned_to_nat(1u); -x_217 = lean_mk_array(x_216, x_215); -x_218 = l_Array_append___rarg(x_62, x_217); -lean_dec(x_217); -x_219 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_219; -x_64 = x_218; -goto block_193; +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_ctor_get(x_181, 0); +lean_inc(x_188); +lean_dec(x_181); +x_189 = l_Lake_LeanConfig_decodeToml___closed__5; +x_190 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_190, 0, x_188); +lean_ctor_set(x_190, 1, x_189); +x_171 = x_190; +goto block_176; } case 3: { -lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_220 = lean_ctor_get(x_198, 0); -lean_inc(x_220); -lean_dec(x_198); -x_221 = l_Lake_LeanConfig_decodeToml___closed__5; -x_222 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_222, 0, x_220); -lean_ctor_set(x_222, 1, x_221); -x_223 = lean_unsigned_to_nat(1u); -x_224 = lean_mk_array(x_223, x_222); -x_225 = l_Array_append___rarg(x_62, x_224); -lean_dec(x_224); -x_226 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_226; -x_64 = x_225; -goto block_193; +lean_object* x_191; lean_object* x_192; lean_object* x_193; +x_191 = lean_ctor_get(x_181, 0); +lean_inc(x_191); +lean_dec(x_181); +x_192 = l_Lake_LeanConfig_decodeToml___closed__5; +x_193 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_193, 0, x_191); +lean_ctor_set(x_193, 1, x_192); +x_171 = x_193; +goto block_176; } case 5: { -lean_object* x_227; lean_object* x_228; -x_227 = lean_ctor_get(x_198, 1); -lean_inc(x_227); -lean_dec(x_198); -x_228 = l_Lake_Toml_decodeArray___at_Lake_PackageConfig_decodeToml___spec__1(x_227); -lean_dec(x_227); -if (lean_obj_tag(x_228) == 0) +lean_object* x_194; lean_object* x_195; +x_194 = lean_ctor_get(x_181, 1); +lean_inc(x_194); +lean_dec(x_181); +x_195 = l_Lake_Toml_decodeArray___at_Lake_PackageConfig_decodeToml___spec__1(x_194); +lean_dec(x_194); +if (lean_obj_tag(x_195) == 0) { -lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_229 = lean_ctor_get(x_228, 0); -lean_inc(x_229); -lean_dec(x_228); -x_230 = l_Array_append___rarg(x_62, x_229); -lean_dec(x_229); -x_231 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_231; -x_64 = x_230; -goto block_193; +lean_object* x_196; lean_object* x_197; lean_object* x_198; +x_196 = lean_ctor_get(x_195, 0); +lean_inc(x_196); +lean_dec(x_195); +x_197 = l_Array_append___rarg(x_63, x_196); +lean_dec(x_196); +x_198 = l_Lake_PackageConfig_decodeToml___closed__17; +x_64 = x_198; +x_65 = x_197; +goto block_170; } else { -lean_object* x_232; -x_232 = lean_ctor_get(x_228, 0); -lean_inc(x_232); -lean_dec(x_228); -x_63 = x_232; -x_64 = x_62; -goto block_193; +lean_object* x_199; +x_199 = lean_ctor_get(x_195, 0); +lean_inc(x_199); +lean_dec(x_195); +x_64 = x_199; +x_65 = x_63; +goto block_170; } } default: { -uint8_t x_233; -x_233 = !lean_is_exclusive(x_198); -if (x_233 == 0) +uint8_t x_200; +x_200 = !lean_is_exclusive(x_181); +if (x_200 == 0) { -lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_234 = lean_ctor_get(x_198, 1); -lean_dec(x_234); -x_235 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_198, 0); -lean_ctor_set(x_198, 1, x_235); -x_236 = lean_unsigned_to_nat(1u); -x_237 = lean_mk_array(x_236, x_198); -x_238 = l_Array_append___rarg(x_62, x_237); -lean_dec(x_237); -x_239 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_239; -x_64 = x_238; -goto block_193; +lean_object* x_201; lean_object* x_202; +x_201 = lean_ctor_get(x_181, 1); +lean_dec(x_201); +x_202 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_181, 0); +lean_ctor_set(x_181, 1, x_202); +x_171 = x_181; +goto block_176; } else { -lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_240 = lean_ctor_get(x_198, 0); -lean_inc(x_240); -lean_dec(x_198); -x_241 = l_Lake_LeanConfig_decodeToml___closed__5; -x_242 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_242, 0, x_240); -lean_ctor_set(x_242, 1, x_241); -x_243 = lean_unsigned_to_nat(1u); -x_244 = lean_mk_array(x_243, x_242); -x_245 = l_Array_append___rarg(x_62, x_244); -lean_dec(x_244); -x_246 = l_Lake_PackageConfig_decodeToml___closed__17; -x_63 = x_246; -x_64 = x_245; -goto block_193; +lean_object* x_203; lean_object* x_204; lean_object* x_205; +x_203 = lean_ctor_get(x_181, 0); +lean_inc(x_203); +lean_dec(x_181); +x_204 = l_Lake_LeanConfig_decodeToml___closed__5; +x_205 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_205, 0, x_203); +lean_ctor_set(x_205, 1, x_204); +x_171 = x_205; +goto block_176; } } } } -block_193: +block_170: { -lean_object* x_65; lean_object* x_66; lean_object* x_159; lean_object* x_160; -x_159 = l_Lake_PackageConfig_decodeToml___closed__11; +lean_object* x_66; lean_object* x_67; lean_object* x_146; lean_object* x_152; lean_object* x_153; +x_152 = l_Lake_PackageConfig_decodeToml___closed__12; lean_inc(x_1); -x_160 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_159, x_1); -if (lean_obj_tag(x_160) == 0) +x_153 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_152, x_1); +if (lean_obj_tag(x_153) == 0) { -lean_object* x_161; -x_161 = l_Lake_PackageConfig_decodeToml___closed__12; -x_65 = x_161; -x_66 = x_64; -goto block_158; +lean_object* x_154; +x_154 = l_Lake_PackageConfig_decodeToml___closed__10; +x_66 = x_154; +x_67 = x_65; +goto block_145; } else { -lean_object* x_162; lean_object* x_163; -x_162 = lean_ctor_get(x_160, 0); -lean_inc(x_162); -lean_dec(x_160); -x_163 = lean_ctor_get(x_162, 1); -lean_inc(x_163); -lean_dec(x_162); -switch (lean_obj_tag(x_163)) { +lean_object* x_155; lean_object* x_156; +x_155 = lean_ctor_get(x_153, 0); +lean_inc(x_155); +lean_dec(x_153); +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +lean_dec(x_155); +switch (lean_obj_tag(x_156)) { case 0: { -lean_object* x_164; -x_164 = lean_ctor_get(x_163, 1); -lean_inc(x_164); -lean_dec(x_163); -x_65 = x_164; -x_66 = x_64; -goto block_158; +lean_object* x_157; +x_157 = lean_ctor_get(x_156, 1); +lean_inc(x_157); +lean_dec(x_156); +x_66 = x_157; +x_67 = x_65; +goto block_145; } case 2: { -lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; -x_165 = lean_ctor_get(x_163, 0); -lean_inc(x_165); -lean_dec(x_163); -x_166 = l_Lake_Glob_decodeToml___closed__2; -x_167 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_167, 0, x_165); -lean_ctor_set(x_167, 1, x_166); -x_168 = lean_unsigned_to_nat(1u); -x_169 = lean_mk_array(x_168, x_167); -x_170 = l_Array_append___rarg(x_64, x_169); -lean_dec(x_169); -x_171 = l_Lake_PackageConfig_decodeToml___closed__12; -x_65 = x_171; -x_66 = x_170; -goto block_158; +lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_158 = lean_ctor_get(x_156, 0); +lean_inc(x_158); +lean_dec(x_156); +x_159 = l_Lake_Glob_decodeToml___closed__2; +x_160 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_160, 0, x_158); +lean_ctor_set(x_160, 1, x_159); +x_146 = x_160; +goto block_151; } case 3: { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_172 = lean_ctor_get(x_163, 0); -lean_inc(x_172); -lean_dec(x_163); -x_173 = l_Lake_Glob_decodeToml___closed__2; -x_174 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_174, 0, x_172); -lean_ctor_set(x_174, 1, x_173); -x_175 = lean_unsigned_to_nat(1u); -x_176 = lean_mk_array(x_175, x_174); -x_177 = l_Array_append___rarg(x_64, x_176); -lean_dec(x_176); -x_178 = l_Lake_PackageConfig_decodeToml___closed__12; -x_65 = x_178; -x_66 = x_177; -goto block_158; +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_156, 0); +lean_inc(x_161); +lean_dec(x_156); +x_162 = l_Lake_Glob_decodeToml___closed__2; +x_163 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_163, 0, x_161); +lean_ctor_set(x_163, 1, x_162); +x_146 = x_163; +goto block_151; } default: { -uint8_t x_179; -x_179 = !lean_is_exclusive(x_163); -if (x_179 == 0) +uint8_t x_164; +x_164 = !lean_is_exclusive(x_156); +if (x_164 == 0) { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_180 = lean_ctor_get(x_163, 1); -lean_dec(x_180); -x_181 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_163, 0); -lean_ctor_set(x_163, 1, x_181); -x_182 = lean_unsigned_to_nat(1u); -x_183 = lean_mk_array(x_182, x_163); -x_184 = l_Array_append___rarg(x_64, x_183); -lean_dec(x_183); -x_185 = l_Lake_PackageConfig_decodeToml___closed__12; -x_65 = x_185; -x_66 = x_184; -goto block_158; +lean_object* x_165; lean_object* x_166; +x_165 = lean_ctor_get(x_156, 1); +lean_dec(x_165); +x_166 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_156, 0); +lean_ctor_set(x_156, 1, x_166); +x_146 = x_156; +goto block_151; } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_186 = lean_ctor_get(x_163, 0); -lean_inc(x_186); -lean_dec(x_163); -x_187 = l_Lake_Glob_decodeToml___closed__2; -x_188 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_188, 0, x_186); -lean_ctor_set(x_188, 1, x_187); -x_189 = lean_unsigned_to_nat(1u); -x_190 = lean_mk_array(x_189, x_188); -x_191 = l_Array_append___rarg(x_64, x_190); -lean_dec(x_190); -x_192 = l_Lake_PackageConfig_decodeToml___closed__12; -x_65 = x_192; -x_66 = x_191; -goto block_158; +lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_156, 0); +lean_inc(x_167); +lean_dec(x_156); +x_168 = l_Lake_Glob_decodeToml___closed__2; +x_169 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +x_146 = x_169; +goto block_151; } } } } -block_158: +block_145: { -uint8_t x_67; lean_object* x_68; lean_object* x_117; lean_object* x_118; -x_117 = l_Lake_PackageConfig_decodeToml___closed__9; +uint8_t x_68; lean_object* x_69; lean_object* x_118; lean_object* x_124; lean_object* x_125; +x_124 = l_Lake_PackageConfig_decodeToml___closed__9; lean_inc(x_1); -x_118 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_41, x_117, x_1); -if (lean_obj_tag(x_118) == 0) +x_125 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_124, x_1); +if (lean_obj_tag(x_125) == 0) { -uint8_t x_119; -x_119 = 1; -x_67 = x_119; -x_68 = x_66; -goto block_116; +uint8_t x_126; +x_126 = 1; +x_68 = x_126; +x_69 = x_67; +goto block_117; } else { -lean_object* x_120; lean_object* x_121; -x_120 = lean_ctor_get(x_118, 0); -lean_inc(x_120); -lean_dec(x_118); -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -lean_dec(x_120); -switch (lean_obj_tag(x_121)) { +lean_object* x_127; lean_object* x_128; +x_127 = lean_ctor_get(x_125, 0); +lean_inc(x_127); +lean_dec(x_125); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +lean_dec(x_127); +switch (lean_obj_tag(x_128)) { case 0: { -uint8_t x_122; -x_122 = !lean_is_exclusive(x_121); -if (x_122 == 0) +uint8_t x_129; +x_129 = !lean_is_exclusive(x_128); +if (x_129 == 0) { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; -x_123 = lean_ctor_get(x_121, 1); -lean_dec(x_123); -x_124 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_121, 1, x_124); -x_125 = lean_unsigned_to_nat(1u); -x_126 = lean_mk_array(x_125, x_121); -x_127 = l_Array_append___rarg(x_66, x_126); -lean_dec(x_126); -x_128 = 1; -x_67 = x_128; -x_68 = x_127; -goto block_116; +lean_object* x_130; lean_object* x_131; +x_130 = lean_ctor_get(x_128, 1); +lean_dec(x_130); +x_131 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_128, 1, x_131); +x_118 = x_128; +goto block_123; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; -x_129 = lean_ctor_get(x_121, 0); -lean_inc(x_129); -lean_dec(x_121); -x_130 = l_Lake_LeanConfig_decodeToml___closed__20; -x_131 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_131, 0, x_129); -lean_ctor_set(x_131, 1, x_130); -x_132 = lean_unsigned_to_nat(1u); -x_133 = lean_mk_array(x_132, x_131); -x_134 = l_Array_append___rarg(x_66, x_133); -lean_dec(x_133); -x_135 = 1; -x_67 = x_135; -x_68 = x_134; -goto block_116; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_128, 0); +lean_inc(x_132); +lean_dec(x_128); +x_133 = l_Lake_LeanConfig_decodeToml___closed__20; +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +x_118 = x_134; +goto block_123; } } case 2: { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_142; -x_136 = lean_ctor_get(x_121, 0); -lean_inc(x_136); -lean_dec(x_121); -x_137 = l_Lake_LeanConfig_decodeToml___closed__20; -x_138 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_138, 0, x_136); -lean_ctor_set(x_138, 1, x_137); -x_139 = lean_unsigned_to_nat(1u); -x_140 = lean_mk_array(x_139, x_138); -x_141 = l_Array_append___rarg(x_66, x_140); -lean_dec(x_140); -x_142 = 1; -x_67 = x_142; -x_68 = x_141; -goto block_116; +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_128, 0); +lean_inc(x_135); +lean_dec(x_128); +x_136 = l_Lake_LeanConfig_decodeToml___closed__20; +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +x_118 = x_137; +goto block_123; } case 3: { -uint8_t x_143; -x_143 = lean_ctor_get_uint8(x_121, sizeof(void*)*1); -lean_dec(x_121); -x_67 = x_143; -x_68 = x_66; -goto block_116; +uint8_t x_138; +x_138 = lean_ctor_get_uint8(x_128, sizeof(void*)*1); +lean_dec(x_128); +x_68 = x_138; +x_69 = x_67; +goto block_117; } default: { -uint8_t x_144; -x_144 = !lean_is_exclusive(x_121); -if (x_144 == 0) +uint8_t x_139; +x_139 = !lean_is_exclusive(x_128); +if (x_139 == 0) { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; uint8_t x_150; -x_145 = lean_ctor_get(x_121, 1); -lean_dec(x_145); -x_146 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_121, 0); -lean_ctor_set(x_121, 1, x_146); -x_147 = lean_unsigned_to_nat(1u); -x_148 = lean_mk_array(x_147, x_121); -x_149 = l_Array_append___rarg(x_66, x_148); -lean_dec(x_148); -x_150 = 1; -x_67 = x_150; -x_68 = x_149; -goto block_116; +lean_object* x_140; lean_object* x_141; +x_140 = lean_ctor_get(x_128, 1); +lean_dec(x_140); +x_141 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_128, 0); +lean_ctor_set(x_128, 1, x_141); +x_118 = x_128; +goto block_123; } else { -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; uint8_t x_157; -x_151 = lean_ctor_get(x_121, 0); -lean_inc(x_151); -lean_dec(x_121); -x_152 = l_Lake_LeanConfig_decodeToml___closed__20; -x_153 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_153, 0, x_151); -lean_ctor_set(x_153, 1, x_152); -x_154 = lean_unsigned_to_nat(1u); -x_155 = lean_mk_array(x_154, x_153); -x_156 = l_Array_append___rarg(x_66, x_155); -lean_dec(x_155); -x_157 = 1; -x_67 = x_157; -x_68 = x_156; -goto block_116; +lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_142 = lean_ctor_get(x_128, 0); +lean_inc(x_142); +lean_dec(x_128); +x_143 = l_Lake_LeanConfig_decodeToml___closed__20; +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_142); +lean_ctor_set(x_144, 1, x_143); +x_118 = x_144; +goto block_123; } } } } -block_116: +block_117: { -lean_object* x_69; lean_object* x_70; lean_object* x_111; +lean_object* x_70; lean_object* x_71; lean_object* x_112; lean_inc(x_1); -x_111 = l_Lake_LeanConfig_decodeToml(x_1); -if (lean_obj_tag(x_111) == 0) +x_112 = l_Lake_LeanConfig_decodeToml(x_1); +if (lean_obj_tag(x_112) == 0) { -lean_object* x_112; lean_object* x_113; lean_object* x_114; -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -lean_dec(x_111); -x_113 = l_Array_append___rarg(x_68, x_112); +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_112, 0); +lean_inc(x_113); lean_dec(x_112); -x_114 = l_Lake_PackageConfig_decodeToml___closed__7; -x_69 = x_114; -x_70 = x_113; -goto block_110; +x_114 = l_Array_append___rarg(x_69, x_113); +lean_dec(x_113); +x_115 = l_Lake_PackageConfig_decodeToml___closed__7; +x_70 = x_115; +x_71 = x_114; +goto block_111; } else { -lean_object* x_115; -x_115 = lean_ctor_get(x_111, 0); -lean_inc(x_115); -lean_dec(x_111); -x_69 = x_115; -x_70 = x_68; -goto block_110; +lean_object* x_116; +x_116 = lean_ctor_get(x_112, 0); +lean_inc(x_116); +lean_dec(x_112); +x_70 = x_116; +x_71 = x_69; +goto block_111; } -block_110: +block_111: { -lean_object* x_71; -x_71 = l_Lake_WorkspaceConfig_decodeToml(x_1); -if (lean_obj_tag(x_71) == 0) +lean_object* x_72; +x_72 = l_Lake_WorkspaceConfig_decodeToml(x_1); +if (lean_obj_tag(x_72) == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -lean_dec(x_71); -x_73 = l_Array_append___rarg(x_70, x_72); +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); lean_dec(x_72); -x_74 = lean_box(0); -if (lean_obj_tag(x_30) == 0) +x_74 = l_Array_append___rarg(x_71, x_73); +lean_dec(x_73); +x_75 = lean_box(0); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_75 = 0; -x_76 = l_Lake_StrPat_decodeToml___closed__6; +uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_76 = 0; +x_77 = l_Lake_StrPat_decodeToml___closed__6; lean_inc(x_11); -x_77 = l_Lean_Name_toString(x_11, x_75, x_76); -x_78 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_79 = lean_string_append(x_78, x_77); -lean_dec(x_77); -x_80 = l_Lake_PackageConfig_decodeToml___closed__5; -x_81 = lean_string_append(x_79, x_80); -x_82 = l_System_Platform_target; -x_83 = lean_string_append(x_81, x_82); -x_84 = l_Lake_PackageConfig_decodeToml___closed__6; -x_85 = lean_string_append(x_83, x_84); -x_86 = l_Lake_decodeLeanOptions___closed__1; -x_87 = lean_alloc_ctor(0, 29, 3); -lean_ctor_set(x_87, 0, x_78); -lean_ctor_set(x_87, 1, x_69); -lean_ctor_set(x_87, 2, x_11); -lean_ctor_set(x_87, 3, x_74); -lean_ctor_set(x_87, 4, x_86); -lean_ctor_set(x_87, 5, x_86); -lean_ctor_set(x_87, 6, x_14); -lean_ctor_set(x_87, 7, x_16); -lean_ctor_set(x_87, 8, x_18); -lean_ctor_set(x_87, 9, x_20); -lean_ctor_set(x_87, 10, x_22); -lean_ctor_set(x_87, 11, x_24); -lean_ctor_set(x_87, 12, x_26); -lean_ctor_set(x_87, 13, x_74); -lean_ctor_set(x_87, 14, x_28); -lean_ctor_set(x_87, 15, x_30); -lean_ctor_set(x_87, 16, x_85); -lean_ctor_set(x_87, 17, x_44); -lean_ctor_set(x_87, 18, x_45); -lean_ctor_set(x_87, 19, x_47); -lean_ctor_set(x_87, 20, x_49); -lean_ctor_set(x_87, 21, x_51); -lean_ctor_set(x_87, 22, x_53); -lean_ctor_set(x_87, 23, x_55); -lean_ctor_set(x_87, 24, x_57); -lean_ctor_set(x_87, 25, x_59); -lean_ctor_set(x_87, 26, x_61); -lean_ctor_set(x_87, 27, x_63); -lean_ctor_set(x_87, 28, x_65); -lean_ctor_set_uint8(x_87, sizeof(void*)*29, x_12); -lean_ctor_set_uint8(x_87, sizeof(void*)*29 + 1, x_32); -lean_ctor_set_uint8(x_87, sizeof(void*)*29 + 2, x_67); -x_3 = x_87; -x_4 = x_73; +x_78 = l_Lean_Name_toString(x_11, x_76, x_77); +x_79 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_80 = lean_string_append(x_79, x_78); +lean_dec(x_78); +x_81 = l_Lake_PackageConfig_decodeToml___closed__5; +x_82 = lean_string_append(x_80, x_81); +x_83 = l_System_Platform_target; +x_84 = lean_string_append(x_82, x_83); +x_85 = l_Lake_PackageConfig_decodeToml___closed__6; +x_86 = lean_string_append(x_84, x_85); +x_87 = l_Lake_decodeLeanOptions___closed__1; +x_88 = lean_alloc_ctor(0, 29, 3); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_70); +lean_ctor_set(x_88, 2, x_11); +lean_ctor_set(x_88, 3, x_75); +lean_ctor_set(x_88, 4, x_87); +lean_ctor_set(x_88, 5, x_87); +lean_ctor_set(x_88, 6, x_15); +lean_ctor_set(x_88, 7, x_17); +lean_ctor_set(x_88, 8, x_19); +lean_ctor_set(x_88, 9, x_21); +lean_ctor_set(x_88, 10, x_23); +lean_ctor_set(x_88, 11, x_25); +lean_ctor_set(x_88, 12, x_27); +lean_ctor_set(x_88, 13, x_75); +lean_ctor_set(x_88, 14, x_29); +lean_ctor_set(x_88, 15, x_31); +lean_ctor_set(x_88, 16, x_86); +lean_ctor_set(x_88, 17, x_45); +lean_ctor_set(x_88, 18, x_46); +lean_ctor_set(x_88, 19, x_48); +lean_ctor_set(x_88, 20, x_50); +lean_ctor_set(x_88, 21, x_52); +lean_ctor_set(x_88, 22, x_54); +lean_ctor_set(x_88, 23, x_56); +lean_ctor_set(x_88, 24, x_58); +lean_ctor_set(x_88, 25, x_60); +lean_ctor_set(x_88, 26, x_62); +lean_ctor_set(x_88, 27, x_64); +lean_ctor_set(x_88, 28, x_66); +lean_ctor_set_uint8(x_88, sizeof(void*)*29, x_12); +lean_ctor_set_uint8(x_88, sizeof(void*)*29 + 1, x_33); +lean_ctor_set_uint8(x_88, sizeof(void*)*29 + 2, x_68); +x_3 = x_88; +x_4 = x_74; goto block_8; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_88 = lean_ctor_get(x_30, 0); -lean_inc(x_88); -x_89 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_90 = l_Lake_decodeLeanOptions___closed__1; -x_91 = lean_alloc_ctor(0, 29, 3); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_69); -lean_ctor_set(x_91, 2, x_11); -lean_ctor_set(x_91, 3, x_74); -lean_ctor_set(x_91, 4, x_90); -lean_ctor_set(x_91, 5, x_90); -lean_ctor_set(x_91, 6, x_14); -lean_ctor_set(x_91, 7, x_16); -lean_ctor_set(x_91, 8, x_18); -lean_ctor_set(x_91, 9, x_20); -lean_ctor_set(x_91, 10, x_22); -lean_ctor_set(x_91, 11, x_24); -lean_ctor_set(x_91, 12, x_26); -lean_ctor_set(x_91, 13, x_74); -lean_ctor_set(x_91, 14, x_28); -lean_ctor_set(x_91, 15, x_30); -lean_ctor_set(x_91, 16, x_88); -lean_ctor_set(x_91, 17, x_44); -lean_ctor_set(x_91, 18, x_45); -lean_ctor_set(x_91, 19, x_47); -lean_ctor_set(x_91, 20, x_49); -lean_ctor_set(x_91, 21, x_51); -lean_ctor_set(x_91, 22, x_53); -lean_ctor_set(x_91, 23, x_55); -lean_ctor_set(x_91, 24, x_57); -lean_ctor_set(x_91, 25, x_59); -lean_ctor_set(x_91, 26, x_61); -lean_ctor_set(x_91, 27, x_63); -lean_ctor_set(x_91, 28, x_65); -lean_ctor_set_uint8(x_91, sizeof(void*)*29, x_12); -lean_ctor_set_uint8(x_91, sizeof(void*)*29 + 1, x_32); -lean_ctor_set_uint8(x_91, sizeof(void*)*29 + 2, x_67); -x_3 = x_91; -x_4 = x_73; +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_89 = lean_ctor_get(x_31, 0); +lean_inc(x_89); +x_90 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_91 = l_Lake_decodeLeanOptions___closed__1; +x_92 = lean_alloc_ctor(0, 29, 3); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_70); +lean_ctor_set(x_92, 2, x_11); +lean_ctor_set(x_92, 3, x_75); +lean_ctor_set(x_92, 4, x_91); +lean_ctor_set(x_92, 5, x_91); +lean_ctor_set(x_92, 6, x_15); +lean_ctor_set(x_92, 7, x_17); +lean_ctor_set(x_92, 8, x_19); +lean_ctor_set(x_92, 9, x_21); +lean_ctor_set(x_92, 10, x_23); +lean_ctor_set(x_92, 11, x_25); +lean_ctor_set(x_92, 12, x_27); +lean_ctor_set(x_92, 13, x_75); +lean_ctor_set(x_92, 14, x_29); +lean_ctor_set(x_92, 15, x_31); +lean_ctor_set(x_92, 16, x_89); +lean_ctor_set(x_92, 17, x_45); +lean_ctor_set(x_92, 18, x_46); +lean_ctor_set(x_92, 19, x_48); +lean_ctor_set(x_92, 20, x_50); +lean_ctor_set(x_92, 21, x_52); +lean_ctor_set(x_92, 22, x_54); +lean_ctor_set(x_92, 23, x_56); +lean_ctor_set(x_92, 24, x_58); +lean_ctor_set(x_92, 25, x_60); +lean_ctor_set(x_92, 26, x_62); +lean_ctor_set(x_92, 27, x_64); +lean_ctor_set(x_92, 28, x_66); +lean_ctor_set_uint8(x_92, sizeof(void*)*29, x_12); +lean_ctor_set_uint8(x_92, sizeof(void*)*29 + 1, x_33); +lean_ctor_set_uint8(x_92, sizeof(void*)*29 + 2, x_68); +x_3 = x_92; +x_4 = x_74; goto block_8; } } else { -lean_object* x_92; lean_object* x_93; -x_92 = lean_ctor_get(x_71, 0); -lean_inc(x_92); -lean_dec(x_71); -x_93 = lean_box(0); -if (lean_obj_tag(x_30) == 0) +lean_object* x_93; lean_object* x_94; +x_93 = lean_ctor_get(x_72, 0); +lean_inc(x_93); +lean_dec(x_72); +x_94 = lean_box(0); +if (lean_obj_tag(x_31) == 0) { -uint8_t x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_94 = 0; -x_95 = l_Lake_StrPat_decodeToml___closed__6; +uint8_t x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_95 = 0; +x_96 = l_Lake_StrPat_decodeToml___closed__6; lean_inc(x_11); -x_96 = l_Lean_Name_toString(x_11, x_94, x_95); -x_97 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_98 = lean_string_append(x_97, x_96); -lean_dec(x_96); -x_99 = l_Lake_PackageConfig_decodeToml___closed__5; -x_100 = lean_string_append(x_98, x_99); -x_101 = l_System_Platform_target; -x_102 = lean_string_append(x_100, x_101); -x_103 = l_Lake_PackageConfig_decodeToml___closed__6; -x_104 = lean_string_append(x_102, x_103); -x_105 = l_Lake_decodeLeanOptions___closed__1; -x_106 = lean_alloc_ctor(0, 29, 3); -lean_ctor_set(x_106, 0, x_92); -lean_ctor_set(x_106, 1, x_69); -lean_ctor_set(x_106, 2, x_11); -lean_ctor_set(x_106, 3, x_93); -lean_ctor_set(x_106, 4, x_105); -lean_ctor_set(x_106, 5, x_105); -lean_ctor_set(x_106, 6, x_14); -lean_ctor_set(x_106, 7, x_16); -lean_ctor_set(x_106, 8, x_18); -lean_ctor_set(x_106, 9, x_20); -lean_ctor_set(x_106, 10, x_22); -lean_ctor_set(x_106, 11, x_24); -lean_ctor_set(x_106, 12, x_26); -lean_ctor_set(x_106, 13, x_93); -lean_ctor_set(x_106, 14, x_28); -lean_ctor_set(x_106, 15, x_30); -lean_ctor_set(x_106, 16, x_104); -lean_ctor_set(x_106, 17, x_44); -lean_ctor_set(x_106, 18, x_45); -lean_ctor_set(x_106, 19, x_47); -lean_ctor_set(x_106, 20, x_49); -lean_ctor_set(x_106, 21, x_51); -lean_ctor_set(x_106, 22, x_53); -lean_ctor_set(x_106, 23, x_55); -lean_ctor_set(x_106, 24, x_57); -lean_ctor_set(x_106, 25, x_59); -lean_ctor_set(x_106, 26, x_61); -lean_ctor_set(x_106, 27, x_63); -lean_ctor_set(x_106, 28, x_65); -lean_ctor_set_uint8(x_106, sizeof(void*)*29, x_12); -lean_ctor_set_uint8(x_106, sizeof(void*)*29 + 1, x_32); -lean_ctor_set_uint8(x_106, sizeof(void*)*29 + 2, x_67); -x_3 = x_106; -x_4 = x_70; +x_97 = l_Lean_Name_toString(x_11, x_95, x_96); +x_98 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_99 = lean_string_append(x_98, x_97); +lean_dec(x_97); +x_100 = l_Lake_PackageConfig_decodeToml___closed__5; +x_101 = lean_string_append(x_99, x_100); +x_102 = l_System_Platform_target; +x_103 = lean_string_append(x_101, x_102); +x_104 = l_Lake_PackageConfig_decodeToml___closed__6; +x_105 = lean_string_append(x_103, x_104); +x_106 = l_Lake_decodeLeanOptions___closed__1; +x_107 = lean_alloc_ctor(0, 29, 3); +lean_ctor_set(x_107, 0, x_93); +lean_ctor_set(x_107, 1, x_70); +lean_ctor_set(x_107, 2, x_11); +lean_ctor_set(x_107, 3, x_94); +lean_ctor_set(x_107, 4, x_106); +lean_ctor_set(x_107, 5, x_106); +lean_ctor_set(x_107, 6, x_15); +lean_ctor_set(x_107, 7, x_17); +lean_ctor_set(x_107, 8, x_19); +lean_ctor_set(x_107, 9, x_21); +lean_ctor_set(x_107, 10, x_23); +lean_ctor_set(x_107, 11, x_25); +lean_ctor_set(x_107, 12, x_27); +lean_ctor_set(x_107, 13, x_94); +lean_ctor_set(x_107, 14, x_29); +lean_ctor_set(x_107, 15, x_31); +lean_ctor_set(x_107, 16, x_105); +lean_ctor_set(x_107, 17, x_45); +lean_ctor_set(x_107, 18, x_46); +lean_ctor_set(x_107, 19, x_48); +lean_ctor_set(x_107, 20, x_50); +lean_ctor_set(x_107, 21, x_52); +lean_ctor_set(x_107, 22, x_54); +lean_ctor_set(x_107, 23, x_56); +lean_ctor_set(x_107, 24, x_58); +lean_ctor_set(x_107, 25, x_60); +lean_ctor_set(x_107, 26, x_62); +lean_ctor_set(x_107, 27, x_64); +lean_ctor_set(x_107, 28, x_66); +lean_ctor_set_uint8(x_107, sizeof(void*)*29, x_12); +lean_ctor_set_uint8(x_107, sizeof(void*)*29 + 1, x_33); +lean_ctor_set_uint8(x_107, sizeof(void*)*29 + 2, x_68); +x_3 = x_107; +x_4 = x_71; goto block_8; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_30, 0); -lean_inc(x_107); -x_108 = l_Lake_decodeLeanOptions___closed__1; -x_109 = lean_alloc_ctor(0, 29, 3); -lean_ctor_set(x_109, 0, x_92); -lean_ctor_set(x_109, 1, x_69); -lean_ctor_set(x_109, 2, x_11); -lean_ctor_set(x_109, 3, x_93); -lean_ctor_set(x_109, 4, x_108); -lean_ctor_set(x_109, 5, x_108); -lean_ctor_set(x_109, 6, x_14); -lean_ctor_set(x_109, 7, x_16); -lean_ctor_set(x_109, 8, x_18); -lean_ctor_set(x_109, 9, x_20); -lean_ctor_set(x_109, 10, x_22); -lean_ctor_set(x_109, 11, x_24); -lean_ctor_set(x_109, 12, x_26); -lean_ctor_set(x_109, 13, x_93); -lean_ctor_set(x_109, 14, x_28); -lean_ctor_set(x_109, 15, x_30); -lean_ctor_set(x_109, 16, x_107); -lean_ctor_set(x_109, 17, x_44); -lean_ctor_set(x_109, 18, x_45); -lean_ctor_set(x_109, 19, x_47); -lean_ctor_set(x_109, 20, x_49); -lean_ctor_set(x_109, 21, x_51); -lean_ctor_set(x_109, 22, x_53); -lean_ctor_set(x_109, 23, x_55); -lean_ctor_set(x_109, 24, x_57); -lean_ctor_set(x_109, 25, x_59); -lean_ctor_set(x_109, 26, x_61); -lean_ctor_set(x_109, 27, x_63); -lean_ctor_set(x_109, 28, x_65); -lean_ctor_set_uint8(x_109, sizeof(void*)*29, x_12); -lean_ctor_set_uint8(x_109, sizeof(void*)*29 + 1, x_32); -lean_ctor_set_uint8(x_109, sizeof(void*)*29 + 2, x_67); -x_3 = x_109; -x_4 = x_70; +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_31, 0); +lean_inc(x_108); +x_109 = l_Lake_decodeLeanOptions___closed__1; +x_110 = lean_alloc_ctor(0, 29, 3); +lean_ctor_set(x_110, 0, x_93); +lean_ctor_set(x_110, 1, x_70); +lean_ctor_set(x_110, 2, x_11); +lean_ctor_set(x_110, 3, x_94); +lean_ctor_set(x_110, 4, x_109); +lean_ctor_set(x_110, 5, x_109); +lean_ctor_set(x_110, 6, x_15); +lean_ctor_set(x_110, 7, x_17); +lean_ctor_set(x_110, 8, x_19); +lean_ctor_set(x_110, 9, x_21); +lean_ctor_set(x_110, 10, x_23); +lean_ctor_set(x_110, 11, x_25); +lean_ctor_set(x_110, 12, x_27); +lean_ctor_set(x_110, 13, x_94); +lean_ctor_set(x_110, 14, x_29); +lean_ctor_set(x_110, 15, x_31); +lean_ctor_set(x_110, 16, x_108); +lean_ctor_set(x_110, 17, x_45); +lean_ctor_set(x_110, 18, x_46); +lean_ctor_set(x_110, 19, x_48); +lean_ctor_set(x_110, 20, x_50); +lean_ctor_set(x_110, 21, x_52); +lean_ctor_set(x_110, 22, x_54); +lean_ctor_set(x_110, 23, x_56); +lean_ctor_set(x_110, 24, x_58); +lean_ctor_set(x_110, 25, x_60); +lean_ctor_set(x_110, 26, x_62); +lean_ctor_set(x_110, 27, x_64); +lean_ctor_set(x_110, 28, x_66); +lean_ctor_set_uint8(x_110, sizeof(void*)*29, x_12); +lean_ctor_set_uint8(x_110, sizeof(void*)*29 + 1, x_33); +lean_ctor_set_uint8(x_110, sizeof(void*)*29 + 2, x_68); +x_3 = x_110; +x_4 = x_71; goto block_8; } } } } +block_123: +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_118); +lean_ctor_set(x_119, 1, x_14); +x_120 = lean_array_mk(x_119); +x_121 = l_Array_append___rarg(x_67, x_120); +lean_dec(x_120); +x_122 = 1; +x_68 = x_122; +x_69 = x_121; +goto block_117; +} } +block_151: +{ +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_147 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_14); +x_148 = lean_array_mk(x_147); +x_149 = l_Array_append___rarg(x_65, x_148); +lean_dec(x_148); +x_150 = l_Lake_PackageConfig_decodeToml___closed__10; +x_66 = x_150; +x_67 = x_149; +goto block_145; } } +block_176: +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_172 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_172, 0, x_171); +lean_ctor_set(x_172, 1, x_14); +x_173 = lean_array_mk(x_172); +x_174 = l_Array_append___rarg(x_63, x_173); +lean_dec(x_173); +x_175 = l_Lake_PackageConfig_decodeToml___closed__17; +x_64 = x_175; +x_65 = x_174; +goto block_170; } } +block_212: +{ +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_208 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_208, 0, x_207); +lean_ctor_set(x_208, 1, x_14); +x_209 = lean_array_mk(x_208); +x_210 = l_Array_append___rarg(x_61, x_209); +lean_dec(x_209); +x_211 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_62 = x_211; +x_63 = x_210; +goto block_206; } } +block_237: +{ +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_233 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_233, 0, x_232); +lean_ctor_set(x_233, 1, x_14); +x_234 = lean_array_mk(x_233); +x_235 = l_Array_append___rarg(x_59, x_234); +lean_dec(x_234); +x_236 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_60 = x_236; +x_61 = x_235; +goto block_231; } } +block_262: +{ +lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; +x_258 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_258, 0, x_257); +lean_ctor_set(x_258, 1, x_14); +x_259 = lean_array_mk(x_258); +x_260 = l_Array_append___rarg(x_57, x_259); +lean_dec(x_259); +x_261 = l_Lake_decodeLeanOptions___closed__1; +x_58 = x_261; +x_59 = x_260; +goto block_256; } } +block_298: +{ +lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; +x_294 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_294, 0, x_293); +lean_ctor_set(x_294, 1, x_14); +x_295 = lean_array_mk(x_294); +x_296 = l_Array_append___rarg(x_55, x_295); +lean_dec(x_295); +x_297 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_56 = x_297; +x_57 = x_296; +goto block_292; } } } } +block_346: +{ +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; +x_342 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_342, 0, x_341); +lean_ctor_set(x_342, 1, x_14); +x_343 = lean_array_mk(x_342); +x_344 = l_Array_append___rarg(x_49, x_343); +lean_dec(x_343); +x_345 = l_Lake_decodeLeanOptions___closed__1; +x_50 = x_345; +x_51 = x_344; +goto block_340; } } +block_382: +{ +lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; +x_378 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_378, 0, x_377); +lean_ctor_set(x_378, 1, x_14); +x_379 = lean_array_mk(x_378); +x_380 = l_Array_append___rarg(x_47, x_379); +lean_dec(x_379); +x_381 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_48 = x_381; +x_49 = x_380; +goto block_376; } } +block_407: +{ +lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; +x_403 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_403, 0, x_402); +lean_ctor_set(x_403, 1, x_14); +x_404 = lean_array_mk(x_403); +x_405 = l_Array_append___rarg(x_38, x_404); +lean_dec(x_404); +x_406 = l_Lake_decodeLeanOptions___closed__1; +x_46 = x_406; +x_47 = x_405; +goto block_401; } } } +block_448: +{ +lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; +x_444 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_444, 0, x_443); +lean_ctor_set(x_444, 1, x_14); +x_445 = lean_array_mk(x_444); +x_446 = l_Array_append___rarg(x_36, x_445); +lean_dec(x_445); +x_447 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_37 = x_447; +x_38 = x_446; +goto block_442; +} +} +block_474: +{ +lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; +x_470 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_470, 0, x_469); +lean_ctor_set(x_470, 1, x_14); +x_471 = lean_array_mk(x_470); +x_472 = l_Array_append___rarg(x_34, x_471); +lean_dec(x_471); +x_473 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_35 = x_473; +x_36 = x_472; +goto block_468; +} +} +block_500: +{ +lean_object* x_496; lean_object* x_497; lean_object* x_498; uint8_t x_499; +x_496 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_496, 0, x_495); +lean_ctor_set(x_496, 1, x_14); +x_497 = lean_array_mk(x_496); +x_498 = l_Array_append___rarg(x_32, x_497); +lean_dec(x_497); +x_499 = 0; +x_33 = x_499; +x_34 = x_498; +goto block_494; +} +} +block_532: +{ +lean_object* x_529; lean_object* x_530; lean_object* x_531; +x_529 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_529, 0, x_528); +lean_ctor_set(x_529, 1, x_14); +x_530 = lean_array_mk(x_529); +x_531 = l_Array_append___rarg(x_30, x_530); +lean_dec(x_530); +x_31 = x_527; +x_32 = x_531; +goto block_523; +} +} +block_572: +{ +lean_object* x_569; lean_object* x_570; lean_object* x_571; +x_569 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_569, 0, x_568); +lean_ctor_set(x_569, 1, x_14); +x_570 = lean_array_mk(x_569); +x_571 = l_Array_append___rarg(x_28, x_570); +lean_dec(x_570); +x_29 = x_567; +x_30 = x_571; +goto block_563; +} +} +block_609: +{ +lean_object* x_605; lean_object* x_606; lean_object* x_607; lean_object* x_608; +x_605 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_605, 0, x_604); +lean_ctor_set(x_605, 1, x_14); +x_606 = lean_array_mk(x_605); +x_607 = l_Array_append___rarg(x_26, x_606); +lean_dec(x_606); +x_608 = l_Lake_defaultIrDir; +x_27 = x_608; +x_28 = x_607; +goto block_603; +} +} +block_635: +{ +lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; +x_631 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_631, 0, x_630); +lean_ctor_set(x_631, 1, x_14); +x_632 = lean_array_mk(x_631); +x_633 = l_Array_append___rarg(x_24, x_632); +lean_dec(x_632); +x_634 = l_Lake_defaultBinDir; +x_25 = x_634; +x_26 = x_633; +goto block_629; } } +block_661: +{ +lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; +x_657 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_657, 0, x_656); +lean_ctor_set(x_657, 1, x_14); +x_658 = lean_array_mk(x_657); +x_659 = l_Array_append___rarg(x_22, x_658); +lean_dec(x_658); +x_660 = l_Lake_defaultNativeLibDir; +x_23 = x_660; +x_24 = x_659; +goto block_655; +} +} +block_687: +{ +lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; +x_683 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_683, 0, x_682); +lean_ctor_set(x_683, 1, x_14); +x_684 = lean_array_mk(x_683); +x_685 = l_Array_append___rarg(x_20, x_684); +lean_dec(x_684); +x_686 = l_Lake_defaultLeanLibDir; +x_21 = x_686; +x_22 = x_685; +goto block_681; +} +} +block_713: +{ +lean_object* x_709; lean_object* x_710; lean_object* x_711; lean_object* x_712; +x_709 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_709, 0, x_708); +lean_ctor_set(x_709, 1, x_14); +x_710 = lean_array_mk(x_709); +x_711 = l_Array_append___rarg(x_18, x_710); +lean_dec(x_710); +x_712 = l_Lake_defaultBuildDir; +x_19 = x_712; +x_20 = x_711; +goto block_707; +} +} +block_739: +{ +lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; +x_735 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_735, 0, x_734); +lean_ctor_set(x_735, 1, x_14); +x_736 = lean_array_mk(x_735); +x_737 = l_Array_append___rarg(x_16, x_736); +lean_dec(x_736); +x_738 = l_Lake_PackageConfig_decodeToml___closed__58; +x_17 = x_738; +x_18 = x_737; +goto block_733; +} +} +block_765: +{ +lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; +x_761 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_761, 0, x_760); +lean_ctor_set(x_761, 1, x_14); +x_762 = lean_array_mk(x_761); +x_763 = l_Array_append___rarg(x_13, x_762); +lean_dec(x_762); +x_764 = l_Lake_decodeLeanOptions___closed__1; +x_15 = x_764; +x_16 = x_763; +goto block_759; +} +} +block_803: +{ +lean_object* x_798; lean_object* x_799; lean_object* x_800; lean_object* x_801; uint8_t x_802; +x_798 = lean_box(0); +x_799 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_799, 0, x_797); +lean_ctor_set(x_799, 1, x_798); +x_800 = lean_array_mk(x_799); +x_801 = l_Array_append___rarg(x_10, x_800); +lean_dec(x_800); +x_802 = 0; +x_12 = x_802; +x_13 = x_801; +goto block_796; } } } @@ -13057,123 +13011,134 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlPackageConfig(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlPackageConfig___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); lean_dec(x_1); -x_28 = l_Lake_PackageConfig_decodeToml(x_27, x_26); -return x_28; +x_22 = l_Lake_PackageConfig_decodeToml(x_21, x_20); +return x_22; } default: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_1); -if (x_29 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_1); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_1, 1); -lean_dec(x_30); -x_31 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_1, 1); +lean_dec(x_24); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_1); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_1, 1, x_25); +x_2 = x_1; +goto block_7; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_36 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_2 = x_28; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } +static lean_object* _init_l_Lake_instDecodeTomlPackageConfig___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlPackageConfig___lambda__1), 1, 0); +return x_1; +} } +static lean_object* _init_l_Lake_instDecodeTomlPackageConfig() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlPackageConfig___closed__1; +return x_1; } } LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_LeanLibConfig_decodeToml___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { @@ -13183,93 +13148,92 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_6); -if (x_9 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_6); +if (x_18 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); -x_12 = l_String_toName(x_11); -if (lean_obj_tag(x_12) == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_6, 0); +x_20 = lean_ctor_get(x_6, 1); +x_21 = l_String_toName(x_20); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_13 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -lean_ctor_set(x_6, 1, x_13); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_6); -x_16 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_16, 0, x_15); -x_17 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_18 = l_Lake_mergeErrors___rarg(x_4, x_16, x_17); -x_2 = x_8; -x_4 = x_18; -goto _start; +lean_object* x_22; +x_22 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +lean_ctor_set(x_6, 1, x_22); +x_9 = x_6; +goto block_17; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_free_object(x_6); -lean_dec(x_10); -x_20 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_20, 0, x_12); -x_21 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_22 = l_Lake_mergeErrors___rarg(x_4, x_20, x_21); +lean_dec(x_19); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_21); +x_24 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_25 = l_Lake_mergeErrors___rarg(x_4, x_23, x_24); x_2 = x_8; -x_4 = x_22; +x_4 = x_25; goto _start; } } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_6, 0); -x_25 = lean_ctor_get(x_6, 1); -lean_inc(x_25); -lean_inc(x_24); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_6, 0); +x_28 = lean_ctor_get(x_6, 1); +lean_inc(x_28); +lean_inc(x_27); lean_dec(x_6); -x_26 = l_String_toName(x_25); -if (lean_obj_tag(x_26) == 0) +x_29 = l_String_toName(x_28); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_27 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_24); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_mk_array(x_29, x_28); -x_31 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_31, 0, x_30); -x_32 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_33 = l_Lake_mergeErrors___rarg(x_4, x_31, x_32); -x_2 = x_8; -x_4 = x_33; -goto _start; +lean_object* x_30; lean_object* x_31; +x_30 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_30); +x_9 = x_31; +goto block_17; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -lean_dec(x_24); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_26); -x_36 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_37 = l_Lake_mergeErrors___rarg(x_4, x_35, x_36); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_27); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_29); +x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); x_2 = x_8; -x_4 = x_37; +x_4 = x_34; goto _start; } } } case 2: { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_6, 0); +lean_inc(x_36); +lean_dec(x_6); +x_37 = l_Lake_Glob_decodeToml___closed__2; +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_9 = x_38; +goto block_17; +} +case 3: +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; x_39 = lean_ctor_get(x_6, 0); lean_inc(x_39); lean_dec(x_6); @@ -13277,80 +13241,55 @@ x_40 = l_Lake_Glob_decodeToml___closed__2; x_41 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_41, 0, x_39); lean_ctor_set(x_41, 1, x_40); -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_mk_array(x_42, x_41); -x_44 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_46 = l_Lake_mergeErrors___rarg(x_4, x_44, x_45); -x_2 = x_8; -x_4 = x_46; -goto _start; -} -case 3: -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_48 = lean_ctor_get(x_6, 0); -lean_inc(x_48); -lean_dec(x_6); -x_49 = l_Lake_Glob_decodeToml___closed__2; -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -x_51 = lean_unsigned_to_nat(1u); -x_52 = lean_mk_array(x_51, x_50); -x_53 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_53, 0, x_52); -x_54 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_55 = l_Lake_mergeErrors___rarg(x_4, x_53, x_54); -x_2 = x_8; -x_4 = x_55; -goto _start; +x_9 = x_41; +goto block_17; } default: { -uint8_t x_57; -x_57 = !lean_is_exclusive(x_6); -if (x_57 == 0) +uint8_t x_42; +x_42 = !lean_is_exclusive(x_6); +if (x_42 == 0) { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_58 = lean_ctor_get(x_6, 1); -lean_dec(x_58); -x_59 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_6, 1); +lean_dec(x_43); +x_44 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_59); -x_60 = lean_unsigned_to_nat(1u); -x_61 = lean_mk_array(x_60, x_6); -x_62 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_62, 0, x_61); -x_63 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_64 = l_Lake_mergeErrors___rarg(x_4, x_62, x_63); -x_2 = x_8; -x_4 = x_64; -goto _start; +lean_ctor_set(x_6, 1, x_44); +x_9 = x_6; +goto block_17; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_66 = lean_ctor_get(x_6, 0); -lean_inc(x_66); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_6, 0); +lean_inc(x_45); lean_dec(x_6); -x_67 = l_Lake_Glob_decodeToml___closed__2; -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -x_69 = lean_unsigned_to_nat(1u); -x_70 = lean_mk_array(x_69, x_68); -x_71 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_71, 0, x_70); -x_72 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_73 = l_Lake_mergeErrors___rarg(x_4, x_71, x_72); -x_2 = x_8; -x_4 = x_73; -goto _start; +x_46 = l_Lake_Glob_decodeToml___closed__2; +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_9 = x_47; +goto block_17; } } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; +} } else { @@ -13438,59 +13377,65 @@ uint8_t x_10; x_10 = !lean_is_exclusive(x_7); if (x_10 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_11 = lean_ctor_get(x_7, 0); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -lean_ctor_set(x_7, 0, x_13); -x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_15 = l_Lake_mergeErrors___rarg(x_4, x_7, x_14); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +lean_ctor_set(x_7, 0, x_14); +x_15 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_16 = l_Lake_mergeErrors___rarg(x_4, x_7, x_15); x_2 = x_9; -x_4 = x_15; +x_4 = x_16; goto _start; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_7, 0); -lean_inc(x_17); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_18 = lean_ctor_get(x_7, 0); +lean_inc(x_18); lean_dec(x_7); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_mk_array(x_18, x_17); -x_20 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_19); -x_21 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_22 = l_Lake_mergeErrors___rarg(x_4, x_20, x_21); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_array_mk(x_20); +x_22 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_24 = l_Lake_mergeErrors___rarg(x_4, x_22, x_23); x_2 = x_9; -x_4 = x_22; +x_4 = x_24; goto _start; } } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_7); -if (x_24 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_7); +if (x_26 == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_26 = l_Lake_mergeErrors___rarg(x_4, x_7, x_25); +lean_object* x_27; lean_object* x_28; +x_27 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_28 = l_Lake_mergeErrors___rarg(x_4, x_7, x_27); x_2 = x_9; -x_4 = x_26; +x_4 = x_28; goto _start; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_7, 0); -lean_inc(x_28); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_7, 0); +lean_inc(x_30); lean_dec(x_7); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -x_30 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_31 = l_Lake_mergeErrors___rarg(x_4, x_29, x_30); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_30); +x_32 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_33 = l_Lake_mergeErrors___rarg(x_4, x_31, x_32); x_2 = x_9; -x_4 = x_31; +x_4 = x_33; goto _start; } } @@ -13712,34 +13657,34 @@ return x_3; LEAN_EXPORT lean_object* l_Lake_LeanLibConfig_decodeToml(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_275; lean_object* x_276; -x_275 = l_Lake_LeanOption_decodeToml___closed__10; +lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_254; lean_object* x_255; +x_254 = l_Lake_LeanOption_decodeToml___closed__10; lean_inc(x_1); -x_276 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_1, x_275, x_2); -if (lean_obj_tag(x_276) == 0) -{ -lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; -x_277 = lean_ctor_get(x_276, 0); -lean_inc(x_277); -lean_dec(x_276); -x_278 = l_Lake_LeanOption_decodeToml___closed__3; -x_279 = l_Array_append___rarg(x_278, x_277); -lean_dec(x_277); -x_280 = lean_box(0); -x_9 = x_280; -x_10 = x_279; -goto block_274; +x_255 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1(x_1, x_254, x_2); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +lean_dec(x_255); +x_257 = l_Lake_LeanOption_decodeToml___closed__3; +x_258 = l_Array_append___rarg(x_257, x_256); +lean_dec(x_256); +x_259 = lean_box(0); +x_9 = x_259; +x_10 = x_258; +goto block_253; } else { -lean_object* x_281; lean_object* x_282; -x_281 = lean_ctor_get(x_276, 0); -lean_inc(x_281); -lean_dec(x_276); -x_282 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_281; -x_10 = x_282; -goto block_274; +lean_object* x_260; lean_object* x_261; +x_260 = lean_ctor_get(x_255, 0); +lean_inc(x_260); +lean_dec(x_255); +x_261 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_260; +x_10 = x_261; +goto block_253; } block_8: { @@ -13762,814 +13707,876 @@ lean_ctor_set(x_7, 0, x_3); return x_7; } } -block_274: +block_253: { -lean_object* x_11; lean_object* x_12; lean_object* x_239; lean_object* x_240; lean_object* x_241; -x_239 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_240 = l_Lake_PackageConfig_decodeToml___closed__59; +lean_object* x_11; lean_object* x_12; lean_object* x_227; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_234 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_235 = l_Lake_PackageConfig_decodeToml___closed__60; lean_inc(x_1); -x_241 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_239, x_240, x_1); -if (lean_obj_tag(x_241) == 0) +x_236 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_234, x_235, x_1); +if (lean_obj_tag(x_236) == 0) { -lean_object* x_242; -x_242 = l_Lake_PackageConfig_decodeToml___closed__60; -x_11 = x_242; +lean_object* x_237; +x_237 = l_Lake_PackageConfig_decodeToml___closed__58; +x_11 = x_237; x_12 = x_10; -goto block_238; +goto block_226; } else { -lean_object* x_243; lean_object* x_244; -x_243 = lean_ctor_get(x_241, 0); -lean_inc(x_243); -lean_dec(x_241); -x_244 = lean_ctor_get(x_243, 1); -lean_inc(x_244); -lean_dec(x_243); -switch (lean_obj_tag(x_244)) { +lean_object* x_238; lean_object* x_239; +x_238 = lean_ctor_get(x_236, 0); +lean_inc(x_238); +lean_dec(x_236); +x_239 = lean_ctor_get(x_238, 1); +lean_inc(x_239); +lean_dec(x_238); +switch (lean_obj_tag(x_239)) { case 0: { -lean_object* x_245; -x_245 = lean_ctor_get(x_244, 1); -lean_inc(x_245); -lean_dec(x_244); -x_11 = x_245; +lean_object* x_240; +x_240 = lean_ctor_get(x_239, 1); +lean_inc(x_240); +lean_dec(x_239); +x_11 = x_240; x_12 = x_10; -goto block_238; +goto block_226; } case 2: { -lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; -x_246 = lean_ctor_get(x_244, 0); -lean_inc(x_246); -lean_dec(x_244); -x_247 = l_Lake_Glob_decodeToml___closed__2; -x_248 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_248, 0, x_246); -lean_ctor_set(x_248, 1, x_247); -x_249 = lean_unsigned_to_nat(1u); -x_250 = lean_mk_array(x_249, x_248); -x_251 = l_Array_append___rarg(x_10, x_250); -lean_dec(x_250); -x_252 = l_Lake_PackageConfig_decodeToml___closed__60; -x_11 = x_252; -x_12 = x_251; -goto block_238; +lean_object* x_241; lean_object* x_242; lean_object* x_243; +x_241 = lean_ctor_get(x_239, 0); +lean_inc(x_241); +lean_dec(x_239); +x_242 = l_Lake_Glob_decodeToml___closed__2; +x_243 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_243, 0, x_241); +lean_ctor_set(x_243, 1, x_242); +x_227 = x_243; +goto block_233; } case 3: { -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_253 = lean_ctor_get(x_244, 0); -lean_inc(x_253); -lean_dec(x_244); -x_254 = l_Lake_Glob_decodeToml___closed__2; -x_255 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_255, 0, x_253); -lean_ctor_set(x_255, 1, x_254); -x_256 = lean_unsigned_to_nat(1u); -x_257 = lean_mk_array(x_256, x_255); -x_258 = l_Array_append___rarg(x_10, x_257); -lean_dec(x_257); -x_259 = l_Lake_PackageConfig_decodeToml___closed__60; -x_11 = x_259; -x_12 = x_258; -goto block_238; +lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_244 = lean_ctor_get(x_239, 0); +lean_inc(x_244); +lean_dec(x_239); +x_245 = l_Lake_Glob_decodeToml___closed__2; +x_246 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_246, 0, x_244); +lean_ctor_set(x_246, 1, x_245); +x_227 = x_246; +goto block_233; } default: { -uint8_t x_260; -x_260 = !lean_is_exclusive(x_244); -if (x_260 == 0) +uint8_t x_247; +x_247 = !lean_is_exclusive(x_239); +if (x_247 == 0) { -lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -x_261 = lean_ctor_get(x_244, 1); -lean_dec(x_261); -x_262 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_244, 0); -lean_ctor_set(x_244, 1, x_262); -x_263 = lean_unsigned_to_nat(1u); -x_264 = lean_mk_array(x_263, x_244); -x_265 = l_Array_append___rarg(x_10, x_264); -lean_dec(x_264); -x_266 = l_Lake_PackageConfig_decodeToml___closed__60; -x_11 = x_266; -x_12 = x_265; -goto block_238; +lean_object* x_248; lean_object* x_249; +x_248 = lean_ctor_get(x_239, 1); +lean_dec(x_248); +x_249 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_239, 0); +lean_ctor_set(x_239, 1, x_249); +x_227 = x_239; +goto block_233; } else { -lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; -x_267 = lean_ctor_get(x_244, 0); -lean_inc(x_267); -lean_dec(x_244); -x_268 = l_Lake_Glob_decodeToml___closed__2; -x_269 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_269, 0, x_267); -lean_ctor_set(x_269, 1, x_268); -x_270 = lean_unsigned_to_nat(1u); -x_271 = lean_mk_array(x_270, x_269); -x_272 = l_Array_append___rarg(x_10, x_271); -lean_dec(x_271); -x_273 = l_Lake_PackageConfig_decodeToml___closed__60; -x_11 = x_273; -x_12 = x_272; -goto block_238; +lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_250 = lean_ctor_get(x_239, 0); +lean_inc(x_250); +lean_dec(x_239); +x_251 = l_Lake_Glob_decodeToml___closed__2; +x_252 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_252, 0, x_250); +lean_ctor_set(x_252, 1, x_251); +x_227 = x_252; +goto block_233; } } } } -block_238: +block_226: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_198; lean_object* x_199; lean_object* x_200; x_13 = lean_box(0); lean_inc(x_9); -x_190 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_190, 0, x_9); -lean_ctor_set(x_190, 1, x_13); -x_191 = lean_array_mk(x_190); -x_192 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_193 = l_Lake_LeanLibConfig_decodeToml___closed__2; +x_191 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_191, 0, x_9); +lean_ctor_set(x_191, 1, x_13); +x_192 = lean_array_mk(x_191); +x_198 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_199 = l_Lake_LeanLibConfig_decodeToml___closed__2; lean_inc(x_1); -x_194 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_192, x_193, x_1); -if (lean_obj_tag(x_194) == 0) +x_200 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_198, x_199, x_1); +if (lean_obj_tag(x_200) == 0) { -x_14 = x_191; +x_14 = x_192; x_15 = x_12; -goto block_189; +goto block_190; } else { -lean_object* x_195; lean_object* x_196; -x_195 = lean_ctor_get(x_194, 0); -lean_inc(x_195); -lean_dec(x_194); -x_196 = lean_ctor_get(x_195, 1); -lean_inc(x_196); -lean_dec(x_195); -switch (lean_obj_tag(x_196)) { +lean_object* x_201; lean_object* x_202; +x_201 = lean_ctor_get(x_200, 0); +lean_inc(x_201); +lean_dec(x_200); +x_202 = lean_ctor_get(x_201, 1); +lean_inc(x_202); +lean_dec(x_201); +switch (lean_obj_tag(x_202)) { case 0: { -uint8_t x_197; -x_197 = !lean_is_exclusive(x_196); -if (x_197 == 0) +uint8_t x_203; +x_203 = !lean_is_exclusive(x_202); +if (x_203 == 0) { -lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_198 = lean_ctor_get(x_196, 1); -lean_dec(x_198); -x_199 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_196, 1, x_199); -x_200 = lean_unsigned_to_nat(1u); -x_201 = lean_mk_array(x_200, x_196); -x_202 = l_Array_append___rarg(x_12, x_201); -lean_dec(x_201); -x_14 = x_191; -x_15 = x_202; -goto block_189; +lean_object* x_204; lean_object* x_205; +x_204 = lean_ctor_get(x_202, 1); +lean_dec(x_204); +x_205 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_202, 1, x_205); +x_193 = x_202; +goto block_197; } else { -lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_203 = lean_ctor_get(x_196, 0); -lean_inc(x_203); -lean_dec(x_196); -x_204 = l_Lake_LeanConfig_decodeToml___closed__5; -x_205 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_205, 0, x_203); -lean_ctor_set(x_205, 1, x_204); -x_206 = lean_unsigned_to_nat(1u); -x_207 = lean_mk_array(x_206, x_205); -x_208 = l_Array_append___rarg(x_12, x_207); -lean_dec(x_207); -x_14 = x_191; -x_15 = x_208; -goto block_189; -} -} -case 2: -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -x_209 = lean_ctor_get(x_196, 0); -lean_inc(x_209); -lean_dec(x_196); +lean_object* x_206; lean_object* x_207; lean_object* x_208; +x_206 = lean_ctor_get(x_202, 0); +lean_inc(x_206); +lean_dec(x_202); +x_207 = l_Lake_LeanConfig_decodeToml___closed__5; +x_208 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_208, 0, x_206); +lean_ctor_set(x_208, 1, x_207); +x_193 = x_208; +goto block_197; +} +} +case 2: +{ +lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_209 = lean_ctor_get(x_202, 0); +lean_inc(x_209); +lean_dec(x_202); x_210 = l_Lake_LeanConfig_decodeToml___closed__5; x_211 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_211, 0, x_209); lean_ctor_set(x_211, 1, x_210); -x_212 = lean_unsigned_to_nat(1u); -x_213 = lean_mk_array(x_212, x_211); -x_214 = l_Array_append___rarg(x_12, x_213); -lean_dec(x_213); -x_14 = x_191; -x_15 = x_214; -goto block_189; +x_193 = x_211; +goto block_197; } case 3: { -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; -x_215 = lean_ctor_get(x_196, 0); -lean_inc(x_215); -lean_dec(x_196); -x_216 = l_Lake_LeanConfig_decodeToml___closed__5; -x_217 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_217, 0, x_215); -lean_ctor_set(x_217, 1, x_216); -x_218 = lean_unsigned_to_nat(1u); -x_219 = lean_mk_array(x_218, x_217); -x_220 = l_Array_append___rarg(x_12, x_219); -lean_dec(x_219); -x_14 = x_191; -x_15 = x_220; -goto block_189; +lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_212 = lean_ctor_get(x_202, 0); +lean_inc(x_212); +lean_dec(x_202); +x_213 = l_Lake_LeanConfig_decodeToml___closed__5; +x_214 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_214, 0, x_212); +lean_ctor_set(x_214, 1, x_213); +x_193 = x_214; +goto block_197; } case 5: { -lean_object* x_221; lean_object* x_222; -x_221 = lean_ctor_get(x_196, 1); -lean_inc(x_221); -lean_dec(x_196); -x_222 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__1(x_221); -lean_dec(x_221); -if (lean_obj_tag(x_222) == 0) +lean_object* x_215; lean_object* x_216; +x_215 = lean_ctor_get(x_202, 1); +lean_inc(x_215); +lean_dec(x_202); +x_216 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__1(x_215); +lean_dec(x_215); +if (lean_obj_tag(x_216) == 0) { -lean_object* x_223; lean_object* x_224; -x_223 = lean_ctor_get(x_222, 0); -lean_inc(x_223); -lean_dec(x_222); -x_224 = l_Array_append___rarg(x_12, x_223); -lean_dec(x_223); -x_14 = x_191; -x_15 = x_224; -goto block_189; +lean_object* x_217; lean_object* x_218; +x_217 = lean_ctor_get(x_216, 0); +lean_inc(x_217); +lean_dec(x_216); +x_218 = l_Array_append___rarg(x_12, x_217); +lean_dec(x_217); +x_14 = x_192; +x_15 = x_218; +goto block_190; } else { -lean_object* x_225; -lean_dec(x_191); -x_225 = lean_ctor_get(x_222, 0); -lean_inc(x_225); -lean_dec(x_222); -x_14 = x_225; +lean_object* x_219; +lean_dec(x_192); +x_219 = lean_ctor_get(x_216, 0); +lean_inc(x_219); +lean_dec(x_216); +x_14 = x_219; x_15 = x_12; -goto block_189; +goto block_190; } } default: { -uint8_t x_226; -x_226 = !lean_is_exclusive(x_196); -if (x_226 == 0) +uint8_t x_220; +x_220 = !lean_is_exclusive(x_202); +if (x_220 == 0) { -lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_227 = lean_ctor_get(x_196, 1); -lean_dec(x_227); -x_228 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_196, 0); -lean_ctor_set(x_196, 1, x_228); -x_229 = lean_unsigned_to_nat(1u); -x_230 = lean_mk_array(x_229, x_196); -x_231 = l_Array_append___rarg(x_12, x_230); -lean_dec(x_230); -x_14 = x_191; -x_15 = x_231; -goto block_189; +lean_object* x_221; lean_object* x_222; +x_221 = lean_ctor_get(x_202, 1); +lean_dec(x_221); +x_222 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_202, 0); +lean_ctor_set(x_202, 1, x_222); +x_193 = x_202; +goto block_197; } else { -lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_232 = lean_ctor_get(x_196, 0); -lean_inc(x_232); -lean_dec(x_196); -x_233 = l_Lake_LeanConfig_decodeToml___closed__5; -x_234 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_234, 0, x_232); -lean_ctor_set(x_234, 1, x_233); -x_235 = lean_unsigned_to_nat(1u); -x_236 = lean_mk_array(x_235, x_234); -x_237 = l_Array_append___rarg(x_12, x_236); -lean_dec(x_236); -x_14 = x_191; -x_15 = x_237; -goto block_189; +lean_object* x_223; lean_object* x_224; lean_object* x_225; +x_223 = lean_ctor_get(x_202, 0); +lean_inc(x_223); +lean_dec(x_202); +x_224 = l_Lake_LeanConfig_decodeToml___closed__5; +x_225 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_225, 0, x_223); +lean_ctor_set(x_225, 1, x_224); +x_193 = x_225; +goto block_197; } } } } -block_189: +block_190: { -lean_object* x_16; lean_object* x_17; size_t x_168; size_t x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_168 = lean_array_size(x_14); -x_169 = 0; +lean_object* x_16; lean_object* x_17; size_t x_129; size_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_129 = lean_array_size(x_14); +x_130 = 0; lean_inc(x_14); -x_170 = l_Array_mapMUnsafe_map___at_Lake_LeanLibConfig_decodeToml___spec__3(x_168, x_169, x_14); -x_171 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_172 = l_Lake_LeanLibConfig_decodeToml___closed__12; +x_131 = l_Array_mapMUnsafe_map___at_Lake_LeanLibConfig_decodeToml___spec__3(x_129, x_130, x_14); +x_132 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_133 = l_Lake_LeanLibConfig_decodeToml___closed__12; lean_inc(x_1); -x_173 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_171, x_172, x_1); -if (lean_obj_tag(x_173) == 0) +x_134 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_132, x_133, x_1); +if (lean_obj_tag(x_134) == 0) { -x_16 = x_170; +x_16 = x_131; x_17 = x_15; -goto block_167; +goto block_128; } else { -lean_object* x_174; lean_object* x_175; -x_174 = lean_ctor_get(x_173, 0); -lean_inc(x_174); -lean_dec(x_173); -x_175 = lean_ctor_get(x_174, 1); -lean_inc(x_175); -lean_dec(x_174); -if (lean_obj_tag(x_175) == 5) +lean_object* x_135; lean_object* x_136; +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +lean_dec(x_134); +x_136 = lean_ctor_get(x_135, 1); +lean_inc(x_136); +lean_dec(x_135); +switch (lean_obj_tag(x_136)) { +case 1: { -lean_object* x_176; lean_object* x_177; -x_176 = lean_ctor_get(x_175, 1); -lean_inc(x_176); -lean_dec(x_175); -x_177 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__4(x_176); -lean_dec(x_176); -if (lean_obj_tag(x_177) == 0) +lean_object* x_137; uint8_t x_138; +lean_inc(x_136); +x_137 = l_Lake_Glob_decodeToml(x_136); +x_138 = !lean_is_exclusive(x_136); +if (x_138 == 0) { -lean_object* x_178; lean_object* x_179; -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -lean_dec(x_177); -x_179 = l_Array_append___rarg(x_15, x_178); -lean_dec(x_178); -x_16 = x_170; -x_17 = x_179; -goto block_167; +lean_object* x_139; lean_object* x_140; +x_139 = lean_ctor_get(x_136, 1); +lean_dec(x_139); +x_140 = lean_ctor_get(x_136, 0); +lean_dec(x_140); +if (lean_obj_tag(x_137) == 0) +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_141 = lean_ctor_get(x_137, 0); +lean_inc(x_141); +lean_dec(x_137); +lean_ctor_set(x_136, 1, x_13); +lean_ctor_set(x_136, 0, x_141); +x_142 = lean_array_mk(x_136); +x_143 = l_Array_append___rarg(x_15, x_142); +lean_dec(x_142); +x_16 = x_131; +x_17 = x_143; +goto block_128; } else { -lean_object* x_180; -lean_dec(x_170); -x_180 = lean_ctor_get(x_177, 0); -lean_inc(x_180); -lean_dec(x_177); -x_16 = x_180; +lean_object* x_144; lean_object* x_145; +lean_dec(x_131); +x_144 = lean_ctor_get(x_137, 0); +lean_inc(x_144); +lean_dec(x_137); +lean_ctor_set(x_136, 1, x_13); +lean_ctor_set(x_136, 0, x_144); +x_145 = lean_array_mk(x_136); +x_16 = x_145; x_17 = x_15; -goto block_167; +goto block_128; } } else { -lean_object* x_181; -x_181 = l_Lake_Glob_decodeToml(x_175); -if (lean_obj_tag(x_181) == 0) +lean_dec(x_136); +if (lean_obj_tag(x_137) == 0) { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_182 = lean_ctor_get(x_181, 0); -lean_inc(x_182); -lean_dec(x_181); -x_183 = lean_unsigned_to_nat(1u); -x_184 = lean_mk_array(x_183, x_182); -x_185 = l_Array_append___rarg(x_15, x_184); -lean_dec(x_184); -x_16 = x_170; -x_17 = x_185; -goto block_167; +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_146 = lean_ctor_get(x_137, 0); +lean_inc(x_146); +lean_dec(x_137); +x_147 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_13); +x_148 = lean_array_mk(x_147); +x_149 = l_Array_append___rarg(x_15, x_148); +lean_dec(x_148); +x_16 = x_131; +x_17 = x_149; +goto block_128; } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; -lean_dec(x_170); -x_186 = lean_ctor_get(x_181, 0); -lean_inc(x_186); -lean_dec(x_181); -x_187 = lean_unsigned_to_nat(1u); -x_188 = lean_mk_array(x_187, x_186); -x_16 = x_188; +lean_object* x_150; lean_object* x_151; lean_object* x_152; +lean_dec(x_131); +x_150 = lean_ctor_get(x_137, 0); +lean_inc(x_150); +lean_dec(x_137); +x_151 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_151, 0, x_150); +lean_ctor_set(x_151, 1, x_13); +x_152 = lean_array_mk(x_151); +x_16 = x_152; x_17 = x_15; -goto block_167; +goto block_128; } } } -block_167: +case 2: { -lean_object* x_18; lean_object* x_19; uint8_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_134 = 0; -x_135 = l_Lake_StrPat_decodeToml___closed__6; -lean_inc(x_9); -x_136 = l_Lean_Name_toString(x_9, x_134, x_135); -x_137 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_138 = l_Lake_LeanLibConfig_decodeToml___closed__10; -lean_inc(x_1); -x_139 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_137, x_138, x_1); -if (lean_obj_tag(x_139) == 0) +lean_object* x_153; +x_153 = l_Lake_Glob_decodeToml(x_136); +if (lean_obj_tag(x_153) == 0) { -x_18 = x_136; -x_19 = x_17; -goto block_133; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +x_155 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_155, 0, x_154); +lean_ctor_set(x_155, 1, x_13); +x_156 = lean_array_mk(x_155); +x_157 = l_Array_append___rarg(x_15, x_156); +lean_dec(x_156); +x_16 = x_131; +x_17 = x_157; +goto block_128; } else { -lean_object* x_140; lean_object* x_141; -x_140 = lean_ctor_get(x_139, 0); -lean_inc(x_140); -lean_dec(x_139); -x_141 = lean_ctor_get(x_140, 1); -lean_inc(x_141); -lean_dec(x_140); -switch (lean_obj_tag(x_141)) { -case 0: -{ -lean_object* x_142; -lean_dec(x_136); -x_142 = lean_ctor_get(x_141, 1); -lean_inc(x_142); -lean_dec(x_141); -x_18 = x_142; -x_19 = x_17; -goto block_133; +lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_131); +x_158 = lean_ctor_get(x_153, 0); +lean_inc(x_158); +lean_dec(x_153); +x_159 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_159, 0, x_158); +lean_ctor_set(x_159, 1, x_13); +x_160 = lean_array_mk(x_159); +x_16 = x_160; +x_17 = x_15; +goto block_128; } -case 2: -{ -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_143 = lean_ctor_get(x_141, 0); -lean_inc(x_143); -lean_dec(x_141); -x_144 = l_Lake_Glob_decodeToml___closed__2; -x_145 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -x_146 = lean_unsigned_to_nat(1u); -x_147 = lean_mk_array(x_146, x_145); -x_148 = l_Array_append___rarg(x_17, x_147); -lean_dec(x_147); -x_18 = x_136; -x_19 = x_148; -goto block_133; } case 3: { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; -x_149 = lean_ctor_get(x_141, 0); -lean_inc(x_149); -lean_dec(x_141); -x_150 = l_Lake_Glob_decodeToml___closed__2; -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); -x_152 = lean_unsigned_to_nat(1u); -x_153 = lean_mk_array(x_152, x_151); -x_154 = l_Array_append___rarg(x_17, x_153); -lean_dec(x_153); -x_18 = x_136; -x_19 = x_154; -goto block_133; -} -default: -{ -uint8_t x_155; -x_155 = !lean_is_exclusive(x_141); -if (x_155 == 0) +lean_object* x_161; +x_161 = l_Lake_Glob_decodeToml(x_136); +if (lean_obj_tag(x_161) == 0) { -lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; -x_156 = lean_ctor_get(x_141, 1); -lean_dec(x_156); -x_157 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_141, 0); -lean_ctor_set(x_141, 1, x_157); -x_158 = lean_unsigned_to_nat(1u); -x_159 = lean_mk_array(x_158, x_141); -x_160 = l_Array_append___rarg(x_17, x_159); -lean_dec(x_159); -x_18 = x_136; -x_19 = x_160; -goto block_133; +lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +lean_dec(x_161); +x_163 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_163, 0, x_162); +lean_ctor_set(x_163, 1, x_13); +x_164 = lean_array_mk(x_163); +x_165 = l_Array_append___rarg(x_15, x_164); +lean_dec(x_164); +x_16 = x_131; +x_17 = x_165; +goto block_128; } else { -lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_161 = lean_ctor_get(x_141, 0); -lean_inc(x_161); -lean_dec(x_141); -x_162 = l_Lake_Glob_decodeToml___closed__2; -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_161); -lean_ctor_set(x_163, 1, x_162); -x_164 = lean_unsigned_to_nat(1u); -x_165 = lean_mk_array(x_164, x_163); -x_166 = l_Array_append___rarg(x_17, x_165); -lean_dec(x_165); -x_18 = x_136; -x_19 = x_166; -goto block_133; -} -} +lean_object* x_166; lean_object* x_167; lean_object* x_168; +lean_dec(x_131); +x_166 = lean_ctor_get(x_161, 0); +lean_inc(x_166); +lean_dec(x_161); +x_167 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_167, 0, x_166); +lean_ctor_set(x_167, 1, x_13); +x_168 = lean_array_mk(x_167); +x_16 = x_168; +x_17 = x_15; +goto block_128; } } -block_133: +case 5: { -uint8_t x_20; lean_object* x_21; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_92 = l_Lake_PackageConfig_decodeToml___closed__62; -lean_inc(x_1); -x_93 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_91, x_92, x_1); -if (lean_obj_tag(x_93) == 0) +lean_object* x_169; lean_object* x_170; +x_169 = lean_ctor_get(x_136, 1); +lean_inc(x_169); +lean_dec(x_136); +x_170 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__4(x_169); +lean_dec(x_169); +if (lean_obj_tag(x_170) == 0) { -uint8_t x_94; -x_94 = 0; -x_20 = x_94; -x_21 = x_19; -goto block_90; +lean_object* x_171; lean_object* x_172; +x_171 = lean_ctor_get(x_170, 0); +lean_inc(x_171); +lean_dec(x_170); +x_172 = l_Array_append___rarg(x_15, x_171); +lean_dec(x_171); +x_16 = x_131; +x_17 = x_172; +goto block_128; } else { -lean_object* x_95; lean_object* x_96; -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -lean_dec(x_93); -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -lean_dec(x_95); -switch (lean_obj_tag(x_96)) { -case 0: +lean_object* x_173; +lean_dec(x_131); +x_173 = lean_ctor_get(x_170, 0); +lean_inc(x_173); +lean_dec(x_170); +x_16 = x_173; +x_17 = x_15; +goto block_128; +} +} +default: { -uint8_t x_97; -x_97 = !lean_is_exclusive(x_96); -if (x_97 == 0) +lean_object* x_174; uint8_t x_175; +lean_inc(x_136); +x_174 = l_Lake_Glob_decodeToml(x_136); +x_175 = !lean_is_exclusive(x_136); +if (x_175 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; -x_98 = lean_ctor_get(x_96, 1); -lean_dec(x_98); -x_99 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_96, 1, x_99); -x_100 = lean_unsigned_to_nat(1u); -x_101 = lean_mk_array(x_100, x_96); -x_102 = l_Array_append___rarg(x_19, x_101); -lean_dec(x_101); -x_103 = 0; -x_20 = x_103; -x_21 = x_102; -goto block_90; -} -else +lean_object* x_176; lean_object* x_177; +x_176 = lean_ctor_get(x_136, 1); +lean_dec(x_176); +x_177 = lean_ctor_get(x_136, 0); +lean_dec(x_177); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; -x_104 = lean_ctor_get(x_96, 0); -lean_inc(x_104); -lean_dec(x_96); -x_105 = l_Lake_LeanConfig_decodeToml___closed__20; -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -x_107 = lean_unsigned_to_nat(1u); -x_108 = lean_mk_array(x_107, x_106); -x_109 = l_Array_append___rarg(x_19, x_108); -lean_dec(x_108); -x_110 = 0; -x_20 = x_110; -x_21 = x_109; -goto block_90; -} +lean_object* x_178; lean_object* x_179; lean_object* x_180; +x_178 = lean_ctor_get(x_174, 0); +lean_inc(x_178); +lean_dec(x_174); +lean_ctor_set_tag(x_136, 1); +lean_ctor_set(x_136, 1, x_13); +lean_ctor_set(x_136, 0, x_178); +x_179 = lean_array_mk(x_136); +x_180 = l_Array_append___rarg(x_15, x_179); +lean_dec(x_179); +x_16 = x_131; +x_17 = x_180; +goto block_128; } -case 2: +else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; uint8_t x_117; -x_111 = lean_ctor_get(x_96, 0); -lean_inc(x_111); -lean_dec(x_96); -x_112 = l_Lake_LeanConfig_decodeToml___closed__20; -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -x_114 = lean_unsigned_to_nat(1u); -x_115 = lean_mk_array(x_114, x_113); -x_116 = l_Array_append___rarg(x_19, x_115); -lean_dec(x_115); -x_117 = 0; -x_20 = x_117; -x_21 = x_116; -goto block_90; +lean_object* x_181; lean_object* x_182; +lean_dec(x_131); +x_181 = lean_ctor_get(x_174, 0); +lean_inc(x_181); +lean_dec(x_174); +lean_ctor_set_tag(x_136, 1); +lean_ctor_set(x_136, 1, x_13); +lean_ctor_set(x_136, 0, x_181); +x_182 = lean_array_mk(x_136); +x_16 = x_182; +x_17 = x_15; +goto block_128; } -case 3: -{ -uint8_t x_118; -x_118 = lean_ctor_get_uint8(x_96, sizeof(void*)*1); -lean_dec(x_96); -x_20 = x_118; -x_21 = x_19; -goto block_90; } -default: +else { -uint8_t x_119; -x_119 = !lean_is_exclusive(x_96); -if (x_119 == 0) +lean_dec(x_136); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; -x_120 = lean_ctor_get(x_96, 1); -lean_dec(x_120); -x_121 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_96, 0); -lean_ctor_set(x_96, 1, x_121); -x_122 = lean_unsigned_to_nat(1u); -x_123 = lean_mk_array(x_122, x_96); -x_124 = l_Array_append___rarg(x_19, x_123); -lean_dec(x_123); -x_125 = 0; -x_20 = x_125; -x_21 = x_124; -goto block_90; +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_183 = lean_ctor_get(x_174, 0); +lean_inc(x_183); +lean_dec(x_174); +x_184 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_184, 0, x_183); +lean_ctor_set(x_184, 1, x_13); +x_185 = lean_array_mk(x_184); +x_186 = l_Array_append___rarg(x_15, x_185); +lean_dec(x_185); +x_16 = x_131; +x_17 = x_186; +goto block_128; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; uint8_t x_132; -x_126 = lean_ctor_get(x_96, 0); -lean_inc(x_126); -lean_dec(x_96); -x_127 = l_Lake_LeanConfig_decodeToml___closed__20; -x_128 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -x_129 = lean_unsigned_to_nat(1u); -x_130 = lean_mk_array(x_129, x_128); -x_131 = l_Array_append___rarg(x_19, x_130); -lean_dec(x_130); -x_132 = 0; -x_20 = x_132; -x_21 = x_131; -goto block_90; +lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_dec(x_131); +x_187 = lean_ctor_get(x_174, 0); +lean_inc(x_187); +lean_dec(x_174); +x_188 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_188, 0, x_187); +lean_ctor_set(x_188, 1, x_13); +x_189 = lean_array_mk(x_188); +x_16 = x_189; +x_17 = x_15; +goto block_128; } } } } -block_90: +} +block_128: { -lean_object* x_22; lean_object* x_23; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_37 = l_Lake_LeanLibConfig_decodeToml___closed__4; +lean_object* x_18; lean_object* x_19; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_102 = 0; +x_103 = l_Lake_StrPat_decodeToml___closed__6; +lean_inc(x_9); +x_104 = l_Lean_Name_toString(x_9, x_102, x_103); +x_110 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_111 = l_Lake_LeanLibConfig_decodeToml___closed__10; lean_inc(x_1); -x_38 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_36, x_37, x_1); -if (lean_obj_tag(x_38) == 0) +x_112 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_110, x_111, x_1); +if (lean_obj_tag(x_112) == 0) { -lean_object* x_39; -x_39 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_39; -x_23 = x_21; -goto block_35; +x_18 = x_104; +x_19 = x_17; +goto block_101; } else { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_38, 0); -lean_inc(x_40); -lean_dec(x_38); -x_41 = lean_ctor_get(x_40, 1); -lean_inc(x_41); -lean_dec(x_40); -switch (lean_obj_tag(x_41)) { +lean_object* x_113; lean_object* x_114; +x_113 = lean_ctor_get(x_112, 0); +lean_inc(x_113); +lean_dec(x_112); +x_114 = lean_ctor_get(x_113, 1); +lean_inc(x_114); +lean_dec(x_113); +switch (lean_obj_tag(x_114)) { case 0: { -uint8_t x_42; -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) +lean_object* x_115; +lean_dec(x_104); +x_115 = lean_ctor_get(x_114, 1); +lean_inc(x_115); +lean_dec(x_114); +x_18 = x_115; +x_19 = x_17; +goto block_101; +} +case 2: { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_43 = lean_ctor_get(x_41, 1); -lean_dec(x_43); -x_44 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_41, 1, x_44); -x_45 = lean_unsigned_to_nat(1u); -x_46 = lean_mk_array(x_45, x_41); -x_47 = l_Array_append___rarg(x_21, x_46); -lean_dec(x_46); -x_48 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_48; -x_23 = x_47; +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_114, 0); +lean_inc(x_116); +lean_dec(x_114); +x_117 = l_Lake_Glob_decodeToml___closed__2; +x_118 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +x_105 = x_118; +goto block_109; +} +case 3: +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_119 = lean_ctor_get(x_114, 0); +lean_inc(x_119); +lean_dec(x_114); +x_120 = l_Lake_Glob_decodeToml___closed__2; +x_121 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +x_105 = x_121; +goto block_109; +} +default: +{ +uint8_t x_122; +x_122 = !lean_is_exclusive(x_114); +if (x_122 == 0) +{ +lean_object* x_123; lean_object* x_124; +x_123 = lean_ctor_get(x_114, 1); +lean_dec(x_123); +x_124 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_114, 0); +lean_ctor_set(x_114, 1, x_124); +x_105 = x_114; +goto block_109; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_114, 0); +lean_inc(x_125); +lean_dec(x_114); +x_126 = l_Lake_Glob_decodeToml___closed__2; +x_127 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +x_105 = x_127; +goto block_109; +} +} +} +} +block_101: +{ +uint8_t x_20; lean_object* x_21; lean_object* x_73; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_80 = l_Lake_PackageConfig_decodeToml___closed__62; +lean_inc(x_1); +x_81 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_79, x_80, x_1); +if (lean_obj_tag(x_81) == 0) +{ +uint8_t x_82; +x_82 = 0; +x_20 = x_82; +x_21 = x_19; +goto block_72; +} +else +{ +lean_object* x_83; lean_object* x_84; +x_83 = lean_ctor_get(x_81, 0); +lean_inc(x_83); +lean_dec(x_81); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +switch (lean_obj_tag(x_84)) { +case 0: +{ +uint8_t x_85; +x_85 = !lean_is_exclusive(x_84); +if (x_85 == 0) +{ +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_84, 1); +lean_dec(x_86); +x_87 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_84, 1, x_87); +x_73 = x_84; +goto block_78; +} +else +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_84, 0); +lean_inc(x_88); +lean_dec(x_84); +x_89 = l_Lake_LeanConfig_decodeToml___closed__20; +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_73 = x_90; +goto block_78; +} +} +case 2: +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_84, 0); +lean_inc(x_91); +lean_dec(x_84); +x_92 = l_Lake_LeanConfig_decodeToml___closed__20; +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_73 = x_93; +goto block_78; +} +case 3: +{ +uint8_t x_94; +x_94 = lean_ctor_get_uint8(x_84, sizeof(void*)*1); +lean_dec(x_84); +x_20 = x_94; +x_21 = x_19; +goto block_72; +} +default: +{ +uint8_t x_95; +x_95 = !lean_is_exclusive(x_84); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; +x_96 = lean_ctor_get(x_84, 1); +lean_dec(x_96); +x_97 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_84, 0); +lean_ctor_set(x_84, 1, x_97); +x_73 = x_84; +goto block_78; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_84, 0); +lean_inc(x_98); +lean_dec(x_84); +x_99 = l_Lake_LeanConfig_decodeToml___closed__20; +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_98); +lean_ctor_set(x_100, 1, x_99); +x_73 = x_100; +goto block_78; +} +} +} +} +block_72: +{ +lean_object* x_22; lean_object* x_23; lean_object* x_36; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_43 = l_Lake_LeanLibConfig_decodeToml___closed__4; +lean_inc(x_1); +x_44 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_42, x_43, x_1); +if (lean_obj_tag(x_44) == 0) +{ +lean_object* x_45; +x_45 = l_Lake_LeanLibConfig_decodeToml___closed__8; +x_22 = x_45; +x_23 = x_21; goto block_35; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_49 = lean_ctor_get(x_41, 0); -lean_inc(x_49); -lean_dec(x_41); +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_44, 0); +lean_inc(x_46); +lean_dec(x_44); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +switch (lean_obj_tag(x_47)) { +case 0: +{ +uint8_t x_48; +x_48 = !lean_is_exclusive(x_47); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; +x_49 = lean_ctor_get(x_47, 1); +lean_dec(x_49); x_50 = l_Lake_LeanConfig_decodeToml___closed__5; -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_unsigned_to_nat(1u); -x_53 = lean_mk_array(x_52, x_51); -x_54 = l_Array_append___rarg(x_21, x_53); -lean_dec(x_53); -x_55 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_55; -x_23 = x_54; -goto block_35; +lean_ctor_set(x_47, 1, x_50); +x_36 = x_47; +goto block_41; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_47, 0); +lean_inc(x_51); +lean_dec(x_47); +x_52 = l_Lake_LeanConfig_decodeToml___closed__5; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_36 = x_53; +goto block_41; } } case 2: { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_41, 0); -lean_inc(x_56); -lean_dec(x_41); -x_57 = l_Lake_LeanConfig_decodeToml___closed__5; -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_unsigned_to_nat(1u); -x_60 = lean_mk_array(x_59, x_58); -x_61 = l_Array_append___rarg(x_21, x_60); -lean_dec(x_60); -x_62 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_62; -x_23 = x_61; -goto block_35; +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_47, 0); +lean_inc(x_54); +lean_dec(x_47); +x_55 = l_Lake_LeanConfig_decodeToml___closed__5; +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +x_36 = x_56; +goto block_41; } case 3: { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_63 = lean_ctor_get(x_41, 0); -lean_inc(x_63); -lean_dec(x_41); -x_64 = l_Lake_LeanConfig_decodeToml___closed__5; -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -x_66 = lean_unsigned_to_nat(1u); -x_67 = lean_mk_array(x_66, x_65); -x_68 = l_Array_append___rarg(x_21, x_67); -lean_dec(x_67); -x_69 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_69; -x_23 = x_68; -goto block_35; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_47, 0); +lean_inc(x_57); +lean_dec(x_47); +x_58 = l_Lake_LeanConfig_decodeToml___closed__5; +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +x_36 = x_59; +goto block_41; } case 5: { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_41, 1); -lean_inc(x_70); -lean_dec(x_41); -x_71 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__1(x_70); -lean_dec(x_70); -if (lean_obj_tag(x_71) == 0) +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_47, 1); +lean_inc(x_60); +lean_dec(x_47); +x_61 = l_Lake_Toml_decodeArray___at_Lake_LeanLibConfig_decodeToml___spec__1(x_60); +lean_dec(x_60); +if (lean_obj_tag(x_61) == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -lean_dec(x_71); -x_73 = l_Array_append___rarg(x_21, x_72); -lean_dec(x_72); -x_74 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_74; -x_23 = x_73; +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +lean_dec(x_61); +x_63 = l_Array_append___rarg(x_21, x_62); +lean_dec(x_62); +x_64 = l_Lake_LeanLibConfig_decodeToml___closed__8; +x_22 = x_64; +x_23 = x_63; goto block_35; } else { -lean_object* x_75; -x_75 = lean_ctor_get(x_71, 0); -lean_inc(x_75); -lean_dec(x_71); -x_22 = x_75; +lean_object* x_65; +x_65 = lean_ctor_get(x_61, 0); +lean_inc(x_65); +lean_dec(x_61); +x_22 = x_65; x_23 = x_21; goto block_35; } } default: { -uint8_t x_76; -x_76 = !lean_is_exclusive(x_41); -if (x_76 == 0) +uint8_t x_66; +x_66 = !lean_is_exclusive(x_47); +if (x_66 == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_77 = lean_ctor_get(x_41, 1); -lean_dec(x_77); -x_78 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_41, 0); -lean_ctor_set(x_41, 1, x_78); -x_79 = lean_unsigned_to_nat(1u); -x_80 = lean_mk_array(x_79, x_41); -x_81 = l_Array_append___rarg(x_21, x_80); -lean_dec(x_80); -x_82 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_82; -x_23 = x_81; -goto block_35; +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_47, 1); +lean_dec(x_67); +x_68 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_47, 0); +lean_ctor_set(x_47, 1, x_68); +x_36 = x_47; +goto block_41; } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_83 = lean_ctor_get(x_41, 0); -lean_inc(x_83); -lean_dec(x_41); -x_84 = l_Lake_LeanConfig_decodeToml___closed__5; -x_85 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -x_86 = lean_unsigned_to_nat(1u); -x_87 = lean_mk_array(x_86, x_85); -x_88 = l_Array_append___rarg(x_21, x_87); -lean_dec(x_87); -x_89 = l_Lake_LeanLibConfig_decodeToml___closed__8; -x_22 = x_89; -x_23 = x_88; -goto block_35; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_47, 0); +lean_inc(x_69); +lean_dec(x_47); +x_70 = l_Lake_LeanConfig_decodeToml___closed__5; +x_71 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +x_36 = x_71; +goto block_41; } } } @@ -14630,10 +14637,79 @@ x_4 = x_23; goto block_8; } } +block_41: +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_13); +x_38 = lean_array_mk(x_37); +x_39 = l_Array_append___rarg(x_21, x_38); +lean_dec(x_38); +x_40 = l_Lake_LeanLibConfig_decodeToml___closed__8; +x_22 = x_40; +x_23 = x_39; +goto block_35; +} +} +block_78: +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_13); +x_75 = lean_array_mk(x_74); +x_76 = l_Array_append___rarg(x_19, x_75); +lean_dec(x_75); +x_77 = 0; +x_20 = x_77; +x_21 = x_76; +goto block_72; +} +} +block_109: +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_13); +x_107 = lean_array_mk(x_106); +x_108 = l_Array_append___rarg(x_17, x_107); +lean_dec(x_107); +x_18 = x_104; +x_19 = x_108; +goto block_101; +} } } +block_197: +{ +lean_object* x_194; lean_object* x_195; lean_object* x_196; +x_194 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_194, 0, x_193); +lean_ctor_set(x_194, 1, x_13); +x_195 = lean_array_mk(x_194); +x_196 = l_Array_append___rarg(x_12, x_195); +lean_dec(x_195); +x_14 = x_192; +x_15 = x_196; +goto block_190; } } +block_233: +{ +lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +x_228 = lean_box(0); +x_229 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_229, 0, x_227); +lean_ctor_set(x_229, 1, x_228); +x_230 = lean_array_mk(x_229); +x_231 = l_Array_append___rarg(x_10, x_230); +lean_dec(x_230); +x_232 = l_Lake_PackageConfig_decodeToml___closed__58; +x_11 = x_232; +x_12 = x_231; +goto block_226; } } } @@ -14704,124 +14780,135 @@ x_4 = l_Lake_LeanLibConfig_decodeToml___lambda__1(x_1, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanLibConfig(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanLibConfig___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); lean_dec(x_1); -x_28 = l_Lake_LeanLibConfig_decodeToml(x_27, x_26); -return x_28; +x_22 = l_Lake_LeanLibConfig_decodeToml(x_21, x_20); +return x_22; } default: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_1); -if (x_29 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_1); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_1, 1); -lean_dec(x_30); -x_31 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_1, 1); +lean_dec(x_24); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_1); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_1, 1, x_25); +x_2 = x_1; +goto block_7; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_36 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_2 = x_28; +goto block_7; +} } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } +static lean_object* _init_l_Lake_instDecodeTomlLeanLibConfig___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlLeanLibConfig___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_instDecodeTomlLeanLibConfig() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlLeanLibConfig___closed__1; +return x_1; +} } static lean_object* _init_l_Lake_LeanExeConfig_decodeToml___closed__1() { _start: @@ -14890,34 +14977,34 @@ return x_3; LEAN_EXPORT lean_object* l_Lake_LeanExeConfig_decodeToml(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_192; lean_object* x_193; -x_192 = l_Lake_LeanOption_decodeToml___closed__10; +lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_152; lean_object* x_153; +x_152 = l_Lake_LeanOption_decodeToml___closed__10; lean_inc(x_1); -x_193 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_192, x_2); -if (lean_obj_tag(x_193) == 0) +x_153 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_152, x_2); +if (lean_obj_tag(x_153) == 0) { -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; -x_194 = lean_ctor_get(x_193, 0); -lean_inc(x_194); -lean_dec(x_193); -x_195 = l_Lake_LeanOption_decodeToml___closed__3; -x_196 = l_Array_append___rarg(x_195, x_194); -lean_dec(x_194); -x_197 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_197; -x_10 = x_196; -goto block_191; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +x_155 = l_Lake_LeanOption_decodeToml___closed__3; +x_156 = l_Array_append___rarg(x_155, x_154); +lean_dec(x_154); +x_157 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_157; +x_10 = x_156; +goto block_151; } else { -lean_object* x_198; lean_object* x_199; -x_198 = lean_ctor_get(x_193, 0); -lean_inc(x_198); -lean_dec(x_193); -x_199 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_198; -x_10 = x_199; -goto block_191; +lean_object* x_158; lean_object* x_159; +x_158 = lean_ctor_get(x_153, 0); +lean_inc(x_158); +lean_dec(x_153); +x_159 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_158; +x_10 = x_159; +goto block_151; } block_8: { @@ -14940,543 +15027,433 @@ lean_ctor_set(x_7, 0, x_3); return x_7; } } -block_191: +block_151: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_156; lean_object* x_157; lean_object* x_158; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_125; lean_object* x_132; lean_object* x_133; lean_object* x_134; x_11 = l_Lake_stringToLegalOrSimpleName(x_9); -x_156 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_157 = l_Lake_PackageConfig_decodeToml___closed__59; +x_132 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_133 = l_Lake_PackageConfig_decodeToml___closed__60; lean_inc(x_1); -x_158 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_156, x_157, x_1); -if (lean_obj_tag(x_158) == 0) +x_134 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_132, x_133, x_1); +if (lean_obj_tag(x_134) == 0) { -lean_object* x_159; -x_159 = l_Lake_PackageConfig_decodeToml___closed__60; -x_12 = x_159; +lean_object* x_135; +x_135 = l_Lake_PackageConfig_decodeToml___closed__58; +x_12 = x_135; x_13 = x_10; -goto block_155; +goto block_124; } else { -lean_object* x_160; lean_object* x_161; -x_160 = lean_ctor_get(x_158, 0); -lean_inc(x_160); -lean_dec(x_158); -x_161 = lean_ctor_get(x_160, 1); -lean_inc(x_161); -lean_dec(x_160); -switch (lean_obj_tag(x_161)) { +lean_object* x_136; lean_object* x_137; +x_136 = lean_ctor_get(x_134, 0); +lean_inc(x_136); +lean_dec(x_134); +x_137 = lean_ctor_get(x_136, 1); +lean_inc(x_137); +lean_dec(x_136); +switch (lean_obj_tag(x_137)) { case 0: { -lean_object* x_162; -x_162 = lean_ctor_get(x_161, 1); -lean_inc(x_162); -lean_dec(x_161); -x_12 = x_162; +lean_object* x_138; +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +x_12 = x_138; x_13 = x_10; -goto block_155; +goto block_124; } case 2: { -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -x_163 = lean_ctor_get(x_161, 0); -lean_inc(x_163); -lean_dec(x_161); -x_164 = l_Lake_Glob_decodeToml___closed__2; -x_165 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_165, 0, x_163); -lean_ctor_set(x_165, 1, x_164); -x_166 = lean_unsigned_to_nat(1u); -x_167 = lean_mk_array(x_166, x_165); -x_168 = l_Array_append___rarg(x_10, x_167); -lean_dec(x_167); -x_169 = l_Lake_PackageConfig_decodeToml___closed__60; -x_12 = x_169; -x_13 = x_168; -goto block_155; +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_137, 0); +lean_inc(x_139); +lean_dec(x_137); +x_140 = l_Lake_Glob_decodeToml___closed__2; +x_141 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_141, 0, x_139); +lean_ctor_set(x_141, 1, x_140); +x_125 = x_141; +goto block_131; } case 3: { -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -x_170 = lean_ctor_get(x_161, 0); -lean_inc(x_170); -lean_dec(x_161); -x_171 = l_Lake_Glob_decodeToml___closed__2; -x_172 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_172, 0, x_170); -lean_ctor_set(x_172, 1, x_171); -x_173 = lean_unsigned_to_nat(1u); -x_174 = lean_mk_array(x_173, x_172); -x_175 = l_Array_append___rarg(x_10, x_174); -lean_dec(x_174); -x_176 = l_Lake_PackageConfig_decodeToml___closed__60; -x_12 = x_176; -x_13 = x_175; -goto block_155; +lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_142 = lean_ctor_get(x_137, 0); +lean_inc(x_142); +lean_dec(x_137); +x_143 = l_Lake_Glob_decodeToml___closed__2; +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_142); +lean_ctor_set(x_144, 1, x_143); +x_125 = x_144; +goto block_131; } default: { -uint8_t x_177; -x_177 = !lean_is_exclusive(x_161); -if (x_177 == 0) +uint8_t x_145; +x_145 = !lean_is_exclusive(x_137); +if (x_145 == 0) { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_178 = lean_ctor_get(x_161, 1); -lean_dec(x_178); -x_179 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_161, 0); -lean_ctor_set(x_161, 1, x_179); -x_180 = lean_unsigned_to_nat(1u); -x_181 = lean_mk_array(x_180, x_161); -x_182 = l_Array_append___rarg(x_10, x_181); -lean_dec(x_181); -x_183 = l_Lake_PackageConfig_decodeToml___closed__60; -x_12 = x_183; -x_13 = x_182; -goto block_155; +lean_object* x_146; lean_object* x_147; +x_146 = lean_ctor_get(x_137, 1); +lean_dec(x_146); +x_147 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_137, 0); +lean_ctor_set(x_137, 1, x_147); +x_125 = x_137; +goto block_131; } else { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_184 = lean_ctor_get(x_161, 0); -lean_inc(x_184); -lean_dec(x_161); -x_185 = l_Lake_Glob_decodeToml___closed__2; -x_186 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_186, 0, x_184); -lean_ctor_set(x_186, 1, x_185); -x_187 = lean_unsigned_to_nat(1u); -x_188 = lean_mk_array(x_187, x_186); -x_189 = l_Array_append___rarg(x_10, x_188); -lean_dec(x_188); -x_190 = l_Lake_PackageConfig_decodeToml___closed__60; -x_12 = x_190; -x_13 = x_189; -goto block_155; +lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_148 = lean_ctor_get(x_137, 0); +lean_inc(x_148); +lean_dec(x_137); +x_149 = l_Lake_Glob_decodeToml___closed__2; +x_150 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 1, x_149); +x_125 = x_150; +goto block_131; } } } } -block_155: +block_124: { -lean_object* x_14; lean_object* x_15; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_111 = l_Lake_LeanExeConfig_decodeToml___closed__7; +lean_object* x_14; lean_object* x_15; lean_object* x_91; lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_98 = l_Lake_LeanExeConfig_decodeToml___closed__7; lean_inc(x_1); -x_112 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_110, x_111, x_1); -if (lean_obj_tag(x_112) == 0) +x_99 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_97, x_98, x_1); +if (lean_obj_tag(x_99) == 0) { lean_inc(x_11); x_14 = x_11; x_15 = x_13; -goto block_109; +goto block_90; } else { -lean_object* x_113; lean_object* x_114; -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -lean_dec(x_112); -x_114 = lean_ctor_get(x_113, 1); -lean_inc(x_114); -lean_dec(x_113); -switch (lean_obj_tag(x_114)) { +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +switch (lean_obj_tag(x_101)) { case 0: { -uint8_t x_115; -x_115 = !lean_is_exclusive(x_114); -if (x_115 == 0) -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_116 = lean_ctor_get(x_114, 0); -x_117 = lean_ctor_get(x_114, 1); -x_118 = l_String_toName(x_117); -if (lean_obj_tag(x_118) == 0) +uint8_t x_102; +x_102 = !lean_is_exclusive(x_101); +if (x_102 == 0) { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_119 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -lean_ctor_set(x_114, 1, x_119); -x_120 = lean_unsigned_to_nat(1u); -x_121 = lean_mk_array(x_120, x_114); -x_122 = l_Array_append___rarg(x_13, x_121); -lean_dec(x_121); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_122; -goto block_109; +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_101, 0); +x_104 = lean_ctor_get(x_101, 1); +x_105 = l_String_toName(x_104); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; +x_106 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +lean_ctor_set(x_101, 1, x_106); +x_91 = x_101; +goto block_96; } else { -lean_free_object(x_114); -lean_dec(x_116); -x_14 = x_118; +lean_free_object(x_101); +lean_dec(x_103); +x_14 = x_105; x_15 = x_13; -goto block_109; +goto block_90; } } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_114, 0); -x_124 = lean_ctor_get(x_114, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_114); -x_125 = l_String_toName(x_124); -if (lean_obj_tag(x_125) == 0) +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_101, 0); +x_108 = lean_ctor_get(x_101, 1); +lean_inc(x_108); +lean_inc(x_107); +lean_dec(x_101); +x_109 = l_String_toName(x_108); +if (lean_obj_tag(x_109) == 0) { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_126 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_123); -lean_ctor_set(x_127, 1, x_126); -x_128 = lean_unsigned_to_nat(1u); -x_129 = lean_mk_array(x_128, x_127); -x_130 = l_Array_append___rarg(x_13, x_129); -lean_dec(x_129); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_130; -goto block_109; +lean_object* x_110; lean_object* x_111; +x_110 = l_Lake_Toml_decodeKeyval___at_Lake_LeanOption_decodeToml___spec__2___closed__1; +x_111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_111, 0, x_107); +lean_ctor_set(x_111, 1, x_110); +x_91 = x_111; +goto block_96; } else { -lean_dec(x_123); -x_14 = x_125; +lean_dec(x_107); +x_14 = x_109; x_15 = x_13; -goto block_109; +goto block_90; } } } case 2: { -lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; -x_131 = lean_ctor_get(x_114, 0); -lean_inc(x_131); -lean_dec(x_114); -x_132 = l_Lake_Glob_decodeToml___closed__2; -x_133 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_133, 0, x_131); -lean_ctor_set(x_133, 1, x_132); -x_134 = lean_unsigned_to_nat(1u); -x_135 = lean_mk_array(x_134, x_133); -x_136 = l_Array_append___rarg(x_13, x_135); -lean_dec(x_135); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_136; -goto block_109; +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_101, 0); +lean_inc(x_112); +lean_dec(x_101); +x_113 = l_Lake_Glob_decodeToml___closed__2; +x_114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +x_91 = x_114; +goto block_96; } case 3: { -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; -x_137 = lean_ctor_get(x_114, 0); -lean_inc(x_137); -lean_dec(x_114); -x_138 = l_Lake_Glob_decodeToml___closed__2; -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -x_140 = lean_unsigned_to_nat(1u); -x_141 = lean_mk_array(x_140, x_139); -x_142 = l_Array_append___rarg(x_13, x_141); -lean_dec(x_141); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_142; -goto block_109; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_101, 0); +lean_inc(x_115); +lean_dec(x_101); +x_116 = l_Lake_Glob_decodeToml___closed__2; +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +x_91 = x_117; +goto block_96; } default: { -uint8_t x_143; -x_143 = !lean_is_exclusive(x_114); -if (x_143 == 0) +uint8_t x_118; +x_118 = !lean_is_exclusive(x_101); +if (x_118 == 0) { -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_144 = lean_ctor_get(x_114, 1); -lean_dec(x_144); -x_145 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_114, 0); -lean_ctor_set(x_114, 1, x_145); -x_146 = lean_unsigned_to_nat(1u); -x_147 = lean_mk_array(x_146, x_114); -x_148 = l_Array_append___rarg(x_13, x_147); -lean_dec(x_147); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_148; -goto block_109; +lean_object* x_119; lean_object* x_120; +x_119 = lean_ctor_get(x_101, 1); +lean_dec(x_119); +x_120 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_101, 0); +lean_ctor_set(x_101, 1, x_120); +x_91 = x_101; +goto block_96; } else { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; -x_149 = lean_ctor_get(x_114, 0); -lean_inc(x_149); -lean_dec(x_114); -x_150 = l_Lake_Glob_decodeToml___closed__2; -x_151 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_151, 0, x_149); -lean_ctor_set(x_151, 1, x_150); -x_152 = lean_unsigned_to_nat(1u); -x_153 = lean_mk_array(x_152, x_151); -x_154 = l_Array_append___rarg(x_13, x_153); -lean_dec(x_153); -lean_inc(x_11); -x_14 = x_11; -x_15 = x_154; -goto block_109; +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_101, 0); +lean_inc(x_121); +lean_dec(x_101); +x_122 = l_Lake_Glob_decodeToml___closed__2; +x_123 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_123, 0, x_121); +lean_ctor_set(x_123, 1, x_122); +x_91 = x_123; +goto block_96; } } } } -block_109: +block_90: { -lean_object* x_16; lean_object* x_17; lean_object* x_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_75 = l_Lake_PackageConfig_decodeToml___closed__5; -x_76 = 0; -x_77 = l_Lake_StrPat_decodeToml___closed__6; +lean_object* x_16; lean_object* x_17; lean_object* x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_62 = l_Lake_PackageConfig_decodeToml___closed__5; +x_63 = 0; +x_64 = l_Lake_StrPat_decodeToml___closed__6; lean_inc(x_11); -x_78 = l_Lean_Name_toStringWithSep(x_75, x_76, x_11, x_77); -x_79 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_80 = l_Lake_LeanExeConfig_decodeToml___closed__5; +x_65 = l_Lean_Name_toStringWithSep(x_62, x_63, x_11, x_64); +x_72 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_73 = l_Lake_LeanExeConfig_decodeToml___closed__5; lean_inc(x_1); -x_81 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_79, x_80, x_1); -if (lean_obj_tag(x_81) == 0) +x_74 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_72, x_73, x_1); +if (lean_obj_tag(x_74) == 0) { -x_16 = x_78; +x_16 = x_65; x_17 = x_15; -goto block_74; +goto block_61; } else { -lean_object* x_82; lean_object* x_83; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -lean_dec(x_81); -x_83 = lean_ctor_get(x_82, 1); -lean_inc(x_83); -lean_dec(x_82); -switch (lean_obj_tag(x_83)) { +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +lean_dec(x_75); +switch (lean_obj_tag(x_76)) { case 0: { -lean_object* x_84; -lean_dec(x_78); -x_84 = lean_ctor_get(x_83, 1); -lean_inc(x_84); -lean_dec(x_83); -x_16 = x_84; +lean_object* x_77; +lean_dec(x_65); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_16 = x_77; x_17 = x_15; -goto block_74; +goto block_61; } case 2: { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_85 = lean_ctor_get(x_83, 0); -lean_inc(x_85); -lean_dec(x_83); -x_86 = l_Lake_Glob_decodeToml___closed__2; -x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_86); -x_88 = lean_unsigned_to_nat(1u); -x_89 = lean_mk_array(x_88, x_87); -x_90 = l_Array_append___rarg(x_15, x_89); -lean_dec(x_89); -x_16 = x_78; -x_17 = x_90; -goto block_74; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_76, 0); +lean_inc(x_78); +lean_dec(x_76); +x_79 = l_Lake_Glob_decodeToml___closed__2; +x_80 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +x_66 = x_80; +goto block_71; } case 3: { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_91 = lean_ctor_get(x_83, 0); -lean_inc(x_91); -lean_dec(x_83); -x_92 = l_Lake_Glob_decodeToml___closed__2; -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -x_94 = lean_unsigned_to_nat(1u); -x_95 = lean_mk_array(x_94, x_93); -x_96 = l_Array_append___rarg(x_15, x_95); -lean_dec(x_95); -x_16 = x_78; -x_17 = x_96; -goto block_74; +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_76, 0); +lean_inc(x_81); +lean_dec(x_76); +x_82 = l_Lake_Glob_decodeToml___closed__2; +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_81); +lean_ctor_set(x_83, 1, x_82); +x_66 = x_83; +goto block_71; } default: { -uint8_t x_97; -x_97 = !lean_is_exclusive(x_83); -if (x_97 == 0) +uint8_t x_84; +x_84 = !lean_is_exclusive(x_76); +if (x_84 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_98 = lean_ctor_get(x_83, 1); -lean_dec(x_98); -x_99 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_83, 0); -lean_ctor_set(x_83, 1, x_99); -x_100 = lean_unsigned_to_nat(1u); -x_101 = lean_mk_array(x_100, x_83); -x_102 = l_Array_append___rarg(x_15, x_101); -lean_dec(x_101); -x_16 = x_78; -x_17 = x_102; -goto block_74; +lean_object* x_85; lean_object* x_86; +x_85 = lean_ctor_get(x_76, 1); +lean_dec(x_85); +x_86 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_76, 0); +lean_ctor_set(x_76, 1, x_86); +x_66 = x_76; +goto block_71; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_103 = lean_ctor_get(x_83, 0); -lean_inc(x_103); -lean_dec(x_83); -x_104 = l_Lake_Glob_decodeToml___closed__2; -x_105 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -x_106 = lean_unsigned_to_nat(1u); -x_107 = lean_mk_array(x_106, x_105); -x_108 = l_Array_append___rarg(x_15, x_107); -lean_dec(x_107); -x_16 = x_78; -x_17 = x_108; -goto block_74; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_76, 0); +lean_inc(x_87); +lean_dec(x_76); +x_88 = l_Lake_Glob_decodeToml___closed__2; +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_66 = x_89; +goto block_71; } } } } -block_74: +block_61: { -uint8_t x_18; lean_object* x_19; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_33 = l_Lake_LeanExeConfig_decodeToml___closed__3; +uint8_t x_18; lean_object* x_19; lean_object* x_32; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_40 = l_Lake_LeanExeConfig_decodeToml___closed__3; lean_inc(x_1); -x_34 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_32, x_33, x_1); -if (lean_obj_tag(x_34) == 0) +x_41 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_39, x_40, x_1); +if (lean_obj_tag(x_41) == 0) { -uint8_t x_35; -x_35 = 0; -x_18 = x_35; +uint8_t x_42; +x_42 = 0; +x_18 = x_42; x_19 = x_17; goto block_31; } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_ctor_get(x_36, 1); -lean_inc(x_37); -lean_dec(x_36); -switch (lean_obj_tag(x_37)) { +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_41, 0); +lean_inc(x_43); +lean_dec(x_41); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +switch (lean_obj_tag(x_44)) { case 0: { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +uint8_t x_45; +x_45 = !lean_is_exclusive(x_44); +if (x_45 == 0) { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_39 = lean_ctor_get(x_37, 1); -lean_dec(x_39); -x_40 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set(x_37, 1, x_40); -x_41 = lean_unsigned_to_nat(1u); -x_42 = lean_mk_array(x_41, x_37); -x_43 = l_Array_append___rarg(x_17, x_42); -lean_dec(x_42); -x_44 = 0; -x_18 = x_44; -x_19 = x_43; -goto block_31; +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_44, 1); +lean_dec(x_46); +x_47 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set(x_44, 1, x_47); +x_32 = x_44; +goto block_38; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; -x_45 = lean_ctor_get(x_37, 0); -lean_inc(x_45); -lean_dec(x_37); -x_46 = l_Lake_LeanConfig_decodeToml___closed__20; -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -x_48 = lean_unsigned_to_nat(1u); -x_49 = lean_mk_array(x_48, x_47); -x_50 = l_Array_append___rarg(x_17, x_49); -lean_dec(x_49); -x_51 = 0; -x_18 = x_51; -x_19 = x_50; -goto block_31; +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_44, 0); +lean_inc(x_48); +lean_dec(x_44); +x_49 = l_Lake_LeanConfig_decodeToml___closed__20; +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +x_32 = x_50; +goto block_38; } } case 2: { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_52 = lean_ctor_get(x_37, 0); -lean_inc(x_52); -lean_dec(x_37); -x_53 = l_Lake_LeanConfig_decodeToml___closed__20; -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_unsigned_to_nat(1u); -x_56 = lean_mk_array(x_55, x_54); -x_57 = l_Array_append___rarg(x_17, x_56); -lean_dec(x_56); -x_58 = 0; -x_18 = x_58; -x_19 = x_57; -goto block_31; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_44, 0); +lean_inc(x_51); +lean_dec(x_44); +x_52 = l_Lake_LeanConfig_decodeToml___closed__20; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_32 = x_53; +goto block_38; } case 3: { -uint8_t x_59; -x_59 = lean_ctor_get_uint8(x_37, sizeof(void*)*1); -lean_dec(x_37); -x_18 = x_59; +uint8_t x_54; +x_54 = lean_ctor_get_uint8(x_44, sizeof(void*)*1); +lean_dec(x_44); +x_18 = x_54; x_19 = x_17; goto block_31; } default: { -uint8_t x_60; -x_60 = !lean_is_exclusive(x_37); -if (x_60 == 0) +uint8_t x_55; +x_55 = !lean_is_exclusive(x_44); +if (x_55 == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; -x_61 = lean_ctor_get(x_37, 1); -lean_dec(x_61); -x_62 = l_Lake_LeanConfig_decodeToml___closed__20; -lean_ctor_set_tag(x_37, 0); -lean_ctor_set(x_37, 1, x_62); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_mk_array(x_63, x_37); -x_65 = l_Array_append___rarg(x_17, x_64); -lean_dec(x_64); -x_66 = 0; -x_18 = x_66; -x_19 = x_65; -goto block_31; +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_44, 1); +lean_dec(x_56); +x_57 = l_Lake_LeanConfig_decodeToml___closed__20; +lean_ctor_set_tag(x_44, 0); +lean_ctor_set(x_44, 1, x_57); +x_32 = x_44; +goto block_38; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -x_67 = lean_ctor_get(x_37, 0); -lean_inc(x_67); -lean_dec(x_37); -x_68 = l_Lake_LeanConfig_decodeToml___closed__20; -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -x_70 = lean_unsigned_to_nat(1u); -x_71 = lean_mk_array(x_70, x_69); -x_72 = l_Array_append___rarg(x_17, x_71); -lean_dec(x_71); -x_73 = 0; -x_18 = x_73; -x_19 = x_72; -goto block_31; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_44, 0); +lean_inc(x_58); +lean_dec(x_44); +x_59 = l_Lake_LeanConfig_decodeToml___closed__20; +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +x_32 = x_60; +goto block_38; } } } @@ -15531,129 +15508,199 @@ x_4 = x_19; goto block_8; } } +block_38: +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_array_mk(x_34); +x_36 = l_Array_append___rarg(x_17, x_35); +lean_dec(x_35); +x_37 = 0; +x_18 = x_37; +x_19 = x_36; +goto block_31; +} +} +block_71: +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_67 = lean_box(0); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +x_69 = lean_array_mk(x_68); +x_70 = l_Array_append___rarg(x_15, x_69); +lean_dec(x_69); +x_16 = x_65; +x_17 = x_70; +goto block_61; +} +} +block_96: +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_92 = lean_box(0); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_94 = lean_array_mk(x_93); +x_95 = l_Array_append___rarg(x_13, x_94); +lean_dec(x_94); +lean_inc(x_11); +x_14 = x_11; +x_15 = x_95; +goto block_90; } } +block_131: +{ +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_126 = lean_box(0); +x_127 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +x_128 = lean_array_mk(x_127); +x_129 = l_Array_append___rarg(x_10, x_128); +lean_dec(x_128); +x_130 = l_Lake_PackageConfig_decodeToml___closed__58; +x_12 = x_130; +x_13 = x_129; +goto block_124; } } } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanExeConfig(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlLeanExeConfig___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); lean_dec(x_1); -x_28 = l_Lake_LeanExeConfig_decodeToml(x_27, x_26); -return x_28; +x_22 = l_Lake_LeanExeConfig_decodeToml(x_21, x_20); +return x_22; } default: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_1); -if (x_29 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_1); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_1, 1); -lean_dec(x_30); -x_31 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_1, 1); +lean_dec(x_24); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_1); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_1, 1, x_25); +x_2 = x_1; +goto block_7; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_36 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_2 = x_28; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} } +static lean_object* _init_l_Lake_instDecodeTomlLeanExeConfig___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlLeanExeConfig___lambda__1), 1, 0); +return x_1; } } +static lean_object* _init_l_Lake_instDecodeTomlLeanExeConfig() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlLeanExeConfig___closed__1; +return x_1; } } LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_DependencySrc_decodeToml___spec__3(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { @@ -15728,87 +15775,84 @@ lean_object* x_3; switch (lean_obj_tag(x_2)) { case 0: { -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_2, 1); +lean_inc(x_12); lean_dec(x_2); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_9); -return x_10; +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_12); +return x_13; } case 2: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_2, 0); -lean_inc(x_11); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); lean_dec(x_2); -x_12 = l_Lake_Glob_decodeToml___closed__2; -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_13); -x_3 = x_15; -goto block_8; +x_15 = l_Lake_Glob_decodeToml___closed__2; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_3 = x_16; +goto block_11; } case 3: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_2, 0); -lean_inc(x_16); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_2, 0); +lean_inc(x_17); lean_dec(x_2); -x_17 = l_Lake_Glob_decodeToml___closed__2; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_18); -x_3 = x_20; -goto block_8; +x_18 = l_Lake_Glob_decodeToml___closed__2; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_3 = x_19; +goto block_11; } default: { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_2); -if (x_21 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_2); +if (x_20 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_2, 1); -lean_dec(x_22); -x_23 = l_Lake_Glob_decodeToml___closed__2; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_2, 1); +lean_dec(x_21); +x_22 = l_Lake_Glob_decodeToml___closed__2; lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_23); -x_24 = lean_unsigned_to_nat(1u); -x_25 = lean_mk_array(x_24, x_2); -x_3 = x_25; -goto block_8; +lean_ctor_set(x_2, 1, x_22); +x_3 = x_2; +goto block_11; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_26 = lean_ctor_get(x_2, 0); -lean_inc(x_26); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_2, 0); +lean_inc(x_23); lean_dec(x_2); -x_27 = l_Lake_Glob_decodeToml___closed__2; -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_mk_array(x_29, x_28); -x_3 = x_30; -goto block_8; +x_24 = l_Lake_Glob_decodeToml___closed__2; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_3 = x_25; +goto block_11; } } } -block_8: +block_11: { -size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; -x_4 = lean_array_size(x_3); -x_5 = 0; -x_6 = l_Array_mapMUnsafe_map___at_Lake_DependencySrc_decodeToml___spec__3(x_1, x_4, x_5, x_3); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_4; lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +x_7 = lean_array_size(x_6); +x_8 = 0; +x_9 = l_Array_mapMUnsafe_map___at_Lake_DependencySrc_decodeToml___spec__3(x_1, x_7, x_8, x_6); +x_10 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; } } } @@ -15821,7 +15865,7 @@ lean_inc(x_2); x_5 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_4, x_2, x_1); if (lean_obj_tag(x_5) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; x_6 = l_Lake_Toml_ppKey(x_2); lean_dec(x_2); x_7 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__2; @@ -15832,25 +15876,28 @@ x_10 = lean_string_append(x_8, x_9); x_11 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_11, 0, x_3); lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_array_mk(x_13); +x_15 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_dec(x_3); -x_15 = lean_ctor_get(x_5, 0); -lean_inc(x_15); -lean_dec(x_5); -x_16 = lean_ctor_get(x_15, 1); +x_16 = lean_ctor_get(x_5, 0); lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lake_Toml_decodeKeyval___at_Lake_DependencySrc_decodeToml___spec__2(x_2, x_16); +lean_dec(x_5); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lake_Toml_decodeKeyval___at_Lake_DependencySrc_decodeToml___spec__2(x_2, x_17); lean_dec(x_2); -return x_17; +return x_18; } } } @@ -15953,9 +16000,11 @@ static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(1u); +x_1 = lean_box(0); x_2 = l_Lake_DependencySrc_decodeToml___closed__10; -x_3 = lean_mk_array(x_1, x_2); +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } @@ -15964,12 +16013,21 @@ static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__12() { { lean_object* x_1; lean_object* x_2; x_1 = l_Lake_DependencySrc_decodeToml___closed__11; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lake_DependencySrc_decodeToml___closed__12; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__13() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__14() { _start: { lean_object* x_1; @@ -15977,7 +16035,7 @@ x_1 = lean_mk_string_unchecked("path", 4, 4); return x_1; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__14() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__15() { _start: { lean_object* x_1; @@ -15985,7 +16043,7 @@ x_1 = lean_mk_string_unchecked("git", 3, 3); return x_1; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__15() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__16() { _start: { lean_object* x_1; @@ -15993,7 +16051,7 @@ x_1 = lean_mk_string_unchecked("expected one of 'path' or 'git'", 31, 31); return x_1; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__16() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__17() { _start: { lean_object* x_1; @@ -16001,17 +16059,17 @@ x_1 = lean_mk_string_unchecked("url", 3, 3); return x_1; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__17() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lake_DependencySrc_decodeToml___closed__16; +x_2 = l_Lake_DependencySrc_decodeToml___closed__17; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__18() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__19() { _start: { lean_object* x_1; @@ -16019,12 +16077,12 @@ x_1 = lean_mk_string_unchecked("dir", 3, 3); return x_1; } } -static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__19() { +static lean_object* _init_l_Lake_DependencySrc_decodeToml___closed__20() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lake_DependencySrc_decodeToml___closed__18; +x_2 = l_Lake_DependencySrc_decodeToml___closed__19; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -16032,566 +16090,548 @@ return x_3; LEAN_EXPORT lean_object* l_Lake_DependencySrc_decodeToml(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_135 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_136 = l_Lake_DependencySrc_decodeToml___closed__6; +lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_99; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_105 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_106 = l_Lake_DependencySrc_decodeToml___closed__6; lean_inc(x_1); -x_137 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_135, x_136, x_1); -if (lean_obj_tag(x_137) == 0) +x_107 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_105, x_106, x_1); +if (lean_obj_tag(x_107) == 0) { -lean_object* x_138; +lean_object* x_108; lean_dec(x_2); lean_dec(x_1); -x_138 = l_Lake_DependencySrc_decodeToml___closed__12; -return x_138; +x_108 = l_Lake_DependencySrc_decodeToml___closed__13; +return x_108; } else { -uint8_t x_139; -x_139 = !lean_is_exclusive(x_137); -if (x_139 == 0) +uint8_t x_109; +x_109 = !lean_is_exclusive(x_107); +if (x_109 == 0) { -lean_object* x_140; lean_object* x_141; -x_140 = lean_ctor_get(x_137, 0); -x_141 = lean_ctor_get(x_140, 1); -lean_inc(x_141); -lean_dec(x_140); -switch (lean_obj_tag(x_141)) { +lean_object* x_110; lean_object* x_111; +x_110 = lean_ctor_get(x_107, 0); +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +lean_dec(x_110); +switch (lean_obj_tag(x_111)) { case 0: { -uint8_t x_142; -x_142 = !lean_is_exclusive(x_141); -if (x_142 == 0) +uint8_t x_112; +x_112 = !lean_is_exclusive(x_111); +if (x_112 == 0) { -lean_object* x_143; lean_object* x_144; lean_object* x_145; uint8_t x_146; -x_143 = lean_ctor_get(x_141, 0); -x_144 = lean_ctor_get(x_141, 1); -x_145 = l_Lake_DependencySrc_decodeToml___closed__13; -x_146 = lean_string_dec_eq(x_144, x_145); -if (x_146 == 0) +lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; +x_113 = lean_ctor_get(x_111, 0); +x_114 = lean_ctor_get(x_111, 1); +x_115 = l_Lake_DependencySrc_decodeToml___closed__14; +x_116 = lean_string_dec_eq(x_114, x_115); +if (x_116 == 0) { -lean_object* x_147; uint8_t x_148; -x_147 = l_Lake_DependencySrc_decodeToml___closed__14; -x_148 = lean_string_dec_eq(x_144, x_147); -lean_dec(x_144); -if (x_148 == 0) +lean_object* x_117; uint8_t x_118; +x_117 = l_Lake_DependencySrc_decodeToml___closed__15; +x_118 = lean_string_dec_eq(x_114, x_117); +lean_dec(x_114); +if (x_118 == 0) { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_dec(x_2); lean_dec(x_1); -x_149 = lean_box(0); -x_150 = l_Lake_DependencySrc_decodeToml___closed__15; -lean_ctor_set(x_141, 1, x_150); -x_151 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_151, 0, x_141); -lean_ctor_set(x_151, 1, x_149); -x_152 = lean_array_mk(x_151); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_152); -return x_137; +x_119 = lean_box(0); +x_120 = l_Lake_DependencySrc_decodeToml___closed__16; +lean_ctor_set(x_111, 1, x_120); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_111); +lean_ctor_set(x_121, 1, x_119); +x_122 = lean_array_mk(x_121); +lean_ctor_set_tag(x_107, 0); +lean_ctor_set(x_107, 0, x_122); +return x_107; } else { -lean_object* x_153; lean_object* x_154; -lean_free_object(x_141); -lean_dec(x_143); -lean_free_object(x_137); -x_153 = l_Lake_DependencySrc_decodeToml___closed__17; +lean_object* x_123; lean_object* x_124; +lean_free_object(x_111); +lean_dec(x_113); +lean_free_object(x_107); +x_123 = l_Lake_DependencySrc_decodeToml___closed__18; lean_inc(x_1); -x_154 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_153, x_2); -if (lean_obj_tag(x_154) == 0) +x_124 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_123, x_2); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_155 = lean_ctor_get(x_154, 0); -lean_inc(x_155); -lean_dec(x_154); -x_156 = l_Lake_LeanOption_decodeToml___closed__3; -x_157 = l_Array_append___rarg(x_156, x_155); -lean_dec(x_155); -x_158 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_158; -x_10 = x_157; -goto block_134; +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_125 = lean_ctor_get(x_124, 0); +lean_inc(x_125); +lean_dec(x_124); +x_126 = l_Lake_LeanOption_decodeToml___closed__3; +x_127 = l_Array_append___rarg(x_126, x_125); +lean_dec(x_125); +x_128 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_128; +x_10 = x_127; +goto block_98; } else { -lean_object* x_159; lean_object* x_160; -x_159 = lean_ctor_get(x_154, 0); -lean_inc(x_159); -lean_dec(x_154); -x_160 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_159; -x_10 = x_160; -goto block_134; +lean_object* x_129; lean_object* x_130; +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_129; +x_10 = x_130; +goto block_98; } } } else { -lean_object* x_161; lean_object* x_162; lean_object* x_163; -lean_free_object(x_141); -lean_dec(x_144); -lean_dec(x_143); +lean_object* x_131; lean_object* x_132; lean_object* x_133; +lean_free_object(x_111); +lean_dec(x_114); +lean_dec(x_113); lean_dec(x_2); -x_161 = l_Lake_DependencySrc_decodeToml___closed__19; -x_162 = lean_box(0); -x_163 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_161, x_162); -if (lean_obj_tag(x_163) == 0) +x_131 = l_Lake_DependencySrc_decodeToml___closed__20; +x_132 = lean_box(0); +x_133 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_131, x_132); +if (lean_obj_tag(x_133) == 0) { -uint8_t x_164; -lean_free_object(x_137); -x_164 = !lean_is_exclusive(x_163); -if (x_164 == 0) +uint8_t x_134; +lean_free_object(x_107); +x_134 = !lean_is_exclusive(x_133); +if (x_134 == 0) { -return x_163; +return x_133; } else { -lean_object* x_165; lean_object* x_166; -x_165 = lean_ctor_get(x_163, 0); -lean_inc(x_165); -lean_dec(x_163); -x_166 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_166, 0, x_165); -return x_166; +lean_object* x_135; lean_object* x_136; +x_135 = lean_ctor_get(x_133, 0); +lean_inc(x_135); +lean_dec(x_133); +x_136 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_136, 0, x_135); +return x_136; } } else { -uint8_t x_167; -x_167 = !lean_is_exclusive(x_163); -if (x_167 == 0) +uint8_t x_137; +x_137 = !lean_is_exclusive(x_133); +if (x_137 == 0) { -lean_object* x_168; -x_168 = lean_ctor_get(x_163, 0); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_168); -lean_ctor_set(x_163, 0, x_137); -return x_163; +lean_object* x_138; +x_138 = lean_ctor_get(x_133, 0); +lean_ctor_set_tag(x_107, 0); +lean_ctor_set(x_107, 0, x_138); +lean_ctor_set(x_133, 0, x_107); +return x_133; } else { -lean_object* x_169; lean_object* x_170; -x_169 = lean_ctor_get(x_163, 0); -lean_inc(x_169); -lean_dec(x_163); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_169); -x_170 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_170, 0, x_137); -return x_170; +lean_object* x_139; lean_object* x_140; +x_139 = lean_ctor_get(x_133, 0); +lean_inc(x_139); +lean_dec(x_133); +lean_ctor_set_tag(x_107, 0); +lean_ctor_set(x_107, 0, x_139); +x_140 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_140, 0, x_107); +return x_140; } } } } else { -lean_object* x_171; lean_object* x_172; lean_object* x_173; uint8_t x_174; -x_171 = lean_ctor_get(x_141, 0); -x_172 = lean_ctor_get(x_141, 1); -lean_inc(x_172); -lean_inc(x_171); -lean_dec(x_141); -x_173 = l_Lake_DependencySrc_decodeToml___closed__13; -x_174 = lean_string_dec_eq(x_172, x_173); -if (x_174 == 0) +lean_object* x_141; lean_object* x_142; lean_object* x_143; uint8_t x_144; +x_141 = lean_ctor_get(x_111, 0); +x_142 = lean_ctor_get(x_111, 1); +lean_inc(x_142); +lean_inc(x_141); +lean_dec(x_111); +x_143 = l_Lake_DependencySrc_decodeToml___closed__14; +x_144 = lean_string_dec_eq(x_142, x_143); +if (x_144 == 0) { -lean_object* x_175; uint8_t x_176; -x_175 = l_Lake_DependencySrc_decodeToml___closed__14; -x_176 = lean_string_dec_eq(x_172, x_175); -lean_dec(x_172); -if (x_176 == 0) +lean_object* x_145; uint8_t x_146; +x_145 = l_Lake_DependencySrc_decodeToml___closed__15; +x_146 = lean_string_dec_eq(x_142, x_145); +lean_dec(x_142); +if (x_146 == 0) { -lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; +lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_2); lean_dec(x_1); -x_177 = lean_box(0); -x_178 = l_Lake_DependencySrc_decodeToml___closed__15; -x_179 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_179, 0, x_171); -lean_ctor_set(x_179, 1, x_178); -x_180 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_180, 0, x_179); -lean_ctor_set(x_180, 1, x_177); -x_181 = lean_array_mk(x_180); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_181); -return x_137; +x_147 = lean_box(0); +x_148 = l_Lake_DependencySrc_decodeToml___closed__16; +x_149 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_141); +lean_ctor_set(x_149, 1, x_148); +x_150 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_147); +x_151 = lean_array_mk(x_150); +lean_ctor_set_tag(x_107, 0); +lean_ctor_set(x_107, 0, x_151); +return x_107; } else { -lean_object* x_182; lean_object* x_183; -lean_dec(x_171); -lean_free_object(x_137); -x_182 = l_Lake_DependencySrc_decodeToml___closed__17; +lean_object* x_152; lean_object* x_153; +lean_dec(x_141); +lean_free_object(x_107); +x_152 = l_Lake_DependencySrc_decodeToml___closed__18; lean_inc(x_1); -x_183 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_182, x_2); -if (lean_obj_tag(x_183) == 0) +x_153 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_152, x_2); +if (lean_obj_tag(x_153) == 0) { -lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_184 = lean_ctor_get(x_183, 0); -lean_inc(x_184); -lean_dec(x_183); -x_185 = l_Lake_LeanOption_decodeToml___closed__3; -x_186 = l_Array_append___rarg(x_185, x_184); -lean_dec(x_184); -x_187 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_187; -x_10 = x_186; -goto block_134; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +x_155 = l_Lake_LeanOption_decodeToml___closed__3; +x_156 = l_Array_append___rarg(x_155, x_154); +lean_dec(x_154); +x_157 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_157; +x_10 = x_156; +goto block_98; } else { -lean_object* x_188; lean_object* x_189; -x_188 = lean_ctor_get(x_183, 0); -lean_inc(x_188); -lean_dec(x_183); -x_189 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_188; -x_10 = x_189; -goto block_134; +lean_object* x_158; lean_object* x_159; +x_158 = lean_ctor_get(x_153, 0); +lean_inc(x_158); +lean_dec(x_153); +x_159 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_158; +x_10 = x_159; +goto block_98; } } } else { -lean_object* x_190; lean_object* x_191; lean_object* x_192; -lean_dec(x_172); -lean_dec(x_171); +lean_object* x_160; lean_object* x_161; lean_object* x_162; +lean_dec(x_142); +lean_dec(x_141); lean_dec(x_2); -x_190 = l_Lake_DependencySrc_decodeToml___closed__19; -x_191 = lean_box(0); -x_192 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_190, x_191); -if (lean_obj_tag(x_192) == 0) -{ -lean_object* x_193; lean_object* x_194; lean_object* x_195; -lean_free_object(x_137); -x_193 = lean_ctor_get(x_192, 0); -lean_inc(x_193); -if (lean_is_exclusive(x_192)) { - lean_ctor_release(x_192, 0); - x_194 = x_192; +x_160 = l_Lake_DependencySrc_decodeToml___closed__20; +x_161 = lean_box(0); +x_162 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_160, x_161); +if (lean_obj_tag(x_162) == 0) +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; +lean_free_object(x_107); +x_163 = lean_ctor_get(x_162, 0); +lean_inc(x_163); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + x_164 = x_162; } else { - lean_dec_ref(x_192); - x_194 = lean_box(0); + lean_dec_ref(x_162); + x_164 = lean_box(0); } -if (lean_is_scalar(x_194)) { - x_195 = lean_alloc_ctor(0, 1, 0); +if (lean_is_scalar(x_164)) { + x_165 = lean_alloc_ctor(0, 1, 0); } else { - x_195 = x_194; + x_165 = x_164; } -lean_ctor_set(x_195, 0, x_193); -return x_195; +lean_ctor_set(x_165, 0, x_163); +return x_165; } else { -lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_196 = lean_ctor_get(x_192, 0); -lean_inc(x_196); -if (lean_is_exclusive(x_192)) { - lean_ctor_release(x_192, 0); - x_197 = x_192; +lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_166 = lean_ctor_get(x_162, 0); +lean_inc(x_166); +if (lean_is_exclusive(x_162)) { + lean_ctor_release(x_162, 0); + x_167 = x_162; } else { - lean_dec_ref(x_192); - x_197 = lean_box(0); + lean_dec_ref(x_162); + x_167 = lean_box(0); } -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_196); -if (lean_is_scalar(x_197)) { - x_198 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set_tag(x_107, 0); +lean_ctor_set(x_107, 0, x_166); +if (lean_is_scalar(x_167)) { + x_168 = lean_alloc_ctor(1, 1, 0); } else { - x_198 = x_197; + x_168 = x_167; } -lean_ctor_set(x_198, 0, x_137); -return x_198; +lean_ctor_set(x_168, 0, x_107); +return x_168; } } } } case 2: { -lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_107); lean_dec(x_2); lean_dec(x_1); -x_199 = lean_ctor_get(x_141, 0); -lean_inc(x_199); -lean_dec(x_141); -x_200 = l_Lake_Glob_decodeToml___closed__2; -x_201 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_201, 0, x_199); -lean_ctor_set(x_201, 1, x_200); -x_202 = lean_unsigned_to_nat(1u); -x_203 = lean_mk_array(x_202, x_201); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_203); -return x_137; +x_169 = lean_ctor_get(x_111, 0); +lean_inc(x_169); +lean_dec(x_111); +x_170 = l_Lake_Glob_decodeToml___closed__2; +x_171 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +x_99 = x_171; +goto block_104; } case 3: { -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; +lean_object* x_172; lean_object* x_173; lean_object* x_174; +lean_free_object(x_107); lean_dec(x_2); lean_dec(x_1); -x_204 = lean_ctor_get(x_141, 0); -lean_inc(x_204); -lean_dec(x_141); -x_205 = l_Lake_Glob_decodeToml___closed__2; -x_206 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_206, 0, x_204); -lean_ctor_set(x_206, 1, x_205); -x_207 = lean_unsigned_to_nat(1u); -x_208 = lean_mk_array(x_207, x_206); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_208); -return x_137; +x_172 = lean_ctor_get(x_111, 0); +lean_inc(x_172); +lean_dec(x_111); +x_173 = l_Lake_Glob_decodeToml___closed__2; +x_174 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_174, 0, x_172); +lean_ctor_set(x_174, 1, x_173); +x_99 = x_174; +goto block_104; } default: { -uint8_t x_209; +uint8_t x_175; +lean_free_object(x_107); lean_dec(x_2); lean_dec(x_1); -x_209 = !lean_is_exclusive(x_141); -if (x_209 == 0) +x_175 = !lean_is_exclusive(x_111); +if (x_175 == 0) { -lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; -x_210 = lean_ctor_get(x_141, 1); -lean_dec(x_210); -x_211 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_141, 0); -lean_ctor_set(x_141, 1, x_211); -x_212 = lean_unsigned_to_nat(1u); -x_213 = lean_mk_array(x_212, x_141); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_213); -return x_137; +lean_object* x_176; lean_object* x_177; +x_176 = lean_ctor_get(x_111, 1); +lean_dec(x_176); +x_177 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_111, 0); +lean_ctor_set(x_111, 1, x_177); +x_99 = x_111; +goto block_104; } else { -lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; -x_214 = lean_ctor_get(x_141, 0); -lean_inc(x_214); -lean_dec(x_141); -x_215 = l_Lake_Glob_decodeToml___closed__2; -x_216 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_216, 0, x_214); -lean_ctor_set(x_216, 1, x_215); -x_217 = lean_unsigned_to_nat(1u); -x_218 = lean_mk_array(x_217, x_216); -lean_ctor_set_tag(x_137, 0); -lean_ctor_set(x_137, 0, x_218); -return x_137; +lean_object* x_178; lean_object* x_179; lean_object* x_180; +x_178 = lean_ctor_get(x_111, 0); +lean_inc(x_178); +lean_dec(x_111); +x_179 = l_Lake_Glob_decodeToml___closed__2; +x_180 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_179); +x_99 = x_180; +goto block_104; } } } } else { -lean_object* x_219; lean_object* x_220; -x_219 = lean_ctor_get(x_137, 0); -lean_inc(x_219); -lean_dec(x_137); -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -lean_dec(x_219); -switch (lean_obj_tag(x_220)) { +lean_object* x_181; lean_object* x_182; +x_181 = lean_ctor_get(x_107, 0); +lean_inc(x_181); +lean_dec(x_107); +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +lean_dec(x_181); +switch (lean_obj_tag(x_182)) { case 0: { -lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; uint8_t x_225; -x_221 = lean_ctor_get(x_220, 0); -lean_inc(x_221); -x_222 = lean_ctor_get(x_220, 1); -lean_inc(x_222); -if (lean_is_exclusive(x_220)) { - lean_ctor_release(x_220, 0); - lean_ctor_release(x_220, 1); - x_223 = x_220; +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; +x_183 = lean_ctor_get(x_182, 0); +lean_inc(x_183); +x_184 = lean_ctor_get(x_182, 1); +lean_inc(x_184); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_185 = x_182; } else { - lean_dec_ref(x_220); - x_223 = lean_box(0); + lean_dec_ref(x_182); + x_185 = lean_box(0); } -x_224 = l_Lake_DependencySrc_decodeToml___closed__13; -x_225 = lean_string_dec_eq(x_222, x_224); -if (x_225 == 0) +x_186 = l_Lake_DependencySrc_decodeToml___closed__14; +x_187 = lean_string_dec_eq(x_184, x_186); +if (x_187 == 0) { -lean_object* x_226; uint8_t x_227; -x_226 = l_Lake_DependencySrc_decodeToml___closed__14; -x_227 = lean_string_dec_eq(x_222, x_226); -lean_dec(x_222); -if (x_227 == 0) +lean_object* x_188; uint8_t x_189; +x_188 = l_Lake_DependencySrc_decodeToml___closed__15; +x_189 = lean_string_dec_eq(x_184, x_188); +lean_dec(x_184); +if (x_189 == 0) { -lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_dec(x_2); lean_dec(x_1); -x_228 = lean_box(0); -x_229 = l_Lake_DependencySrc_decodeToml___closed__15; -if (lean_is_scalar(x_223)) { - x_230 = lean_alloc_ctor(0, 2, 0); +x_190 = lean_box(0); +x_191 = l_Lake_DependencySrc_decodeToml___closed__16; +if (lean_is_scalar(x_185)) { + x_192 = lean_alloc_ctor(0, 2, 0); } else { - x_230 = x_223; -} -lean_ctor_set(x_230, 0, x_221); -lean_ctor_set(x_230, 1, x_229); -x_231 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_231, 0, x_230); -lean_ctor_set(x_231, 1, x_228); -x_232 = lean_array_mk(x_231); -x_233 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_233, 0, x_232); -return x_233; + x_192 = x_185; +} +lean_ctor_set(x_192, 0, x_183); +lean_ctor_set(x_192, 1, x_191); +x_193 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_193, 0, x_192); +lean_ctor_set(x_193, 1, x_190); +x_194 = lean_array_mk(x_193); +x_195 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_195, 0, x_194); +return x_195; } else { -lean_object* x_234; lean_object* x_235; -lean_dec(x_223); -lean_dec(x_221); -x_234 = l_Lake_DependencySrc_decodeToml___closed__17; +lean_object* x_196; lean_object* x_197; +lean_dec(x_185); +lean_dec(x_183); +x_196 = l_Lake_DependencySrc_decodeToml___closed__18; lean_inc(x_1); -x_235 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_234, x_2); -if (lean_obj_tag(x_235) == 0) +x_197 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_196, x_2); +if (lean_obj_tag(x_197) == 0) { -lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_236 = lean_ctor_get(x_235, 0); -lean_inc(x_236); -lean_dec(x_235); -x_237 = l_Lake_LeanOption_decodeToml___closed__3; -x_238 = l_Array_append___rarg(x_237, x_236); -lean_dec(x_236); -x_239 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_239; -x_10 = x_238; -goto block_134; +lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_198 = lean_ctor_get(x_197, 0); +lean_inc(x_198); +lean_dec(x_197); +x_199 = l_Lake_LeanOption_decodeToml___closed__3; +x_200 = l_Array_append___rarg(x_199, x_198); +lean_dec(x_198); +x_201 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_201; +x_10 = x_200; +goto block_98; } else { -lean_object* x_240; lean_object* x_241; -x_240 = lean_ctor_get(x_235, 0); -lean_inc(x_240); -lean_dec(x_235); -x_241 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_240; -x_10 = x_241; -goto block_134; +lean_object* x_202; lean_object* x_203; +x_202 = lean_ctor_get(x_197, 0); +lean_inc(x_202); +lean_dec(x_197); +x_203 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_202; +x_10 = x_203; +goto block_98; } } } else { -lean_object* x_242; lean_object* x_243; lean_object* x_244; -lean_dec(x_223); -lean_dec(x_222); -lean_dec(x_221); +lean_object* x_204; lean_object* x_205; lean_object* x_206; +lean_dec(x_185); +lean_dec(x_184); +lean_dec(x_183); lean_dec(x_2); -x_242 = l_Lake_DependencySrc_decodeToml___closed__19; -x_243 = lean_box(0); -x_244 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_242, x_243); -if (lean_obj_tag(x_244) == 0) -{ -lean_object* x_245; lean_object* x_246; lean_object* x_247; -x_245 = lean_ctor_get(x_244, 0); -lean_inc(x_245); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - x_246 = x_244; +x_204 = l_Lake_DependencySrc_decodeToml___closed__20; +x_205 = lean_box(0); +x_206 = l_Lake_Toml_Table_decode___at_Lake_DependencySrc_decodeToml___spec__1(x_1, x_204, x_205); +if (lean_obj_tag(x_206) == 0) +{ +lean_object* x_207; lean_object* x_208; lean_object* x_209; +x_207 = lean_ctor_get(x_206, 0); +lean_inc(x_207); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + x_208 = x_206; } else { - lean_dec_ref(x_244); - x_246 = lean_box(0); + lean_dec_ref(x_206); + x_208 = lean_box(0); } -if (lean_is_scalar(x_246)) { - x_247 = lean_alloc_ctor(0, 1, 0); +if (lean_is_scalar(x_208)) { + x_209 = lean_alloc_ctor(0, 1, 0); } else { - x_247 = x_246; + x_209 = x_208; } -lean_ctor_set(x_247, 0, x_245); -return x_247; +lean_ctor_set(x_209, 0, x_207); +return x_209; } else { -lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; -x_248 = lean_ctor_get(x_244, 0); -lean_inc(x_248); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - x_249 = x_244; +lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_210 = lean_ctor_get(x_206, 0); +lean_inc(x_210); +if (lean_is_exclusive(x_206)) { + lean_ctor_release(x_206, 0); + x_211 = x_206; } else { - lean_dec_ref(x_244); - x_249 = lean_box(0); + lean_dec_ref(x_206); + x_211 = lean_box(0); } -x_250 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_250, 0, x_248); -if (lean_is_scalar(x_249)) { - x_251 = lean_alloc_ctor(1, 1, 0); +x_212 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_212, 0, x_210); +if (lean_is_scalar(x_211)) { + x_213 = lean_alloc_ctor(1, 1, 0); } else { - x_251 = x_249; + x_213 = x_211; } -lean_ctor_set(x_251, 0, x_250); -return x_251; +lean_ctor_set(x_213, 0, x_212); +return x_213; } } } case 2: { -lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; +lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_dec(x_2); lean_dec(x_1); -x_252 = lean_ctor_get(x_220, 0); -lean_inc(x_252); -lean_dec(x_220); -x_253 = l_Lake_Glob_decodeToml___closed__2; -x_254 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_254, 0, x_252); -lean_ctor_set(x_254, 1, x_253); -x_255 = lean_unsigned_to_nat(1u); -x_256 = lean_mk_array(x_255, x_254); -x_257 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_257, 0, x_256); -return x_257; +x_214 = lean_ctor_get(x_182, 0); +lean_inc(x_214); +lean_dec(x_182); +x_215 = l_Lake_Glob_decodeToml___closed__2; +x_216 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_216, 0, x_214); +lean_ctor_set(x_216, 1, x_215); +x_99 = x_216; +goto block_104; } case 3: { -lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_dec(x_2); lean_dec(x_1); -x_258 = lean_ctor_get(x_220, 0); -lean_inc(x_258); -lean_dec(x_220); -x_259 = l_Lake_Glob_decodeToml___closed__2; -x_260 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_260, 0, x_258); -lean_ctor_set(x_260, 1, x_259); -x_261 = lean_unsigned_to_nat(1u); -x_262 = lean_mk_array(x_261, x_260); -x_263 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_263, 0, x_262); -return x_263; +x_217 = lean_ctor_get(x_182, 0); +lean_inc(x_217); +lean_dec(x_182); +x_218 = l_Lake_Glob_decodeToml___closed__2; +x_219 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +x_99 = x_219; +goto block_104; } default: { -lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_dec(x_2); lean_dec(x_1); -x_264 = lean_ctor_get(x_220, 0); -lean_inc(x_264); -if (lean_is_exclusive(x_220)) { - lean_ctor_release(x_220, 0); - lean_ctor_release(x_220, 1); - x_265 = x_220; +x_220 = lean_ctor_get(x_182, 0); +lean_inc(x_220); +if (lean_is_exclusive(x_182)) { + lean_ctor_release(x_182, 0); + lean_ctor_release(x_182, 1); + x_221 = x_182; } else { - lean_dec_ref(x_220); - x_265 = lean_box(0); + lean_dec_ref(x_182); + x_221 = lean_box(0); } -x_266 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_265)) { - x_267 = lean_alloc_ctor(0, 2, 0); +x_222 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_221)) { + x_223 = lean_alloc_ctor(0, 2, 0); } else { - x_267 = x_265; - lean_ctor_set_tag(x_267, 0); + x_223 = x_221; + lean_ctor_set_tag(x_223, 0); } -lean_ctor_set(x_267, 0, x_264); -lean_ctor_set(x_267, 1, x_266); -x_268 = lean_unsigned_to_nat(1u); -x_269 = lean_mk_array(x_268, x_267); -x_270 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_270, 0, x_269); -return x_270; +lean_ctor_set(x_223, 0, x_220); +lean_ctor_set(x_223, 1, x_222); +x_99 = x_223; +goto block_104; } } } @@ -16617,463 +16657,409 @@ lean_ctor_set(x_7, 0, x_3); return x_7; } } -block_134: +block_98: { -lean_object* x_11; lean_object* x_12; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_79 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_80 = l_Lake_DependencySrc_decodeToml___closed__4; +lean_object* x_11; lean_object* x_12; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_58 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_59 = l_Lake_DependencySrc_decodeToml___closed__4; lean_inc(x_1); -x_81 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_79, x_80, x_1); -x_82 = lean_box(0); -if (lean_obj_tag(x_81) == 0) +x_60 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_58, x_59, x_1); +x_61 = lean_box(0); +if (lean_obj_tag(x_60) == 0) { -x_11 = x_82; +x_11 = x_61; x_12 = x_10; -goto block_78; +goto block_57; } else { -uint8_t x_83; -x_83 = !lean_is_exclusive(x_81); -if (x_83 == 0) +uint8_t x_68; +x_68 = !lean_is_exclusive(x_60); +if (x_68 == 0) { -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_81, 0); -x_85 = lean_ctor_get(x_84, 1); -lean_inc(x_85); -lean_dec(x_84); -switch (lean_obj_tag(x_85)) { +lean_object* x_69; lean_object* x_70; +x_69 = lean_ctor_get(x_60, 0); +x_70 = lean_ctor_get(x_69, 1); +lean_inc(x_70); +lean_dec(x_69); +switch (lean_obj_tag(x_70)) { case 0: { -lean_object* x_86; -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -lean_dec(x_85); -lean_ctor_set(x_81, 0, x_86); -x_11 = x_81; +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +lean_ctor_set(x_60, 0, x_71); +x_11 = x_60; x_12 = x_10; -goto block_78; +goto block_57; } case 2: { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -lean_free_object(x_81); -x_87 = lean_ctor_get(x_85, 0); -lean_inc(x_87); -lean_dec(x_85); -x_88 = l_Lake_Glob_decodeToml___closed__2; -x_89 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -x_90 = lean_unsigned_to_nat(1u); -x_91 = lean_mk_array(x_90, x_89); -x_92 = l_Array_append___rarg(x_10, x_91); -lean_dec(x_91); -x_11 = x_82; -x_12 = x_92; -goto block_78; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_60); +x_72 = lean_ctor_get(x_70, 0); +lean_inc(x_72); +lean_dec(x_70); +x_73 = l_Lake_Glob_decodeToml___closed__2; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +x_62 = x_74; +goto block_67; } case 3: { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -lean_free_object(x_81); -x_93 = lean_ctor_get(x_85, 0); -lean_inc(x_93); -lean_dec(x_85); -x_94 = l_Lake_Glob_decodeToml___closed__2; -x_95 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -x_96 = lean_unsigned_to_nat(1u); -x_97 = lean_mk_array(x_96, x_95); -x_98 = l_Array_append___rarg(x_10, x_97); -lean_dec(x_97); -x_11 = x_82; -x_12 = x_98; -goto block_78; +lean_object* x_75; lean_object* x_76; lean_object* x_77; +lean_free_object(x_60); +x_75 = lean_ctor_get(x_70, 0); +lean_inc(x_75); +lean_dec(x_70); +x_76 = l_Lake_Glob_decodeToml___closed__2; +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +x_62 = x_77; +goto block_67; } default: { -uint8_t x_99; -lean_free_object(x_81); -x_99 = !lean_is_exclusive(x_85); -if (x_99 == 0) +uint8_t x_78; +lean_free_object(x_60); +x_78 = !lean_is_exclusive(x_70); +if (x_78 == 0) { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_100 = lean_ctor_get(x_85, 1); -lean_dec(x_100); -x_101 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_85, 0); -lean_ctor_set(x_85, 1, x_101); -x_102 = lean_unsigned_to_nat(1u); -x_103 = lean_mk_array(x_102, x_85); -x_104 = l_Array_append___rarg(x_10, x_103); -lean_dec(x_103); -x_11 = x_82; -x_12 = x_104; -goto block_78; +lean_object* x_79; lean_object* x_80; +x_79 = lean_ctor_get(x_70, 1); +lean_dec(x_79); +x_80 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_70, 0); +lean_ctor_set(x_70, 1, x_80); +x_62 = x_70; +goto block_67; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_105 = lean_ctor_get(x_85, 0); -lean_inc(x_105); -lean_dec(x_85); -x_106 = l_Lake_Glob_decodeToml___closed__2; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -x_108 = lean_unsigned_to_nat(1u); -x_109 = lean_mk_array(x_108, x_107); -x_110 = l_Array_append___rarg(x_10, x_109); -lean_dec(x_109); -x_11 = x_82; -x_12 = x_110; -goto block_78; +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_70, 0); +lean_inc(x_81); +lean_dec(x_70); +x_82 = l_Lake_Glob_decodeToml___closed__2; +x_83 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_83, 0, x_81); +lean_ctor_set(x_83, 1, x_82); +x_62 = x_83; +goto block_67; } } } } else { -lean_object* x_111; lean_object* x_112; -x_111 = lean_ctor_get(x_81, 0); -lean_inc(x_111); -lean_dec(x_81); -x_112 = lean_ctor_get(x_111, 1); -lean_inc(x_112); -lean_dec(x_111); -switch (lean_obj_tag(x_112)) { +lean_object* x_84; lean_object* x_85; +x_84 = lean_ctor_get(x_60, 0); +lean_inc(x_84); +lean_dec(x_60); +x_85 = lean_ctor_get(x_84, 1); +lean_inc(x_85); +lean_dec(x_84); +switch (lean_obj_tag(x_85)) { case 0: { -lean_object* x_113; lean_object* x_114; -x_113 = lean_ctor_get(x_112, 1); -lean_inc(x_113); -lean_dec(x_112); -x_114 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_114, 0, x_113); -x_11 = x_114; +lean_object* x_86; lean_object* x_87; +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_87, 0, x_86); +x_11 = x_87; x_12 = x_10; -goto block_78; +goto block_57; } case 2: { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_115 = lean_ctor_get(x_112, 0); -lean_inc(x_115); -lean_dec(x_112); -x_116 = l_Lake_Glob_decodeToml___closed__2; -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_115); -lean_ctor_set(x_117, 1, x_116); -x_118 = lean_unsigned_to_nat(1u); -x_119 = lean_mk_array(x_118, x_117); -x_120 = l_Array_append___rarg(x_10, x_119); -lean_dec(x_119); -x_11 = x_82; -x_12 = x_120; -goto block_78; +lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_88 = lean_ctor_get(x_85, 0); +lean_inc(x_88); +lean_dec(x_85); +x_89 = l_Lake_Glob_decodeToml___closed__2; +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_62 = x_90; +goto block_67; } case 3: { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_121 = lean_ctor_get(x_112, 0); -lean_inc(x_121); -lean_dec(x_112); -x_122 = l_Lake_Glob_decodeToml___closed__2; -x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); -x_124 = lean_unsigned_to_nat(1u); -x_125 = lean_mk_array(x_124, x_123); -x_126 = l_Array_append___rarg(x_10, x_125); -lean_dec(x_125); -x_11 = x_82; -x_12 = x_126; -goto block_78; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_85, 0); +lean_inc(x_91); +lean_dec(x_85); +x_92 = l_Lake_Glob_decodeToml___closed__2; +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_62 = x_93; +goto block_67; } default: { -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_127 = lean_ctor_get(x_112, 0); -lean_inc(x_127); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_128 = x_112; +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_94 = lean_ctor_get(x_85, 0); +lean_inc(x_94); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_95 = x_85; } else { - lean_dec_ref(x_112); - x_128 = lean_box(0); + lean_dec_ref(x_85); + x_95 = lean_box(0); } -x_129 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_128)) { - x_130 = lean_alloc_ctor(0, 2, 0); +x_96 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); } else { - x_130 = x_128; - lean_ctor_set_tag(x_130, 0); + x_97 = x_95; + lean_ctor_set_tag(x_97, 0); } -lean_ctor_set(x_130, 0, x_127); -lean_ctor_set(x_130, 1, x_129); -x_131 = lean_unsigned_to_nat(1u); -x_132 = lean_mk_array(x_131, x_130); -x_133 = l_Array_append___rarg(x_10, x_132); -lean_dec(x_132); -x_11 = x_82; -x_12 = x_133; -goto block_78; +lean_ctor_set(x_97, 0, x_94); +lean_ctor_set(x_97, 1, x_96); +x_62 = x_97; +goto block_67; } } } } -block_78: +block_57: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_13 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; x_14 = l_Lake_DependencySrc_decodeToml___closed__2; x_15 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_13, x_14, x_1); x_16 = lean_box(0); if (lean_obj_tag(x_15) == 0) { -lean_object* x_17; -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_9); -lean_ctor_set(x_17, 1, x_11); -lean_ctor_set(x_17, 2, x_16); -x_3 = x_17; +lean_object* x_24; +x_24 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_24, 0, x_9); +lean_ctor_set(x_24, 1, x_11); +lean_ctor_set(x_24, 2, x_16); +x_3 = x_24; x_4 = x_12; goto block_8; } else { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_15); -if (x_18 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_15); +if (x_25 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_15, 0); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -switch (lean_obj_tag(x_20)) { +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_15, 0); +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +switch (lean_obj_tag(x_27)) { case 0: { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -lean_ctor_set(x_15, 0, x_21); -x_22 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_22, 0, x_9); -lean_ctor_set(x_22, 1, x_11); -lean_ctor_set(x_22, 2, x_15); -x_3 = x_22; -x_4 = x_12; -goto block_8; -} -case 2: -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -lean_free_object(x_15); -x_23 = lean_ctor_get(x_20, 0); -lean_inc(x_23); -lean_dec(x_20); -x_24 = l_Lake_Glob_decodeToml___closed__2; -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_25); -x_28 = l_Array_append___rarg(x_12, x_27); +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); lean_dec(x_27); +lean_ctor_set(x_15, 0, x_28); x_29 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_29, 0, x_9); lean_ctor_set(x_29, 1, x_11); -lean_ctor_set(x_29, 2, x_16); +lean_ctor_set(x_29, 2, x_15); x_3 = x_29; -x_4 = x_28; +x_4 = x_12; goto block_8; } -case 3: +case 2: { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_free_object(x_15); -x_30 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_27, 0); lean_inc(x_30); -lean_dec(x_20); +lean_dec(x_27); x_31 = l_Lake_Glob_decodeToml___closed__2; x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_30); lean_ctor_set(x_32, 1, x_31); -x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_mk_array(x_33, x_32); -x_35 = l_Array_append___rarg(x_12, x_34); -lean_dec(x_34); -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_9); -lean_ctor_set(x_36, 1, x_11); -lean_ctor_set(x_36, 2, x_16); -x_3 = x_36; -x_4 = x_35; -goto block_8; +x_17 = x_32; +goto block_23; +} +case 3: +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +lean_free_object(x_15); +x_33 = lean_ctor_get(x_27, 0); +lean_inc(x_33); +lean_dec(x_27); +x_34 = l_Lake_Glob_decodeToml___closed__2; +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_17 = x_35; +goto block_23; } default: { -uint8_t x_37; +uint8_t x_36; lean_free_object(x_15); -x_37 = !lean_is_exclusive(x_20); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_27); +if (x_36 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_38 = lean_ctor_get(x_20, 1); -lean_dec(x_38); -x_39 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_20, 0); -lean_ctor_set(x_20, 1, x_39); -x_40 = lean_unsigned_to_nat(1u); -x_41 = lean_mk_array(x_40, x_20); -x_42 = l_Array_append___rarg(x_12, x_41); -lean_dec(x_41); -x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_9); -lean_ctor_set(x_43, 1, x_11); -lean_ctor_set(x_43, 2, x_16); -x_3 = x_43; -x_4 = x_42; -goto block_8; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_27, 1); +lean_dec(x_37); +x_38 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_27, 0); +lean_ctor_set(x_27, 1, x_38); +x_17 = x_27; +goto block_23; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_44 = lean_ctor_get(x_20, 0); -lean_inc(x_44); -lean_dec(x_20); -x_45 = l_Lake_Glob_decodeToml___closed__2; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_unsigned_to_nat(1u); -x_48 = lean_mk_array(x_47, x_46); -x_49 = l_Array_append___rarg(x_12, x_48); -lean_dec(x_48); -x_50 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_50, 0, x_9); -lean_ctor_set(x_50, 1, x_11); -lean_ctor_set(x_50, 2, x_16); -x_3 = x_50; -x_4 = x_49; -goto block_8; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_27, 0); +lean_inc(x_39); +lean_dec(x_27); +x_40 = l_Lake_Glob_decodeToml___closed__2; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_17 = x_41; +goto block_23; } } } } else { -lean_object* x_51; lean_object* x_52; -x_51 = lean_ctor_get(x_15, 0); -lean_inc(x_51); +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_15, 0); +lean_inc(x_42); lean_dec(x_15); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -lean_dec(x_51); -switch (lean_obj_tag(x_52)) { +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +switch (lean_obj_tag(x_43)) { case 0: { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_53); -x_55 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_55, 0, x_9); -lean_ctor_set(x_55, 1, x_11); -lean_ctor_set(x_55, 2, x_54); -x_3 = x_55; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_46, 0, x_9); +lean_ctor_set(x_46, 1, x_11); +lean_ctor_set(x_46, 2, x_45); +x_3 = x_46; x_4 = x_12; goto block_8; } case 2: { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_52, 0); -lean_inc(x_56); -lean_dec(x_52); -x_57 = l_Lake_Glob_decodeToml___closed__2; -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_unsigned_to_nat(1u); -x_60 = lean_mk_array(x_59, x_58); -x_61 = l_Array_append___rarg(x_12, x_60); -lean_dec(x_60); -x_62 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_62, 0, x_9); -lean_ctor_set(x_62, 1, x_11); -lean_ctor_set(x_62, 2, x_16); -x_3 = x_62; -x_4 = x_61; -goto block_8; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_43, 0); +lean_inc(x_47); +lean_dec(x_43); +x_48 = l_Lake_Glob_decodeToml___closed__2; +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_17 = x_49; +goto block_23; } case 3: { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_63 = lean_ctor_get(x_52, 0); -lean_inc(x_63); -lean_dec(x_52); -x_64 = l_Lake_Glob_decodeToml___closed__2; -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -x_66 = lean_unsigned_to_nat(1u); -x_67 = lean_mk_array(x_66, x_65); -x_68 = l_Array_append___rarg(x_12, x_67); -lean_dec(x_67); -x_69 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_69, 0, x_9); -lean_ctor_set(x_69, 1, x_11); -lean_ctor_set(x_69, 2, x_16); -x_3 = x_69; -x_4 = x_68; -goto block_8; +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_43, 0); +lean_inc(x_50); +lean_dec(x_43); +x_51 = l_Lake_Glob_decodeToml___closed__2; +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +x_17 = x_52; +goto block_23; } default: { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_70 = lean_ctor_get(x_52, 0); -lean_inc(x_70); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_71 = x_52; +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_43, 0); +lean_inc(x_53); +if (lean_is_exclusive(x_43)) { + lean_ctor_release(x_43, 0); + lean_ctor_release(x_43, 1); + x_54 = x_43; } else { - lean_dec_ref(x_52); - x_71 = lean_box(0); + lean_dec_ref(x_43); + x_54 = lean_box(0); } -x_72 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_71)) { - x_73 = lean_alloc_ctor(0, 2, 0); +x_55 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(0, 2, 0); } else { - x_73 = x_71; - lean_ctor_set_tag(x_73, 0); -} -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_72); -x_74 = lean_unsigned_to_nat(1u); -x_75 = lean_mk_array(x_74, x_73); -x_76 = l_Array_append___rarg(x_12, x_75); -lean_dec(x_75); -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_9); -lean_ctor_set(x_77, 1, x_11); -lean_ctor_set(x_77, 2, x_16); -x_3 = x_77; -x_4 = x_76; -goto block_8; + x_56 = x_54; + lean_ctor_set_tag(x_56, 0); } +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_55); +x_17 = x_56; +goto block_23; } } } } +block_23: +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_18 = lean_box(0); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_array_mk(x_19); +x_21 = l_Array_append___rarg(x_12, x_20); +lean_dec(x_20); +x_22 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_22, 0, x_9); +lean_ctor_set(x_22, 1, x_11); +lean_ctor_set(x_22, 2, x_16); +x_3 = x_22; +x_4 = x_21; +goto block_8; +} +} +block_67: +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_63 = lean_box(0); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +x_65 = lean_array_mk(x_64); +x_66 = l_Array_append___rarg(x_10, x_65); +lean_dec(x_65); +x_11 = x_61; +x_12 = x_66; +goto block_57; +} +} +block_104: +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_100 = lean_box(0); +x_101 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_101, 0, x_99); +lean_ctor_set(x_101, 1, x_100); +x_102 = lean_array_mk(x_101); +x_103 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_103, 0, x_102); +return x_103; } } } @@ -17099,124 +17085,135 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependencySrc(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependencySrc___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); lean_dec(x_1); -x_28 = l_Lake_DependencySrc_decodeToml(x_27, x_26); -return x_28; +x_22 = l_Lake_DependencySrc_decodeToml(x_21, x_20); +return x_22; } default: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_1); -if (x_29 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_1); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_1, 1); -lean_dec(x_30); -x_31 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_1, 1); +lean_dec(x_24); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_1); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_1, 1, x_25); +x_2 = x_1; +goto block_7; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_36 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_2 = x_28; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } +static lean_object* _init_l_Lake_instDecodeTomlDependencySrc___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlDependencySrc___lambda__1), 1, 0); +return x_1; } } +static lean_object* _init_l_Lake_instDecodeTomlDependencySrc() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlDependencySrc___closed__1; +return x_1; +} } LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: @@ -17233,209 +17230,116 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; uint8_t x_9; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); -x_9 = !lean_is_exclusive(x_6); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_6, 0); -x_11 = lean_ctor_get(x_6, 1); +x_9 = lean_ctor_get(x_6, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_6, 1); +lean_inc(x_10); +if (lean_is_exclusive(x_6)) { + lean_ctor_release(x_6, 0); + lean_ctor_release(x_6, 1); + x_11 = x_6; +} else { + lean_dec_ref(x_6); + x_11 = lean_box(0); +} x_12 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2___lambda__1), 3, 1); -lean_closure_set(x_12, 0, x_10); -switch (lean_obj_tag(x_11)) { +lean_closure_set(x_12, 0, x_9); +switch (lean_obj_tag(x_10)) { case 0: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -lean_free_object(x_6); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_dec(x_11); -x_14 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Lake_mergeErrors___rarg(x_4, x_14, x_12); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_dec(x_10); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lake_mergeErrors___rarg(x_4, x_22, x_12); x_2 = x_8; -x_4 = x_15; +x_4 = x_23; goto _start; } case 2: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_11, 0); -lean_inc(x_17); -lean_dec(x_11); -x_18 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_6, 1, x_18); -lean_ctor_set(x_6, 0, x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_6); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -x_22 = l_Lake_mergeErrors___rarg(x_4, x_21, x_12); -x_2 = x_8; -x_4 = x_22; -goto _start; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_10, 0); +lean_inc(x_25); +lean_dec(x_10); +x_26 = l_Lake_Glob_decodeToml___closed__2; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_13 = x_27; +goto block_20; } case 3: { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_11, 0); -lean_inc(x_24); -lean_dec(x_11); -x_25 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_6, 1, x_25); -lean_ctor_set(x_6, 0, x_24); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_6); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -x_29 = l_Lake_mergeErrors___rarg(x_4, x_28, x_12); -x_2 = x_8; -x_4 = x_29; -goto _start; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_10, 0); +lean_inc(x_28); +lean_dec(x_10); +x_29 = l_Lake_Glob_decodeToml___closed__2; +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_13 = x_30; +goto block_20; } default: { uint8_t x_31; -lean_free_object(x_6); -x_31 = !lean_is_exclusive(x_11); +x_31 = !lean_is_exclusive(x_10); if (x_31 == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_32 = lean_ctor_get(x_11, 1); +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_10, 1); lean_dec(x_32); x_33 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_11, 0); -lean_ctor_set(x_11, 1, x_33); -x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_mk_array(x_34, x_11); -x_36 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_36, 0, x_35); -x_37 = l_Lake_mergeErrors___rarg(x_4, x_36, x_12); -x_2 = x_8; -x_4 = x_37; -goto _start; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_39 = lean_ctor_get(x_11, 0); -lean_inc(x_39); -lean_dec(x_11); -x_40 = l_Lake_Glob_decodeToml___closed__2; -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_unsigned_to_nat(1u); -x_43 = lean_mk_array(x_42, x_41); -x_44 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = l_Lake_mergeErrors___rarg(x_4, x_44, x_12); -x_2 = x_8; -x_4 = x_45; -goto _start; -} -} -} +lean_ctor_set_tag(x_10, 0); +lean_ctor_set(x_10, 1, x_33); +x_13 = x_10; +goto block_20; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_6, 0); -x_48 = lean_ctor_get(x_6, 1); -lean_inc(x_48); -lean_inc(x_47); -lean_dec(x_6); -x_49 = lean_alloc_closure((void*)(l_Array_foldlMUnsafe_fold___at_Lake_Dependency_decodeToml___spec__2___lambda__1), 3, 1); -lean_closure_set(x_49, 0, x_47); -switch (lean_obj_tag(x_48)) { -case 0: -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -x_51 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_51, 0, x_50); -x_52 = l_Lake_mergeErrors___rarg(x_4, x_51, x_49); -x_2 = x_8; -x_4 = x_52; -goto _start; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_10, 0); +lean_inc(x_34); +lean_dec(x_10); +x_35 = l_Lake_Glob_decodeToml___closed__2; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_13 = x_36; +goto block_20; } -case 2: -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_54 = lean_ctor_get(x_48, 0); -lean_inc(x_54); -lean_dec(x_48); -x_55 = l_Lake_Glob_decodeToml___closed__2; -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -x_57 = lean_unsigned_to_nat(1u); -x_58 = lean_mk_array(x_57, x_56); -x_59 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_59, 0, x_58); -x_60 = l_Lake_mergeErrors___rarg(x_4, x_59, x_49); -x_2 = x_8; -x_4 = x_60; -goto _start; } -case 3: -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_62 = lean_ctor_get(x_48, 0); -lean_inc(x_62); -lean_dec(x_48); -x_63 = l_Lake_Glob_decodeToml___closed__2; -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_mk_array(x_65, x_64); -x_67 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = l_Lake_mergeErrors___rarg(x_4, x_67, x_49); -x_2 = x_8; -x_4 = x_68; -goto _start; } -default: +block_20: { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_70 = lean_ctor_get(x_48, 0); -lean_inc(x_70); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_71 = x_48; -} else { - lean_dec_ref(x_48); - x_71 = lean_box(0); -} -x_72 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_71)) { - x_73 = lean_alloc_ctor(0, 2, 0); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_14 = lean_box(0); +if (lean_is_scalar(x_11)) { + x_15 = lean_alloc_ctor(1, 2, 0); } else { - x_73 = x_71; - lean_ctor_set_tag(x_73, 0); + x_15 = x_11; + lean_ctor_set_tag(x_15, 1); } -lean_ctor_set(x_73, 0, x_70); -lean_ctor_set(x_73, 1, x_72); -x_74 = lean_unsigned_to_nat(1u); -x_75 = lean_mk_array(x_74, x_73); -x_76 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_76, 0, x_75); -x_77 = l_Lake_mergeErrors___rarg(x_4, x_76, x_49); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_array_mk(x_15); +x_17 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_17, 0, x_16); +x_18 = l_Lake_mergeErrors___rarg(x_4, x_17, x_12); x_2 = x_8; -x_4 = x_77; +x_4 = x_18; goto _start; } } -} -} else { return x_4; @@ -17491,3489 +17395,7320 @@ return x_12; } } } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__1() { -_start: +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("options", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_Dependency_decodeToml___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("git#", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("scope", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_Dependency_decodeToml___closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_DependencySrc_decodeToml___closed__15; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("source", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_Dependency_decodeToml___closed__7; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("expected string or table", 24, 24); +return x_1; +} +} +static lean_object* _init_l_Lake_Dependency_decodeToml___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lake_DependencySrc_decodeToml___closed__14; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lake_Dependency_decodeToml(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_1642; lean_object* x_1643; +x_1642 = l_Lake_LeanOption_decodeToml___closed__10; +lean_inc(x_1); +x_1643 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_1642, x_2); +if (lean_obj_tag(x_1643) == 0) +{ +lean_object* x_1644; lean_object* x_1645; lean_object* x_1646; lean_object* x_1647; +x_1644 = lean_ctor_get(x_1643, 0); +lean_inc(x_1644); +lean_dec(x_1643); +x_1645 = l_Lake_LeanOption_decodeToml___closed__3; +x_1646 = l_Array_append___rarg(x_1645, x_1644); +lean_dec(x_1644); +x_1647 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_9 = x_1647; +x_10 = x_1646; +goto block_1641; +} +else +{ +lean_object* x_1648; lean_object* x_1649; +x_1648 = lean_ctor_get(x_1643, 0); +lean_inc(x_1648); +lean_dec(x_1643); +x_1649 = l_Lake_LeanOption_decodeToml___closed__3; +x_9 = x_1648; +x_10 = x_1649; +goto block_1641; +} +block_8: +{ +uint8_t x_5; +x_5 = l_Array_isEmpty___rarg(x_4); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_3); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_4); +return x_6; +} +else +{ +lean_object* x_7; +lean_dec(x_4); +x_7 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_7, 0, x_3); +return x_7; +} +} +block_1641: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_1601; lean_object* x_1602; lean_object* x_1603; lean_object* x_1604; lean_object* x_1605; +x_11 = l_Lake_stringToLegalOrSimpleName(x_9); +x_1601 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_1602 = l_Lake_DependencySrc_decodeToml___closed__4; +lean_inc(x_1); +x_1603 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1601, x_1602, x_1); +x_1604 = lean_box(0); +if (lean_obj_tag(x_1603) == 0) +{ +x_12 = x_1604; +x_13 = x_10; +goto block_1600; +} +else +{ +uint8_t x_1611; +x_1611 = !lean_is_exclusive(x_1603); +if (x_1611 == 0) +{ +lean_object* x_1612; lean_object* x_1613; +x_1612 = lean_ctor_get(x_1603, 0); +x_1613 = lean_ctor_get(x_1612, 1); +lean_inc(x_1613); +lean_dec(x_1612); +switch (lean_obj_tag(x_1613)) { +case 0: +{ +lean_object* x_1614; +x_1614 = lean_ctor_get(x_1613, 1); +lean_inc(x_1614); +lean_dec(x_1613); +lean_ctor_set(x_1603, 0, x_1614); +x_12 = x_1603; +x_13 = x_10; +goto block_1600; +} +case 2: +{ +lean_object* x_1615; lean_object* x_1616; lean_object* x_1617; +lean_free_object(x_1603); +x_1615 = lean_ctor_get(x_1613, 0); +lean_inc(x_1615); +lean_dec(x_1613); +x_1616 = l_Lake_Glob_decodeToml___closed__2; +x_1617 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1617, 0, x_1615); +lean_ctor_set(x_1617, 1, x_1616); +x_1605 = x_1617; +goto block_1610; +} +case 3: +{ +lean_object* x_1618; lean_object* x_1619; lean_object* x_1620; +lean_free_object(x_1603); +x_1618 = lean_ctor_get(x_1613, 0); +lean_inc(x_1618); +lean_dec(x_1613); +x_1619 = l_Lake_Glob_decodeToml___closed__2; +x_1620 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1620, 0, x_1618); +lean_ctor_set(x_1620, 1, x_1619); +x_1605 = x_1620; +goto block_1610; +} +default: +{ +uint8_t x_1621; +lean_free_object(x_1603); +x_1621 = !lean_is_exclusive(x_1613); +if (x_1621 == 0) +{ +lean_object* x_1622; lean_object* x_1623; +x_1622 = lean_ctor_get(x_1613, 1); +lean_dec(x_1622); +x_1623 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1613, 0); +lean_ctor_set(x_1613, 1, x_1623); +x_1605 = x_1613; +goto block_1610; +} +else +{ +lean_object* x_1624; lean_object* x_1625; lean_object* x_1626; +x_1624 = lean_ctor_get(x_1613, 0); +lean_inc(x_1624); +lean_dec(x_1613); +x_1625 = l_Lake_Glob_decodeToml___closed__2; +x_1626 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1626, 0, x_1624); +lean_ctor_set(x_1626, 1, x_1625); +x_1605 = x_1626; +goto block_1610; +} +} +} +} +else +{ +lean_object* x_1627; lean_object* x_1628; +x_1627 = lean_ctor_get(x_1603, 0); +lean_inc(x_1627); +lean_dec(x_1603); +x_1628 = lean_ctor_get(x_1627, 1); +lean_inc(x_1628); +lean_dec(x_1627); +switch (lean_obj_tag(x_1628)) { +case 0: +{ +lean_object* x_1629; lean_object* x_1630; +x_1629 = lean_ctor_get(x_1628, 1); +lean_inc(x_1629); +lean_dec(x_1628); +x_1630 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1630, 0, x_1629); +x_12 = x_1630; +x_13 = x_10; +goto block_1600; +} +case 2: +{ +lean_object* x_1631; lean_object* x_1632; lean_object* x_1633; +x_1631 = lean_ctor_get(x_1628, 0); +lean_inc(x_1631); +lean_dec(x_1628); +x_1632 = l_Lake_Glob_decodeToml___closed__2; +x_1633 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1633, 0, x_1631); +lean_ctor_set(x_1633, 1, x_1632); +x_1605 = x_1633; +goto block_1610; +} +case 3: +{ +lean_object* x_1634; lean_object* x_1635; lean_object* x_1636; +x_1634 = lean_ctor_get(x_1628, 0); +lean_inc(x_1634); +lean_dec(x_1628); +x_1635 = l_Lake_Glob_decodeToml___closed__2; +x_1636 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1636, 0, x_1634); +lean_ctor_set(x_1636, 1, x_1635); +x_1605 = x_1636; +goto block_1610; +} +default: +{ +lean_object* x_1637; lean_object* x_1638; lean_object* x_1639; lean_object* x_1640; +x_1637 = lean_ctor_get(x_1628, 0); +lean_inc(x_1637); +if (lean_is_exclusive(x_1628)) { + lean_ctor_release(x_1628, 0); + lean_ctor_release(x_1628, 1); + x_1638 = x_1628; +} else { + lean_dec_ref(x_1628); + x_1638 = lean_box(0); +} +x_1639 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1638)) { + x_1640 = lean_alloc_ctor(0, 2, 0); +} else { + x_1640 = x_1638; + lean_ctor_set_tag(x_1640, 0); +} +lean_ctor_set(x_1640, 0, x_1637); +lean_ctor_set(x_1640, 1, x_1639); +x_1605 = x_1640; +goto block_1610; +} +} +} +} +block_1600: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_148; lean_object* x_149; lean_object* x_395; lean_object* x_396; lean_object* x_1174; lean_object* x_1175; lean_object* x_1176; lean_object* x_1177; lean_object* x_1178; +x_1174 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_1175 = l_Lake_Dependency_decodeToml___closed__10; +lean_inc(x_1); +x_1176 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1175, x_1); +x_1177 = lean_box(0); +if (lean_obj_tag(x_1176) == 0) +{ +lean_object* x_1184; lean_object* x_1185; +x_1184 = l_Lake_Dependency_decodeToml___closed__6; +lean_inc(x_1); +x_1185 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1184, x_1); +if (lean_obj_tag(x_1185) == 0) +{ +lean_object* x_1186; lean_object* x_1187; lean_object* x_1188; +x_1186 = l_Lake_Dependency_decodeToml___closed__8; +lean_inc(x_1); +x_1187 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1186, x_1); +if (lean_obj_tag(x_1187) == 0) +{ +x_14 = x_1177; +x_15 = x_13; +goto block_147; +} +else +{ +uint8_t x_1194; +x_1194 = !lean_is_exclusive(x_1187); +if (x_1194 == 0) +{ +lean_object* x_1195; lean_object* x_1196; +x_1195 = lean_ctor_get(x_1187, 0); +x_1196 = lean_ctor_get(x_1195, 1); +lean_inc(x_1196); +lean_dec(x_1195); +switch (lean_obj_tag(x_1196)) { +case 0: +{ +uint8_t x_1197; +lean_free_object(x_1187); +x_1197 = !lean_is_exclusive(x_1196); +if (x_1197 == 0) +{ +lean_object* x_1198; lean_object* x_1199; +x_1198 = lean_ctor_get(x_1196, 1); +lean_dec(x_1198); +x_1199 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1196, 1, x_1199); +x_1188 = x_1196; +goto block_1193; +} +else +{ +lean_object* x_1200; lean_object* x_1201; lean_object* x_1202; +x_1200 = lean_ctor_get(x_1196, 0); +lean_inc(x_1200); +lean_dec(x_1196); +x_1201 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1202 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1202, 0, x_1200); +lean_ctor_set(x_1202, 1, x_1201); +x_1188 = x_1202; +goto block_1193; +} +} +case 2: +{ +lean_object* x_1203; lean_object* x_1204; lean_object* x_1205; +lean_free_object(x_1187); +x_1203 = lean_ctor_get(x_1196, 0); +lean_inc(x_1203); +lean_dec(x_1196); +x_1204 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1205 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1205, 0, x_1203); +lean_ctor_set(x_1205, 1, x_1204); +x_1188 = x_1205; +goto block_1193; +} +case 3: +{ +lean_object* x_1206; lean_object* x_1207; lean_object* x_1208; +lean_free_object(x_1187); +x_1206 = lean_ctor_get(x_1196, 0); +lean_inc(x_1206); +lean_dec(x_1196); +x_1207 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1208 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1208, 0, x_1206); +lean_ctor_set(x_1208, 1, x_1207); +x_1188 = x_1208; +goto block_1193; +} +case 6: +{ +lean_object* x_1209; lean_object* x_1210; lean_object* x_1211; +x_1209 = lean_ctor_get(x_1196, 0); +lean_inc(x_1209); +x_1210 = lean_ctor_get(x_1196, 1); +lean_inc(x_1210); +lean_dec(x_1196); +x_1211 = l_Lake_DependencySrc_decodeToml(x_1210, x_1209); +if (lean_obj_tag(x_1211) == 0) +{ +lean_object* x_1212; lean_object* x_1213; +lean_free_object(x_1187); +x_1212 = lean_ctor_get(x_1211, 0); +lean_inc(x_1212); +lean_dec(x_1211); +x_1213 = l_Array_append___rarg(x_13, x_1212); +lean_dec(x_1212); +x_14 = x_1177; +x_15 = x_1213; +goto block_147; +} +else +{ +lean_object* x_1214; +x_1214 = lean_ctor_get(x_1211, 0); +lean_inc(x_1214); +lean_dec(x_1211); +lean_ctor_set(x_1187, 0, x_1214); +x_14 = x_1187; +x_15 = x_13; +goto block_147; +} +} +default: +{ +uint8_t x_1215; +lean_free_object(x_1187); +x_1215 = !lean_is_exclusive(x_1196); +if (x_1215 == 0) +{ +lean_object* x_1216; lean_object* x_1217; +x_1216 = lean_ctor_get(x_1196, 1); +lean_dec(x_1216); +x_1217 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_1196, 0); +lean_ctor_set(x_1196, 1, x_1217); +x_1188 = x_1196; +goto block_1193; +} +else +{ +lean_object* x_1218; lean_object* x_1219; lean_object* x_1220; +x_1218 = lean_ctor_get(x_1196, 0); +lean_inc(x_1218); +lean_dec(x_1196); +x_1219 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1220 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1220, 0, x_1218); +lean_ctor_set(x_1220, 1, x_1219); +x_1188 = x_1220; +goto block_1193; +} +} +} +} +else +{ +lean_object* x_1221; lean_object* x_1222; +x_1221 = lean_ctor_get(x_1187, 0); +lean_inc(x_1221); +lean_dec(x_1187); +x_1222 = lean_ctor_get(x_1221, 1); +lean_inc(x_1222); +lean_dec(x_1221); +switch (lean_obj_tag(x_1222)) { +case 0: +{ +lean_object* x_1223; lean_object* x_1224; lean_object* x_1225; lean_object* x_1226; +x_1223 = lean_ctor_get(x_1222, 0); +lean_inc(x_1223); +if (lean_is_exclusive(x_1222)) { + lean_ctor_release(x_1222, 0); + lean_ctor_release(x_1222, 1); + x_1224 = x_1222; +} else { + lean_dec_ref(x_1222); + x_1224 = lean_box(0); +} +x_1225 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1224)) { + x_1226 = lean_alloc_ctor(0, 2, 0); +} else { + x_1226 = x_1224; +} +lean_ctor_set(x_1226, 0, x_1223); +lean_ctor_set(x_1226, 1, x_1225); +x_1188 = x_1226; +goto block_1193; +} +case 2: +{ +lean_object* x_1227; lean_object* x_1228; lean_object* x_1229; +x_1227 = lean_ctor_get(x_1222, 0); +lean_inc(x_1227); +lean_dec(x_1222); +x_1228 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1229 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1229, 0, x_1227); +lean_ctor_set(x_1229, 1, x_1228); +x_1188 = x_1229; +goto block_1193; +} +case 3: +{ +lean_object* x_1230; lean_object* x_1231; lean_object* x_1232; +x_1230 = lean_ctor_get(x_1222, 0); +lean_inc(x_1230); +lean_dec(x_1222); +x_1231 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1232 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1232, 0, x_1230); +lean_ctor_set(x_1232, 1, x_1231); +x_1188 = x_1232; +goto block_1193; +} +case 6: +{ +lean_object* x_1233; lean_object* x_1234; lean_object* x_1235; +x_1233 = lean_ctor_get(x_1222, 0); +lean_inc(x_1233); +x_1234 = lean_ctor_get(x_1222, 1); +lean_inc(x_1234); +lean_dec(x_1222); +x_1235 = l_Lake_DependencySrc_decodeToml(x_1234, x_1233); +if (lean_obj_tag(x_1235) == 0) +{ +lean_object* x_1236; lean_object* x_1237; +x_1236 = lean_ctor_get(x_1235, 0); +lean_inc(x_1236); +lean_dec(x_1235); +x_1237 = l_Array_append___rarg(x_13, x_1236); +lean_dec(x_1236); +x_14 = x_1177; +x_15 = x_1237; +goto block_147; +} +else +{ +lean_object* x_1238; lean_object* x_1239; +x_1238 = lean_ctor_get(x_1235, 0); +lean_inc(x_1238); +lean_dec(x_1235); +x_1239 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1239, 0, x_1238); +x_14 = x_1239; +x_15 = x_13; +goto block_147; +} +} +default: +{ +lean_object* x_1240; lean_object* x_1241; lean_object* x_1242; lean_object* x_1243; +x_1240 = lean_ctor_get(x_1222, 0); +lean_inc(x_1240); +if (lean_is_exclusive(x_1222)) { + lean_ctor_release(x_1222, 0); + lean_ctor_release(x_1222, 1); + x_1241 = x_1222; +} else { + lean_dec_ref(x_1222); + x_1241 = lean_box(0); +} +x_1242 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1241)) { + x_1243 = lean_alloc_ctor(0, 2, 0); +} else { + x_1243 = x_1241; + lean_ctor_set_tag(x_1243, 0); +} +lean_ctor_set(x_1243, 0, x_1240); +lean_ctor_set(x_1243, 1, x_1242); +x_1188 = x_1243; +goto block_1193; +} +} +} +} +block_1193: +{ +lean_object* x_1189; lean_object* x_1190; lean_object* x_1191; lean_object* x_1192; +x_1189 = lean_box(0); +x_1190 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1190, 0, x_1188); +lean_ctor_set(x_1190, 1, x_1189); +x_1191 = lean_array_mk(x_1190); +x_1192 = l_Array_append___rarg(x_13, x_1191); +lean_dec(x_1191); +x_14 = x_1177; +x_15 = x_1192; +goto block_147; +} +} +else +{ +lean_object* x_1244; lean_object* x_1245; lean_object* x_1246; +x_1244 = lean_ctor_get(x_1185, 0); +lean_inc(x_1244); +if (lean_is_exclusive(x_1185)) { + lean_ctor_release(x_1185, 0); + x_1245 = x_1185; +} else { + lean_dec_ref(x_1185); + x_1245 = lean_box(0); +} +x_1246 = lean_ctor_get(x_1244, 1); +lean_inc(x_1246); +lean_dec(x_1244); +switch (lean_obj_tag(x_1246)) { +case 0: +{ +lean_object* x_1247; lean_object* x_1248; lean_object* x_1249; lean_object* x_1250; lean_object* x_1251; +x_1247 = lean_ctor_get(x_1246, 1); +lean_inc(x_1247); +if (lean_is_exclusive(x_1246)) { + lean_ctor_release(x_1246, 0); + lean_ctor_release(x_1246, 1); + x_1248 = x_1246; +} else { + lean_dec_ref(x_1246); + x_1248 = lean_box(0); +} +x_1249 = l_Lake_DependencySrc_decodeToml___closed__2; +lean_inc(x_1); +x_1250 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1249, x_1); +if (lean_obj_tag(x_1250) == 0) +{ +lean_object* x_1259; lean_object* x_1260; +lean_dec(x_1248); +lean_dec(x_1245); +lean_inc(x_12); +x_1259 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1259, 0, x_1247); +lean_ctor_set(x_1259, 1, x_12); +lean_ctor_set(x_1259, 2, x_1177); +x_1260 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1260, 0, x_1259); +x_14 = x_1260; +x_15 = x_13; +goto block_147; +} +else +{ +uint8_t x_1261; +x_1261 = !lean_is_exclusive(x_1250); +if (x_1261 == 0) +{ +lean_object* x_1262; lean_object* x_1263; +x_1262 = lean_ctor_get(x_1250, 0); +x_1263 = lean_ctor_get(x_1262, 1); +lean_inc(x_1263); +lean_dec(x_1262); +switch (lean_obj_tag(x_1263)) { +case 0: +{ +lean_object* x_1264; lean_object* x_1265; lean_object* x_1266; +lean_dec(x_1248); +lean_dec(x_1245); +x_1264 = lean_ctor_get(x_1263, 1); +lean_inc(x_1264); +lean_dec(x_1263); +lean_ctor_set(x_1250, 0, x_1264); +lean_inc(x_12); +x_1265 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1265, 0, x_1247); +lean_ctor_set(x_1265, 1, x_12); +lean_ctor_set(x_1265, 2, x_1250); +x_1266 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1266, 0, x_1265); +x_14 = x_1266; +x_15 = x_13; +goto block_147; +} +case 2: +{ +lean_object* x_1267; lean_object* x_1268; lean_object* x_1269; +lean_free_object(x_1250); +x_1267 = lean_ctor_get(x_1263, 0); +lean_inc(x_1267); +lean_dec(x_1263); +x_1268 = l_Lake_Glob_decodeToml___closed__2; +x_1269 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1269, 0, x_1267); +lean_ctor_set(x_1269, 1, x_1268); +x_1251 = x_1269; +goto block_1258; +} +case 3: +{ +lean_object* x_1270; lean_object* x_1271; lean_object* x_1272; +lean_free_object(x_1250); +x_1270 = lean_ctor_get(x_1263, 0); +lean_inc(x_1270); +lean_dec(x_1263); +x_1271 = l_Lake_Glob_decodeToml___closed__2; +x_1272 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1272, 0, x_1270); +lean_ctor_set(x_1272, 1, x_1271); +x_1251 = x_1272; +goto block_1258; +} +default: +{ +uint8_t x_1273; +lean_free_object(x_1250); +x_1273 = !lean_is_exclusive(x_1263); +if (x_1273 == 0) +{ +lean_object* x_1274; lean_object* x_1275; +x_1274 = lean_ctor_get(x_1263, 1); +lean_dec(x_1274); +x_1275 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1263, 0); +lean_ctor_set(x_1263, 1, x_1275); +x_1251 = x_1263; +goto block_1258; +} +else +{ +lean_object* x_1276; lean_object* x_1277; lean_object* x_1278; +x_1276 = lean_ctor_get(x_1263, 0); +lean_inc(x_1276); +lean_dec(x_1263); +x_1277 = l_Lake_Glob_decodeToml___closed__2; +x_1278 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1278, 0, x_1276); +lean_ctor_set(x_1278, 1, x_1277); +x_1251 = x_1278; +goto block_1258; +} +} +} +} +else +{ +lean_object* x_1279; lean_object* x_1280; +x_1279 = lean_ctor_get(x_1250, 0); +lean_inc(x_1279); +lean_dec(x_1250); +x_1280 = lean_ctor_get(x_1279, 1); +lean_inc(x_1280); +lean_dec(x_1279); +switch (lean_obj_tag(x_1280)) { +case 0: +{ +lean_object* x_1281; lean_object* x_1282; lean_object* x_1283; lean_object* x_1284; +lean_dec(x_1248); +lean_dec(x_1245); +x_1281 = lean_ctor_get(x_1280, 1); +lean_inc(x_1281); +lean_dec(x_1280); +x_1282 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1282, 0, x_1281); +lean_inc(x_12); +x_1283 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1283, 0, x_1247); +lean_ctor_set(x_1283, 1, x_12); +lean_ctor_set(x_1283, 2, x_1282); +x_1284 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1284, 0, x_1283); +x_14 = x_1284; +x_15 = x_13; +goto block_147; +} +case 2: +{ +lean_object* x_1285; lean_object* x_1286; lean_object* x_1287; +x_1285 = lean_ctor_get(x_1280, 0); +lean_inc(x_1285); +lean_dec(x_1280); +x_1286 = l_Lake_Glob_decodeToml___closed__2; +x_1287 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1287, 0, x_1285); +lean_ctor_set(x_1287, 1, x_1286); +x_1251 = x_1287; +goto block_1258; +} +case 3: +{ +lean_object* x_1288; lean_object* x_1289; lean_object* x_1290; +x_1288 = lean_ctor_get(x_1280, 0); +lean_inc(x_1288); +lean_dec(x_1280); +x_1289 = l_Lake_Glob_decodeToml___closed__2; +x_1290 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1290, 0, x_1288); +lean_ctor_set(x_1290, 1, x_1289); +x_1251 = x_1290; +goto block_1258; +} +default: +{ +lean_object* x_1291; lean_object* x_1292; lean_object* x_1293; lean_object* x_1294; +x_1291 = lean_ctor_get(x_1280, 0); +lean_inc(x_1291); +if (lean_is_exclusive(x_1280)) { + lean_ctor_release(x_1280, 0); + lean_ctor_release(x_1280, 1); + x_1292 = x_1280; +} else { + lean_dec_ref(x_1280); + x_1292 = lean_box(0); +} +x_1293 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1292)) { + x_1294 = lean_alloc_ctor(0, 2, 0); +} else { + x_1294 = x_1292; + lean_ctor_set_tag(x_1294, 0); +} +lean_ctor_set(x_1294, 0, x_1291); +lean_ctor_set(x_1294, 1, x_1293); +x_1251 = x_1294; +goto block_1258; +} +} +} +} +block_1258: +{ +lean_object* x_1252; lean_object* x_1253; lean_object* x_1254; lean_object* x_1255; lean_object* x_1256; lean_object* x_1257; +x_1252 = lean_box(0); +if (lean_is_scalar(x_1248)) { + x_1253 = lean_alloc_ctor(1, 2, 0); +} else { + x_1253 = x_1248; + lean_ctor_set_tag(x_1253, 1); +} +lean_ctor_set(x_1253, 0, x_1251); +lean_ctor_set(x_1253, 1, x_1252); +x_1254 = lean_array_mk(x_1253); +x_1255 = l_Array_append___rarg(x_13, x_1254); +lean_dec(x_1254); +lean_inc(x_12); +x_1256 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1256, 0, x_1247); +lean_ctor_set(x_1256, 1, x_12); +lean_ctor_set(x_1256, 2, x_1177); +if (lean_is_scalar(x_1245)) { + x_1257 = lean_alloc_ctor(1, 1, 0); +} else { + x_1257 = x_1245; +} +lean_ctor_set(x_1257, 0, x_1256); +x_14 = x_1257; +x_15 = x_1255; +goto block_147; +} +} +case 2: +{ +lean_object* x_1295; lean_object* x_1296; lean_object* x_1297; lean_object* x_1298; +lean_dec(x_1245); +x_1295 = lean_ctor_get(x_1246, 0); +lean_inc(x_1295); +lean_dec(x_1246); +x_1296 = l_Lake_Dependency_decodeToml___closed__9; +x_1297 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1297, 0, x_1295); +lean_ctor_set(x_1297, 1, x_1296); +x_1298 = lean_array_push(x_13, x_1297); +x_148 = x_1177; +x_149 = x_1298; +goto block_394; +} +case 3: +{ +lean_object* x_1299; lean_object* x_1300; lean_object* x_1301; lean_object* x_1302; +lean_dec(x_1245); +x_1299 = lean_ctor_get(x_1246, 0); +lean_inc(x_1299); +lean_dec(x_1246); +x_1300 = l_Lake_Dependency_decodeToml___closed__9; +x_1301 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1301, 0, x_1299); +lean_ctor_set(x_1301, 1, x_1300); +x_1302 = lean_array_push(x_13, x_1301); +x_148 = x_1177; +x_149 = x_1302; +goto block_394; +} +case 6: +{ +lean_object* x_1303; lean_object* x_1304; lean_object* x_1305; lean_object* x_1306; lean_object* x_1307; lean_object* x_1556; lean_object* x_1557; +x_1303 = lean_ctor_get(x_1246, 0); +lean_inc(x_1303); +x_1304 = lean_ctor_get(x_1246, 1); +lean_inc(x_1304); +if (lean_is_exclusive(x_1246)) { + lean_ctor_release(x_1246, 0); + lean_ctor_release(x_1246, 1); + x_1305 = x_1246; +} else { + lean_dec_ref(x_1246); + x_1305 = lean_box(0); +} +x_1556 = l_Lake_DependencySrc_decodeToml___closed__18; +lean_inc(x_1304); +x_1557 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1304, x_1556, x_1303); +if (lean_obj_tag(x_1557) == 0) +{ +lean_object* x_1558; lean_object* x_1559; lean_object* x_1560; +x_1558 = lean_ctor_get(x_1557, 0); +lean_inc(x_1558); +lean_dec(x_1557); +x_1559 = l_Array_append___rarg(x_13, x_1558); +lean_dec(x_1558); +x_1560 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1306 = x_1560; +x_1307 = x_1559; +goto block_1555; +} +else +{ +lean_object* x_1561; +x_1561 = lean_ctor_get(x_1557, 0); +lean_inc(x_1561); +lean_dec(x_1557); +x_1306 = x_1561; +x_1307 = x_13; +goto block_1555; +} +block_1555: +{ +lean_object* x_1308; lean_object* x_1309; lean_object* x_1310; +x_1308 = l_Lake_DependencySrc_decodeToml___closed__2; +x_1309 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1308, x_1304); +if (lean_obj_tag(x_1309) == 0) +{ +lean_object* x_1318; lean_object* x_1319; lean_object* x_1320; lean_object* x_1321; lean_object* x_1408; lean_object* x_1415; lean_object* x_1416; +lean_dec(x_1305); +lean_dec(x_1245); +x_1318 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1318, 0, x_1306); +lean_ctor_set(x_1318, 1, x_12); +lean_ctor_set(x_1318, 2, x_1177); +x_1319 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1319, 0, x_1318); +x_1415 = l_Lake_Dependency_decodeToml___closed__5; +lean_inc(x_1); +x_1416 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1415, x_1); +if (lean_obj_tag(x_1416) == 0) +{ +lean_object* x_1417; lean_object* x_1418; lean_object* x_1462; lean_object* x_1463; lean_object* x_1468; lean_object* x_1469; lean_object* x_1470; +x_1468 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_1469 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1468, x_1); +if (lean_obj_tag(x_1469) == 0) +{ +x_1417 = x_1177; +x_1418 = x_1307; +goto block_1461; +} +else +{ +uint8_t x_1476; +x_1476 = !lean_is_exclusive(x_1469); +if (x_1476 == 0) +{ +lean_object* x_1477; lean_object* x_1478; +x_1477 = lean_ctor_get(x_1469, 0); +x_1478 = lean_ctor_get(x_1477, 1); +lean_inc(x_1478); +lean_dec(x_1477); +switch (lean_obj_tag(x_1478)) { +case 0: +{ +lean_object* x_1479; +x_1479 = lean_ctor_get(x_1478, 1); +lean_inc(x_1479); +lean_dec(x_1478); +lean_ctor_set(x_1469, 0, x_1479); +x_1462 = x_1469; +x_1463 = x_1307; +goto block_1467; +} +case 2: +{ +lean_object* x_1480; lean_object* x_1481; lean_object* x_1482; +lean_free_object(x_1469); +x_1480 = lean_ctor_get(x_1478, 0); +lean_inc(x_1480); +lean_dec(x_1478); +x_1481 = l_Lake_Glob_decodeToml___closed__2; +x_1482 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1482, 0, x_1480); +lean_ctor_set(x_1482, 1, x_1481); +x_1470 = x_1482; +goto block_1475; +} +case 3: +{ +lean_object* x_1483; lean_object* x_1484; lean_object* x_1485; +lean_free_object(x_1469); +x_1483 = lean_ctor_get(x_1478, 0); +lean_inc(x_1483); +lean_dec(x_1478); +x_1484 = l_Lake_Glob_decodeToml___closed__2; +x_1485 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1485, 0, x_1483); +lean_ctor_set(x_1485, 1, x_1484); +x_1470 = x_1485; +goto block_1475; +} +default: +{ +uint8_t x_1486; +lean_free_object(x_1469); +x_1486 = !lean_is_exclusive(x_1478); +if (x_1486 == 0) +{ +lean_object* x_1487; lean_object* x_1488; +x_1487 = lean_ctor_get(x_1478, 1); +lean_dec(x_1487); +x_1488 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1478, 0); +lean_ctor_set(x_1478, 1, x_1488); +x_1470 = x_1478; +goto block_1475; +} +else +{ +lean_object* x_1489; lean_object* x_1490; lean_object* x_1491; +x_1489 = lean_ctor_get(x_1478, 0); +lean_inc(x_1489); +lean_dec(x_1478); +x_1490 = l_Lake_Glob_decodeToml___closed__2; +x_1491 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1491, 0, x_1489); +lean_ctor_set(x_1491, 1, x_1490); +x_1470 = x_1491; +goto block_1475; +} +} +} +} +else +{ +lean_object* x_1492; lean_object* x_1493; +x_1492 = lean_ctor_get(x_1469, 0); +lean_inc(x_1492); +lean_dec(x_1469); +x_1493 = lean_ctor_get(x_1492, 1); +lean_inc(x_1493); +lean_dec(x_1492); +switch (lean_obj_tag(x_1493)) { +case 0: +{ +lean_object* x_1494; lean_object* x_1495; +x_1494 = lean_ctor_get(x_1493, 1); +lean_inc(x_1494); +lean_dec(x_1493); +x_1495 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1495, 0, x_1494); +x_1462 = x_1495; +x_1463 = x_1307; +goto block_1467; +} +case 2: +{ +lean_object* x_1496; lean_object* x_1497; lean_object* x_1498; +x_1496 = lean_ctor_get(x_1493, 0); +lean_inc(x_1496); +lean_dec(x_1493); +x_1497 = l_Lake_Glob_decodeToml___closed__2; +x_1498 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1498, 0, x_1496); +lean_ctor_set(x_1498, 1, x_1497); +x_1470 = x_1498; +goto block_1475; +} +case 3: +{ +lean_object* x_1499; lean_object* x_1500; lean_object* x_1501; +x_1499 = lean_ctor_get(x_1493, 0); +lean_inc(x_1499); +lean_dec(x_1493); +x_1500 = l_Lake_Glob_decodeToml___closed__2; +x_1501 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1501, 0, x_1499); +lean_ctor_set(x_1501, 1, x_1500); +x_1470 = x_1501; +goto block_1475; +} +default: +{ +lean_object* x_1502; lean_object* x_1503; lean_object* x_1504; lean_object* x_1505; +x_1502 = lean_ctor_get(x_1493, 0); +lean_inc(x_1502); +if (lean_is_exclusive(x_1493)) { + lean_ctor_release(x_1493, 0); + lean_ctor_release(x_1493, 1); + x_1503 = x_1493; +} else { + lean_dec_ref(x_1493); + x_1503 = lean_box(0); +} +x_1504 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1503)) { + x_1505 = lean_alloc_ctor(0, 2, 0); +} else { + x_1505 = x_1503; + lean_ctor_set_tag(x_1505, 0); +} +lean_ctor_set(x_1505, 0, x_1502); +lean_ctor_set(x_1505, 1, x_1504); +x_1470 = x_1505; +goto block_1475; +} +} +} +} +block_1461: +{ +lean_object* x_1419; lean_object* x_1420; lean_object* x_1428; lean_object* x_1429; +x_1419 = lean_box(0); +x_1428 = l_Lake_Dependency_decodeToml___closed__2; +x_1429 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1428, x_1); +if (lean_obj_tag(x_1429) == 0) +{ +lean_object* x_1430; lean_object* x_1431; +x_1430 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1431 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1431, 0, x_11); +lean_ctor_set(x_1431, 1, x_1430); +lean_ctor_set(x_1431, 2, x_1417); +lean_ctor_set(x_1431, 3, x_1319); +lean_ctor_set(x_1431, 4, x_1419); +x_3 = x_1431; +x_4 = x_1418; +goto block_8; +} +else +{ +lean_object* x_1432; lean_object* x_1433; +x_1432 = lean_ctor_get(x_1429, 0); +lean_inc(x_1432); +lean_dec(x_1429); +x_1433 = lean_ctor_get(x_1432, 1); +lean_inc(x_1433); +lean_dec(x_1432); +switch (lean_obj_tag(x_1433)) { +case 0: +{ +uint8_t x_1434; +x_1434 = !lean_is_exclusive(x_1433); +if (x_1434 == 0) +{ +lean_object* x_1435; lean_object* x_1436; +x_1435 = lean_ctor_get(x_1433, 1); +lean_dec(x_1435); +x_1436 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1433, 1, x_1436); +x_1420 = x_1433; +goto block_1427; +} +else +{ +lean_object* x_1437; lean_object* x_1438; lean_object* x_1439; +x_1437 = lean_ctor_get(x_1433, 0); +lean_inc(x_1437); +lean_dec(x_1433); +x_1438 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1439 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1439, 0, x_1437); +lean_ctor_set(x_1439, 1, x_1438); +x_1420 = x_1439; +goto block_1427; +} +} +case 2: +{ +lean_object* x_1440; lean_object* x_1441; lean_object* x_1442; +x_1440 = lean_ctor_get(x_1433, 0); +lean_inc(x_1440); +lean_dec(x_1433); +x_1441 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1442 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1442, 0, x_1440); +lean_ctor_set(x_1442, 1, x_1441); +x_1420 = x_1442; +goto block_1427; +} +case 3: +{ +lean_object* x_1443; lean_object* x_1444; lean_object* x_1445; +x_1443 = lean_ctor_get(x_1433, 0); +lean_inc(x_1443); +lean_dec(x_1433); +x_1444 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1445 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1445, 0, x_1443); +lean_ctor_set(x_1445, 1, x_1444); +x_1420 = x_1445; +goto block_1427; +} +case 6: +{ +lean_object* x_1446; lean_object* x_1447; +x_1446 = lean_ctor_get(x_1433, 1); +lean_inc(x_1446); +lean_dec(x_1433); +x_1447 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_1446); +lean_dec(x_1446); +if (lean_obj_tag(x_1447) == 0) +{ +lean_object* x_1448; lean_object* x_1449; lean_object* x_1450; lean_object* x_1451; +x_1448 = lean_ctor_get(x_1447, 0); +lean_inc(x_1448); +lean_dec(x_1447); +x_1449 = l_Array_append___rarg(x_1418, x_1448); +lean_dec(x_1448); +x_1450 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1451 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1451, 0, x_11); +lean_ctor_set(x_1451, 1, x_1450); +lean_ctor_set(x_1451, 2, x_1417); +lean_ctor_set(x_1451, 3, x_1319); +lean_ctor_set(x_1451, 4, x_1419); +x_3 = x_1451; +x_4 = x_1449; +goto block_8; +} +else +{ +lean_object* x_1452; lean_object* x_1453; lean_object* x_1454; +x_1452 = lean_ctor_get(x_1447, 0); +lean_inc(x_1452); +lean_dec(x_1447); +x_1453 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1454 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1454, 0, x_11); +lean_ctor_set(x_1454, 1, x_1453); +lean_ctor_set(x_1454, 2, x_1417); +lean_ctor_set(x_1454, 3, x_1319); +lean_ctor_set(x_1454, 4, x_1452); +x_3 = x_1454; +x_4 = x_1418; +goto block_8; +} +} +default: +{ +uint8_t x_1455; +x_1455 = !lean_is_exclusive(x_1433); +if (x_1455 == 0) +{ +lean_object* x_1456; lean_object* x_1457; +x_1456 = lean_ctor_get(x_1433, 1); +lean_dec(x_1456); +x_1457 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_1433, 0); +lean_ctor_set(x_1433, 1, x_1457); +x_1420 = x_1433; +goto block_1427; +} +else +{ +lean_object* x_1458; lean_object* x_1459; lean_object* x_1460; +x_1458 = lean_ctor_get(x_1433, 0); +lean_inc(x_1458); +lean_dec(x_1433); +x_1459 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1460 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1460, 0, x_1458); +lean_ctor_set(x_1460, 1, x_1459); +x_1420 = x_1460; +goto block_1427; +} +} +} +} +block_1427: +{ +lean_object* x_1421; lean_object* x_1422; lean_object* x_1423; lean_object* x_1424; lean_object* x_1425; lean_object* x_1426; +x_1421 = lean_box(0); +x_1422 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1422, 0, x_1420); +lean_ctor_set(x_1422, 1, x_1421); +x_1423 = lean_array_mk(x_1422); +x_1424 = l_Array_append___rarg(x_1418, x_1423); +lean_dec(x_1423); +x_1425 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1426 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1426, 0, x_11); +lean_ctor_set(x_1426, 1, x_1425); +lean_ctor_set(x_1426, 2, x_1417); +lean_ctor_set(x_1426, 3, x_1319); +lean_ctor_set(x_1426, 4, x_1419); +x_3 = x_1426; +x_4 = x_1424; +goto block_8; +} +} +block_1467: +{ +if (lean_obj_tag(x_1462) == 0) +{ +x_1417 = x_1177; +x_1418 = x_1463; +goto block_1461; +} +else +{ +uint8_t x_1464; +x_1464 = !lean_is_exclusive(x_1462); +if (x_1464 == 0) +{ +x_1417 = x_1462; +x_1418 = x_1463; +goto block_1461; +} +else +{ +lean_object* x_1465; lean_object* x_1466; +x_1465 = lean_ctor_get(x_1462, 0); +lean_inc(x_1465); +lean_dec(x_1462); +x_1466 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1466, 0, x_1465); +x_1417 = x_1466; +x_1418 = x_1463; +goto block_1461; +} +} +} +block_1475: +{ +lean_object* x_1471; lean_object* x_1472; lean_object* x_1473; lean_object* x_1474; +x_1471 = lean_box(0); +x_1472 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1472, 0, x_1470); +lean_ctor_set(x_1472, 1, x_1471); +x_1473 = lean_array_mk(x_1472); +x_1474 = l_Array_append___rarg(x_1307, x_1473); +lean_dec(x_1473); +x_1462 = x_1177; +x_1463 = x_1474; +goto block_1467; +} +} +else +{ +lean_object* x_1506; lean_object* x_1507; +x_1506 = lean_ctor_get(x_1416, 0); +lean_inc(x_1506); +lean_dec(x_1416); +x_1507 = lean_ctor_get(x_1506, 1); +lean_inc(x_1507); +lean_dec(x_1506); +switch (lean_obj_tag(x_1507)) { +case 0: +{ +lean_object* x_1508; +x_1508 = lean_ctor_get(x_1507, 1); +lean_inc(x_1508); +lean_dec(x_1507); +x_1320 = x_1508; +x_1321 = x_1307; +goto block_1407; +} +case 2: +{ +lean_object* x_1509; lean_object* x_1510; lean_object* x_1511; +x_1509 = lean_ctor_get(x_1507, 0); +lean_inc(x_1509); +lean_dec(x_1507); +x_1510 = l_Lake_Glob_decodeToml___closed__2; +x_1511 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1511, 0, x_1509); +lean_ctor_set(x_1511, 1, x_1510); +x_1408 = x_1511; +goto block_1414; +} +case 3: +{ +lean_object* x_1512; lean_object* x_1513; lean_object* x_1514; +x_1512 = lean_ctor_get(x_1507, 0); +lean_inc(x_1512); +lean_dec(x_1507); +x_1513 = l_Lake_Glob_decodeToml___closed__2; +x_1514 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1514, 0, x_1512); +lean_ctor_set(x_1514, 1, x_1513); +x_1408 = x_1514; +goto block_1414; +} +default: +{ +uint8_t x_1515; +x_1515 = !lean_is_exclusive(x_1507); +if (x_1515 == 0) +{ +lean_object* x_1516; lean_object* x_1517; +x_1516 = lean_ctor_get(x_1507, 1); +lean_dec(x_1516); +x_1517 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1507, 0); +lean_ctor_set(x_1507, 1, x_1517); +x_1408 = x_1507; +goto block_1414; +} +else +{ +lean_object* x_1518; lean_object* x_1519; lean_object* x_1520; +x_1518 = lean_ctor_get(x_1507, 0); +lean_inc(x_1518); +lean_dec(x_1507); +x_1519 = l_Lake_Glob_decodeToml___closed__2; +x_1520 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1520, 0, x_1518); +lean_ctor_set(x_1520, 1, x_1519); +x_1408 = x_1520; +goto block_1414; +} +} +} +} +block_1407: +{ +lean_object* x_1322; lean_object* x_1323; lean_object* x_1363; lean_object* x_1364; lean_object* x_1369; lean_object* x_1370; lean_object* x_1371; +x_1369 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_1370 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1369, x_1); +if (lean_obj_tag(x_1370) == 0) +{ +x_1363 = x_1177; +x_1364 = x_1321; +goto block_1368; +} +else +{ +uint8_t x_1377; +x_1377 = !lean_is_exclusive(x_1370); +if (x_1377 == 0) +{ +lean_object* x_1378; lean_object* x_1379; +x_1378 = lean_ctor_get(x_1370, 0); +x_1379 = lean_ctor_get(x_1378, 1); +lean_inc(x_1379); +lean_dec(x_1378); +switch (lean_obj_tag(x_1379)) { +case 0: +{ +lean_object* x_1380; +x_1380 = lean_ctor_get(x_1379, 1); +lean_inc(x_1380); +lean_dec(x_1379); +lean_ctor_set(x_1370, 0, x_1380); +x_1363 = x_1370; +x_1364 = x_1321; +goto block_1368; +} +case 2: +{ +lean_object* x_1381; lean_object* x_1382; lean_object* x_1383; +lean_free_object(x_1370); +x_1381 = lean_ctor_get(x_1379, 0); +lean_inc(x_1381); +lean_dec(x_1379); +x_1382 = l_Lake_Glob_decodeToml___closed__2; +x_1383 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1383, 0, x_1381); +lean_ctor_set(x_1383, 1, x_1382); +x_1371 = x_1383; +goto block_1376; +} +case 3: +{ +lean_object* x_1384; lean_object* x_1385; lean_object* x_1386; +lean_free_object(x_1370); +x_1384 = lean_ctor_get(x_1379, 0); +lean_inc(x_1384); +lean_dec(x_1379); +x_1385 = l_Lake_Glob_decodeToml___closed__2; +x_1386 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1386, 0, x_1384); +lean_ctor_set(x_1386, 1, x_1385); +x_1371 = x_1386; +goto block_1376; +} +default: +{ +uint8_t x_1387; +lean_free_object(x_1370); +x_1387 = !lean_is_exclusive(x_1379); +if (x_1387 == 0) +{ +lean_object* x_1388; lean_object* x_1389; +x_1388 = lean_ctor_get(x_1379, 1); +lean_dec(x_1388); +x_1389 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1379, 0); +lean_ctor_set(x_1379, 1, x_1389); +x_1371 = x_1379; +goto block_1376; +} +else +{ +lean_object* x_1390; lean_object* x_1391; lean_object* x_1392; +x_1390 = lean_ctor_get(x_1379, 0); +lean_inc(x_1390); +lean_dec(x_1379); +x_1391 = l_Lake_Glob_decodeToml___closed__2; +x_1392 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1392, 0, x_1390); +lean_ctor_set(x_1392, 1, x_1391); +x_1371 = x_1392; +goto block_1376; +} +} +} +} +else +{ +lean_object* x_1393; lean_object* x_1394; +x_1393 = lean_ctor_get(x_1370, 0); +lean_inc(x_1393); +lean_dec(x_1370); +x_1394 = lean_ctor_get(x_1393, 1); +lean_inc(x_1394); +lean_dec(x_1393); +switch (lean_obj_tag(x_1394)) { +case 0: +{ +lean_object* x_1395; lean_object* x_1396; +x_1395 = lean_ctor_get(x_1394, 1); +lean_inc(x_1395); +lean_dec(x_1394); +x_1396 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1396, 0, x_1395); +x_1363 = x_1396; +x_1364 = x_1321; +goto block_1368; +} +case 2: +{ +lean_object* x_1397; lean_object* x_1398; lean_object* x_1399; +x_1397 = lean_ctor_get(x_1394, 0); +lean_inc(x_1397); +lean_dec(x_1394); +x_1398 = l_Lake_Glob_decodeToml___closed__2; +x_1399 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1399, 0, x_1397); +lean_ctor_set(x_1399, 1, x_1398); +x_1371 = x_1399; +goto block_1376; +} +case 3: +{ +lean_object* x_1400; lean_object* x_1401; lean_object* x_1402; +x_1400 = lean_ctor_get(x_1394, 0); +lean_inc(x_1400); +lean_dec(x_1394); +x_1401 = l_Lake_Glob_decodeToml___closed__2; +x_1402 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1402, 0, x_1400); +lean_ctor_set(x_1402, 1, x_1401); +x_1371 = x_1402; +goto block_1376; +} +default: +{ +lean_object* x_1403; lean_object* x_1404; lean_object* x_1405; lean_object* x_1406; +x_1403 = lean_ctor_get(x_1394, 0); +lean_inc(x_1403); +if (lean_is_exclusive(x_1394)) { + lean_ctor_release(x_1394, 0); + lean_ctor_release(x_1394, 1); + x_1404 = x_1394; +} else { + lean_dec_ref(x_1394); + x_1404 = lean_box(0); +} +x_1405 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1404)) { + x_1406 = lean_alloc_ctor(0, 2, 0); +} else { + x_1406 = x_1404; + lean_ctor_set_tag(x_1406, 0); +} +lean_ctor_set(x_1406, 0, x_1403); +lean_ctor_set(x_1406, 1, x_1405); +x_1371 = x_1406; +goto block_1376; +} +} +} +} +block_1362: +{ +lean_object* x_1324; lean_object* x_1325; lean_object* x_1332; lean_object* x_1333; +x_1324 = lean_box(0); +x_1332 = l_Lake_Dependency_decodeToml___closed__2; +x_1333 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1174, x_1332, x_1); +if (lean_obj_tag(x_1333) == 0) +{ +lean_object* x_1334; +x_1334 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1334, 0, x_11); +lean_ctor_set(x_1334, 1, x_1320); +lean_ctor_set(x_1334, 2, x_1322); +lean_ctor_set(x_1334, 3, x_1319); +lean_ctor_set(x_1334, 4, x_1324); +x_3 = x_1334; +x_4 = x_1323; +goto block_8; +} +else +{ +lean_object* x_1335; lean_object* x_1336; +x_1335 = lean_ctor_get(x_1333, 0); +lean_inc(x_1335); +lean_dec(x_1333); +x_1336 = lean_ctor_get(x_1335, 1); +lean_inc(x_1336); +lean_dec(x_1335); +switch (lean_obj_tag(x_1336)) { +case 0: +{ +uint8_t x_1337; +x_1337 = !lean_is_exclusive(x_1336); +if (x_1337 == 0) +{ +lean_object* x_1338; lean_object* x_1339; +x_1338 = lean_ctor_get(x_1336, 1); +lean_dec(x_1338); +x_1339 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1336, 1, x_1339); +x_1325 = x_1336; +goto block_1331; +} +else +{ +lean_object* x_1340; lean_object* x_1341; lean_object* x_1342; +x_1340 = lean_ctor_get(x_1336, 0); +lean_inc(x_1340); +lean_dec(x_1336); +x_1341 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1342 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1342, 0, x_1340); +lean_ctor_set(x_1342, 1, x_1341); +x_1325 = x_1342; +goto block_1331; +} +} +case 2: +{ +lean_object* x_1343; lean_object* x_1344; lean_object* x_1345; +x_1343 = lean_ctor_get(x_1336, 0); +lean_inc(x_1343); +lean_dec(x_1336); +x_1344 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1345 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1345, 0, x_1343); +lean_ctor_set(x_1345, 1, x_1344); +x_1325 = x_1345; +goto block_1331; +} +case 3: +{ +lean_object* x_1346; lean_object* x_1347; lean_object* x_1348; +x_1346 = lean_ctor_get(x_1336, 0); +lean_inc(x_1346); +lean_dec(x_1336); +x_1347 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1348 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1348, 0, x_1346); +lean_ctor_set(x_1348, 1, x_1347); +x_1325 = x_1348; +goto block_1331; +} +case 6: +{ +lean_object* x_1349; lean_object* x_1350; +x_1349 = lean_ctor_get(x_1336, 1); +lean_inc(x_1349); +lean_dec(x_1336); +x_1350 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_1349); +lean_dec(x_1349); +if (lean_obj_tag(x_1350) == 0) +{ +lean_object* x_1351; lean_object* x_1352; lean_object* x_1353; +x_1351 = lean_ctor_get(x_1350, 0); +lean_inc(x_1351); +lean_dec(x_1350); +x_1352 = l_Array_append___rarg(x_1323, x_1351); +lean_dec(x_1351); +x_1353 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1353, 0, x_11); +lean_ctor_set(x_1353, 1, x_1320); +lean_ctor_set(x_1353, 2, x_1322); +lean_ctor_set(x_1353, 3, x_1319); +lean_ctor_set(x_1353, 4, x_1324); +x_3 = x_1353; +x_4 = x_1352; +goto block_8; +} +else +{ +lean_object* x_1354; lean_object* x_1355; +x_1354 = lean_ctor_get(x_1350, 0); +lean_inc(x_1354); +lean_dec(x_1350); +x_1355 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1355, 0, x_11); +lean_ctor_set(x_1355, 1, x_1320); +lean_ctor_set(x_1355, 2, x_1322); +lean_ctor_set(x_1355, 3, x_1319); +lean_ctor_set(x_1355, 4, x_1354); +x_3 = x_1355; +x_4 = x_1323; +goto block_8; +} +} +default: +{ +uint8_t x_1356; +x_1356 = !lean_is_exclusive(x_1336); +if (x_1356 == 0) +{ +lean_object* x_1357; lean_object* x_1358; +x_1357 = lean_ctor_get(x_1336, 1); +lean_dec(x_1357); +x_1358 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_1336, 0); +lean_ctor_set(x_1336, 1, x_1358); +x_1325 = x_1336; +goto block_1331; +} +else +{ +lean_object* x_1359; lean_object* x_1360; lean_object* x_1361; +x_1359 = lean_ctor_get(x_1336, 0); +lean_inc(x_1359); +lean_dec(x_1336); +x_1360 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1361 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1361, 0, x_1359); +lean_ctor_set(x_1361, 1, x_1360); +x_1325 = x_1361; +goto block_1331; +} +} +} +} +block_1331: +{ +lean_object* x_1326; lean_object* x_1327; lean_object* x_1328; lean_object* x_1329; lean_object* x_1330; +x_1326 = lean_box(0); +x_1327 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1327, 0, x_1325); +lean_ctor_set(x_1327, 1, x_1326); +x_1328 = lean_array_mk(x_1327); +x_1329 = l_Array_append___rarg(x_1323, x_1328); +lean_dec(x_1328); +x_1330 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1330, 0, x_11); +lean_ctor_set(x_1330, 1, x_1320); +lean_ctor_set(x_1330, 2, x_1322); +lean_ctor_set(x_1330, 3, x_1319); +lean_ctor_set(x_1330, 4, x_1324); +x_3 = x_1330; +x_4 = x_1329; +goto block_8; +} +} +block_1368: +{ +if (lean_obj_tag(x_1363) == 0) +{ +x_1322 = x_1177; +x_1323 = x_1364; +goto block_1362; +} +else +{ +uint8_t x_1365; +x_1365 = !lean_is_exclusive(x_1363); +if (x_1365 == 0) +{ +x_1322 = x_1363; +x_1323 = x_1364; +goto block_1362; +} +else +{ +lean_object* x_1366; lean_object* x_1367; +x_1366 = lean_ctor_get(x_1363, 0); +lean_inc(x_1366); +lean_dec(x_1363); +x_1367 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1367, 0, x_1366); +x_1322 = x_1367; +x_1323 = x_1364; +goto block_1362; +} +} +} +block_1376: +{ +lean_object* x_1372; lean_object* x_1373; lean_object* x_1374; lean_object* x_1375; +x_1372 = lean_box(0); +x_1373 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1373, 0, x_1371); +lean_ctor_set(x_1373, 1, x_1372); +x_1374 = lean_array_mk(x_1373); +x_1375 = l_Array_append___rarg(x_1321, x_1374); +lean_dec(x_1374); +x_1363 = x_1177; +x_1364 = x_1375; +goto block_1368; +} +} +block_1414: +{ +lean_object* x_1409; lean_object* x_1410; lean_object* x_1411; lean_object* x_1412; lean_object* x_1413; +x_1409 = lean_box(0); +x_1410 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1410, 0, x_1408); +lean_ctor_set(x_1410, 1, x_1409); +x_1411 = lean_array_mk(x_1410); +x_1412 = l_Array_append___rarg(x_1307, x_1411); +lean_dec(x_1411); +x_1413 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1320 = x_1413; +x_1321 = x_1412; +goto block_1407; +} +} +else +{ +uint8_t x_1521; +x_1521 = !lean_is_exclusive(x_1309); +if (x_1521 == 0) +{ +lean_object* x_1522; lean_object* x_1523; +x_1522 = lean_ctor_get(x_1309, 0); +x_1523 = lean_ctor_get(x_1522, 1); +lean_inc(x_1523); +lean_dec(x_1522); +switch (lean_obj_tag(x_1523)) { +case 0: +{ +lean_object* x_1524; lean_object* x_1525; lean_object* x_1526; +lean_dec(x_1305); +lean_dec(x_1245); +x_1524 = lean_ctor_get(x_1523, 1); +lean_inc(x_1524); +lean_dec(x_1523); +lean_ctor_set(x_1309, 0, x_1524); +lean_inc(x_12); +x_1525 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1525, 0, x_1306); +lean_ctor_set(x_1525, 1, x_12); +lean_ctor_set(x_1525, 2, x_1309); +x_1526 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1526, 0, x_1525); +x_14 = x_1526; +x_15 = x_1307; +goto block_147; +} +case 2: +{ +lean_object* x_1527; lean_object* x_1528; lean_object* x_1529; +lean_free_object(x_1309); +x_1527 = lean_ctor_get(x_1523, 0); +lean_inc(x_1527); +lean_dec(x_1523); +x_1528 = l_Lake_Glob_decodeToml___closed__2; +x_1529 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1529, 0, x_1527); +lean_ctor_set(x_1529, 1, x_1528); +x_1310 = x_1529; +goto block_1317; +} +case 3: +{ +lean_object* x_1530; lean_object* x_1531; lean_object* x_1532; +lean_free_object(x_1309); +x_1530 = lean_ctor_get(x_1523, 0); +lean_inc(x_1530); +lean_dec(x_1523); +x_1531 = l_Lake_Glob_decodeToml___closed__2; +x_1532 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1532, 0, x_1530); +lean_ctor_set(x_1532, 1, x_1531); +x_1310 = x_1532; +goto block_1317; +} +default: +{ +uint8_t x_1533; +lean_free_object(x_1309); +x_1533 = !lean_is_exclusive(x_1523); +if (x_1533 == 0) +{ +lean_object* x_1534; lean_object* x_1535; +x_1534 = lean_ctor_get(x_1523, 1); +lean_dec(x_1534); +x_1535 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1523, 0); +lean_ctor_set(x_1523, 1, x_1535); +x_1310 = x_1523; +goto block_1317; +} +else +{ +lean_object* x_1536; lean_object* x_1537; lean_object* x_1538; +x_1536 = lean_ctor_get(x_1523, 0); +lean_inc(x_1536); +lean_dec(x_1523); +x_1537 = l_Lake_Glob_decodeToml___closed__2; +x_1538 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1538, 0, x_1536); +lean_ctor_set(x_1538, 1, x_1537); +x_1310 = x_1538; +goto block_1317; +} +} +} +} +else +{ +lean_object* x_1539; lean_object* x_1540; +x_1539 = lean_ctor_get(x_1309, 0); +lean_inc(x_1539); +lean_dec(x_1309); +x_1540 = lean_ctor_get(x_1539, 1); +lean_inc(x_1540); +lean_dec(x_1539); +switch (lean_obj_tag(x_1540)) { +case 0: +{ +lean_object* x_1541; lean_object* x_1542; lean_object* x_1543; lean_object* x_1544; +lean_dec(x_1305); +lean_dec(x_1245); +x_1541 = lean_ctor_get(x_1540, 1); +lean_inc(x_1541); +lean_dec(x_1540); +x_1542 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1542, 0, x_1541); +lean_inc(x_12); +x_1543 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1543, 0, x_1306); +lean_ctor_set(x_1543, 1, x_12); +lean_ctor_set(x_1543, 2, x_1542); +x_1544 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1544, 0, x_1543); +x_14 = x_1544; +x_15 = x_1307; +goto block_147; +} +case 2: +{ +lean_object* x_1545; lean_object* x_1546; lean_object* x_1547; +x_1545 = lean_ctor_get(x_1540, 0); +lean_inc(x_1545); +lean_dec(x_1540); +x_1546 = l_Lake_Glob_decodeToml___closed__2; +x_1547 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1547, 0, x_1545); +lean_ctor_set(x_1547, 1, x_1546); +x_1310 = x_1547; +goto block_1317; +} +case 3: +{ +lean_object* x_1548; lean_object* x_1549; lean_object* x_1550; +x_1548 = lean_ctor_get(x_1540, 0); +lean_inc(x_1548); +lean_dec(x_1540); +x_1549 = l_Lake_Glob_decodeToml___closed__2; +x_1550 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1550, 0, x_1548); +lean_ctor_set(x_1550, 1, x_1549); +x_1310 = x_1550; +goto block_1317; +} +default: +{ +lean_object* x_1551; lean_object* x_1552; lean_object* x_1553; lean_object* x_1554; +x_1551 = lean_ctor_get(x_1540, 0); +lean_inc(x_1551); +if (lean_is_exclusive(x_1540)) { + lean_ctor_release(x_1540, 0); + lean_ctor_release(x_1540, 1); + x_1552 = x_1540; +} else { + lean_dec_ref(x_1540); + x_1552 = lean_box(0); +} +x_1553 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1552)) { + x_1554 = lean_alloc_ctor(0, 2, 0); +} else { + x_1554 = x_1552; + lean_ctor_set_tag(x_1554, 0); +} +lean_ctor_set(x_1554, 0, x_1551); +lean_ctor_set(x_1554, 1, x_1553); +x_1310 = x_1554; +goto block_1317; +} +} +} +} +block_1317: +{ +lean_object* x_1311; lean_object* x_1312; lean_object* x_1313; lean_object* x_1314; lean_object* x_1315; lean_object* x_1316; +x_1311 = lean_box(0); +if (lean_is_scalar(x_1305)) { + x_1312 = lean_alloc_ctor(1, 2, 0); +} else { + x_1312 = x_1305; + lean_ctor_set_tag(x_1312, 1); +} +lean_ctor_set(x_1312, 0, x_1310); +lean_ctor_set(x_1312, 1, x_1311); +x_1313 = lean_array_mk(x_1312); +x_1314 = l_Array_append___rarg(x_1307, x_1313); +lean_dec(x_1313); +lean_inc(x_12); +x_1315 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_1315, 0, x_1306); +lean_ctor_set(x_1315, 1, x_12); +lean_ctor_set(x_1315, 2, x_1177); +if (lean_is_scalar(x_1245)) { + x_1316 = lean_alloc_ctor(1, 1, 0); +} else { + x_1316 = x_1245; +} +lean_ctor_set(x_1316, 0, x_1315); +x_14 = x_1316; +x_15 = x_1314; +goto block_147; +} +} +} +default: +{ +uint8_t x_1562; +lean_dec(x_1245); +x_1562 = !lean_is_exclusive(x_1246); +if (x_1562 == 0) +{ +lean_object* x_1563; lean_object* x_1564; lean_object* x_1565; +x_1563 = lean_ctor_get(x_1246, 1); +lean_dec(x_1563); +x_1564 = l_Lake_Dependency_decodeToml___closed__9; +lean_ctor_set_tag(x_1246, 0); +lean_ctor_set(x_1246, 1, x_1564); +x_1565 = lean_array_push(x_13, x_1246); +x_148 = x_1177; +x_149 = x_1565; +goto block_394; +} +else +{ +lean_object* x_1566; lean_object* x_1567; lean_object* x_1568; lean_object* x_1569; +x_1566 = lean_ctor_get(x_1246, 0); +lean_inc(x_1566); +lean_dec(x_1246); +x_1567 = l_Lake_Dependency_decodeToml___closed__9; +x_1568 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1568, 0, x_1566); +lean_ctor_set(x_1568, 1, x_1567); +x_1569 = lean_array_push(x_13, x_1568); +x_148 = x_1177; +x_149 = x_1569; +goto block_394; +} +} +} +} +} +else +{ +uint8_t x_1570; +x_1570 = !lean_is_exclusive(x_1176); +if (x_1570 == 0) +{ +lean_object* x_1571; lean_object* x_1572; +x_1571 = lean_ctor_get(x_1176, 0); +x_1572 = lean_ctor_get(x_1571, 1); +lean_inc(x_1572); +lean_dec(x_1571); +switch (lean_obj_tag(x_1572)) { +case 0: +{ +lean_object* x_1573; +x_1573 = lean_ctor_get(x_1572, 1); +lean_inc(x_1573); +lean_dec(x_1572); +lean_ctor_set(x_1176, 0, x_1573); +x_395 = x_1176; +x_396 = x_13; +goto block_1173; +} +case 2: +{ +lean_object* x_1574; lean_object* x_1575; lean_object* x_1576; +lean_free_object(x_1176); +x_1574 = lean_ctor_get(x_1572, 0); +lean_inc(x_1574); +lean_dec(x_1572); +x_1575 = l_Lake_Glob_decodeToml___closed__2; +x_1576 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1576, 0, x_1574); +lean_ctor_set(x_1576, 1, x_1575); +x_1178 = x_1576; +goto block_1183; +} +case 3: +{ +lean_object* x_1577; lean_object* x_1578; lean_object* x_1579; +lean_free_object(x_1176); +x_1577 = lean_ctor_get(x_1572, 0); +lean_inc(x_1577); +lean_dec(x_1572); +x_1578 = l_Lake_Glob_decodeToml___closed__2; +x_1579 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1579, 0, x_1577); +lean_ctor_set(x_1579, 1, x_1578); +x_1178 = x_1579; +goto block_1183; +} +default: +{ +uint8_t x_1580; +lean_free_object(x_1176); +x_1580 = !lean_is_exclusive(x_1572); +if (x_1580 == 0) +{ +lean_object* x_1581; lean_object* x_1582; +x_1581 = lean_ctor_get(x_1572, 1); +lean_dec(x_1581); +x_1582 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_1572, 0); +lean_ctor_set(x_1572, 1, x_1582); +x_1178 = x_1572; +goto block_1183; +} +else +{ +lean_object* x_1583; lean_object* x_1584; lean_object* x_1585; +x_1583 = lean_ctor_get(x_1572, 0); +lean_inc(x_1583); +lean_dec(x_1572); +x_1584 = l_Lake_Glob_decodeToml___closed__2; +x_1585 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1585, 0, x_1583); +lean_ctor_set(x_1585, 1, x_1584); +x_1178 = x_1585; +goto block_1183; +} +} +} +} +else +{ +lean_object* x_1586; lean_object* x_1587; +x_1586 = lean_ctor_get(x_1176, 0); +lean_inc(x_1586); +lean_dec(x_1176); +x_1587 = lean_ctor_get(x_1586, 1); +lean_inc(x_1587); +lean_dec(x_1586); +switch (lean_obj_tag(x_1587)) { +case 0: +{ +lean_object* x_1588; lean_object* x_1589; +x_1588 = lean_ctor_get(x_1587, 1); +lean_inc(x_1588); +lean_dec(x_1587); +x_1589 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1589, 0, x_1588); +x_395 = x_1589; +x_396 = x_13; +goto block_1173; +} +case 2: +{ +lean_object* x_1590; lean_object* x_1591; lean_object* x_1592; +x_1590 = lean_ctor_get(x_1587, 0); +lean_inc(x_1590); +lean_dec(x_1587); +x_1591 = l_Lake_Glob_decodeToml___closed__2; +x_1592 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1592, 0, x_1590); +lean_ctor_set(x_1592, 1, x_1591); +x_1178 = x_1592; +goto block_1183; +} +case 3: +{ +lean_object* x_1593; lean_object* x_1594; lean_object* x_1595; +x_1593 = lean_ctor_get(x_1587, 0); +lean_inc(x_1593); +lean_dec(x_1587); +x_1594 = l_Lake_Glob_decodeToml___closed__2; +x_1595 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1595, 0, x_1593); +lean_ctor_set(x_1595, 1, x_1594); +x_1178 = x_1595; +goto block_1183; +} +default: +{ +lean_object* x_1596; lean_object* x_1597; lean_object* x_1598; lean_object* x_1599; +x_1596 = lean_ctor_get(x_1587, 0); +lean_inc(x_1596); +if (lean_is_exclusive(x_1587)) { + lean_ctor_release(x_1587, 0); + lean_ctor_release(x_1587, 1); + x_1597 = x_1587; +} else { + lean_dec_ref(x_1587); + x_1597 = lean_box(0); +} +x_1598 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1597)) { + x_1599 = lean_alloc_ctor(0, 2, 0); +} else { + x_1599 = x_1597; + lean_ctor_set_tag(x_1599, 0); +} +lean_ctor_set(x_1599, 0, x_1596); +lean_ctor_set(x_1599, 1, x_1598); +x_1178 = x_1599; +goto block_1183; +} +} +} +} +block_147: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_121; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_129 = l_Lake_Dependency_decodeToml___closed__5; +lean_inc(x_1); +x_130 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_128, x_129, x_1); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; +x_131 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_16 = x_131; +x_17 = x_15; +goto block_120; +} +else +{ +lean_object* x_132; lean_object* x_133; +x_132 = lean_ctor_get(x_130, 0); +lean_inc(x_132); +lean_dec(x_130); +x_133 = lean_ctor_get(x_132, 1); +lean_inc(x_133); +lean_dec(x_132); +switch (lean_obj_tag(x_133)) { +case 0: +{ +lean_object* x_134; +x_134 = lean_ctor_get(x_133, 1); +lean_inc(x_134); +lean_dec(x_133); +x_16 = x_134; +x_17 = x_15; +goto block_120; +} +case 2: +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_133, 0); +lean_inc(x_135); +lean_dec(x_133); +x_136 = l_Lake_Glob_decodeToml___closed__2; +x_137 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +x_121 = x_137; +goto block_127; +} +case 3: +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_133, 0); +lean_inc(x_138); +lean_dec(x_133); +x_139 = l_Lake_Glob_decodeToml___closed__2; +x_140 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_140, 0, x_138); +lean_ctor_set(x_140, 1, x_139); +x_121 = x_140; +goto block_127; +} +default: +{ +uint8_t x_141; +x_141 = !lean_is_exclusive(x_133); +if (x_141 == 0) +{ +lean_object* x_142; lean_object* x_143; +x_142 = lean_ctor_get(x_133, 1); +lean_dec(x_142); +x_143 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_133, 0); +lean_ctor_set(x_133, 1, x_143); +x_121 = x_133; +goto block_127; +} +else +{ +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_133, 0); +lean_inc(x_144); +lean_dec(x_133); +x_145 = l_Lake_Glob_decodeToml___closed__2; +x_146 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_121 = x_146; +goto block_127; +} +} +} +} +block_120: +{ +lean_object* x_18; lean_object* x_19; lean_object* x_60; lean_object* x_61; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_80 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_81 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_82 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_80, x_81, x_1); +x_83 = lean_box(0); +if (lean_obj_tag(x_82) == 0) +{ +x_60 = x_83; +x_61 = x_17; +goto block_79; +} +else +{ +uint8_t x_90; +x_90 = !lean_is_exclusive(x_82); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; +x_91 = lean_ctor_get(x_82, 0); +x_92 = lean_ctor_get(x_91, 1); +lean_inc(x_92); +lean_dec(x_91); +switch (lean_obj_tag(x_92)) { +case 0: +{ +lean_object* x_93; +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +lean_ctor_set(x_82, 0, x_93); +x_60 = x_82; +x_61 = x_17; +goto block_79; +} +case 2: +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_free_object(x_82); +x_94 = lean_ctor_get(x_92, 0); +lean_inc(x_94); +lean_dec(x_92); +x_95 = l_Lake_Glob_decodeToml___closed__2; +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_84 = x_96; +goto block_89; +} +case 3: +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_free_object(x_82); +x_97 = lean_ctor_get(x_92, 0); +lean_inc(x_97); +lean_dec(x_92); +x_98 = l_Lake_Glob_decodeToml___closed__2; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +x_84 = x_99; +goto block_89; +} +default: +{ +uint8_t x_100; +lean_free_object(x_82); +x_100 = !lean_is_exclusive(x_92); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; +x_101 = lean_ctor_get(x_92, 1); +lean_dec(x_101); +x_102 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_92, 0); +lean_ctor_set(x_92, 1, x_102); +x_84 = x_92; +goto block_89; +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_103 = lean_ctor_get(x_92, 0); +lean_inc(x_103); +lean_dec(x_92); +x_104 = l_Lake_Glob_decodeToml___closed__2; +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +x_84 = x_105; +goto block_89; +} +} +} +} +else +{ +lean_object* x_106; lean_object* x_107; +x_106 = lean_ctor_get(x_82, 0); +lean_inc(x_106); +lean_dec(x_82); +x_107 = lean_ctor_get(x_106, 1); +lean_inc(x_107); +lean_dec(x_106); +switch (lean_obj_tag(x_107)) { +case 0: +{ +lean_object* x_108; lean_object* x_109; +x_108 = lean_ctor_get(x_107, 1); +lean_inc(x_108); +lean_dec(x_107); +x_109 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_109, 0, x_108); +x_60 = x_109; +x_61 = x_17; +goto block_79; +} +case 2: +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_107, 0); +lean_inc(x_110); +lean_dec(x_107); +x_111 = l_Lake_Glob_decodeToml___closed__2; +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +x_84 = x_112; +goto block_89; +} +case 3: +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_107, 0); +lean_inc(x_113); +lean_dec(x_107); +x_114 = l_Lake_Glob_decodeToml___closed__2; +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +x_84 = x_115; +goto block_89; +} +default: +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_116 = lean_ctor_get(x_107, 0); +lean_inc(x_116); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_117 = x_107; +} else { + lean_dec_ref(x_107); + x_117 = lean_box(0); +} +x_118 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_117)) { + x_119 = lean_alloc_ctor(0, 2, 0); +} else { + x_119 = x_117; + lean_ctor_set_tag(x_119, 0); +} +lean_ctor_set(x_119, 0, x_116); +lean_ctor_set(x_119, 1, x_118); +x_84 = x_119; +goto block_89; +} +} +} +} +block_59: +{ +lean_object* x_20; lean_object* x_21; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_20 = lean_box(0); +x_28 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_29 = l_Lake_Dependency_decodeToml___closed__2; +x_30 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_28, x_29, x_1); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; +x_31 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_31, 0, x_11); +lean_ctor_set(x_31, 1, x_16); +lean_ctor_set(x_31, 2, x_18); +lean_ctor_set(x_31, 3, x_14); +lean_ctor_set(x_31, 4, x_20); +x_3 = x_31; +x_4 = x_19; +goto block_8; +} +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_30, 0); +lean_inc(x_32); +lean_dec(x_30); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +switch (lean_obj_tag(x_33)) { +case 0: +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_33, 1); +lean_dec(x_35); +x_36 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_33, 1, x_36); +x_21 = x_33; +goto block_27; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_33, 0); +lean_inc(x_37); +lean_dec(x_33); +x_38 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +x_21 = x_39; +goto block_27; +} +} +case 2: +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_33, 0); +lean_inc(x_40); +lean_dec(x_33); +x_41 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_21 = x_42; +goto block_27; +} +case 3: +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_33, 0); +lean_inc(x_43); +lean_dec(x_33); +x_44 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +x_21 = x_45; +goto block_27; +} +case 6: +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_33, 1); +lean_inc(x_46); +lean_dec(x_33); +x_47 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_46); +lean_dec(x_46); +if (lean_obj_tag(x_47) == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +lean_dec(x_47); +x_49 = l_Array_append___rarg(x_19, x_48); +lean_dec(x_48); +x_50 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_50, 0, x_11); +lean_ctor_set(x_50, 1, x_16); +lean_ctor_set(x_50, 2, x_18); +lean_ctor_set(x_50, 3, x_14); +lean_ctor_set(x_50, 4, x_20); +x_3 = x_50; +x_4 = x_49; +goto block_8; +} +else +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_47, 0); +lean_inc(x_51); +lean_dec(x_47); +x_52 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_52, 0, x_11); +lean_ctor_set(x_52, 1, x_16); +lean_ctor_set(x_52, 2, x_18); +lean_ctor_set(x_52, 3, x_14); +lean_ctor_set(x_52, 4, x_51); +x_3 = x_52; +x_4 = x_19; +goto block_8; +} +} +default: +{ +uint8_t x_53; +x_53 = !lean_is_exclusive(x_33); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; +x_54 = lean_ctor_get(x_33, 1); +lean_dec(x_54); +x_55 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_33, 0); +lean_ctor_set(x_33, 1, x_55); +x_21 = x_33; +goto block_27; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_33, 0); +lean_inc(x_56); +lean_dec(x_33); +x_57 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +x_21 = x_58; +goto block_27; +} +} +} +} +block_27: +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_array_mk(x_23); +x_25 = l_Array_append___rarg(x_19, x_24); +lean_dec(x_24); +x_26 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_26, 0, x_11); +lean_ctor_set(x_26, 1, x_16); +lean_ctor_set(x_26, 2, x_18); +lean_ctor_set(x_26, 3, x_14); +lean_ctor_set(x_26, 4, x_20); +x_3 = x_26; +x_4 = x_25; +goto block_8; +} +} +block_79: +{ +if (lean_obj_tag(x_60) == 0) +{ +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_62; +x_62 = lean_box(0); +x_18 = x_62; +x_19 = x_61; +goto block_59; +} +else +{ +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_63; +x_63 = !lean_is_exclusive(x_12); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_64 = lean_ctor_get(x_12, 0); +x_65 = l_Lake_Dependency_decodeToml___closed__3; +x_66 = lean_string_append(x_65, x_64); +lean_dec(x_64); +x_67 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_68 = lean_string_append(x_66, x_67); +lean_ctor_set(x_12, 0, x_68); +x_18 = x_12; +x_19 = x_61; +goto block_59; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_69 = lean_ctor_get(x_12, 0); +lean_inc(x_69); +lean_dec(x_12); +x_70 = l_Lake_Dependency_decodeToml___closed__3; +x_71 = lean_string_append(x_70, x_69); +lean_dec(x_69); +x_72 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_73 = lean_string_append(x_71, x_72); +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_73); +x_18 = x_74; +x_19 = x_61; +goto block_59; +} +} +else +{ +lean_object* x_75; +lean_dec(x_12); +x_75 = lean_box(0); +x_18 = x_75; +x_19 = x_61; +goto block_59; +} +} +} +else +{ +uint8_t x_76; +lean_dec(x_12); +x_76 = !lean_is_exclusive(x_60); +if (x_76 == 0) +{ +x_18 = x_60; +x_19 = x_61; +goto block_59; +} +else +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_60, 0); +lean_inc(x_77); +lean_dec(x_60); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_77); +x_18 = x_78; +x_19 = x_61; +goto block_59; +} +} +} +block_89: +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_85 = lean_box(0); +x_86 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_85); +x_87 = lean_array_mk(x_86); +x_88 = l_Array_append___rarg(x_17, x_87); +lean_dec(x_87); +x_60 = x_83; +x_61 = x_88; +goto block_79; +} +} +block_127: +{ +lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_122 = lean_box(0); +x_123 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_123, 0, x_121); +lean_ctor_set(x_123, 1, x_122); +x_124 = lean_array_mk(x_123); +x_125 = l_Array_append___rarg(x_15, x_124); +lean_dec(x_124); +x_126 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_16 = x_126; +x_17 = x_125; +goto block_120; +} +} +block_394: +{ +lean_object* x_150; lean_object* x_151; lean_object* x_254; lean_object* x_261; lean_object* x_262; lean_object* x_263; +x_261 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_262 = l_Lake_Dependency_decodeToml___closed__5; +lean_inc(x_1); +x_263 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_261, x_262, x_1); +if (lean_obj_tag(x_263) == 0) +{ +lean_object* x_264; lean_object* x_265; lean_object* x_309; lean_object* x_310; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; +x_328 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_329 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_261, x_328, x_1); +x_330 = lean_box(0); +if (lean_obj_tag(x_329) == 0) +{ +if (lean_obj_tag(x_12) == 0) +{ +x_264 = x_330; +x_265 = x_149; +goto block_308; +} +else +{ +uint8_t x_337; +x_337 = !lean_is_exclusive(x_12); +if (x_337 == 0) +{ +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; +x_338 = lean_ctor_get(x_12, 0); +x_339 = l_Lake_Dependency_decodeToml___closed__3; +x_340 = lean_string_append(x_339, x_338); +lean_dec(x_338); +x_341 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_342 = lean_string_append(x_340, x_341); +lean_ctor_set(x_12, 0, x_342); +x_264 = x_12; +x_265 = x_149; +goto block_308; +} +else +{ +lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; +x_343 = lean_ctor_get(x_12, 0); +lean_inc(x_343); +lean_dec(x_12); +x_344 = l_Lake_Dependency_decodeToml___closed__3; +x_345 = lean_string_append(x_344, x_343); +lean_dec(x_343); +x_346 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_347 = lean_string_append(x_345, x_346); +x_348 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_348, 0, x_347); +x_264 = x_348; +x_265 = x_149; +goto block_308; +} +} +} +else +{ +uint8_t x_349; +x_349 = !lean_is_exclusive(x_329); +if (x_349 == 0) +{ +lean_object* x_350; lean_object* x_351; +x_350 = lean_ctor_get(x_329, 0); +x_351 = lean_ctor_get(x_350, 1); +lean_inc(x_351); +lean_dec(x_350); +switch (lean_obj_tag(x_351)) { +case 0: +{ +lean_object* x_352; +x_352 = lean_ctor_get(x_351, 1); +lean_inc(x_352); +lean_dec(x_351); +lean_ctor_set(x_329, 0, x_352); +x_309 = x_329; +x_310 = x_149; +goto block_327; +} +case 2: +{ +lean_object* x_353; lean_object* x_354; lean_object* x_355; +lean_free_object(x_329); +x_353 = lean_ctor_get(x_351, 0); +lean_inc(x_353); +lean_dec(x_351); +x_354 = l_Lake_Glob_decodeToml___closed__2; +x_355 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_355, 0, x_353); +lean_ctor_set(x_355, 1, x_354); +x_331 = x_355; +goto block_336; +} +case 3: +{ +lean_object* x_356; lean_object* x_357; lean_object* x_358; +lean_free_object(x_329); +x_356 = lean_ctor_get(x_351, 0); +lean_inc(x_356); +lean_dec(x_351); +x_357 = l_Lake_Glob_decodeToml___closed__2; +x_358 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_358, 0, x_356); +lean_ctor_set(x_358, 1, x_357); +x_331 = x_358; +goto block_336; +} +default: +{ +uint8_t x_359; +lean_free_object(x_329); +x_359 = !lean_is_exclusive(x_351); +if (x_359 == 0) +{ +lean_object* x_360; lean_object* x_361; +x_360 = lean_ctor_get(x_351, 1); +lean_dec(x_360); +x_361 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_351, 0); +lean_ctor_set(x_351, 1, x_361); +x_331 = x_351; +goto block_336; +} +else +{ +lean_object* x_362; lean_object* x_363; lean_object* x_364; +x_362 = lean_ctor_get(x_351, 0); +lean_inc(x_362); +lean_dec(x_351); +x_363 = l_Lake_Glob_decodeToml___closed__2; +x_364 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_364, 0, x_362); +lean_ctor_set(x_364, 1, x_363); +x_331 = x_364; +goto block_336; +} +} +} +} +else +{ +lean_object* x_365; lean_object* x_366; +x_365 = lean_ctor_get(x_329, 0); +lean_inc(x_365); +lean_dec(x_329); +x_366 = lean_ctor_get(x_365, 1); +lean_inc(x_366); +lean_dec(x_365); +switch (lean_obj_tag(x_366)) { +case 0: +{ +lean_object* x_367; lean_object* x_368; +x_367 = lean_ctor_get(x_366, 1); +lean_inc(x_367); +lean_dec(x_366); +x_368 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_368, 0, x_367); +x_309 = x_368; +x_310 = x_149; +goto block_327; +} +case 2: +{ +lean_object* x_369; lean_object* x_370; lean_object* x_371; +x_369 = lean_ctor_get(x_366, 0); +lean_inc(x_369); +lean_dec(x_366); +x_370 = l_Lake_Glob_decodeToml___closed__2; +x_371 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_371, 0, x_369); +lean_ctor_set(x_371, 1, x_370); +x_331 = x_371; +goto block_336; +} +case 3: +{ +lean_object* x_372; lean_object* x_373; lean_object* x_374; +x_372 = lean_ctor_get(x_366, 0); +lean_inc(x_372); +lean_dec(x_366); +x_373 = l_Lake_Glob_decodeToml___closed__2; +x_374 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_374, 0, x_372); +lean_ctor_set(x_374, 1, x_373); +x_331 = x_374; +goto block_336; +} +default: +{ +lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; +x_375 = lean_ctor_get(x_366, 0); +lean_inc(x_375); +if (lean_is_exclusive(x_366)) { + lean_ctor_release(x_366, 0); + lean_ctor_release(x_366, 1); + x_376 = x_366; +} else { + lean_dec_ref(x_366); + x_376 = lean_box(0); +} +x_377 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_376)) { + x_378 = lean_alloc_ctor(0, 2, 0); +} else { + x_378 = x_376; + lean_ctor_set_tag(x_378, 0); +} +lean_ctor_set(x_378, 0, x_375); +lean_ctor_set(x_378, 1, x_377); +x_331 = x_378; +goto block_336; +} +} +} +} +block_308: +{ +lean_object* x_266; lean_object* x_267; lean_object* x_275; lean_object* x_276; +x_266 = lean_box(0); +x_275 = l_Lake_Dependency_decodeToml___closed__2; +x_276 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_261, x_275, x_1); +if (lean_obj_tag(x_276) == 0) +{ +lean_object* x_277; lean_object* x_278; +x_277 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_278 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_278, 0, x_11); +lean_ctor_set(x_278, 1, x_277); +lean_ctor_set(x_278, 2, x_264); +lean_ctor_set(x_278, 3, x_148); +lean_ctor_set(x_278, 4, x_266); +x_3 = x_278; +x_4 = x_265; +goto block_8; +} +else +{ +lean_object* x_279; lean_object* x_280; +x_279 = lean_ctor_get(x_276, 0); +lean_inc(x_279); +lean_dec(x_276); +x_280 = lean_ctor_get(x_279, 1); +lean_inc(x_280); +lean_dec(x_279); +switch (lean_obj_tag(x_280)) { +case 0: +{ +uint8_t x_281; +x_281 = !lean_is_exclusive(x_280); +if (x_281 == 0) +{ +lean_object* x_282; lean_object* x_283; +x_282 = lean_ctor_get(x_280, 1); +lean_dec(x_282); +x_283 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_280, 1, x_283); +x_267 = x_280; +goto block_274; +} +else +{ +lean_object* x_284; lean_object* x_285; lean_object* x_286; +x_284 = lean_ctor_get(x_280, 0); +lean_inc(x_284); +lean_dec(x_280); +x_285 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_286 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_286, 0, x_284); +lean_ctor_set(x_286, 1, x_285); +x_267 = x_286; +goto block_274; +} +} +case 2: +{ +lean_object* x_287; lean_object* x_288; lean_object* x_289; +x_287 = lean_ctor_get(x_280, 0); +lean_inc(x_287); +lean_dec(x_280); +x_288 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_289 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_289, 0, x_287); +lean_ctor_set(x_289, 1, x_288); +x_267 = x_289; +goto block_274; +} +case 3: +{ +lean_object* x_290; lean_object* x_291; lean_object* x_292; +x_290 = lean_ctor_get(x_280, 0); +lean_inc(x_290); +lean_dec(x_280); +x_291 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_292 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_292, 0, x_290); +lean_ctor_set(x_292, 1, x_291); +x_267 = x_292; +goto block_274; +} +case 6: +{ +lean_object* x_293; lean_object* x_294; +x_293 = lean_ctor_get(x_280, 1); +lean_inc(x_293); +lean_dec(x_280); +x_294 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_293); +lean_dec(x_293); +if (lean_obj_tag(x_294) == 0) +{ +lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_295 = lean_ctor_get(x_294, 0); +lean_inc(x_295); +lean_dec(x_294); +x_296 = l_Array_append___rarg(x_265, x_295); +lean_dec(x_295); +x_297 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_298 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_298, 0, x_11); +lean_ctor_set(x_298, 1, x_297); +lean_ctor_set(x_298, 2, x_264); +lean_ctor_set(x_298, 3, x_148); +lean_ctor_set(x_298, 4, x_266); +x_3 = x_298; +x_4 = x_296; +goto block_8; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; +x_299 = lean_ctor_get(x_294, 0); +lean_inc(x_299); +lean_dec(x_294); +x_300 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_301 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_301, 0, x_11); +lean_ctor_set(x_301, 1, x_300); +lean_ctor_set(x_301, 2, x_264); +lean_ctor_set(x_301, 3, x_148); +lean_ctor_set(x_301, 4, x_299); +x_3 = x_301; +x_4 = x_265; +goto block_8; +} +} +default: +{ +uint8_t x_302; +x_302 = !lean_is_exclusive(x_280); +if (x_302 == 0) +{ +lean_object* x_303; lean_object* x_304; +x_303 = lean_ctor_get(x_280, 1); +lean_dec(x_303); +x_304 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_280, 0); +lean_ctor_set(x_280, 1, x_304); +x_267 = x_280; +goto block_274; +} +else +{ +lean_object* x_305; lean_object* x_306; lean_object* x_307; +x_305 = lean_ctor_get(x_280, 0); +lean_inc(x_305); +lean_dec(x_280); +x_306 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_307 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_307, 0, x_305); +lean_ctor_set(x_307, 1, x_306); +x_267 = x_307; +goto block_274; +} +} +} +} +block_274: +{ +lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; +x_268 = lean_box(0); +x_269 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_269, 0, x_267); +lean_ctor_set(x_269, 1, x_268); +x_270 = lean_array_mk(x_269); +x_271 = l_Array_append___rarg(x_265, x_270); +lean_dec(x_270); +x_272 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_273 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_273, 0, x_11); +lean_ctor_set(x_273, 1, x_272); +lean_ctor_set(x_273, 2, x_264); +lean_ctor_set(x_273, 3, x_148); +lean_ctor_set(x_273, 4, x_266); +x_3 = x_273; +x_4 = x_271; +goto block_8; +} +} +block_327: +{ +if (lean_obj_tag(x_309) == 0) +{ +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_311; +x_311 = lean_box(0); +x_264 = x_311; +x_265 = x_310; +goto block_308; +} +else +{ +uint8_t x_312; +x_312 = !lean_is_exclusive(x_12); +if (x_312 == 0) +{ +lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; +x_313 = lean_ctor_get(x_12, 0); +x_314 = l_Lake_Dependency_decodeToml___closed__3; +x_315 = lean_string_append(x_314, x_313); +lean_dec(x_313); +x_316 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_317 = lean_string_append(x_315, x_316); +lean_ctor_set(x_12, 0, x_317); +x_264 = x_12; +x_265 = x_310; +goto block_308; +} +else +{ +lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; +x_318 = lean_ctor_get(x_12, 0); +lean_inc(x_318); +lean_dec(x_12); +x_319 = l_Lake_Dependency_decodeToml___closed__3; +x_320 = lean_string_append(x_319, x_318); +lean_dec(x_318); +x_321 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_322 = lean_string_append(x_320, x_321); +x_323 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_323, 0, x_322); +x_264 = x_323; +x_265 = x_310; +goto block_308; +} +} +} +else +{ +uint8_t x_324; +lean_dec(x_12); +x_324 = !lean_is_exclusive(x_309); +if (x_324 == 0) +{ +x_264 = x_309; +x_265 = x_310; +goto block_308; +} +else +{ +lean_object* x_325; lean_object* x_326; +x_325 = lean_ctor_get(x_309, 0); +lean_inc(x_325); +lean_dec(x_309); +x_326 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_326, 0, x_325); +x_264 = x_326; +x_265 = x_310; +goto block_308; +} +} +} +block_336: +{ +lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; +x_332 = lean_box(0); +x_333 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_333, 0, x_331); +lean_ctor_set(x_333, 1, x_332); +x_334 = lean_array_mk(x_333); +x_335 = l_Array_append___rarg(x_149, x_334); +lean_dec(x_334); +x_309 = x_330; +x_310 = x_335; +goto block_327; +} +} +else +{ +lean_object* x_379; lean_object* x_380; +x_379 = lean_ctor_get(x_263, 0); +lean_inc(x_379); +lean_dec(x_263); +x_380 = lean_ctor_get(x_379, 1); +lean_inc(x_380); +lean_dec(x_379); +switch (lean_obj_tag(x_380)) { +case 0: +{ +lean_object* x_381; +x_381 = lean_ctor_get(x_380, 1); +lean_inc(x_381); +lean_dec(x_380); +x_150 = x_381; +x_151 = x_149; +goto block_253; +} +case 2: +{ +lean_object* x_382; lean_object* x_383; lean_object* x_384; +x_382 = lean_ctor_get(x_380, 0); +lean_inc(x_382); +lean_dec(x_380); +x_383 = l_Lake_Glob_decodeToml___closed__2; +x_384 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_384, 0, x_382); +lean_ctor_set(x_384, 1, x_383); +x_254 = x_384; +goto block_260; +} +case 3: +{ +lean_object* x_385; lean_object* x_386; lean_object* x_387; +x_385 = lean_ctor_get(x_380, 0); +lean_inc(x_385); +lean_dec(x_380); +x_386 = l_Lake_Glob_decodeToml___closed__2; +x_387 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_387, 0, x_385); +lean_ctor_set(x_387, 1, x_386); +x_254 = x_387; +goto block_260; +} +default: +{ +uint8_t x_388; +x_388 = !lean_is_exclusive(x_380); +if (x_388 == 0) +{ +lean_object* x_389; lean_object* x_390; +x_389 = lean_ctor_get(x_380, 1); +lean_dec(x_389); +x_390 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_380, 0); +lean_ctor_set(x_380, 1, x_390); +x_254 = x_380; +goto block_260; +} +else +{ +lean_object* x_391; lean_object* x_392; lean_object* x_393; +x_391 = lean_ctor_get(x_380, 0); +lean_inc(x_391); +lean_dec(x_380); +x_392 = l_Lake_Glob_decodeToml___closed__2; +x_393 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_393, 0, x_391); +lean_ctor_set(x_393, 1, x_392); +x_254 = x_393; +goto block_260; +} +} +} +} +block_253: +{ +lean_object* x_152; lean_object* x_153; lean_object* x_194; lean_object* x_195; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; +x_213 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_214 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_215 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_213, x_214, x_1); +x_216 = lean_box(0); +if (lean_obj_tag(x_215) == 0) +{ +x_194 = x_216; +x_195 = x_151; +goto block_212; +} +else +{ +uint8_t x_223; +x_223 = !lean_is_exclusive(x_215); +if (x_223 == 0) +{ +lean_object* x_224; lean_object* x_225; +x_224 = lean_ctor_get(x_215, 0); +x_225 = lean_ctor_get(x_224, 1); +lean_inc(x_225); +lean_dec(x_224); +switch (lean_obj_tag(x_225)) { +case 0: +{ +lean_object* x_226; +x_226 = lean_ctor_get(x_225, 1); +lean_inc(x_226); +lean_dec(x_225); +lean_ctor_set(x_215, 0, x_226); +x_194 = x_215; +x_195 = x_151; +goto block_212; +} +case 2: +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; +lean_free_object(x_215); +x_227 = lean_ctor_get(x_225, 0); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lake_Glob_decodeToml___closed__2; +x_229 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_229, 0, x_227); +lean_ctor_set(x_229, 1, x_228); +x_217 = x_229; +goto block_222; +} +case 3: +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_free_object(x_215); +x_230 = lean_ctor_get(x_225, 0); +lean_inc(x_230); +lean_dec(x_225); +x_231 = l_Lake_Glob_decodeToml___closed__2; +x_232 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_232, 0, x_230); +lean_ctor_set(x_232, 1, x_231); +x_217 = x_232; +goto block_222; +} +default: +{ +uint8_t x_233; +lean_free_object(x_215); +x_233 = !lean_is_exclusive(x_225); +if (x_233 == 0) +{ +lean_object* x_234; lean_object* x_235; +x_234 = lean_ctor_get(x_225, 1); +lean_dec(x_234); +x_235 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_225, 0); +lean_ctor_set(x_225, 1, x_235); +x_217 = x_225; +goto block_222; +} +else +{ +lean_object* x_236; lean_object* x_237; lean_object* x_238; +x_236 = lean_ctor_get(x_225, 0); +lean_inc(x_236); +lean_dec(x_225); +x_237 = l_Lake_Glob_decodeToml___closed__2; +x_238 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_238, 0, x_236); +lean_ctor_set(x_238, 1, x_237); +x_217 = x_238; +goto block_222; +} +} +} +} +else +{ +lean_object* x_239; lean_object* x_240; +x_239 = lean_ctor_get(x_215, 0); +lean_inc(x_239); +lean_dec(x_215); +x_240 = lean_ctor_get(x_239, 1); +lean_inc(x_240); +lean_dec(x_239); +switch (lean_obj_tag(x_240)) { +case 0: +{ +lean_object* x_241; lean_object* x_242; +x_241 = lean_ctor_get(x_240, 1); +lean_inc(x_241); +lean_dec(x_240); +x_242 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_242, 0, x_241); +x_194 = x_242; +x_195 = x_151; +goto block_212; +} +case 2: +{ +lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_243 = lean_ctor_get(x_240, 0); +lean_inc(x_243); +lean_dec(x_240); +x_244 = l_Lake_Glob_decodeToml___closed__2; +x_245 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_245, 0, x_243); +lean_ctor_set(x_245, 1, x_244); +x_217 = x_245; +goto block_222; +} +case 3: +{ +lean_object* x_246; lean_object* x_247; lean_object* x_248; +x_246 = lean_ctor_get(x_240, 0); +lean_inc(x_246); +lean_dec(x_240); +x_247 = l_Lake_Glob_decodeToml___closed__2; +x_248 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_248, 0, x_246); +lean_ctor_set(x_248, 1, x_247); +x_217 = x_248; +goto block_222; +} +default: +{ +lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; +x_249 = lean_ctor_get(x_240, 0); +lean_inc(x_249); +if (lean_is_exclusive(x_240)) { + lean_ctor_release(x_240, 0); + lean_ctor_release(x_240, 1); + x_250 = x_240; +} else { + lean_dec_ref(x_240); + x_250 = lean_box(0); +} +x_251 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_250)) { + x_252 = lean_alloc_ctor(0, 2, 0); +} else { + x_252 = x_250; + lean_ctor_set_tag(x_252, 0); +} +lean_ctor_set(x_252, 0, x_249); +lean_ctor_set(x_252, 1, x_251); +x_217 = x_252; +goto block_222; +} +} +} +} +block_193: +{ +lean_object* x_154; lean_object* x_155; lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_154 = lean_box(0); +x_162 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_163 = l_Lake_Dependency_decodeToml___closed__2; +x_164 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_162, x_163, x_1); +if (lean_obj_tag(x_164) == 0) +{ +lean_object* x_165; +x_165 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_165, 0, x_11); +lean_ctor_set(x_165, 1, x_150); +lean_ctor_set(x_165, 2, x_152); +lean_ctor_set(x_165, 3, x_148); +lean_ctor_set(x_165, 4, x_154); +x_3 = x_165; +x_4 = x_153; +goto block_8; +} +else +{ +lean_object* x_166; lean_object* x_167; +x_166 = lean_ctor_get(x_164, 0); +lean_inc(x_166); +lean_dec(x_164); +x_167 = lean_ctor_get(x_166, 1); +lean_inc(x_167); +lean_dec(x_166); +switch (lean_obj_tag(x_167)) { +case 0: +{ +uint8_t x_168; +x_168 = !lean_is_exclusive(x_167); +if (x_168 == 0) +{ +lean_object* x_169; lean_object* x_170; +x_169 = lean_ctor_get(x_167, 1); +lean_dec(x_169); +x_170 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_167, 1, x_170); +x_155 = x_167; +goto block_161; +} +else +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_171 = lean_ctor_get(x_167, 0); +lean_inc(x_171); +lean_dec(x_167); +x_172 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_173 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_173, 0, x_171); +lean_ctor_set(x_173, 1, x_172); +x_155 = x_173; +goto block_161; +} +} +case 2: +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; +x_174 = lean_ctor_get(x_167, 0); +lean_inc(x_174); +lean_dec(x_167); +x_175 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_176 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_176, 0, x_174); +lean_ctor_set(x_176, 1, x_175); +x_155 = x_176; +goto block_161; +} +case 3: +{ +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_167, 0); +lean_inc(x_177); +lean_dec(x_167); +x_178 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_179 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +x_155 = x_179; +goto block_161; +} +case 6: +{ +lean_object* x_180; lean_object* x_181; +x_180 = lean_ctor_get(x_167, 1); +lean_inc(x_180); +lean_dec(x_167); +x_181 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_180); +lean_dec(x_180); +if (lean_obj_tag(x_181) == 0) +{ +lean_object* x_182; lean_object* x_183; lean_object* x_184; +x_182 = lean_ctor_get(x_181, 0); +lean_inc(x_182); +lean_dec(x_181); +x_183 = l_Array_append___rarg(x_153, x_182); +lean_dec(x_182); +x_184 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_184, 0, x_11); +lean_ctor_set(x_184, 1, x_150); +lean_ctor_set(x_184, 2, x_152); +lean_ctor_set(x_184, 3, x_148); +lean_ctor_set(x_184, 4, x_154); +x_3 = x_184; +x_4 = x_183; +goto block_8; +} +else +{ +lean_object* x_185; lean_object* x_186; +x_185 = lean_ctor_get(x_181, 0); +lean_inc(x_185); +lean_dec(x_181); +x_186 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_186, 0, x_11); +lean_ctor_set(x_186, 1, x_150); +lean_ctor_set(x_186, 2, x_152); +lean_ctor_set(x_186, 3, x_148); +lean_ctor_set(x_186, 4, x_185); +x_3 = x_186; +x_4 = x_153; +goto block_8; +} +} +default: +{ +uint8_t x_187; +x_187 = !lean_is_exclusive(x_167); +if (x_187 == 0) +{ +lean_object* x_188; lean_object* x_189; +x_188 = lean_ctor_get(x_167, 1); +lean_dec(x_188); +x_189 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_167, 0); +lean_ctor_set(x_167, 1, x_189); +x_155 = x_167; +goto block_161; +} +else +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; +x_190 = lean_ctor_get(x_167, 0); +lean_inc(x_190); +lean_dec(x_167); +x_191 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_192 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_192, 0, x_190); +lean_ctor_set(x_192, 1, x_191); +x_155 = x_192; +goto block_161; +} +} +} +} +block_161: +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +x_156 = lean_box(0); +x_157 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +x_158 = lean_array_mk(x_157); +x_159 = l_Array_append___rarg(x_153, x_158); +lean_dec(x_158); +x_160 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_160, 0, x_11); +lean_ctor_set(x_160, 1, x_150); +lean_ctor_set(x_160, 2, x_152); +lean_ctor_set(x_160, 3, x_148); +lean_ctor_set(x_160, 4, x_154); +x_3 = x_160; +x_4 = x_159; +goto block_8; +} +} +block_212: +{ +if (lean_obj_tag(x_194) == 0) +{ +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_196; +x_196 = lean_box(0); +x_152 = x_196; +x_153 = x_195; +goto block_193; +} +else +{ +uint8_t x_197; +x_197 = !lean_is_exclusive(x_12); +if (x_197 == 0) +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; +x_198 = lean_ctor_get(x_12, 0); +x_199 = l_Lake_Dependency_decodeToml___closed__3; +x_200 = lean_string_append(x_199, x_198); +lean_dec(x_198); +x_201 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_202 = lean_string_append(x_200, x_201); +lean_ctor_set(x_12, 0, x_202); +x_152 = x_12; +x_153 = x_195; +goto block_193; +} +else +{ +lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; +x_203 = lean_ctor_get(x_12, 0); +lean_inc(x_203); +lean_dec(x_12); +x_204 = l_Lake_Dependency_decodeToml___closed__3; +x_205 = lean_string_append(x_204, x_203); +lean_dec(x_203); +x_206 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_207 = lean_string_append(x_205, x_206); +x_208 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_208, 0, x_207); +x_152 = x_208; +x_153 = x_195; +goto block_193; +} +} +} +else +{ +uint8_t x_209; +lean_dec(x_12); +x_209 = !lean_is_exclusive(x_194); +if (x_209 == 0) +{ +x_152 = x_194; +x_153 = x_195; +goto block_193; +} +else +{ +lean_object* x_210; lean_object* x_211; +x_210 = lean_ctor_get(x_194, 0); +lean_inc(x_210); +lean_dec(x_194); +x_211 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_211, 0, x_210); +x_152 = x_211; +x_153 = x_195; +goto block_193; +} +} +} +block_222: +{ +lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +x_218 = lean_box(0); +x_219 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +x_220 = lean_array_mk(x_219); +x_221 = l_Array_append___rarg(x_151, x_220); +lean_dec(x_220); +x_194 = x_216; +x_195 = x_221; +goto block_212; +} +} +block_260: +{ +lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; +x_255 = lean_box(0); +x_256 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_256, 0, x_254); +lean_ctor_set(x_256, 1, x_255); +x_257 = lean_array_mk(x_256); +x_258 = l_Array_append___rarg(x_149, x_257); +lean_dec(x_257); +x_259 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_150 = x_259; +x_151 = x_258; +goto block_253; +} +} +block_1173: +{ +if (lean_obj_tag(x_395) == 0) +{ +lean_object* x_397; lean_object* x_398; lean_object* x_399; +x_397 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_398 = l_Lake_Dependency_decodeToml___closed__6; +lean_inc(x_1); +x_399 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_398, x_1); +if (lean_obj_tag(x_399) == 0) +{ +lean_object* x_400; lean_object* x_401; lean_object* x_402; lean_object* x_403; +x_400 = l_Lake_Dependency_decodeToml___closed__8; +lean_inc(x_1); +x_401 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_400, x_1); +x_402 = lean_box(0); +if (lean_obj_tag(x_401) == 0) +{ +x_14 = x_402; +x_15 = x_396; +goto block_147; +} +else +{ +uint8_t x_409; +x_409 = !lean_is_exclusive(x_401); +if (x_409 == 0) +{ +lean_object* x_410; lean_object* x_411; +x_410 = lean_ctor_get(x_401, 0); +x_411 = lean_ctor_get(x_410, 1); +lean_inc(x_411); +lean_dec(x_410); +switch (lean_obj_tag(x_411)) { +case 0: +{ +uint8_t x_412; +lean_free_object(x_401); +x_412 = !lean_is_exclusive(x_411); +if (x_412 == 0) +{ +lean_object* x_413; lean_object* x_414; +x_413 = lean_ctor_get(x_411, 1); +lean_dec(x_413); +x_414 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_411, 1, x_414); +x_403 = x_411; +goto block_408; +} +else +{ +lean_object* x_415; lean_object* x_416; lean_object* x_417; +x_415 = lean_ctor_get(x_411, 0); +lean_inc(x_415); +lean_dec(x_411); +x_416 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_417 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_417, 0, x_415); +lean_ctor_set(x_417, 1, x_416); +x_403 = x_417; +goto block_408; +} +} +case 2: +{ +lean_object* x_418; lean_object* x_419; lean_object* x_420; +lean_free_object(x_401); +x_418 = lean_ctor_get(x_411, 0); +lean_inc(x_418); +lean_dec(x_411); +x_419 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_420 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_420, 0, x_418); +lean_ctor_set(x_420, 1, x_419); +x_403 = x_420; +goto block_408; +} +case 3: +{ +lean_object* x_421; lean_object* x_422; lean_object* x_423; +lean_free_object(x_401); +x_421 = lean_ctor_get(x_411, 0); +lean_inc(x_421); +lean_dec(x_411); +x_422 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_423 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_423, 0, x_421); +lean_ctor_set(x_423, 1, x_422); +x_403 = x_423; +goto block_408; +} +case 6: +{ +lean_object* x_424; lean_object* x_425; lean_object* x_426; +x_424 = lean_ctor_get(x_411, 0); +lean_inc(x_424); +x_425 = lean_ctor_get(x_411, 1); +lean_inc(x_425); +lean_dec(x_411); +x_426 = l_Lake_DependencySrc_decodeToml(x_425, x_424); +if (lean_obj_tag(x_426) == 0) +{ +lean_object* x_427; lean_object* x_428; +lean_free_object(x_401); +x_427 = lean_ctor_get(x_426, 0); +lean_inc(x_427); +lean_dec(x_426); +x_428 = l_Array_append___rarg(x_396, x_427); +lean_dec(x_427); +x_14 = x_402; +x_15 = x_428; +goto block_147; +} +else +{ +lean_object* x_429; +x_429 = lean_ctor_get(x_426, 0); +lean_inc(x_429); +lean_dec(x_426); +lean_ctor_set(x_401, 0, x_429); +x_14 = x_401; +x_15 = x_396; +goto block_147; +} +} +default: +{ +uint8_t x_430; +lean_free_object(x_401); +x_430 = !lean_is_exclusive(x_411); +if (x_430 == 0) +{ +lean_object* x_431; lean_object* x_432; +x_431 = lean_ctor_get(x_411, 1); +lean_dec(x_431); +x_432 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_411, 0); +lean_ctor_set(x_411, 1, x_432); +x_403 = x_411; +goto block_408; +} +else +{ +lean_object* x_433; lean_object* x_434; lean_object* x_435; +x_433 = lean_ctor_get(x_411, 0); +lean_inc(x_433); +lean_dec(x_411); +x_434 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_435 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_435, 0, x_433); +lean_ctor_set(x_435, 1, x_434); +x_403 = x_435; +goto block_408; +} +} +} +} +else +{ +lean_object* x_436; lean_object* x_437; +x_436 = lean_ctor_get(x_401, 0); +lean_inc(x_436); +lean_dec(x_401); +x_437 = lean_ctor_get(x_436, 1); +lean_inc(x_437); +lean_dec(x_436); +switch (lean_obj_tag(x_437)) { +case 0: +{ +lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; +x_438 = lean_ctor_get(x_437, 0); +lean_inc(x_438); +if (lean_is_exclusive(x_437)) { + lean_ctor_release(x_437, 0); + lean_ctor_release(x_437, 1); + x_439 = x_437; +} else { + lean_dec_ref(x_437); + x_439 = lean_box(0); +} +x_440 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_439)) { + x_441 = lean_alloc_ctor(0, 2, 0); +} else { + x_441 = x_439; +} +lean_ctor_set(x_441, 0, x_438); +lean_ctor_set(x_441, 1, x_440); +x_403 = x_441; +goto block_408; +} +case 2: +{ +lean_object* x_442; lean_object* x_443; lean_object* x_444; +x_442 = lean_ctor_get(x_437, 0); +lean_inc(x_442); +lean_dec(x_437); +x_443 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_444 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_444, 0, x_442); +lean_ctor_set(x_444, 1, x_443); +x_403 = x_444; +goto block_408; +} +case 3: +{ +lean_object* x_445; lean_object* x_446; lean_object* x_447; +x_445 = lean_ctor_get(x_437, 0); +lean_inc(x_445); +lean_dec(x_437); +x_446 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_447 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_447, 0, x_445); +lean_ctor_set(x_447, 1, x_446); +x_403 = x_447; +goto block_408; +} +case 6: +{ +lean_object* x_448; lean_object* x_449; lean_object* x_450; +x_448 = lean_ctor_get(x_437, 0); +lean_inc(x_448); +x_449 = lean_ctor_get(x_437, 1); +lean_inc(x_449); +lean_dec(x_437); +x_450 = l_Lake_DependencySrc_decodeToml(x_449, x_448); +if (lean_obj_tag(x_450) == 0) +{ +lean_object* x_451; lean_object* x_452; +x_451 = lean_ctor_get(x_450, 0); +lean_inc(x_451); +lean_dec(x_450); +x_452 = l_Array_append___rarg(x_396, x_451); +lean_dec(x_451); +x_14 = x_402; +x_15 = x_452; +goto block_147; +} +else +{ +lean_object* x_453; lean_object* x_454; +x_453 = lean_ctor_get(x_450, 0); +lean_inc(x_453); +lean_dec(x_450); +x_454 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_454, 0, x_453); +x_14 = x_454; +x_15 = x_396; +goto block_147; +} +} +default: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("options", 7, 7); -return x_1; +lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; +x_455 = lean_ctor_get(x_437, 0); +lean_inc(x_455); +if (lean_is_exclusive(x_437)) { + lean_ctor_release(x_437, 0); + lean_ctor_release(x_437, 1); + x_456 = x_437; +} else { + lean_dec_ref(x_437); + x_456 = lean_box(0); } +x_457 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_456)) { + x_458 = lean_alloc_ctor(0, 2, 0); +} else { + x_458 = x_456; + lean_ctor_set_tag(x_458, 0); } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_Dependency_decodeToml___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_ctor_set(x_458, 0, x_455); +lean_ctor_set(x_458, 1, x_457); +x_403 = x_458; +goto block_408; } } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("git#", 4, 4); -return x_1; } } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__4() { -_start: +block_408: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("scope", 5, 5); -return x_1; +lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; +x_404 = lean_box(0); +x_405 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_405, 0, x_403); +lean_ctor_set(x_405, 1, x_404); +x_406 = lean_array_mk(x_405); +x_407 = l_Array_append___rarg(x_396, x_406); +lean_dec(x_406); +x_14 = x_402; +x_15 = x_407; +goto block_147; } } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_Dependency_decodeToml___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_459; lean_object* x_460; lean_object* x_461; +x_459 = lean_ctor_get(x_399, 0); +lean_inc(x_459); +if (lean_is_exclusive(x_399)) { + lean_ctor_release(x_399, 0); + x_460 = x_399; +} else { + lean_dec_ref(x_399); + x_460 = lean_box(0); } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__6() { -_start: +x_461 = lean_ctor_get(x_459, 1); +lean_inc(x_461); +lean_dec(x_459); +switch (lean_obj_tag(x_461)) { +case 0: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_DependencySrc_decodeToml___closed__14; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_462; lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; +x_462 = lean_ctor_get(x_461, 1); +lean_inc(x_462); +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + lean_ctor_release(x_461, 1); + x_463 = x_461; +} else { + lean_dec_ref(x_461); + x_463 = lean_box(0); } +x_464 = l_Lake_DependencySrc_decodeToml___closed__2; +lean_inc(x_1); +x_465 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_464, x_1); +x_466 = lean_box(0); +if (lean_obj_tag(x_465) == 0) +{ +lean_object* x_475; lean_object* x_476; +lean_dec(x_463); +lean_dec(x_460); +lean_inc(x_12); +x_475 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_475, 0, x_462); +lean_ctor_set(x_475, 1, x_12); +lean_ctor_set(x_475, 2, x_466); +x_476 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_476, 0, x_475); +x_14 = x_476; +x_15 = x_396; +goto block_147; } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__7() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("source", 6, 6); -return x_1; +uint8_t x_477; +x_477 = !lean_is_exclusive(x_465); +if (x_477 == 0) +{ +lean_object* x_478; lean_object* x_479; +x_478 = lean_ctor_get(x_465, 0); +x_479 = lean_ctor_get(x_478, 1); +lean_inc(x_479); +lean_dec(x_478); +switch (lean_obj_tag(x_479)) { +case 0: +{ +lean_object* x_480; lean_object* x_481; lean_object* x_482; +lean_dec(x_463); +lean_dec(x_460); +x_480 = lean_ctor_get(x_479, 1); +lean_inc(x_480); +lean_dec(x_479); +lean_ctor_set(x_465, 0, x_480); +lean_inc(x_12); +x_481 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_481, 0, x_462); +lean_ctor_set(x_481, 1, x_12); +lean_ctor_set(x_481, 2, x_465); +x_482 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_482, 0, x_481); +x_14 = x_482; +x_15 = x_396; +goto block_147; } +case 2: +{ +lean_object* x_483; lean_object* x_484; lean_object* x_485; +lean_free_object(x_465); +x_483 = lean_ctor_get(x_479, 0); +lean_inc(x_483); +lean_dec(x_479); +x_484 = l_Lake_Glob_decodeToml___closed__2; +x_485 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_485, 0, x_483); +lean_ctor_set(x_485, 1, x_484); +x_467 = x_485; +goto block_474; } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__8() { -_start: +case 3: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_Dependency_decodeToml___closed__7; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_486; lean_object* x_487; lean_object* x_488; +lean_free_object(x_465); +x_486 = lean_ctor_get(x_479, 0); +lean_inc(x_486); +lean_dec(x_479); +x_487 = l_Lake_Glob_decodeToml___closed__2; +x_488 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_488, 0, x_486); +lean_ctor_set(x_488, 1, x_487); +x_467 = x_488; +goto block_474; } +default: +{ +uint8_t x_489; +lean_free_object(x_465); +x_489 = !lean_is_exclusive(x_479); +if (x_489 == 0) +{ +lean_object* x_490; lean_object* x_491; +x_490 = lean_ctor_get(x_479, 1); +lean_dec(x_490); +x_491 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_479, 0); +lean_ctor_set(x_479, 1, x_491); +x_467 = x_479; +goto block_474; } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__9() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("expected string or table", 24, 24); -return x_1; +lean_object* x_492; lean_object* x_493; lean_object* x_494; +x_492 = lean_ctor_get(x_479, 0); +lean_inc(x_492); +lean_dec(x_479); +x_493 = l_Lake_Glob_decodeToml___closed__2; +x_494 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_494, 0, x_492); +lean_ctor_set(x_494, 1, x_493); +x_467 = x_494; +goto block_474; } } -static lean_object* _init_l_Lake_Dependency_decodeToml___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lake_DependencySrc_decodeToml___closed__13; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; } } -LEAN_EXPORT lean_object* l_Lake_Dependency_decodeToml(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_9; lean_object* x_10; lean_object* x_906; lean_object* x_907; -x_906 = l_Lake_LeanOption_decodeToml___closed__10; -lean_inc(x_1); -x_907 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_1, x_906, x_2); -if (lean_obj_tag(x_907) == 0) -{ -lean_object* x_908; lean_object* x_909; lean_object* x_910; lean_object* x_911; -x_908 = lean_ctor_get(x_907, 0); -lean_inc(x_908); -lean_dec(x_907); -x_909 = l_Lake_LeanOption_decodeToml___closed__3; -x_910 = l_Array_append___rarg(x_909, x_908); -lean_dec(x_908); -x_911 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_9 = x_911; -x_10 = x_910; -goto block_905; +lean_object* x_495; lean_object* x_496; +x_495 = lean_ctor_get(x_465, 0); +lean_inc(x_495); +lean_dec(x_465); +x_496 = lean_ctor_get(x_495, 1); +lean_inc(x_496); +lean_dec(x_495); +switch (lean_obj_tag(x_496)) { +case 0: +{ +lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; +lean_dec(x_463); +lean_dec(x_460); +x_497 = lean_ctor_get(x_496, 1); +lean_inc(x_497); +lean_dec(x_496); +x_498 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_498, 0, x_497); +lean_inc(x_12); +x_499 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_499, 0, x_462); +lean_ctor_set(x_499, 1, x_12); +lean_ctor_set(x_499, 2, x_498); +x_500 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_500, 0, x_499); +x_14 = x_500; +x_15 = x_396; +goto block_147; } -else +case 2: { -lean_object* x_912; lean_object* x_913; -x_912 = lean_ctor_get(x_907, 0); -lean_inc(x_912); -lean_dec(x_907); -x_913 = l_Lake_LeanOption_decodeToml___closed__3; -x_9 = x_912; -x_10 = x_913; -goto block_905; +lean_object* x_501; lean_object* x_502; lean_object* x_503; +x_501 = lean_ctor_get(x_496, 0); +lean_inc(x_501); +lean_dec(x_496); +x_502 = l_Lake_Glob_decodeToml___closed__2; +x_503 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_503, 0, x_501); +lean_ctor_set(x_503, 1, x_502); +x_467 = x_503; +goto block_474; } -block_8: +case 3: { -uint8_t x_5; -x_5 = l_Array_isEmpty___rarg(x_4); -if (x_5 == 0) +lean_object* x_504; lean_object* x_505; lean_object* x_506; +x_504 = lean_ctor_get(x_496, 0); +lean_inc(x_504); +lean_dec(x_496); +x_505 = l_Lake_Glob_decodeToml___closed__2; +x_506 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_506, 0, x_504); +lean_ctor_set(x_506, 1, x_505); +x_467 = x_506; +goto block_474; +} +default: { -lean_object* x_6; -lean_dec(x_3); -x_6 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_6, 0, x_4); -return x_6; +lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; +x_507 = lean_ctor_get(x_496, 0); +lean_inc(x_507); +if (lean_is_exclusive(x_496)) { + lean_ctor_release(x_496, 0); + lean_ctor_release(x_496, 1); + x_508 = x_496; +} else { + lean_dec_ref(x_496); + x_508 = lean_box(0); } -else +x_509 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_508)) { + x_510 = lean_alloc_ctor(0, 2, 0); +} else { + x_510 = x_508; + lean_ctor_set_tag(x_510, 0); +} +lean_ctor_set(x_510, 0, x_507); +lean_ctor_set(x_510, 1, x_509); +x_467 = x_510; +goto block_474; +} +} +} +} +block_474: { -lean_object* x_7; -lean_dec(x_4); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_3); -return x_7; +lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; +x_468 = lean_box(0); +if (lean_is_scalar(x_463)) { + x_469 = lean_alloc_ctor(1, 2, 0); +} else { + x_469 = x_463; + lean_ctor_set_tag(x_469, 1); +} +lean_ctor_set(x_469, 0, x_467); +lean_ctor_set(x_469, 1, x_468); +x_470 = lean_array_mk(x_469); +x_471 = l_Array_append___rarg(x_396, x_470); +lean_dec(x_470); +lean_inc(x_12); +x_472 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_472, 0, x_462); +lean_ctor_set(x_472, 1, x_12); +lean_ctor_set(x_472, 2, x_466); +if (lean_is_scalar(x_460)) { + x_473 = lean_alloc_ctor(1, 1, 0); +} else { + x_473 = x_460; +} +lean_ctor_set(x_473, 0, x_472); +x_14 = x_473; +x_15 = x_471; +goto block_147; } } -block_905: +case 2: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; -x_11 = l_Lake_stringToLegalOrSimpleName(x_9); -x_850 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_851 = l_Lake_DependencySrc_decodeToml___closed__4; +lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; +lean_dec(x_460); +x_511 = lean_ctor_get(x_461, 0); +lean_inc(x_511); +lean_dec(x_461); +x_512 = l_Lake_Dependency_decodeToml___closed__9; +x_513 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_513, 0, x_511); +lean_ctor_set(x_513, 1, x_512); +x_514 = lean_array_push(x_396, x_513); +x_515 = lean_box(0); +x_148 = x_515; +x_149 = x_514; +goto block_394; +} +case 3: +{ +lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; +lean_dec(x_460); +x_516 = lean_ctor_get(x_461, 0); +lean_inc(x_516); +lean_dec(x_461); +x_517 = l_Lake_Dependency_decodeToml___closed__9; +x_518 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_518, 0, x_516); +lean_ctor_set(x_518, 1, x_517); +x_519 = lean_array_push(x_396, x_518); +x_520 = lean_box(0); +x_148 = x_520; +x_149 = x_519; +goto block_394; +} +case 6: +{ +lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_775; lean_object* x_776; +x_521 = lean_ctor_get(x_461, 0); +lean_inc(x_521); +x_522 = lean_ctor_get(x_461, 1); +lean_inc(x_522); +if (lean_is_exclusive(x_461)) { + lean_ctor_release(x_461, 0); + lean_ctor_release(x_461, 1); + x_523 = x_461; +} else { + lean_dec_ref(x_461); + x_523 = lean_box(0); +} +x_775 = l_Lake_DependencySrc_decodeToml___closed__18; +lean_inc(x_522); +x_776 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_522, x_775, x_521); +if (lean_obj_tag(x_776) == 0) +{ +lean_object* x_777; lean_object* x_778; lean_object* x_779; +x_777 = lean_ctor_get(x_776, 0); +lean_inc(x_777); +lean_dec(x_776); +x_778 = l_Array_append___rarg(x_396, x_777); +lean_dec(x_777); +x_779 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_524 = x_779; +x_525 = x_778; +goto block_774; +} +else +{ +lean_object* x_780; +x_780 = lean_ctor_get(x_776, 0); +lean_inc(x_780); +lean_dec(x_776); +x_524 = x_780; +x_525 = x_396; +goto block_774; +} +block_774: +{ +lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; +x_526 = l_Lake_DependencySrc_decodeToml___closed__2; +x_527 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_526, x_522); +x_528 = lean_box(0); +if (lean_obj_tag(x_527) == 0) +{ +lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_627; lean_object* x_634; lean_object* x_635; +lean_dec(x_523); +lean_dec(x_460); +x_537 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_537, 0, x_524); +lean_ctor_set(x_537, 1, x_12); +lean_ctor_set(x_537, 2, x_528); +x_538 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_538, 0, x_537); +x_634 = l_Lake_Dependency_decodeToml___closed__5; lean_inc(x_1); -x_852 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_850, x_851, x_1); -x_853 = lean_box(0); -if (lean_obj_tag(x_852) == 0) +x_635 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_634, x_1); +if (lean_obj_tag(x_635) == 0) { -x_12 = x_853; -x_13 = x_10; -goto block_849; +lean_object* x_636; lean_object* x_637; lean_object* x_681; lean_object* x_682; lean_object* x_687; lean_object* x_688; lean_object* x_689; +x_687 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_688 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_687, x_1); +if (lean_obj_tag(x_688) == 0) +{ +x_636 = x_528; +x_637 = x_525; +goto block_680; } else { -uint8_t x_854; -x_854 = !lean_is_exclusive(x_852); -if (x_854 == 0) +uint8_t x_695; +x_695 = !lean_is_exclusive(x_688); +if (x_695 == 0) { -lean_object* x_855; lean_object* x_856; -x_855 = lean_ctor_get(x_852, 0); -x_856 = lean_ctor_get(x_855, 1); -lean_inc(x_856); -lean_dec(x_855); -switch (lean_obj_tag(x_856)) { +lean_object* x_696; lean_object* x_697; +x_696 = lean_ctor_get(x_688, 0); +x_697 = lean_ctor_get(x_696, 1); +lean_inc(x_697); +lean_dec(x_696); +switch (lean_obj_tag(x_697)) { case 0: { -lean_object* x_857; -x_857 = lean_ctor_get(x_856, 1); -lean_inc(x_857); -lean_dec(x_856); -lean_ctor_set(x_852, 0, x_857); -x_12 = x_852; -x_13 = x_10; -goto block_849; +lean_object* x_698; +x_698 = lean_ctor_get(x_697, 1); +lean_inc(x_698); +lean_dec(x_697); +lean_ctor_set(x_688, 0, x_698); +x_681 = x_688; +x_682 = x_525; +goto block_686; } case 2: { -lean_object* x_858; lean_object* x_859; lean_object* x_860; lean_object* x_861; lean_object* x_862; lean_object* x_863; -lean_free_object(x_852); -x_858 = lean_ctor_get(x_856, 0); -lean_inc(x_858); -lean_dec(x_856); -x_859 = l_Lake_Glob_decodeToml___closed__2; -x_860 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_860, 0, x_858); -lean_ctor_set(x_860, 1, x_859); -x_861 = lean_unsigned_to_nat(1u); -x_862 = lean_mk_array(x_861, x_860); -x_863 = l_Array_append___rarg(x_10, x_862); -lean_dec(x_862); -x_12 = x_853; -x_13 = x_863; -goto block_849; +lean_object* x_699; lean_object* x_700; lean_object* x_701; +lean_free_object(x_688); +x_699 = lean_ctor_get(x_697, 0); +lean_inc(x_699); +lean_dec(x_697); +x_700 = l_Lake_Glob_decodeToml___closed__2; +x_701 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_701, 0, x_699); +lean_ctor_set(x_701, 1, x_700); +x_689 = x_701; +goto block_694; } case 3: { -lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; lean_object* x_869; -lean_free_object(x_852); -x_864 = lean_ctor_get(x_856, 0); -lean_inc(x_864); -lean_dec(x_856); -x_865 = l_Lake_Glob_decodeToml___closed__2; -x_866 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_866, 0, x_864); -lean_ctor_set(x_866, 1, x_865); -x_867 = lean_unsigned_to_nat(1u); -x_868 = lean_mk_array(x_867, x_866); -x_869 = l_Array_append___rarg(x_10, x_868); -lean_dec(x_868); -x_12 = x_853; -x_13 = x_869; -goto block_849; +lean_object* x_702; lean_object* x_703; lean_object* x_704; +lean_free_object(x_688); +x_702 = lean_ctor_get(x_697, 0); +lean_inc(x_702); +lean_dec(x_697); +x_703 = l_Lake_Glob_decodeToml___closed__2; +x_704 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_704, 0, x_702); +lean_ctor_set(x_704, 1, x_703); +x_689 = x_704; +goto block_694; } default: { -uint8_t x_870; -lean_free_object(x_852); -x_870 = !lean_is_exclusive(x_856); -if (x_870 == 0) +uint8_t x_705; +lean_free_object(x_688); +x_705 = !lean_is_exclusive(x_697); +if (x_705 == 0) { -lean_object* x_871; lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; -x_871 = lean_ctor_get(x_856, 1); -lean_dec(x_871); -x_872 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_856, 0); -lean_ctor_set(x_856, 1, x_872); -x_873 = lean_unsigned_to_nat(1u); -x_874 = lean_mk_array(x_873, x_856); -x_875 = l_Array_append___rarg(x_10, x_874); -lean_dec(x_874); -x_12 = x_853; -x_13 = x_875; -goto block_849; -} -else -{ -lean_object* x_876; lean_object* x_877; lean_object* x_878; lean_object* x_879; lean_object* x_880; lean_object* x_881; -x_876 = lean_ctor_get(x_856, 0); -lean_inc(x_876); -lean_dec(x_856); -x_877 = l_Lake_Glob_decodeToml___closed__2; -x_878 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_878, 0, x_876); -lean_ctor_set(x_878, 1, x_877); -x_879 = lean_unsigned_to_nat(1u); -x_880 = lean_mk_array(x_879, x_878); -x_881 = l_Array_append___rarg(x_10, x_880); -lean_dec(x_880); -x_12 = x_853; -x_13 = x_881; -goto block_849; +lean_object* x_706; lean_object* x_707; +x_706 = lean_ctor_get(x_697, 1); +lean_dec(x_706); +x_707 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_697, 0); +lean_ctor_set(x_697, 1, x_707); +x_689 = x_697; +goto block_694; +} +else +{ +lean_object* x_708; lean_object* x_709; lean_object* x_710; +x_708 = lean_ctor_get(x_697, 0); +lean_inc(x_708); +lean_dec(x_697); +x_709 = l_Lake_Glob_decodeToml___closed__2; +x_710 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_710, 0, x_708); +lean_ctor_set(x_710, 1, x_709); +x_689 = x_710; +goto block_694; } } } } else { -lean_object* x_882; lean_object* x_883; -x_882 = lean_ctor_get(x_852, 0); -lean_inc(x_882); -lean_dec(x_852); -x_883 = lean_ctor_get(x_882, 1); -lean_inc(x_883); -lean_dec(x_882); -switch (lean_obj_tag(x_883)) { +lean_object* x_711; lean_object* x_712; +x_711 = lean_ctor_get(x_688, 0); +lean_inc(x_711); +lean_dec(x_688); +x_712 = lean_ctor_get(x_711, 1); +lean_inc(x_712); +lean_dec(x_711); +switch (lean_obj_tag(x_712)) { case 0: { -lean_object* x_884; lean_object* x_885; -x_884 = lean_ctor_get(x_883, 1); -lean_inc(x_884); -lean_dec(x_883); -x_885 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_885, 0, x_884); -x_12 = x_885; -x_13 = x_10; -goto block_849; +lean_object* x_713; lean_object* x_714; +x_713 = lean_ctor_get(x_712, 1); +lean_inc(x_713); +lean_dec(x_712); +x_714 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_714, 0, x_713); +x_681 = x_714; +x_682 = x_525; +goto block_686; } case 2: { -lean_object* x_886; lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; -x_886 = lean_ctor_get(x_883, 0); -lean_inc(x_886); -lean_dec(x_883); -x_887 = l_Lake_Glob_decodeToml___closed__2; -x_888 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_888, 0, x_886); -lean_ctor_set(x_888, 1, x_887); -x_889 = lean_unsigned_to_nat(1u); -x_890 = lean_mk_array(x_889, x_888); -x_891 = l_Array_append___rarg(x_10, x_890); -lean_dec(x_890); -x_12 = x_853; -x_13 = x_891; -goto block_849; +lean_object* x_715; lean_object* x_716; lean_object* x_717; +x_715 = lean_ctor_get(x_712, 0); +lean_inc(x_715); +lean_dec(x_712); +x_716 = l_Lake_Glob_decodeToml___closed__2; +x_717 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_717, 0, x_715); +lean_ctor_set(x_717, 1, x_716); +x_689 = x_717; +goto block_694; } case 3: { -lean_object* x_892; lean_object* x_893; lean_object* x_894; lean_object* x_895; lean_object* x_896; lean_object* x_897; -x_892 = lean_ctor_get(x_883, 0); -lean_inc(x_892); -lean_dec(x_883); -x_893 = l_Lake_Glob_decodeToml___closed__2; -x_894 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_894, 0, x_892); -lean_ctor_set(x_894, 1, x_893); -x_895 = lean_unsigned_to_nat(1u); -x_896 = lean_mk_array(x_895, x_894); -x_897 = l_Array_append___rarg(x_10, x_896); -lean_dec(x_896); -x_12 = x_853; -x_13 = x_897; -goto block_849; +lean_object* x_718; lean_object* x_719; lean_object* x_720; +x_718 = lean_ctor_get(x_712, 0); +lean_inc(x_718); +lean_dec(x_712); +x_719 = l_Lake_Glob_decodeToml___closed__2; +x_720 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_720, 0, x_718); +lean_ctor_set(x_720, 1, x_719); +x_689 = x_720; +goto block_694; } default: { -lean_object* x_898; lean_object* x_899; lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; -x_898 = lean_ctor_get(x_883, 0); -lean_inc(x_898); -if (lean_is_exclusive(x_883)) { - lean_ctor_release(x_883, 0); - lean_ctor_release(x_883, 1); - x_899 = x_883; +lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; +x_721 = lean_ctor_get(x_712, 0); +lean_inc(x_721); +if (lean_is_exclusive(x_712)) { + lean_ctor_release(x_712, 0); + lean_ctor_release(x_712, 1); + x_722 = x_712; } else { - lean_dec_ref(x_883); - x_899 = lean_box(0); + lean_dec_ref(x_712); + x_722 = lean_box(0); } -x_900 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_899)) { - x_901 = lean_alloc_ctor(0, 2, 0); +x_723 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_722)) { + x_724 = lean_alloc_ctor(0, 2, 0); } else { - x_901 = x_899; - lean_ctor_set_tag(x_901, 0); + x_724 = x_722; + lean_ctor_set_tag(x_724, 0); } -lean_ctor_set(x_901, 0, x_898); -lean_ctor_set(x_901, 1, x_900); -x_902 = lean_unsigned_to_nat(1u); -x_903 = lean_mk_array(x_902, x_901); -x_904 = l_Array_append___rarg(x_10, x_903); -lean_dec(x_903); -x_12 = x_853; -x_13 = x_904; -goto block_849; +lean_ctor_set(x_724, 0, x_721); +lean_ctor_set(x_724, 1, x_723); +x_689 = x_724; +goto block_694; } } } } -block_849: +block_680: { -lean_object* x_14; lean_object* x_15; lean_object* x_189; lean_object* x_190; lean_object* x_514; lean_object* x_515; lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; -x_794 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_795 = l_Lake_Dependency_decodeToml___closed__10; -lean_inc(x_1); -x_796 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_794, x_795, x_1); -x_797 = lean_box(0); -if (lean_obj_tag(x_796) == 0) +lean_object* x_638; lean_object* x_639; lean_object* x_647; lean_object* x_648; +x_638 = lean_box(0); +x_647 = l_Lake_Dependency_decodeToml___closed__2; +x_648 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_647, x_1); +if (lean_obj_tag(x_648) == 0) { -x_514 = x_797; -x_515 = x_13; -goto block_793; +lean_object* x_649; lean_object* x_650; +x_649 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_650 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_650, 0, x_11); +lean_ctor_set(x_650, 1, x_649); +lean_ctor_set(x_650, 2, x_636); +lean_ctor_set(x_650, 3, x_538); +lean_ctor_set(x_650, 4, x_638); +x_3 = x_650; +x_4 = x_637; +goto block_8; } else { -uint8_t x_798; -x_798 = !lean_is_exclusive(x_796); -if (x_798 == 0) -{ -lean_object* x_799; lean_object* x_800; -x_799 = lean_ctor_get(x_796, 0); -x_800 = lean_ctor_get(x_799, 1); -lean_inc(x_800); -lean_dec(x_799); -switch (lean_obj_tag(x_800)) { +lean_object* x_651; lean_object* x_652; +x_651 = lean_ctor_get(x_648, 0); +lean_inc(x_651); +lean_dec(x_648); +x_652 = lean_ctor_get(x_651, 1); +lean_inc(x_652); +lean_dec(x_651); +switch (lean_obj_tag(x_652)) { case 0: { -lean_object* x_801; -x_801 = lean_ctor_get(x_800, 1); -lean_inc(x_801); -lean_dec(x_800); -lean_ctor_set(x_796, 0, x_801); -x_514 = x_796; -x_515 = x_13; -goto block_793; +uint8_t x_653; +x_653 = !lean_is_exclusive(x_652); +if (x_653 == 0) +{ +lean_object* x_654; lean_object* x_655; +x_654 = lean_ctor_get(x_652, 1); +lean_dec(x_654); +x_655 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_652, 1, x_655); +x_639 = x_652; +goto block_646; +} +else +{ +lean_object* x_656; lean_object* x_657; lean_object* x_658; +x_656 = lean_ctor_get(x_652, 0); +lean_inc(x_656); +lean_dec(x_652); +x_657 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_658 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_658, 0, x_656); +lean_ctor_set(x_658, 1, x_657); +x_639 = x_658; +goto block_646; +} } case 2: { -lean_object* x_802; lean_object* x_803; lean_object* x_804; lean_object* x_805; lean_object* x_806; lean_object* x_807; -lean_free_object(x_796); -x_802 = lean_ctor_get(x_800, 0); -lean_inc(x_802); -lean_dec(x_800); -x_803 = l_Lake_Glob_decodeToml___closed__2; -x_804 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_804, 0, x_802); -lean_ctor_set(x_804, 1, x_803); -x_805 = lean_unsigned_to_nat(1u); -x_806 = lean_mk_array(x_805, x_804); -x_807 = l_Array_append___rarg(x_13, x_806); -lean_dec(x_806); -x_514 = x_797; -x_515 = x_807; -goto block_793; +lean_object* x_659; lean_object* x_660; lean_object* x_661; +x_659 = lean_ctor_get(x_652, 0); +lean_inc(x_659); +lean_dec(x_652); +x_660 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_661 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_661, 0, x_659); +lean_ctor_set(x_661, 1, x_660); +x_639 = x_661; +goto block_646; } case 3: { -lean_object* x_808; lean_object* x_809; lean_object* x_810; lean_object* x_811; lean_object* x_812; lean_object* x_813; -lean_free_object(x_796); -x_808 = lean_ctor_get(x_800, 0); -lean_inc(x_808); -lean_dec(x_800); -x_809 = l_Lake_Glob_decodeToml___closed__2; -x_810 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_810, 0, x_808); -lean_ctor_set(x_810, 1, x_809); -x_811 = lean_unsigned_to_nat(1u); -x_812 = lean_mk_array(x_811, x_810); -x_813 = l_Array_append___rarg(x_13, x_812); -lean_dec(x_812); -x_514 = x_797; -x_515 = x_813; -goto block_793; +lean_object* x_662; lean_object* x_663; lean_object* x_664; +x_662 = lean_ctor_get(x_652, 0); +lean_inc(x_662); +lean_dec(x_652); +x_663 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_664 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_664, 0, x_662); +lean_ctor_set(x_664, 1, x_663); +x_639 = x_664; +goto block_646; +} +case 6: +{ +lean_object* x_665; lean_object* x_666; +x_665 = lean_ctor_get(x_652, 1); +lean_inc(x_665); +lean_dec(x_652); +x_666 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_665); +lean_dec(x_665); +if (lean_obj_tag(x_666) == 0) +{ +lean_object* x_667; lean_object* x_668; lean_object* x_669; lean_object* x_670; +x_667 = lean_ctor_get(x_666, 0); +lean_inc(x_667); +lean_dec(x_666); +x_668 = l_Array_append___rarg(x_637, x_667); +lean_dec(x_667); +x_669 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_670 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_670, 0, x_11); +lean_ctor_set(x_670, 1, x_669); +lean_ctor_set(x_670, 2, x_636); +lean_ctor_set(x_670, 3, x_538); +lean_ctor_set(x_670, 4, x_638); +x_3 = x_670; +x_4 = x_668; +goto block_8; +} +else +{ +lean_object* x_671; lean_object* x_672; lean_object* x_673; +x_671 = lean_ctor_get(x_666, 0); +lean_inc(x_671); +lean_dec(x_666); +x_672 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_673 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_673, 0, x_11); +lean_ctor_set(x_673, 1, x_672); +lean_ctor_set(x_673, 2, x_636); +lean_ctor_set(x_673, 3, x_538); +lean_ctor_set(x_673, 4, x_671); +x_3 = x_673; +x_4 = x_637; +goto block_8; +} +} +default: +{ +uint8_t x_674; +x_674 = !lean_is_exclusive(x_652); +if (x_674 == 0) +{ +lean_object* x_675; lean_object* x_676; +x_675 = lean_ctor_get(x_652, 1); +lean_dec(x_675); +x_676 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_652, 0); +lean_ctor_set(x_652, 1, x_676); +x_639 = x_652; +goto block_646; +} +else +{ +lean_object* x_677; lean_object* x_678; lean_object* x_679; +x_677 = lean_ctor_get(x_652, 0); +lean_inc(x_677); +lean_dec(x_652); +x_678 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_679 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_679, 0, x_677); +lean_ctor_set(x_679, 1, x_678); +x_639 = x_679; +goto block_646; } -default: -{ -uint8_t x_814; -lean_free_object(x_796); -x_814 = !lean_is_exclusive(x_800); -if (x_814 == 0) -{ -lean_object* x_815; lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; -x_815 = lean_ctor_get(x_800, 1); -lean_dec(x_815); -x_816 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_800, 0); -lean_ctor_set(x_800, 1, x_816); -x_817 = lean_unsigned_to_nat(1u); -x_818 = lean_mk_array(x_817, x_800); -x_819 = l_Array_append___rarg(x_13, x_818); -lean_dec(x_818); -x_514 = x_797; -x_515 = x_819; -goto block_793; -} -else -{ -lean_object* x_820; lean_object* x_821; lean_object* x_822; lean_object* x_823; lean_object* x_824; lean_object* x_825; -x_820 = lean_ctor_get(x_800, 0); -lean_inc(x_820); -lean_dec(x_800); -x_821 = l_Lake_Glob_decodeToml___closed__2; -x_822 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_822, 0, x_820); -lean_ctor_set(x_822, 1, x_821); -x_823 = lean_unsigned_to_nat(1u); -x_824 = lean_mk_array(x_823, x_822); -x_825 = l_Array_append___rarg(x_13, x_824); -lean_dec(x_824); -x_514 = x_797; -x_515 = x_825; -goto block_793; } } } +block_646: +{ +lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; +x_640 = lean_box(0); +x_641 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_641, 0, x_639); +lean_ctor_set(x_641, 1, x_640); +x_642 = lean_array_mk(x_641); +x_643 = l_Array_append___rarg(x_637, x_642); +lean_dec(x_642); +x_644 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_645 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_645, 0, x_11); +lean_ctor_set(x_645, 1, x_644); +lean_ctor_set(x_645, 2, x_636); +lean_ctor_set(x_645, 3, x_538); +lean_ctor_set(x_645, 4, x_638); +x_3 = x_645; +x_4 = x_643; +goto block_8; } -else +} +block_686: { -lean_object* x_826; lean_object* x_827; -x_826 = lean_ctor_get(x_796, 0); -lean_inc(x_826); -lean_dec(x_796); -x_827 = lean_ctor_get(x_826, 1); -lean_inc(x_827); -lean_dec(x_826); -switch (lean_obj_tag(x_827)) { -case 0: +if (lean_obj_tag(x_681) == 0) { -lean_object* x_828; lean_object* x_829; -x_828 = lean_ctor_get(x_827, 1); -lean_inc(x_828); -lean_dec(x_827); -x_829 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_829, 0, x_828); -x_514 = x_829; -x_515 = x_13; -goto block_793; +x_636 = x_528; +x_637 = x_682; +goto block_680; } -case 2: +else { -lean_object* x_830; lean_object* x_831; lean_object* x_832; lean_object* x_833; lean_object* x_834; lean_object* x_835; -x_830 = lean_ctor_get(x_827, 0); -lean_inc(x_830); -lean_dec(x_827); -x_831 = l_Lake_Glob_decodeToml___closed__2; -x_832 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_832, 0, x_830); -lean_ctor_set(x_832, 1, x_831); -x_833 = lean_unsigned_to_nat(1u); -x_834 = lean_mk_array(x_833, x_832); -x_835 = l_Array_append___rarg(x_13, x_834); -lean_dec(x_834); -x_514 = x_797; -x_515 = x_835; -goto block_793; -} -case 3: +uint8_t x_683; +x_683 = !lean_is_exclusive(x_681); +if (x_683 == 0) { -lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; -x_836 = lean_ctor_get(x_827, 0); -lean_inc(x_836); -lean_dec(x_827); -x_837 = l_Lake_Glob_decodeToml___closed__2; -x_838 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_838, 0, x_836); -lean_ctor_set(x_838, 1, x_837); -x_839 = lean_unsigned_to_nat(1u); -x_840 = lean_mk_array(x_839, x_838); -x_841 = l_Array_append___rarg(x_13, x_840); -lean_dec(x_840); -x_514 = x_797; -x_515 = x_841; -goto block_793; +x_636 = x_681; +x_637 = x_682; +goto block_680; } -default: +else { -lean_object* x_842; lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; -x_842 = lean_ctor_get(x_827, 0); -lean_inc(x_842); -if (lean_is_exclusive(x_827)) { - lean_ctor_release(x_827, 0); - lean_ctor_release(x_827, 1); - x_843 = x_827; -} else { - lean_dec_ref(x_827); - x_843 = lean_box(0); -} -x_844 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_843)) { - x_845 = lean_alloc_ctor(0, 2, 0); -} else { - x_845 = x_843; - lean_ctor_set_tag(x_845, 0); -} -lean_ctor_set(x_845, 0, x_842); -lean_ctor_set(x_845, 1, x_844); -x_846 = lean_unsigned_to_nat(1u); -x_847 = lean_mk_array(x_846, x_845); -x_848 = l_Array_append___rarg(x_13, x_847); -lean_dec(x_847); -x_514 = x_797; -x_515 = x_848; -goto block_793; -} +lean_object* x_684; lean_object* x_685; +x_684 = lean_ctor_get(x_681, 0); +lean_inc(x_684); +lean_dec(x_681); +x_685 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_685, 0, x_684); +x_636 = x_685; +x_637 = x_682; +goto block_680; } } } -block_188: -{ -lean_object* x_16; lean_object* x_17; lean_object* x_153; lean_object* x_154; lean_object* x_155; -x_153 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_154 = l_Lake_Dependency_decodeToml___closed__5; -lean_inc(x_1); -x_155 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_153, x_154, x_1); -if (lean_obj_tag(x_155) == 0) +block_694: { -lean_object* x_156; -x_156 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_16 = x_156; -x_17 = x_15; -goto block_152; +lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; +x_690 = lean_box(0); +x_691 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_691, 0, x_689); +lean_ctor_set(x_691, 1, x_690); +x_692 = lean_array_mk(x_691); +x_693 = l_Array_append___rarg(x_525, x_692); +lean_dec(x_692); +x_681 = x_528; +x_682 = x_693; +goto block_686; +} } else { -lean_object* x_157; lean_object* x_158; -x_157 = lean_ctor_get(x_155, 0); -lean_inc(x_157); -lean_dec(x_155); -x_158 = lean_ctor_get(x_157, 1); -lean_inc(x_158); -lean_dec(x_157); -switch (lean_obj_tag(x_158)) { +lean_object* x_725; lean_object* x_726; +x_725 = lean_ctor_get(x_635, 0); +lean_inc(x_725); +lean_dec(x_635); +x_726 = lean_ctor_get(x_725, 1); +lean_inc(x_726); +lean_dec(x_725); +switch (lean_obj_tag(x_726)) { case 0: { -lean_object* x_159; -x_159 = lean_ctor_get(x_158, 1); -lean_inc(x_159); -lean_dec(x_158); -x_16 = x_159; -x_17 = x_15; -goto block_152; +lean_object* x_727; +x_727 = lean_ctor_get(x_726, 1); +lean_inc(x_727); +lean_dec(x_726); +x_539 = x_727; +x_540 = x_525; +goto block_626; } case 2: { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_160 = lean_ctor_get(x_158, 0); -lean_inc(x_160); -lean_dec(x_158); -x_161 = l_Lake_Glob_decodeToml___closed__2; -x_162 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_162, 0, x_160); -lean_ctor_set(x_162, 1, x_161); -x_163 = lean_unsigned_to_nat(1u); -x_164 = lean_mk_array(x_163, x_162); -x_165 = l_Array_append___rarg(x_15, x_164); -lean_dec(x_164); -x_166 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_16 = x_166; -x_17 = x_165; -goto block_152; +lean_object* x_728; lean_object* x_729; lean_object* x_730; +x_728 = lean_ctor_get(x_726, 0); +lean_inc(x_728); +lean_dec(x_726); +x_729 = l_Lake_Glob_decodeToml___closed__2; +x_730 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_730, 0, x_728); +lean_ctor_set(x_730, 1, x_729); +x_627 = x_730; +goto block_633; } case 3: { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_167 = lean_ctor_get(x_158, 0); -lean_inc(x_167); -lean_dec(x_158); -x_168 = l_Lake_Glob_decodeToml___closed__2; -x_169 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_169, 0, x_167); -lean_ctor_set(x_169, 1, x_168); -x_170 = lean_unsigned_to_nat(1u); -x_171 = lean_mk_array(x_170, x_169); -x_172 = l_Array_append___rarg(x_15, x_171); -lean_dec(x_171); -x_173 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_16 = x_173; -x_17 = x_172; -goto block_152; +lean_object* x_731; lean_object* x_732; lean_object* x_733; +x_731 = lean_ctor_get(x_726, 0); +lean_inc(x_731); +lean_dec(x_726); +x_732 = l_Lake_Glob_decodeToml___closed__2; +x_733 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_733, 0, x_731); +lean_ctor_set(x_733, 1, x_732); +x_627 = x_733; +goto block_633; } default: { -uint8_t x_174; -x_174 = !lean_is_exclusive(x_158); -if (x_174 == 0) +uint8_t x_734; +x_734 = !lean_is_exclusive(x_726); +if (x_734 == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; -x_175 = lean_ctor_get(x_158, 1); -lean_dec(x_175); -x_176 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_158, 0); -lean_ctor_set(x_158, 1, x_176); -x_177 = lean_unsigned_to_nat(1u); -x_178 = lean_mk_array(x_177, x_158); -x_179 = l_Array_append___rarg(x_15, x_178); -lean_dec(x_178); -x_180 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_16 = x_180; -x_17 = x_179; -goto block_152; +lean_object* x_735; lean_object* x_736; +x_735 = lean_ctor_get(x_726, 1); +lean_dec(x_735); +x_736 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_726, 0); +lean_ctor_set(x_726, 1, x_736); +x_627 = x_726; +goto block_633; } else { -lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_181 = lean_ctor_get(x_158, 0); -lean_inc(x_181); -lean_dec(x_158); -x_182 = l_Lake_Glob_decodeToml___closed__2; -x_183 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -x_184 = lean_unsigned_to_nat(1u); -x_185 = lean_mk_array(x_184, x_183); -x_186 = l_Array_append___rarg(x_15, x_185); -lean_dec(x_185); -x_187 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_16 = x_187; -x_17 = x_186; -goto block_152; +lean_object* x_737; lean_object* x_738; lean_object* x_739; +x_737 = lean_ctor_get(x_726, 0); +lean_inc(x_737); +lean_dec(x_726); +x_738 = l_Lake_Glob_decodeToml___closed__2; +x_739 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_739, 0, x_737); +lean_ctor_set(x_739, 1, x_738); +x_627 = x_739; +goto block_633; } } } } -block_152: +block_626: { -lean_object* x_18; lean_object* x_19; lean_object* x_77; lean_object* x_78; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_97 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_98 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_object* x_541; lean_object* x_542; lean_object* x_582; lean_object* x_583; lean_object* x_588; lean_object* x_589; lean_object* x_590; +x_588 = l_Lake_PackageConfig_decodeToml___closed__29; lean_inc(x_1); -x_99 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_97, x_98, x_1); -x_100 = lean_box(0); -if (lean_obj_tag(x_99) == 0) +x_589 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_588, x_1); +if (lean_obj_tag(x_589) == 0) { -x_77 = x_100; -x_78 = x_17; -goto block_96; +x_582 = x_528; +x_583 = x_540; +goto block_587; } else { -uint8_t x_101; -x_101 = !lean_is_exclusive(x_99); -if (x_101 == 0) +uint8_t x_596; +x_596 = !lean_is_exclusive(x_589); +if (x_596 == 0) { -lean_object* x_102; lean_object* x_103; -x_102 = lean_ctor_get(x_99, 0); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -switch (lean_obj_tag(x_103)) { +lean_object* x_597; lean_object* x_598; +x_597 = lean_ctor_get(x_589, 0); +x_598 = lean_ctor_get(x_597, 1); +lean_inc(x_598); +lean_dec(x_597); +switch (lean_obj_tag(x_598)) { case 0: { -lean_object* x_104; -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); -lean_ctor_set(x_99, 0, x_104); -x_77 = x_99; -x_78 = x_17; -goto block_96; +lean_object* x_599; +x_599 = lean_ctor_get(x_598, 1); +lean_inc(x_599); +lean_dec(x_598); +lean_ctor_set(x_589, 0, x_599); +x_582 = x_589; +x_583 = x_540; +goto block_587; } case 2: { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -lean_free_object(x_99); -x_105 = lean_ctor_get(x_103, 0); -lean_inc(x_105); -lean_dec(x_103); -x_106 = l_Lake_Glob_decodeToml___closed__2; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -x_108 = lean_unsigned_to_nat(1u); -x_109 = lean_mk_array(x_108, x_107); -x_110 = l_Array_append___rarg(x_17, x_109); -lean_dec(x_109); -x_77 = x_100; -x_78 = x_110; -goto block_96; +lean_object* x_600; lean_object* x_601; lean_object* x_602; +lean_free_object(x_589); +x_600 = lean_ctor_get(x_598, 0); +lean_inc(x_600); +lean_dec(x_598); +x_601 = l_Lake_Glob_decodeToml___closed__2; +x_602 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_602, 0, x_600); +lean_ctor_set(x_602, 1, x_601); +x_590 = x_602; +goto block_595; } case 3: { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -lean_free_object(x_99); -x_111 = lean_ctor_get(x_103, 0); -lean_inc(x_111); -lean_dec(x_103); -x_112 = l_Lake_Glob_decodeToml___closed__2; -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -x_114 = lean_unsigned_to_nat(1u); -x_115 = lean_mk_array(x_114, x_113); -x_116 = l_Array_append___rarg(x_17, x_115); -lean_dec(x_115); -x_77 = x_100; -x_78 = x_116; -goto block_96; +lean_object* x_603; lean_object* x_604; lean_object* x_605; +lean_free_object(x_589); +x_603 = lean_ctor_get(x_598, 0); +lean_inc(x_603); +lean_dec(x_598); +x_604 = l_Lake_Glob_decodeToml___closed__2; +x_605 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_605, 0, x_603); +lean_ctor_set(x_605, 1, x_604); +x_590 = x_605; +goto block_595; } default: { -uint8_t x_117; -lean_free_object(x_99); -x_117 = !lean_is_exclusive(x_103); -if (x_117 == 0) +uint8_t x_606; +lean_free_object(x_589); +x_606 = !lean_is_exclusive(x_598); +if (x_606 == 0) { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_118 = lean_ctor_get(x_103, 1); -lean_dec(x_118); -x_119 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_103, 0); -lean_ctor_set(x_103, 1, x_119); -x_120 = lean_unsigned_to_nat(1u); -x_121 = lean_mk_array(x_120, x_103); -x_122 = l_Array_append___rarg(x_17, x_121); -lean_dec(x_121); -x_77 = x_100; -x_78 = x_122; -goto block_96; +lean_object* x_607; lean_object* x_608; +x_607 = lean_ctor_get(x_598, 1); +lean_dec(x_607); +x_608 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_598, 0); +lean_ctor_set(x_598, 1, x_608); +x_590 = x_598; +goto block_595; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_123 = lean_ctor_get(x_103, 0); -lean_inc(x_123); -lean_dec(x_103); -x_124 = l_Lake_Glob_decodeToml___closed__2; -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -x_126 = lean_unsigned_to_nat(1u); -x_127 = lean_mk_array(x_126, x_125); -x_128 = l_Array_append___rarg(x_17, x_127); -lean_dec(x_127); -x_77 = x_100; -x_78 = x_128; -goto block_96; +lean_object* x_609; lean_object* x_610; lean_object* x_611; +x_609 = lean_ctor_get(x_598, 0); +lean_inc(x_609); +lean_dec(x_598); +x_610 = l_Lake_Glob_decodeToml___closed__2; +x_611 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_611, 0, x_609); +lean_ctor_set(x_611, 1, x_610); +x_590 = x_611; +goto block_595; } } } } else { -lean_object* x_129; lean_object* x_130; -x_129 = lean_ctor_get(x_99, 0); -lean_inc(x_129); -lean_dec(x_99); -x_130 = lean_ctor_get(x_129, 1); -lean_inc(x_130); -lean_dec(x_129); -switch (lean_obj_tag(x_130)) { +lean_object* x_612; lean_object* x_613; +x_612 = lean_ctor_get(x_589, 0); +lean_inc(x_612); +lean_dec(x_589); +x_613 = lean_ctor_get(x_612, 1); +lean_inc(x_613); +lean_dec(x_612); +switch (lean_obj_tag(x_613)) { case 0: { -lean_object* x_131; lean_object* x_132; -x_131 = lean_ctor_get(x_130, 1); -lean_inc(x_131); -lean_dec(x_130); -x_132 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_132, 0, x_131); -x_77 = x_132; -x_78 = x_17; -goto block_96; +lean_object* x_614; lean_object* x_615; +x_614 = lean_ctor_get(x_613, 1); +lean_inc(x_614); +lean_dec(x_613); +x_615 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_615, 0, x_614); +x_582 = x_615; +x_583 = x_540; +goto block_587; } case 2: { -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; -x_133 = lean_ctor_get(x_130, 0); -lean_inc(x_133); -lean_dec(x_130); -x_134 = l_Lake_Glob_decodeToml___closed__2; -x_135 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -x_136 = lean_unsigned_to_nat(1u); -x_137 = lean_mk_array(x_136, x_135); -x_138 = l_Array_append___rarg(x_17, x_137); -lean_dec(x_137); -x_77 = x_100; -x_78 = x_138; -goto block_96; +lean_object* x_616; lean_object* x_617; lean_object* x_618; +x_616 = lean_ctor_get(x_613, 0); +lean_inc(x_616); +lean_dec(x_613); +x_617 = l_Lake_Glob_decodeToml___closed__2; +x_618 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_618, 0, x_616); +lean_ctor_set(x_618, 1, x_617); +x_590 = x_618; +goto block_595; } case 3: { -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_139 = lean_ctor_get(x_130, 0); -lean_inc(x_139); -lean_dec(x_130); -x_140 = l_Lake_Glob_decodeToml___closed__2; -x_141 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -x_142 = lean_unsigned_to_nat(1u); -x_143 = lean_mk_array(x_142, x_141); -x_144 = l_Array_append___rarg(x_17, x_143); -lean_dec(x_143); -x_77 = x_100; -x_78 = x_144; -goto block_96; +lean_object* x_619; lean_object* x_620; lean_object* x_621; +x_619 = lean_ctor_get(x_613, 0); +lean_inc(x_619); +lean_dec(x_613); +x_620 = l_Lake_Glob_decodeToml___closed__2; +x_621 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_621, 0, x_619); +lean_ctor_set(x_621, 1, x_620); +x_590 = x_621; +goto block_595; } default: { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_145 = lean_ctor_get(x_130, 0); -lean_inc(x_145); -if (lean_is_exclusive(x_130)) { - lean_ctor_release(x_130, 0); - lean_ctor_release(x_130, 1); - x_146 = x_130; +lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; +x_622 = lean_ctor_get(x_613, 0); +lean_inc(x_622); +if (lean_is_exclusive(x_613)) { + lean_ctor_release(x_613, 0); + lean_ctor_release(x_613, 1); + x_623 = x_613; } else { - lean_dec_ref(x_130); - x_146 = lean_box(0); + lean_dec_ref(x_613); + x_623 = lean_box(0); } -x_147 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_146)) { - x_148 = lean_alloc_ctor(0, 2, 0); +x_624 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_623)) { + x_625 = lean_alloc_ctor(0, 2, 0); } else { - x_148 = x_146; - lean_ctor_set_tag(x_148, 0); -} -lean_ctor_set(x_148, 0, x_145); -lean_ctor_set(x_148, 1, x_147); -x_149 = lean_unsigned_to_nat(1u); -x_150 = lean_mk_array(x_149, x_148); -x_151 = l_Array_append___rarg(x_17, x_150); -lean_dec(x_150); -x_77 = x_100; -x_78 = x_151; -goto block_96; + x_625 = x_623; + lean_ctor_set_tag(x_625, 0); } +lean_ctor_set(x_625, 0, x_622); +lean_ctor_set(x_625, 1, x_624); +x_590 = x_625; +goto block_595; } } } -block_76: +} +block_581: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = lean_box(0); -x_21 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_22 = l_Lake_Dependency_decodeToml___closed__2; -x_23 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_21, x_22, x_1); -if (lean_obj_tag(x_23) == 0) +lean_object* x_543; lean_object* x_544; lean_object* x_551; lean_object* x_552; +x_543 = lean_box(0); +x_551 = l_Lake_Dependency_decodeToml___closed__2; +x_552 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_397, x_551, x_1); +if (lean_obj_tag(x_552) == 0) { -lean_object* x_24; -x_24 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_24, 0, x_11); -lean_ctor_set(x_24, 1, x_16); -lean_ctor_set(x_24, 2, x_18); -lean_ctor_set(x_24, 3, x_14); -lean_ctor_set(x_24, 4, x_20); -x_3 = x_24; -x_4 = x_19; +lean_object* x_553; +x_553 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_553, 0, x_11); +lean_ctor_set(x_553, 1, x_539); +lean_ctor_set(x_553, 2, x_541); +lean_ctor_set(x_553, 3, x_538); +lean_ctor_set(x_553, 4, x_543); +x_3 = x_553; +x_4 = x_542; goto block_8; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_23, 0); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -switch (lean_obj_tag(x_26)) { +lean_object* x_554; lean_object* x_555; +x_554 = lean_ctor_get(x_552, 0); +lean_inc(x_554); +lean_dec(x_552); +x_555 = lean_ctor_get(x_554, 1); +lean_inc(x_555); +lean_dec(x_554); +switch (lean_obj_tag(x_555)) { case 0: { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) +uint8_t x_556; +x_556 = !lean_is_exclusive(x_555); +if (x_556 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_28 = lean_ctor_get(x_26, 1); -lean_dec(x_28); -x_29 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_26, 1, x_29); -x_30 = lean_unsigned_to_nat(1u); -x_31 = lean_mk_array(x_30, x_26); -x_32 = l_Array_append___rarg(x_19, x_31); -lean_dec(x_31); -x_33 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_33, 0, x_11); -lean_ctor_set(x_33, 1, x_16); -lean_ctor_set(x_33, 2, x_18); -lean_ctor_set(x_33, 3, x_14); -lean_ctor_set(x_33, 4, x_20); -x_3 = x_33; -x_4 = x_32; -goto block_8; +lean_object* x_557; lean_object* x_558; +x_557 = lean_ctor_get(x_555, 1); +lean_dec(x_557); +x_558 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_555, 1, x_558); +x_544 = x_555; +goto block_550; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_34 = lean_ctor_get(x_26, 0); -lean_inc(x_34); -lean_dec(x_26); -x_35 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = l_Array_append___rarg(x_19, x_38); -lean_dec(x_38); -x_40 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_40, 0, x_11); -lean_ctor_set(x_40, 1, x_16); -lean_ctor_set(x_40, 2, x_18); -lean_ctor_set(x_40, 3, x_14); -lean_ctor_set(x_40, 4, x_20); -x_3 = x_40; -x_4 = x_39; -goto block_8; +lean_object* x_559; lean_object* x_560; lean_object* x_561; +x_559 = lean_ctor_get(x_555, 0); +lean_inc(x_559); +lean_dec(x_555); +x_560 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_561 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_561, 0, x_559); +lean_ctor_set(x_561, 1, x_560); +x_544 = x_561; +goto block_550; } } case 2: { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_41 = lean_ctor_get(x_26, 0); -lean_inc(x_41); -lean_dec(x_26); -x_42 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_unsigned_to_nat(1u); -x_45 = lean_mk_array(x_44, x_43); -x_46 = l_Array_append___rarg(x_19, x_45); -lean_dec(x_45); -x_47 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_47, 0, x_11); -lean_ctor_set(x_47, 1, x_16); -lean_ctor_set(x_47, 2, x_18); -lean_ctor_set(x_47, 3, x_14); -lean_ctor_set(x_47, 4, x_20); -x_3 = x_47; -x_4 = x_46; -goto block_8; +lean_object* x_562; lean_object* x_563; lean_object* x_564; +x_562 = lean_ctor_get(x_555, 0); +lean_inc(x_562); +lean_dec(x_555); +x_563 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_564 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_564, 0, x_562); +lean_ctor_set(x_564, 1, x_563); +x_544 = x_564; +goto block_550; } case 3: { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_48 = lean_ctor_get(x_26, 0); -lean_inc(x_48); -lean_dec(x_26); -x_49 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -x_51 = lean_unsigned_to_nat(1u); -x_52 = lean_mk_array(x_51, x_50); -x_53 = l_Array_append___rarg(x_19, x_52); -lean_dec(x_52); -x_54 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_54, 0, x_11); -lean_ctor_set(x_54, 1, x_16); -lean_ctor_set(x_54, 2, x_18); -lean_ctor_set(x_54, 3, x_14); -lean_ctor_set(x_54, 4, x_20); -x_3 = x_54; -x_4 = x_53; -goto block_8; +lean_object* x_565; lean_object* x_566; lean_object* x_567; +x_565 = lean_ctor_get(x_555, 0); +lean_inc(x_565); +lean_dec(x_555); +x_566 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_567 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_567, 0, x_565); +lean_ctor_set(x_567, 1, x_566); +x_544 = x_567; +goto block_550; } case 6: { -lean_object* x_55; lean_object* x_56; -x_55 = lean_ctor_get(x_26, 1); -lean_inc(x_55); -lean_dec(x_26); -x_56 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_55); -lean_dec(x_55); -if (lean_obj_tag(x_56) == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -lean_dec(x_56); -x_58 = l_Array_append___rarg(x_19, x_57); -lean_dec(x_57); -x_59 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_59, 0, x_11); -lean_ctor_set(x_59, 1, x_16); -lean_ctor_set(x_59, 2, x_18); -lean_ctor_set(x_59, 3, x_14); -lean_ctor_set(x_59, 4, x_20); -x_3 = x_59; -x_4 = x_58; +lean_object* x_568; lean_object* x_569; +x_568 = lean_ctor_get(x_555, 1); +lean_inc(x_568); +lean_dec(x_555); +x_569 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_568); +lean_dec(x_568); +if (lean_obj_tag(x_569) == 0) +{ +lean_object* x_570; lean_object* x_571; lean_object* x_572; +x_570 = lean_ctor_get(x_569, 0); +lean_inc(x_570); +lean_dec(x_569); +x_571 = l_Array_append___rarg(x_542, x_570); +lean_dec(x_570); +x_572 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_572, 0, x_11); +lean_ctor_set(x_572, 1, x_539); +lean_ctor_set(x_572, 2, x_541); +lean_ctor_set(x_572, 3, x_538); +lean_ctor_set(x_572, 4, x_543); +x_3 = x_572; +x_4 = x_571; goto block_8; } else { -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_56, 0); -lean_inc(x_60); -lean_dec(x_56); -x_61 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_61, 0, x_11); -lean_ctor_set(x_61, 1, x_16); -lean_ctor_set(x_61, 2, x_18); -lean_ctor_set(x_61, 3, x_14); -lean_ctor_set(x_61, 4, x_60); -x_3 = x_61; -x_4 = x_19; +lean_object* x_573; lean_object* x_574; +x_573 = lean_ctor_get(x_569, 0); +lean_inc(x_573); +lean_dec(x_569); +x_574 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_574, 0, x_11); +lean_ctor_set(x_574, 1, x_539); +lean_ctor_set(x_574, 2, x_541); +lean_ctor_set(x_574, 3, x_538); +lean_ctor_set(x_574, 4, x_573); +x_3 = x_574; +x_4 = x_542; goto block_8; } } default: { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_26); -if (x_62 == 0) +uint8_t x_575; +x_575 = !lean_is_exclusive(x_555); +if (x_575 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_63 = lean_ctor_get(x_26, 1); -lean_dec(x_63); -x_64 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set_tag(x_26, 0); -lean_ctor_set(x_26, 1, x_64); -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_mk_array(x_65, x_26); -x_67 = l_Array_append___rarg(x_19, x_66); -lean_dec(x_66); -x_68 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_68, 0, x_11); -lean_ctor_set(x_68, 1, x_16); -lean_ctor_set(x_68, 2, x_18); -lean_ctor_set(x_68, 3, x_14); -lean_ctor_set(x_68, 4, x_20); -x_3 = x_68; -x_4 = x_67; -goto block_8; +lean_object* x_576; lean_object* x_577; +x_576 = lean_ctor_get(x_555, 1); +lean_dec(x_576); +x_577 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_555, 0); +lean_ctor_set(x_555, 1, x_577); +x_544 = x_555; +goto block_550; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_69 = lean_ctor_get(x_26, 0); -lean_inc(x_69); -lean_dec(x_26); -x_70 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_71 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -x_72 = lean_unsigned_to_nat(1u); -x_73 = lean_mk_array(x_72, x_71); -x_74 = l_Array_append___rarg(x_19, x_73); -lean_dec(x_73); -x_75 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_75, 0, x_11); -lean_ctor_set(x_75, 1, x_16); -lean_ctor_set(x_75, 2, x_18); -lean_ctor_set(x_75, 3, x_14); -lean_ctor_set(x_75, 4, x_20); -x_3 = x_75; -x_4 = x_74; +lean_object* x_578; lean_object* x_579; lean_object* x_580; +x_578 = lean_ctor_get(x_555, 0); +lean_inc(x_578); +lean_dec(x_555); +x_579 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_580 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_580, 0, x_578); +lean_ctor_set(x_580, 1, x_579); +x_544 = x_580; +goto block_550; +} +} +} +} +block_550: +{ +lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; +x_545 = lean_box(0); +x_546 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_546, 0, x_544); +lean_ctor_set(x_546, 1, x_545); +x_547 = lean_array_mk(x_546); +x_548 = l_Array_append___rarg(x_542, x_547); +lean_dec(x_547); +x_549 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_549, 0, x_11); +lean_ctor_set(x_549, 1, x_539); +lean_ctor_set(x_549, 2, x_541); +lean_ctor_set(x_549, 3, x_538); +lean_ctor_set(x_549, 4, x_543); +x_3 = x_549; +x_4 = x_548; goto block_8; } } +block_587: +{ +if (lean_obj_tag(x_582) == 0) +{ +x_541 = x_528; +x_542 = x_583; +goto block_581; +} +else +{ +uint8_t x_584; +x_584 = !lean_is_exclusive(x_582); +if (x_584 == 0) +{ +x_541 = x_582; +x_542 = x_583; +goto block_581; +} +else +{ +lean_object* x_585; lean_object* x_586; +x_585 = lean_ctor_get(x_582, 0); +lean_inc(x_585); +lean_dec(x_582); +x_586 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_586, 0, x_585); +x_541 = x_586; +x_542 = x_583; +goto block_581; +} +} +} +block_595: +{ +lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; +x_591 = lean_box(0); +x_592 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_592, 0, x_590); +lean_ctor_set(x_592, 1, x_591); +x_593 = lean_array_mk(x_592); +x_594 = l_Array_append___rarg(x_540, x_593); +lean_dec(x_593); +x_582 = x_528; +x_583 = x_594; +goto block_587; +} +} +block_633: +{ +lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; +x_628 = lean_box(0); +x_629 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_629, 0, x_627); +lean_ctor_set(x_629, 1, x_628); +x_630 = lean_array_mk(x_629); +x_631 = l_Array_append___rarg(x_525, x_630); +lean_dec(x_630); +x_632 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_539 = x_632; +x_540 = x_631; +goto block_626; +} +} +else +{ +uint8_t x_740; +x_740 = !lean_is_exclusive(x_527); +if (x_740 == 0) +{ +lean_object* x_741; lean_object* x_742; +x_741 = lean_ctor_get(x_527, 0); +x_742 = lean_ctor_get(x_741, 1); +lean_inc(x_742); +lean_dec(x_741); +switch (lean_obj_tag(x_742)) { +case 0: +{ +lean_object* x_743; lean_object* x_744; lean_object* x_745; +lean_dec(x_523); +lean_dec(x_460); +x_743 = lean_ctor_get(x_742, 1); +lean_inc(x_743); +lean_dec(x_742); +lean_ctor_set(x_527, 0, x_743); +lean_inc(x_12); +x_744 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_744, 0, x_524); +lean_ctor_set(x_744, 1, x_12); +lean_ctor_set(x_744, 2, x_527); +x_745 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_745, 0, x_744); +x_14 = x_745; +x_15 = x_525; +goto block_147; } +case 2: +{ +lean_object* x_746; lean_object* x_747; lean_object* x_748; +lean_free_object(x_527); +x_746 = lean_ctor_get(x_742, 0); +lean_inc(x_746); +lean_dec(x_742); +x_747 = l_Lake_Glob_decodeToml___closed__2; +x_748 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_748, 0, x_746); +lean_ctor_set(x_748, 1, x_747); +x_529 = x_748; +goto block_536; } +case 3: +{ +lean_object* x_749; lean_object* x_750; lean_object* x_751; +lean_free_object(x_527); +x_749 = lean_ctor_get(x_742, 0); +lean_inc(x_749); +lean_dec(x_742); +x_750 = l_Lake_Glob_decodeToml___closed__2; +x_751 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_751, 0, x_749); +lean_ctor_set(x_751, 1, x_750); +x_529 = x_751; +goto block_536; } -block_96: +default: { -if (lean_obj_tag(x_77) == 0) +uint8_t x_752; +lean_free_object(x_527); +x_752 = !lean_is_exclusive(x_742); +if (x_752 == 0) { -if (lean_obj_tag(x_12) == 0) +lean_object* x_753; lean_object* x_754; +x_753 = lean_ctor_get(x_742, 1); +lean_dec(x_753); +x_754 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_742, 0); +lean_ctor_set(x_742, 1, x_754); +x_529 = x_742; +goto block_536; +} +else { -lean_object* x_79; -x_79 = lean_box(0); -x_18 = x_79; -x_19 = x_78; -goto block_76; +lean_object* x_755; lean_object* x_756; lean_object* x_757; +x_755 = lean_ctor_get(x_742, 0); +lean_inc(x_755); +lean_dec(x_742); +x_756 = l_Lake_Glob_decodeToml___closed__2; +x_757 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_757, 0, x_755); +lean_ctor_set(x_757, 1, x_756); +x_529 = x_757; +goto block_536; +} +} +} } else { -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_80; -x_80 = !lean_is_exclusive(x_12); -if (x_80 == 0) +lean_object* x_758; lean_object* x_759; +x_758 = lean_ctor_get(x_527, 0); +lean_inc(x_758); +lean_dec(x_527); +x_759 = lean_ctor_get(x_758, 1); +lean_inc(x_759); +lean_dec(x_758); +switch (lean_obj_tag(x_759)) { +case 0: { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_81 = lean_ctor_get(x_12, 0); -x_82 = l_Lake_Dependency_decodeToml___closed__3; -x_83 = lean_string_append(x_82, x_81); -lean_dec(x_81); -x_84 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_85 = lean_string_append(x_83, x_84); -lean_ctor_set(x_12, 0, x_85); -x_18 = x_12; -x_19 = x_78; -goto block_76; +lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; +lean_dec(x_523); +lean_dec(x_460); +x_760 = lean_ctor_get(x_759, 1); +lean_inc(x_760); +lean_dec(x_759); +x_761 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_761, 0, x_760); +lean_inc(x_12); +x_762 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_762, 0, x_524); +lean_ctor_set(x_762, 1, x_12); +lean_ctor_set(x_762, 2, x_761); +x_763 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_763, 0, x_762); +x_14 = x_763; +x_15 = x_525; +goto block_147; } -else +case 2: { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_86 = lean_ctor_get(x_12, 0); -lean_inc(x_86); -lean_dec(x_12); -x_87 = l_Lake_Dependency_decodeToml___closed__3; -x_88 = lean_string_append(x_87, x_86); -lean_dec(x_86); -x_89 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_90 = lean_string_append(x_88, x_89); -x_91 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_91, 0, x_90); -x_18 = x_91; -x_19 = x_78; -goto block_76; +lean_object* x_764; lean_object* x_765; lean_object* x_766; +x_764 = lean_ctor_get(x_759, 0); +lean_inc(x_764); +lean_dec(x_759); +x_765 = l_Lake_Glob_decodeToml___closed__2; +x_766 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_766, 0, x_764); +lean_ctor_set(x_766, 1, x_765); +x_529 = x_766; +goto block_536; } +case 3: +{ +lean_object* x_767; lean_object* x_768; lean_object* x_769; +x_767 = lean_ctor_get(x_759, 0); +lean_inc(x_767); +lean_dec(x_759); +x_768 = l_Lake_Glob_decodeToml___closed__2; +x_769 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_769, 0, x_767); +lean_ctor_set(x_769, 1, x_768); +x_529 = x_769; +goto block_536; } -else +default: { -lean_object* x_92; -lean_dec(x_12); -x_92 = lean_box(0); -x_18 = x_92; -x_19 = x_78; -goto block_76; +lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; +x_770 = lean_ctor_get(x_759, 0); +lean_inc(x_770); +if (lean_is_exclusive(x_759)) { + lean_ctor_release(x_759, 0); + lean_ctor_release(x_759, 1); + x_771 = x_759; +} else { + lean_dec_ref(x_759); + x_771 = lean_box(0); } +x_772 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_771)) { + x_773 = lean_alloc_ctor(0, 2, 0); +} else { + x_773 = x_771; + lean_ctor_set_tag(x_773, 0); } +lean_ctor_set(x_773, 0, x_770); +lean_ctor_set(x_773, 1, x_772); +x_529 = x_773; +goto block_536; } -else -{ -uint8_t x_93; -lean_dec(x_12); -x_93 = !lean_is_exclusive(x_77); -if (x_93 == 0) -{ -x_18 = x_77; -x_19 = x_78; -goto block_76; } -else +} +} +block_536: { -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_77, 0); -lean_inc(x_94); -lean_dec(x_77); -x_95 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_95, 0, x_94); -x_18 = x_95; -x_19 = x_78; -goto block_76; +lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; +x_530 = lean_box(0); +if (lean_is_scalar(x_523)) { + x_531 = lean_alloc_ctor(1, 2, 0); +} else { + x_531 = x_523; + lean_ctor_set_tag(x_531, 1); } +lean_ctor_set(x_531, 0, x_529); +lean_ctor_set(x_531, 1, x_530); +x_532 = lean_array_mk(x_531); +x_533 = l_Array_append___rarg(x_525, x_532); +lean_dec(x_532); +lean_inc(x_12); +x_534 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_534, 0, x_524); +lean_ctor_set(x_534, 1, x_12); +lean_ctor_set(x_534, 2, x_528); +if (lean_is_scalar(x_460)) { + x_535 = lean_alloc_ctor(1, 1, 0); +} else { + x_535 = x_460; } +lean_ctor_set(x_535, 0, x_534); +x_14 = x_535; +x_15 = x_533; +goto block_147; } } } -block_513: -{ -lean_object* x_191; lean_object* x_192; lean_object* x_327; lean_object* x_328; lean_object* x_329; -x_327 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_328 = l_Lake_Dependency_decodeToml___closed__5; -lean_inc(x_1); -x_329 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_327, x_328, x_1); -if (lean_obj_tag(x_329) == 0) -{ -lean_object* x_330; lean_object* x_331; lean_object* x_397; lean_object* x_398; lean_object* x_416; lean_object* x_417; lean_object* x_418; -x_416 = l_Lake_PackageConfig_decodeToml___closed__29; -lean_inc(x_1); -x_417 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_327, x_416, x_1); -x_418 = lean_box(0); -if (lean_obj_tag(x_417) == 0) +default: { -if (lean_obj_tag(x_12) == 0) +uint8_t x_781; +lean_dec(x_460); +x_781 = !lean_is_exclusive(x_461); +if (x_781 == 0) { -x_330 = x_418; -x_331 = x_190; -goto block_396; +lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; +x_782 = lean_ctor_get(x_461, 1); +lean_dec(x_782); +x_783 = l_Lake_Dependency_decodeToml___closed__9; +lean_ctor_set_tag(x_461, 0); +lean_ctor_set(x_461, 1, x_783); +x_784 = lean_array_push(x_396, x_461); +x_785 = lean_box(0); +x_148 = x_785; +x_149 = x_784; +goto block_394; } else { -uint8_t x_419; -x_419 = !lean_is_exclusive(x_12); -if (x_419 == 0) -{ -lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; -x_420 = lean_ctor_get(x_12, 0); -x_421 = l_Lake_Dependency_decodeToml___closed__3; -x_422 = lean_string_append(x_421, x_420); -lean_dec(x_420); -x_423 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_424 = lean_string_append(x_422, x_423); -lean_ctor_set(x_12, 0, x_424); -x_330 = x_12; -x_331 = x_190; -goto block_396; +lean_object* x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; +x_786 = lean_ctor_get(x_461, 0); +lean_inc(x_786); +lean_dec(x_461); +x_787 = l_Lake_Dependency_decodeToml___closed__9; +x_788 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_788, 0, x_786); +lean_ctor_set(x_788, 1, x_787); +x_789 = lean_array_push(x_396, x_788); +x_790 = lean_box(0); +x_148 = x_790; +x_149 = x_789; +goto block_394; +} +} +} +} } else { -lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; -x_425 = lean_ctor_get(x_12, 0); -lean_inc(x_425); +uint8_t x_791; lean_dec(x_12); -x_426 = l_Lake_Dependency_decodeToml___closed__3; -x_427 = lean_string_append(x_426, x_425); -lean_dec(x_425); -x_428 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_429 = lean_string_append(x_427, x_428); -x_430 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_430, 0, x_429); -x_330 = x_430; -x_331 = x_190; -goto block_396; -} -} +x_791 = !lean_is_exclusive(x_395); +if (x_791 == 0) +{ +lean_object* x_792; lean_object* x_793; lean_object* x_794; lean_object* x_795; lean_object* x_886; lean_object* x_893; lean_object* x_894; lean_object* x_895; +x_792 = lean_ctor_get(x_395, 0); +x_793 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_793, 0, x_792); +lean_ctor_set(x_395, 0, x_793); +x_893 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_894 = l_Lake_Dependency_decodeToml___closed__5; +lean_inc(x_1); +x_895 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_893, x_894, x_1); +if (lean_obj_tag(x_895) == 0) +{ +lean_object* x_896; lean_object* x_897; lean_object* x_941; lean_object* x_942; lean_object* x_948; lean_object* x_949; lean_object* x_950; lean_object* x_951; +x_948 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_inc(x_1); +x_949 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_893, x_948, x_1); +x_950 = lean_box(0); +if (lean_obj_tag(x_949) == 0) +{ +x_896 = x_950; +x_897 = x_396; +goto block_940; } else { -uint8_t x_431; -x_431 = !lean_is_exclusive(x_417); -if (x_431 == 0) +uint8_t x_957; +x_957 = !lean_is_exclusive(x_949); +if (x_957 == 0) { -lean_object* x_432; lean_object* x_433; -x_432 = lean_ctor_get(x_417, 0); -x_433 = lean_ctor_get(x_432, 1); -lean_inc(x_433); -lean_dec(x_432); -switch (lean_obj_tag(x_433)) { +lean_object* x_958; lean_object* x_959; +x_958 = lean_ctor_get(x_949, 0); +x_959 = lean_ctor_get(x_958, 1); +lean_inc(x_959); +lean_dec(x_958); +switch (lean_obj_tag(x_959)) { case 0: { -lean_object* x_434; -x_434 = lean_ctor_get(x_433, 1); -lean_inc(x_434); -lean_dec(x_433); -lean_ctor_set(x_417, 0, x_434); -x_397 = x_417; -x_398 = x_190; -goto block_415; +lean_object* x_960; +x_960 = lean_ctor_get(x_959, 1); +lean_inc(x_960); +lean_dec(x_959); +lean_ctor_set(x_949, 0, x_960); +x_941 = x_949; +x_942 = x_396; +goto block_947; } case 2: { -lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; -lean_free_object(x_417); -x_435 = lean_ctor_get(x_433, 0); -lean_inc(x_435); -lean_dec(x_433); -x_436 = l_Lake_Glob_decodeToml___closed__2; -x_437 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_437, 0, x_435); -lean_ctor_set(x_437, 1, x_436); -x_438 = lean_unsigned_to_nat(1u); -x_439 = lean_mk_array(x_438, x_437); -x_440 = l_Array_append___rarg(x_190, x_439); -lean_dec(x_439); -x_397 = x_418; -x_398 = x_440; -goto block_415; +lean_object* x_961; lean_object* x_962; lean_object* x_963; +lean_free_object(x_949); +x_961 = lean_ctor_get(x_959, 0); +lean_inc(x_961); +lean_dec(x_959); +x_962 = l_Lake_Glob_decodeToml___closed__2; +x_963 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_963, 0, x_961); +lean_ctor_set(x_963, 1, x_962); +x_951 = x_963; +goto block_956; } case 3: { -lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; -lean_free_object(x_417); -x_441 = lean_ctor_get(x_433, 0); -lean_inc(x_441); -lean_dec(x_433); -x_442 = l_Lake_Glob_decodeToml___closed__2; -x_443 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_443, 0, x_441); -lean_ctor_set(x_443, 1, x_442); -x_444 = lean_unsigned_to_nat(1u); -x_445 = lean_mk_array(x_444, x_443); -x_446 = l_Array_append___rarg(x_190, x_445); -lean_dec(x_445); -x_397 = x_418; -x_398 = x_446; -goto block_415; +lean_object* x_964; lean_object* x_965; lean_object* x_966; +lean_free_object(x_949); +x_964 = lean_ctor_get(x_959, 0); +lean_inc(x_964); +lean_dec(x_959); +x_965 = l_Lake_Glob_decodeToml___closed__2; +x_966 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_966, 0, x_964); +lean_ctor_set(x_966, 1, x_965); +x_951 = x_966; +goto block_956; } default: { -uint8_t x_447; -lean_free_object(x_417); -x_447 = !lean_is_exclusive(x_433); -if (x_447 == 0) +uint8_t x_967; +lean_free_object(x_949); +x_967 = !lean_is_exclusive(x_959); +if (x_967 == 0) { -lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; -x_448 = lean_ctor_get(x_433, 1); -lean_dec(x_448); -x_449 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_433, 0); -lean_ctor_set(x_433, 1, x_449); -x_450 = lean_unsigned_to_nat(1u); -x_451 = lean_mk_array(x_450, x_433); -x_452 = l_Array_append___rarg(x_190, x_451); -lean_dec(x_451); -x_397 = x_418; -x_398 = x_452; -goto block_415; +lean_object* x_968; lean_object* x_969; +x_968 = lean_ctor_get(x_959, 1); +lean_dec(x_968); +x_969 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_959, 0); +lean_ctor_set(x_959, 1, x_969); +x_951 = x_959; +goto block_956; } else { -lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; -x_453 = lean_ctor_get(x_433, 0); -lean_inc(x_453); -lean_dec(x_433); -x_454 = l_Lake_Glob_decodeToml___closed__2; -x_455 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_455, 0, x_453); -lean_ctor_set(x_455, 1, x_454); -x_456 = lean_unsigned_to_nat(1u); -x_457 = lean_mk_array(x_456, x_455); -x_458 = l_Array_append___rarg(x_190, x_457); -lean_dec(x_457); -x_397 = x_418; -x_398 = x_458; -goto block_415; +lean_object* x_970; lean_object* x_971; lean_object* x_972; +x_970 = lean_ctor_get(x_959, 0); +lean_inc(x_970); +lean_dec(x_959); +x_971 = l_Lake_Glob_decodeToml___closed__2; +x_972 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_972, 0, x_970); +lean_ctor_set(x_972, 1, x_971); +x_951 = x_972; +goto block_956; } } } } else { -lean_object* x_459; lean_object* x_460; -x_459 = lean_ctor_get(x_417, 0); -lean_inc(x_459); -lean_dec(x_417); -x_460 = lean_ctor_get(x_459, 1); -lean_inc(x_460); -lean_dec(x_459); -switch (lean_obj_tag(x_460)) { +lean_object* x_973; lean_object* x_974; +x_973 = lean_ctor_get(x_949, 0); +lean_inc(x_973); +lean_dec(x_949); +x_974 = lean_ctor_get(x_973, 1); +lean_inc(x_974); +lean_dec(x_973); +switch (lean_obj_tag(x_974)) { case 0: { -lean_object* x_461; lean_object* x_462; -x_461 = lean_ctor_get(x_460, 1); -lean_inc(x_461); -lean_dec(x_460); -x_462 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_462, 0, x_461); -x_397 = x_462; -x_398 = x_190; -goto block_415; +lean_object* x_975; lean_object* x_976; +x_975 = lean_ctor_get(x_974, 1); +lean_inc(x_975); +lean_dec(x_974); +x_976 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_976, 0, x_975); +x_941 = x_976; +x_942 = x_396; +goto block_947; } case 2: { -lean_object* x_463; lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; -x_463 = lean_ctor_get(x_460, 0); -lean_inc(x_463); -lean_dec(x_460); -x_464 = l_Lake_Glob_decodeToml___closed__2; -x_465 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_465, 0, x_463); -lean_ctor_set(x_465, 1, x_464); -x_466 = lean_unsigned_to_nat(1u); -x_467 = lean_mk_array(x_466, x_465); -x_468 = l_Array_append___rarg(x_190, x_467); -lean_dec(x_467); -x_397 = x_418; -x_398 = x_468; -goto block_415; +lean_object* x_977; lean_object* x_978; lean_object* x_979; +x_977 = lean_ctor_get(x_974, 0); +lean_inc(x_977); +lean_dec(x_974); +x_978 = l_Lake_Glob_decodeToml___closed__2; +x_979 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_979, 0, x_977); +lean_ctor_set(x_979, 1, x_978); +x_951 = x_979; +goto block_956; } case 3: { -lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; lean_object* x_473; lean_object* x_474; -x_469 = lean_ctor_get(x_460, 0); -lean_inc(x_469); -lean_dec(x_460); -x_470 = l_Lake_Glob_decodeToml___closed__2; -x_471 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_471, 0, x_469); -lean_ctor_set(x_471, 1, x_470); -x_472 = lean_unsigned_to_nat(1u); -x_473 = lean_mk_array(x_472, x_471); -x_474 = l_Array_append___rarg(x_190, x_473); -lean_dec(x_473); -x_397 = x_418; -x_398 = x_474; -goto block_415; +lean_object* x_980; lean_object* x_981; lean_object* x_982; +x_980 = lean_ctor_get(x_974, 0); +lean_inc(x_980); +lean_dec(x_974); +x_981 = l_Lake_Glob_decodeToml___closed__2; +x_982 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_982, 0, x_980); +lean_ctor_set(x_982, 1, x_981); +x_951 = x_982; +goto block_956; } default: { -lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; lean_object* x_480; lean_object* x_481; -x_475 = lean_ctor_get(x_460, 0); -lean_inc(x_475); -if (lean_is_exclusive(x_460)) { - lean_ctor_release(x_460, 0); - lean_ctor_release(x_460, 1); - x_476 = x_460; +lean_object* x_983; lean_object* x_984; lean_object* x_985; lean_object* x_986; +x_983 = lean_ctor_get(x_974, 0); +lean_inc(x_983); +if (lean_is_exclusive(x_974)) { + lean_ctor_release(x_974, 0); + lean_ctor_release(x_974, 1); + x_984 = x_974; } else { - lean_dec_ref(x_460); - x_476 = lean_box(0); + lean_dec_ref(x_974); + x_984 = lean_box(0); } -x_477 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_476)) { - x_478 = lean_alloc_ctor(0, 2, 0); +x_985 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_984)) { + x_986 = lean_alloc_ctor(0, 2, 0); } else { - x_478 = x_476; - lean_ctor_set_tag(x_478, 0); -} -lean_ctor_set(x_478, 0, x_475); -lean_ctor_set(x_478, 1, x_477); -x_479 = lean_unsigned_to_nat(1u); -x_480 = lean_mk_array(x_479, x_478); -x_481 = l_Array_append___rarg(x_190, x_480); -lean_dec(x_480); -x_397 = x_418; -x_398 = x_481; -goto block_415; + x_986 = x_984; + lean_ctor_set_tag(x_986, 0); } +lean_ctor_set(x_986, 0, x_983); +lean_ctor_set(x_986, 1, x_985); +x_951 = x_986; +goto block_956; } } } -block_396: +} +block_940: { -lean_object* x_332; lean_object* x_333; lean_object* x_334; -x_332 = lean_box(0); -x_333 = l_Lake_Dependency_decodeToml___closed__2; -x_334 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_327, x_333, x_1); -if (lean_obj_tag(x_334) == 0) +lean_object* x_898; lean_object* x_899; lean_object* x_907; lean_object* x_908; +x_898 = lean_box(0); +x_907 = l_Lake_Dependency_decodeToml___closed__2; +x_908 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_893, x_907, x_1); +if (lean_obj_tag(x_908) == 0) { -lean_object* x_335; lean_object* x_336; -x_335 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_336 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_336, 0, x_11); -lean_ctor_set(x_336, 1, x_335); -lean_ctor_set(x_336, 2, x_330); -lean_ctor_set(x_336, 3, x_189); -lean_ctor_set(x_336, 4, x_332); -x_3 = x_336; -x_4 = x_331; +lean_object* x_909; lean_object* x_910; +x_909 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_910 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_910, 0, x_11); +lean_ctor_set(x_910, 1, x_909); +lean_ctor_set(x_910, 2, x_896); +lean_ctor_set(x_910, 3, x_395); +lean_ctor_set(x_910, 4, x_898); +x_3 = x_910; +x_4 = x_897; goto block_8; } else { -lean_object* x_337; lean_object* x_338; -x_337 = lean_ctor_get(x_334, 0); -lean_inc(x_337); -lean_dec(x_334); -x_338 = lean_ctor_get(x_337, 1); -lean_inc(x_338); -lean_dec(x_337); -switch (lean_obj_tag(x_338)) { +lean_object* x_911; lean_object* x_912; +x_911 = lean_ctor_get(x_908, 0); +lean_inc(x_911); +lean_dec(x_908); +x_912 = lean_ctor_get(x_911, 1); +lean_inc(x_912); +lean_dec(x_911); +switch (lean_obj_tag(x_912)) { case 0: { -uint8_t x_339; -x_339 = !lean_is_exclusive(x_338); -if (x_339 == 0) -{ -lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; -x_340 = lean_ctor_get(x_338, 1); -lean_dec(x_340); -x_341 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_338, 1, x_341); -x_342 = lean_unsigned_to_nat(1u); -x_343 = lean_mk_array(x_342, x_338); -x_344 = l_Array_append___rarg(x_331, x_343); -lean_dec(x_343); -x_345 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_346 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_346, 0, x_11); -lean_ctor_set(x_346, 1, x_345); -lean_ctor_set(x_346, 2, x_330); -lean_ctor_set(x_346, 3, x_189); -lean_ctor_set(x_346, 4, x_332); -x_3 = x_346; -x_4 = x_344; -goto block_8; +uint8_t x_913; +x_913 = !lean_is_exclusive(x_912); +if (x_913 == 0) +{ +lean_object* x_914; lean_object* x_915; +x_914 = lean_ctor_get(x_912, 1); +lean_dec(x_914); +x_915 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_912, 1, x_915); +x_899 = x_912; +goto block_906; } else { -lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; -x_347 = lean_ctor_get(x_338, 0); -lean_inc(x_347); -lean_dec(x_338); -x_348 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_349 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_349, 0, x_347); -lean_ctor_set(x_349, 1, x_348); -x_350 = lean_unsigned_to_nat(1u); -x_351 = lean_mk_array(x_350, x_349); -x_352 = l_Array_append___rarg(x_331, x_351); -lean_dec(x_351); -x_353 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_354 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_354, 0, x_11); -lean_ctor_set(x_354, 1, x_353); -lean_ctor_set(x_354, 2, x_330); -lean_ctor_set(x_354, 3, x_189); -lean_ctor_set(x_354, 4, x_332); -x_3 = x_354; -x_4 = x_352; -goto block_8; +lean_object* x_916; lean_object* x_917; lean_object* x_918; +x_916 = lean_ctor_get(x_912, 0); +lean_inc(x_916); +lean_dec(x_912); +x_917 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_918 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_918, 0, x_916); +lean_ctor_set(x_918, 1, x_917); +x_899 = x_918; +goto block_906; } } case 2: { -lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; -x_355 = lean_ctor_get(x_338, 0); -lean_inc(x_355); -lean_dec(x_338); -x_356 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_357 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_357, 0, x_355); -lean_ctor_set(x_357, 1, x_356); -x_358 = lean_unsigned_to_nat(1u); -x_359 = lean_mk_array(x_358, x_357); -x_360 = l_Array_append___rarg(x_331, x_359); -lean_dec(x_359); -x_361 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_362 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_362, 0, x_11); -lean_ctor_set(x_362, 1, x_361); -lean_ctor_set(x_362, 2, x_330); -lean_ctor_set(x_362, 3, x_189); -lean_ctor_set(x_362, 4, x_332); -x_3 = x_362; -x_4 = x_360; -goto block_8; +lean_object* x_919; lean_object* x_920; lean_object* x_921; +x_919 = lean_ctor_get(x_912, 0); +lean_inc(x_919); +lean_dec(x_912); +x_920 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_921 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_921, 0, x_919); +lean_ctor_set(x_921, 1, x_920); +x_899 = x_921; +goto block_906; } case 3: { -lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; -x_363 = lean_ctor_get(x_338, 0); -lean_inc(x_363); -lean_dec(x_338); -x_364 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_365 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_365, 0, x_363); -lean_ctor_set(x_365, 1, x_364); -x_366 = lean_unsigned_to_nat(1u); -x_367 = lean_mk_array(x_366, x_365); -x_368 = l_Array_append___rarg(x_331, x_367); -lean_dec(x_367); -x_369 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_370 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_370, 0, x_11); -lean_ctor_set(x_370, 1, x_369); -lean_ctor_set(x_370, 2, x_330); -lean_ctor_set(x_370, 3, x_189); -lean_ctor_set(x_370, 4, x_332); -x_3 = x_370; -x_4 = x_368; -goto block_8; +lean_object* x_922; lean_object* x_923; lean_object* x_924; +x_922 = lean_ctor_get(x_912, 0); +lean_inc(x_922); +lean_dec(x_912); +x_923 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_924 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_924, 0, x_922); +lean_ctor_set(x_924, 1, x_923); +x_899 = x_924; +goto block_906; } case 6: { -lean_object* x_371; lean_object* x_372; -x_371 = lean_ctor_get(x_338, 1); -lean_inc(x_371); -lean_dec(x_338); -x_372 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_371); -lean_dec(x_371); -if (lean_obj_tag(x_372) == 0) +lean_object* x_925; lean_object* x_926; +x_925 = lean_ctor_get(x_912, 1); +lean_inc(x_925); +lean_dec(x_912); +x_926 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_925); +lean_dec(x_925); +if (lean_obj_tag(x_926) == 0) { -lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; -x_373 = lean_ctor_get(x_372, 0); -lean_inc(x_373); -lean_dec(x_372); -x_374 = l_Array_append___rarg(x_331, x_373); -lean_dec(x_373); -x_375 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_376 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_376, 0, x_11); -lean_ctor_set(x_376, 1, x_375); -lean_ctor_set(x_376, 2, x_330); -lean_ctor_set(x_376, 3, x_189); -lean_ctor_set(x_376, 4, x_332); -x_3 = x_376; -x_4 = x_374; +lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; +x_927 = lean_ctor_get(x_926, 0); +lean_inc(x_927); +lean_dec(x_926); +x_928 = l_Array_append___rarg(x_897, x_927); +lean_dec(x_927); +x_929 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_930 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_930, 0, x_11); +lean_ctor_set(x_930, 1, x_929); +lean_ctor_set(x_930, 2, x_896); +lean_ctor_set(x_930, 3, x_395); +lean_ctor_set(x_930, 4, x_898); +x_3 = x_930; +x_4 = x_928; goto block_8; } else { -lean_object* x_377; lean_object* x_378; lean_object* x_379; -x_377 = lean_ctor_get(x_372, 0); -lean_inc(x_377); -lean_dec(x_372); -x_378 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_379 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_379, 0, x_11); -lean_ctor_set(x_379, 1, x_378); -lean_ctor_set(x_379, 2, x_330); -lean_ctor_set(x_379, 3, x_189); -lean_ctor_set(x_379, 4, x_377); -x_3 = x_379; -x_4 = x_331; +lean_object* x_931; lean_object* x_932; lean_object* x_933; +x_931 = lean_ctor_get(x_926, 0); +lean_inc(x_931); +lean_dec(x_926); +x_932 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_933 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_933, 0, x_11); +lean_ctor_set(x_933, 1, x_932); +lean_ctor_set(x_933, 2, x_896); +lean_ctor_set(x_933, 3, x_395); +lean_ctor_set(x_933, 4, x_931); +x_3 = x_933; +x_4 = x_897; goto block_8; } } default: { -uint8_t x_380; -x_380 = !lean_is_exclusive(x_338); -if (x_380 == 0) -{ -lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; -x_381 = lean_ctor_get(x_338, 1); -lean_dec(x_381); -x_382 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set_tag(x_338, 0); -lean_ctor_set(x_338, 1, x_382); -x_383 = lean_unsigned_to_nat(1u); -x_384 = lean_mk_array(x_383, x_338); -x_385 = l_Array_append___rarg(x_331, x_384); -lean_dec(x_384); -x_386 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_387 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_387, 0, x_11); -lean_ctor_set(x_387, 1, x_386); -lean_ctor_set(x_387, 2, x_330); -lean_ctor_set(x_387, 3, x_189); -lean_ctor_set(x_387, 4, x_332); -x_3 = x_387; -x_4 = x_385; -goto block_8; +uint8_t x_934; +x_934 = !lean_is_exclusive(x_912); +if (x_934 == 0) +{ +lean_object* x_935; lean_object* x_936; +x_935 = lean_ctor_get(x_912, 1); +lean_dec(x_935); +x_936 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_912, 0); +lean_ctor_set(x_912, 1, x_936); +x_899 = x_912; +goto block_906; } else { -lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; -x_388 = lean_ctor_get(x_338, 0); -lean_inc(x_388); -lean_dec(x_338); -x_389 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_390 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_390, 0, x_388); -lean_ctor_set(x_390, 1, x_389); -x_391 = lean_unsigned_to_nat(1u); -x_392 = lean_mk_array(x_391, x_390); -x_393 = l_Array_append___rarg(x_331, x_392); -lean_dec(x_392); -x_394 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_395 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_395, 0, x_11); -lean_ctor_set(x_395, 1, x_394); -lean_ctor_set(x_395, 2, x_330); -lean_ctor_set(x_395, 3, x_189); -lean_ctor_set(x_395, 4, x_332); -x_3 = x_395; -x_4 = x_393; -goto block_8; -} +lean_object* x_937; lean_object* x_938; lean_object* x_939; +x_937 = lean_ctor_get(x_912, 0); +lean_inc(x_937); +lean_dec(x_912); +x_938 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_939 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_939, 0, x_937); +lean_ctor_set(x_939, 1, x_938); +x_899 = x_939; +goto block_906; } } } } -block_415: +block_906: { -if (lean_obj_tag(x_397) == 0) +lean_object* x_900; lean_object* x_901; lean_object* x_902; lean_object* x_903; lean_object* x_904; lean_object* x_905; +x_900 = lean_box(0); +x_901 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_901, 0, x_899); +lean_ctor_set(x_901, 1, x_900); +x_902 = lean_array_mk(x_901); +x_903 = l_Array_append___rarg(x_897, x_902); +lean_dec(x_902); +x_904 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_905 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_905, 0, x_11); +lean_ctor_set(x_905, 1, x_904); +lean_ctor_set(x_905, 2, x_896); +lean_ctor_set(x_905, 3, x_395); +lean_ctor_set(x_905, 4, x_898); +x_3 = x_905; +x_4 = x_903; +goto block_8; +} +} +block_947: { -if (lean_obj_tag(x_12) == 0) +if (lean_obj_tag(x_941) == 0) { -lean_object* x_399; -x_399 = lean_box(0); -x_330 = x_399; -x_331 = x_398; -goto block_396; +lean_object* x_943; +x_943 = lean_box(0); +x_896 = x_943; +x_897 = x_942; +goto block_940; } else { -uint8_t x_400; -x_400 = !lean_is_exclusive(x_12); -if (x_400 == 0) +uint8_t x_944; +x_944 = !lean_is_exclusive(x_941); +if (x_944 == 0) { -lean_object* x_401; lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; -x_401 = lean_ctor_get(x_12, 0); -x_402 = l_Lake_Dependency_decodeToml___closed__3; -x_403 = lean_string_append(x_402, x_401); -lean_dec(x_401); -x_404 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_405 = lean_string_append(x_403, x_404); -lean_ctor_set(x_12, 0, x_405); -x_330 = x_12; -x_331 = x_398; -goto block_396; +x_896 = x_941; +x_897 = x_942; +goto block_940; } else { -lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; -x_406 = lean_ctor_get(x_12, 0); -lean_inc(x_406); -lean_dec(x_12); -x_407 = l_Lake_Dependency_decodeToml___closed__3; -x_408 = lean_string_append(x_407, x_406); -lean_dec(x_406); -x_409 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_410 = lean_string_append(x_408, x_409); -x_411 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_411, 0, x_410); -x_330 = x_411; -x_331 = x_398; -goto block_396; -} +lean_object* x_945; lean_object* x_946; +x_945 = lean_ctor_get(x_941, 0); +lean_inc(x_945); +lean_dec(x_941); +x_946 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_946, 0, x_945); +x_896 = x_946; +x_897 = x_942; +goto block_940; } } -else -{ -uint8_t x_412; -lean_dec(x_12); -x_412 = !lean_is_exclusive(x_397); -if (x_412 == 0) -{ -x_330 = x_397; -x_331 = x_398; -goto block_396; } -else +block_956: { -lean_object* x_413; lean_object* x_414; -x_413 = lean_ctor_get(x_397, 0); -lean_inc(x_413); -lean_dec(x_397); -x_414 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_414, 0, x_413); -x_330 = x_414; -x_331 = x_398; -goto block_396; -} -} +lean_object* x_952; lean_object* x_953; lean_object* x_954; lean_object* x_955; +x_952 = lean_box(0); +x_953 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_953, 0, x_951); +lean_ctor_set(x_953, 1, x_952); +x_954 = lean_array_mk(x_953); +x_955 = l_Array_append___rarg(x_396, x_954); +lean_dec(x_954); +x_941 = x_950; +x_942 = x_955; +goto block_947; } } else { -lean_object* x_482; lean_object* x_483; -x_482 = lean_ctor_get(x_329, 0); -lean_inc(x_482); -lean_dec(x_329); -x_483 = lean_ctor_get(x_482, 1); -lean_inc(x_483); -lean_dec(x_482); -switch (lean_obj_tag(x_483)) { +lean_object* x_987; lean_object* x_988; +x_987 = lean_ctor_get(x_895, 0); +lean_inc(x_987); +lean_dec(x_895); +x_988 = lean_ctor_get(x_987, 1); +lean_inc(x_988); +lean_dec(x_987); +switch (lean_obj_tag(x_988)) { case 0: { -lean_object* x_484; -x_484 = lean_ctor_get(x_483, 1); -lean_inc(x_484); -lean_dec(x_483); -x_191 = x_484; -x_192 = x_190; -goto block_326; +lean_object* x_989; +x_989 = lean_ctor_get(x_988, 1); +lean_inc(x_989); +lean_dec(x_988); +x_794 = x_989; +x_795 = x_396; +goto block_885; } case 2: { -lean_object* x_485; lean_object* x_486; lean_object* x_487; lean_object* x_488; lean_object* x_489; lean_object* x_490; lean_object* x_491; -x_485 = lean_ctor_get(x_483, 0); -lean_inc(x_485); -lean_dec(x_483); -x_486 = l_Lake_Glob_decodeToml___closed__2; -x_487 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_487, 0, x_485); -lean_ctor_set(x_487, 1, x_486); -x_488 = lean_unsigned_to_nat(1u); -x_489 = lean_mk_array(x_488, x_487); -x_490 = l_Array_append___rarg(x_190, x_489); -lean_dec(x_489); -x_491 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_191 = x_491; -x_192 = x_490; -goto block_326; +lean_object* x_990; lean_object* x_991; lean_object* x_992; +x_990 = lean_ctor_get(x_988, 0); +lean_inc(x_990); +lean_dec(x_988); +x_991 = l_Lake_Glob_decodeToml___closed__2; +x_992 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_992, 0, x_990); +lean_ctor_set(x_992, 1, x_991); +x_886 = x_992; +goto block_892; } case 3: { -lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; -x_492 = lean_ctor_get(x_483, 0); -lean_inc(x_492); -lean_dec(x_483); -x_493 = l_Lake_Glob_decodeToml___closed__2; -x_494 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_494, 0, x_492); -lean_ctor_set(x_494, 1, x_493); -x_495 = lean_unsigned_to_nat(1u); -x_496 = lean_mk_array(x_495, x_494); -x_497 = l_Array_append___rarg(x_190, x_496); -lean_dec(x_496); -x_498 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_191 = x_498; -x_192 = x_497; -goto block_326; +lean_object* x_993; lean_object* x_994; lean_object* x_995; +x_993 = lean_ctor_get(x_988, 0); +lean_inc(x_993); +lean_dec(x_988); +x_994 = l_Lake_Glob_decodeToml___closed__2; +x_995 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_995, 0, x_993); +lean_ctor_set(x_995, 1, x_994); +x_886 = x_995; +goto block_892; } default: { -uint8_t x_499; -x_499 = !lean_is_exclusive(x_483); -if (x_499 == 0) -{ -lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; -x_500 = lean_ctor_get(x_483, 1); -lean_dec(x_500); -x_501 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_483, 0); -lean_ctor_set(x_483, 1, x_501); -x_502 = lean_unsigned_to_nat(1u); -x_503 = lean_mk_array(x_502, x_483); -x_504 = l_Array_append___rarg(x_190, x_503); -lean_dec(x_503); -x_505 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_191 = x_505; -x_192 = x_504; -goto block_326; +uint8_t x_996; +x_996 = !lean_is_exclusive(x_988); +if (x_996 == 0) +{ +lean_object* x_997; lean_object* x_998; +x_997 = lean_ctor_get(x_988, 1); +lean_dec(x_997); +x_998 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_988, 0); +lean_ctor_set(x_988, 1, x_998); +x_886 = x_988; +goto block_892; } else { -lean_object* x_506; lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; -x_506 = lean_ctor_get(x_483, 0); -lean_inc(x_506); -lean_dec(x_483); -x_507 = l_Lake_Glob_decodeToml___closed__2; -x_508 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_508, 0, x_506); -lean_ctor_set(x_508, 1, x_507); -x_509 = lean_unsigned_to_nat(1u); -x_510 = lean_mk_array(x_509, x_508); -x_511 = l_Array_append___rarg(x_190, x_510); -lean_dec(x_510); -x_512 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_191 = x_512; -x_192 = x_511; -goto block_326; +lean_object* x_999; lean_object* x_1000; lean_object* x_1001; +x_999 = lean_ctor_get(x_988, 0); +lean_inc(x_999); +lean_dec(x_988); +x_1000 = l_Lake_Glob_decodeToml___closed__2; +x_1001 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1001, 0, x_999); +lean_ctor_set(x_1001, 1, x_1000); +x_886 = x_1001; +goto block_892; } } } } -block_326: +block_885: { -lean_object* x_193; lean_object* x_194; lean_object* x_252; lean_object* x_253; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; -x_271 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_272 = l_Lake_PackageConfig_decodeToml___closed__29; +lean_object* x_796; lean_object* x_797; lean_object* x_838; lean_object* x_839; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; +x_845 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_846 = l_Lake_PackageConfig_decodeToml___closed__29; lean_inc(x_1); -x_273 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_271, x_272, x_1); -x_274 = lean_box(0); -if (lean_obj_tag(x_273) == 0) +x_847 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_845, x_846, x_1); +x_848 = lean_box(0); +if (lean_obj_tag(x_847) == 0) { -x_252 = x_274; -x_253 = x_192; -goto block_270; +x_838 = x_848; +x_839 = x_795; +goto block_844; } else { -uint8_t x_275; -x_275 = !lean_is_exclusive(x_273); -if (x_275 == 0) +uint8_t x_855; +x_855 = !lean_is_exclusive(x_847); +if (x_855 == 0) { -lean_object* x_276; lean_object* x_277; -x_276 = lean_ctor_get(x_273, 0); -x_277 = lean_ctor_get(x_276, 1); -lean_inc(x_277); -lean_dec(x_276); -switch (lean_obj_tag(x_277)) { +lean_object* x_856; lean_object* x_857; +x_856 = lean_ctor_get(x_847, 0); +x_857 = lean_ctor_get(x_856, 1); +lean_inc(x_857); +lean_dec(x_856); +switch (lean_obj_tag(x_857)) { case 0: { -lean_object* x_278; -x_278 = lean_ctor_get(x_277, 1); -lean_inc(x_278); -lean_dec(x_277); -lean_ctor_set(x_273, 0, x_278); -x_252 = x_273; -x_253 = x_192; -goto block_270; +lean_object* x_858; +x_858 = lean_ctor_get(x_857, 1); +lean_inc(x_858); +lean_dec(x_857); +lean_ctor_set(x_847, 0, x_858); +x_838 = x_847; +x_839 = x_795; +goto block_844; } case 2: { -lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -lean_free_object(x_273); -x_279 = lean_ctor_get(x_277, 0); -lean_inc(x_279); -lean_dec(x_277); -x_280 = l_Lake_Glob_decodeToml___closed__2; -x_281 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_281, 0, x_279); -lean_ctor_set(x_281, 1, x_280); -x_282 = lean_unsigned_to_nat(1u); -x_283 = lean_mk_array(x_282, x_281); -x_284 = l_Array_append___rarg(x_192, x_283); -lean_dec(x_283); -x_252 = x_274; -x_253 = x_284; -goto block_270; +lean_object* x_859; lean_object* x_860; lean_object* x_861; +lean_free_object(x_847); +x_859 = lean_ctor_get(x_857, 0); +lean_inc(x_859); +lean_dec(x_857); +x_860 = l_Lake_Glob_decodeToml___closed__2; +x_861 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_861, 0, x_859); +lean_ctor_set(x_861, 1, x_860); +x_849 = x_861; +goto block_854; } case 3: { -lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; -lean_free_object(x_273); -x_285 = lean_ctor_get(x_277, 0); -lean_inc(x_285); -lean_dec(x_277); -x_286 = l_Lake_Glob_decodeToml___closed__2; -x_287 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_287, 0, x_285); -lean_ctor_set(x_287, 1, x_286); -x_288 = lean_unsigned_to_nat(1u); -x_289 = lean_mk_array(x_288, x_287); -x_290 = l_Array_append___rarg(x_192, x_289); -lean_dec(x_289); -x_252 = x_274; -x_253 = x_290; -goto block_270; +lean_object* x_862; lean_object* x_863; lean_object* x_864; +lean_free_object(x_847); +x_862 = lean_ctor_get(x_857, 0); +lean_inc(x_862); +lean_dec(x_857); +x_863 = l_Lake_Glob_decodeToml___closed__2; +x_864 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_864, 0, x_862); +lean_ctor_set(x_864, 1, x_863); +x_849 = x_864; +goto block_854; } default: { -uint8_t x_291; -lean_free_object(x_273); -x_291 = !lean_is_exclusive(x_277); -if (x_291 == 0) -{ -lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; -x_292 = lean_ctor_get(x_277, 1); -lean_dec(x_292); -x_293 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_277, 0); -lean_ctor_set(x_277, 1, x_293); -x_294 = lean_unsigned_to_nat(1u); -x_295 = lean_mk_array(x_294, x_277); -x_296 = l_Array_append___rarg(x_192, x_295); -lean_dec(x_295); -x_252 = x_274; -x_253 = x_296; -goto block_270; +uint8_t x_865; +lean_free_object(x_847); +x_865 = !lean_is_exclusive(x_857); +if (x_865 == 0) +{ +lean_object* x_866; lean_object* x_867; +x_866 = lean_ctor_get(x_857, 1); +lean_dec(x_866); +x_867 = l_Lake_Glob_decodeToml___closed__2; +lean_ctor_set_tag(x_857, 0); +lean_ctor_set(x_857, 1, x_867); +x_849 = x_857; +goto block_854; } else { -lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; -x_297 = lean_ctor_get(x_277, 0); -lean_inc(x_297); -lean_dec(x_277); -x_298 = l_Lake_Glob_decodeToml___closed__2; -x_299 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_299, 0, x_297); -lean_ctor_set(x_299, 1, x_298); -x_300 = lean_unsigned_to_nat(1u); -x_301 = lean_mk_array(x_300, x_299); -x_302 = l_Array_append___rarg(x_192, x_301); -lean_dec(x_301); -x_252 = x_274; -x_253 = x_302; -goto block_270; +lean_object* x_868; lean_object* x_869; lean_object* x_870; +x_868 = lean_ctor_get(x_857, 0); +lean_inc(x_868); +lean_dec(x_857); +x_869 = l_Lake_Glob_decodeToml___closed__2; +x_870 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_870, 0, x_868); +lean_ctor_set(x_870, 1, x_869); +x_849 = x_870; +goto block_854; } } } } else { -lean_object* x_303; lean_object* x_304; -x_303 = lean_ctor_get(x_273, 0); -lean_inc(x_303); -lean_dec(x_273); -x_304 = lean_ctor_get(x_303, 1); -lean_inc(x_304); -lean_dec(x_303); -switch (lean_obj_tag(x_304)) { +lean_object* x_871; lean_object* x_872; +x_871 = lean_ctor_get(x_847, 0); +lean_inc(x_871); +lean_dec(x_847); +x_872 = lean_ctor_get(x_871, 1); +lean_inc(x_872); +lean_dec(x_871); +switch (lean_obj_tag(x_872)) { case 0: { -lean_object* x_305; lean_object* x_306; -x_305 = lean_ctor_get(x_304, 1); -lean_inc(x_305); -lean_dec(x_304); -x_306 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_306, 0, x_305); -x_252 = x_306; -x_253 = x_192; -goto block_270; +lean_object* x_873; lean_object* x_874; +x_873 = lean_ctor_get(x_872, 1); +lean_inc(x_873); +lean_dec(x_872); +x_874 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_874, 0, x_873); +x_838 = x_874; +x_839 = x_795; +goto block_844; } case 2: { -lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; -x_307 = lean_ctor_get(x_304, 0); -lean_inc(x_307); -lean_dec(x_304); -x_308 = l_Lake_Glob_decodeToml___closed__2; -x_309 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_309, 0, x_307); -lean_ctor_set(x_309, 1, x_308); -x_310 = lean_unsigned_to_nat(1u); -x_311 = lean_mk_array(x_310, x_309); -x_312 = l_Array_append___rarg(x_192, x_311); -lean_dec(x_311); -x_252 = x_274; -x_253 = x_312; -goto block_270; +lean_object* x_875; lean_object* x_876; lean_object* x_877; +x_875 = lean_ctor_get(x_872, 0); +lean_inc(x_875); +lean_dec(x_872); +x_876 = l_Lake_Glob_decodeToml___closed__2; +x_877 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_877, 0, x_875); +lean_ctor_set(x_877, 1, x_876); +x_849 = x_877; +goto block_854; } case 3: { -lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; -x_313 = lean_ctor_get(x_304, 0); -lean_inc(x_313); -lean_dec(x_304); -x_314 = l_Lake_Glob_decodeToml___closed__2; -x_315 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_315, 0, x_313); -lean_ctor_set(x_315, 1, x_314); -x_316 = lean_unsigned_to_nat(1u); -x_317 = lean_mk_array(x_316, x_315); -x_318 = l_Array_append___rarg(x_192, x_317); -lean_dec(x_317); -x_252 = x_274; -x_253 = x_318; -goto block_270; +lean_object* x_878; lean_object* x_879; lean_object* x_880; +x_878 = lean_ctor_get(x_872, 0); +lean_inc(x_878); +lean_dec(x_872); +x_879 = l_Lake_Glob_decodeToml___closed__2; +x_880 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_880, 0, x_878); +lean_ctor_set(x_880, 1, x_879); +x_849 = x_880; +goto block_854; } default: { -lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; -x_319 = lean_ctor_get(x_304, 0); -lean_inc(x_319); -if (lean_is_exclusive(x_304)) { - lean_ctor_release(x_304, 0); - lean_ctor_release(x_304, 1); - x_320 = x_304; +lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; +x_881 = lean_ctor_get(x_872, 0); +lean_inc(x_881); +if (lean_is_exclusive(x_872)) { + lean_ctor_release(x_872, 0); + lean_ctor_release(x_872, 1); + x_882 = x_872; } else { - lean_dec_ref(x_304); - x_320 = lean_box(0); + lean_dec_ref(x_872); + x_882 = lean_box(0); } -x_321 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_320)) { - x_322 = lean_alloc_ctor(0, 2, 0); +x_883 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_882)) { + x_884 = lean_alloc_ctor(0, 2, 0); } else { - x_322 = x_320; - lean_ctor_set_tag(x_322, 0); -} -lean_ctor_set(x_322, 0, x_319); -lean_ctor_set(x_322, 1, x_321); -x_323 = lean_unsigned_to_nat(1u); -x_324 = lean_mk_array(x_323, x_322); -x_325 = l_Array_append___rarg(x_192, x_324); -lean_dec(x_324); -x_252 = x_274; -x_253 = x_325; -goto block_270; + x_884 = x_882; + lean_ctor_set_tag(x_884, 0); +} +lean_ctor_set(x_884, 0, x_881); +lean_ctor_set(x_884, 1, x_883); +x_849 = x_884; +goto block_854; } } } } -block_251: +block_837: { -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_195 = lean_box(0); -x_196 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_197 = l_Lake_Dependency_decodeToml___closed__2; -x_198 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_196, x_197, x_1); -if (lean_obj_tag(x_198) == 0) +lean_object* x_798; lean_object* x_799; lean_object* x_806; lean_object* x_807; lean_object* x_808; +x_798 = lean_box(0); +x_806 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_807 = l_Lake_Dependency_decodeToml___closed__2; +x_808 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_806, x_807, x_1); +if (lean_obj_tag(x_808) == 0) { -lean_object* x_199; -x_199 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_199, 0, x_11); -lean_ctor_set(x_199, 1, x_191); -lean_ctor_set(x_199, 2, x_193); -lean_ctor_set(x_199, 3, x_189); -lean_ctor_set(x_199, 4, x_195); -x_3 = x_199; -x_4 = x_194; +lean_object* x_809; +x_809 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_809, 0, x_11); +lean_ctor_set(x_809, 1, x_794); +lean_ctor_set(x_809, 2, x_796); +lean_ctor_set(x_809, 3, x_395); +lean_ctor_set(x_809, 4, x_798); +x_3 = x_809; +x_4 = x_797; goto block_8; } else { -lean_object* x_200; lean_object* x_201; -x_200 = lean_ctor_get(x_198, 0); -lean_inc(x_200); -lean_dec(x_198); -x_201 = lean_ctor_get(x_200, 1); -lean_inc(x_201); -lean_dec(x_200); -switch (lean_obj_tag(x_201)) { +lean_object* x_810; lean_object* x_811; +x_810 = lean_ctor_get(x_808, 0); +lean_inc(x_810); +lean_dec(x_808); +x_811 = lean_ctor_get(x_810, 1); +lean_inc(x_811); +lean_dec(x_810); +switch (lean_obj_tag(x_811)) { case 0: { -uint8_t x_202; -x_202 = !lean_is_exclusive(x_201); -if (x_202 == 0) +uint8_t x_812; +x_812 = !lean_is_exclusive(x_811); +if (x_812 == 0) { -lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_203 = lean_ctor_get(x_201, 1); -lean_dec(x_203); -x_204 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_201, 1, x_204); -x_205 = lean_unsigned_to_nat(1u); -x_206 = lean_mk_array(x_205, x_201); -x_207 = l_Array_append___rarg(x_194, x_206); -lean_dec(x_206); -x_208 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_208, 0, x_11); -lean_ctor_set(x_208, 1, x_191); -lean_ctor_set(x_208, 2, x_193); -lean_ctor_set(x_208, 3, x_189); -lean_ctor_set(x_208, 4, x_195); -x_3 = x_208; -x_4 = x_207; -goto block_8; +lean_object* x_813; lean_object* x_814; +x_813 = lean_ctor_get(x_811, 1); +lean_dec(x_813); +x_814 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_811, 1, x_814); +x_799 = x_811; +goto block_805; } else { -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; -x_209 = lean_ctor_get(x_201, 0); -lean_inc(x_209); -lean_dec(x_201); -x_210 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_211 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_211, 0, x_209); -lean_ctor_set(x_211, 1, x_210); -x_212 = lean_unsigned_to_nat(1u); -x_213 = lean_mk_array(x_212, x_211); -x_214 = l_Array_append___rarg(x_194, x_213); -lean_dec(x_213); -x_215 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_215, 0, x_11); -lean_ctor_set(x_215, 1, x_191); -lean_ctor_set(x_215, 2, x_193); -lean_ctor_set(x_215, 3, x_189); -lean_ctor_set(x_215, 4, x_195); -x_3 = x_215; -x_4 = x_214; -goto block_8; +lean_object* x_815; lean_object* x_816; lean_object* x_817; +x_815 = lean_ctor_get(x_811, 0); +lean_inc(x_815); +lean_dec(x_811); +x_816 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_817 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_817, 0, x_815); +lean_ctor_set(x_817, 1, x_816); +x_799 = x_817; +goto block_805; } } case 2: { -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; -x_216 = lean_ctor_get(x_201, 0); -lean_inc(x_216); -lean_dec(x_201); -x_217 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_218 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_218, 0, x_216); -lean_ctor_set(x_218, 1, x_217); -x_219 = lean_unsigned_to_nat(1u); -x_220 = lean_mk_array(x_219, x_218); -x_221 = l_Array_append___rarg(x_194, x_220); -lean_dec(x_220); -x_222 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_222, 0, x_11); -lean_ctor_set(x_222, 1, x_191); -lean_ctor_set(x_222, 2, x_193); -lean_ctor_set(x_222, 3, x_189); -lean_ctor_set(x_222, 4, x_195); -x_3 = x_222; -x_4 = x_221; -goto block_8; +lean_object* x_818; lean_object* x_819; lean_object* x_820; +x_818 = lean_ctor_get(x_811, 0); +lean_inc(x_818); +lean_dec(x_811); +x_819 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_820 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_820, 0, x_818); +lean_ctor_set(x_820, 1, x_819); +x_799 = x_820; +goto block_805; } case 3: { -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_223 = lean_ctor_get(x_201, 0); -lean_inc(x_223); -lean_dec(x_201); -x_224 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_225 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_225, 0, x_223); -lean_ctor_set(x_225, 1, x_224); -x_226 = lean_unsigned_to_nat(1u); -x_227 = lean_mk_array(x_226, x_225); -x_228 = l_Array_append___rarg(x_194, x_227); -lean_dec(x_227); -x_229 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_229, 0, x_11); -lean_ctor_set(x_229, 1, x_191); -lean_ctor_set(x_229, 2, x_193); -lean_ctor_set(x_229, 3, x_189); -lean_ctor_set(x_229, 4, x_195); -x_3 = x_229; -x_4 = x_228; -goto block_8; +lean_object* x_821; lean_object* x_822; lean_object* x_823; +x_821 = lean_ctor_get(x_811, 0); +lean_inc(x_821); +lean_dec(x_811); +x_822 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_823 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_823, 0, x_821); +lean_ctor_set(x_823, 1, x_822); +x_799 = x_823; +goto block_805; } case 6: { -lean_object* x_230; lean_object* x_231; -x_230 = lean_ctor_get(x_201, 1); -lean_inc(x_230); -lean_dec(x_201); -x_231 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_230); -lean_dec(x_230); -if (lean_obj_tag(x_231) == 0) +lean_object* x_824; lean_object* x_825; +x_824 = lean_ctor_get(x_811, 1); +lean_inc(x_824); +lean_dec(x_811); +x_825 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_824); +lean_dec(x_824); +if (lean_obj_tag(x_825) == 0) { -lean_object* x_232; lean_object* x_233; lean_object* x_234; -x_232 = lean_ctor_get(x_231, 0); -lean_inc(x_232); -lean_dec(x_231); -x_233 = l_Array_append___rarg(x_194, x_232); -lean_dec(x_232); -x_234 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_234, 0, x_11); -lean_ctor_set(x_234, 1, x_191); -lean_ctor_set(x_234, 2, x_193); -lean_ctor_set(x_234, 3, x_189); -lean_ctor_set(x_234, 4, x_195); -x_3 = x_234; -x_4 = x_233; +lean_object* x_826; lean_object* x_827; lean_object* x_828; +x_826 = lean_ctor_get(x_825, 0); +lean_inc(x_826); +lean_dec(x_825); +x_827 = l_Array_append___rarg(x_797, x_826); +lean_dec(x_826); +x_828 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_828, 0, x_11); +lean_ctor_set(x_828, 1, x_794); +lean_ctor_set(x_828, 2, x_796); +lean_ctor_set(x_828, 3, x_395); +lean_ctor_set(x_828, 4, x_798); +x_3 = x_828; +x_4 = x_827; goto block_8; } else { -lean_object* x_235; lean_object* x_236; -x_235 = lean_ctor_get(x_231, 0); -lean_inc(x_235); -lean_dec(x_231); -x_236 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_236, 0, x_11); -lean_ctor_set(x_236, 1, x_191); -lean_ctor_set(x_236, 2, x_193); -lean_ctor_set(x_236, 3, x_189); -lean_ctor_set(x_236, 4, x_235); -x_3 = x_236; -x_4 = x_194; +lean_object* x_829; lean_object* x_830; +x_829 = lean_ctor_get(x_825, 0); +lean_inc(x_829); +lean_dec(x_825); +x_830 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_830, 0, x_11); +lean_ctor_set(x_830, 1, x_794); +lean_ctor_set(x_830, 2, x_796); +lean_ctor_set(x_830, 3, x_395); +lean_ctor_set(x_830, 4, x_829); +x_3 = x_830; +x_4 = x_797; goto block_8; } } default: { -uint8_t x_237; -x_237 = !lean_is_exclusive(x_201); -if (x_237 == 0) +uint8_t x_831; +x_831 = !lean_is_exclusive(x_811); +if (x_831 == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; -x_238 = lean_ctor_get(x_201, 1); -lean_dec(x_238); -x_239 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set_tag(x_201, 0); -lean_ctor_set(x_201, 1, x_239); -x_240 = lean_unsigned_to_nat(1u); -x_241 = lean_mk_array(x_240, x_201); -x_242 = l_Array_append___rarg(x_194, x_241); -lean_dec(x_241); -x_243 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_243, 0, x_11); -lean_ctor_set(x_243, 1, x_191); -lean_ctor_set(x_243, 2, x_193); -lean_ctor_set(x_243, 3, x_189); -lean_ctor_set(x_243, 4, x_195); -x_3 = x_243; -x_4 = x_242; -goto block_8; +lean_object* x_832; lean_object* x_833; +x_832 = lean_ctor_get(x_811, 1); +lean_dec(x_832); +x_833 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set_tag(x_811, 0); +lean_ctor_set(x_811, 1, x_833); +x_799 = x_811; +goto block_805; } else { -lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_244 = lean_ctor_get(x_201, 0); -lean_inc(x_244); -lean_dec(x_201); -x_245 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_246 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_246, 0, x_244); -lean_ctor_set(x_246, 1, x_245); -x_247 = lean_unsigned_to_nat(1u); -x_248 = lean_mk_array(x_247, x_246); -x_249 = l_Array_append___rarg(x_194, x_248); -lean_dec(x_248); -x_250 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_250, 0, x_11); -lean_ctor_set(x_250, 1, x_191); -lean_ctor_set(x_250, 2, x_193); -lean_ctor_set(x_250, 3, x_189); -lean_ctor_set(x_250, 4, x_195); -x_3 = x_250; -x_4 = x_249; -goto block_8; -} +lean_object* x_834; lean_object* x_835; lean_object* x_836; +x_834 = lean_ctor_get(x_811, 0); +lean_inc(x_834); +lean_dec(x_811); +x_835 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_836 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_836, 0, x_834); +lean_ctor_set(x_836, 1, x_835); +x_799 = x_836; +goto block_805; } } } } -block_270: -{ -if (lean_obj_tag(x_252) == 0) -{ -if (lean_obj_tag(x_12) == 0) +block_805: { -lean_object* x_254; -x_254 = lean_box(0); -x_193 = x_254; -x_194 = x_253; -goto block_251; +lean_object* x_800; lean_object* x_801; lean_object* x_802; lean_object* x_803; lean_object* x_804; +x_800 = lean_box(0); +x_801 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_801, 0, x_799); +lean_ctor_set(x_801, 1, x_800); +x_802 = lean_array_mk(x_801); +x_803 = l_Array_append___rarg(x_797, x_802); +lean_dec(x_802); +x_804 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_804, 0, x_11); +lean_ctor_set(x_804, 1, x_794); +lean_ctor_set(x_804, 2, x_796); +lean_ctor_set(x_804, 3, x_395); +lean_ctor_set(x_804, 4, x_798); +x_3 = x_804; +x_4 = x_803; +goto block_8; } -else -{ -uint8_t x_255; -x_255 = !lean_is_exclusive(x_12); -if (x_255 == 0) -{ -lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; -x_256 = lean_ctor_get(x_12, 0); -x_257 = l_Lake_Dependency_decodeToml___closed__3; -x_258 = lean_string_append(x_257, x_256); -lean_dec(x_256); -x_259 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_260 = lean_string_append(x_258, x_259); -lean_ctor_set(x_12, 0, x_260); -x_193 = x_12; -x_194 = x_253; -goto block_251; } -else +block_844: { -lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -x_261 = lean_ctor_get(x_12, 0); -lean_inc(x_261); -lean_dec(x_12); -x_262 = l_Lake_Dependency_decodeToml___closed__3; -x_263 = lean_string_append(x_262, x_261); -lean_dec(x_261); -x_264 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_265 = lean_string_append(x_263, x_264); -x_266 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_266, 0, x_265); -x_193 = x_266; -x_194 = x_253; -goto block_251; -} -} +if (lean_obj_tag(x_838) == 0) +{ +lean_object* x_840; +x_840 = lean_box(0); +x_796 = x_840; +x_797 = x_839; +goto block_837; } else { -uint8_t x_267; -lean_dec(x_12); -x_267 = !lean_is_exclusive(x_252); -if (x_267 == 0) +uint8_t x_841; +x_841 = !lean_is_exclusive(x_838); +if (x_841 == 0) { -x_193 = x_252; -x_194 = x_253; -goto block_251; +x_796 = x_838; +x_797 = x_839; +goto block_837; } else { -lean_object* x_268; lean_object* x_269; -x_268 = lean_ctor_get(x_252, 0); -lean_inc(x_268); -lean_dec(x_252); -x_269 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_269, 0, x_268); -x_193 = x_269; -x_194 = x_253; -goto block_251; +lean_object* x_842; lean_object* x_843; +x_842 = lean_ctor_get(x_838, 0); +lean_inc(x_842); +lean_dec(x_838); +x_843 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_843, 0, x_842); +x_796 = x_843; +x_797 = x_839; +goto block_837; } } } +block_854: +{ +lean_object* x_850; lean_object* x_851; lean_object* x_852; lean_object* x_853; +x_850 = lean_box(0); +x_851 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_851, 0, x_849); +lean_ctor_set(x_851, 1, x_850); +x_852 = lean_array_mk(x_851); +x_853 = l_Array_append___rarg(x_795, x_852); +lean_dec(x_852); +x_838 = x_848; +x_839 = x_853; +goto block_844; } } -block_793: +block_892: { -if (lean_obj_tag(x_514) == 0) -{ -lean_object* x_516; lean_object* x_517; lean_object* x_518; -x_516 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_517 = l_Lake_Dependency_decodeToml___closed__6; +lean_object* x_887; lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; +x_887 = lean_box(0); +x_888 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_888, 0, x_886); +lean_ctor_set(x_888, 1, x_887); +x_889 = lean_array_mk(x_888); +x_890 = l_Array_append___rarg(x_396, x_889); +lean_dec(x_889); +x_891 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_794 = x_891; +x_795 = x_890; +goto block_885; +} +} +else +{ +lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; lean_object* x_1005; lean_object* x_1006; lean_object* x_1078; lean_object* x_1085; lean_object* x_1086; lean_object* x_1087; +x_1002 = lean_ctor_get(x_395, 0); +lean_inc(x_1002); +lean_dec(x_395); +x_1003 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_1003, 0, x_1002); +x_1004 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1004, 0, x_1003); +x_1085 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_1086 = l_Lake_Dependency_decodeToml___closed__5; lean_inc(x_1); -x_518 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_516, x_517, x_1); -if (lean_obj_tag(x_518) == 0) +x_1087 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1085, x_1086, x_1); +if (lean_obj_tag(x_1087) == 0) { -lean_object* x_519; lean_object* x_520; lean_object* x_521; -x_519 = l_Lake_Dependency_decodeToml___closed__8; +lean_object* x_1088; lean_object* x_1089; lean_object* x_1129; lean_object* x_1130; lean_object* x_1136; lean_object* x_1137; lean_object* x_1138; lean_object* x_1139; +x_1136 = l_Lake_PackageConfig_decodeToml___closed__29; lean_inc(x_1); -x_520 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_516, x_519, x_1); -x_521 = lean_box(0); -if (lean_obj_tag(x_520) == 0) +x_1137 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1085, x_1136, x_1); +x_1138 = lean_box(0); +if (lean_obj_tag(x_1137) == 0) { -x_14 = x_521; -x_15 = x_515; -goto block_188; +x_1088 = x_1138; +x_1089 = x_396; +goto block_1128; } else { -uint8_t x_522; -x_522 = !lean_is_exclusive(x_520); -if (x_522 == 0) -{ -lean_object* x_523; lean_object* x_524; -x_523 = lean_ctor_get(x_520, 0); -x_524 = lean_ctor_get(x_523, 1); -lean_inc(x_524); -lean_dec(x_523); -switch (lean_obj_tag(x_524)) { -case 0: -{ -uint8_t x_525; -lean_free_object(x_520); -x_525 = !lean_is_exclusive(x_524); -if (x_525 == 0) -{ -lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; lean_object* x_530; -x_526 = lean_ctor_get(x_524, 1); -lean_dec(x_526); -x_527 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_524, 1, x_527); -x_528 = lean_unsigned_to_nat(1u); -x_529 = lean_mk_array(x_528, x_524); -x_530 = l_Array_append___rarg(x_515, x_529); -lean_dec(x_529); -x_14 = x_521; -x_15 = x_530; -goto block_188; +lean_object* x_1145; lean_object* x_1146; lean_object* x_1147; +x_1145 = lean_ctor_get(x_1137, 0); +lean_inc(x_1145); +if (lean_is_exclusive(x_1137)) { + lean_ctor_release(x_1137, 0); + x_1146 = x_1137; +} else { + lean_dec_ref(x_1137); + x_1146 = lean_box(0); } -else +x_1147 = lean_ctor_get(x_1145, 1); +lean_inc(x_1147); +lean_dec(x_1145); +switch (lean_obj_tag(x_1147)) { +case 0: { -lean_object* x_531; lean_object* x_532; lean_object* x_533; lean_object* x_534; lean_object* x_535; lean_object* x_536; -x_531 = lean_ctor_get(x_524, 0); -lean_inc(x_531); -lean_dec(x_524); -x_532 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_533 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_533, 0, x_531); -lean_ctor_set(x_533, 1, x_532); -x_534 = lean_unsigned_to_nat(1u); -x_535 = lean_mk_array(x_534, x_533); -x_536 = l_Array_append___rarg(x_515, x_535); -lean_dec(x_535); -x_14 = x_521; -x_15 = x_536; -goto block_188; +lean_object* x_1148; lean_object* x_1149; +x_1148 = lean_ctor_get(x_1147, 1); +lean_inc(x_1148); +lean_dec(x_1147); +if (lean_is_scalar(x_1146)) { + x_1149 = lean_alloc_ctor(1, 1, 0); +} else { + x_1149 = x_1146; } +lean_ctor_set(x_1149, 0, x_1148); +x_1129 = x_1149; +x_1130 = x_396; +goto block_1135; } case 2: { -lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; -lean_free_object(x_520); -x_537 = lean_ctor_get(x_524, 0); -lean_inc(x_537); -lean_dec(x_524); -x_538 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_539 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_539, 0, x_537); -lean_ctor_set(x_539, 1, x_538); -x_540 = lean_unsigned_to_nat(1u); -x_541 = lean_mk_array(x_540, x_539); -x_542 = l_Array_append___rarg(x_515, x_541); -lean_dec(x_541); -x_14 = x_521; -x_15 = x_542; -goto block_188; +lean_object* x_1150; lean_object* x_1151; lean_object* x_1152; +lean_dec(x_1146); +x_1150 = lean_ctor_get(x_1147, 0); +lean_inc(x_1150); +lean_dec(x_1147); +x_1151 = l_Lake_Glob_decodeToml___closed__2; +x_1152 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1152, 0, x_1150); +lean_ctor_set(x_1152, 1, x_1151); +x_1139 = x_1152; +goto block_1144; } case 3: { -lean_object* x_543; lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; -lean_free_object(x_520); -x_543 = lean_ctor_get(x_524, 0); -lean_inc(x_543); -lean_dec(x_524); -x_544 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_545 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_545, 0, x_543); -lean_ctor_set(x_545, 1, x_544); -x_546 = lean_unsigned_to_nat(1u); -x_547 = lean_mk_array(x_546, x_545); -x_548 = l_Array_append___rarg(x_515, x_547); -lean_dec(x_547); -x_14 = x_521; -x_15 = x_548; -goto block_188; -} -case 6: -{ -lean_object* x_549; lean_object* x_550; lean_object* x_551; -x_549 = lean_ctor_get(x_524, 0); -lean_inc(x_549); -x_550 = lean_ctor_get(x_524, 1); -lean_inc(x_550); -lean_dec(x_524); -x_551 = l_Lake_DependencySrc_decodeToml(x_550, x_549); -if (lean_obj_tag(x_551) == 0) -{ -lean_object* x_552; lean_object* x_553; -lean_free_object(x_520); -x_552 = lean_ctor_get(x_551, 0); -lean_inc(x_552); -lean_dec(x_551); -x_553 = l_Array_append___rarg(x_515, x_552); -lean_dec(x_552); -x_14 = x_521; -x_15 = x_553; -goto block_188; -} -else -{ -lean_object* x_554; -x_554 = lean_ctor_get(x_551, 0); -lean_inc(x_554); -lean_dec(x_551); -lean_ctor_set(x_520, 0, x_554); -x_14 = x_520; -x_15 = x_515; -goto block_188; -} +lean_object* x_1153; lean_object* x_1154; lean_object* x_1155; +lean_dec(x_1146); +x_1153 = lean_ctor_get(x_1147, 0); +lean_inc(x_1153); +lean_dec(x_1147); +x_1154 = l_Lake_Glob_decodeToml___closed__2; +x_1155 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1155, 0, x_1153); +lean_ctor_set(x_1155, 1, x_1154); +x_1139 = x_1155; +goto block_1144; } default: { -uint8_t x_555; -lean_free_object(x_520); -x_555 = !lean_is_exclusive(x_524); -if (x_555 == 0) -{ -lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_559; lean_object* x_560; -x_556 = lean_ctor_get(x_524, 1); -lean_dec(x_556); -x_557 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set_tag(x_524, 0); -lean_ctor_set(x_524, 1, x_557); -x_558 = lean_unsigned_to_nat(1u); -x_559 = lean_mk_array(x_558, x_524); -x_560 = l_Array_append___rarg(x_515, x_559); -lean_dec(x_559); -x_14 = x_521; -x_15 = x_560; -goto block_188; -} -else -{ -lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; -x_561 = lean_ctor_get(x_524, 0); -lean_inc(x_561); -lean_dec(x_524); -x_562 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_563 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_563, 0, x_561); -lean_ctor_set(x_563, 1, x_562); -x_564 = lean_unsigned_to_nat(1u); -x_565 = lean_mk_array(x_564, x_563); -x_566 = l_Array_append___rarg(x_515, x_565); -lean_dec(x_565); -x_14 = x_521; -x_15 = x_566; -goto block_188; -} -} +lean_object* x_1156; lean_object* x_1157; lean_object* x_1158; lean_object* x_1159; +lean_dec(x_1146); +x_1156 = lean_ctor_get(x_1147, 0); +lean_inc(x_1156); +if (lean_is_exclusive(x_1147)) { + lean_ctor_release(x_1147, 0); + lean_ctor_release(x_1147, 1); + x_1157 = x_1147; +} else { + lean_dec_ref(x_1147); + x_1157 = lean_box(0); } +x_1158 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1157)) { + x_1159 = lean_alloc_ctor(0, 2, 0); +} else { + x_1159 = x_1157; + lean_ctor_set_tag(x_1159, 0); +} +lean_ctor_set(x_1159, 0, x_1156); +lean_ctor_set(x_1159, 1, x_1158); +x_1139 = x_1159; +goto block_1144; +} +} +} +block_1128: +{ +lean_object* x_1090; lean_object* x_1091; lean_object* x_1099; lean_object* x_1100; +x_1090 = lean_box(0); +x_1099 = l_Lake_Dependency_decodeToml___closed__2; +x_1100 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1085, x_1099, x_1); +if (lean_obj_tag(x_1100) == 0) +{ +lean_object* x_1101; lean_object* x_1102; +x_1101 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1102 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1102, 0, x_11); +lean_ctor_set(x_1102, 1, x_1101); +lean_ctor_set(x_1102, 2, x_1088); +lean_ctor_set(x_1102, 3, x_1004); +lean_ctor_set(x_1102, 4, x_1090); +x_3 = x_1102; +x_4 = x_1089; +goto block_8; } else { -lean_object* x_567; lean_object* x_568; -x_567 = lean_ctor_get(x_520, 0); -lean_inc(x_567); -lean_dec(x_520); -x_568 = lean_ctor_get(x_567, 1); -lean_inc(x_568); -lean_dec(x_567); -switch (lean_obj_tag(x_568)) { +lean_object* x_1103; lean_object* x_1104; +x_1103 = lean_ctor_get(x_1100, 0); +lean_inc(x_1103); +lean_dec(x_1100); +x_1104 = lean_ctor_get(x_1103, 1); +lean_inc(x_1104); +lean_dec(x_1103); +switch (lean_obj_tag(x_1104)) { case 0: { -lean_object* x_569; lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; -x_569 = lean_ctor_get(x_568, 0); -lean_inc(x_569); -if (lean_is_exclusive(x_568)) { - lean_ctor_release(x_568, 0); - lean_ctor_release(x_568, 1); - x_570 = x_568; +lean_object* x_1105; lean_object* x_1106; lean_object* x_1107; lean_object* x_1108; +x_1105 = lean_ctor_get(x_1104, 0); +lean_inc(x_1105); +if (lean_is_exclusive(x_1104)) { + lean_ctor_release(x_1104, 0); + lean_ctor_release(x_1104, 1); + x_1106 = x_1104; } else { - lean_dec_ref(x_568); - x_570 = lean_box(0); + lean_dec_ref(x_1104); + x_1106 = lean_box(0); } -x_571 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -if (lean_is_scalar(x_570)) { - x_572 = lean_alloc_ctor(0, 2, 0); +x_1107 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1106)) { + x_1108 = lean_alloc_ctor(0, 2, 0); } else { - x_572 = x_570; + x_1108 = x_1106; } -lean_ctor_set(x_572, 0, x_569); -lean_ctor_set(x_572, 1, x_571); -x_573 = lean_unsigned_to_nat(1u); -x_574 = lean_mk_array(x_573, x_572); -x_575 = l_Array_append___rarg(x_515, x_574); -lean_dec(x_574); -x_14 = x_521; -x_15 = x_575; -goto block_188; +lean_ctor_set(x_1108, 0, x_1105); +lean_ctor_set(x_1108, 1, x_1107); +x_1091 = x_1108; +goto block_1098; } case 2: { -lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; -x_576 = lean_ctor_get(x_568, 0); -lean_inc(x_576); -lean_dec(x_568); -x_577 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_578 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_578, 0, x_576); -lean_ctor_set(x_578, 1, x_577); -x_579 = lean_unsigned_to_nat(1u); -x_580 = lean_mk_array(x_579, x_578); -x_581 = l_Array_append___rarg(x_515, x_580); -lean_dec(x_580); -x_14 = x_521; -x_15 = x_581; -goto block_188; +lean_object* x_1109; lean_object* x_1110; lean_object* x_1111; +x_1109 = lean_ctor_get(x_1104, 0); +lean_inc(x_1109); +lean_dec(x_1104); +x_1110 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1111 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1111, 0, x_1109); +lean_ctor_set(x_1111, 1, x_1110); +x_1091 = x_1111; +goto block_1098; } case 3: { -lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; lean_object* x_587; -x_582 = lean_ctor_get(x_568, 0); -lean_inc(x_582); -lean_dec(x_568); -x_583 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_584 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_584, 0, x_582); -lean_ctor_set(x_584, 1, x_583); -x_585 = lean_unsigned_to_nat(1u); -x_586 = lean_mk_array(x_585, x_584); -x_587 = l_Array_append___rarg(x_515, x_586); -lean_dec(x_586); -x_14 = x_521; -x_15 = x_587; -goto block_188; +lean_object* x_1112; lean_object* x_1113; lean_object* x_1114; +x_1112 = lean_ctor_get(x_1104, 0); +lean_inc(x_1112); +lean_dec(x_1104); +x_1113 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1114 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1114, 0, x_1112); +lean_ctor_set(x_1114, 1, x_1113); +x_1091 = x_1114; +goto block_1098; } case 6: { -lean_object* x_588; lean_object* x_589; lean_object* x_590; -x_588 = lean_ctor_get(x_568, 0); -lean_inc(x_588); -x_589 = lean_ctor_get(x_568, 1); -lean_inc(x_589); -lean_dec(x_568); -x_590 = l_Lake_DependencySrc_decodeToml(x_589, x_588); -if (lean_obj_tag(x_590) == 0) -{ -lean_object* x_591; lean_object* x_592; -x_591 = lean_ctor_get(x_590, 0); -lean_inc(x_591); -lean_dec(x_590); -x_592 = l_Array_append___rarg(x_515, x_591); -lean_dec(x_591); -x_14 = x_521; -x_15 = x_592; -goto block_188; +lean_object* x_1115; lean_object* x_1116; +x_1115 = lean_ctor_get(x_1104, 1); +lean_inc(x_1115); +lean_dec(x_1104); +x_1116 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_1115); +lean_dec(x_1115); +if (lean_obj_tag(x_1116) == 0) +{ +lean_object* x_1117; lean_object* x_1118; lean_object* x_1119; lean_object* x_1120; +x_1117 = lean_ctor_get(x_1116, 0); +lean_inc(x_1117); +lean_dec(x_1116); +x_1118 = l_Array_append___rarg(x_1089, x_1117); +lean_dec(x_1117); +x_1119 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1120 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1120, 0, x_11); +lean_ctor_set(x_1120, 1, x_1119); +lean_ctor_set(x_1120, 2, x_1088); +lean_ctor_set(x_1120, 3, x_1004); +lean_ctor_set(x_1120, 4, x_1090); +x_3 = x_1120; +x_4 = x_1118; +goto block_8; } else { -lean_object* x_593; lean_object* x_594; -x_593 = lean_ctor_get(x_590, 0); -lean_inc(x_593); -lean_dec(x_590); -x_594 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_594, 0, x_593); -x_14 = x_594; -x_15 = x_515; -goto block_188; +lean_object* x_1121; lean_object* x_1122; lean_object* x_1123; +x_1121 = lean_ctor_get(x_1116, 0); +lean_inc(x_1121); +lean_dec(x_1116); +x_1122 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1123 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1123, 0, x_11); +lean_ctor_set(x_1123, 1, x_1122); +lean_ctor_set(x_1123, 2, x_1088); +lean_ctor_set(x_1123, 3, x_1004); +lean_ctor_set(x_1123, 4, x_1121); +x_3 = x_1123; +x_4 = x_1089; +goto block_8; } } default: { -lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; -x_595 = lean_ctor_get(x_568, 0); -lean_inc(x_595); -if (lean_is_exclusive(x_568)) { - lean_ctor_release(x_568, 0); - lean_ctor_release(x_568, 1); - x_596 = x_568; +lean_object* x_1124; lean_object* x_1125; lean_object* x_1126; lean_object* x_1127; +x_1124 = lean_ctor_get(x_1104, 0); +lean_inc(x_1124); +if (lean_is_exclusive(x_1104)) { + lean_ctor_release(x_1104, 0); + lean_ctor_release(x_1104, 1); + x_1125 = x_1104; } else { - lean_dec_ref(x_568); - x_596 = lean_box(0); + lean_dec_ref(x_1104); + x_1125 = lean_box(0); } -x_597 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -if (lean_is_scalar(x_596)) { - x_598 = lean_alloc_ctor(0, 2, 0); +x_1126 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1125)) { + x_1127 = lean_alloc_ctor(0, 2, 0); } else { - x_598 = x_596; - lean_ctor_set_tag(x_598, 0); -} -lean_ctor_set(x_598, 0, x_595); -lean_ctor_set(x_598, 1, x_597); -x_599 = lean_unsigned_to_nat(1u); -x_600 = lean_mk_array(x_599, x_598); -x_601 = l_Array_append___rarg(x_515, x_600); -lean_dec(x_600); -x_14 = x_521; -x_15 = x_601; -goto block_188; -} -} -} -} + x_1127 = x_1125; + lean_ctor_set_tag(x_1127, 0); +} +lean_ctor_set(x_1127, 0, x_1124); +lean_ctor_set(x_1127, 1, x_1126); +x_1091 = x_1127; +goto block_1098; +} +} +} +block_1098: +{ +lean_object* x_1092; lean_object* x_1093; lean_object* x_1094; lean_object* x_1095; lean_object* x_1096; lean_object* x_1097; +x_1092 = lean_box(0); +x_1093 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1093, 0, x_1091); +lean_ctor_set(x_1093, 1, x_1092); +x_1094 = lean_array_mk(x_1093); +x_1095 = l_Array_append___rarg(x_1089, x_1094); +lean_dec(x_1094); +x_1096 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1097 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1097, 0, x_11); +lean_ctor_set(x_1097, 1, x_1096); +lean_ctor_set(x_1097, 2, x_1088); +lean_ctor_set(x_1097, 3, x_1004); +lean_ctor_set(x_1097, 4, x_1090); +x_3 = x_1097; +x_4 = x_1095; +goto block_8; } -else -{ -lean_object* x_602; lean_object* x_603; lean_object* x_604; -x_602 = lean_ctor_get(x_518, 0); -lean_inc(x_602); -if (lean_is_exclusive(x_518)) { - lean_ctor_release(x_518, 0); - x_603 = x_518; -} else { - lean_dec_ref(x_518); - x_603 = lean_box(0); } -x_604 = lean_ctor_get(x_602, 1); -lean_inc(x_604); -lean_dec(x_602); -switch (lean_obj_tag(x_604)) { -case 0: -{ -uint8_t x_605; -x_605 = !lean_is_exclusive(x_604); -if (x_605 == 0) +block_1135: { -lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_613; lean_object* x_614; lean_object* x_615; -x_606 = lean_ctor_get(x_604, 1); -x_607 = lean_ctor_get(x_604, 0); -lean_dec(x_607); -x_613 = l_Lake_DependencySrc_decodeToml___closed__2; -lean_inc(x_1); -x_614 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_516, x_613, x_1); -x_615 = lean_box(0); -if (lean_obj_tag(x_614) == 0) +if (lean_obj_tag(x_1129) == 0) { -lean_free_object(x_604); -x_608 = x_615; -x_609 = x_515; -goto block_612; +lean_object* x_1131; +x_1131 = lean_box(0); +x_1088 = x_1131; +x_1089 = x_1130; +goto block_1128; } else { -uint8_t x_616; -x_616 = !lean_is_exclusive(x_614); -if (x_616 == 0) -{ -lean_object* x_617; lean_object* x_618; -x_617 = lean_ctor_get(x_614, 0); -x_618 = lean_ctor_get(x_617, 1); -lean_inc(x_618); -lean_dec(x_617); -switch (lean_obj_tag(x_618)) { -case 0: -{ -lean_object* x_619; -lean_free_object(x_604); -x_619 = lean_ctor_get(x_618, 1); -lean_inc(x_619); -lean_dec(x_618); -lean_ctor_set(x_614, 0, x_619); -x_608 = x_614; -x_609 = x_515; -goto block_612; -} -case 2: -{ -lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; -lean_free_object(x_614); -x_620 = lean_ctor_get(x_618, 0); -lean_inc(x_620); -lean_dec(x_618); -x_621 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_604, 1, x_621); -lean_ctor_set(x_604, 0, x_620); -x_622 = lean_unsigned_to_nat(1u); -x_623 = lean_mk_array(x_622, x_604); -x_624 = l_Array_append___rarg(x_515, x_623); -lean_dec(x_623); -x_608 = x_615; -x_609 = x_624; -goto block_612; +lean_object* x_1132; lean_object* x_1133; lean_object* x_1134; +x_1132 = lean_ctor_get(x_1129, 0); +lean_inc(x_1132); +if (lean_is_exclusive(x_1129)) { + lean_ctor_release(x_1129, 0); + x_1133 = x_1129; +} else { + lean_dec_ref(x_1129); + x_1133 = lean_box(0); } -case 3: -{ -lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; -lean_free_object(x_614); -x_625 = lean_ctor_get(x_618, 0); -lean_inc(x_625); -lean_dec(x_618); -x_626 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_604, 1, x_626); -lean_ctor_set(x_604, 0, x_625); -x_627 = lean_unsigned_to_nat(1u); -x_628 = lean_mk_array(x_627, x_604); -x_629 = l_Array_append___rarg(x_515, x_628); -lean_dec(x_628); -x_608 = x_615; -x_609 = x_629; -goto block_612; +if (lean_is_scalar(x_1133)) { + x_1134 = lean_alloc_ctor(1, 1, 0); +} else { + x_1134 = x_1133; } -default: -{ -uint8_t x_630; -lean_free_object(x_614); -lean_free_object(x_604); -x_630 = !lean_is_exclusive(x_618); -if (x_630 == 0) -{ -lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; lean_object* x_635; -x_631 = lean_ctor_get(x_618, 1); -lean_dec(x_631); -x_632 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_618, 0); -lean_ctor_set(x_618, 1, x_632); -x_633 = lean_unsigned_to_nat(1u); -x_634 = lean_mk_array(x_633, x_618); -x_635 = l_Array_append___rarg(x_515, x_634); -lean_dec(x_634); -x_608 = x_615; -x_609 = x_635; -goto block_612; -} -else -{ -lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; -x_636 = lean_ctor_get(x_618, 0); -lean_inc(x_636); -lean_dec(x_618); -x_637 = l_Lake_Glob_decodeToml___closed__2; -x_638 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_638, 0, x_636); -lean_ctor_set(x_638, 1, x_637); -x_639 = lean_unsigned_to_nat(1u); -x_640 = lean_mk_array(x_639, x_638); -x_641 = l_Array_append___rarg(x_515, x_640); -lean_dec(x_640); -x_608 = x_615; -x_609 = x_641; -goto block_612; +lean_ctor_set(x_1134, 0, x_1132); +x_1088 = x_1134; +x_1089 = x_1130; +goto block_1128; } } +block_1144: +{ +lean_object* x_1140; lean_object* x_1141; lean_object* x_1142; lean_object* x_1143; +x_1140 = lean_box(0); +x_1141 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1141, 0, x_1139); +lean_ctor_set(x_1141, 1, x_1140); +x_1142 = lean_array_mk(x_1141); +x_1143 = l_Array_append___rarg(x_396, x_1142); +lean_dec(x_1142); +x_1129 = x_1138; +x_1130 = x_1143; +goto block_1135; } } else { -lean_object* x_642; lean_object* x_643; -x_642 = lean_ctor_get(x_614, 0); -lean_inc(x_642); -lean_dec(x_614); -x_643 = lean_ctor_get(x_642, 1); -lean_inc(x_643); -lean_dec(x_642); -switch (lean_obj_tag(x_643)) { +lean_object* x_1160; lean_object* x_1161; +x_1160 = lean_ctor_get(x_1087, 0); +lean_inc(x_1160); +lean_dec(x_1087); +x_1161 = lean_ctor_get(x_1160, 1); +lean_inc(x_1161); +lean_dec(x_1160); +switch (lean_obj_tag(x_1161)) { case 0: { -lean_object* x_644; lean_object* x_645; -lean_free_object(x_604); -x_644 = lean_ctor_get(x_643, 1); -lean_inc(x_644); -lean_dec(x_643); -x_645 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_645, 0, x_644); -x_608 = x_645; -x_609 = x_515; -goto block_612; +lean_object* x_1162; +x_1162 = lean_ctor_get(x_1161, 1); +lean_inc(x_1162); +lean_dec(x_1161); +x_1005 = x_1162; +x_1006 = x_396; +goto block_1077; } case 2: { -lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; -x_646 = lean_ctor_get(x_643, 0); -lean_inc(x_646); -lean_dec(x_643); -x_647 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_604, 1, x_647); -lean_ctor_set(x_604, 0, x_646); -x_648 = lean_unsigned_to_nat(1u); -x_649 = lean_mk_array(x_648, x_604); -x_650 = l_Array_append___rarg(x_515, x_649); -lean_dec(x_649); -x_608 = x_615; -x_609 = x_650; -goto block_612; +lean_object* x_1163; lean_object* x_1164; lean_object* x_1165; +x_1163 = lean_ctor_get(x_1161, 0); +lean_inc(x_1163); +lean_dec(x_1161); +x_1164 = l_Lake_Glob_decodeToml___closed__2; +x_1165 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1165, 0, x_1163); +lean_ctor_set(x_1165, 1, x_1164); +x_1078 = x_1165; +goto block_1084; } case 3: { -lean_object* x_651; lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; -x_651 = lean_ctor_get(x_643, 0); -lean_inc(x_651); -lean_dec(x_643); -x_652 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set(x_604, 1, x_652); -lean_ctor_set(x_604, 0, x_651); -x_653 = lean_unsigned_to_nat(1u); -x_654 = lean_mk_array(x_653, x_604); -x_655 = l_Array_append___rarg(x_515, x_654); -lean_dec(x_654); -x_608 = x_615; -x_609 = x_655; -goto block_612; +lean_object* x_1166; lean_object* x_1167; lean_object* x_1168; +x_1166 = lean_ctor_get(x_1161, 0); +lean_inc(x_1166); +lean_dec(x_1161); +x_1167 = l_Lake_Glob_decodeToml___closed__2; +x_1168 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1168, 0, x_1166); +lean_ctor_set(x_1168, 1, x_1167); +x_1078 = x_1168; +goto block_1084; } default: { -lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; lean_object* x_661; lean_object* x_662; -lean_free_object(x_604); -x_656 = lean_ctor_get(x_643, 0); -lean_inc(x_656); -if (lean_is_exclusive(x_643)) { - lean_ctor_release(x_643, 0); - lean_ctor_release(x_643, 1); - x_657 = x_643; +lean_object* x_1169; lean_object* x_1170; lean_object* x_1171; lean_object* x_1172; +x_1169 = lean_ctor_get(x_1161, 0); +lean_inc(x_1169); +if (lean_is_exclusive(x_1161)) { + lean_ctor_release(x_1161, 0); + lean_ctor_release(x_1161, 1); + x_1170 = x_1161; } else { - lean_dec_ref(x_643); - x_657 = lean_box(0); + lean_dec_ref(x_1161); + x_1170 = lean_box(0); } -x_658 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_657)) { - x_659 = lean_alloc_ctor(0, 2, 0); +x_1171 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1170)) { + x_1172 = lean_alloc_ctor(0, 2, 0); } else { - x_659 = x_657; - lean_ctor_set_tag(x_659, 0); + x_1172 = x_1170; + lean_ctor_set_tag(x_1172, 0); } -lean_ctor_set(x_659, 0, x_656); -lean_ctor_set(x_659, 1, x_658); -x_660 = lean_unsigned_to_nat(1u); -x_661 = lean_mk_array(x_660, x_659); -x_662 = l_Array_append___rarg(x_515, x_661); -lean_dec(x_661); -x_608 = x_615; -x_609 = x_662; -goto block_612; +lean_ctor_set(x_1172, 0, x_1169); +lean_ctor_set(x_1172, 1, x_1171); +x_1078 = x_1172; +goto block_1084; } } } -} -block_612: -{ -lean_object* x_610; lean_object* x_611; -lean_inc(x_12); -x_610 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_610, 0, x_606); -lean_ctor_set(x_610, 1, x_12); -lean_ctor_set(x_610, 2, x_608); -if (lean_is_scalar(x_603)) { - x_611 = lean_alloc_ctor(1, 1, 0); -} else { - x_611 = x_603; -} -lean_ctor_set(x_611, 0, x_610); -x_14 = x_611; -x_15 = x_609; -goto block_188; -} -} -else +block_1077: { -lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_669; lean_object* x_670; lean_object* x_671; -x_663 = lean_ctor_get(x_604, 1); -lean_inc(x_663); -lean_dec(x_604); -x_669 = l_Lake_DependencySrc_decodeToml___closed__2; +lean_object* x_1007; lean_object* x_1008; lean_object* x_1045; lean_object* x_1046; lean_object* x_1052; lean_object* x_1053; lean_object* x_1054; lean_object* x_1055; lean_object* x_1056; +x_1052 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_1053 = l_Lake_PackageConfig_decodeToml___closed__29; lean_inc(x_1); -x_670 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_516, x_669, x_1); -x_671 = lean_box(0); -if (lean_obj_tag(x_670) == 0) +x_1054 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1052, x_1053, x_1); +x_1055 = lean_box(0); +if (lean_obj_tag(x_1054) == 0) { -x_664 = x_671; -x_665 = x_515; -goto block_668; +x_1045 = x_1055; +x_1046 = x_1006; +goto block_1051; } else { -lean_object* x_672; lean_object* x_673; lean_object* x_674; -x_672 = lean_ctor_get(x_670, 0); -lean_inc(x_672); -if (lean_is_exclusive(x_670)) { - lean_ctor_release(x_670, 0); - x_673 = x_670; +lean_object* x_1062; lean_object* x_1063; lean_object* x_1064; +x_1062 = lean_ctor_get(x_1054, 0); +lean_inc(x_1062); +if (lean_is_exclusive(x_1054)) { + lean_ctor_release(x_1054, 0); + x_1063 = x_1054; } else { - lean_dec_ref(x_670); - x_673 = lean_box(0); + lean_dec_ref(x_1054); + x_1063 = lean_box(0); } -x_674 = lean_ctor_get(x_672, 1); -lean_inc(x_674); -lean_dec(x_672); -switch (lean_obj_tag(x_674)) { +x_1064 = lean_ctor_get(x_1062, 1); +lean_inc(x_1064); +lean_dec(x_1062); +switch (lean_obj_tag(x_1064)) { case 0: { -lean_object* x_675; lean_object* x_676; -x_675 = lean_ctor_get(x_674, 1); -lean_inc(x_675); -lean_dec(x_674); -if (lean_is_scalar(x_673)) { - x_676 = lean_alloc_ctor(1, 1, 0); +lean_object* x_1065; lean_object* x_1066; +x_1065 = lean_ctor_get(x_1064, 1); +lean_inc(x_1065); +lean_dec(x_1064); +if (lean_is_scalar(x_1063)) { + x_1066 = lean_alloc_ctor(1, 1, 0); } else { - x_676 = x_673; + x_1066 = x_1063; } -lean_ctor_set(x_676, 0, x_675); -x_664 = x_676; -x_665 = x_515; -goto block_668; +lean_ctor_set(x_1066, 0, x_1065); +x_1045 = x_1066; +x_1046 = x_1006; +goto block_1051; } case 2: { -lean_object* x_677; lean_object* x_678; lean_object* x_679; lean_object* x_680; lean_object* x_681; lean_object* x_682; -lean_dec(x_673); -x_677 = lean_ctor_get(x_674, 0); -lean_inc(x_677); -lean_dec(x_674); -x_678 = l_Lake_Glob_decodeToml___closed__2; -x_679 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_679, 0, x_677); -lean_ctor_set(x_679, 1, x_678); -x_680 = lean_unsigned_to_nat(1u); -x_681 = lean_mk_array(x_680, x_679); -x_682 = l_Array_append___rarg(x_515, x_681); -lean_dec(x_681); -x_664 = x_671; -x_665 = x_682; -goto block_668; +lean_object* x_1067; lean_object* x_1068; lean_object* x_1069; +lean_dec(x_1063); +x_1067 = lean_ctor_get(x_1064, 0); +lean_inc(x_1067); +lean_dec(x_1064); +x_1068 = l_Lake_Glob_decodeToml___closed__2; +x_1069 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1069, 0, x_1067); +lean_ctor_set(x_1069, 1, x_1068); +x_1056 = x_1069; +goto block_1061; } case 3: { -lean_object* x_683; lean_object* x_684; lean_object* x_685; lean_object* x_686; lean_object* x_687; lean_object* x_688; -lean_dec(x_673); -x_683 = lean_ctor_get(x_674, 0); -lean_inc(x_683); -lean_dec(x_674); -x_684 = l_Lake_Glob_decodeToml___closed__2; -x_685 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_685, 0, x_683); -lean_ctor_set(x_685, 1, x_684); -x_686 = lean_unsigned_to_nat(1u); -x_687 = lean_mk_array(x_686, x_685); -x_688 = l_Array_append___rarg(x_515, x_687); -lean_dec(x_687); -x_664 = x_671; -x_665 = x_688; -goto block_668; +lean_object* x_1070; lean_object* x_1071; lean_object* x_1072; +lean_dec(x_1063); +x_1070 = lean_ctor_get(x_1064, 0); +lean_inc(x_1070); +lean_dec(x_1064); +x_1071 = l_Lake_Glob_decodeToml___closed__2; +x_1072 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1072, 0, x_1070); +lean_ctor_set(x_1072, 1, x_1071); +x_1056 = x_1072; +goto block_1061; } default: { -lean_object* x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; lean_object* x_694; lean_object* x_695; -lean_dec(x_673); -x_689 = lean_ctor_get(x_674, 0); -lean_inc(x_689); -if (lean_is_exclusive(x_674)) { - lean_ctor_release(x_674, 0); - lean_ctor_release(x_674, 1); - x_690 = x_674; +lean_object* x_1073; lean_object* x_1074; lean_object* x_1075; lean_object* x_1076; +lean_dec(x_1063); +x_1073 = lean_ctor_get(x_1064, 0); +lean_inc(x_1073); +if (lean_is_exclusive(x_1064)) { + lean_ctor_release(x_1064, 0); + lean_ctor_release(x_1064, 1); + x_1074 = x_1064; } else { - lean_dec_ref(x_674); - x_690 = lean_box(0); + lean_dec_ref(x_1064); + x_1074 = lean_box(0); } -x_691 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_690)) { - x_692 = lean_alloc_ctor(0, 2, 0); +x_1075 = l_Lake_Glob_decodeToml___closed__2; +if (lean_is_scalar(x_1074)) { + x_1076 = lean_alloc_ctor(0, 2, 0); } else { - x_692 = x_690; - lean_ctor_set_tag(x_692, 0); -} -lean_ctor_set(x_692, 0, x_689); -lean_ctor_set(x_692, 1, x_691); -x_693 = lean_unsigned_to_nat(1u); -x_694 = lean_mk_array(x_693, x_692); -x_695 = l_Array_append___rarg(x_515, x_694); -lean_dec(x_694); -x_664 = x_671; -x_665 = x_695; -goto block_668; -} -} + x_1076 = x_1074; + lean_ctor_set_tag(x_1076, 0); +} +lean_ctor_set(x_1076, 0, x_1073); +lean_ctor_set(x_1076, 1, x_1075); +x_1056 = x_1076; +goto block_1061; +} +} +} +block_1044: +{ +lean_object* x_1009; lean_object* x_1010; lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; +x_1009 = lean_box(0); +x_1017 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_1018 = l_Lake_Dependency_decodeToml___closed__2; +x_1019 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_1017, x_1018, x_1); +if (lean_obj_tag(x_1019) == 0) +{ +lean_object* x_1020; +x_1020 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1020, 0, x_11); +lean_ctor_set(x_1020, 1, x_1005); +lean_ctor_set(x_1020, 2, x_1007); +lean_ctor_set(x_1020, 3, x_1004); +lean_ctor_set(x_1020, 4, x_1009); +x_3 = x_1020; +x_4 = x_1008; +goto block_8; } -block_668: +else { -lean_object* x_666; lean_object* x_667; -lean_inc(x_12); -x_666 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_666, 0, x_663); -lean_ctor_set(x_666, 1, x_12); -lean_ctor_set(x_666, 2, x_664); -if (lean_is_scalar(x_603)) { - x_667 = lean_alloc_ctor(1, 1, 0); +lean_object* x_1021; lean_object* x_1022; +x_1021 = lean_ctor_get(x_1019, 0); +lean_inc(x_1021); +lean_dec(x_1019); +x_1022 = lean_ctor_get(x_1021, 1); +lean_inc(x_1022); +lean_dec(x_1021); +switch (lean_obj_tag(x_1022)) { +case 0: +{ +lean_object* x_1023; lean_object* x_1024; lean_object* x_1025; lean_object* x_1026; +x_1023 = lean_ctor_get(x_1022, 0); +lean_inc(x_1023); +if (lean_is_exclusive(x_1022)) { + lean_ctor_release(x_1022, 0); + lean_ctor_release(x_1022, 1); + x_1024 = x_1022; } else { - x_667 = x_603; -} -lean_ctor_set(x_667, 0, x_666); -x_14 = x_667; -x_15 = x_665; -goto block_188; + lean_dec_ref(x_1022); + x_1024 = lean_box(0); } +x_1025 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1024)) { + x_1026 = lean_alloc_ctor(0, 2, 0); +} else { + x_1026 = x_1024; } +lean_ctor_set(x_1026, 0, x_1023); +lean_ctor_set(x_1026, 1, x_1025); +x_1010 = x_1026; +goto block_1016; } case 2: { -lean_object* x_696; lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; -lean_dec(x_603); -x_696 = lean_ctor_get(x_604, 0); -lean_inc(x_696); -lean_dec(x_604); -x_697 = l_Lake_Dependency_decodeToml___closed__9; -x_698 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_698, 0, x_696); -lean_ctor_set(x_698, 1, x_697); -x_699 = lean_array_push(x_515, x_698); -x_700 = lean_box(0); -x_189 = x_700; -x_190 = x_699; -goto block_513; +lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; +x_1027 = lean_ctor_get(x_1022, 0); +lean_inc(x_1027); +lean_dec(x_1022); +x_1028 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1029 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1029, 0, x_1027); +lean_ctor_set(x_1029, 1, x_1028); +x_1010 = x_1029; +goto block_1016; } case 3: { -lean_object* x_701; lean_object* x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; -lean_dec(x_603); -x_701 = lean_ctor_get(x_604, 0); -lean_inc(x_701); -lean_dec(x_604); -x_702 = l_Lake_Dependency_decodeToml___closed__9; -x_703 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_703, 0, x_701); -lean_ctor_set(x_703, 1, x_702); -x_704 = lean_array_push(x_515, x_703); -x_705 = lean_box(0); -x_189 = x_705; -x_190 = x_704; -goto block_513; +lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; +x_1030 = lean_ctor_get(x_1022, 0); +lean_inc(x_1030); +lean_dec(x_1022); +x_1031 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_1032 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1032, 0, x_1030); +lean_ctor_set(x_1032, 1, x_1031); +x_1010 = x_1032; +goto block_1016; } case 6: { -lean_object* x_706; lean_object* x_707; lean_object* x_708; lean_object* x_709; lean_object* x_710; lean_object* x_771; lean_object* x_772; -x_706 = lean_ctor_get(x_604, 0); -lean_inc(x_706); -x_707 = lean_ctor_get(x_604, 1); -lean_inc(x_707); -if (lean_is_exclusive(x_604)) { - lean_ctor_release(x_604, 0); - lean_ctor_release(x_604, 1); - x_708 = x_604; -} else { - lean_dec_ref(x_604); - x_708 = lean_box(0); -} -x_771 = l_Lake_DependencySrc_decodeToml___closed__17; -lean_inc(x_707); -x_772 = l_Lake_Toml_Table_decode___at_Lake_PackageConfig_decodeToml___spec__3(x_707, x_771, x_706); -if (lean_obj_tag(x_772) == 0) -{ -lean_object* x_773; lean_object* x_774; lean_object* x_775; -x_773 = lean_ctor_get(x_772, 0); -lean_inc(x_773); -lean_dec(x_772); -x_774 = l_Array_append___rarg(x_515, x_773); -lean_dec(x_773); -x_775 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; -x_709 = x_775; -x_710 = x_774; -goto block_770; +lean_object* x_1033; lean_object* x_1034; +x_1033 = lean_ctor_get(x_1022, 1); +lean_inc(x_1033); +lean_dec(x_1022); +x_1034 = l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1(x_1033); +lean_dec(x_1033); +if (lean_obj_tag(x_1034) == 0) +{ +lean_object* x_1035; lean_object* x_1036; lean_object* x_1037; +x_1035 = lean_ctor_get(x_1034, 0); +lean_inc(x_1035); +lean_dec(x_1034); +x_1036 = l_Array_append___rarg(x_1008, x_1035); +lean_dec(x_1035); +x_1037 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1037, 0, x_11); +lean_ctor_set(x_1037, 1, x_1005); +lean_ctor_set(x_1037, 2, x_1007); +lean_ctor_set(x_1037, 3, x_1004); +lean_ctor_set(x_1037, 4, x_1009); +x_3 = x_1037; +x_4 = x_1036; +goto block_8; } else { -lean_object* x_776; -x_776 = lean_ctor_get(x_772, 0); -lean_inc(x_776); -lean_dec(x_772); -x_709 = x_776; -x_710 = x_515; -goto block_770; -} -block_770: -{ -lean_object* x_711; lean_object* x_712; lean_object* x_716; lean_object* x_717; lean_object* x_718; -x_716 = l_Lake_DependencySrc_decodeToml___closed__2; -x_717 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_516, x_716, x_707); -x_718 = lean_box(0); -if (lean_obj_tag(x_717) == 0) -{ -lean_dec(x_708); -x_711 = x_718; -x_712 = x_710; -goto block_715; +lean_object* x_1038; lean_object* x_1039; +x_1038 = lean_ctor_get(x_1034, 0); +lean_inc(x_1038); +lean_dec(x_1034); +x_1039 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1039, 0, x_11); +lean_ctor_set(x_1039, 1, x_1005); +lean_ctor_set(x_1039, 2, x_1007); +lean_ctor_set(x_1039, 3, x_1004); +lean_ctor_set(x_1039, 4, x_1038); +x_3 = x_1039; +x_4 = x_1008; +goto block_8; } -else -{ -uint8_t x_719; -x_719 = !lean_is_exclusive(x_717); -if (x_719 == 0) -{ -lean_object* x_720; lean_object* x_721; -x_720 = lean_ctor_get(x_717, 0); -x_721 = lean_ctor_get(x_720, 1); -lean_inc(x_721); -lean_dec(x_720); -switch (lean_obj_tag(x_721)) { -case 0: -{ -lean_object* x_722; -lean_dec(x_708); -x_722 = lean_ctor_get(x_721, 1); -lean_inc(x_722); -lean_dec(x_721); -lean_ctor_set(x_717, 0, x_722); -x_711 = x_717; -x_712 = x_710; -goto block_715; } -case 2: +default: { -lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; lean_object* x_728; -lean_free_object(x_717); -x_723 = lean_ctor_get(x_721, 0); -lean_inc(x_723); -lean_dec(x_721); -x_724 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_708)) { - x_725 = lean_alloc_ctor(0, 2, 0); +lean_object* x_1040; lean_object* x_1041; lean_object* x_1042; lean_object* x_1043; +x_1040 = lean_ctor_get(x_1022, 0); +lean_inc(x_1040); +if (lean_is_exclusive(x_1022)) { + lean_ctor_release(x_1022, 0); + lean_ctor_release(x_1022, 1); + x_1041 = x_1022; } else { - x_725 = x_708; - lean_ctor_set_tag(x_725, 0); -} -lean_ctor_set(x_725, 0, x_723); -lean_ctor_set(x_725, 1, x_724); -x_726 = lean_unsigned_to_nat(1u); -x_727 = lean_mk_array(x_726, x_725); -x_728 = l_Array_append___rarg(x_710, x_727); -lean_dec(x_727); -x_711 = x_718; -x_712 = x_728; -goto block_715; + lean_dec_ref(x_1022); + x_1041 = lean_box(0); } -case 3: -{ -lean_object* x_729; lean_object* x_730; lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; -lean_free_object(x_717); -x_729 = lean_ctor_get(x_721, 0); -lean_inc(x_729); -lean_dec(x_721); -x_730 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_708)) { - x_731 = lean_alloc_ctor(0, 2, 0); +x_1042 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +if (lean_is_scalar(x_1041)) { + x_1043 = lean_alloc_ctor(0, 2, 0); } else { - x_731 = x_708; - lean_ctor_set_tag(x_731, 0); -} -lean_ctor_set(x_731, 0, x_729); -lean_ctor_set(x_731, 1, x_730); -x_732 = lean_unsigned_to_nat(1u); -x_733 = lean_mk_array(x_732, x_731); -x_734 = l_Array_append___rarg(x_710, x_733); -lean_dec(x_733); -x_711 = x_718; -x_712 = x_734; -goto block_715; -} -default: -{ -uint8_t x_735; -lean_free_object(x_717); -lean_dec(x_708); -x_735 = !lean_is_exclusive(x_721); -if (x_735 == 0) -{ -lean_object* x_736; lean_object* x_737; lean_object* x_738; lean_object* x_739; lean_object* x_740; -x_736 = lean_ctor_get(x_721, 1); -lean_dec(x_736); -x_737 = l_Lake_Glob_decodeToml___closed__2; -lean_ctor_set_tag(x_721, 0); -lean_ctor_set(x_721, 1, x_737); -x_738 = lean_unsigned_to_nat(1u); -x_739 = lean_mk_array(x_738, x_721); -x_740 = l_Array_append___rarg(x_710, x_739); -lean_dec(x_739); -x_711 = x_718; -x_712 = x_740; -goto block_715; -} -else -{ -lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; -x_741 = lean_ctor_get(x_721, 0); -lean_inc(x_741); -lean_dec(x_721); -x_742 = l_Lake_Glob_decodeToml___closed__2; -x_743 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_743, 0, x_741); -lean_ctor_set(x_743, 1, x_742); -x_744 = lean_unsigned_to_nat(1u); -x_745 = lean_mk_array(x_744, x_743); -x_746 = l_Array_append___rarg(x_710, x_745); -lean_dec(x_745); -x_711 = x_718; -x_712 = x_746; -goto block_715; -} -} + x_1043 = x_1041; + lean_ctor_set_tag(x_1043, 0); } +lean_ctor_set(x_1043, 0, x_1040); +lean_ctor_set(x_1043, 1, x_1042); +x_1010 = x_1043; +goto block_1016; +} +} +} +block_1016: +{ +lean_object* x_1011; lean_object* x_1012; lean_object* x_1013; lean_object* x_1014; lean_object* x_1015; +x_1011 = lean_box(0); +x_1012 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1012, 0, x_1010); +lean_ctor_set(x_1012, 1, x_1011); +x_1013 = lean_array_mk(x_1012); +x_1014 = l_Array_append___rarg(x_1008, x_1013); +lean_dec(x_1013); +x_1015 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_1015, 0, x_11); +lean_ctor_set(x_1015, 1, x_1005); +lean_ctor_set(x_1015, 2, x_1007); +lean_ctor_set(x_1015, 3, x_1004); +lean_ctor_set(x_1015, 4, x_1009); +x_3 = x_1015; +x_4 = x_1014; +goto block_8; } -else -{ -lean_object* x_747; lean_object* x_748; -x_747 = lean_ctor_get(x_717, 0); -lean_inc(x_747); -lean_dec(x_717); -x_748 = lean_ctor_get(x_747, 1); -lean_inc(x_748); -lean_dec(x_747); -switch (lean_obj_tag(x_748)) { -case 0: -{ -lean_object* x_749; lean_object* x_750; -lean_dec(x_708); -x_749 = lean_ctor_get(x_748, 1); -lean_inc(x_749); -lean_dec(x_748); -x_750 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_750, 0, x_749); -x_711 = x_750; -x_712 = x_710; -goto block_715; } -case 2: +block_1051: { -lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; -x_751 = lean_ctor_get(x_748, 0); -lean_inc(x_751); -lean_dec(x_748); -x_752 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_708)) { - x_753 = lean_alloc_ctor(0, 2, 0); -} else { - x_753 = x_708; - lean_ctor_set_tag(x_753, 0); -} -lean_ctor_set(x_753, 0, x_751); -lean_ctor_set(x_753, 1, x_752); -x_754 = lean_unsigned_to_nat(1u); -x_755 = lean_mk_array(x_754, x_753); -x_756 = l_Array_append___rarg(x_710, x_755); -lean_dec(x_755); -x_711 = x_718; -x_712 = x_756; -goto block_715; -} -case 3: +if (lean_obj_tag(x_1045) == 0) { -lean_object* x_757; lean_object* x_758; lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; -x_757 = lean_ctor_get(x_748, 0); -lean_inc(x_757); -lean_dec(x_748); -x_758 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_708)) { - x_759 = lean_alloc_ctor(0, 2, 0); -} else { - x_759 = x_708; - lean_ctor_set_tag(x_759, 0); -} -lean_ctor_set(x_759, 0, x_757); -lean_ctor_set(x_759, 1, x_758); -x_760 = lean_unsigned_to_nat(1u); -x_761 = lean_mk_array(x_760, x_759); -x_762 = l_Array_append___rarg(x_710, x_761); -lean_dec(x_761); -x_711 = x_718; -x_712 = x_762; -goto block_715; +lean_object* x_1047; +x_1047 = lean_box(0); +x_1007 = x_1047; +x_1008 = x_1046; +goto block_1044; } -default: +else { -lean_object* x_763; lean_object* x_764; lean_object* x_765; lean_object* x_766; lean_object* x_767; lean_object* x_768; lean_object* x_769; -lean_dec(x_708); -x_763 = lean_ctor_get(x_748, 0); -lean_inc(x_763); -if (lean_is_exclusive(x_748)) { - lean_ctor_release(x_748, 0); - lean_ctor_release(x_748, 1); - x_764 = x_748; +lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; +x_1048 = lean_ctor_get(x_1045, 0); +lean_inc(x_1048); +if (lean_is_exclusive(x_1045)) { + lean_ctor_release(x_1045, 0); + x_1049 = x_1045; } else { - lean_dec_ref(x_748); - x_764 = lean_box(0); + lean_dec_ref(x_1045); + x_1049 = lean_box(0); } -x_765 = l_Lake_Glob_decodeToml___closed__2; -if (lean_is_scalar(x_764)) { - x_766 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_1049)) { + x_1050 = lean_alloc_ctor(1, 1, 0); } else { - x_766 = x_764; - lean_ctor_set_tag(x_766, 0); -} -lean_ctor_set(x_766, 0, x_763); -lean_ctor_set(x_766, 1, x_765); -x_767 = lean_unsigned_to_nat(1u); -x_768 = lean_mk_array(x_767, x_766); -x_769 = l_Array_append___rarg(x_710, x_768); -lean_dec(x_768); -x_711 = x_718; -x_712 = x_769; -goto block_715; -} -} -} + x_1050 = x_1049; } -block_715: -{ -lean_object* x_713; lean_object* x_714; -lean_inc(x_12); -x_713 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_713, 0, x_709); -lean_ctor_set(x_713, 1, x_12); -lean_ctor_set(x_713, 2, x_711); -if (lean_is_scalar(x_603)) { - x_714 = lean_alloc_ctor(1, 1, 0); -} else { - x_714 = x_603; +lean_ctor_set(x_1050, 0, x_1048); +x_1007 = x_1050; +x_1008 = x_1046; +goto block_1044; +} +} +block_1061: +{ +lean_object* x_1057; lean_object* x_1058; lean_object* x_1059; lean_object* x_1060; +x_1057 = lean_box(0); +x_1058 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1058, 0, x_1056); +lean_ctor_set(x_1058, 1, x_1057); +x_1059 = lean_array_mk(x_1058); +x_1060 = l_Array_append___rarg(x_1006, x_1059); +lean_dec(x_1059); +x_1045 = x_1055; +x_1046 = x_1060; +goto block_1051; +} +} +block_1084: +{ +lean_object* x_1079; lean_object* x_1080; lean_object* x_1081; lean_object* x_1082; lean_object* x_1083; +x_1079 = lean_box(0); +x_1080 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1080, 0, x_1078); +lean_ctor_set(x_1080, 1, x_1079); +x_1081 = lean_array_mk(x_1080); +x_1082 = l_Array_append___rarg(x_396, x_1081); +lean_dec(x_1081); +x_1083 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__3; +x_1005 = x_1083; +x_1006 = x_1082; +goto block_1077; } -lean_ctor_set(x_714, 0, x_713); -x_14 = x_714; -x_15 = x_712; -goto block_188; } } } -default: +block_1183: { -uint8_t x_777; -lean_dec(x_603); -x_777 = !lean_is_exclusive(x_604); -if (x_777 == 0) -{ -lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; -x_778 = lean_ctor_get(x_604, 1); -lean_dec(x_778); -x_779 = l_Lake_Dependency_decodeToml___closed__9; -lean_ctor_set_tag(x_604, 0); -lean_ctor_set(x_604, 1, x_779); -x_780 = lean_array_push(x_515, x_604); -x_781 = lean_box(0); -x_189 = x_781; -x_190 = x_780; -goto block_513; -} -else -{ -lean_object* x_782; lean_object* x_783; lean_object* x_784; lean_object* x_785; lean_object* x_786; -x_782 = lean_ctor_get(x_604, 0); -lean_inc(x_782); -lean_dec(x_604); -x_783 = l_Lake_Dependency_decodeToml___closed__9; -x_784 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_784, 0, x_782); -lean_ctor_set(x_784, 1, x_783); -x_785 = lean_array_push(x_515, x_784); -x_786 = lean_box(0); -x_189 = x_786; -x_190 = x_785; -goto block_513; -} -} -} +lean_object* x_1179; lean_object* x_1180; lean_object* x_1181; lean_object* x_1182; +x_1179 = lean_box(0); +x_1180 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1180, 0, x_1178); +lean_ctor_set(x_1180, 1, x_1179); +x_1181 = lean_array_mk(x_1180); +x_1182 = l_Array_append___rarg(x_13, x_1181); +lean_dec(x_1181); +x_395 = x_1177; +x_396 = x_1182; +goto block_1173; } } -else -{ -uint8_t x_787; -x_787 = !lean_is_exclusive(x_514); -if (x_787 == 0) -{ -lean_object* x_788; lean_object* x_789; -x_788 = lean_ctor_get(x_514, 0); -x_789 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_789, 0, x_788); -lean_ctor_set(x_514, 0, x_789); -x_14 = x_514; -x_15 = x_515; -goto block_188; -} -else +block_1610: { -lean_object* x_790; lean_object* x_791; lean_object* x_792; -x_790 = lean_ctor_get(x_514, 0); -lean_inc(x_790); -lean_dec(x_514); -x_791 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_791, 0, x_790); -x_792 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_792, 0, x_791); -x_14 = x_792; -x_15 = x_515; -goto block_188; -} -} -} +lean_object* x_1606; lean_object* x_1607; lean_object* x_1608; lean_object* x_1609; +x_1606 = lean_box(0); +x_1607 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1607, 0, x_1605); +lean_ctor_set(x_1607, 1, x_1606); +x_1608 = lean_array_mk(x_1607); +x_1609 = l_Array_append___rarg(x_10, x_1608); +lean_dec(x_1608); +x_12 = x_1604; +x_13 = x_1609; +goto block_1600; } } } @@ -21000,123 +24735,134 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependency(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_instDecodeTomlDependency___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); -x_15 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_15 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_1, 1); -lean_inc(x_27); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_1, 1); +lean_inc(x_21); lean_dec(x_1); -x_28 = l_Lake_Dependency_decodeToml(x_27, x_26); -return x_28; +x_22 = l_Lake_Dependency_decodeToml(x_21, x_20); +return x_22; } default: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_1); -if (x_29 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_1); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_1, 1); -lean_dec(x_30); -x_31 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_1, 1); +lean_dec(x_24); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_1); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_1, 1, x_25); +x_2 = x_1; +goto block_7; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_1, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); lean_dec(x_1); -x_36 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_2 = x_28; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } } +static lean_object* _init_l_Lake_instDecodeTomlDependency___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_instDecodeTomlDependency___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_instDecodeTomlDependency() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_instDecodeTomlDependency___closed__1; +return x_1; } } LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__1(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { @@ -22041,151 +25787,125 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_6); -if (x_9 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_6); +if (x_18 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_6, 1); -lean_dec(x_10); -x_11 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_6, 1, x_11); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_6); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_16 = l_Lake_mergeErrors___rarg(x_4, x_14, x_15); -x_2 = x_8; -x_4 = x_16; -goto _start; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_6, 1); +lean_dec(x_19); +x_20 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_6, 1, x_20); +x_9 = x_6; +goto block_17; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_18 = lean_ctor_get(x_6, 0); -lean_inc(x_18); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); lean_dec(x_6); -x_19 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_mk_array(x_21, x_20); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_25 = l_Lake_mergeErrors___rarg(x_4, x_23, x_24); -x_2 = x_8; -x_4 = x_25; -goto _start; +x_22 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_9 = x_23; +goto block_17; } } case 2: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_6, 0); +lean_inc(x_24); +lean_dec(x_6); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_9 = x_26; +goto block_17; +} +case 3: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; x_27 = lean_ctor_get(x_6, 0); lean_inc(x_27); lean_dec(x_6); -x_28 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_28 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); -x_30 = lean_unsigned_to_nat(1u); -x_31 = lean_mk_array(x_30, x_29); -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); -x_2 = x_8; -x_4 = x_34; -goto _start; -} -case 3: -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_36 = lean_ctor_get(x_6, 0); -lean_inc(x_36); -lean_dec(x_6); -x_37 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_mk_array(x_39, x_38); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -x_42 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_43 = l_Lake_mergeErrors___rarg(x_4, x_41, x_42); -x_2 = x_8; -x_4 = x_43; -goto _start; +x_9 = x_29; +goto block_17; } case 6: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = lean_ctor_get(x_6, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_6, 1); -lean_inc(x_46); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_6, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_6, 1); +lean_inc(x_31); lean_dec(x_6); -x_47 = l_Lake_Dependency_decodeToml(x_46, x_45); -x_48 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_49 = l_Lake_mergeErrors___rarg(x_4, x_47, x_48); +x_32 = l_Lake_Dependency_decodeToml(x_31, x_30); +x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); x_2 = x_8; -x_4 = x_49; +x_4 = x_34; goto _start; } default: { -uint8_t x_51; -x_51 = !lean_is_exclusive(x_6); -if (x_51 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_6); +if (x_36 == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_6, 1); -lean_dec(x_52); -x_53 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_6, 1); +lean_dec(x_37); +x_38 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_53); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_mk_array(x_54, x_6); -x_56 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_56, 0, x_55); -x_57 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_58 = l_Lake_mergeErrors___rarg(x_4, x_56, x_57); -x_2 = x_8; -x_4 = x_58; -goto _start; +lean_ctor_set(x_6, 1, x_38); +x_9 = x_6; +goto block_17; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_ctor_get(x_6, 0); -lean_inc(x_60); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_6, 0); +lean_inc(x_39); lean_dec(x_6); -x_61 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_mk_array(x_63, x_62); -x_65 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_67 = l_Lake_mergeErrors___rarg(x_4, x_65, x_66); -x_2 = x_8; -x_4 = x_67; -goto _start; +x_40 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_9 = x_41; +goto block_17; +} } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; } } else @@ -22262,151 +25982,125 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_6); -if (x_9 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_6); +if (x_18 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_6, 1); -lean_dec(x_10); -x_11 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_6, 1, x_11); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_6); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_16 = l_Lake_mergeErrors___rarg(x_4, x_14, x_15); -x_2 = x_8; -x_4 = x_16; -goto _start; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_6, 1); +lean_dec(x_19); +x_20 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_6, 1, x_20); +x_9 = x_6; +goto block_17; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_18 = lean_ctor_get(x_6, 0); -lean_inc(x_18); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); lean_dec(x_6); -x_19 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_mk_array(x_21, x_20); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_25 = l_Lake_mergeErrors___rarg(x_4, x_23, x_24); -x_2 = x_8; -x_4 = x_25; -goto _start; +x_22 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_9 = x_23; +goto block_17; } } case 2: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_6, 0); +lean_inc(x_24); +lean_dec(x_6); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_9 = x_26; +goto block_17; +} +case 3: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; x_27 = lean_ctor_get(x_6, 0); lean_inc(x_27); lean_dec(x_6); -x_28 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_28 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); -x_30 = lean_unsigned_to_nat(1u); -x_31 = lean_mk_array(x_30, x_29); -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); -x_2 = x_8; -x_4 = x_34; -goto _start; -} -case 3: -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_36 = lean_ctor_get(x_6, 0); -lean_inc(x_36); -lean_dec(x_6); -x_37 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_mk_array(x_39, x_38); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -x_42 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_43 = l_Lake_mergeErrors___rarg(x_4, x_41, x_42); -x_2 = x_8; -x_4 = x_43; -goto _start; +x_9 = x_29; +goto block_17; } case 6: -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = lean_ctor_get(x_6, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_6, 1); -lean_inc(x_46); +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_6, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_6, 1); +lean_inc(x_31); lean_dec(x_6); -x_47 = l_Lake_LeanExeConfig_decodeToml(x_46, x_45); -x_48 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_49 = l_Lake_mergeErrors___rarg(x_4, x_47, x_48); +x_32 = l_Lake_LeanExeConfig_decodeToml(x_31, x_30); +x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); x_2 = x_8; -x_4 = x_49; +x_4 = x_34; goto _start; } default: { -uint8_t x_51; -x_51 = !lean_is_exclusive(x_6); -if (x_51 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_6); +if (x_36 == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_6, 1); -lean_dec(x_52); -x_53 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_6, 1); +lean_dec(x_37); +x_38 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_53); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_mk_array(x_54, x_6); -x_56 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_56, 0, x_55); -x_57 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_58 = l_Lake_mergeErrors___rarg(x_4, x_56, x_57); -x_2 = x_8; -x_4 = x_58; -goto _start; +lean_ctor_set(x_6, 1, x_38); +x_9 = x_6; +goto block_17; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_ctor_get(x_6, 0); -lean_inc(x_60); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_6, 0); +lean_inc(x_39); lean_dec(x_6); -x_61 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_mk_array(x_63, x_62); -x_65 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_67 = l_Lake_mergeErrors___rarg(x_4, x_65, x_66); -x_2 = x_8; -x_4 = x_67; -goto _start; +x_40 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_9 = x_41; +goto block_17; +} } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; } } else @@ -22483,151 +26177,125 @@ uint8_t x_5; x_5 = lean_usize_dec_eq(x_2, x_3); if (x_5 == 0) { -lean_object* x_6; size_t x_7; size_t x_8; +lean_object* x_6; size_t x_7; size_t x_8; lean_object* x_9; x_6 = lean_array_uget(x_1, x_2); x_7 = 1; x_8 = lean_usize_add(x_2, x_7); switch (lean_obj_tag(x_6)) { case 0: { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_6); -if (x_9 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_6); +if (x_18 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_10 = lean_ctor_get(x_6, 1); -lean_dec(x_10); -x_11 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -lean_ctor_set(x_6, 1, x_11); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_6); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -x_15 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_16 = l_Lake_mergeErrors___rarg(x_4, x_14, x_15); -x_2 = x_8; -x_4 = x_16; -goto _start; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_6, 1); +lean_dec(x_19); +x_20 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +lean_ctor_set(x_6, 1, x_20); +x_9 = x_6; +goto block_17; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_18 = lean_ctor_get(x_6, 0); -lean_inc(x_18); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_6, 0); +lean_inc(x_21); lean_dec(x_6); -x_19 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_mk_array(x_21, x_20); -x_23 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_23, 0, x_22); -x_24 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_25 = l_Lake_mergeErrors___rarg(x_4, x_23, x_24); -x_2 = x_8; -x_4 = x_25; -goto _start; +x_22 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +x_9 = x_23; +goto block_17; } } case 2: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_6, 0); +lean_inc(x_24); +lean_dec(x_6); +x_25 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +x_9 = x_26; +goto block_17; +} +case 3: +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; x_27 = lean_ctor_get(x_6, 0); lean_inc(x_27); lean_dec(x_6); -x_28 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +x_28 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; x_29 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_29, 0, x_27); lean_ctor_set(x_29, 1, x_28); -x_30 = lean_unsigned_to_nat(1u); -x_31 = lean_mk_array(x_30, x_29); -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); -x_2 = x_8; -x_4 = x_34; -goto _start; -} -case 3: -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_36 = lean_ctor_get(x_6, 0); -lean_inc(x_36); -lean_dec(x_6); -x_37 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_mk_array(x_39, x_38); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -x_42 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_43 = l_Lake_mergeErrors___rarg(x_4, x_41, x_42); -x_2 = x_8; -x_4 = x_43; -goto _start; +x_9 = x_29; +goto block_17; } case 6: { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_45 = lean_ctor_get(x_6, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_6, 1); -lean_inc(x_46); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_6, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_6, 1); +lean_inc(x_31); lean_dec(x_6); -x_47 = l_Lake_LeanLibConfig_decodeToml(x_46, x_45); -x_48 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_49 = l_Lake_mergeErrors___rarg(x_4, x_47, x_48); +x_32 = l_Lake_LeanLibConfig_decodeToml(x_31, x_30); +x_33 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_34 = l_Lake_mergeErrors___rarg(x_4, x_32, x_33); x_2 = x_8; -x_4 = x_49; +x_4 = x_34; goto _start; } default: { -uint8_t x_51; -x_51 = !lean_is_exclusive(x_6); -if (x_51 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_6); +if (x_36 == 0) { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_52 = lean_ctor_get(x_6, 1); -lean_dec(x_52); -x_53 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_6, 1); +lean_dec(x_37); +x_38 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; lean_ctor_set_tag(x_6, 0); -lean_ctor_set(x_6, 1, x_53); -x_54 = lean_unsigned_to_nat(1u); -x_55 = lean_mk_array(x_54, x_6); -x_56 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_56, 0, x_55); -x_57 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_58 = l_Lake_mergeErrors___rarg(x_4, x_56, x_57); -x_2 = x_8; -x_4 = x_58; -goto _start; +lean_ctor_set(x_6, 1, x_38); +x_9 = x_6; +goto block_17; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_ctor_get(x_6, 0); -lean_inc(x_60); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_6, 0); +lean_inc(x_39); lean_dec(x_6); -x_61 = l_Lake_instDecodeTomlWorkspaceConfig___closed__1; -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_mk_array(x_63, x_62); -x_65 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; -x_67 = l_Lake_mergeErrors___rarg(x_4, x_65, x_66); -x_2 = x_8; -x_4 = x_67; -goto _start; +x_40 = l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_9 = x_41; +goto block_17; +} } } +block_17: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_13, 0, x_12); +x_14 = l_Array_foldlMUnsafe_fold___at_Lake_decodeLeanOptions___spec__2___closed__1; +x_15 = l_Lake_mergeErrors___rarg(x_4, x_13, x_14); +x_2 = x_8; +x_4 = x_15; +goto _start; } } else @@ -22889,94 +26557,94 @@ return x_9; LEAN_EXPORT lean_object* l_Lake_loadTomlConfig(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; lean_object* x_685; -x_680 = lean_ctor_get(x_1, 2); -lean_inc(x_680); -x_681 = lean_ctor_get(x_1, 3); -lean_inc(x_681); -x_682 = l_System_FilePath_join(x_680, x_681); -lean_dec(x_681); -x_683 = lean_ctor_get(x_1, 4); -lean_inc(x_683); -x_684 = l_System_FilePath_join(x_682, x_683); -lean_dec(x_683); -x_685 = l_IO_FS_readFile(x_684, x_3); -lean_dec(x_684); -if (lean_obj_tag(x_685) == 0) -{ -uint8_t x_686; -x_686 = !lean_is_exclusive(x_685); -if (x_686 == 0) -{ -lean_object* x_687; -x_687 = lean_ctor_get(x_685, 1); -lean_ctor_set(x_685, 1, x_2); -x_4 = x_685; -x_5 = x_687; -goto block_679; -} -else -{ -lean_object* x_688; lean_object* x_689; lean_object* x_690; -x_688 = lean_ctor_get(x_685, 0); -x_689 = lean_ctor_get(x_685, 1); -lean_inc(x_689); -lean_inc(x_688); -lean_dec(x_685); -x_690 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_690, 0, x_688); -lean_ctor_set(x_690, 1, x_2); -x_4 = x_690; -x_5 = x_689; -goto block_679; -} -} -else -{ -uint8_t x_691; -x_691 = !lean_is_exclusive(x_685); -if (x_691 == 0) -{ -lean_object* x_692; lean_object* x_693; lean_object* x_694; uint8_t x_695; lean_object* x_696; lean_object* x_697; lean_object* x_698; -x_692 = lean_ctor_get(x_685, 0); -x_693 = lean_ctor_get(x_685, 1); -x_694 = lean_io_error_to_string(x_692); -x_695 = 3; -x_696 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_696, 0, x_694); -lean_ctor_set_uint8(x_696, sizeof(void*)*1, x_695); -x_697 = lean_array_get_size(x_2); -x_698 = lean_array_push(x_2, x_696); -lean_ctor_set(x_685, 1, x_698); -lean_ctor_set(x_685, 0, x_697); -x_4 = x_685; -x_5 = x_693; -goto block_679; -} -else -{ -lean_object* x_699; lean_object* x_700; lean_object* x_701; uint8_t x_702; lean_object* x_703; lean_object* x_704; lean_object* x_705; lean_object* x_706; -x_699 = lean_ctor_get(x_685, 0); -x_700 = lean_ctor_get(x_685, 1); -lean_inc(x_700); -lean_inc(x_699); -lean_dec(x_685); -x_701 = lean_io_error_to_string(x_699); -x_702 = 3; -x_703 = lean_alloc_ctor(0, 1, 1); -lean_ctor_set(x_703, 0, x_701); -lean_ctor_set_uint8(x_703, sizeof(void*)*1, x_702); -x_704 = lean_array_get_size(x_2); -x_705 = lean_array_push(x_2, x_703); -x_706 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_706, 0, x_704); -lean_ctor_set(x_706, 1, x_705); -x_4 = x_706; -x_5 = x_700; -goto block_679; -} +lean_object* x_4; lean_object* x_5; lean_object* x_576; lean_object* x_577; lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; +x_576 = lean_ctor_get(x_1, 2); +lean_inc(x_576); +x_577 = lean_ctor_get(x_1, 3); +lean_inc(x_577); +x_578 = l_System_FilePath_join(x_576, x_577); +lean_dec(x_577); +x_579 = lean_ctor_get(x_1, 4); +lean_inc(x_579); +x_580 = l_System_FilePath_join(x_578, x_579); +lean_dec(x_579); +x_581 = l_IO_FS_readFile(x_580, x_3); +lean_dec(x_580); +if (lean_obj_tag(x_581) == 0) +{ +uint8_t x_582; +x_582 = !lean_is_exclusive(x_581); +if (x_582 == 0) +{ +lean_object* x_583; +x_583 = lean_ctor_get(x_581, 1); +lean_ctor_set(x_581, 1, x_2); +x_4 = x_581; +x_5 = x_583; +goto block_575; } -block_679: +else +{ +lean_object* x_584; lean_object* x_585; lean_object* x_586; +x_584 = lean_ctor_get(x_581, 0); +x_585 = lean_ctor_get(x_581, 1); +lean_inc(x_585); +lean_inc(x_584); +lean_dec(x_581); +x_586 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_586, 0, x_584); +lean_ctor_set(x_586, 1, x_2); +x_4 = x_586; +x_5 = x_585; +goto block_575; +} +} +else +{ +uint8_t x_587; +x_587 = !lean_is_exclusive(x_581); +if (x_587 == 0) +{ +lean_object* x_588; lean_object* x_589; lean_object* x_590; uint8_t x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; +x_588 = lean_ctor_get(x_581, 0); +x_589 = lean_ctor_get(x_581, 1); +x_590 = lean_io_error_to_string(x_588); +x_591 = 3; +x_592 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_592, 0, x_590); +lean_ctor_set_uint8(x_592, sizeof(void*)*1, x_591); +x_593 = lean_array_get_size(x_2); +x_594 = lean_array_push(x_2, x_592); +lean_ctor_set(x_581, 1, x_594); +lean_ctor_set(x_581, 0, x_593); +x_4 = x_581; +x_5 = x_589; +goto block_575; +} +else +{ +lean_object* x_595; lean_object* x_596; lean_object* x_597; uint8_t x_598; lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; +x_595 = lean_ctor_get(x_581, 0); +x_596 = lean_ctor_get(x_581, 1); +lean_inc(x_596); +lean_inc(x_595); +lean_dec(x_581); +x_597 = lean_io_error_to_string(x_595); +x_598 = 3; +x_599 = lean_alloc_ctor(0, 1, 1); +lean_ctor_set(x_599, 0, x_597); +lean_ctor_set_uint8(x_599, sizeof(void*)*1, x_598); +x_600 = lean_array_get_size(x_2); +x_601 = lean_array_push(x_2, x_599); +x_602 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_602, 0, x_600); +lean_ctor_set(x_602, 1, x_601); +x_4 = x_602; +x_5 = x_596; +goto block_575; +} +} +block_575: { if (lean_obj_tag(x_4) == 0) { @@ -22984,7 +26652,7 @@ uint8_t x_6; x_6 = !lean_is_exclusive(x_4); if (x_6 == 0) { -lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_363; +lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_295; x_7 = lean_ctor_get(x_4, 0); x_8 = lean_ctor_get(x_1, 4); lean_inc(x_8); @@ -22992,38 +26660,38 @@ x_9 = 1; lean_inc(x_8); x_10 = l_Lean_Parser_mkInputContext(x_7, x_8, x_9); lean_inc(x_10); -x_363 = l_Lake_Toml_loadToml(x_10, x_5); -if (lean_obj_tag(x_363) == 0) +x_295 = l_Lake_Toml_loadToml(x_10, x_5); +if (lean_obj_tag(x_295) == 0) { -lean_object* x_364; lean_object* x_365; lean_object* x_366; -x_364 = lean_ctor_get(x_363, 0); -lean_inc(x_364); -x_365 = lean_ctor_get(x_363, 1); -lean_inc(x_365); -lean_dec(x_363); -x_366 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_366, 0, x_364); -lean_ctor_set(x_4, 0, x_366); +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_298, 0, x_296); +lean_ctor_set(x_4, 0, x_298); x_11 = x_4; -x_12 = x_365; -goto block_362; +x_12 = x_297; +goto block_294; } else { -lean_object* x_367; lean_object* x_368; lean_object* x_369; -x_367 = lean_ctor_get(x_363, 0); -lean_inc(x_367); -x_368 = lean_ctor_get(x_363, 1); -lean_inc(x_368); -lean_dec(x_363); -x_369 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_369, 0, x_367); -lean_ctor_set(x_4, 0, x_369); +lean_object* x_299; lean_object* x_300; lean_object* x_301; +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +lean_dec(x_295); +x_301 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_301, 0, x_299); +lean_ctor_set(x_4, 0, x_301); x_11 = x_4; -x_12 = x_368; -goto block_362; +x_12 = x_300; +goto block_294; } -block_362: +block_294: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_13 = lean_ctor_get(x_11, 0); @@ -23206,748 +26874,608 @@ return x_77; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_354; lean_object* x_355; +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_286; lean_object* x_287; x_78 = lean_ctor_get(x_13, 0); lean_inc(x_78); lean_dec(x_13); -x_354 = lean_box(0); +x_286 = lean_box(0); lean_inc(x_78); -x_355 = l_Lake_PackageConfig_decodeToml(x_78, x_354); -if (lean_obj_tag(x_355) == 0) +x_287 = l_Lake_PackageConfig_decodeToml(x_78, x_286); +if (lean_obj_tag(x_287) == 0) { -lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; -x_356 = lean_ctor_get(x_355, 0); -lean_inc(x_356); -lean_dec(x_355); -x_357 = l_Lake_decodeLeanOptions___closed__1; -x_358 = l_Array_append___rarg(x_357, x_356); -lean_dec(x_356); -x_359 = l_Lake_loadTomlConfig___closed__11; -x_79 = x_359; -x_80 = x_358; -goto block_353; +lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +x_289 = l_Lake_decodeLeanOptions___closed__1; +x_290 = l_Array_append___rarg(x_289, x_288); +lean_dec(x_288); +x_291 = l_Lake_loadTomlConfig___closed__11; +x_79 = x_291; +x_80 = x_290; +goto block_285; } else { -lean_object* x_360; lean_object* x_361; -x_360 = lean_ctor_get(x_355, 0); -lean_inc(x_360); -lean_dec(x_355); -x_361 = l_Lake_decodeLeanOptions___closed__1; -x_79 = x_360; -x_80 = x_361; -goto block_353; -} -block_353: -{ -lean_object* x_81; lean_object* x_82; lean_object* x_287; lean_object* x_288; lean_object* x_299; lean_object* x_300; lean_object* x_301; -x_299 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_300 = l_Lake_loadTomlConfig___closed__9; +lean_object* x_292; lean_object* x_293; +x_292 = lean_ctor_get(x_287, 0); +lean_inc(x_292); +lean_dec(x_287); +x_293 = l_Lake_decodeLeanOptions___closed__1; +x_79 = x_292; +x_80 = x_293; +goto block_285; +} +block_285: +{ +lean_object* x_81; lean_object* x_82; lean_object* x_236; lean_object* x_237; lean_object* x_248; lean_object* x_249; lean_object* x_255; lean_object* x_256; lean_object* x_257; +x_248 = lean_box(0); +x_255 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_256 = l_Lake_loadTomlConfig___closed__9; lean_inc(x_78); -x_301 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_299, x_300, x_78); -if (lean_obj_tag(x_301) == 0) +x_257 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_255, x_256, x_78); +if (lean_obj_tag(x_257) == 0) { -lean_object* x_302; -x_302 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_302; -x_288 = x_80; -goto block_298; +lean_object* x_258; +x_258 = l_Lake_decodeLeanOptions___closed__1; +x_236 = x_258; +x_237 = x_80; +goto block_247; } else { -lean_object* x_303; lean_object* x_304; -x_303 = lean_ctor_get(x_301, 0); -lean_inc(x_303); -lean_dec(x_301); -x_304 = lean_ctor_get(x_303, 1); -lean_inc(x_304); -lean_dec(x_303); -switch (lean_obj_tag(x_304)) { +lean_object* x_259; lean_object* x_260; +x_259 = lean_ctor_get(x_257, 0); +lean_inc(x_259); +lean_dec(x_257); +x_260 = lean_ctor_get(x_259, 1); +lean_inc(x_260); +lean_dec(x_259); +switch (lean_obj_tag(x_260)) { case 0: { -uint8_t x_305; -x_305 = !lean_is_exclusive(x_304); -if (x_305 == 0) +uint8_t x_261; +x_261 = !lean_is_exclusive(x_260); +if (x_261 == 0) { -lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; -x_306 = lean_ctor_get(x_304, 1); -lean_dec(x_306); -x_307 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_304, 1, x_307); -x_308 = lean_unsigned_to_nat(1u); -x_309 = lean_mk_array(x_308, x_304); -x_310 = l_Array_append___rarg(x_80, x_309); -lean_dec(x_309); -x_311 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_311; -x_288 = x_310; -goto block_298; +lean_object* x_262; lean_object* x_263; +x_262 = lean_ctor_get(x_260, 1); +lean_dec(x_262); +x_263 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_260, 1, x_263); +x_249 = x_260; +goto block_254; } else { -lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; -x_312 = lean_ctor_get(x_304, 0); -lean_inc(x_312); -lean_dec(x_304); -x_313 = l_Lake_LeanConfig_decodeToml___closed__5; -x_314 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_314, 0, x_312); -lean_ctor_set(x_314, 1, x_313); -x_315 = lean_unsigned_to_nat(1u); -x_316 = lean_mk_array(x_315, x_314); -x_317 = l_Array_append___rarg(x_80, x_316); -lean_dec(x_316); -x_318 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_318; -x_288 = x_317; -goto block_298; +lean_object* x_264; lean_object* x_265; lean_object* x_266; +x_264 = lean_ctor_get(x_260, 0); +lean_inc(x_264); +lean_dec(x_260); +x_265 = l_Lake_LeanConfig_decodeToml___closed__5; +x_266 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_266, 0, x_264); +lean_ctor_set(x_266, 1, x_265); +x_249 = x_266; +goto block_254; } } case 2: { -lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; -x_319 = lean_ctor_get(x_304, 0); -lean_inc(x_319); -lean_dec(x_304); -x_320 = l_Lake_LeanConfig_decodeToml___closed__5; -x_321 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_321, 0, x_319); -lean_ctor_set(x_321, 1, x_320); -x_322 = lean_unsigned_to_nat(1u); -x_323 = lean_mk_array(x_322, x_321); -x_324 = l_Array_append___rarg(x_80, x_323); -lean_dec(x_323); -x_325 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_325; -x_288 = x_324; -goto block_298; +lean_object* x_267; lean_object* x_268; lean_object* x_269; +x_267 = lean_ctor_get(x_260, 0); +lean_inc(x_267); +lean_dec(x_260); +x_268 = l_Lake_LeanConfig_decodeToml___closed__5; +x_269 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_269, 0, x_267); +lean_ctor_set(x_269, 1, x_268); +x_249 = x_269; +goto block_254; } case 3: { -lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; -x_326 = lean_ctor_get(x_304, 0); -lean_inc(x_326); -lean_dec(x_304); -x_327 = l_Lake_LeanConfig_decodeToml___closed__5; -x_328 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_328, 0, x_326); -lean_ctor_set(x_328, 1, x_327); -x_329 = lean_unsigned_to_nat(1u); -x_330 = lean_mk_array(x_329, x_328); -x_331 = l_Array_append___rarg(x_80, x_330); -lean_dec(x_330); -x_332 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_332; -x_288 = x_331; -goto block_298; +lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_270 = lean_ctor_get(x_260, 0); +lean_inc(x_270); +lean_dec(x_260); +x_271 = l_Lake_LeanConfig_decodeToml___closed__5; +x_272 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_272, 0, x_270); +lean_ctor_set(x_272, 1, x_271); +x_249 = x_272; +goto block_254; } case 5: { -lean_object* x_333; lean_object* x_334; -x_333 = lean_ctor_get(x_304, 1); -lean_inc(x_333); -lean_dec(x_304); -x_334 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__15(x_333); -lean_dec(x_333); -if (lean_obj_tag(x_334) == 0) +lean_object* x_273; lean_object* x_274; +x_273 = lean_ctor_get(x_260, 1); +lean_inc(x_273); +lean_dec(x_260); +x_274 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__15(x_273); +lean_dec(x_273); +if (lean_obj_tag(x_274) == 0) { -lean_object* x_335; lean_object* x_336; lean_object* x_337; -x_335 = lean_ctor_get(x_334, 0); -lean_inc(x_335); -lean_dec(x_334); -x_336 = l_Array_append___rarg(x_80, x_335); -lean_dec(x_335); -x_337 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_337; -x_288 = x_336; -goto block_298; +lean_object* x_275; lean_object* x_276; lean_object* x_277; +x_275 = lean_ctor_get(x_274, 0); +lean_inc(x_275); +lean_dec(x_274); +x_276 = l_Array_append___rarg(x_80, x_275); +lean_dec(x_275); +x_277 = l_Lake_decodeLeanOptions___closed__1; +x_236 = x_277; +x_237 = x_276; +goto block_247; } else { -lean_object* x_338; -x_338 = lean_ctor_get(x_334, 0); -lean_inc(x_338); -lean_dec(x_334); -x_287 = x_338; -x_288 = x_80; -goto block_298; +lean_object* x_278; +x_278 = lean_ctor_get(x_274, 0); +lean_inc(x_278); +lean_dec(x_274); +x_236 = x_278; +x_237 = x_80; +goto block_247; } } default: { -uint8_t x_339; -x_339 = !lean_is_exclusive(x_304); -if (x_339 == 0) -{ -lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; -x_340 = lean_ctor_get(x_304, 1); -lean_dec(x_340); -x_341 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_304, 0); -lean_ctor_set(x_304, 1, x_341); -x_342 = lean_unsigned_to_nat(1u); -x_343 = lean_mk_array(x_342, x_304); -x_344 = l_Array_append___rarg(x_80, x_343); -lean_dec(x_343); -x_345 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_345; -x_288 = x_344; -goto block_298; +uint8_t x_279; +x_279 = !lean_is_exclusive(x_260); +if (x_279 == 0) +{ +lean_object* x_280; lean_object* x_281; +x_280 = lean_ctor_get(x_260, 1); +lean_dec(x_280); +x_281 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_260, 0); +lean_ctor_set(x_260, 1, x_281); +x_249 = x_260; +goto block_254; } else { -lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; -x_346 = lean_ctor_get(x_304, 0); -lean_inc(x_346); -lean_dec(x_304); -x_347 = l_Lake_LeanConfig_decodeToml___closed__5; -x_348 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_348, 0, x_346); -lean_ctor_set(x_348, 1, x_347); -x_349 = lean_unsigned_to_nat(1u); -x_350 = lean_mk_array(x_349, x_348); -x_351 = l_Array_append___rarg(x_80, x_350); -lean_dec(x_350); -x_352 = l_Lake_decodeLeanOptions___closed__1; -x_287 = x_352; -x_288 = x_351; -goto block_298; +lean_object* x_282; lean_object* x_283; lean_object* x_284; +x_282 = lean_ctor_get(x_260, 0); +lean_inc(x_282); +lean_dec(x_260); +x_283 = l_Lake_LeanConfig_decodeToml___closed__5; +x_284 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_284, 0, x_282); +lean_ctor_set(x_284, 1, x_283); +x_249 = x_284; +goto block_254; } } } } -block_286: +block_235: { -lean_object* x_83; lean_object* x_84; lean_object* x_220; lean_object* x_221; lean_object* x_232; lean_object* x_233; lean_object* x_234; -x_232 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_233 = l_Lake_loadTomlConfig___closed__7; +lean_object* x_83; lean_object* x_84; lean_object* x_186; lean_object* x_187; lean_object* x_198; lean_object* x_199; lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_198 = lean_box(0); +x_205 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_206 = l_Lake_loadTomlConfig___closed__7; lean_inc(x_78); -x_234 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_232, x_233, x_78); -if (lean_obj_tag(x_234) == 0) +x_207 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_205, x_206, x_78); +if (lean_obj_tag(x_207) == 0) { -lean_object* x_235; -x_235 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_235; -x_221 = x_82; -goto block_231; +lean_object* x_208; +x_208 = l_Lake_decodeLeanOptions___closed__1; +x_186 = x_208; +x_187 = x_82; +goto block_197; } else { -lean_object* x_236; lean_object* x_237; -x_236 = lean_ctor_get(x_234, 0); -lean_inc(x_236); -lean_dec(x_234); -x_237 = lean_ctor_get(x_236, 1); -lean_inc(x_237); -lean_dec(x_236); -switch (lean_obj_tag(x_237)) { +lean_object* x_209; lean_object* x_210; +x_209 = lean_ctor_get(x_207, 0); +lean_inc(x_209); +lean_dec(x_207); +x_210 = lean_ctor_get(x_209, 1); +lean_inc(x_210); +lean_dec(x_209); +switch (lean_obj_tag(x_210)) { case 0: { -uint8_t x_238; -x_238 = !lean_is_exclusive(x_237); -if (x_238 == 0) +uint8_t x_211; +x_211 = !lean_is_exclusive(x_210); +if (x_211 == 0) { -lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -x_239 = lean_ctor_get(x_237, 1); -lean_dec(x_239); -x_240 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_237, 1, x_240); -x_241 = lean_unsigned_to_nat(1u); -x_242 = lean_mk_array(x_241, x_237); -x_243 = l_Array_append___rarg(x_82, x_242); -lean_dec(x_242); -x_244 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_244; -x_221 = x_243; -goto block_231; +lean_object* x_212; lean_object* x_213; +x_212 = lean_ctor_get(x_210, 1); +lean_dec(x_212); +x_213 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_210, 1, x_213); +x_199 = x_210; +goto block_204; } else { -lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; -x_245 = lean_ctor_get(x_237, 0); -lean_inc(x_245); -lean_dec(x_237); -x_246 = l_Lake_LeanConfig_decodeToml___closed__5; -x_247 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_247, 0, x_245); -lean_ctor_set(x_247, 1, x_246); -x_248 = lean_unsigned_to_nat(1u); -x_249 = lean_mk_array(x_248, x_247); -x_250 = l_Array_append___rarg(x_82, x_249); -lean_dec(x_249); -x_251 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_251; -x_221 = x_250; -goto block_231; +lean_object* x_214; lean_object* x_215; lean_object* x_216; +x_214 = lean_ctor_get(x_210, 0); +lean_inc(x_214); +lean_dec(x_210); +x_215 = l_Lake_LeanConfig_decodeToml___closed__5; +x_216 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_216, 0, x_214); +lean_ctor_set(x_216, 1, x_215); +x_199 = x_216; +goto block_204; } } case 2: { -lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; -x_252 = lean_ctor_get(x_237, 0); -lean_inc(x_252); -lean_dec(x_237); -x_253 = l_Lake_LeanConfig_decodeToml___closed__5; -x_254 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_254, 0, x_252); -lean_ctor_set(x_254, 1, x_253); -x_255 = lean_unsigned_to_nat(1u); -x_256 = lean_mk_array(x_255, x_254); -x_257 = l_Array_append___rarg(x_82, x_256); -lean_dec(x_256); -x_258 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_258; -x_221 = x_257; -goto block_231; +lean_object* x_217; lean_object* x_218; lean_object* x_219; +x_217 = lean_ctor_get(x_210, 0); +lean_inc(x_217); +lean_dec(x_210); +x_218 = l_Lake_LeanConfig_decodeToml___closed__5; +x_219 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_219, 0, x_217); +lean_ctor_set(x_219, 1, x_218); +x_199 = x_219; +goto block_204; } case 3: { -lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; -x_259 = lean_ctor_get(x_237, 0); -lean_inc(x_259); -lean_dec(x_237); -x_260 = l_Lake_LeanConfig_decodeToml___closed__5; -x_261 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_261, 0, x_259); -lean_ctor_set(x_261, 1, x_260); -x_262 = lean_unsigned_to_nat(1u); -x_263 = lean_mk_array(x_262, x_261); -x_264 = l_Array_append___rarg(x_82, x_263); -lean_dec(x_263); -x_265 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_265; -x_221 = x_264; -goto block_231; +lean_object* x_220; lean_object* x_221; lean_object* x_222; +x_220 = lean_ctor_get(x_210, 0); +lean_inc(x_220); +lean_dec(x_210); +x_221 = l_Lake_LeanConfig_decodeToml___closed__5; +x_222 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_222, 0, x_220); +lean_ctor_set(x_222, 1, x_221); +x_199 = x_222; +goto block_204; } case 5: { -lean_object* x_266; lean_object* x_267; -x_266 = lean_ctor_get(x_237, 1); -lean_inc(x_266); -lean_dec(x_237); -x_267 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__12(x_266); -lean_dec(x_266); -if (lean_obj_tag(x_267) == 0) +lean_object* x_223; lean_object* x_224; +x_223 = lean_ctor_get(x_210, 1); +lean_inc(x_223); +lean_dec(x_210); +x_224 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__12(x_223); +lean_dec(x_223); +if (lean_obj_tag(x_224) == 0) { -lean_object* x_268; lean_object* x_269; lean_object* x_270; -x_268 = lean_ctor_get(x_267, 0); -lean_inc(x_268); -lean_dec(x_267); -x_269 = l_Array_append___rarg(x_82, x_268); -lean_dec(x_268); -x_270 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_270; -x_221 = x_269; -goto block_231; +lean_object* x_225; lean_object* x_226; lean_object* x_227; +x_225 = lean_ctor_get(x_224, 0); +lean_inc(x_225); +lean_dec(x_224); +x_226 = l_Array_append___rarg(x_82, x_225); +lean_dec(x_225); +x_227 = l_Lake_decodeLeanOptions___closed__1; +x_186 = x_227; +x_187 = x_226; +goto block_197; } else { -lean_object* x_271; -x_271 = lean_ctor_get(x_267, 0); -lean_inc(x_271); -lean_dec(x_267); -x_220 = x_271; -x_221 = x_82; -goto block_231; +lean_object* x_228; +x_228 = lean_ctor_get(x_224, 0); +lean_inc(x_228); +lean_dec(x_224); +x_186 = x_228; +x_187 = x_82; +goto block_197; } } default: { -uint8_t x_272; -x_272 = !lean_is_exclusive(x_237); -if (x_272 == 0) +uint8_t x_229; +x_229 = !lean_is_exclusive(x_210); +if (x_229 == 0) { -lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; -x_273 = lean_ctor_get(x_237, 1); -lean_dec(x_273); -x_274 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_237, 0); -lean_ctor_set(x_237, 1, x_274); -x_275 = lean_unsigned_to_nat(1u); -x_276 = lean_mk_array(x_275, x_237); -x_277 = l_Array_append___rarg(x_82, x_276); -lean_dec(x_276); -x_278 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_278; -x_221 = x_277; -goto block_231; +lean_object* x_230; lean_object* x_231; +x_230 = lean_ctor_get(x_210, 1); +lean_dec(x_230); +x_231 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_210, 0); +lean_ctor_set(x_210, 1, x_231); +x_199 = x_210; +goto block_204; } else { -lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; -x_279 = lean_ctor_get(x_237, 0); -lean_inc(x_279); -lean_dec(x_237); -x_280 = l_Lake_LeanConfig_decodeToml___closed__5; -x_281 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_281, 0, x_279); -lean_ctor_set(x_281, 1, x_280); -x_282 = lean_unsigned_to_nat(1u); -x_283 = lean_mk_array(x_282, x_281); -x_284 = l_Array_append___rarg(x_82, x_283); -lean_dec(x_283); -x_285 = l_Lake_decodeLeanOptions___closed__1; -x_220 = x_285; -x_221 = x_284; -goto block_231; +lean_object* x_232; lean_object* x_233; lean_object* x_234; +x_232 = lean_ctor_get(x_210, 0); +lean_inc(x_232); +lean_dec(x_210); +x_233 = l_Lake_LeanConfig_decodeToml___closed__5; +x_234 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_234, 0, x_232); +lean_ctor_set(x_234, 1, x_233); +x_199 = x_234; +goto block_204; } } } } -block_219: +block_185: { -lean_object* x_85; lean_object* x_86; lean_object* x_165; lean_object* x_166; lean_object* x_167; -x_165 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_166 = l_Lake_loadTomlConfig___closed__5; +lean_object* x_85; lean_object* x_86; lean_object* x_148; lean_object* x_149; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_148 = lean_box(0); +x_155 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_156 = l_Lake_loadTomlConfig___closed__5; lean_inc(x_78); -x_167 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_165, x_166, x_78); -if (lean_obj_tag(x_167) == 0) +x_157 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_155, x_156, x_78); +if (lean_obj_tag(x_157) == 0) { -lean_object* x_168; -x_168 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_168; +lean_object* x_158; +x_158 = l_Lake_decodeLeanOptions___closed__1; +x_85 = x_158; x_86 = x_84; -goto block_164; +goto block_147; } else { -lean_object* x_169; lean_object* x_170; -x_169 = lean_ctor_get(x_167, 0); -lean_inc(x_169); -lean_dec(x_167); -x_170 = lean_ctor_get(x_169, 1); -lean_inc(x_170); -lean_dec(x_169); -switch (lean_obj_tag(x_170)) { +lean_object* x_159; lean_object* x_160; +x_159 = lean_ctor_get(x_157, 0); +lean_inc(x_159); +lean_dec(x_157); +x_160 = lean_ctor_get(x_159, 1); +lean_inc(x_160); +lean_dec(x_159); +switch (lean_obj_tag(x_160)) { case 0: { -uint8_t x_171; -x_171 = !lean_is_exclusive(x_170); -if (x_171 == 0) +uint8_t x_161; +x_161 = !lean_is_exclusive(x_160); +if (x_161 == 0) { -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; -x_172 = lean_ctor_get(x_170, 1); -lean_dec(x_172); -x_173 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_170, 1, x_173); -x_174 = lean_unsigned_to_nat(1u); -x_175 = lean_mk_array(x_174, x_170); -x_176 = l_Array_append___rarg(x_84, x_175); -lean_dec(x_175); -x_177 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_177; -x_86 = x_176; -goto block_164; +lean_object* x_162; lean_object* x_163; +x_162 = lean_ctor_get(x_160, 1); +lean_dec(x_162); +x_163 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_160, 1, x_163); +x_149 = x_160; +goto block_154; } else { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_178 = lean_ctor_get(x_170, 0); -lean_inc(x_178); -lean_dec(x_170); -x_179 = l_Lake_LeanConfig_decodeToml___closed__5; -x_180 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_180, 0, x_178); -lean_ctor_set(x_180, 1, x_179); -x_181 = lean_unsigned_to_nat(1u); -x_182 = lean_mk_array(x_181, x_180); -x_183 = l_Array_append___rarg(x_84, x_182); -lean_dec(x_182); -x_184 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_184; -x_86 = x_183; -goto block_164; +lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +lean_dec(x_160); +x_165 = l_Lake_LeanConfig_decodeToml___closed__5; +x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_166, 0, x_164); +lean_ctor_set(x_166, 1, x_165); +x_149 = x_166; +goto block_154; } } case 2: { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_185 = lean_ctor_get(x_170, 0); -lean_inc(x_185); -lean_dec(x_170); -x_186 = l_Lake_LeanConfig_decodeToml___closed__5; -x_187 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -x_188 = lean_unsigned_to_nat(1u); -x_189 = lean_mk_array(x_188, x_187); -x_190 = l_Array_append___rarg(x_84, x_189); -lean_dec(x_189); -x_191 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_191; -x_86 = x_190; -goto block_164; +lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_167 = lean_ctor_get(x_160, 0); +lean_inc(x_167); +lean_dec(x_160); +x_168 = l_Lake_LeanConfig_decodeToml___closed__5; +x_169 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_169, 0, x_167); +lean_ctor_set(x_169, 1, x_168); +x_149 = x_169; +goto block_154; } case 3: { -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_192 = lean_ctor_get(x_170, 0); -lean_inc(x_192); -lean_dec(x_170); -x_193 = l_Lake_LeanConfig_decodeToml___closed__5; -x_194 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_194, 0, x_192); -lean_ctor_set(x_194, 1, x_193); -x_195 = lean_unsigned_to_nat(1u); -x_196 = lean_mk_array(x_195, x_194); -x_197 = l_Array_append___rarg(x_84, x_196); -lean_dec(x_196); -x_198 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_198; -x_86 = x_197; -goto block_164; +lean_object* x_170; lean_object* x_171; lean_object* x_172; +x_170 = lean_ctor_get(x_160, 0); +lean_inc(x_170); +lean_dec(x_160); +x_171 = l_Lake_LeanConfig_decodeToml___closed__5; +x_172 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_172, 0, x_170); +lean_ctor_set(x_172, 1, x_171); +x_149 = x_172; +goto block_154; } case 5: { -lean_object* x_199; lean_object* x_200; -x_199 = lean_ctor_get(x_170, 1); -lean_inc(x_199); -lean_dec(x_170); -x_200 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_199); -lean_dec(x_199); -if (lean_obj_tag(x_200) == 0) +lean_object* x_173; lean_object* x_174; +x_173 = lean_ctor_get(x_160, 1); +lean_inc(x_173); +lean_dec(x_160); +x_174 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_173); +lean_dec(x_173); +if (lean_obj_tag(x_174) == 0) { -lean_object* x_201; lean_object* x_202; lean_object* x_203; -x_201 = lean_ctor_get(x_200, 0); -lean_inc(x_201); -lean_dec(x_200); -x_202 = l_Array_append___rarg(x_84, x_201); -lean_dec(x_201); -x_203 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_203; -x_86 = x_202; -goto block_164; +lean_object* x_175; lean_object* x_176; lean_object* x_177; +x_175 = lean_ctor_get(x_174, 0); +lean_inc(x_175); +lean_dec(x_174); +x_176 = l_Array_append___rarg(x_84, x_175); +lean_dec(x_175); +x_177 = l_Lake_decodeLeanOptions___closed__1; +x_85 = x_177; +x_86 = x_176; +goto block_147; } else { -lean_object* x_204; -x_204 = lean_ctor_get(x_200, 0); -lean_inc(x_204); -lean_dec(x_200); -x_85 = x_204; +lean_object* x_178; +x_178 = lean_ctor_get(x_174, 0); +lean_inc(x_178); +lean_dec(x_174); +x_85 = x_178; x_86 = x_84; -goto block_164; +goto block_147; } } default: { -uint8_t x_205; -x_205 = !lean_is_exclusive(x_170); -if (x_205 == 0) +uint8_t x_179; +x_179 = !lean_is_exclusive(x_160); +if (x_179 == 0) { -lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; -x_206 = lean_ctor_get(x_170, 1); -lean_dec(x_206); -x_207 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_170, 0); -lean_ctor_set(x_170, 1, x_207); -x_208 = lean_unsigned_to_nat(1u); -x_209 = lean_mk_array(x_208, x_170); -x_210 = l_Array_append___rarg(x_84, x_209); -lean_dec(x_209); -x_211 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_211; -x_86 = x_210; -goto block_164; +lean_object* x_180; lean_object* x_181; +x_180 = lean_ctor_get(x_160, 1); +lean_dec(x_180); +x_181 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_160, 0); +lean_ctor_set(x_160, 1, x_181); +x_149 = x_160; +goto block_154; } else { -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; -x_212 = lean_ctor_get(x_170, 0); -lean_inc(x_212); -lean_dec(x_170); -x_213 = l_Lake_LeanConfig_decodeToml___closed__5; -x_214 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_214, 0, x_212); -lean_ctor_set(x_214, 1, x_213); -x_215 = lean_unsigned_to_nat(1u); -x_216 = lean_mk_array(x_215, x_214); -x_217 = l_Array_append___rarg(x_84, x_216); -lean_dec(x_216); -x_218 = l_Lake_decodeLeanOptions___closed__1; -x_85 = x_218; -x_86 = x_217; -goto block_164; +lean_object* x_182; lean_object* x_183; lean_object* x_184; +x_182 = lean_ctor_get(x_160, 0); +lean_inc(x_182); +lean_dec(x_160); +x_183 = l_Lake_LeanConfig_decodeToml___closed__5; +x_184 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_184, 0, x_182); +lean_ctor_set(x_184, 1, x_183); +x_149 = x_184; +goto block_154; } } } } -block_164: +block_147: { -size_t x_87; size_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_110; lean_object* x_111; lean_object* x_112; +size_t x_87; size_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_110; lean_object* x_111; lean_object* x_117; lean_object* x_118; lean_object* x_119; x_87 = lean_array_size(x_85); x_88 = 0; x_89 = l_Array_mapMUnsafe_map___at_Lake_loadTomlConfig___spec__8(x_87, x_88, x_85); -x_110 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_111 = l_Lake_loadTomlConfig___closed__3; -x_112 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_110, x_111, x_78); -if (lean_obj_tag(x_112) == 0) -{ -lean_object* x_113; -x_113 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_113; +x_110 = lean_box(0); +x_117 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_118 = l_Lake_loadTomlConfig___closed__3; +x_119 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_117, x_118, x_78); +if (lean_obj_tag(x_119) == 0) +{ +lean_object* x_120; +x_120 = l_Lake_decodeLeanOptions___closed__1; +x_90 = x_120; x_91 = x_86; goto block_109; } else { -lean_object* x_114; lean_object* x_115; -x_114 = lean_ctor_get(x_112, 0); -lean_inc(x_114); -lean_dec(x_112); -x_115 = lean_ctor_get(x_114, 1); -lean_inc(x_115); -lean_dec(x_114); -switch (lean_obj_tag(x_115)) { +lean_object* x_121; lean_object* x_122; +x_121 = lean_ctor_get(x_119, 0); +lean_inc(x_121); +lean_dec(x_119); +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +lean_dec(x_121); +switch (lean_obj_tag(x_122)) { case 0: { -uint8_t x_116; -x_116 = !lean_is_exclusive(x_115); -if (x_116 == 0) +uint8_t x_123; +x_123 = !lean_is_exclusive(x_122); +if (x_123 == 0) { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_117 = lean_ctor_get(x_115, 1); -lean_dec(x_117); -x_118 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set(x_115, 1, x_118); -x_119 = lean_unsigned_to_nat(1u); -x_120 = lean_mk_array(x_119, x_115); -x_121 = l_Array_append___rarg(x_86, x_120); -lean_dec(x_120); -x_122 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_122; -x_91 = x_121; -goto block_109; +lean_object* x_124; lean_object* x_125; +x_124 = lean_ctor_get(x_122, 1); +lean_dec(x_124); +x_125 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set(x_122, 1, x_125); +x_111 = x_122; +goto block_116; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_123 = lean_ctor_get(x_115, 0); -lean_inc(x_123); -lean_dec(x_115); -x_124 = l_Lake_LeanConfig_decodeToml___closed__5; -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -x_126 = lean_unsigned_to_nat(1u); -x_127 = lean_mk_array(x_126, x_125); -x_128 = l_Array_append___rarg(x_86, x_127); -lean_dec(x_127); -x_129 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_129; -x_91 = x_128; -goto block_109; +lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_126 = lean_ctor_get(x_122, 0); +lean_inc(x_126); +lean_dec(x_122); +x_127 = l_Lake_LeanConfig_decodeToml___closed__5; +x_128 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); +x_111 = x_128; +goto block_116; } } case 2: { -lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; -x_130 = lean_ctor_get(x_115, 0); -lean_inc(x_130); -lean_dec(x_115); -x_131 = l_Lake_LeanConfig_decodeToml___closed__5; -x_132 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -x_133 = lean_unsigned_to_nat(1u); -x_134 = lean_mk_array(x_133, x_132); -x_135 = l_Array_append___rarg(x_86, x_134); -lean_dec(x_134); -x_136 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_136; -x_91 = x_135; -goto block_109; +lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_129 = lean_ctor_get(x_122, 0); +lean_inc(x_129); +lean_dec(x_122); +x_130 = l_Lake_LeanConfig_decodeToml___closed__5; +x_131 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_131, 0, x_129); +lean_ctor_set(x_131, 1, x_130); +x_111 = x_131; +goto block_116; } case 3: { -lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_137 = lean_ctor_get(x_115, 0); -lean_inc(x_137); -lean_dec(x_115); -x_138 = l_Lake_LeanConfig_decodeToml___closed__5; -x_139 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -x_140 = lean_unsigned_to_nat(1u); -x_141 = lean_mk_array(x_140, x_139); -x_142 = l_Array_append___rarg(x_86, x_141); -lean_dec(x_141); -x_143 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_143; -x_91 = x_142; -goto block_109; +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_122, 0); +lean_inc(x_132); +lean_dec(x_122); +x_133 = l_Lake_LeanConfig_decodeToml___closed__5; +x_134 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +x_111 = x_134; +goto block_116; } case 5: { -lean_object* x_144; lean_object* x_145; -x_144 = lean_ctor_get(x_115, 1); -lean_inc(x_144); -lean_dec(x_115); -x_145 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__9(x_144); -lean_dec(x_144); -if (lean_obj_tag(x_145) == 0) +lean_object* x_135; lean_object* x_136; +x_135 = lean_ctor_get(x_122, 1); +lean_inc(x_135); +lean_dec(x_122); +x_136 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__9(x_135); +lean_dec(x_135); +if (lean_obj_tag(x_136) == 0) { -lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -lean_dec(x_145); -x_147 = l_Array_append___rarg(x_86, x_146); -lean_dec(x_146); -x_148 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_148; -x_91 = x_147; +lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = l_Array_append___rarg(x_86, x_137); +lean_dec(x_137); +x_139 = l_Lake_decodeLeanOptions___closed__1; +x_90 = x_139; +x_91 = x_138; goto block_109; } else { -lean_object* x_149; -x_149 = lean_ctor_get(x_145, 0); -lean_inc(x_149); -lean_dec(x_145); -x_90 = x_149; +lean_object* x_140; +x_140 = lean_ctor_get(x_136, 0); +lean_inc(x_140); +lean_dec(x_136); +x_90 = x_140; x_91 = x_86; goto block_109; } } default: { -uint8_t x_150; -x_150 = !lean_is_exclusive(x_115); -if (x_150 == 0) -{ -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_151 = lean_ctor_get(x_115, 1); -lean_dec(x_151); -x_152 = l_Lake_LeanConfig_decodeToml___closed__5; -lean_ctor_set_tag(x_115, 0); -lean_ctor_set(x_115, 1, x_152); -x_153 = lean_unsigned_to_nat(1u); -x_154 = lean_mk_array(x_153, x_115); -x_155 = l_Array_append___rarg(x_86, x_154); -lean_dec(x_154); -x_156 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_156; -x_91 = x_155; -goto block_109; +uint8_t x_141; +x_141 = !lean_is_exclusive(x_122); +if (x_141 == 0) +{ +lean_object* x_142; lean_object* x_143; +x_142 = lean_ctor_get(x_122, 1); +lean_dec(x_142); +x_143 = l_Lake_LeanConfig_decodeToml___closed__5; +lean_ctor_set_tag(x_122, 0); +lean_ctor_set(x_122, 1, x_143); +x_111 = x_122; +goto block_116; } else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_157 = lean_ctor_get(x_115, 0); -lean_inc(x_157); -lean_dec(x_115); -x_158 = l_Lake_LeanConfig_decodeToml___closed__5; -x_159 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_159, 0, x_157); -lean_ctor_set(x_159, 1, x_158); -x_160 = lean_unsigned_to_nat(1u); -x_161 = lean_mk_array(x_160, x_159); -x_162 = l_Array_append___rarg(x_86, x_161); -lean_dec(x_161); -x_163 = l_Lake_decodeLeanOptions___closed__1; -x_90 = x_163; -x_91 = x_162; -goto block_109; +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_122, 0); +lean_inc(x_144); +lean_dec(x_122); +x_145 = l_Lake_LeanConfig_decodeToml___closed__5; +x_146 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_111 = x_146; +goto block_116; } } } @@ -24035,92 +27563,148 @@ x_17 = x_91; goto block_46; } } +block_116: +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_112 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_110); +x_113 = lean_array_mk(x_112); +x_114 = l_Array_append___rarg(x_86, x_113); +lean_dec(x_113); +x_115 = l_Lake_decodeLeanOptions___closed__1; +x_90 = x_115; +x_91 = x_114; +goto block_109; } } -block_231: +block_154: { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; uint8_t x_226; -x_222 = lean_array_get_size(x_220); -x_223 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_224 = l_Lake_RBArray_mkEmpty___rarg(x_223, x_222); -x_225 = lean_unsigned_to_nat(0u); -x_226 = lean_nat_dec_lt(x_225, x_222); -if (x_226 == 0) +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +x_150 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_148); +x_151 = lean_array_mk(x_150); +x_152 = l_Array_append___rarg(x_84, x_151); +lean_dec(x_151); +x_153 = l_Lake_decodeLeanOptions___closed__1; +x_85 = x_153; +x_86 = x_152; +goto block_147; +} +} +block_197: { -lean_dec(x_222); -lean_dec(x_220); -x_83 = x_224; -x_84 = x_221; -goto block_219; +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; uint8_t x_192; +x_188 = lean_array_get_size(x_186); +x_189 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_190 = l_Lake_RBArray_mkEmpty___rarg(x_189, x_188); +x_191 = lean_unsigned_to_nat(0u); +x_192 = lean_nat_dec_lt(x_191, x_188); +if (x_192 == 0) +{ +lean_dec(x_188); +lean_dec(x_186); +x_83 = x_190; +x_84 = x_187; +goto block_185; } else { -uint8_t x_227; -x_227 = lean_nat_dec_le(x_222, x_222); -if (x_227 == 0) +uint8_t x_193; +x_193 = lean_nat_dec_le(x_188, x_188); +if (x_193 == 0) { -lean_dec(x_222); -lean_dec(x_220); -x_83 = x_224; -x_84 = x_221; -goto block_219; +lean_dec(x_188); +lean_dec(x_186); +x_83 = x_190; +x_84 = x_187; +goto block_185; } else { -size_t x_228; size_t x_229; lean_object* x_230; -x_228 = 0; -x_229 = lean_usize_of_nat(x_222); -lean_dec(x_222); -x_230 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__11(x_220, x_228, x_229, x_224); -lean_dec(x_220); -x_83 = x_230; -x_84 = x_221; -goto block_219; +size_t x_194; size_t x_195; lean_object* x_196; +x_194 = 0; +x_195 = lean_usize_of_nat(x_188); +lean_dec(x_188); +x_196 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__11(x_186, x_194, x_195, x_190); +lean_dec(x_186); +x_83 = x_196; +x_84 = x_187; +goto block_185; } } } +block_204: +{ +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_198); +x_201 = lean_array_mk(x_200); +x_202 = l_Array_append___rarg(x_82, x_201); +lean_dec(x_201); +x_203 = l_Lake_decodeLeanOptions___closed__1; +x_186 = x_203; +x_187 = x_202; +goto block_197; +} } -block_298: +block_247: { -lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; uint8_t x_293; -x_289 = lean_array_get_size(x_287); -x_290 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_291 = l_Lake_RBArray_mkEmpty___rarg(x_290, x_289); -x_292 = lean_unsigned_to_nat(0u); -x_293 = lean_nat_dec_lt(x_292, x_289); -if (x_293 == 0) +lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; uint8_t x_242; +x_238 = lean_array_get_size(x_236); +x_239 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_240 = l_Lake_RBArray_mkEmpty___rarg(x_239, x_238); +x_241 = lean_unsigned_to_nat(0u); +x_242 = lean_nat_dec_lt(x_241, x_238); +if (x_242 == 0) { -lean_dec(x_289); -lean_dec(x_287); -x_81 = x_291; -x_82 = x_288; -goto block_286; +lean_dec(x_238); +lean_dec(x_236); +x_81 = x_240; +x_82 = x_237; +goto block_235; } else { -uint8_t x_294; -x_294 = lean_nat_dec_le(x_289, x_289); -if (x_294 == 0) +uint8_t x_243; +x_243 = lean_nat_dec_le(x_238, x_238); +if (x_243 == 0) { -lean_dec(x_289); -lean_dec(x_287); -x_81 = x_291; -x_82 = x_288; -goto block_286; +lean_dec(x_238); +lean_dec(x_236); +x_81 = x_240; +x_82 = x_237; +goto block_235; } else { -size_t x_295; size_t x_296; lean_object* x_297; -x_295 = 0; -x_296 = lean_usize_of_nat(x_289); -lean_dec(x_289); -x_297 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__14(x_287, x_295, x_296, x_291); -lean_dec(x_287); -x_81 = x_297; -x_82 = x_288; -goto block_286; +size_t x_244; size_t x_245; lean_object* x_246; +x_244 = 0; +x_245 = lean_usize_of_nat(x_238); +lean_dec(x_238); +x_246 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__14(x_236, x_244, x_245, x_240); +lean_dec(x_236); +x_81 = x_246; +x_82 = x_237; +goto block_235; +} } } +block_254: +{ +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; +x_250 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_250, 0, x_249); +lean_ctor_set(x_250, 1, x_248); +x_251 = lean_array_mk(x_250); +x_252 = l_Array_append___rarg(x_80, x_251); +lean_dec(x_251); +x_253 = l_Lake_decodeLeanOptions___closed__1; +x_236 = x_253; +x_237 = x_252; +goto block_247; } } } @@ -24272,1154 +27856,1118 @@ return x_45; } else { -lean_object* x_370; lean_object* x_371; lean_object* x_372; uint8_t x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_664; -x_370 = lean_ctor_get(x_4, 0); -x_371 = lean_ctor_get(x_4, 1); -lean_inc(x_371); -lean_inc(x_370); +lean_object* x_302; lean_object* x_303; lean_object* x_304; uint8_t x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_560; +x_302 = lean_ctor_get(x_4, 0); +x_303 = lean_ctor_get(x_4, 1); +lean_inc(x_303); +lean_inc(x_302); lean_dec(x_4); -x_372 = lean_ctor_get(x_1, 4); -lean_inc(x_372); -x_373 = 1; -lean_inc(x_372); -x_374 = l_Lean_Parser_mkInputContext(x_370, x_372, x_373); -lean_inc(x_374); -x_664 = l_Lake_Toml_loadToml(x_374, x_5); -if (lean_obj_tag(x_664) == 0) -{ -lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; -x_665 = lean_ctor_get(x_664, 0); -lean_inc(x_665); -x_666 = lean_ctor_get(x_664, 1); -lean_inc(x_666); -lean_dec(x_664); -x_667 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_667, 0, x_665); -x_668 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_668, 0, x_667); -lean_ctor_set(x_668, 1, x_371); -x_375 = x_668; -x_376 = x_666; -goto block_663; -} -else +x_304 = lean_ctor_get(x_1, 4); +lean_inc(x_304); +x_305 = 1; +lean_inc(x_304); +x_306 = l_Lean_Parser_mkInputContext(x_302, x_304, x_305); +lean_inc(x_306); +x_560 = l_Lake_Toml_loadToml(x_306, x_5); +if (lean_obj_tag(x_560) == 0) { -lean_object* x_669; lean_object* x_670; lean_object* x_671; lean_object* x_672; -x_669 = lean_ctor_get(x_664, 0); -lean_inc(x_669); -x_670 = lean_ctor_get(x_664, 1); -lean_inc(x_670); -lean_dec(x_664); -x_671 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_671, 0, x_669); -x_672 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_672, 0, x_671); -lean_ctor_set(x_672, 1, x_371); -x_375 = x_672; -x_376 = x_670; -goto block_663; +lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; +x_561 = lean_ctor_get(x_560, 0); +lean_inc(x_561); +x_562 = lean_ctor_get(x_560, 1); +lean_inc(x_562); +lean_dec(x_560); +x_563 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_563, 0, x_561); +x_564 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_564, 0, x_563); +lean_ctor_set(x_564, 1, x_303); +x_307 = x_564; +x_308 = x_562; +goto block_559; } -block_663: +else { -lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; -x_377 = lean_ctor_get(x_375, 0); -lean_inc(x_377); -x_378 = lean_ctor_get(x_375, 1); -lean_inc(x_378); -if (lean_is_exclusive(x_375)) { - lean_ctor_release(x_375, 0); - lean_ctor_release(x_375, 1); - x_379 = x_375; +lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; +x_565 = lean_ctor_get(x_560, 0); +lean_inc(x_565); +x_566 = lean_ctor_get(x_560, 1); +lean_inc(x_566); +lean_dec(x_560); +x_567 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_567, 0, x_565); +x_568 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_568, 0, x_567); +lean_ctor_set(x_568, 1, x_303); +x_307 = x_568; +x_308 = x_566; +goto block_559; +} +block_559: +{ +lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; +x_309 = lean_ctor_get(x_307, 0); +lean_inc(x_309); +x_310 = lean_ctor_get(x_307, 1); +lean_inc(x_310); +if (lean_is_exclusive(x_307)) { + lean_ctor_release(x_307, 0); + lean_ctor_release(x_307, 1); + x_311 = x_307; } else { - lean_dec_ref(x_375); - x_379 = lean_box(0); + lean_dec_ref(x_307); + x_311 = lean_box(0); } -if (lean_obj_tag(x_377) == 0) +if (lean_obj_tag(x_309) == 0) { -lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; -lean_dec(x_379); -lean_dec(x_374); -lean_dec(x_372); +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; +lean_dec(x_311); +lean_dec(x_306); +lean_dec(x_304); lean_dec(x_1); -x_406 = lean_ctor_get(x_377, 0); -lean_inc(x_406); -lean_dec(x_377); -x_407 = lean_array_get_size(x_378); -x_408 = l_Lake_loadTomlConfig___closed__1; -x_409 = l_Lean_MessageLog_forM___at_Lake_loadTomlConfig___spec__2(x_406, x_408, x_378, x_376); -lean_dec(x_406); -if (lean_obj_tag(x_409) == 0) -{ -lean_object* x_410; -x_410 = lean_ctor_get(x_409, 0); -lean_inc(x_410); -if (lean_obj_tag(x_410) == 0) -{ -lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; -x_411 = lean_ctor_get(x_409, 1); -lean_inc(x_411); -if (lean_is_exclusive(x_409)) { - lean_ctor_release(x_409, 0); - lean_ctor_release(x_409, 1); - x_412 = x_409; +x_338 = lean_ctor_get(x_309, 0); +lean_inc(x_338); +lean_dec(x_309); +x_339 = lean_array_get_size(x_310); +x_340 = l_Lake_loadTomlConfig___closed__1; +x_341 = l_Lean_MessageLog_forM___at_Lake_loadTomlConfig___spec__2(x_338, x_340, x_310, x_308); +lean_dec(x_338); +if (lean_obj_tag(x_341) == 0) +{ +lean_object* x_342; +x_342 = lean_ctor_get(x_341, 0); +lean_inc(x_342); +if (lean_obj_tag(x_342) == 0) +{ +lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; +x_343 = lean_ctor_get(x_341, 1); +lean_inc(x_343); +if (lean_is_exclusive(x_341)) { + lean_ctor_release(x_341, 0); + lean_ctor_release(x_341, 1); + x_344 = x_341; } else { - lean_dec_ref(x_409); - x_412 = lean_box(0); -} -x_413 = lean_ctor_get(x_410, 1); -lean_inc(x_413); -if (lean_is_exclusive(x_410)) { - lean_ctor_release(x_410, 0); - lean_ctor_release(x_410, 1); - x_414 = x_410; + lean_dec_ref(x_341); + x_344 = lean_box(0); +} +x_345 = lean_ctor_get(x_342, 1); +lean_inc(x_345); +if (lean_is_exclusive(x_342)) { + lean_ctor_release(x_342, 0); + lean_ctor_release(x_342, 1); + x_346 = x_342; } else { - lean_dec_ref(x_410); - x_414 = lean_box(0); + lean_dec_ref(x_342); + x_346 = lean_box(0); } -if (lean_is_scalar(x_414)) { - x_415 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_346)) { + x_347 = lean_alloc_ctor(1, 2, 0); } else { - x_415 = x_414; - lean_ctor_set_tag(x_415, 1); + x_347 = x_346; + lean_ctor_set_tag(x_347, 1); } -lean_ctor_set(x_415, 0, x_407); -lean_ctor_set(x_415, 1, x_413); -if (lean_is_scalar(x_412)) { - x_416 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_347, 0, x_339); +lean_ctor_set(x_347, 1, x_345); +if (lean_is_scalar(x_344)) { + x_348 = lean_alloc_ctor(0, 2, 0); } else { - x_416 = x_412; + x_348 = x_344; } -lean_ctor_set(x_416, 0, x_415); -lean_ctor_set(x_416, 1, x_411); -return x_416; +lean_ctor_set(x_348, 0, x_347); +lean_ctor_set(x_348, 1, x_343); +return x_348; } else { -lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; -x_417 = lean_ctor_get(x_409, 1); -lean_inc(x_417); -if (lean_is_exclusive(x_409)) { - lean_ctor_release(x_409, 0); - lean_ctor_release(x_409, 1); - x_418 = x_409; +lean_object* x_349; lean_object* x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; +x_349 = lean_ctor_get(x_341, 1); +lean_inc(x_349); +if (lean_is_exclusive(x_341)) { + lean_ctor_release(x_341, 0); + lean_ctor_release(x_341, 1); + x_350 = x_341; } else { - lean_dec_ref(x_409); - x_418 = lean_box(0); + lean_dec_ref(x_341); + x_350 = lean_box(0); } -x_419 = lean_ctor_get(x_410, 1); -lean_inc(x_419); -if (lean_is_exclusive(x_410)) { - lean_ctor_release(x_410, 0); - lean_ctor_release(x_410, 1); - x_420 = x_410; +x_351 = lean_ctor_get(x_342, 1); +lean_inc(x_351); +if (lean_is_exclusive(x_342)) { + lean_ctor_release(x_342, 0); + lean_ctor_release(x_342, 1); + x_352 = x_342; } else { - lean_dec_ref(x_410); - x_420 = lean_box(0); + lean_dec_ref(x_342); + x_352 = lean_box(0); } -if (lean_is_scalar(x_420)) { - x_421 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_352)) { + x_353 = lean_alloc_ctor(1, 2, 0); } else { - x_421 = x_420; + x_353 = x_352; } -lean_ctor_set(x_421, 0, x_407); -lean_ctor_set(x_421, 1, x_419); -if (lean_is_scalar(x_418)) { - x_422 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_353, 0, x_339); +lean_ctor_set(x_353, 1, x_351); +if (lean_is_scalar(x_350)) { + x_354 = lean_alloc_ctor(0, 2, 0); } else { - x_422 = x_418; + x_354 = x_350; } -lean_ctor_set(x_422, 0, x_421); -lean_ctor_set(x_422, 1, x_417); -return x_422; +lean_ctor_set(x_354, 0, x_353); +lean_ctor_set(x_354, 1, x_349); +return x_354; } } else { -lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; -lean_dec(x_407); -x_423 = lean_ctor_get(x_409, 0); -lean_inc(x_423); -x_424 = lean_ctor_get(x_409, 1); -lean_inc(x_424); -if (lean_is_exclusive(x_409)) { - lean_ctor_release(x_409, 0); - lean_ctor_release(x_409, 1); - x_425 = x_409; +lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; +lean_dec(x_339); +x_355 = lean_ctor_get(x_341, 0); +lean_inc(x_355); +x_356 = lean_ctor_get(x_341, 1); +lean_inc(x_356); +if (lean_is_exclusive(x_341)) { + lean_ctor_release(x_341, 0); + lean_ctor_release(x_341, 1); + x_357 = x_341; } else { - lean_dec_ref(x_409); - x_425 = lean_box(0); + lean_dec_ref(x_341); + x_357 = lean_box(0); } -if (lean_is_scalar(x_425)) { - x_426 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_357)) { + x_358 = lean_alloc_ctor(1, 2, 0); } else { - x_426 = x_425; + x_358 = x_357; } -lean_ctor_set(x_426, 0, x_423); -lean_ctor_set(x_426, 1, x_424); -return x_426; +lean_ctor_set(x_358, 0, x_355); +lean_ctor_set(x_358, 1, x_356); +return x_358; } } else { -lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_655; lean_object* x_656; -x_427 = lean_ctor_get(x_377, 0); -lean_inc(x_427); -lean_dec(x_377); -x_655 = lean_box(0); -lean_inc(x_427); -x_656 = l_Lake_PackageConfig_decodeToml(x_427, x_655); -if (lean_obj_tag(x_656) == 0) +lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_551; lean_object* x_552; +x_359 = lean_ctor_get(x_309, 0); +lean_inc(x_359); +lean_dec(x_309); +x_551 = lean_box(0); +lean_inc(x_359); +x_552 = l_Lake_PackageConfig_decodeToml(x_359, x_551); +if (lean_obj_tag(x_552) == 0) { -lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; -x_657 = lean_ctor_get(x_656, 0); -lean_inc(x_657); -lean_dec(x_656); -x_658 = l_Lake_decodeLeanOptions___closed__1; -x_659 = l_Array_append___rarg(x_658, x_657); -lean_dec(x_657); -x_660 = l_Lake_loadTomlConfig___closed__11; -x_428 = x_660; -x_429 = x_659; -goto block_654; -} -else -{ -lean_object* x_661; lean_object* x_662; -x_661 = lean_ctor_get(x_656, 0); -lean_inc(x_661); -lean_dec(x_656); -x_662 = l_Lake_decodeLeanOptions___closed__1; -x_428 = x_661; -x_429 = x_662; -goto block_654; -} -block_654: -{ -lean_object* x_430; lean_object* x_431; lean_object* x_600; lean_object* x_601; lean_object* x_612; lean_object* x_613; lean_object* x_614; -x_612 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_613 = l_Lake_loadTomlConfig___closed__9; -lean_inc(x_427); -x_614 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_612, x_613, x_427); -if (lean_obj_tag(x_614) == 0) +lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; +x_553 = lean_ctor_get(x_552, 0); +lean_inc(x_553); +lean_dec(x_552); +x_554 = l_Lake_decodeLeanOptions___closed__1; +x_555 = l_Array_append___rarg(x_554, x_553); +lean_dec(x_553); +x_556 = l_Lake_loadTomlConfig___closed__11; +x_360 = x_556; +x_361 = x_555; +goto block_550; +} +else +{ +lean_object* x_557; lean_object* x_558; +x_557 = lean_ctor_get(x_552, 0); +lean_inc(x_557); +lean_dec(x_552); +x_558 = l_Lake_decodeLeanOptions___closed__1; +x_360 = x_557; +x_361 = x_558; +goto block_550; +} +block_550: +{ +lean_object* x_362; lean_object* x_363; lean_object* x_505; lean_object* x_506; lean_object* x_517; lean_object* x_518; lean_object* x_524; lean_object* x_525; lean_object* x_526; +x_517 = lean_box(0); +x_524 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_525 = l_Lake_loadTomlConfig___closed__9; +lean_inc(x_359); +x_526 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_524, x_525, x_359); +if (lean_obj_tag(x_526) == 0) { -lean_object* x_615; -x_615 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_615; -x_601 = x_429; -goto block_611; +lean_object* x_527; +x_527 = l_Lake_decodeLeanOptions___closed__1; +x_505 = x_527; +x_506 = x_361; +goto block_516; } else { -lean_object* x_616; lean_object* x_617; -x_616 = lean_ctor_get(x_614, 0); -lean_inc(x_616); -lean_dec(x_614); -x_617 = lean_ctor_get(x_616, 1); -lean_inc(x_617); -lean_dec(x_616); -switch (lean_obj_tag(x_617)) { +lean_object* x_528; lean_object* x_529; +x_528 = lean_ctor_get(x_526, 0); +lean_inc(x_528); +lean_dec(x_526); +x_529 = lean_ctor_get(x_528, 1); +lean_inc(x_529); +lean_dec(x_528); +switch (lean_obj_tag(x_529)) { case 0: { -lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; lean_object* x_624; lean_object* x_625; -x_618 = lean_ctor_get(x_617, 0); -lean_inc(x_618); -if (lean_is_exclusive(x_617)) { - lean_ctor_release(x_617, 0); - lean_ctor_release(x_617, 1); - x_619 = x_617; +lean_object* x_530; lean_object* x_531; lean_object* x_532; lean_object* x_533; +x_530 = lean_ctor_get(x_529, 0); +lean_inc(x_530); +if (lean_is_exclusive(x_529)) { + lean_ctor_release(x_529, 0); + lean_ctor_release(x_529, 1); + x_531 = x_529; } else { - lean_dec_ref(x_617); - x_619 = lean_box(0); + lean_dec_ref(x_529); + x_531 = lean_box(0); } -x_620 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_619)) { - x_621 = lean_alloc_ctor(0, 2, 0); +x_532 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_531)) { + x_533 = lean_alloc_ctor(0, 2, 0); } else { - x_621 = x_619; + x_533 = x_531; } -lean_ctor_set(x_621, 0, x_618); -lean_ctor_set(x_621, 1, x_620); -x_622 = lean_unsigned_to_nat(1u); -x_623 = lean_mk_array(x_622, x_621); -x_624 = l_Array_append___rarg(x_429, x_623); -lean_dec(x_623); -x_625 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_625; -x_601 = x_624; -goto block_611; +lean_ctor_set(x_533, 0, x_530); +lean_ctor_set(x_533, 1, x_532); +x_518 = x_533; +goto block_523; } case 2: { -lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; lean_object* x_631; lean_object* x_632; -x_626 = lean_ctor_get(x_617, 0); -lean_inc(x_626); -lean_dec(x_617); -x_627 = l_Lake_LeanConfig_decodeToml___closed__5; -x_628 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_628, 0, x_626); -lean_ctor_set(x_628, 1, x_627); -x_629 = lean_unsigned_to_nat(1u); -x_630 = lean_mk_array(x_629, x_628); -x_631 = l_Array_append___rarg(x_429, x_630); -lean_dec(x_630); -x_632 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_632; -x_601 = x_631; -goto block_611; +lean_object* x_534; lean_object* x_535; lean_object* x_536; +x_534 = lean_ctor_get(x_529, 0); +lean_inc(x_534); +lean_dec(x_529); +x_535 = l_Lake_LeanConfig_decodeToml___closed__5; +x_536 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_536, 0, x_534); +lean_ctor_set(x_536, 1, x_535); +x_518 = x_536; +goto block_523; } case 3: { -lean_object* x_633; lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; -x_633 = lean_ctor_get(x_617, 0); -lean_inc(x_633); -lean_dec(x_617); -x_634 = l_Lake_LeanConfig_decodeToml___closed__5; -x_635 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_635, 0, x_633); -lean_ctor_set(x_635, 1, x_634); -x_636 = lean_unsigned_to_nat(1u); -x_637 = lean_mk_array(x_636, x_635); -x_638 = l_Array_append___rarg(x_429, x_637); -lean_dec(x_637); -x_639 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_639; -x_601 = x_638; -goto block_611; +lean_object* x_537; lean_object* x_538; lean_object* x_539; +x_537 = lean_ctor_get(x_529, 0); +lean_inc(x_537); +lean_dec(x_529); +x_538 = l_Lake_LeanConfig_decodeToml___closed__5; +x_539 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_539, 0, x_537); +lean_ctor_set(x_539, 1, x_538); +x_518 = x_539; +goto block_523; } case 5: { -lean_object* x_640; lean_object* x_641; -x_640 = lean_ctor_get(x_617, 1); -lean_inc(x_640); -lean_dec(x_617); -x_641 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__15(x_640); -lean_dec(x_640); -if (lean_obj_tag(x_641) == 0) +lean_object* x_540; lean_object* x_541; +x_540 = lean_ctor_get(x_529, 1); +lean_inc(x_540); +lean_dec(x_529); +x_541 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__15(x_540); +lean_dec(x_540); +if (lean_obj_tag(x_541) == 0) { -lean_object* x_642; lean_object* x_643; lean_object* x_644; -x_642 = lean_ctor_get(x_641, 0); -lean_inc(x_642); -lean_dec(x_641); -x_643 = l_Array_append___rarg(x_429, x_642); -lean_dec(x_642); -x_644 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_644; -x_601 = x_643; -goto block_611; +lean_object* x_542; lean_object* x_543; lean_object* x_544; +x_542 = lean_ctor_get(x_541, 0); +lean_inc(x_542); +lean_dec(x_541); +x_543 = l_Array_append___rarg(x_361, x_542); +lean_dec(x_542); +x_544 = l_Lake_decodeLeanOptions___closed__1; +x_505 = x_544; +x_506 = x_543; +goto block_516; } else { -lean_object* x_645; -x_645 = lean_ctor_get(x_641, 0); -lean_inc(x_645); -lean_dec(x_641); -x_600 = x_645; -x_601 = x_429; -goto block_611; +lean_object* x_545; +x_545 = lean_ctor_get(x_541, 0); +lean_inc(x_545); +lean_dec(x_541); +x_505 = x_545; +x_506 = x_361; +goto block_516; } } default: { -lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; lean_object* x_650; lean_object* x_651; lean_object* x_652; lean_object* x_653; -x_646 = lean_ctor_get(x_617, 0); -lean_inc(x_646); -if (lean_is_exclusive(x_617)) { - lean_ctor_release(x_617, 0); - lean_ctor_release(x_617, 1); - x_647 = x_617; +lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; +x_546 = lean_ctor_get(x_529, 0); +lean_inc(x_546); +if (lean_is_exclusive(x_529)) { + lean_ctor_release(x_529, 0); + lean_ctor_release(x_529, 1); + x_547 = x_529; } else { - lean_dec_ref(x_617); - x_647 = lean_box(0); + lean_dec_ref(x_529); + x_547 = lean_box(0); } -x_648 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_647)) { - x_649 = lean_alloc_ctor(0, 2, 0); +x_548 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_547)) { + x_549 = lean_alloc_ctor(0, 2, 0); } else { - x_649 = x_647; - lean_ctor_set_tag(x_649, 0); -} -lean_ctor_set(x_649, 0, x_646); -lean_ctor_set(x_649, 1, x_648); -x_650 = lean_unsigned_to_nat(1u); -x_651 = lean_mk_array(x_650, x_649); -x_652 = l_Array_append___rarg(x_429, x_651); -lean_dec(x_651); -x_653 = l_Lake_decodeLeanOptions___closed__1; -x_600 = x_653; -x_601 = x_652; -goto block_611; + x_549 = x_547; + lean_ctor_set_tag(x_549, 0); } +lean_ctor_set(x_549, 0, x_546); +lean_ctor_set(x_549, 1, x_548); +x_518 = x_549; +goto block_523; } } -block_599: +} +block_504: { -lean_object* x_432; lean_object* x_433; lean_object* x_545; lean_object* x_546; lean_object* x_557; lean_object* x_558; lean_object* x_559; -x_557 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_558 = l_Lake_loadTomlConfig___closed__7; -lean_inc(x_427); -x_559 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_557, x_558, x_427); -if (lean_obj_tag(x_559) == 0) +lean_object* x_364; lean_object* x_365; lean_object* x_459; lean_object* x_460; lean_object* x_471; lean_object* x_472; lean_object* x_478; lean_object* x_479; lean_object* x_480; +x_471 = lean_box(0); +x_478 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_479 = l_Lake_loadTomlConfig___closed__7; +lean_inc(x_359); +x_480 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_478, x_479, x_359); +if (lean_obj_tag(x_480) == 0) { -lean_object* x_560; -x_560 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_560; -x_546 = x_431; -goto block_556; +lean_object* x_481; +x_481 = l_Lake_decodeLeanOptions___closed__1; +x_459 = x_481; +x_460 = x_363; +goto block_470; } else { -lean_object* x_561; lean_object* x_562; -x_561 = lean_ctor_get(x_559, 0); -lean_inc(x_561); -lean_dec(x_559); -x_562 = lean_ctor_get(x_561, 1); -lean_inc(x_562); -lean_dec(x_561); -switch (lean_obj_tag(x_562)) { +lean_object* x_482; lean_object* x_483; +x_482 = lean_ctor_get(x_480, 0); +lean_inc(x_482); +lean_dec(x_480); +x_483 = lean_ctor_get(x_482, 1); +lean_inc(x_483); +lean_dec(x_482); +switch (lean_obj_tag(x_483)) { case 0: { -lean_object* x_563; lean_object* x_564; lean_object* x_565; lean_object* x_566; lean_object* x_567; lean_object* x_568; lean_object* x_569; lean_object* x_570; -x_563 = lean_ctor_get(x_562, 0); -lean_inc(x_563); -if (lean_is_exclusive(x_562)) { - lean_ctor_release(x_562, 0); - lean_ctor_release(x_562, 1); - x_564 = x_562; +lean_object* x_484; lean_object* x_485; lean_object* x_486; lean_object* x_487; +x_484 = lean_ctor_get(x_483, 0); +lean_inc(x_484); +if (lean_is_exclusive(x_483)) { + lean_ctor_release(x_483, 0); + lean_ctor_release(x_483, 1); + x_485 = x_483; } else { - lean_dec_ref(x_562); - x_564 = lean_box(0); + lean_dec_ref(x_483); + x_485 = lean_box(0); } -x_565 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_564)) { - x_566 = lean_alloc_ctor(0, 2, 0); +x_486 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_485)) { + x_487 = lean_alloc_ctor(0, 2, 0); } else { - x_566 = x_564; + x_487 = x_485; } -lean_ctor_set(x_566, 0, x_563); -lean_ctor_set(x_566, 1, x_565); -x_567 = lean_unsigned_to_nat(1u); -x_568 = lean_mk_array(x_567, x_566); -x_569 = l_Array_append___rarg(x_431, x_568); -lean_dec(x_568); -x_570 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_570; -x_546 = x_569; -goto block_556; +lean_ctor_set(x_487, 0, x_484); +lean_ctor_set(x_487, 1, x_486); +x_472 = x_487; +goto block_477; } case 2: { -lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_577; -x_571 = lean_ctor_get(x_562, 0); -lean_inc(x_571); -lean_dec(x_562); -x_572 = l_Lake_LeanConfig_decodeToml___closed__5; -x_573 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_573, 0, x_571); -lean_ctor_set(x_573, 1, x_572); -x_574 = lean_unsigned_to_nat(1u); -x_575 = lean_mk_array(x_574, x_573); -x_576 = l_Array_append___rarg(x_431, x_575); -lean_dec(x_575); -x_577 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_577; -x_546 = x_576; -goto block_556; +lean_object* x_488; lean_object* x_489; lean_object* x_490; +x_488 = lean_ctor_get(x_483, 0); +lean_inc(x_488); +lean_dec(x_483); +x_489 = l_Lake_LeanConfig_decodeToml___closed__5; +x_490 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_490, 0, x_488); +lean_ctor_set(x_490, 1, x_489); +x_472 = x_490; +goto block_477; } case 3: { -lean_object* x_578; lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; lean_object* x_584; -x_578 = lean_ctor_get(x_562, 0); -lean_inc(x_578); -lean_dec(x_562); -x_579 = l_Lake_LeanConfig_decodeToml___closed__5; -x_580 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_580, 0, x_578); -lean_ctor_set(x_580, 1, x_579); -x_581 = lean_unsigned_to_nat(1u); -x_582 = lean_mk_array(x_581, x_580); -x_583 = l_Array_append___rarg(x_431, x_582); -lean_dec(x_582); -x_584 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_584; -x_546 = x_583; -goto block_556; +lean_object* x_491; lean_object* x_492; lean_object* x_493; +x_491 = lean_ctor_get(x_483, 0); +lean_inc(x_491); +lean_dec(x_483); +x_492 = l_Lake_LeanConfig_decodeToml___closed__5; +x_493 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_493, 0, x_491); +lean_ctor_set(x_493, 1, x_492); +x_472 = x_493; +goto block_477; } case 5: { -lean_object* x_585; lean_object* x_586; -x_585 = lean_ctor_get(x_562, 1); -lean_inc(x_585); -lean_dec(x_562); -x_586 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__12(x_585); -lean_dec(x_585); -if (lean_obj_tag(x_586) == 0) -{ -lean_object* x_587; lean_object* x_588; lean_object* x_589; -x_587 = lean_ctor_get(x_586, 0); -lean_inc(x_587); -lean_dec(x_586); -x_588 = l_Array_append___rarg(x_431, x_587); -lean_dec(x_587); -x_589 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_589; -x_546 = x_588; -goto block_556; -} -else -{ -lean_object* x_590; -x_590 = lean_ctor_get(x_586, 0); -lean_inc(x_590); -lean_dec(x_586); -x_545 = x_590; -x_546 = x_431; -goto block_556; +lean_object* x_494; lean_object* x_495; +x_494 = lean_ctor_get(x_483, 1); +lean_inc(x_494); +lean_dec(x_483); +x_495 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__12(x_494); +lean_dec(x_494); +if (lean_obj_tag(x_495) == 0) +{ +lean_object* x_496; lean_object* x_497; lean_object* x_498; +x_496 = lean_ctor_get(x_495, 0); +lean_inc(x_496); +lean_dec(x_495); +x_497 = l_Array_append___rarg(x_363, x_496); +lean_dec(x_496); +x_498 = l_Lake_decodeLeanOptions___closed__1; +x_459 = x_498; +x_460 = x_497; +goto block_470; +} +else +{ +lean_object* x_499; +x_499 = lean_ctor_get(x_495, 0); +lean_inc(x_499); +lean_dec(x_495); +x_459 = x_499; +x_460 = x_363; +goto block_470; } } default: { -lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; lean_object* x_598; -x_591 = lean_ctor_get(x_562, 0); -lean_inc(x_591); -if (lean_is_exclusive(x_562)) { - lean_ctor_release(x_562, 0); - lean_ctor_release(x_562, 1); - x_592 = x_562; +lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; +x_500 = lean_ctor_get(x_483, 0); +lean_inc(x_500); +if (lean_is_exclusive(x_483)) { + lean_ctor_release(x_483, 0); + lean_ctor_release(x_483, 1); + x_501 = x_483; } else { - lean_dec_ref(x_562); - x_592 = lean_box(0); + lean_dec_ref(x_483); + x_501 = lean_box(0); } -x_593 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_592)) { - x_594 = lean_alloc_ctor(0, 2, 0); +x_502 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_501)) { + x_503 = lean_alloc_ctor(0, 2, 0); } else { - x_594 = x_592; - lean_ctor_set_tag(x_594, 0); + x_503 = x_501; + lean_ctor_set_tag(x_503, 0); } -lean_ctor_set(x_594, 0, x_591); -lean_ctor_set(x_594, 1, x_593); -x_595 = lean_unsigned_to_nat(1u); -x_596 = lean_mk_array(x_595, x_594); -x_597 = l_Array_append___rarg(x_431, x_596); -lean_dec(x_596); -x_598 = l_Lake_decodeLeanOptions___closed__1; -x_545 = x_598; -x_546 = x_597; -goto block_556; +lean_ctor_set(x_503, 0, x_500); +lean_ctor_set(x_503, 1, x_502); +x_472 = x_503; +goto block_477; } } } -block_544: +block_458: { -lean_object* x_434; lean_object* x_435; lean_object* x_502; lean_object* x_503; lean_object* x_504; -x_502 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_503 = l_Lake_loadTomlConfig___closed__5; -lean_inc(x_427); -x_504 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_502, x_503, x_427); -if (lean_obj_tag(x_504) == 0) +lean_object* x_366; lean_object* x_367; lean_object* x_425; lean_object* x_426; lean_object* x_432; lean_object* x_433; lean_object* x_434; +x_425 = lean_box(0); +x_432 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_433 = l_Lake_loadTomlConfig___closed__5; +lean_inc(x_359); +x_434 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_432, x_433, x_359); +if (lean_obj_tag(x_434) == 0) { -lean_object* x_505; -x_505 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_505; -x_435 = x_433; -goto block_501; +lean_object* x_435; +x_435 = l_Lake_decodeLeanOptions___closed__1; +x_366 = x_435; +x_367 = x_365; +goto block_424; } else { -lean_object* x_506; lean_object* x_507; -x_506 = lean_ctor_get(x_504, 0); -lean_inc(x_506); -lean_dec(x_504); -x_507 = lean_ctor_get(x_506, 1); -lean_inc(x_507); -lean_dec(x_506); -switch (lean_obj_tag(x_507)) { +lean_object* x_436; lean_object* x_437; +x_436 = lean_ctor_get(x_434, 0); +lean_inc(x_436); +lean_dec(x_434); +x_437 = lean_ctor_get(x_436, 1); +lean_inc(x_437); +lean_dec(x_436); +switch (lean_obj_tag(x_437)) { case 0: { -lean_object* x_508; lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; -x_508 = lean_ctor_get(x_507, 0); -lean_inc(x_508); -if (lean_is_exclusive(x_507)) { - lean_ctor_release(x_507, 0); - lean_ctor_release(x_507, 1); - x_509 = x_507; +lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_441; +x_438 = lean_ctor_get(x_437, 0); +lean_inc(x_438); +if (lean_is_exclusive(x_437)) { + lean_ctor_release(x_437, 0); + lean_ctor_release(x_437, 1); + x_439 = x_437; } else { - lean_dec_ref(x_507); - x_509 = lean_box(0); + lean_dec_ref(x_437); + x_439 = lean_box(0); } -x_510 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_509)) { - x_511 = lean_alloc_ctor(0, 2, 0); +x_440 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_439)) { + x_441 = lean_alloc_ctor(0, 2, 0); } else { - x_511 = x_509; -} -lean_ctor_set(x_511, 0, x_508); -lean_ctor_set(x_511, 1, x_510); -x_512 = lean_unsigned_to_nat(1u); -x_513 = lean_mk_array(x_512, x_511); -x_514 = l_Array_append___rarg(x_433, x_513); -lean_dec(x_513); -x_515 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_515; -x_435 = x_514; -goto block_501; + x_441 = x_439; +} +lean_ctor_set(x_441, 0, x_438); +lean_ctor_set(x_441, 1, x_440); +x_426 = x_441; +goto block_431; } case 2: { -lean_object* x_516; lean_object* x_517; lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; -x_516 = lean_ctor_get(x_507, 0); -lean_inc(x_516); -lean_dec(x_507); -x_517 = l_Lake_LeanConfig_decodeToml___closed__5; -x_518 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_518, 0, x_516); -lean_ctor_set(x_518, 1, x_517); -x_519 = lean_unsigned_to_nat(1u); -x_520 = lean_mk_array(x_519, x_518); -x_521 = l_Array_append___rarg(x_433, x_520); -lean_dec(x_520); -x_522 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_522; -x_435 = x_521; -goto block_501; +lean_object* x_442; lean_object* x_443; lean_object* x_444; +x_442 = lean_ctor_get(x_437, 0); +lean_inc(x_442); +lean_dec(x_437); +x_443 = l_Lake_LeanConfig_decodeToml___closed__5; +x_444 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_444, 0, x_442); +lean_ctor_set(x_444, 1, x_443); +x_426 = x_444; +goto block_431; } case 3: { -lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; lean_object* x_528; lean_object* x_529; -x_523 = lean_ctor_get(x_507, 0); -lean_inc(x_523); -lean_dec(x_507); -x_524 = l_Lake_LeanConfig_decodeToml___closed__5; -x_525 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_525, 0, x_523); -lean_ctor_set(x_525, 1, x_524); -x_526 = lean_unsigned_to_nat(1u); -x_527 = lean_mk_array(x_526, x_525); -x_528 = l_Array_append___rarg(x_433, x_527); -lean_dec(x_527); -x_529 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_529; -x_435 = x_528; -goto block_501; +lean_object* x_445; lean_object* x_446; lean_object* x_447; +x_445 = lean_ctor_get(x_437, 0); +lean_inc(x_445); +lean_dec(x_437); +x_446 = l_Lake_LeanConfig_decodeToml___closed__5; +x_447 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_447, 0, x_445); +lean_ctor_set(x_447, 1, x_446); +x_426 = x_447; +goto block_431; } case 5: { -lean_object* x_530; lean_object* x_531; -x_530 = lean_ctor_get(x_507, 1); -lean_inc(x_530); -lean_dec(x_507); -x_531 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_530); -lean_dec(x_530); -if (lean_obj_tag(x_531) == 0) +lean_object* x_448; lean_object* x_449; +x_448 = lean_ctor_get(x_437, 1); +lean_inc(x_448); +lean_dec(x_437); +x_449 = l_Lake_Toml_decodeArray___at_Lake_StrPat_decodeToml___spec__1(x_448); +lean_dec(x_448); +if (lean_obj_tag(x_449) == 0) { -lean_object* x_532; lean_object* x_533; lean_object* x_534; -x_532 = lean_ctor_get(x_531, 0); -lean_inc(x_532); -lean_dec(x_531); -x_533 = l_Array_append___rarg(x_433, x_532); -lean_dec(x_532); -x_534 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_534; -x_435 = x_533; -goto block_501; +lean_object* x_450; lean_object* x_451; lean_object* x_452; +x_450 = lean_ctor_get(x_449, 0); +lean_inc(x_450); +lean_dec(x_449); +x_451 = l_Array_append___rarg(x_365, x_450); +lean_dec(x_450); +x_452 = l_Lake_decodeLeanOptions___closed__1; +x_366 = x_452; +x_367 = x_451; +goto block_424; } else { -lean_object* x_535; -x_535 = lean_ctor_get(x_531, 0); -lean_inc(x_535); -lean_dec(x_531); -x_434 = x_535; -x_435 = x_433; -goto block_501; +lean_object* x_453; +x_453 = lean_ctor_get(x_449, 0); +lean_inc(x_453); +lean_dec(x_449); +x_366 = x_453; +x_367 = x_365; +goto block_424; } } default: { -lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; lean_object* x_541; lean_object* x_542; lean_object* x_543; -x_536 = lean_ctor_get(x_507, 0); -lean_inc(x_536); -if (lean_is_exclusive(x_507)) { - lean_ctor_release(x_507, 0); - lean_ctor_release(x_507, 1); - x_537 = x_507; +lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; +x_454 = lean_ctor_get(x_437, 0); +lean_inc(x_454); +if (lean_is_exclusive(x_437)) { + lean_ctor_release(x_437, 0); + lean_ctor_release(x_437, 1); + x_455 = x_437; } else { - lean_dec_ref(x_507); - x_537 = lean_box(0); + lean_dec_ref(x_437); + x_455 = lean_box(0); } -x_538 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_537)) { - x_539 = lean_alloc_ctor(0, 2, 0); +x_456 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_455)) { + x_457 = lean_alloc_ctor(0, 2, 0); } else { - x_539 = x_537; - lean_ctor_set_tag(x_539, 0); + x_457 = x_455; + lean_ctor_set_tag(x_457, 0); } -lean_ctor_set(x_539, 0, x_536); -lean_ctor_set(x_539, 1, x_538); -x_540 = lean_unsigned_to_nat(1u); -x_541 = lean_mk_array(x_540, x_539); -x_542 = l_Array_append___rarg(x_433, x_541); -lean_dec(x_541); -x_543 = l_Lake_decodeLeanOptions___closed__1; -x_434 = x_543; -x_435 = x_542; -goto block_501; +lean_ctor_set(x_457, 0, x_454); +lean_ctor_set(x_457, 1, x_456); +x_426 = x_457; +goto block_431; } } } -block_501: +block_424: { -size_t x_436; size_t x_437; lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_459; lean_object* x_460; lean_object* x_461; -x_436 = lean_array_size(x_434); -x_437 = 0; -x_438 = l_Array_mapMUnsafe_map___at_Lake_loadTomlConfig___spec__8(x_436, x_437, x_434); -x_459 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_460 = l_Lake_loadTomlConfig___closed__3; -x_461 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_459, x_460, x_427); -if (lean_obj_tag(x_461) == 0) +size_t x_368; size_t x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_391; lean_object* x_392; lean_object* x_398; lean_object* x_399; lean_object* x_400; +x_368 = lean_array_size(x_366); +x_369 = 0; +x_370 = l_Array_mapMUnsafe_map___at_Lake_loadTomlConfig___spec__8(x_368, x_369, x_366); +x_391 = lean_box(0); +x_398 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_399 = l_Lake_loadTomlConfig___closed__3; +x_400 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_398, x_399, x_359); +if (lean_obj_tag(x_400) == 0) { -lean_object* x_462; -x_462 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_462; -x_440 = x_435; -goto block_458; +lean_object* x_401; +x_401 = l_Lake_decodeLeanOptions___closed__1; +x_371 = x_401; +x_372 = x_367; +goto block_390; } else { -lean_object* x_463; lean_object* x_464; -x_463 = lean_ctor_get(x_461, 0); -lean_inc(x_463); -lean_dec(x_461); -x_464 = lean_ctor_get(x_463, 1); -lean_inc(x_464); -lean_dec(x_463); -switch (lean_obj_tag(x_464)) { +lean_object* x_402; lean_object* x_403; +x_402 = lean_ctor_get(x_400, 0); +lean_inc(x_402); +lean_dec(x_400); +x_403 = lean_ctor_get(x_402, 1); +lean_inc(x_403); +lean_dec(x_402); +switch (lean_obj_tag(x_403)) { case 0: { -lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; lean_object* x_472; -x_465 = lean_ctor_get(x_464, 0); -lean_inc(x_465); -if (lean_is_exclusive(x_464)) { - lean_ctor_release(x_464, 0); - lean_ctor_release(x_464, 1); - x_466 = x_464; +lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; +x_404 = lean_ctor_get(x_403, 0); +lean_inc(x_404); +if (lean_is_exclusive(x_403)) { + lean_ctor_release(x_403, 0); + lean_ctor_release(x_403, 1); + x_405 = x_403; } else { - lean_dec_ref(x_464); - x_466 = lean_box(0); + lean_dec_ref(x_403); + x_405 = lean_box(0); } -x_467 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_466)) { - x_468 = lean_alloc_ctor(0, 2, 0); +x_406 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_405)) { + x_407 = lean_alloc_ctor(0, 2, 0); } else { - x_468 = x_466; + x_407 = x_405; } -lean_ctor_set(x_468, 0, x_465); -lean_ctor_set(x_468, 1, x_467); -x_469 = lean_unsigned_to_nat(1u); -x_470 = lean_mk_array(x_469, x_468); -x_471 = l_Array_append___rarg(x_435, x_470); -lean_dec(x_470); -x_472 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_472; -x_440 = x_471; -goto block_458; +lean_ctor_set(x_407, 0, x_404); +lean_ctor_set(x_407, 1, x_406); +x_392 = x_407; +goto block_397; } case 2: { -lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; -x_473 = lean_ctor_get(x_464, 0); -lean_inc(x_473); -lean_dec(x_464); -x_474 = l_Lake_LeanConfig_decodeToml___closed__5; -x_475 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_475, 0, x_473); -lean_ctor_set(x_475, 1, x_474); -x_476 = lean_unsigned_to_nat(1u); -x_477 = lean_mk_array(x_476, x_475); -x_478 = l_Array_append___rarg(x_435, x_477); -lean_dec(x_477); -x_479 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_479; -x_440 = x_478; -goto block_458; +lean_object* x_408; lean_object* x_409; lean_object* x_410; +x_408 = lean_ctor_get(x_403, 0); +lean_inc(x_408); +lean_dec(x_403); +x_409 = l_Lake_LeanConfig_decodeToml___closed__5; +x_410 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_410, 0, x_408); +lean_ctor_set(x_410, 1, x_409); +x_392 = x_410; +goto block_397; } case 3: { -lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; -x_480 = lean_ctor_get(x_464, 0); -lean_inc(x_480); -lean_dec(x_464); -x_481 = l_Lake_LeanConfig_decodeToml___closed__5; -x_482 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_482, 0, x_480); -lean_ctor_set(x_482, 1, x_481); -x_483 = lean_unsigned_to_nat(1u); -x_484 = lean_mk_array(x_483, x_482); -x_485 = l_Array_append___rarg(x_435, x_484); -lean_dec(x_484); -x_486 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_486; -x_440 = x_485; -goto block_458; +lean_object* x_411; lean_object* x_412; lean_object* x_413; +x_411 = lean_ctor_get(x_403, 0); +lean_inc(x_411); +lean_dec(x_403); +x_412 = l_Lake_LeanConfig_decodeToml___closed__5; +x_413 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_413, 0, x_411); +lean_ctor_set(x_413, 1, x_412); +x_392 = x_413; +goto block_397; } case 5: { -lean_object* x_487; lean_object* x_488; -x_487 = lean_ctor_get(x_464, 1); -lean_inc(x_487); -lean_dec(x_464); -x_488 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__9(x_487); -lean_dec(x_487); -if (lean_obj_tag(x_488) == 0) -{ -lean_object* x_489; lean_object* x_490; lean_object* x_491; -x_489 = lean_ctor_get(x_488, 0); -lean_inc(x_489); -lean_dec(x_488); -x_490 = l_Array_append___rarg(x_435, x_489); -lean_dec(x_489); -x_491 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_491; -x_440 = x_490; -goto block_458; +lean_object* x_414; lean_object* x_415; +x_414 = lean_ctor_get(x_403, 1); +lean_inc(x_414); +lean_dec(x_403); +x_415 = l_Lake_Toml_decodeArray___at_Lake_loadTomlConfig___spec__9(x_414); +lean_dec(x_414); +if (lean_obj_tag(x_415) == 0) +{ +lean_object* x_416; lean_object* x_417; lean_object* x_418; +x_416 = lean_ctor_get(x_415, 0); +lean_inc(x_416); +lean_dec(x_415); +x_417 = l_Array_append___rarg(x_367, x_416); +lean_dec(x_416); +x_418 = l_Lake_decodeLeanOptions___closed__1; +x_371 = x_418; +x_372 = x_417; +goto block_390; } else { -lean_object* x_492; -x_492 = lean_ctor_get(x_488, 0); -lean_inc(x_492); -lean_dec(x_488); -x_439 = x_492; -x_440 = x_435; -goto block_458; +lean_object* x_419; +x_419 = lean_ctor_get(x_415, 0); +lean_inc(x_419); +lean_dec(x_415); +x_371 = x_419; +x_372 = x_367; +goto block_390; } } default: { -lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_500; -x_493 = lean_ctor_get(x_464, 0); -lean_inc(x_493); -if (lean_is_exclusive(x_464)) { - lean_ctor_release(x_464, 0); - lean_ctor_release(x_464, 1); - x_494 = x_464; +lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; +x_420 = lean_ctor_get(x_403, 0); +lean_inc(x_420); +if (lean_is_exclusive(x_403)) { + lean_ctor_release(x_403, 0); + lean_ctor_release(x_403, 1); + x_421 = x_403; } else { - lean_dec_ref(x_464); - x_494 = lean_box(0); + lean_dec_ref(x_403); + x_421 = lean_box(0); } -x_495 = l_Lake_LeanConfig_decodeToml___closed__5; -if (lean_is_scalar(x_494)) { - x_496 = lean_alloc_ctor(0, 2, 0); +x_422 = l_Lake_LeanConfig_decodeToml___closed__5; +if (lean_is_scalar(x_421)) { + x_423 = lean_alloc_ctor(0, 2, 0); } else { - x_496 = x_494; - lean_ctor_set_tag(x_496, 0); -} -lean_ctor_set(x_496, 0, x_493); -lean_ctor_set(x_496, 1, x_495); -x_497 = lean_unsigned_to_nat(1u); -x_498 = lean_mk_array(x_497, x_496); -x_499 = l_Array_append___rarg(x_435, x_498); -lean_dec(x_498); -x_500 = l_Lake_decodeLeanOptions___closed__1; -x_439 = x_500; -x_440 = x_499; -goto block_458; + x_423 = x_421; + lean_ctor_set_tag(x_423, 0); } +lean_ctor_set(x_423, 0, x_420); +lean_ctor_set(x_423, 1, x_422); +x_392 = x_423; +goto block_397; } } -block_458: +} +block_390: { -lean_object* x_441; lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; -x_441 = lean_ctor_get(x_1, 2); -lean_inc(x_441); -x_442 = lean_ctor_get(x_1, 3); -lean_inc(x_442); -x_443 = l_System_FilePath_join(x_441, x_442); -x_444 = lean_ctor_get(x_428, 3); -lean_inc(x_444); -x_445 = lean_ctor_get(x_1, 8); -lean_inc(x_445); -x_446 = lean_ctor_get(x_1, 9); -lean_inc(x_446); +lean_object* x_373; lean_object* x_374; lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; +x_373 = lean_ctor_get(x_1, 2); +lean_inc(x_373); +x_374 = lean_ctor_get(x_1, 3); +lean_inc(x_374); +x_375 = l_System_FilePath_join(x_373, x_374); +x_376 = lean_ctor_get(x_360, 3); +lean_inc(x_376); +x_377 = lean_ctor_get(x_1, 8); +lean_inc(x_377); +x_378 = lean_ctor_get(x_1, 9); +lean_inc(x_378); lean_dec(x_1); -x_447 = lean_box(0); -if (lean_obj_tag(x_444) == 0) +x_379 = lean_box(0); +if (lean_obj_tag(x_376) == 0) +{ +lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; +x_380 = lean_ctor_get(x_360, 17); +lean_inc(x_380); +x_381 = lean_ctor_get(x_360, 19); +lean_inc(x_381); +x_382 = l_Lake_defaultManifestFile; +x_383 = l_Lake_decodeLeanOptions___closed__1; +x_384 = lean_alloc_ctor(0, 18, 0); +lean_ctor_set(x_384, 0, x_375); +lean_ctor_set(x_384, 1, x_374); +lean_ctor_set(x_384, 2, x_360); +lean_ctor_set(x_384, 3, x_304); +lean_ctor_set(x_384, 4, x_382); +lean_ctor_set(x_384, 5, x_377); +lean_ctor_set(x_384, 6, x_378); +lean_ctor_set(x_384, 7, x_371); +lean_ctor_set(x_384, 8, x_362); +lean_ctor_set(x_384, 9, x_364); +lean_ctor_set(x_384, 10, x_379); +lean_ctor_set(x_384, 11, x_379); +lean_ctor_set(x_384, 12, x_370); +lean_ctor_set(x_384, 13, x_379); +lean_ctor_set(x_384, 14, x_383); +lean_ctor_set(x_384, 15, x_383); +lean_ctor_set(x_384, 16, x_380); +lean_ctor_set(x_384, 17, x_381); +x_312 = x_384; +x_313 = x_372; +goto block_337; +} +else +{ +lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; +x_385 = lean_ctor_get(x_360, 17); +lean_inc(x_385); +x_386 = lean_ctor_get(x_360, 19); +lean_inc(x_386); +x_387 = lean_ctor_get(x_376, 0); +lean_inc(x_387); +lean_dec(x_376); +x_388 = l_Lake_decodeLeanOptions___closed__1; +x_389 = lean_alloc_ctor(0, 18, 0); +lean_ctor_set(x_389, 0, x_375); +lean_ctor_set(x_389, 1, x_374); +lean_ctor_set(x_389, 2, x_360); +lean_ctor_set(x_389, 3, x_304); +lean_ctor_set(x_389, 4, x_387); +lean_ctor_set(x_389, 5, x_377); +lean_ctor_set(x_389, 6, x_378); +lean_ctor_set(x_389, 7, x_371); +lean_ctor_set(x_389, 8, x_362); +lean_ctor_set(x_389, 9, x_364); +lean_ctor_set(x_389, 10, x_379); +lean_ctor_set(x_389, 11, x_379); +lean_ctor_set(x_389, 12, x_370); +lean_ctor_set(x_389, 13, x_379); +lean_ctor_set(x_389, 14, x_388); +lean_ctor_set(x_389, 15, x_388); +lean_ctor_set(x_389, 16, x_385); +lean_ctor_set(x_389, 17, x_386); +x_312 = x_389; +x_313 = x_372; +goto block_337; +} +} +block_397: +{ +lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; +x_393 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_393, 0, x_392); +lean_ctor_set(x_393, 1, x_391); +x_394 = lean_array_mk(x_393); +x_395 = l_Array_append___rarg(x_367, x_394); +lean_dec(x_394); +x_396 = l_Lake_decodeLeanOptions___closed__1; +x_371 = x_396; +x_372 = x_395; +goto block_390; +} +} +block_431: { -lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; -x_448 = lean_ctor_get(x_428, 17); -lean_inc(x_448); -x_449 = lean_ctor_get(x_428, 19); -lean_inc(x_449); -x_450 = l_Lake_defaultManifestFile; -x_451 = l_Lake_decodeLeanOptions___closed__1; -x_452 = lean_alloc_ctor(0, 18, 0); -lean_ctor_set(x_452, 0, x_443); -lean_ctor_set(x_452, 1, x_442); -lean_ctor_set(x_452, 2, x_428); -lean_ctor_set(x_452, 3, x_372); -lean_ctor_set(x_452, 4, x_450); -lean_ctor_set(x_452, 5, x_445); -lean_ctor_set(x_452, 6, x_446); -lean_ctor_set(x_452, 7, x_439); -lean_ctor_set(x_452, 8, x_430); -lean_ctor_set(x_452, 9, x_432); -lean_ctor_set(x_452, 10, x_447); -lean_ctor_set(x_452, 11, x_447); -lean_ctor_set(x_452, 12, x_438); -lean_ctor_set(x_452, 13, x_447); -lean_ctor_set(x_452, 14, x_451); -lean_ctor_set(x_452, 15, x_451); -lean_ctor_set(x_452, 16, x_448); -lean_ctor_set(x_452, 17, x_449); -x_380 = x_452; -x_381 = x_440; -goto block_405; -} -else -{ -lean_object* x_453; lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; -x_453 = lean_ctor_get(x_428, 17); -lean_inc(x_453); -x_454 = lean_ctor_get(x_428, 19); -lean_inc(x_454); -x_455 = lean_ctor_get(x_444, 0); -lean_inc(x_455); -lean_dec(x_444); -x_456 = l_Lake_decodeLeanOptions___closed__1; -x_457 = lean_alloc_ctor(0, 18, 0); -lean_ctor_set(x_457, 0, x_443); -lean_ctor_set(x_457, 1, x_442); -lean_ctor_set(x_457, 2, x_428); -lean_ctor_set(x_457, 3, x_372); -lean_ctor_set(x_457, 4, x_455); -lean_ctor_set(x_457, 5, x_445); -lean_ctor_set(x_457, 6, x_446); -lean_ctor_set(x_457, 7, x_439); -lean_ctor_set(x_457, 8, x_430); -lean_ctor_set(x_457, 9, x_432); -lean_ctor_set(x_457, 10, x_447); -lean_ctor_set(x_457, 11, x_447); -lean_ctor_set(x_457, 12, x_438); -lean_ctor_set(x_457, 13, x_447); -lean_ctor_set(x_457, 14, x_456); -lean_ctor_set(x_457, 15, x_456); -lean_ctor_set(x_457, 16, x_453); -lean_ctor_set(x_457, 17, x_454); -x_380 = x_457; -x_381 = x_440; -goto block_405; -} -} -} -} -block_556: -{ -lean_object* x_547; lean_object* x_548; lean_object* x_549; lean_object* x_550; uint8_t x_551; -x_547 = lean_array_get_size(x_545); -x_548 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_549 = l_Lake_RBArray_mkEmpty___rarg(x_548, x_547); -x_550 = lean_unsigned_to_nat(0u); -x_551 = lean_nat_dec_lt(x_550, x_547); -if (x_551 == 0) +lean_object* x_427; lean_object* x_428; lean_object* x_429; lean_object* x_430; +x_427 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_427, 0, x_426); +lean_ctor_set(x_427, 1, x_425); +x_428 = lean_array_mk(x_427); +x_429 = l_Array_append___rarg(x_365, x_428); +lean_dec(x_428); +x_430 = l_Lake_decodeLeanOptions___closed__1; +x_366 = x_430; +x_367 = x_429; +goto block_424; +} +} +block_470: { -lean_dec(x_547); -lean_dec(x_545); -x_432 = x_549; -x_433 = x_546; -goto block_544; +lean_object* x_461; lean_object* x_462; lean_object* x_463; lean_object* x_464; uint8_t x_465; +x_461 = lean_array_get_size(x_459); +x_462 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_463 = l_Lake_RBArray_mkEmpty___rarg(x_462, x_461); +x_464 = lean_unsigned_to_nat(0u); +x_465 = lean_nat_dec_lt(x_464, x_461); +if (x_465 == 0) +{ +lean_dec(x_461); +lean_dec(x_459); +x_364 = x_463; +x_365 = x_460; +goto block_458; } else { -uint8_t x_552; -x_552 = lean_nat_dec_le(x_547, x_547); -if (x_552 == 0) +uint8_t x_466; +x_466 = lean_nat_dec_le(x_461, x_461); +if (x_466 == 0) { -lean_dec(x_547); -lean_dec(x_545); -x_432 = x_549; -x_433 = x_546; -goto block_544; +lean_dec(x_461); +lean_dec(x_459); +x_364 = x_463; +x_365 = x_460; +goto block_458; } else { -size_t x_553; size_t x_554; lean_object* x_555; -x_553 = 0; -x_554 = lean_usize_of_nat(x_547); -lean_dec(x_547); -x_555 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__11(x_545, x_553, x_554, x_549); -lean_dec(x_545); -x_432 = x_555; -x_433 = x_546; -goto block_544; +size_t x_467; size_t x_468; lean_object* x_469; +x_467 = 0; +x_468 = lean_usize_of_nat(x_461); +lean_dec(x_461); +x_469 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__11(x_459, x_467, x_468, x_463); +lean_dec(x_459); +x_364 = x_469; +x_365 = x_460; +goto block_458; +} } } +block_477: +{ +lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; +x_473 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_473, 0, x_472); +lean_ctor_set(x_473, 1, x_471); +x_474 = lean_array_mk(x_473); +x_475 = l_Array_append___rarg(x_363, x_474); +lean_dec(x_474); +x_476 = l_Lake_decodeLeanOptions___closed__1; +x_459 = x_476; +x_460 = x_475; +goto block_470; } } -block_611: +block_516: { -lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; uint8_t x_606; -x_602 = lean_array_get_size(x_600); -x_603 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; -x_604 = l_Lake_RBArray_mkEmpty___rarg(x_603, x_602); -x_605 = lean_unsigned_to_nat(0u); -x_606 = lean_nat_dec_lt(x_605, x_602); -if (x_606 == 0) +lean_object* x_507; lean_object* x_508; lean_object* x_509; lean_object* x_510; uint8_t x_511; +x_507 = lean_array_get_size(x_505); +x_508 = l_Lake_Toml_Table_decode___at_Lake_LeanOption_decodeToml___spec__1___closed__1; +x_509 = l_Lake_RBArray_mkEmpty___rarg(x_508, x_507); +x_510 = lean_unsigned_to_nat(0u); +x_511 = lean_nat_dec_lt(x_510, x_507); +if (x_511 == 0) { -lean_dec(x_602); -lean_dec(x_600); -x_430 = x_604; -x_431 = x_601; -goto block_599; +lean_dec(x_507); +lean_dec(x_505); +x_362 = x_509; +x_363 = x_506; +goto block_504; } else { -uint8_t x_607; -x_607 = lean_nat_dec_le(x_602, x_602); -if (x_607 == 0) +uint8_t x_512; +x_512 = lean_nat_dec_le(x_507, x_507); +if (x_512 == 0) { -lean_dec(x_602); -lean_dec(x_600); -x_430 = x_604; -x_431 = x_601; -goto block_599; +lean_dec(x_507); +lean_dec(x_505); +x_362 = x_509; +x_363 = x_506; +goto block_504; } else { -size_t x_608; size_t x_609; lean_object* x_610; -x_608 = 0; -x_609 = lean_usize_of_nat(x_602); -lean_dec(x_602); -x_610 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__14(x_600, x_608, x_609, x_604); -lean_dec(x_600); -x_430 = x_610; -x_431 = x_601; -goto block_599; +size_t x_513; size_t x_514; lean_object* x_515; +x_513 = 0; +x_514 = lean_usize_of_nat(x_507); +lean_dec(x_507); +x_515 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__14(x_505, x_513, x_514, x_509); +lean_dec(x_505); +x_362 = x_515; +x_363 = x_506; +goto block_504; +} } } +block_523: +{ +lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; +x_519 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_519, 0, x_518); +lean_ctor_set(x_519, 1, x_517); +x_520 = lean_array_mk(x_519); +x_521 = l_Array_append___rarg(x_361, x_520); +lean_dec(x_520); +x_522 = l_Lake_decodeLeanOptions___closed__1; +x_505 = x_522; +x_506 = x_521; +goto block_516; } } } -block_405: +block_337: { -uint8_t x_382; -x_382 = l_Array_isEmpty___rarg(x_381); -if (x_382 == 0) +uint8_t x_314; +x_314 = l_Array_isEmpty___rarg(x_313); +if (x_314 == 0) { -lean_object* x_383; lean_object* x_384; uint8_t x_385; lean_object* x_386; -lean_dec(x_380); -x_383 = lean_array_get_size(x_381); -x_384 = lean_unsigned_to_nat(0u); -x_385 = lean_nat_dec_lt(x_384, x_383); -x_386 = lean_array_get_size(x_378); -if (x_385 == 0) -{ -lean_object* x_387; lean_object* x_388; -lean_dec(x_383); -lean_dec(x_381); -lean_dec(x_374); -if (lean_is_scalar(x_379)) { - x_387 = lean_alloc_ctor(1, 2, 0); +lean_object* x_315; lean_object* x_316; uint8_t x_317; lean_object* x_318; +lean_dec(x_312); +x_315 = lean_array_get_size(x_313); +x_316 = lean_unsigned_to_nat(0u); +x_317 = lean_nat_dec_lt(x_316, x_315); +x_318 = lean_array_get_size(x_310); +if (x_317 == 0) +{ +lean_object* x_319; lean_object* x_320; +lean_dec(x_315); +lean_dec(x_313); +lean_dec(x_306); +if (lean_is_scalar(x_311)) { + x_319 = lean_alloc_ctor(1, 2, 0); } else { - x_387 = x_379; - lean_ctor_set_tag(x_387, 1); + x_319 = x_311; + lean_ctor_set_tag(x_319, 1); } -lean_ctor_set(x_387, 0, x_386); -lean_ctor_set(x_387, 1, x_378); -x_388 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_388, 0, x_387); -lean_ctor_set(x_388, 1, x_376); -return x_388; +lean_ctor_set(x_319, 0, x_318); +lean_ctor_set(x_319, 1, x_310); +x_320 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_320, 0, x_319); +lean_ctor_set(x_320, 1, x_308); +return x_320; } else { -uint8_t x_389; -x_389 = lean_nat_dec_le(x_383, x_383); -if (x_389 == 0) +uint8_t x_321; +x_321 = lean_nat_dec_le(x_315, x_315); +if (x_321 == 0) { -lean_object* x_390; lean_object* x_391; -lean_dec(x_383); -lean_dec(x_381); -lean_dec(x_374); -if (lean_is_scalar(x_379)) { - x_390 = lean_alloc_ctor(1, 2, 0); +lean_object* x_322; lean_object* x_323; +lean_dec(x_315); +lean_dec(x_313); +lean_dec(x_306); +if (lean_is_scalar(x_311)) { + x_322 = lean_alloc_ctor(1, 2, 0); } else { - x_390 = x_379; - lean_ctor_set_tag(x_390, 1); + x_322 = x_311; + lean_ctor_set_tag(x_322, 1); } -lean_ctor_set(x_390, 0, x_386); -lean_ctor_set(x_390, 1, x_378); -x_391 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_391, 0, x_390); -lean_ctor_set(x_391, 1, x_376); -return x_391; +lean_ctor_set(x_322, 0, x_318); +lean_ctor_set(x_322, 1, x_310); +x_323 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_323, 0, x_322); +lean_ctor_set(x_323, 1, x_308); +return x_323; } else { -size_t x_392; size_t x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; lean_object* x_401; lean_object* x_402; -lean_dec(x_379); -x_392 = 0; -x_393 = lean_usize_of_nat(x_383); -lean_dec(x_383); -x_394 = lean_box(0); -x_395 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__1(x_374, x_381, x_392, x_393, x_394, x_378, x_376); -lean_dec(x_381); -x_396 = lean_ctor_get(x_395, 0); -lean_inc(x_396); -x_397 = lean_ctor_get(x_395, 1); -lean_inc(x_397); -if (lean_is_exclusive(x_395)) { - lean_ctor_release(x_395, 0); - lean_ctor_release(x_395, 1); - x_398 = x_395; +size_t x_324; size_t x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; +lean_dec(x_311); +x_324 = 0; +x_325 = lean_usize_of_nat(x_315); +lean_dec(x_315); +x_326 = lean_box(0); +x_327 = l_Array_foldlMUnsafe_fold___at_Lake_loadTomlConfig___spec__1(x_306, x_313, x_324, x_325, x_326, x_310, x_308); +lean_dec(x_313); +x_328 = lean_ctor_get(x_327, 0); +lean_inc(x_328); +x_329 = lean_ctor_get(x_327, 1); +lean_inc(x_329); +if (lean_is_exclusive(x_327)) { + lean_ctor_release(x_327, 0); + lean_ctor_release(x_327, 1); + x_330 = x_327; } else { - lean_dec_ref(x_395); - x_398 = lean_box(0); -} -x_399 = lean_ctor_get(x_396, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_396)) { - lean_ctor_release(x_396, 0); - lean_ctor_release(x_396, 1); - x_400 = x_396; + lean_dec_ref(x_327); + x_330 = lean_box(0); +} +x_331 = lean_ctor_get(x_328, 1); +lean_inc(x_331); +if (lean_is_exclusive(x_328)) { + lean_ctor_release(x_328, 0); + lean_ctor_release(x_328, 1); + x_332 = x_328; } else { - lean_dec_ref(x_396); - x_400 = lean_box(0); + lean_dec_ref(x_328); + x_332 = lean_box(0); } -if (lean_is_scalar(x_400)) { - x_401 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_332)) { + x_333 = lean_alloc_ctor(1, 2, 0); } else { - x_401 = x_400; - lean_ctor_set_tag(x_401, 1); + x_333 = x_332; + lean_ctor_set_tag(x_333, 1); } -lean_ctor_set(x_401, 0, x_386); -lean_ctor_set(x_401, 1, x_399); -if (lean_is_scalar(x_398)) { - x_402 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_333, 0, x_318); +lean_ctor_set(x_333, 1, x_331); +if (lean_is_scalar(x_330)) { + x_334 = lean_alloc_ctor(0, 2, 0); } else { - x_402 = x_398; + x_334 = x_330; } -lean_ctor_set(x_402, 0, x_401); -lean_ctor_set(x_402, 1, x_397); -return x_402; +lean_ctor_set(x_334, 0, x_333); +lean_ctor_set(x_334, 1, x_329); +return x_334; } } } else { -lean_object* x_403; lean_object* x_404; -lean_dec(x_381); -lean_dec(x_374); -if (lean_is_scalar(x_379)) { - x_403 = lean_alloc_ctor(0, 2, 0); +lean_object* x_335; lean_object* x_336; +lean_dec(x_313); +lean_dec(x_306); +if (lean_is_scalar(x_311)) { + x_335 = lean_alloc_ctor(0, 2, 0); } else { - x_403 = x_379; + x_335 = x_311; } -lean_ctor_set(x_403, 0, x_380); -lean_ctor_set(x_403, 1, x_378); -x_404 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_404, 0, x_403); -lean_ctor_set(x_404, 1, x_376); -return x_404; +lean_ctor_set(x_335, 0, x_312); +lean_ctor_set(x_335, 1, x_310); +x_336 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_336, 0, x_335); +lean_ctor_set(x_336, 1, x_308); +return x_336; } } } @@ -25427,32 +28975,32 @@ return x_404; } else { -uint8_t x_673; +uint8_t x_569; lean_dec(x_1); -x_673 = !lean_is_exclusive(x_4); -if (x_673 == 0) +x_569 = !lean_is_exclusive(x_4); +if (x_569 == 0) { -lean_object* x_674; -x_674 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_674, 0, x_4); -lean_ctor_set(x_674, 1, x_5); -return x_674; +lean_object* x_570; +x_570 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_570, 0, x_4); +lean_ctor_set(x_570, 1, x_5); +return x_570; } else { -lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; -x_675 = lean_ctor_get(x_4, 0); -x_676 = lean_ctor_get(x_4, 1); -lean_inc(x_676); -lean_inc(x_675); +lean_object* x_571; lean_object* x_572; lean_object* x_573; lean_object* x_574; +x_571 = lean_ctor_get(x_4, 0); +x_572 = lean_ctor_get(x_4, 1); +lean_inc(x_572); +lean_inc(x_571); lean_dec(x_4); -x_677 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_677, 0, x_675); -lean_ctor_set(x_677, 1, x_676); -x_678 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_678, 0, x_677); -lean_ctor_set(x_678, 1, x_5); -return x_678; +x_573 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_573, 0, x_571); +lean_ctor_set(x_573, 1, x_572); +x_574 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_574, 0, x_573); +lean_ctor_set(x_574, 1, x_5); +return x_574; } } } @@ -25699,10 +29247,10 @@ lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__3); l_Lake_LeanOption_decodeToml___closed__4 = _init_l_Lake_LeanOption_decodeToml___closed__4(); lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__4); l_Lake_LeanOption_decodeToml___closed__5 = _init_l_Lake_LeanOption_decodeToml___closed__5(); -lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__5); l_Lake_LeanOption_decodeToml___closed__6 = _init_l_Lake_LeanOption_decodeToml___closed__6(); lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__6); l_Lake_LeanOption_decodeToml___closed__7 = _init_l_Lake_LeanOption_decodeToml___closed__7(); +lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__7); l_Lake_LeanOption_decodeToml___closed__8 = _init_l_Lake_LeanOption_decodeToml___closed__8(); lean_mark_persistent(l_Lake_LeanOption_decodeToml___closed__8); l_Lake_LeanOption_decodeToml___closed__9 = _init_l_Lake_LeanOption_decodeToml___closed__9(); @@ -25777,8 +29325,16 @@ l_Lake_WorkspaceConfig_decodeToml___closed__1 = _init_l_Lake_WorkspaceConfig_dec lean_mark_persistent(l_Lake_WorkspaceConfig_decodeToml___closed__1); l_Lake_WorkspaceConfig_decodeToml___closed__2 = _init_l_Lake_WorkspaceConfig_decodeToml___closed__2(); lean_mark_persistent(l_Lake_WorkspaceConfig_decodeToml___closed__2); +l_Lake_WorkspaceConfig_decodeToml___closed__3 = _init_l_Lake_WorkspaceConfig_decodeToml___closed__3(); +lean_mark_persistent(l_Lake_WorkspaceConfig_decodeToml___closed__3); +l_Lake_WorkspaceConfig_decodeToml___closed__4 = _init_l_Lake_WorkspaceConfig_decodeToml___closed__4(); +lean_mark_persistent(l_Lake_WorkspaceConfig_decodeToml___closed__4); +l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1 = _init_l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlWorkspaceConfig___lambda__1___closed__1); l_Lake_instDecodeTomlWorkspaceConfig___closed__1 = _init_l_Lake_instDecodeTomlWorkspaceConfig___closed__1(); lean_mark_persistent(l_Lake_instDecodeTomlWorkspaceConfig___closed__1); +l_Lake_instDecodeTomlWorkspaceConfig = _init_l_Lake_instDecodeTomlWorkspaceConfig(); +lean_mark_persistent(l_Lake_instDecodeTomlWorkspaceConfig); l_Lake_LeanConfig_decodeToml___closed__1 = _init_l_Lake_LeanConfig_decodeToml___closed__1(); lean_mark_persistent(l_Lake_LeanConfig_decodeToml___closed__1); l_Lake_LeanConfig_decodeToml___closed__2 = _init_l_Lake_LeanConfig_decodeToml___closed__2(); @@ -25827,6 +29383,10 @@ l_Lake_LeanConfig_decodeToml___closed__23 = _init_l_Lake_LeanConfig_decodeToml__ lean_mark_persistent(l_Lake_LeanConfig_decodeToml___closed__23); l_Lake_LeanConfig_decodeToml___closed__24 = _init_l_Lake_LeanConfig_decodeToml___closed__24(); lean_mark_persistent(l_Lake_LeanConfig_decodeToml___closed__24); +l_Lake_instDecodeTomlLeanConfig___closed__1 = _init_l_Lake_instDecodeTomlLeanConfig___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanConfig___closed__1); +l_Lake_instDecodeTomlLeanConfig = _init_l_Lake_instDecodeTomlLeanConfig(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanConfig); l_Lake_PackageConfig_decodeToml___closed__1 = _init_l_Lake_PackageConfig_decodeToml___closed__1(); lean_mark_persistent(l_Lake_PackageConfig_decodeToml___closed__1); l_Lake_PackageConfig_decodeToml___closed__2 = _init_l_Lake_PackageConfig_decodeToml___closed__2(); @@ -25949,6 +29509,10 @@ l_Lake_PackageConfig_decodeToml___closed__61 = _init_l_Lake_PackageConfig_decode lean_mark_persistent(l_Lake_PackageConfig_decodeToml___closed__61); l_Lake_PackageConfig_decodeToml___closed__62 = _init_l_Lake_PackageConfig_decodeToml___closed__62(); lean_mark_persistent(l_Lake_PackageConfig_decodeToml___closed__62); +l_Lake_instDecodeTomlPackageConfig___closed__1 = _init_l_Lake_instDecodeTomlPackageConfig___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlPackageConfig___closed__1); +l_Lake_instDecodeTomlPackageConfig = _init_l_Lake_instDecodeTomlPackageConfig(); +lean_mark_persistent(l_Lake_instDecodeTomlPackageConfig); l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__1 = _init_l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__1(); lean_mark_persistent(l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__1); l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__2 = _init_l_Lake_LeanLibConfig_decodeToml___lambda__1___closed__2(); @@ -25981,6 +29545,10 @@ l_Lake_LeanLibConfig_decodeToml___closed__11 = _init_l_Lake_LeanLibConfig_decode lean_mark_persistent(l_Lake_LeanLibConfig_decodeToml___closed__11); l_Lake_LeanLibConfig_decodeToml___closed__12 = _init_l_Lake_LeanLibConfig_decodeToml___closed__12(); lean_mark_persistent(l_Lake_LeanLibConfig_decodeToml___closed__12); +l_Lake_instDecodeTomlLeanLibConfig___closed__1 = _init_l_Lake_instDecodeTomlLeanLibConfig___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanLibConfig___closed__1); +l_Lake_instDecodeTomlLeanLibConfig = _init_l_Lake_instDecodeTomlLeanLibConfig(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanLibConfig); l_Lake_LeanExeConfig_decodeToml___closed__1 = _init_l_Lake_LeanExeConfig_decodeToml___closed__1(); lean_mark_persistent(l_Lake_LeanExeConfig_decodeToml___closed__1); l_Lake_LeanExeConfig_decodeToml___closed__2 = _init_l_Lake_LeanExeConfig_decodeToml___closed__2(); @@ -25995,6 +29563,10 @@ l_Lake_LeanExeConfig_decodeToml___closed__6 = _init_l_Lake_LeanExeConfig_decodeT lean_mark_persistent(l_Lake_LeanExeConfig_decodeToml___closed__6); l_Lake_LeanExeConfig_decodeToml___closed__7 = _init_l_Lake_LeanExeConfig_decodeToml___closed__7(); lean_mark_persistent(l_Lake_LeanExeConfig_decodeToml___closed__7); +l_Lake_instDecodeTomlLeanExeConfig___closed__1 = _init_l_Lake_instDecodeTomlLeanExeConfig___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanExeConfig___closed__1); +l_Lake_instDecodeTomlLeanExeConfig = _init_l_Lake_instDecodeTomlLeanExeConfig(); +lean_mark_persistent(l_Lake_instDecodeTomlLeanExeConfig); l_Lake_DependencySrc_decodeToml___closed__1 = _init_l_Lake_DependencySrc_decodeToml___closed__1(); lean_mark_persistent(l_Lake_DependencySrc_decodeToml___closed__1); l_Lake_DependencySrc_decodeToml___closed__2 = _init_l_Lake_DependencySrc_decodeToml___closed__2(); @@ -26033,6 +29605,12 @@ l_Lake_DependencySrc_decodeToml___closed__18 = _init_l_Lake_DependencySrc_decode lean_mark_persistent(l_Lake_DependencySrc_decodeToml___closed__18); l_Lake_DependencySrc_decodeToml___closed__19 = _init_l_Lake_DependencySrc_decodeToml___closed__19(); lean_mark_persistent(l_Lake_DependencySrc_decodeToml___closed__19); +l_Lake_DependencySrc_decodeToml___closed__20 = _init_l_Lake_DependencySrc_decodeToml___closed__20(); +lean_mark_persistent(l_Lake_DependencySrc_decodeToml___closed__20); +l_Lake_instDecodeTomlDependencySrc___closed__1 = _init_l_Lake_instDecodeTomlDependencySrc___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlDependencySrc___closed__1); +l_Lake_instDecodeTomlDependencySrc = _init_l_Lake_instDecodeTomlDependencySrc(); +lean_mark_persistent(l_Lake_instDecodeTomlDependencySrc); l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1___closed__1 = _init_l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1___closed__1(); lean_mark_persistent(l_Lake_Toml_Table_decodeNameMap___at_Lake_Dependency_decodeToml___spec__1___closed__1); l_Lake_Dependency_decodeToml___closed__1 = _init_l_Lake_Dependency_decodeToml___closed__1(); @@ -26055,6 +29633,10 @@ l_Lake_Dependency_decodeToml___closed__9 = _init_l_Lake_Dependency_decodeToml___ lean_mark_persistent(l_Lake_Dependency_decodeToml___closed__9); l_Lake_Dependency_decodeToml___closed__10 = _init_l_Lake_Dependency_decodeToml___closed__10(); lean_mark_persistent(l_Lake_Dependency_decodeToml___closed__10); +l_Lake_instDecodeTomlDependency___closed__1 = _init_l_Lake_instDecodeTomlDependency___closed__1(); +lean_mark_persistent(l_Lake_instDecodeTomlDependency___closed__1); +l_Lake_instDecodeTomlDependency = _init_l_Lake_instDecodeTomlDependency(); +lean_mark_persistent(l_Lake_instDecodeTomlDependency); l_Lake_loadTomlConfig___closed__1 = _init_l_Lake_loadTomlConfig___closed__1(); lean_mark_persistent(l_Lake_loadTomlConfig___closed__1); l_Lake_loadTomlConfig___closed__2 = _init_l_Lake_loadTomlConfig___closed__2(); diff --git a/stage0/stdlib/Lake/Toml/Decode.c b/stage0/stdlib/Lake/Toml/Decode.c index 3d630bc1c0d5..8f71331d8092 100644 --- a/stage0/stdlib/Lake/Toml/Decode.c +++ b/stage0/stdlib/Lake/Toml/Decode.c @@ -13,25 +13,26 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlName(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlName; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_Table_decodeNameMap___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_decode(lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lake_instMonadLiftExceptArray__lake(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlBool(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlBool; LEAN_EXPORT lean_object* l_Lake_Toml_Table_tryDecodeD(lean_object*); +static lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1; lean_object* l_Array_push___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlTable(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlTable; lean_object* l_Lake_Toml_ppKey(lean_object*); LEAN_EXPORT lean_object* l_Lake_optDecodeD___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Toml_Value_decodeName___closed__1; static lean_object* l_Lake_Toml_Value_decodeString___closed__1; -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFilePath(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFilePath; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___rarg(lean_object*, lean_object*); -lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_tryDecode_x3f(lean_object*); +static lean_object* l_Lake_Toml_Value_instDecodeTomlNat___closed__1; LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeString(lean_object*); LEAN_EXPORT lean_object* l_Lake_optDecode_x3f(lean_object*, lean_object*, lean_object*); @@ -43,7 +44,11 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_Table_decodeNa LEAN_EXPORT lean_object* l_Lake_mergeErrors(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_decodeArray___spec__1___rarg___closed__1; LEAN_EXPORT lean_object* l_Lake_tryDecodeD___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlString___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_optDecodeD(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFloat___lambda__1(lean_object*); +static lean_object* l_Lake_Toml_Value_instDecodeTomlTable___closed__1; LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArray___rarg(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); static lean_object* l_Lake_ensureDecode___rarg___closed__1; @@ -58,10 +63,13 @@ LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeNat(lean_object*); lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_Table_decodeNameMap___spec__1(lean_object*); lean_object* l_Lean_Name_quickCmp___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlNat___lambda__1(lean_object*); lean_object* l_Except_pure___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeDateTime(lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlInt(lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlNat(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlInt; +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlNat; +static lean_object* l_Lake_Toml_Value_instDecodeTomlBool___closed__1; +static lean_object* l_Lake_Toml_Value_instDecodeTomlString___closed__1; LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArrayOrSingleton(lean_object*); static lean_object* l_Lake_Toml_Value_decodeNat___closed__1; LEAN_EXPORT lean_object* l_Lake_optDecode_x3f___rarg(lean_object*, lean_object*, lean_object*); @@ -71,19 +79,23 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1 static lean_object* l_Lake_Toml_Value_decodeBool___closed__1; static lean_object* l_Lake_Toml_Table_decode_x3f___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_decodeArray___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFloat(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFloat; lean_object* l_Lean_RBNode_insert___at_Lean_NameMap_insert___spec__1___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_tryDecodeD___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_tryDecode(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeFloat(lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlString(lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg___lambda__1(lean_object*, lean_object*); +static lean_object* l_Lake_Toml_Value_instDecodeTomlFloat___closed__1; +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlString; +LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg(lean_object*); static lean_object* l_Lake_Toml_Table_decodeValue___closed__3; LEAN_EXPORT lean_object* l_Lake_Toml_decodeArray___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray___rarg(lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_tryDecode(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lake_Toml_decodeArray___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lake_Toml_Value_instDecodeTomlInt___closed__1; +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlBool___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeValueArray(lean_object*); lean_object* lean_nat_abs(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -92,8 +104,9 @@ static lean_object* l_Lake_Toml_Value_decodeDateTime___closed__1; LEAN_EXPORT lean_object* l_Lake_tryDecode___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_decodeToml(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_decode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime; LEAN_EXPORT lean_object* l_Lake_ensureDecode___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlName___lambda__1(lean_object*); static lean_object* l_Lake_Toml_Table_decodeValue___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1(lean_object*, size_t, size_t, lean_object*); @@ -108,9 +121,11 @@ lean_object* l_String_toName(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray(lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_tryDecodeD___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlInt___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_optDecode(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeName(lean_object*); static lean_object* l_Lake_Toml_Value_decodeValueArray___closed__1; +lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lake_instMonadLiftExceptArray__lake___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_optDecode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Toml_Value_decodeNat___closed__2; @@ -130,9 +145,11 @@ LEAN_EXPORT lean_object* l_Lake_decodeToml___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_decodeKeyval(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeBool(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlTable___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_decodeNameMap___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lake_Toml_Table_tryDecode_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lake_Toml_Value_decodeInt___closed__1; +static lean_object* l_Lake_Toml_Value_instDecodeTomlName___closed__1; uint8_t l_Array_isEmpty___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lake_instMonadLiftExceptArray__lake___rarg(lean_object* x_1) { _start: @@ -143,43 +160,49 @@ uint8_t x_2; x_2 = !lean_is_exclusive(x_1); if (x_2 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_3 = lean_ctor_get(x_1, 0); -x_4 = lean_unsigned_to_nat(1u); -x_5 = lean_mk_array(x_4, x_3); -lean_ctor_set(x_1, 0, x_5); +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +lean_ctor_set(x_1, 0, x_6); return x_1; } else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_6 = lean_ctor_get(x_1, 0); -lean_inc(x_6); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); lean_dec(x_1); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_mk_array(x_7, x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_7); +lean_ctor_set(x_9, 1, x_8); +x_10 = lean_array_mk(x_9); +x_11 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } else { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_1); -if (x_10 == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_1); +if (x_12 == 0) { return x_1; } else { -lean_object* x_11; lean_object* x_12; -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); lean_dec(x_1); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -return x_12; +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +return x_14; } } } @@ -882,39 +905,24 @@ return x_19; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlString(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlString___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_2; lean_object* x_3; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -lean_dec(x_1); -x_3 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_3, 0, x_2); -return x_3; -} -case 2: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_1, 1); +lean_inc(x_8); lean_dec(x_1); -x_5 = l_Lake_Toml_Value_decodeString___closed__1; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_mk_array(x_7, x_6); -x_9 = lean_alloc_ctor(0, 1, 0); +x_9 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_9, 0, x_8); return x_9; } -case 3: +case 2: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_10; lean_object* x_11; lean_object* x_12; x_10 = lean_ctor_get(x_1, 0); lean_inc(x_10); lean_dec(x_1); @@ -922,11 +930,21 @@ x_11 = l_Lake_Toml_Value_decodeString___closed__1; x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_10); lean_ctor_set(x_12, 1, x_11); -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_mk_array(x_13, x_12); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +x_2 = x_12; +goto block_7; +} +case 3: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +lean_dec(x_1); +x_14 = l_Lake_Toml_Value_decodeString___closed__1; +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +x_2 = x_15; +goto block_7; } default: { @@ -934,120 +952,66 @@ uint8_t x_16; x_16 = !lean_is_exclusive(x_1); if (x_16 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_17; lean_object* x_18; x_17 = lean_ctor_get(x_1, 1); lean_dec(x_17); x_18 = l_Lake_Toml_Value_decodeString___closed__1; lean_ctor_set_tag(x_1, 0); lean_ctor_set(x_1, 1, x_18); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_1); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -return x_21; +x_2 = x_1; +goto block_7; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_22 = lean_ctor_get(x_1, 0); -lean_inc(x_22); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); lean_dec(x_1); -x_23 = l_Lake_Toml_Value_decodeString___closed__1; -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_mk_array(x_25, x_24); -x_27 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; +x_20 = l_Lake_Toml_Value_decodeString___closed__1; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_2 = x_21; +goto block_7; +} } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFilePath(lean_object* x_1) { +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlString___closed__1() { _start: { -switch (lean_obj_tag(x_1)) { -case 0: -{ -lean_object* x_2; lean_object* x_3; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -lean_dec(x_1); -x_3 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_3, 0, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlString___lambda__1), 1, 0); +return x_1; } -case 2: -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_4 = lean_ctor_get(x_1, 0); -lean_inc(x_4); -lean_dec(x_1); -x_5 = l_Lake_Toml_Value_decodeString___closed__1; -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_4); -lean_ctor_set(x_6, 1, x_5); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_mk_array(x_7, x_6); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; } -case 3: +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlString() { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -lean_dec(x_1); -x_11 = l_Lake_Toml_Value_decodeString___closed__1; -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_10); -lean_ctor_set(x_12, 1, x_11); -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_mk_array(x_13, x_12); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlString___closed__1; +return x_1; } -default: -{ -uint8_t x_16; -x_16 = !lean_is_exclusive(x_1); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_1, 1); -lean_dec(x_17); -x_18 = l_Lake_Toml_Value_decodeString___closed__1; -lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_18); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_1); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -return x_21; } -else +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlFilePath() { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_22 = lean_ctor_get(x_1, 0); -lean_inc(x_22); -lean_dec(x_1); -x_23 = l_Lake_Toml_Value_decodeString___closed__1; -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_mk_array(x_25, x_24); -x_27 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; -} -} -} +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlString___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeName___closed__1() { @@ -1183,76 +1147,71 @@ return x_31; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlName(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlName___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -x_4 = lean_ctor_get(x_1, 1); -x_5 = l_String_toName(x_4); -if (lean_obj_tag(x_5) == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +x_11 = l_String_toName(x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; -x_6 = l_Lake_Toml_Value_decodeName___closed__1; -lean_ctor_set(x_1, 1, x_6); -x_7 = lean_unsigned_to_nat(1u); -x_8 = lean_mk_array(x_7, x_1); -x_9 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_9, 0, x_8); -return x_9; +lean_object* x_12; +x_12 = l_Lake_Toml_Value_decodeName___closed__1; +lean_ctor_set(x_1, 1, x_12); +x_2 = x_1; +goto block_7; } else { -lean_object* x_10; +lean_object* x_13; lean_free_object(x_1); -lean_dec(x_3); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_5); -return x_10; +lean_dec(x_9); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_11); +return x_13; } } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_1, 0); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -lean_inc(x_11); +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_1, 0); +x_15 = lean_ctor_get(x_1, 1); +lean_inc(x_15); +lean_inc(x_14); lean_dec(x_1); -x_13 = l_String_toName(x_12); -if (lean_obj_tag(x_13) == 0) +x_16 = l_String_toName(x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_14 = l_Lake_Toml_Value_decodeName___closed__1; -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_11); -lean_ctor_set(x_15, 1, x_14); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_mk_array(x_16, x_15); -x_18 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_18, 0, x_17); -return x_18; +lean_object* x_17; lean_object* x_18; +x_17 = l_Lake_Toml_Value_decodeName___closed__1; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_14); +lean_ctor_set(x_18, 1, x_17); +x_2 = x_18; +goto block_7; } else { lean_object* x_19; -lean_dec(x_11); +lean_dec(x_14); x_19 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_19, 0, x_13); +lean_ctor_set(x_19, 0, x_16); return x_19; } } } case 2: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_object* x_20; lean_object* x_21; lean_object* x_22; x_20 = lean_ctor_get(x_1, 0); lean_inc(x_20); lean_dec(x_1); @@ -1260,64 +1219,80 @@ x_21 = l_Lake_Toml_Value_decodeString___closed__1; x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_2 = x_22; +goto block_7; } case 3: { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_26 = lean_ctor_get(x_1, 0); -lean_inc(x_26); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); lean_dec(x_1); -x_27 = l_Lake_Toml_Value_decodeString___closed__1; -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_unsigned_to_nat(1u); -x_30 = lean_mk_array(x_29, x_28); -x_31 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_31, 0, x_30); -return x_31; +x_24 = l_Lake_Toml_Value_decodeString___closed__1; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_2 = x_25; +goto block_7; } default: { -uint8_t x_32; -x_32 = !lean_is_exclusive(x_1); -if (x_32 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_1); +if (x_26 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_33 = lean_ctor_get(x_1, 1); -lean_dec(x_33); -x_34 = l_Lake_Toml_Value_decodeString___closed__1; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_1, 1); +lean_dec(x_27); +x_28 = l_Lake_Toml_Value_decodeString___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_34); -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_mk_array(x_35, x_1); -x_37 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_37, 0, x_36); -return x_37; +lean_ctor_set(x_1, 1, x_28); +x_2 = x_1; +goto block_7; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_38 = lean_ctor_get(x_1, 0); -lean_inc(x_38); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_1, 0); +lean_inc(x_29); lean_dec(x_1); -x_39 = l_Lake_Toml_Value_decodeString___closed__1; -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -x_41 = lean_unsigned_to_nat(1u); -x_42 = lean_mk_array(x_41, x_40); -x_43 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_43, 0, x_42); -return x_43; +x_30 = l_Lake_Toml_Value_decodeString___closed__1; +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +x_2 = x_31; +goto block_7; +} } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +} +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlName___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlName___lambda__1), 1, 0); +return x_1; +} } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlName() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlName___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeInt___closed__1() { @@ -1434,43 +1409,38 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlInt(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlInt___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeInt___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeInt___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeInt___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; -} +x_12 = l_Lake_Toml_Value_decodeInt___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; +} } case 1: { @@ -1484,7 +1454,7 @@ return x_15; } case 2: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_object* x_16; lean_object* x_17; lean_object* x_18; x_16 = lean_ctor_get(x_1, 0); lean_inc(x_16); lean_dec(x_1); @@ -1492,65 +1462,81 @@ x_17 = l_Lake_Toml_Value_decodeInt___closed__1; x_18 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_18, 0, x_16); lean_ctor_set(x_18, 1, x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_mk_array(x_19, x_18); -x_21 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_21, 0, x_20); -return x_21; +x_2 = x_18; +goto block_7; } case 3: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_22 = lean_ctor_get(x_1, 0); -lean_inc(x_22); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_1, 0); +lean_inc(x_19); lean_dec(x_1); -x_23 = l_Lake_Toml_Value_decodeInt___closed__1; -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_unsigned_to_nat(1u); -x_26 = lean_mk_array(x_25, x_24); -x_27 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; +x_20 = l_Lake_Toml_Value_decodeInt___closed__1; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_2 = x_21; +goto block_7; } default: { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_1); -if (x_28 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_1, 1); -lean_dec(x_29); -x_30 = l_Lake_Toml_Value_decodeInt___closed__1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = l_Lake_Toml_Value_decodeInt___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_mk_array(x_31, x_1); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +lean_ctor_set(x_1, 1, x_24); +x_2 = x_1; +goto block_7; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); lean_dec(x_1); -x_35 = l_Lake_Toml_Value_decodeInt___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_39, 0, x_38); -return x_39; +x_26 = l_Lake_Toml_Value_decodeInt___closed__1; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_2 = x_27; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlInt___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlInt___lambda__1), 1, 0); +return x_1; } } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlInt() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlInt___closed__1; +return x_1; +} } static lean_object* _init_l_Lake_Toml_Value_decodeNat___closed__1() { _start: @@ -1733,42 +1719,37 @@ return x_43; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlNat(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlNat___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeNat___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeNat___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeNat___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_Toml_Value_decodeNat___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 1: @@ -1795,122 +1776,132 @@ return x_20; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_21; lean_dec(x_16); x_21 = l_Lake_Toml_Value_decodeNat___closed__1; lean_ctor_set_tag(x_1, 0); lean_ctor_set(x_1, 1, x_21); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_mk_array(x_22, x_1); -x_24 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_24, 0, x_23); -return x_24; +x_2 = x_1; +goto block_7; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_25 = lean_ctor_get(x_1, 0); -x_26 = lean_ctor_get(x_1, 1); -lean_inc(x_26); -lean_inc(x_25); +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_22 = lean_ctor_get(x_1, 0); +x_23 = lean_ctor_get(x_1, 1); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_1); -x_27 = l_Lake_Toml_Value_decodeNat___closed__2; -x_28 = lean_int_dec_lt(x_26, x_27); -if (x_28 == 0) +x_24 = l_Lake_Toml_Value_decodeNat___closed__2; +x_25 = lean_int_dec_lt(x_23, x_24); +if (x_25 == 0) { -lean_object* x_29; lean_object* x_30; -lean_dec(x_25); -x_29 = lean_nat_abs(x_26); -lean_dec(x_26); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -return x_30; +lean_object* x_26; lean_object* x_27; +lean_dec(x_22); +x_26 = lean_nat_abs(x_23); +lean_dec(x_23); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_26); +return x_27; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_dec(x_26); -x_31 = l_Lake_Toml_Value_decodeNat___closed__1; -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_25); -lean_ctor_set(x_32, 1, x_31); -x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_mk_array(x_33, x_32); -x_35 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_35, 0, x_34); -return x_35; +lean_object* x_28; lean_object* x_29; +lean_dec(x_23); +x_28 = l_Lake_Toml_Value_decodeNat___closed__1; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_22); +lean_ctor_set(x_29, 1, x_28); +x_2 = x_29; +goto block_7; } } } case 2: { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_36 = lean_ctor_get(x_1, 0); -lean_inc(x_36); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_1, 0); +lean_inc(x_30); lean_dec(x_1); -x_37 = l_Lake_Toml_Value_decodeNat___closed__1; -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_mk_array(x_39, x_38); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -return x_41; +x_31 = l_Lake_Toml_Value_decodeNat___closed__1; +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_2 = x_32; +goto block_7; } case 3: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_42 = lean_ctor_get(x_1, 0); -lean_inc(x_42); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_1, 0); +lean_inc(x_33); lean_dec(x_1); -x_43 = l_Lake_Toml_Value_decodeNat___closed__1; -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_unsigned_to_nat(1u); -x_46 = lean_mk_array(x_45, x_44); -x_47 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_47, 0, x_46); -return x_47; +x_34 = l_Lake_Toml_Value_decodeNat___closed__1; +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_2 = x_35; +goto block_7; } default: { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_1); -if (x_48 == 0) +uint8_t x_36; +x_36 = !lean_is_exclusive(x_1); +if (x_36 == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_49 = lean_ctor_get(x_1, 1); -lean_dec(x_49); -x_50 = l_Lake_Toml_Value_decodeNat___closed__1; +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_1, 1); +lean_dec(x_37); +x_38 = l_Lake_Toml_Value_decodeNat___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_50); -x_51 = lean_unsigned_to_nat(1u); -x_52 = lean_mk_array(x_51, x_1); -x_53 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_53, 0, x_52); -return x_53; +lean_ctor_set(x_1, 1, x_38); +x_2 = x_1; +goto block_7; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_54 = lean_ctor_get(x_1, 0); -lean_inc(x_54); +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_1, 0); +lean_inc(x_39); lean_dec(x_1); -x_55 = l_Lake_Toml_Value_decodeNat___closed__1; -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -x_57 = lean_unsigned_to_nat(1u); -x_58 = lean_mk_array(x_57, x_56); -x_59 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_59, 0, x_58); -return x_59; +x_40 = l_Lake_Toml_Value_decodeNat___closed__1; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_2 = x_41; +goto block_7; } } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +} +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlNat___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlNat___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlNat() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlNat___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeFloat___closed__1() { @@ -2013,42 +2004,37 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFloat(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlFloat___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeFloat___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeFloat___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeFloat___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_Toml_Value_decodeFloat___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: @@ -2063,7 +2049,7 @@ return x_16; } case 3: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_object* x_17; lean_object* x_18; lean_object* x_19; x_17 = lean_ctor_get(x_1, 0); lean_inc(x_17); lean_dec(x_1); @@ -2071,48 +2057,67 @@ x_18 = l_Lake_Toml_Value_decodeFloat___closed__1; x_19 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); -x_20 = lean_unsigned_to_nat(1u); -x_21 = lean_mk_array(x_20, x_19); -x_22 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_22, 0, x_21); -return x_22; +x_2 = x_19; +goto block_7; } default: { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_1); -if (x_23 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_1); +if (x_20 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_1, 1); -lean_dec(x_24); -x_25 = l_Lake_Toml_Value_decodeFloat___closed__1; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_1, 1); +lean_dec(x_21); +x_22 = l_Lake_Toml_Value_decodeFloat___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_25); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_1); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -return x_28; +lean_ctor_set(x_1, 1, x_22); +x_2 = x_1; +goto block_7; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_29 = lean_ctor_get(x_1, 0); -lean_inc(x_29); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); lean_dec(x_1); -x_30 = l_Lake_Toml_Value_decodeFloat___closed__1; -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_31); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +x_24 = l_Lake_Toml_Value_decodeFloat___closed__1; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_2 = x_25; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlFloat___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlFloat___lambda__1), 1, 0); +return x_1; } } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlFloat() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlFloat___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeBool___closed__1() { @@ -2215,47 +2220,42 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlBool(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlBool___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeBool___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeBool___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeBool___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_Toml_Value_decodeBool___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); @@ -2263,58 +2263,77 @@ x_15 = l_Lake_Toml_Value_decodeBool___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -uint8_t x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); +uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); lean_dec(x_1); -x_21 = lean_box(x_20); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -return x_22; +x_18 = lean_box(x_17); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_18); +return x_19; } default: { -uint8_t x_23; -x_23 = !lean_is_exclusive(x_1); -if (x_23 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_1); +if (x_20 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_1, 1); -lean_dec(x_24); -x_25 = l_Lake_Toml_Value_decodeBool___closed__1; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_1, 1); +lean_dec(x_21); +x_22 = l_Lake_Toml_Value_decodeBool___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_25); -x_26 = lean_unsigned_to_nat(1u); -x_27 = lean_mk_array(x_26, x_1); -x_28 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_28, 0, x_27); -return x_28; +lean_ctor_set(x_1, 1, x_22); +x_2 = x_1; +goto block_7; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_29 = lean_ctor_get(x_1, 0); -lean_inc(x_29); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_1, 0); +lean_inc(x_23); lean_dec(x_1); -x_30 = l_Lake_Toml_Value_decodeBool___closed__1; -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_31); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +x_24 = l_Lake_Toml_Value_decodeBool___closed__1; +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +x_2 = x_25; +goto block_7; } } } +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} +} +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlBool___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlBool___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlBool() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlBool___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeDateTime___closed__1() { @@ -2431,47 +2450,42 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlDateTime___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeDateTime___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeDateTime___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeDateTime___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_Toml_Value_decodeDateTime___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); @@ -2479,74 +2493,90 @@ x_15 = l_Lake_Toml_Value_decodeDateTime___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_Toml_Value_decodeDateTime___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_Toml_Value_decodeDateTime___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 4: { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_1, 1); -lean_inc(x_26); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); lean_dec(x_1); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_20); +return x_21; } default: { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_1); -if (x_28 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_1, 1); -lean_dec(x_29); -x_30 = l_Lake_Toml_Value_decodeDateTime___closed__1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = l_Lake_Toml_Value_decodeDateTime___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_mk_array(x_31, x_1); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +lean_ctor_set(x_1, 1, x_24); +x_2 = x_1; +goto block_7; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); lean_dec(x_1); -x_35 = l_Lake_Toml_Value_decodeDateTime___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_39, 0, x_38); -return x_39; +x_26 = l_Lake_Toml_Value_decodeDateTime___closed__1; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_2 = x_27; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} +} } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlDateTime___lambda__1), 1, 0); +return x_1; } } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlDateTime() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1; +return x_1; } } static lean_object* _init_l_Lake_Toml_Value_decodeValueArray___closed__1() { @@ -2666,45 +2696,40 @@ return x_27; LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArray___rarg(lean_object* x_1, lean_object* x_2) { _start: { +lean_object* x_3; switch (lean_obj_tag(x_2)) { case 0: { -uint8_t x_3; +uint8_t x_9; lean_dec(x_1); -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +x_9 = !lean_is_exclusive(x_2); +if (x_9 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = lean_ctor_get(x_2, 1); -lean_dec(x_4); -x_5 = l_Lake_Toml_Value_decodeValueArray___closed__1; -lean_ctor_set(x_2, 1, x_5); -x_6 = lean_unsigned_to_nat(1u); -x_7 = lean_mk_array(x_6, x_2); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_2, 1); +lean_dec(x_10); +x_11 = l_Lake_Toml_Value_decodeValueArray___closed__1; +lean_ctor_set(x_2, 1, x_11); +x_3 = x_2; +goto block_8; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_2, 0); -lean_inc(x_9); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); lean_dec(x_2); -x_10 = l_Lake_Toml_Value_decodeValueArray___closed__1; -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_13 = l_Lake_Toml_Value_decodeValueArray___closed__1; +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_3 = x_14; +goto block_8; } } case 2: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); @@ -2713,163 +2738,457 @@ x_16 = l_Lake_Toml_Value_decodeValueArray___closed__1; x_17 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_mk_array(x_18, x_17); -x_20 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +x_3 = x_17; +goto block_8; } case 3: { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_dec(x_1); -x_21 = lean_ctor_get(x_2, 0); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); +lean_dec(x_2); +x_19 = l_Lake_Toml_Value_decodeValueArray___closed__1; +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_3 = x_20; +goto block_8; +} +case 5: +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_2, 1); lean_inc(x_21); lean_dec(x_2); -x_22 = l_Lake_Toml_Value_decodeValueArray___closed__1; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_unsigned_to_nat(1u); -x_25 = lean_mk_array(x_24, x_23); -x_26 = lean_alloc_ctor(0, 1, 0); +x_22 = l_Lake_Toml_decodeArray___rarg(x_1, x_21); +lean_dec(x_21); +return x_22; +} +default: +{ +uint8_t x_23; +lean_dec(x_1); +x_23 = !lean_is_exclusive(x_2); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_2, 1); +lean_dec(x_24); +x_25 = l_Lake_Toml_Value_decodeValueArray___closed__1; +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 1, x_25); +x_3 = x_2; +goto block_8; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_2, 0); +lean_inc(x_26); +lean_dec(x_2); +x_27 = l_Lake_Toml_Value_decodeValueArray___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_3 = x_28; +goto block_8; +} +} +} +block_8: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArray(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_decodeArray___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_decodeArray___rarg), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlArray___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArrayOrSingleton___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +switch (lean_obj_tag(x_2)) { +case 1: +{ +lean_object* x_3; uint8_t x_4; +lean_inc(x_2); +x_3 = lean_apply_1(x_1, x_2); +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_2, 1); +lean_dec(x_5); +x_6 = lean_ctor_get(x_2, 0); +lean_dec(x_6); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_7; +lean_free_object(x_2); +x_7 = !lean_is_exclusive(x_3); +if (x_7 == 0) +{ +return x_3; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_9, 0, x_8); +return x_9; +} +} +else +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_box(0); +lean_ctor_set(x_2, 1, x_12); +lean_ctor_set(x_2, 0, x_11); +x_13 = lean_array_mk(x_2); +lean_ctor_set(x_3, 0, x_13); +return x_3; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_3, 0); +lean_inc(x_14); +lean_dec(x_3); +x_15 = lean_box(0); +lean_ctor_set(x_2, 1, x_15); +lean_ctor_set(x_2, 0, x_14); +x_16 = lean_array_mk(x_2); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_16); +return x_17; +} +} +} +else +{ +lean_dec(x_2); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_3, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + x_19 = x_3; +} else { + lean_dec_ref(x_3); + x_19 = lean_box(0); +} +if (lean_is_scalar(x_19)) { + x_20 = lean_alloc_ctor(0, 1, 0); +} else { + x_20 = x_19; +} +lean_ctor_set(x_20, 0, x_18); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_21 = lean_ctor_get(x_3, 0); +lean_inc(x_21); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + x_22 = x_3; +} else { + lean_dec_ref(x_3); + x_22 = lean_box(0); +} +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_21); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_array_mk(x_24); +if (lean_is_scalar(x_22)) { + x_26 = lean_alloc_ctor(1, 1, 0); +} else { + x_26 = x_22; +} lean_ctor_set(x_26, 0, x_25); return x_26; } -case 5: +} +} +case 2: { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_2, 1); -lean_inc(x_27); -lean_dec(x_2); -x_28 = l_Lake_Toml_decodeArray___rarg(x_1, x_27); +lean_object* x_27; +x_27 = lean_apply_1(x_1, x_2); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +return x_27; +} +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); lean_dec(x_27); -return x_28; +x_30 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_30, 0, x_29); +return x_30; } -default: +} +else { -uint8_t x_29; -lean_dec(x_1); -x_29 = !lean_is_exclusive(x_2); -if (x_29 == 0) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_27); +if (x_31 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_2, 1); -lean_dec(x_30); -x_31 = l_Lake_Toml_Value_decodeValueArray___closed__1; -lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_2); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_27, 0); +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_array_mk(x_34); +lean_ctor_set(x_27, 0, x_35); +return x_27; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_2, 0); -lean_inc(x_35); -lean_dec(x_2); -x_36 = l_Lake_Toml_Value_decodeValueArray___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_36 = lean_ctor_get(x_27, 0); +lean_inc(x_36); +lean_dec(x_27); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_array_mk(x_38); +x_40 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_40, 0, x_39); return x_40; } } } +case 3: +{ +lean_object* x_41; +x_41 = lean_apply_1(x_1, x_2); +if (lean_obj_tag(x_41) == 0) +{ +uint8_t x_42; +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) +{ +return x_41; } -} -LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArray(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_decodeArray___rarg), 2, 0); -return x_2; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_41, 0); +lean_inc(x_43); +lean_dec(x_41); +x_44 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_44, 0, x_43); +return x_44; } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray___rarg(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_decodeArray___rarg), 2, 1); -lean_closure_set(x_2, 0, x_1); -return x_2; -} +uint8_t x_45; +x_45 = !lean_is_exclusive(x_41); +if (x_45 == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_41, 0); +x_47 = lean_box(0); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +x_49 = lean_array_mk(x_48); +lean_ctor_set(x_41, 0, x_49); +return x_41; } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlArray(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlArray___rarg), 1, 0); -return x_2; +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_50 = lean_ctor_get(x_41, 0); +lean_inc(x_50); +lean_dec(x_41); +x_51 = lean_box(0); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +x_53 = lean_array_mk(x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +return x_54; } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_decodeArrayOrSingleton___rarg(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 5) +} +case 5: { -lean_object* x_3; lean_object* x_4; -x_3 = lean_ctor_get(x_2, 1); -lean_inc(x_3); +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_2, 1); +lean_inc(x_55); lean_dec(x_2); -x_4 = l_Lake_Toml_decodeArray___rarg(x_1, x_3); -lean_dec(x_3); -return x_4; +x_56 = l_Lake_Toml_decodeArray___rarg(x_1, x_55); +lean_dec(x_55); +return x_56; } -else +default: { -lean_object* x_5; -x_5 = lean_apply_1(x_1, x_2); -if (lean_obj_tag(x_5) == 0) +lean_object* x_57; uint8_t x_58; +lean_inc(x_2); +x_57 = lean_apply_1(x_1, x_2); +x_58 = !lean_is_exclusive(x_2); +if (x_58 == 0) { -uint8_t x_6; -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) +lean_object* x_59; lean_object* x_60; +x_59 = lean_ctor_get(x_2, 1); +lean_dec(x_59); +x_60 = lean_ctor_get(x_2, 0); +lean_dec(x_60); +if (lean_obj_tag(x_57) == 0) { -return x_5; +uint8_t x_61; +lean_free_object(x_2); +x_61 = !lean_is_exclusive(x_57); +if (x_61 == 0) +{ +return x_57; } else { -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_62; lean_object* x_63; +x_62 = lean_ctor_get(x_57, 0); +lean_inc(x_62); +lean_dec(x_57); +x_63 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_63, 0, x_62); +return x_63; } } else { -uint8_t x_9; -x_9 = !lean_is_exclusive(x_5); -if (x_9 == 0) +uint8_t x_64; +x_64 = !lean_is_exclusive(x_57); +if (x_64 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_ctor_get(x_5, 0); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -lean_ctor_set(x_5, 0, x_12); -return x_5; +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_57, 0); +x_66 = lean_box(0); +lean_ctor_set_tag(x_2, 1); +lean_ctor_set(x_2, 1, x_66); +lean_ctor_set(x_2, 0, x_65); +x_67 = lean_array_mk(x_2); +lean_ctor_set(x_57, 0, x_67); +return x_57; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_5, 0); -lean_inc(x_13); -lean_dec(x_5); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_mk_array(x_14, x_13); -x_16 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_16, 0, x_15); -return x_16; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_68 = lean_ctor_get(x_57, 0); +lean_inc(x_68); +lean_dec(x_57); +x_69 = lean_box(0); +lean_ctor_set_tag(x_2, 1); +lean_ctor_set(x_2, 1, x_69); +lean_ctor_set(x_2, 0, x_68); +x_70 = lean_array_mk(x_2); +x_71 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_71, 0, x_70); +return x_71; +} +} +} +else +{ +lean_dec(x_2); +if (lean_obj_tag(x_57) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_57, 0); +lean_inc(x_72); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + x_73 = x_57; +} else { + lean_dec_ref(x_57); + x_73 = lean_box(0); +} +if (lean_is_scalar(x_73)) { + x_74 = lean_alloc_ctor(0, 1, 0); +} else { + x_74 = x_73; +} +lean_ctor_set(x_74, 0, x_72); +return x_74; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_75 = lean_ctor_get(x_57, 0); +lean_inc(x_75); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + x_76 = x_57; +} else { + lean_dec_ref(x_57); + x_76 = lean_box(0); +} +x_77 = lean_box(0); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_75); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_array_mk(x_78); +if (lean_is_scalar(x_76)) { + x_80 = lean_alloc_ctor(1, 1, 0); +} else { + x_80 = x_76; +} +lean_ctor_set(x_80, 0, x_79); +return x_80; +} } } } @@ -2997,47 +3316,42 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlTable(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lake_Toml_Value_instDecodeTomlTable___lambda__1(lean_object* x_1) { _start: { +lean_object* x_2; switch (lean_obj_tag(x_1)) { case 0: { -uint8_t x_2; -x_2 = !lean_is_exclusive(x_1); -if (x_2 == 0) +uint8_t x_8; +x_8 = !lean_is_exclusive(x_1); +if (x_8 == 0) { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_3 = lean_ctor_get(x_1, 1); -lean_dec(x_3); -x_4 = l_Lake_Toml_Value_decodeTable___closed__1; -lean_ctor_set(x_1, 1, x_4); -x_5 = lean_unsigned_to_nat(1u); -x_6 = lean_mk_array(x_5, x_1); -x_7 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 1); +lean_dec(x_9); +x_10 = l_Lake_Toml_Value_decodeTable___closed__1; +lean_ctor_set(x_1, 1, x_10); +x_2 = x_1; +goto block_7; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); lean_dec(x_1); -x_9 = l_Lake_Toml_Value_decodeTable___closed__1; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_unsigned_to_nat(1u); -x_12 = lean_mk_array(x_11, x_10); -x_13 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; +x_12 = l_Lake_Toml_Value_decodeTable___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_2 = x_13; +goto block_7; } } case 2: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_ctor_get(x_1, 0); lean_inc(x_14); lean_dec(x_1); @@ -3045,74 +3359,90 @@ x_15 = l_Lake_Toml_Value_decodeTable___closed__1; x_16 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_mk_array(x_17, x_16); -x_19 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_19, 0, x_18); -return x_19; +x_2 = x_16; +goto block_7; } case 3: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_1, 0); -lean_inc(x_20); +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_1, 0); +lean_inc(x_17); lean_dec(x_1); -x_21 = l_Lake_Toml_Value_decodeTable___closed__1; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -x_23 = lean_unsigned_to_nat(1u); -x_24 = lean_mk_array(x_23, x_22); -x_25 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_25, 0, x_24); -return x_25; +x_18 = l_Lake_Toml_Value_decodeTable___closed__1; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_2 = x_19; +goto block_7; } case 6: { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_1, 1); -lean_inc(x_26); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_1, 1); +lean_inc(x_20); lean_dec(x_1); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_26); -return x_27; +x_21 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_21, 0, x_20); +return x_21; } default: { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_1); -if (x_28 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_1, 1); -lean_dec(x_29); -x_30 = l_Lake_Toml_Value_decodeTable___closed__1; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = l_Lake_Toml_Value_decodeTable___closed__1; lean_ctor_set_tag(x_1, 0); -lean_ctor_set(x_1, 1, x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_mk_array(x_31, x_1); -x_33 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_33, 0, x_32); -return x_33; +lean_ctor_set(x_1, 1, x_24); +x_2 = x_1; +goto block_7; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_1, 0); +lean_inc(x_25); lean_dec(x_1); -x_35 = l_Lake_Toml_Value_decodeTable___closed__1; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_37 = lean_unsigned_to_nat(1u); -x_38 = lean_mk_array(x_37, x_36); -x_39 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_39, 0, x_38); -return x_39; +x_26 = l_Lake_Toml_Value_decodeTable___closed__1; +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_2 = x_27; +goto block_7; +} +} +} +block_7: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_mk(x_4); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; +} } } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlTable___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lake_Toml_Value_instDecodeTomlTable___lambda__1), 1, 0); +return x_1; +} } +static lean_object* _init_l_Lake_Toml_Value_instDecodeTomlTable() { +_start: +{ +lean_object* x_1; +x_1 = l_Lake_Toml_Value_instDecodeTomlTable___closed__1; +return x_1; } } static lean_object* _init_l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__1() { @@ -3369,7 +3699,7 @@ lean_inc(x_3); x_6 = l_Lake_Toml_RBDict_findEntry_x3f___rarg(x_5, x_3, x_2); if (lean_obj_tag(x_6) == 0) { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_dec(x_1); x_7 = l_Lake_Toml_ppKey(x_3); lean_dec(x_3); @@ -3381,25 +3711,28 @@ x_11 = lean_string_append(x_9, x_10); x_12 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_12, 0, x_4); lean_ctor_set(x_12, 1, x_11); -x_13 = lean_unsigned_to_nat(1u); -x_14 = lean_mk_array(x_13, x_12); -x_15 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_array_mk(x_14); +x_16 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_16, 0, x_15); +return x_16; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_dec(x_4); -x_16 = lean_ctor_get(x_6, 0); -lean_inc(x_16); -lean_dec(x_6); -x_17 = lean_ctor_get(x_16, 1); +x_17 = lean_ctor_get(x_6, 0); lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lake_Toml_decodeKeyval___rarg(x_1, x_3, x_17); +lean_dec(x_6); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lake_Toml_decodeKeyval___rarg(x_1, x_3, x_18); lean_dec(x_3); -return x_18; +return x_19; } } } @@ -3688,48 +4021,43 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { +lean_object* x_3; switch (lean_obj_tag(x_2)) { case 0: { -uint8_t x_3; +uint8_t x_9; lean_dec(x_1); -x_3 = !lean_is_exclusive(x_2); -if (x_3 == 0) +x_9 = !lean_is_exclusive(x_2); +if (x_9 == 0) { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_4 = lean_ctor_get(x_2, 1); -lean_dec(x_4); -x_5 = l_Lake_Toml_Value_decodeTable___closed__1; -lean_ctor_set(x_2, 1, x_5); -x_6 = lean_unsigned_to_nat(1u); -x_7 = lean_mk_array(x_6, x_2); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_2, 1); +lean_dec(x_10); +x_11 = l_Lake_Toml_Value_decodeTable___closed__1; +lean_ctor_set(x_2, 1, x_11); +x_3 = x_2; +goto block_8; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_9 = lean_ctor_get(x_2, 0); -lean_inc(x_9); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); lean_dec(x_2); -x_10 = l_Lake_Toml_Value_decodeTable___closed__1; -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_9); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_unsigned_to_nat(1u); -x_13 = lean_mk_array(x_12, x_11); -x_14 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_14, 0, x_13); -return x_14; +x_13 = l_Lake_Toml_Value_decodeTable___closed__1; +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_3 = x_14; +goto block_8; } } case 2: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_dec(x_1); x_15 = lean_ctor_get(x_2, 0); lean_inc(x_15); @@ -3738,83 +4066,92 @@ x_16 = l_Lake_Toml_Value_decodeTable___closed__1; x_17 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = lean_unsigned_to_nat(1u); -x_19 = lean_mk_array(x_18, x_17); -x_20 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_19); -return x_20; +x_3 = x_17; +goto block_8; } case 3: { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_dec(x_1); -x_21 = lean_ctor_get(x_2, 0); -lean_inc(x_21); +x_18 = lean_ctor_get(x_2, 0); +lean_inc(x_18); lean_dec(x_2); -x_22 = l_Lake_Toml_Value_decodeTable___closed__1; -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_unsigned_to_nat(1u); -x_25 = lean_mk_array(x_24, x_23); -x_26 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_26, 0, x_25); -return x_26; +x_19 = l_Lake_Toml_Value_decodeTable___closed__1; +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_3 = x_20; +goto block_8; } case 6: { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_2, 1); -lean_inc(x_27); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_2, 1); +lean_inc(x_21); lean_dec(x_2); -x_28 = l_Lake_Toml_Table_decodeNameMap___rarg(x_1, x_27); -lean_dec(x_27); -return x_28; +x_22 = l_Lake_Toml_Table_decodeNameMap___rarg(x_1, x_21); +lean_dec(x_21); +return x_22; } default: { -uint8_t x_29; +uint8_t x_23; lean_dec(x_1); -x_29 = !lean_is_exclusive(x_2); -if (x_29 == 0) +x_23 = !lean_is_exclusive(x_2); +if (x_23 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_30 = lean_ctor_get(x_2, 1); -lean_dec(x_30); -x_31 = l_Lake_Toml_Value_decodeTable___closed__1; +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_2, 1); +lean_dec(x_24); +x_25 = l_Lake_Toml_Value_decodeTable___closed__1; lean_ctor_set_tag(x_2, 0); -lean_ctor_set(x_2, 1, x_31); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_mk_array(x_32, x_2); -x_34 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_34, 0, x_33); -return x_34; +lean_ctor_set(x_2, 1, x_25); +x_3 = x_2; +goto block_8; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_35 = lean_ctor_get(x_2, 0); -lean_inc(x_35); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_2, 0); +lean_inc(x_26); lean_dec(x_2); -x_36 = l_Lake_Toml_Value_decodeTable___closed__1; -x_37 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_unsigned_to_nat(1u); -x_39 = lean_mk_array(x_38, x_37); -x_40 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_40, 0, x_39); -return x_40; +x_27 = l_Lake_Toml_Value_decodeTable___closed__1; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_3 = x_28; +goto block_8; +} +} +} +block_8: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_3); +lean_ctor_set(x_5, 1, x_4); +x_6 = lean_array_mk(x_5); +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_6); +return x_7; } } } +LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Table_instDecodeTomlNameMap___rarg___lambda__1), 2, 1); +lean_closure_set(x_2, 0, x_1); +return x_2; } } LEAN_EXPORT lean_object* l_Lake_Toml_Table_instDecodeTomlNameMap(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Table_instDecodeTomlNameMap___rarg), 2, 0); +x_2 = lean_alloc_closure((void*)(l_Lake_Toml_Table_instDecodeTomlNameMap___rarg), 1, 0); return x_2; } } @@ -4045,24 +4382,58 @@ l_Lake_Toml_instDecodeTomlValue = _init_l_Lake_Toml_instDecodeTomlValue(); lean_mark_persistent(l_Lake_Toml_instDecodeTomlValue); l_Lake_Toml_Value_decodeString___closed__1 = _init_l_Lake_Toml_Value_decodeString___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeString___closed__1); +l_Lake_Toml_Value_instDecodeTomlString___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlString___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlString___closed__1); +l_Lake_Toml_Value_instDecodeTomlString = _init_l_Lake_Toml_Value_instDecodeTomlString(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlString); +l_Lake_Toml_Value_instDecodeTomlFilePath = _init_l_Lake_Toml_Value_instDecodeTomlFilePath(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlFilePath); l_Lake_Toml_Value_decodeName___closed__1 = _init_l_Lake_Toml_Value_decodeName___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeName___closed__1); +l_Lake_Toml_Value_instDecodeTomlName___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlName___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlName___closed__1); +l_Lake_Toml_Value_instDecodeTomlName = _init_l_Lake_Toml_Value_instDecodeTomlName(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlName); l_Lake_Toml_Value_decodeInt___closed__1 = _init_l_Lake_Toml_Value_decodeInt___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeInt___closed__1); +l_Lake_Toml_Value_instDecodeTomlInt___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlInt___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlInt___closed__1); +l_Lake_Toml_Value_instDecodeTomlInt = _init_l_Lake_Toml_Value_instDecodeTomlInt(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlInt); l_Lake_Toml_Value_decodeNat___closed__1 = _init_l_Lake_Toml_Value_decodeNat___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeNat___closed__1); l_Lake_Toml_Value_decodeNat___closed__2 = _init_l_Lake_Toml_Value_decodeNat___closed__2(); lean_mark_persistent(l_Lake_Toml_Value_decodeNat___closed__2); +l_Lake_Toml_Value_instDecodeTomlNat___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlNat___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlNat___closed__1); +l_Lake_Toml_Value_instDecodeTomlNat = _init_l_Lake_Toml_Value_instDecodeTomlNat(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlNat); l_Lake_Toml_Value_decodeFloat___closed__1 = _init_l_Lake_Toml_Value_decodeFloat___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeFloat___closed__1); +l_Lake_Toml_Value_instDecodeTomlFloat___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlFloat___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlFloat___closed__1); +l_Lake_Toml_Value_instDecodeTomlFloat = _init_l_Lake_Toml_Value_instDecodeTomlFloat(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlFloat); l_Lake_Toml_Value_decodeBool___closed__1 = _init_l_Lake_Toml_Value_decodeBool___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeBool___closed__1); +l_Lake_Toml_Value_instDecodeTomlBool___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlBool___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlBool___closed__1); +l_Lake_Toml_Value_instDecodeTomlBool = _init_l_Lake_Toml_Value_instDecodeTomlBool(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlBool); l_Lake_Toml_Value_decodeDateTime___closed__1 = _init_l_Lake_Toml_Value_decodeDateTime___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeDateTime___closed__1); +l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlDateTime___closed__1); +l_Lake_Toml_Value_instDecodeTomlDateTime = _init_l_Lake_Toml_Value_instDecodeTomlDateTime(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlDateTime); l_Lake_Toml_Value_decodeValueArray___closed__1 = _init_l_Lake_Toml_Value_decodeValueArray___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeValueArray___closed__1); l_Lake_Toml_Value_decodeTable___closed__1 = _init_l_Lake_Toml_Value_decodeTable___closed__1(); lean_mark_persistent(l_Lake_Toml_Value_decodeTable___closed__1); +l_Lake_Toml_Value_instDecodeTomlTable___closed__1 = _init_l_Lake_Toml_Value_instDecodeTomlTable___closed__1(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlTable___closed__1); +l_Lake_Toml_Value_instDecodeTomlTable = _init_l_Lake_Toml_Value_instDecodeTomlTable(); +lean_mark_persistent(l_Lake_Toml_Value_instDecodeTomlTable); l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__1(); lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__1); l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lake_Toml_decodeKeyval___spec__1___closed__2(); diff --git a/stage0/stdlib/Lean/AddDecl.c b/stage0/stdlib/Lean/AddDecl.c index 894099034125..caae9a7477cf 100644 --- a/stage0/stdlib/Lean/AddDecl.c +++ b/stage0/stdlib/Lean/AddDecl.c @@ -38,7 +38,6 @@ extern lean_object* l_Lean_trace_profiler_useHeartbeats; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_addDecl___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_addDecl___spec__4___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Environment_compileDecl(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_AddDecl___hyg_5____closed__4; size_t lean_usize_of_nat(lean_object*); @@ -73,7 +72,6 @@ static lean_object* l_Lean_initFn____x40_Lean_AddDecl___hyg_5____closed__6; double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Environment_addDecl___closed__1; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_addDecl___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Environment_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_withTraceNode___at_Lean_addDecl___spec__4___lambda__3___closed__2; static lean_object* l_Lean_logWarning___at_Lean_addDecl___spec__3___closed__1; static lean_object* l_Lean_initFn____x40_Lean_AddDecl___hyg_5____closed__2; @@ -91,7 +89,6 @@ uint8_t l_Lean_Declaration_foldExprM___at_Lean_Declaration_hasSorry___spec__1(le LEAN_EXPORT lean_object* l_Lean_addDecl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_withTraceNode___at_Lean_addDecl___spec__4___lambda__4___closed__4; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_addDecl___spec__4___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Environment_addAndCompile___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_profileitM___at_Lean_addDecl___spec__6(lean_object*); extern lean_object* l_Lean_trace_profiler; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); @@ -234,52 +231,6 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Environment_addAndCompile(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Environment_addDecl(x_1, x_2, x_3, x_4); -if (lean_obj_tag(x_5) == 0) -{ -uint8_t x_6; -lean_dec(x_3); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -return x_5; -} -else -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -x_8 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_8, 0, x_7); -return x_8; -} -} -else -{ -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_5, 0); -lean_inc(x_9); -lean_dec(x_5); -x_10 = l_Lean_Environment_compileDecl(x_9, x_2, x_3); -return x_10; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Environment_addAndCompile___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_Environment_addAndCompile(x_1, x_2, x_3, x_4); -lean_dec(x_4); -lean_dec(x_2); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_addDecl___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { diff --git a/stage0/stdlib/Lean/BuiltinDocAttr.c b/stage0/stdlib/Lean/BuiltinDocAttr.c index c479d0196197..08a0431de253 100644 --- a/stage0/stdlib/Lean/BuiltinDocAttr.c +++ b/stage0/stdlib/Lean/BuiltinDocAttr.c @@ -39,7 +39,6 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_BuiltinDocAttr___hyg_207____closed__11; uint8_t l_Lean_TagDeclarationExtension_isTagged(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkStrLit(lean_object*); -LEAN_EXPORT lean_object* l_Lean_declareBuiltinDocStringAndRanges___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_is_aux_recursor(lean_object*, lean_object*); static lean_object* l_Lean_declareBuiltinDocStringAndRanges___lambda__1___closed__5; @@ -507,6 +506,8 @@ lean_inc(x_7); if (lean_obj_tag(x_7) == 0) { uint8_t x_8; +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_1); x_8 = !lean_is_exclusive(x_6); if (x_8 == 0) @@ -800,6 +801,8 @@ x_25 = lean_array_mk(x_5); x_26 = l_Lean_declareBuiltinDocStringAndRanges___closed__5; x_27 = l_Lean_mkAppN(x_26, x_25); lean_dec(x_25); +lean_inc(x_3); +lean_inc(x_2); x_28 = l_Lean_declareBuiltin(x_21, x_27, x_2, x_3, x_17); if (lean_obj_tag(x_28) == 0) { @@ -816,6 +819,8 @@ return x_31; else { uint8_t x_32; +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); x_32 = !lean_is_exclusive(x_28); if (x_32 == 0) @@ -863,6 +868,8 @@ x_44 = lean_array_mk(x_5); x_45 = l_Lean_declareBuiltinDocStringAndRanges___closed__5; x_46 = l_Lean_mkAppN(x_45, x_44); lean_dec(x_44); +lean_inc(x_3); +lean_inc(x_2); x_47 = l_Lean_declareBuiltin(x_39, x_46, x_2, x_3, x_36); if (lean_obj_tag(x_47) == 0) { @@ -879,6 +886,8 @@ return x_50; else { lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); x_51 = lean_ctor_get(x_47, 0); lean_inc(x_51); @@ -969,6 +978,8 @@ x_74 = lean_array_mk(x_73); x_75 = l_Lean_declareBuiltinDocStringAndRanges___closed__5; x_76 = l_Lean_mkAppN(x_75, x_74); lean_dec(x_74); +lean_inc(x_3); +lean_inc(x_2); x_77 = l_Lean_declareBuiltin(x_68, x_76, x_2, x_3, x_64); if (lean_obj_tag(x_77) == 0) { @@ -985,6 +996,8 @@ return x_80; else { lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); x_81 = lean_ctor_get(x_77, 0); lean_inc(x_81); @@ -1057,22 +1070,10 @@ LEAN_EXPORT lean_object* l_Lean_declareBuiltinDocStringAndRanges___lambda__1___b { lean_object* x_6; x_6 = l_Lean_declareBuiltinDocStringAndRanges___lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_declareBuiltinDocStringAndRanges___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; -x_5 = l_Lean_declareBuiltinDocStringAndRanges(x_1, x_2, x_3, x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_5; -} -} LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_BuiltinDocAttr___hyg_207____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { @@ -1086,12 +1087,12 @@ x_8 = lean_ctor_get(x_7, 1); lean_inc(x_8); lean_dec(x_7); x_9 = l_Lean_declareBuiltinDocStringAndRanges(x_1, x_4, x_5, x_8); -lean_dec(x_4); return x_9; } else { uint8_t x_10; +lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); x_10 = !lean_is_exclusive(x_7); @@ -1331,7 +1332,6 @@ uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); x_8 = l_Lean_initFn____x40_Lean_BuiltinDocAttr___hyg_207____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); return x_8; } } diff --git a/stage0/stdlib/Lean/Compiler/IR/Basic.c b/stage0/stdlib/Lean/Compiler/IR/Basic.c index 76831e084c37..4df4a9690020 100644 --- a/stage0/stdlib/Lean/Compiler/IR/Basic.c +++ b/stage0/stdlib/Lean/Compiler/IR/Basic.c @@ -5352,7 +5352,7 @@ x_13 = l_Lean_IR_reshapeAux___closed__2; x_14 = lean_string_append(x_12, x_13); x_15 = l_Lean_IR_reshapeAux___closed__3; x_16 = l_Lean_IR_reshapeAux___closed__4; -x_17 = lean_unsigned_to_nat(272u); +x_17 = lean_unsigned_to_nat(271u); x_18 = lean_unsigned_to_nat(4u); x_19 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_15, x_16, x_17, x_18, x_14); lean_dec(x_14); diff --git a/stage0/stdlib/Lean/Compiler/InitAttr.c b/stage0/stdlib/Lean/Compiler/InitAttr.c index d5cd21b8faca..cb929d77d1cd 100644 --- a/stage0/stdlib/Lean/Compiler/InitAttr.c +++ b/stage0/stdlib/Lean/Compiler/InitAttr.c @@ -18,16 +18,13 @@ static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed_ static lean_object* l_Lean_initFn____x40_Lean_Compiler_InitAttr___hyg_1154____closed__1; static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__27; lean_object* lean_mk_empty_array_with_capacity(lean_object*); -static lean_object* l_Lean_declareBuiltin___closed__10; lean_object* l_Lean_isInitializerExecutionEnabled(lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); static lean_object* l_Lean_registerInitAttrUnsafe___closed__2; static lean_object* l_Lean_initFn____x40_Lean_Compiler_InitAttr___hyg_1182____closed__4; -lean_object* l_Lean_MessageData_toString(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_registerInitAttr___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Compiler_InitAttr_0__Lean_getIOTypeArg(lean_object*); LEAN_EXPORT lean_object* l_Lean_setBuiltinInitAttr(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_declareBuiltin___closed__13; LEAN_EXPORT lean_object* l_Lean_registerInitAttrUnsafe___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_getInitFnNameForCore_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__29; @@ -77,7 +74,6 @@ static lean_object* l___private_Lean_Compiler_InitAttr_0__Lean_getIOTypeArg___cl LEAN_EXPORT lean_object* l_Lean_isIOUnitRegularInitFn___boxed(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_registerInitAttrUnsafe___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_declareBuiltin___closed__8; uint8_t lean_expr_eqv(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_get_init_fn_name_for(lean_object*, lean_object*); @@ -96,7 +92,6 @@ static lean_object* l_Lean_declareBuiltin___closed__2; lean_object* l_Lean_MessageData_ofFormat(lean_object*); static lean_object* l_Lean_registerInitAttrUnsafe___lambda__1___closed__5; static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__3; -static lean_object* l_Lean_declareBuiltin___closed__9; static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_registerInitAttrUnsafe___spec__6___closed__1; static lean_object* l_Lean_getRegularInitFnNameFor_x3f___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); @@ -141,14 +136,12 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_registerInitAttr static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__21; LEAN_EXPORT lean_object* l_Lean_regularInitAttr; static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__13; -lean_object* l_Lean_Environment_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_registerInitAttrUnsafe___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_registerInitAttrUnsafe___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_registerInitAttrUnsafe___lambda__1___closed__8; extern lean_object* l_Lean_NameSet_empty; static lean_object* l___private_Lean_Compiler_InitAttr_0__Lean_isUnitType___closed__1; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_declareBuiltin___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_registerInitAttrUnsafe___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Compiler_InitAttr___hyg_1182_(lean_object*); @@ -163,10 +156,8 @@ LEAN_EXPORT lean_object* l_Lean_getConstInfo___at_Lean_registerInitAttrUnsafe___ static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__7; LEAN_EXPORT lean_object* l_Lean_hasInitAttr___boxed(lean_object*, lean_object*); uint8_t l_Lean_NameSet_contains(lean_object*, lean_object*); -static lean_object* l_Lean_declareBuiltin___closed__11; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_registerInitAttrUnsafe___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); -static lean_object* l_Lean_declareBuiltin___closed__12; lean_object* l_Lean_registerParametricAttribute___rarg(lean_object*, lean_object*); static lean_object* l_Lean_declareBuiltin___closed__7; lean_object* l___private_Lean_MonadEnv_0__Lean_mkAuxNameAux(lean_object*, lean_object*, lean_object*); @@ -192,13 +183,12 @@ uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_registerInitAttrUnsafe___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_isIOUnitBuiltinInitFn___boxed(lean_object*, lean_object*); +lean_object* l_Lean_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_registerInitAttrUnsafe___lambda__1___closed__4; LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_ofExcept___at_Lean_registerInitAttrUnsafe___spec__5(lean_object*, lean_object*); -lean_object* l_Lean_throwError___at___private_Lean_ReducibilityAttrs_0__Lean_validate___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_declareBuiltin___closed__6; -lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); static lean_object* l___auto____x40_Lean_Compiler_InitAttr___hyg_1141____closed__8; lean_object* l_Lean_Attribute_Builtin_getIdent_x3f(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); @@ -3721,70 +3711,18 @@ x_3 = l_Lean_Expr_app___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_declareBuiltin___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to emit registration code for builtin '", 46, 46); -return x_1; -} -} -static lean_object* _init_l_Lean_declareBuiltin___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_declareBuiltin___closed__8; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_declareBuiltin___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("': ", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_declareBuiltin___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_declareBuiltin___closed__10; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_declareBuiltin___closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_declareBuiltin___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_declareBuiltin___closed__12; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Lean_declareBuiltin(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; x_6 = l_Lean_declareBuiltin___closed__2; -lean_inc(x_1); x_7 = l_Lean_Name_append(x_6, x_1); x_8 = lean_unsigned_to_nat(1u); x_9 = l_Lean_mkAuxName___at_Lean_declareBuiltin___spec__1(x_7, x_8, x_3, x_4, x_5); x_10 = !lean_is_exclusive(x_9); if (x_10 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_11 = lean_ctor_get(x_9, 0); x_12 = lean_ctor_get(x_9, 1); x_13 = lean_box(0); @@ -3807,509 +3745,317 @@ lean_ctor_set(x_18, 3, x_9); lean_ctor_set_uint8(x_18, sizeof(void*)*4, x_17); x_19 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_19, 0, x_18); -x_20 = lean_st_ref_get(x_4, x_12); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +lean_inc(x_4); +lean_inc(x_3); +x_20 = l_Lean_addAndCompile(x_19, x_3, x_4, x_12); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_box(0); -x_26 = l_Lean_Environment_addAndCompile(x_24, x_13, x_19, x_25); -if (lean_obj_tag(x_26) == 0) +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_get(x_4, x_21); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -lean_dec(x_11); -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -lean_dec(x_26); -x_28 = l_Lean_KernelException_toMessageData(x_27, x_13); -x_29 = l_Lean_MessageData_toString(x_28, x_23); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; +x_28 = lean_box(0); +x_29 = l_Lean_ParametricAttribute_setParam___rarg(x_27, x_26, x_11, x_28); +x_30 = lean_ctor_get(x_3, 5); +lean_inc(x_30); +x_31 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_29, x_25); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_31 = lean_ctor_get(x_29, 0); -x_32 = lean_ctor_get(x_29, 1); -x_33 = l_Lean_MessageData_ofName(x_1); -x_34 = l_Lean_declareBuiltin___closed__9; -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_33); -lean_ctor_set(x_29, 0, x_34); -x_35 = l_Lean_declareBuiltin___closed__11; -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_35); -lean_ctor_set(x_20, 0, x_29); -x_36 = l_Lean_stringToMessageData(x_31); +lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_30); +lean_free_object(x_22); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); lean_dec(x_31); -x_37 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_37, 0, x_20); -lean_ctor_set(x_37, 1, x_36); -x_38 = l_Lean_declareBuiltin___closed__13; -x_39 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -x_40 = l_Lean_throwError___at___private_Lean_ReducibilityAttrs_0__Lean_validate___spec__3(x_39, x_3, x_4, x_32); -return x_40; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_41 = lean_ctor_get(x_29, 0); -x_42 = lean_ctor_get(x_29, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_29); -x_43 = l_Lean_MessageData_ofName(x_1); -x_44 = l_Lean_declareBuiltin___closed__9; -x_45 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_43); -x_46 = l_Lean_declareBuiltin___closed__11; -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_46); -lean_ctor_set(x_20, 0, x_45); -x_47 = l_Lean_stringToMessageData(x_41); -lean_dec(x_41); -x_48 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_48, 0, x_20); -lean_ctor_set(x_48, 1, x_47); -x_49 = l_Lean_declareBuiltin___closed__13; -x_50 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -x_51 = l_Lean_throwError___at___private_Lean_ReducibilityAttrs_0__Lean_validate___spec__3(x_50, x_3, x_4, x_42); -return x_51; -} -} -else -{ -uint8_t x_52; -lean_dec(x_1); -x_52 = !lean_is_exclusive(x_26); -if (x_52 == 0) -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_53 = lean_ctor_get(x_26, 0); -x_54 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; -x_55 = lean_box(0); -x_56 = l_Lean_ParametricAttribute_setParam___rarg(x_54, x_53, x_11, x_55); -x_57 = lean_ctor_get(x_3, 5); -x_58 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_56, x_23); -if (lean_obj_tag(x_58) == 0) -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; -lean_free_object(x_26); -lean_free_object(x_20); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_59, x_3, x_4, x_60); -return x_61; +x_34 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_32, x_3, x_4, x_33); +lean_dec(x_4); +lean_dec(x_3); +return x_34; } else { -uint8_t x_62; -x_62 = !lean_is_exclusive(x_58); -if (x_62 == 0) +uint8_t x_35; +lean_dec(x_4); +lean_dec(x_3); +x_35 = !lean_is_exclusive(x_31); +if (x_35 == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_58, 0); -x_64 = lean_io_error_to_string(x_63); -lean_ctor_set_tag(x_26, 3); -lean_ctor_set(x_26, 0, x_64); -x_65 = l_Lean_MessageData_ofFormat(x_26); -lean_inc(x_57); -lean_ctor_set(x_20, 1, x_65); -lean_ctor_set(x_20, 0, x_57); -lean_ctor_set(x_58, 0, x_20); -return x_58; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_31, 0); +x_37 = lean_io_error_to_string(x_36); +x_38 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = l_Lean_MessageData_ofFormat(x_38); +lean_ctor_set(x_22, 1, x_39); +lean_ctor_set(x_22, 0, x_30); +lean_ctor_set(x_31, 0, x_22); +return x_31; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_66 = lean_ctor_get(x_58, 0); -x_67 = lean_ctor_get(x_58, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_58); -x_68 = lean_io_error_to_string(x_66); -lean_ctor_set_tag(x_26, 3); -lean_ctor_set(x_26, 0, x_68); -x_69 = l_Lean_MessageData_ofFormat(x_26); -lean_inc(x_57); -lean_ctor_set(x_20, 1, x_69); -lean_ctor_set(x_20, 0, x_57); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_20); -lean_ctor_set(x_70, 1, x_67); -return x_70; +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_31, 0); +x_41 = lean_ctor_get(x_31, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_31); +x_42 = lean_io_error_to_string(x_40); +x_43 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_43, 0, x_42); +x_44 = l_Lean_MessageData_ofFormat(x_43); +lean_ctor_set(x_22, 1, x_44); +lean_ctor_set(x_22, 0, x_30); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_22); +lean_ctor_set(x_45, 1, x_41); +return x_45; } } } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_71 = lean_ctor_get(x_26, 0); -lean_inc(x_71); -lean_dec(x_26); -x_72 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; -x_73 = lean_box(0); -x_74 = l_Lean_ParametricAttribute_setParam___rarg(x_72, x_71, x_11, x_73); -x_75 = lean_ctor_get(x_3, 5); -x_76 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_74, x_23); -if (lean_obj_tag(x_76) == 0) -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; -lean_free_object(x_20); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); -lean_inc(x_78); -lean_dec(x_76); -x_79 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_77, x_3, x_4, x_78); -return x_79; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_46 = lean_ctor_get(x_22, 0); +x_47 = lean_ctor_get(x_22, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_22); +x_48 = lean_ctor_get(x_46, 0); +lean_inc(x_48); +lean_dec(x_46); +x_49 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; +x_50 = lean_box(0); +x_51 = l_Lean_ParametricAttribute_setParam___rarg(x_49, x_48, x_11, x_50); +x_52 = lean_ctor_get(x_3, 5); +lean_inc(x_52); +x_53 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_51, x_47); +if (lean_obj_tag(x_53) == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_dec(x_52); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +x_56 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_54, x_3, x_4, x_55); +lean_dec(x_4); +lean_dec(x_3); +return x_56; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_80 = lean_ctor_get(x_76, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_76, 1); -lean_inc(x_81); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_82 = x_76; +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_dec(x_4); +lean_dec(x_3); +x_57 = lean_ctor_get(x_53, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_53, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_59 = x_53; } else { - lean_dec_ref(x_76); - x_82 = lean_box(0); -} -x_83 = lean_io_error_to_string(x_80); -x_84 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_84, 0, x_83); -x_85 = l_Lean_MessageData_ofFormat(x_84); -lean_inc(x_75); -lean_ctor_set(x_20, 1, x_85); -lean_ctor_set(x_20, 0, x_75); -if (lean_is_scalar(x_82)) { - x_86 = lean_alloc_ctor(1, 2, 0); + lean_dec_ref(x_53); + x_59 = lean_box(0); +} +x_60 = lean_io_error_to_string(x_57); +x_61 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_62 = l_Lean_MessageData_ofFormat(x_61); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_52); +lean_ctor_set(x_63, 1, x_62); +if (lean_is_scalar(x_59)) { + x_64 = lean_alloc_ctor(1, 2, 0); } else { - x_86 = x_82; + x_64 = x_59; } -lean_ctor_set(x_86, 0, x_20); -lean_ctor_set(x_86, 1, x_81); -return x_86; +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_58); +return x_64; } } } +else +{ +uint8_t x_65; +lean_dec(x_11); +lean_dec(x_4); +lean_dec(x_3); +x_65 = !lean_is_exclusive(x_20); +if (x_65 == 0) +{ +return x_20; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_87 = lean_ctor_get(x_20, 0); -x_88 = lean_ctor_get(x_20, 1); -lean_inc(x_88); -lean_inc(x_87); +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_20, 0); +x_67 = lean_ctor_get(x_20, 1); +lean_inc(x_67); +lean_inc(x_66); lean_dec(x_20); -x_89 = lean_ctor_get(x_87, 0); -lean_inc(x_89); -lean_dec(x_87); -x_90 = lean_box(0); -x_91 = l_Lean_Environment_addAndCompile(x_89, x_13, x_19, x_90); -if (lean_obj_tag(x_91) == 0) -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -lean_dec(x_11); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -lean_dec(x_91); -x_93 = l_Lean_KernelException_toMessageData(x_92, x_13); -x_94 = l_Lean_MessageData_toString(x_93, x_88); -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - x_97 = x_94; -} else { - lean_dec_ref(x_94); - x_97 = lean_box(0); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; } -x_98 = l_Lean_MessageData_ofName(x_1); -x_99 = l_Lean_declareBuiltin___closed__9; -if (lean_is_scalar(x_97)) { - x_100 = lean_alloc_ctor(7, 2, 0); -} else { - x_100 = x_97; - lean_ctor_set_tag(x_100, 7); } -lean_ctor_set(x_100, 0, x_99); -lean_ctor_set(x_100, 1, x_98); -x_101 = l_Lean_declareBuiltin___closed__11; -x_102 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_102, 0, x_100); -lean_ctor_set(x_102, 1, x_101); -x_103 = l_Lean_stringToMessageData(x_95); -lean_dec(x_95); -x_104 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_104, 0, x_102); -lean_ctor_set(x_104, 1, x_103); -x_105 = l_Lean_declareBuiltin___closed__13; -x_106 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -x_107 = l_Lean_throwError___at___private_Lean_ReducibilityAttrs_0__Lean_validate___spec__3(x_106, x_3, x_4, x_96); -return x_107; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_1); -x_108 = lean_ctor_get(x_91, 0); -lean_inc(x_108); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - x_109 = x_91; -} else { - lean_dec_ref(x_91); - x_109 = lean_box(0); -} -x_110 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; -x_111 = lean_box(0); -x_112 = l_Lean_ParametricAttribute_setParam___rarg(x_110, x_108, x_11, x_111); -x_113 = lean_ctor_get(x_3, 5); -x_114 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_112, x_88); -if (lean_obj_tag(x_114) == 0) -{ -lean_object* x_115; lean_object* x_116; lean_object* x_117; -lean_dec(x_109); -x_115 = lean_ctor_get(x_114, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_114, 1); -lean_inc(x_116); -lean_dec(x_114); -x_117 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_115, x_3, x_4, x_116); -return x_117; -} -else +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_69 = lean_ctor_get(x_9, 0); +x_70 = lean_ctor_get(x_9, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_9); +x_71 = lean_box(0); +x_72 = l_Lean_declareBuiltin___closed__7; +lean_inc(x_69); +x_73 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_73, 0, x_69); +lean_ctor_set(x_73, 1, x_71); +lean_ctor_set(x_73, 2, x_72); +lean_inc(x_69); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_69); +lean_ctor_set(x_74, 1, x_71); +x_75 = lean_box(0); +x_76 = 1; +x_77 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_77, 0, x_73); +lean_ctor_set(x_77, 1, x_2); +lean_ctor_set(x_77, 2, x_75); +lean_ctor_set(x_77, 3, x_74); +lean_ctor_set_uint8(x_77, sizeof(void*)*4, x_76); +x_78 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_78, 0, x_77); +lean_inc(x_4); +lean_inc(x_3); +x_79 = l_Lean_addAndCompile(x_78, x_3, x_4, x_70); +if (lean_obj_tag(x_79) == 0) { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_118 = lean_ctor_get(x_114, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_114, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_114)) { - lean_ctor_release(x_114, 0); - lean_ctor_release(x_114, 1); - x_120 = x_114; -} else { - lean_dec_ref(x_114); - x_120 = lean_box(0); -} -x_121 = lean_io_error_to_string(x_118); -if (lean_is_scalar(x_109)) { - x_122 = lean_alloc_ctor(3, 1, 0); -} else { - x_122 = x_109; - lean_ctor_set_tag(x_122, 3); -} -lean_ctor_set(x_122, 0, x_121); -x_123 = l_Lean_MessageData_ofFormat(x_122); -lean_inc(x_113); -x_124 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_124, 0, x_113); -lean_ctor_set(x_124, 1, x_123); -if (lean_is_scalar(x_120)) { - x_125 = lean_alloc_ctor(1, 2, 0); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_80 = lean_ctor_get(x_79, 1); +lean_inc(x_80); +lean_dec(x_79); +x_81 = lean_st_ref_get(x_4, x_80); +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_84 = x_81; } else { - x_125 = x_120; -} -lean_ctor_set(x_125, 0, x_124); -lean_ctor_set(x_125, 1, x_119); -return x_125; -} -} + lean_dec_ref(x_81); + x_84 = lean_box(0); } +x_85 = lean_ctor_get(x_82, 0); +lean_inc(x_85); +lean_dec(x_82); +x_86 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; +x_87 = lean_box(0); +x_88 = l_Lean_ParametricAttribute_setParam___rarg(x_86, x_85, x_69, x_87); +x_89 = lean_ctor_get(x_3, 5); +lean_inc(x_89); +x_90 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_88, x_83); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_89); +lean_dec(x_84); +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_91, x_3, x_4, x_92); +lean_dec(x_4); +lean_dec(x_3); +return x_93; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint8_t x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; -x_126 = lean_ctor_get(x_9, 0); -x_127 = lean_ctor_get(x_9, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_9); -x_128 = lean_box(0); -x_129 = l_Lean_declareBuiltin___closed__7; -lean_inc(x_126); -x_130 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_130, 0, x_126); -lean_ctor_set(x_130, 1, x_128); -lean_ctor_set(x_130, 2, x_129); -lean_inc(x_126); -x_131 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_131, 0, x_126); -lean_ctor_set(x_131, 1, x_128); -x_132 = lean_box(0); -x_133 = 1; -x_134 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_134, 0, x_130); -lean_ctor_set(x_134, 1, x_2); -lean_ctor_set(x_134, 2, x_132); -lean_ctor_set(x_134, 3, x_131); -lean_ctor_set_uint8(x_134, sizeof(void*)*4, x_133); -x_135 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_135, 0, x_134); -x_136 = lean_st_ref_get(x_4, x_127); -x_137 = lean_ctor_get(x_136, 0); -lean_inc(x_137); -x_138 = lean_ctor_get(x_136, 1); -lean_inc(x_138); -if (lean_is_exclusive(x_136)) { - lean_ctor_release(x_136, 0); - lean_ctor_release(x_136, 1); - x_139 = x_136; +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_dec(x_4); +lean_dec(x_3); +x_94 = lean_ctor_get(x_90, 0); +lean_inc(x_94); +x_95 = lean_ctor_get(x_90, 1); +lean_inc(x_95); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_96 = x_90; } else { - lean_dec_ref(x_136); - x_139 = lean_box(0); -} -x_140 = lean_ctor_get(x_137, 0); -lean_inc(x_140); -lean_dec(x_137); -x_141 = lean_box(0); -x_142 = l_Lean_Environment_addAndCompile(x_140, x_128, x_135, x_141); -if (lean_obj_tag(x_142) == 0) -{ -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -lean_dec(x_126); -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -lean_dec(x_142); -x_144 = l_Lean_KernelException_toMessageData(x_143, x_128); -x_145 = l_Lean_MessageData_toString(x_144, x_138); -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_145, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_145)) { - lean_ctor_release(x_145, 0); - lean_ctor_release(x_145, 1); - x_148 = x_145; + lean_dec_ref(x_90); + x_96 = lean_box(0); +} +x_97 = lean_io_error_to_string(x_94); +x_98 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_98, 0, x_97); +x_99 = l_Lean_MessageData_ofFormat(x_98); +if (lean_is_scalar(x_84)) { + x_100 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_145); - x_148 = lean_box(0); + x_100 = x_84; } -x_149 = l_Lean_MessageData_ofName(x_1); -x_150 = l_Lean_declareBuiltin___closed__9; -if (lean_is_scalar(x_148)) { - x_151 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_100, 0, x_89); +lean_ctor_set(x_100, 1, x_99); +if (lean_is_scalar(x_96)) { + x_101 = lean_alloc_ctor(1, 2, 0); } else { - x_151 = x_148; - lean_ctor_set_tag(x_151, 7); -} -lean_ctor_set(x_151, 0, x_150); -lean_ctor_set(x_151, 1, x_149); -x_152 = l_Lean_declareBuiltin___closed__11; -if (lean_is_scalar(x_139)) { - x_153 = lean_alloc_ctor(7, 2, 0); -} else { - x_153 = x_139; - lean_ctor_set_tag(x_153, 7); + x_101 = x_96; } -lean_ctor_set(x_153, 0, x_151); -lean_ctor_set(x_153, 1, x_152); -x_154 = l_Lean_stringToMessageData(x_146); -lean_dec(x_146); -x_155 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_154); -x_156 = l_Lean_declareBuiltin___closed__13; -x_157 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_157, 0, x_155); -lean_ctor_set(x_157, 1, x_156); -x_158 = l_Lean_throwError___at___private_Lean_ReducibilityAttrs_0__Lean_validate___spec__3(x_157, x_3, x_4, x_147); -return x_158; +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_95); +return x_101; } -else -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -lean_dec(x_1); -x_159 = lean_ctor_get(x_142, 0); -lean_inc(x_159); -if (lean_is_exclusive(x_142)) { - lean_ctor_release(x_142, 0); - x_160 = x_142; -} else { - lean_dec_ref(x_142); - x_160 = lean_box(0); -} -x_161 = l_Lean_getBuiltinInitFnNameFor_x3f___closed__1; -x_162 = lean_box(0); -x_163 = l_Lean_ParametricAttribute_setParam___rarg(x_161, x_159, x_126, x_162); -x_164 = lean_ctor_get(x_3, 5); -x_165 = l_IO_ofExcept___at_Lean_declareBuiltin___spec__2(x_163, x_138); -if (lean_obj_tag(x_165) == 0) -{ -lean_object* x_166; lean_object* x_167; lean_object* x_168; -lean_dec(x_160); -lean_dec(x_139); -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_165, 1); -lean_inc(x_167); -lean_dec(x_165); -x_168 = l_Lean_setEnv___at_Lean_compileDecl___spec__11(x_166, x_3, x_4, x_167); -return x_168; } else { -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -x_169 = lean_ctor_get(x_165, 0); -lean_inc(x_169); -x_170 = lean_ctor_get(x_165, 1); -lean_inc(x_170); -if (lean_is_exclusive(x_165)) { - lean_ctor_release(x_165, 0); - lean_ctor_release(x_165, 1); - x_171 = x_165; -} else { - lean_dec_ref(x_165); - x_171 = lean_box(0); -} -x_172 = lean_io_error_to_string(x_169); -if (lean_is_scalar(x_160)) { - x_173 = lean_alloc_ctor(3, 1, 0); -} else { - x_173 = x_160; - lean_ctor_set_tag(x_173, 3); -} -lean_ctor_set(x_173, 0, x_172); -x_174 = l_Lean_MessageData_ofFormat(x_173); -lean_inc(x_164); -if (lean_is_scalar(x_139)) { - x_175 = lean_alloc_ctor(0, 2, 0); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_69); +lean_dec(x_4); +lean_dec(x_3); +x_102 = lean_ctor_get(x_79, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_79, 1); +lean_inc(x_103); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_104 = x_79; } else { - x_175 = x_139; + lean_dec_ref(x_79); + x_104 = lean_box(0); } -lean_ctor_set(x_175, 0, x_164); -lean_ctor_set(x_175, 1, x_174); -if (lean_is_scalar(x_171)) { - x_176 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_104)) { + x_105 = lean_alloc_ctor(1, 2, 0); } else { - x_176 = x_171; -} -lean_ctor_set(x_176, 0, x_175); -lean_ctor_set(x_176, 1, x_170); -return x_176; + x_105 = x_104; } +lean_ctor_set(x_105, 0, x_102); +lean_ctor_set(x_105, 1, x_103); +return x_105; } } } @@ -4324,16 +4070,6 @@ lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_declareBuiltin___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l_Lean_declareBuiltin(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_6; -} -} lean_object* initialize_Lean_AddDecl(uint8_t builtin, lean_object*); lean_object* initialize_Lean_MonadEnv(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_InfoTree_Main(uint8_t builtin, lean_object*); @@ -4498,18 +4234,6 @@ l_Lean_declareBuiltin___closed__6 = _init_l_Lean_declareBuiltin___closed__6(); lean_mark_persistent(l_Lean_declareBuiltin___closed__6); l_Lean_declareBuiltin___closed__7 = _init_l_Lean_declareBuiltin___closed__7(); lean_mark_persistent(l_Lean_declareBuiltin___closed__7); -l_Lean_declareBuiltin___closed__8 = _init_l_Lean_declareBuiltin___closed__8(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__8); -l_Lean_declareBuiltin___closed__9 = _init_l_Lean_declareBuiltin___closed__9(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__9); -l_Lean_declareBuiltin___closed__10 = _init_l_Lean_declareBuiltin___closed__10(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__10); -l_Lean_declareBuiltin___closed__11 = _init_l_Lean_declareBuiltin___closed__11(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__11); -l_Lean_declareBuiltin___closed__12 = _init_l_Lean_declareBuiltin___closed__12(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__12); -l_Lean_declareBuiltin___closed__13 = _init_l_Lean_declareBuiltin___closed__13(); -lean_mark_persistent(l_Lean_declareBuiltin___closed__13); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Compiler/LCNF/MonoTypes.c b/stage0/stdlib/Lean/Compiler/LCNF/MonoTypes.c index 0e4347ce734e..fcc1b169299d 100644 --- a/stage0/stdlib/Lean/Compiler/LCNF/MonoTypes.c +++ b/stage0/stdlib/Lean/Compiler/LCNF/MonoTypes.c @@ -38,7 +38,6 @@ lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*) lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Compiler_LCNF_getOtherDeclBaseType___spec__1(lean_object*, lean_object*); lean_object* l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); -static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1; extern lean_object* l_Lean_Compiler_LCNF_erasedExpr; lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__10; @@ -68,7 +67,6 @@ LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_instReprTrivialStructureInfo; static lean_object* l_Lean_Compiler_LCNF_toMonoType_visitApp___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Compiler_LCNF_hasTrivialStructure_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644_(lean_object*); static uint64_t l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__6; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_hasTrivialStructure_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_LCNF_toMonoType___closed__1; @@ -143,6 +141,7 @@ LEAN_EXPORT lean_object* l_panic___at_Lean_Compiler_LCNF_getRelevantCtorFields__ lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_toMonoType_visitApp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633_(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Compiler_LCNF_toMonoType_visitApp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -164,6 +163,7 @@ static lean_object* l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__1; static lean_object* l___private_Lean_Compiler_LCNF_MonoTypes_0__Lean_Compiler_LCNF_reprTrivialStructureInfo____x40_Lean_Compiler_LCNF_MonoTypes___hyg_253____closed__19; LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_hasTrivialStructure_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Compiler_LCNF_MonoTypes_0__Lean_Compiler_LCNF_reprTrivialStructureInfo____x40_Lean_Compiler_LCNF_MonoTypes___hyg_253____closed__13; +static lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1; static lean_object* _init_l_panic___at_Lean_Compiler_LCNF_getRelevantCtorFields___spec__1___closed__1() { _start: { @@ -1880,7 +1880,7 @@ static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Compiler_LCNF_t lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__1; x_2 = l_Array_forIn_x27Unsafe_loop___at_Lean_Compiler_LCNF_toMonoType_visitApp___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(99u); +x_3 = lean_unsigned_to_nat(97u); x_4 = lean_unsigned_to_nat(50u); x_5 = l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2805,7 +2805,7 @@ x_1 = l_Lean_Compiler_LCNF_getRelevantCtorFields___closed__8; return x_1; } } -static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1() { +static lean_object* _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -2815,11 +2815,11 @@ lean_closure_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1; +x_2 = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1; x_3 = l_Lean_EnvExtensionInterfaceUnsafe_registerExt___rarg(x_2, x_1); return x_3; } @@ -3374,9 +3374,9 @@ l_Lean_Compiler_LCNF_toMonoType___closed__1 = _init_l_Lean_Compiler_LCNF_toMonoT lean_mark_persistent(l_Lean_Compiler_LCNF_toMonoType___closed__1); l_Lean_Compiler_LCNF_instInhabitedMonoTypeExtState = _init_l_Lean_Compiler_LCNF_instInhabitedMonoTypeExtState(); lean_mark_persistent(l_Lean_Compiler_LCNF_instInhabitedMonoTypeExtState); -l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1(); -lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644____closed__1); -if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1644_(lean_io_mk_world()); +l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1 = _init_l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1(); +lean_mark_persistent(l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633____closed__1); +if (builtin) {res = l_Lean_Compiler_LCNF_initFn____x40_Lean_Compiler_LCNF_MonoTypes___hyg_1633_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Compiler_LCNF_monoTypeExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Compiler_LCNF_monoTypeExt); diff --git a/stage0/stdlib/Lean/Compiler/Old.c b/stage0/stdlib/Lean/Compiler/Old.c index 8159c99833fe..b142c0130f53 100644 --- a/stage0/stdlib/Lean/Compiler/Old.c +++ b/stage0/stdlib/Lean/Compiler/Old.c @@ -24,11 +24,7 @@ lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Compiler_getDeclNamesForCodeGen(lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Compiler_checkIsDefinition___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecl(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecl___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Compiler_isEagerLambdaLiftingName___closed__1; -lean_object* lean_compile_decls(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecls___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Compiler_checkIsDefinition___closed__5; static lean_object* l_Lean_Compiler_checkIsDefinition___closed__4; @@ -475,35 +471,6 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecls___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = lean_compile_decls(x_1, x_2, x_3); -lean_dec(x_3); -lean_dec(x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; lean_object* x_5; -x_4 = l_Lean_Compiler_getDeclNamesForCodeGen(x_3); -x_5 = lean_compile_decls(x_1, x_2, x_4); -lean_dec(x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Environment_compileDecl___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_Environment_compileDecl(x_1, x_2, x_3); -lean_dec(x_2); -return x_4; -} -} lean_object* initialize_Lean_Environment(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Compiler_Old(uint8_t builtin, lean_object* w) { diff --git a/stage0/stdlib/Lean/CoreM.c b/stage0/stdlib/Lean/CoreM.c index 5da8820315a8..7331574a0b9c 100644 --- a/stage0/stdlib/Lean/CoreM.c +++ b/stage0/stdlib/Lean/CoreM.c @@ -255,7 +255,6 @@ uint8_t lean_string_validate_utf8(lean_object*); static lean_object* l_Lean_Core_initFn____x40_Lean_CoreM___hyg_185____closed__15; LEAN_EXPORT lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_instMonadRefCoreM___closed__1; -lean_object* l_Lean_Environment_compileDecl(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Kernel_enableDiag(lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Lean_Core_instMonadRecDepthCoreM___lambda__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_CoreM_0__Lean_supportedRecursors___closed__15; @@ -348,7 +347,6 @@ static lean_object* l_Lean_compileDecl___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_compileDecl___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_useDiagnosticMsg___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_compile_decls(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Core_wrapAsyncAsSnapshot___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Core_instInhabitedCoreM___rarg___closed__2; static lean_object* l_Lean_withTraceNode___at_Lean_Core_wrapAsyncAsSnapshot___spec__1___lambda__4___closed__2; @@ -389,6 +387,7 @@ static lean_object* l___private_Lean_CoreM_0__Lean_supportedRecursors___closed__ LEAN_EXPORT lean_object* l_Lean_Core_instantiateValueLevelParams___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_MessageData_hasTag(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_compileDeclsOld___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Core_instMonadTraceCoreM___closed__1; static lean_object* l___auto____x40_Lean_CoreM___hyg_4099____closed__10; @@ -744,6 +743,7 @@ LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_CoreM_0__Lean_checkUn static lean_object* l_Lean_Core_instMonadEnvCoreM___closed__3; LEAN_EXPORT lean_object* l_Lean_Core_logSnapshotTask(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*); +lean_object* lean_compile_decls(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Core_initFn____x40_Lean_CoreM___hyg_2952_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_CoreM___hyg_80____closed__2; static lean_object* l_Lean_Core_initFn____x40_Lean_CoreM___hyg_3066____closed__1; @@ -20045,6 +20045,16 @@ x_5 = lean_lcnf_compile_decls(x_1, x_2, x_3, x_4); return x_5; } } +LEAN_EXPORT lean_object* l_Lean_compileDeclsOld___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_compile_decls(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_2); +return x_4; +} +} LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_compileDecl___spec__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -22803,7 +22813,7 @@ x_8 = lean_ctor_get(x_6, 0); x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); lean_dec(x_8); -x_10 = l_Lean_Environment_compileDecl(x_9, x_1, x_2); +x_10 = lean_compile_decls(x_9, x_1, x_2); lean_ctor_set(x_6, 0, x_10); return x_6; } @@ -22818,7 +22828,7 @@ lean_dec(x_6); x_13 = lean_ctor_get(x_11, 0); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Environment_compileDecl(x_13, x_1, x_2); +x_14 = lean_compile_decls(x_13, x_1, x_2); x_15 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_15, 0, x_14); lean_ctor_set(x_15, 1, x_12); @@ -22840,12 +22850,12 @@ LEAN_EXPORT lean_object* l_Lean_compileDecl___lambda__3(lean_object* x_1, lean_o _start: { lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_13; +lean_inc(x_1); x_8 = lean_alloc_closure((void*)(l_Lean_compileDecl___lambda__1___boxed), 5, 1); lean_closure_set(x_8, 0, x_1); -lean_inc(x_3); x_9 = lean_alloc_closure((void*)(l_Lean_compileDecl___lambda__2___boxed), 5, 2); lean_closure_set(x_9, 0, x_2); -lean_closure_set(x_9, 1, x_3); +lean_closure_set(x_9, 1, x_1); x_10 = l_Lean_compileDecl___lambda__3___closed__1; x_11 = 1; x_12 = l_Lean_initFn____x40_Lean_CoreM___hyg_80____closed__3; @@ -23272,6 +23282,7 @@ lean_object* x_6; x_6 = l_Lean_compileDecl___lambda__2(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); return x_6; } diff --git a/stage0/stdlib/Lean/Data/AssocList.c b/stage0/stdlib/Lean/Data/AssocList.c index ba6b7bea5779..4b19b02a8fb9 100644 --- a/stage0/stdlib/Lean/Data/AssocList.c +++ b/stage0/stdlib/Lean/Data/AssocList.c @@ -42,11 +42,13 @@ LEAN_EXPORT lean_object* l_Lean_AssocList_insert(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_mapVal___rarg(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_AssocList_any___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_insertNew___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_insertNew(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_instForInProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_AssocList_toList___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_toAssocList_x27___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_AssocList_toList___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_AssocList_insert___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_AssocList_contains___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_toAssocList_x27___rarg___boxed(lean_object*); @@ -94,7 +96,7 @@ x_3 = lean_box(0); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_AssocList_insert___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_AssocList_insertNew___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; @@ -105,11 +107,11 @@ lean_ctor_set(x_4, 2, x_1); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_AssocList_insert(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_AssocList_insertNew(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Lean_AssocList_insert___rarg), 3, 0); +x_3 = lean_alloc_closure((void*)(l_Lean_AssocList_insertNew___rarg), 3, 0); return x_3; } } @@ -765,6 +767,40 @@ x_3 = lean_alloc_closure((void*)(l_Lean_AssocList_replace___rarg), 4, 0); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +lean_inc(x_2); +lean_inc(x_3); +lean_inc(x_1); +x_5 = l_Lean_AssocList_contains___rarg(x_1, x_3, x_2); +if (x_5 == 0) +{ +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_6, 0, x_3); +lean_ctor_set(x_6, 1, x_4); +lean_ctor_set(x_6, 2, x_2); +return x_6; +} +else +{ +lean_object* x_7; +x_7 = l_Lean_AssocList_replace___rarg(x_1, x_3, x_4, x_2); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_insert(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_AssocList_insert___rarg), 4, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_AssocList_erase___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { diff --git a/stage0/stdlib/Lean/Elab/App.c b/stage0/stdlib/Lean/Elab/App.c index 000d0ab12645..2c841594b174 100644 --- a/stage0/stdlib/Lean/Elab/App.c +++ b/stage0/stdlib/Lean/Elab/App.c @@ -108,7 +108,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Elab_Term_instToStringNamedArg___lambda__1(lean_object*); lean_object* l_Lean_RBNode_find___at_Lean_Elab_Term_resolveLocalName___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Elab_Term_getElabElimExprInfo___spec__6(lean_object*, lean_object*, lean_object*); @@ -118,7 +117,6 @@ static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__3; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__5; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__7; LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Term_ElabElim_finalize___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instToStringNamedArg___closed__1; static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__8___closed__2; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__3; @@ -157,7 +155,6 @@ uint8_t l_Lean_Exception_isInterrupt(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_findNamedArgDependsOnCurrent_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__5___closed__4; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13; lean_object* l_Lean_Elab_Term_synthesizeSyntheticMVars(uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Elab_Term_ElabElim_revertArgs___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_formatStxAux(lean_object*, uint8_t, lean_object*, lean_object*); @@ -207,7 +204,6 @@ LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Elab_Term_ElabElim_ lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_consumeImplicits___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_reprElabElimInfo____x40_Lean_Elab_App___hyg_7113____closed__19; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9; lean_object* l_Lean_Syntax_getId(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -228,7 +224,7 @@ lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*) static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__7; static lean_object* l___regBuiltin_Lean_Elab_Term_elabDotIdent__1___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Term_synthesizeAppInstMVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Term_resolveLocalName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_getElabElimExprInfo___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_shouldElabAsElim___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_findNamedArgDependsOnCurrent_x3f___spec__4(lean_object*, lean_object*, lean_object*); @@ -272,6 +268,7 @@ lean_object* l_instInhabitedReaderT___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__1; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Term_ElabAppArgs_trySynthesizeAppInstMVars___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3; lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_proj___override(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getPos_x3f(lean_object*, uint8_t); @@ -445,6 +442,7 @@ LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_App_0__Lean_El LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_nestedExceptionToMessageData___at___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___spec__10___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeAppInstMVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9; lean_object* l_Lean_Elab_Term_elabTermEnsuringType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabAppArgs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forInAux___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -469,19 +467,18 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicitUniv_declRange__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringNamedArg(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabProj_declRange__1___closed__3; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10; LEAN_EXPORT lean_object* l_Lean_computeStructureResolutionOrder_selectParent___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lean_Elab_Term_elabLetDeclCore___spec__2___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_instInhabitedElabElimInfo___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10; lean_object* l_Lean_getPathToBaseStructure_x3f(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux___spec__5___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncRecDepth___at_Lean_Elab_Term_ElabElim_revertArgs___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_insert___at___private_Lean_Structure_0__Lean_setStructureResolutionOrder___spec__1(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Elab_instInhabitedInfoTree; size_t lean_usize_of_nat(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14; LEAN_EXPORT lean_object* l_Lean_throwMaxRecDepthAt___at___private_Lean_Elab_App_0__Lean_Elab_Term_addLValArg_go___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instToStringArg(lean_object*); LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Elab_Term_ElabAppArgs_trySynthesizeAppInstMVars___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -509,6 +506,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_elabExplicitUnivs(lean_object*, lean_o LEAN_EXPORT lean_object* l_Lean_setEnv___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_qsort_sort___at_Lean_computeStructureResolutionOrder___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitLet___at_Lean_Elab_Term_ElabElim_revertArgs___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -535,7 +533,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_throwLValEr LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12; lean_object* l_Lean_Elab_Term_mkInstMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_8237____lambda__2___closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_synthesizeAppInstMVars(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -768,6 +765,7 @@ uint8_t l_Lean_BinderInfo_isInstImplicit(uint8_t); lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_processImplicitArg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4; lean_object* l_Lean_Elab_Term_tryPostponeIfMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabIdent__1___closed__3; static lean_object* l_Subarray_forInUnsafe_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__3___closed__3; @@ -838,7 +836,6 @@ static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__6___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId___boxed(lean_object**); static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__12___closed__2; static lean_object* l_List_foldlM___at_Lean_Elab_Term_ElabElim_revertArgs___spec__17___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_instInhabitedElabElimInfo; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_Elab_Term_ElabElim_mkMotive___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -856,7 +853,7 @@ lean_object* l_Array_mapMUnsafe_map___at_Lean_computeStructureResolutionOrder___ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_addLValArg___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_throwInvalidNamedArg___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult_isResultType___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1; lean_object* l_Lean_Elab_Term_postponeElabTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_findNamedArgDependsOnCurrent_x3f___spec__18___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_fvarId(lean_object*); @@ -876,6 +873,7 @@ static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_throwInvalidFiel uint8_t l_Lean_LocalDecl_isAuxDecl(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_getBindingName(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicitUniv_declRange__1___closed__1; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_addLValArg_go___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -884,6 +882,7 @@ lean_object* l_Lean_registerTagAttribute(lean_object*, lean_object*, lean_object lean_object* l_Lean_CollectFVars_main(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_transform_visit_visitPost___at_Lean_Elab_Term_ElabElim_revertArgs___spec__3(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___spec__4___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_nextArgHole_x3f___boxed(lean_object*); extern lean_object* l_Std_Format_defWidth; @@ -909,13 +908,13 @@ uint8_t l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1( LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_8237____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabApp_declRange__1___closed__5; extern lean_object* l_Lean_recOnSuffix; static lean_object* l_Lean_Elab_Term_throwInvalidNamedArg___rarg___closed__7; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___lambda__1___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_saveArgInfo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906_(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabApp__1___closed__2; LEAN_EXPORT lean_object* l_Lean_computeStructureResolutionOrder_selectParent___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLValsAux_loop___lambda__3___closed__2; @@ -941,8 +940,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_throwInvali lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___spec__1(lean_object*); static lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lean_Elab_Term_ElabElim_mkMotive___spec__1___rarg___closed__2; +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11; LEAN_EXPORT lean_object* l_Lean_Elab_Term_mkFreshBinderName___at_Lean_Elab_Term_ElabElim_mkMotive___spec__1___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11; LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_shouldPropagateExpectedTypeFor___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_getSuccesses___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1011,10 +1010,12 @@ static lean_object* l_Lean_exprDependsOn___at___private_Lean_Elab_App_0__Lean_El LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Term_getElabElimExprInfo___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabElim_main___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_throwInvalidFieldNotation___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabPipeProj__1___closed__3; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_shouldPropagateExpectedTypeFor___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___rarg___lambda__1(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14; lean_object* l_Lean_Elab_Term_addTermInfo_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_hasArgsToProcess___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1088,16 +1089,15 @@ static lean_object* l___regBuiltin_Lean_Elab_Term_elabProj_declRange__1___closed extern lean_object* l_Lean_brecOnSuffix; static lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicit_declRange__1___closed__1; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___rarg___closed__3; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__21(lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15; lean_object* lean_environment_main_module(lean_object*); static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_8237____lambda__2___closed__15; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___closed__9; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__18; lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicitUniv_declRange__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880_(lean_object*); static lean_object* l_Lean_Elab_Term_elabAppArgs___lambda__5___closed__4; LEAN_EXPORT lean_object* l_Lean_addTrace___at___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_forallTelescope___at_Lean_Elab_Term_ElabElim_finalize___spec__9___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1234,6 +1234,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs lean_object* l_Lean_toMessageList(lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_getSuccesses___spec__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppLVals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_shouldElabAsElim___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Term_elabLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_propagateExpectedType___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1301,15 +1302,12 @@ static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_8237____l LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___lambda__3___closed__2; -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_isNextOutParamOfLocalInstanceAndResult_hasLocalInstaceWithOutParams(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Elab_Util_0__Lean_Elab_evalSyntaxConstantUnsafe(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasFVar(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__9(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_List_foldlM___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId___spec__1___lambda__1___boxed(lean_object**); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Term_getElabElimExprInfo___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_findMethod_x3f___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedName; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___lambda__5___closed__1; @@ -1385,7 +1383,6 @@ uint8_t l_Lean_isAuxRecursorWithSuffix(lean_object*, lean_object*, lean_object*) lean_object* lean_array_get_size(lean_object*); lean_object* l_Lean_LocalDecl_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_normalizeFunType___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_finalize___closed__1; static lean_object* l___regBuiltin_Lean_Elab_Term_elabApp_declRange__1___closed__2; @@ -1436,7 +1433,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Term_ElabAppArgs_synthesizeAppInstMVars___r LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_getSuccesses___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_compileDecl___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Term_elabExplicit_declRange__1(lean_object*); -static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7; static lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValAux___lambda__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_fTypeHasOptAutoParams(lean_object*); uint8_t l_Lean_Expr_isConst(lean_object*); @@ -1485,6 +1481,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_transform___at_Lean_Elab_Term_ElabElim_reve LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Term_throwInvalidNamedArg(lean_object*); static lean_object* l_Lean_Elab_Term_ElabElim_finalize___lambda__13___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_withMCtx___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux___spec__3(lean_object*); @@ -1533,6 +1530,7 @@ LEAN_EXPORT lean_object* l_Lean_getRefPos___at___private_Lean_Elab_App_0__Lean_E lean_object* l_Lean_Elab_Term_resolveName_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_addInstMVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_ElabAppArgs_shouldPropagateExpectedTypeFor___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_hasOptAutoParams___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -55112,20 +55110,6 @@ x_14 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go(x_3, x_5, x return x_14; } } -LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_box(0); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_1); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_9); -return x_12; -} -} static lean_object* _init_l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__1() { _start: { @@ -55180,7 +55164,7 @@ return x_2; LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_103; +lean_object* x_12; lean_object* x_13; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_104; x_23 = l_Lean_instantiateMVars___at_Lean_Elab_Term_MVarErrorInfo_logError___spec__1(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11); x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); @@ -55203,241 +55187,772 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_28); -x_103 = l_Lean_Elab_Term_tryPostponeIfMVar(x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_25); -if (lean_obj_tag(x_103) == 0) +x_104 = l_Lean_Elab_Term_tryPostponeIfMVar(x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_25); +if (lean_obj_tag(x_104) == 0) { -lean_object* x_104; lean_object* x_105; -x_104 = lean_ctor_get(x_103, 1); -lean_inc(x_104); -lean_dec(x_103); -x_105 = l_Lean_Expr_cleanupAnnotations(x_28); -if (lean_obj_tag(x_105) == 4) +lean_object* x_105; lean_object* x_106; +x_105 = lean_ctor_get(x_104, 1); +lean_inc(x_105); +lean_dec(x_104); +x_106 = l_Lean_Expr_cleanupAnnotations(x_28); +if (lean_obj_tag(x_106) == 4) { -lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; uint8_t x_111; -x_106 = lean_ctor_get(x_105, 0); -lean_inc(x_106); -lean_dec(x_105); -x_107 = l_Lean_Syntax_getId(x_1); -x_108 = lean_erase_macro_scopes(x_107); -x_109 = l_Lean_Name_append(x_106, x_108); -x_110 = lean_st_ref_get(x_10, x_104); -x_111 = !lean_is_exclusive(x_110); -if (x_111 == 0) +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; uint8_t x_112; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +lean_dec(x_106); +x_108 = l_Lean_Syntax_getId(x_1); +x_109 = lean_erase_macro_scopes(x_108); +x_110 = l_Lean_Name_append(x_107, x_109); +x_111 = lean_st_ref_get(x_10, x_105); +x_112 = !lean_is_exclusive(x_111); +if (x_112 == 0) +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; +x_113 = lean_ctor_get(x_111, 0); +x_114 = lean_ctor_get(x_111, 1); +x_115 = lean_ctor_get(x_113, 0); +lean_inc(x_115); +lean_dec(x_113); +x_116 = l_Lean_Environment_contains(x_115, x_110); +if (x_116 == 0) { -lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; -x_112 = lean_ctor_get(x_110, 0); -x_113 = lean_ctor_get(x_110, 1); -x_114 = lean_ctor_get(x_112, 0); -lean_inc(x_114); -lean_dec(x_112); -x_115 = l_Lean_Environment_contains(x_114, x_109); -if (x_115 == 0) -{ -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_116 = l_Lean_MessageData_ofName(x_109); -x_117 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; -lean_ctor_set_tag(x_110, 7); -lean_ctor_set(x_110, 1, x_116); -lean_ctor_set(x_110, 0, x_117); -x_118 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; -x_119 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_119, 0, x_110); -lean_ctor_set(x_119, 1, x_118); +lean_object* x_117; lean_object* x_118; +lean_inc(x_9); +lean_inc(x_7); +lean_inc(x_5); +lean_inc(x_110); +x_117 = l_Lean_Elab_Term_resolveLocalName(x_110, x_5, x_6, x_7, x_8, x_9, x_10, x_114); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +if (lean_obj_tag(x_118) == 0) +{ +uint8_t x_119; +x_119 = !lean_is_exclusive(x_117); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_120 = lean_ctor_get(x_117, 1); +x_121 = lean_ctor_get(x_117, 0); +lean_dec(x_121); +x_122 = l_Lean_MessageData_ofName(x_110); +x_123 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +lean_ctor_set_tag(x_117, 7); +lean_ctor_set(x_117, 1, x_122); +lean_ctor_set(x_117, 0, x_123); +x_124 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_124); +lean_ctor_set(x_111, 0, x_117); lean_inc(x_3); -x_120 = l_Lean_indentExpr(x_3); -x_121 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_121, 0, x_119); -lean_ctor_set(x_121, 1, x_120); -x_122 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; -x_123 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); +x_125 = l_Lean_indentExpr(x_3); +x_126 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_126, 0, x_111); +lean_ctor_set(x_126, 1, x_125); +x_127 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +x_128 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); lean_inc(x_5); -x_124 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_123, x_5, x_6, x_7, x_8, x_9, x_10, x_113); -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_29 = x_125; -x_30 = x_126; -goto block_102; +x_129 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_128, x_5, x_6, x_7, x_8, x_9, x_10, x_120); +x_130 = lean_ctor_get(x_129, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_129, 1); +lean_inc(x_131); +lean_dec(x_129); +x_29 = x_130; +x_30 = x_131; +goto block_103; } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -lean_free_object(x_110); +lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_132 = lean_ctor_get(x_117, 1); +lean_inc(x_132); +lean_dec(x_117); +x_133 = l_Lean_MessageData_ofName(x_110); +x_134 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +x_135 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_135, 0, x_134); +lean_ctor_set(x_135, 1, x_133); +x_136 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_136); +lean_ctor_set(x_111, 0, x_135); +lean_inc(x_3); +x_137 = l_Lean_indentExpr(x_3); +x_138 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_138, 0, x_111); +lean_ctor_set(x_138, 1, x_137); +x_139 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +x_140 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_140, 0, x_138); +lean_ctor_set(x_140, 1, x_139); +lean_inc(x_5); +x_141 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_140, x_5, x_6, x_7, x_8, x_9, x_10, x_132); +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +lean_dec(x_141); +x_29 = x_142; +x_30 = x_143; +goto block_103; +} +} +else +{ +lean_object* x_144; lean_object* x_145; +x_144 = lean_ctor_get(x_118, 0); +lean_inc(x_144); +lean_dec(x_118); +x_145 = lean_ctor_get(x_144, 1); +lean_inc(x_145); +if (lean_obj_tag(x_145) == 0) +{ +lean_object* x_146; uint8_t x_147; +lean_free_object(x_111); +lean_dec(x_110); lean_dec(x_26); lean_dec(x_24); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_127 = lean_box(0); -x_128 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2(x_109, x_127, x_5, x_6, x_7, x_8, x_9, x_10, x_113); +x_146 = lean_ctor_get(x_117, 1); +lean_inc(x_146); +lean_dec(x_117); +x_147 = !lean_is_exclusive(x_144); +if (x_147 == 0) +{ +lean_object* x_148; lean_object* x_149; +x_148 = lean_ctor_get(x_144, 1); +lean_dec(x_148); +x_149 = lean_box(0); +lean_ctor_set_tag(x_144, 1); +lean_ctor_set(x_144, 1, x_149); +x_12 = x_144; +x_13 = x_146; +goto block_22; +} +else +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_150 = lean_ctor_get(x_144, 0); +lean_inc(x_150); +lean_dec(x_144); +x_151 = lean_box(0); +x_152 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +x_12 = x_152; +x_13 = x_146; +goto block_22; +} +} +else +{ +uint8_t x_153; +x_153 = !lean_is_exclusive(x_144); +if (x_153 == 0) +{ +lean_object* x_154; lean_object* x_155; uint8_t x_156; +x_154 = lean_ctor_get(x_144, 1); +lean_dec(x_154); +x_155 = lean_ctor_get(x_144, 0); +lean_dec(x_155); +x_156 = !lean_is_exclusive(x_145); +if (x_156 == 0) +{ +lean_object* x_157; lean_object* x_158; uint8_t x_159; +x_157 = lean_ctor_get(x_145, 1); +lean_dec(x_157); +x_158 = lean_ctor_get(x_145, 0); +lean_dec(x_158); +x_159 = !lean_is_exclusive(x_117); +if (x_159 == 0) +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_160 = lean_ctor_get(x_117, 1); +x_161 = lean_ctor_get(x_117, 0); +lean_dec(x_161); +x_162 = l_Lean_MessageData_ofName(x_110); +x_163 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +lean_ctor_set_tag(x_145, 7); +lean_ctor_set(x_145, 1, x_162); +lean_ctor_set(x_145, 0, x_163); +x_164 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +lean_ctor_set_tag(x_144, 7); +lean_ctor_set(x_144, 1, x_164); +lean_ctor_set(x_144, 0, x_145); +lean_inc(x_3); +x_165 = l_Lean_indentExpr(x_3); +lean_ctor_set_tag(x_117, 7); +lean_ctor_set(x_117, 1, x_165); +lean_ctor_set(x_117, 0, x_144); +x_166 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_166); +lean_ctor_set(x_111, 0, x_117); +lean_inc(x_5); +x_167 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_111, x_5, x_6, x_7, x_8, x_9, x_10, x_160); +x_168 = lean_ctor_get(x_167, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_167, 1); +lean_inc(x_169); +lean_dec(x_167); +x_29 = x_168; +x_30 = x_169; +goto block_103; +} +else +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_170 = lean_ctor_get(x_117, 1); +lean_inc(x_170); +lean_dec(x_117); +x_171 = l_Lean_MessageData_ofName(x_110); +x_172 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +lean_ctor_set_tag(x_145, 7); +lean_ctor_set(x_145, 1, x_171); +lean_ctor_set(x_145, 0, x_172); +x_173 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +lean_ctor_set_tag(x_144, 7); +lean_ctor_set(x_144, 1, x_173); +lean_ctor_set(x_144, 0, x_145); +lean_inc(x_3); +x_174 = l_Lean_indentExpr(x_3); +x_175 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_175, 0, x_144); +lean_ctor_set(x_175, 1, x_174); +x_176 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_176); +lean_ctor_set(x_111, 0, x_175); +lean_inc(x_5); +x_177 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_111, x_5, x_6, x_7, x_8, x_9, x_10, x_170); +x_178 = lean_ctor_get(x_177, 0); +lean_inc(x_178); +x_179 = lean_ctor_get(x_177, 1); +lean_inc(x_179); +lean_dec(x_177); +x_29 = x_178; +x_30 = x_179; +goto block_103; +} +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_145); +x_180 = lean_ctor_get(x_117, 1); +lean_inc(x_180); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_181 = x_117; +} else { + lean_dec_ref(x_117); + x_181 = lean_box(0); +} +x_182 = l_Lean_MessageData_ofName(x_110); +x_183 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +x_184 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_184, 0, x_183); +lean_ctor_set(x_184, 1, x_182); +x_185 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +lean_ctor_set_tag(x_144, 7); +lean_ctor_set(x_144, 1, x_185); +lean_ctor_set(x_144, 0, x_184); +lean_inc(x_3); +x_186 = l_Lean_indentExpr(x_3); +if (lean_is_scalar(x_181)) { + x_187 = lean_alloc_ctor(7, 2, 0); +} else { + x_187 = x_181; + lean_ctor_set_tag(x_187, 7); +} +lean_ctor_set(x_187, 0, x_144); +lean_ctor_set(x_187, 1, x_186); +x_188 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_188); +lean_ctor_set(x_111, 0, x_187); +lean_inc(x_5); +x_189 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_111, x_5, x_6, x_7, x_8, x_9, x_10, x_180); +x_190 = lean_ctor_get(x_189, 0); +lean_inc(x_190); +x_191 = lean_ctor_get(x_189, 1); +lean_inc(x_191); +lean_dec(x_189); +x_29 = x_190; +x_30 = x_191; +goto block_103; +} +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; +lean_dec(x_144); +if (lean_is_exclusive(x_145)) { + lean_ctor_release(x_145, 0); + lean_ctor_release(x_145, 1); + x_192 = x_145; +} else { + lean_dec_ref(x_145); + x_192 = lean_box(0); +} +x_193 = lean_ctor_get(x_117, 1); +lean_inc(x_193); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_194 = x_117; +} else { + lean_dec_ref(x_117); + x_194 = lean_box(0); +} +x_195 = l_Lean_MessageData_ofName(x_110); +x_196 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +if (lean_is_scalar(x_192)) { + x_197 = lean_alloc_ctor(7, 2, 0); +} else { + x_197 = x_192; + lean_ctor_set_tag(x_197, 7); +} +lean_ctor_set(x_197, 0, x_196); +lean_ctor_set(x_197, 1, x_195); +x_198 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +x_199 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_inc(x_3); +x_200 = l_Lean_indentExpr(x_3); +if (lean_is_scalar(x_194)) { + x_201 = lean_alloc_ctor(7, 2, 0); +} else { + x_201 = x_194; + lean_ctor_set_tag(x_201, 7); +} +lean_ctor_set(x_201, 0, x_199); +lean_ctor_set(x_201, 1, x_200); +x_202 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +lean_ctor_set_tag(x_111, 7); +lean_ctor_set(x_111, 1, x_202); +lean_ctor_set(x_111, 0, x_201); +lean_inc(x_5); +x_203 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_111, x_5, x_6, x_7, x_8, x_9, x_10, x_193); +x_204 = lean_ctor_get(x_203, 0); +lean_inc(x_204); +x_205 = lean_ctor_get(x_203, 1); +lean_inc(x_205); +lean_dec(x_203); +x_29 = x_204; +x_30 = x_205; +goto block_103; +} +} +} +} +else +{ +lean_object* x_206; lean_object* x_207; +lean_free_object(x_111); +x_206 = lean_box(0); +lean_inc(x_9); +lean_inc(x_5); +x_207 = l_Lean_Elab_Term_mkConst(x_110, x_206, x_5, x_6, x_7, x_8, x_9, x_10, x_114); +if (lean_obj_tag(x_207) == 0) +{ +uint8_t x_208; +lean_dec(x_26); +lean_dec(x_24); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -lean_dec(x_128); -x_12 = x_129; -x_13 = x_130; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_208 = !lean_is_exclusive(x_207); +if (x_208 == 0) +{ +lean_object* x_209; lean_object* x_210; +x_209 = lean_ctor_get(x_207, 1); +x_210 = lean_box(0); +lean_ctor_set(x_207, 1, x_210); +x_12 = x_207; +x_13 = x_209; +goto block_22; +} +else +{ +lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_211 = lean_ctor_get(x_207, 0); +x_212 = lean_ctor_get(x_207, 1); +lean_inc(x_212); +lean_inc(x_211); +lean_dec(x_207); +x_213 = lean_box(0); +x_214 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_214, 0, x_211); +lean_ctor_set(x_214, 1, x_213); +x_12 = x_214; +x_13 = x_212; goto block_22; } } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; -x_131 = lean_ctor_get(x_110, 0); -x_132 = lean_ctor_get(x_110, 1); -lean_inc(x_132); -lean_inc(x_131); -lean_dec(x_110); -x_133 = lean_ctor_get(x_131, 0); -lean_inc(x_133); -lean_dec(x_131); -x_134 = l_Lean_Environment_contains(x_133, x_109); -if (x_134 == 0) +lean_object* x_215; lean_object* x_216; +x_215 = lean_ctor_get(x_207, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_207, 1); +lean_inc(x_216); +lean_dec(x_207); +x_29 = x_215; +x_30 = x_216; +goto block_103; +} +} +} +else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_135 = l_Lean_MessageData_ofName(x_109); -x_136 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; -x_137 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_135); -x_138 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; -x_139 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); +lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; +x_217 = lean_ctor_get(x_111, 0); +x_218 = lean_ctor_get(x_111, 1); +lean_inc(x_218); +lean_inc(x_217); +lean_dec(x_111); +x_219 = lean_ctor_get(x_217, 0); +lean_inc(x_219); +lean_dec(x_217); +x_220 = l_Lean_Environment_contains(x_219, x_110); +if (x_220 == 0) +{ +lean_object* x_221; lean_object* x_222; +lean_inc(x_9); +lean_inc(x_7); +lean_inc(x_5); +lean_inc(x_110); +x_221 = l_Lean_Elab_Term_resolveLocalName(x_110, x_5, x_6, x_7, x_8, x_9, x_10, x_218); +x_222 = lean_ctor_get(x_221, 0); +lean_inc(x_222); +if (lean_obj_tag(x_222) == 0) +{ +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_223 = lean_ctor_get(x_221, 1); +lean_inc(x_223); +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + lean_ctor_release(x_221, 1); + x_224 = x_221; +} else { + lean_dec_ref(x_221); + x_224 = lean_box(0); +} +x_225 = l_Lean_MessageData_ofName(x_110); +x_226 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +if (lean_is_scalar(x_224)) { + x_227 = lean_alloc_ctor(7, 2, 0); +} else { + x_227 = x_224; + lean_ctor_set_tag(x_227, 7); +} +lean_ctor_set(x_227, 0, x_226); +lean_ctor_set(x_227, 1, x_225); +x_228 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +x_229 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_229, 0, x_227); +lean_ctor_set(x_229, 1, x_228); lean_inc(x_3); -x_140 = l_Lean_indentExpr(x_3); -x_141 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -x_142 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; -x_143 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_143, 0, x_141); -lean_ctor_set(x_143, 1, x_142); +x_230 = l_Lean_indentExpr(x_3); +x_231 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_231, 0, x_229); +lean_ctor_set(x_231, 1, x_230); +x_232 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +x_233 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_233, 0, x_231); +lean_ctor_set(x_233, 1, x_232); lean_inc(x_5); -x_144 = l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(x_143, x_5, x_6, x_7, x_8, x_9, x_10, x_132); -x_145 = lean_ctor_get(x_144, 0); -lean_inc(x_145); -x_146 = lean_ctor_get(x_144, 1); -lean_inc(x_146); -lean_dec(x_144); -x_29 = x_145; -x_30 = x_146; -goto block_102; +x_234 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_233, x_5, x_6, x_7, x_8, x_9, x_10, x_223); +x_235 = lean_ctor_get(x_234, 0); +lean_inc(x_235); +x_236 = lean_ctor_get(x_234, 1); +lean_inc(x_236); +lean_dec(x_234); +x_29 = x_235; +x_30 = x_236; +goto block_103; } else { -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +lean_object* x_237; lean_object* x_238; +x_237 = lean_ctor_get(x_222, 0); +lean_inc(x_237); +lean_dec(x_222); +x_238 = lean_ctor_get(x_237, 1); +lean_inc(x_238); +if (lean_obj_tag(x_238) == 0) +{ +lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; +lean_dec(x_110); lean_dec(x_26); lean_dec(x_24); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_147 = lean_box(0); -x_148 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2(x_109, x_147, x_5, x_6, x_7, x_8, x_9, x_10, x_132); +x_239 = lean_ctor_get(x_221, 1); +lean_inc(x_239); +lean_dec(x_221); +x_240 = lean_ctor_get(x_237, 0); +lean_inc(x_240); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + x_241 = x_237; +} else { + lean_dec_ref(x_237); + x_241 = lean_box(0); +} +x_242 = lean_box(0); +if (lean_is_scalar(x_241)) { + x_243 = lean_alloc_ctor(1, 2, 0); +} else { + x_243 = x_241; + lean_ctor_set_tag(x_243, 1); +} +lean_ctor_set(x_243, 0, x_240); +lean_ctor_set(x_243, 1, x_242); +x_12 = x_243; +x_13 = x_239; +goto block_22; +} +else +{ +lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + x_244 = x_237; +} else { + lean_dec_ref(x_237); + x_244 = lean_box(0); +} +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_245 = x_238; +} else { + lean_dec_ref(x_238); + x_245 = lean_box(0); +} +x_246 = lean_ctor_get(x_221, 1); +lean_inc(x_246); +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + lean_ctor_release(x_221, 1); + x_247 = x_221; +} else { + lean_dec_ref(x_221); + x_247 = lean_box(0); +} +x_248 = l_Lean_MessageData_ofName(x_110); +x_249 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__4; +if (lean_is_scalar(x_245)) { + x_250 = lean_alloc_ctor(7, 2, 0); +} else { + x_250 = x_245; + lean_ctor_set_tag(x_250, 7); +} +lean_ctor_set(x_250, 0, x_249); +lean_ctor_set(x_250, 1, x_248); +x_251 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__6; +if (lean_is_scalar(x_244)) { + x_252 = lean_alloc_ctor(7, 2, 0); +} else { + x_252 = x_244; + lean_ctor_set_tag(x_252, 7); +} +lean_ctor_set(x_252, 0, x_250); +lean_ctor_set(x_252, 1, x_251); +lean_inc(x_3); +x_253 = l_Lean_indentExpr(x_3); +if (lean_is_scalar(x_247)) { + x_254 = lean_alloc_ctor(7, 2, 0); +} else { + x_254 = x_247; + lean_ctor_set_tag(x_254, 7); +} +lean_ctor_set(x_254, 0, x_252); +lean_ctor_set(x_254, 1, x_253); +x_255 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +x_256 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_256, 0, x_254); +lean_ctor_set(x_256, 1, x_255); +lean_inc(x_5); +x_257 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_256, x_5, x_6, x_7, x_8, x_9, x_10, x_246); +x_258 = lean_ctor_get(x_257, 0); +lean_inc(x_258); +x_259 = lean_ctor_get(x_257, 1); +lean_inc(x_259); +lean_dec(x_257); +x_29 = x_258; +x_30 = x_259; +goto block_103; +} +} +} +else +{ +lean_object* x_260; lean_object* x_261; +x_260 = lean_box(0); +lean_inc(x_9); +lean_inc(x_5); +x_261 = l_Lean_Elab_Term_mkConst(x_110, x_260, x_5, x_6, x_7, x_8, x_9, x_10, x_218); +if (lean_obj_tag(x_261) == 0) +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; +lean_dec(x_26); +lean_dec(x_24); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_149 = lean_ctor_get(x_148, 0); -lean_inc(x_149); -x_150 = lean_ctor_get(x_148, 1); -lean_inc(x_150); -lean_dec(x_148); -x_12 = x_149; -x_13 = x_150; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_262 = lean_ctor_get(x_261, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_261, 1); +lean_inc(x_263); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + lean_ctor_release(x_261, 1); + x_264 = x_261; +} else { + lean_dec_ref(x_261); + x_264 = lean_box(0); +} +x_265 = lean_box(0); +if (lean_is_scalar(x_264)) { + x_266 = lean_alloc_ctor(0, 2, 0); +} else { + x_266 = x_264; +} +lean_ctor_set(x_266, 0, x_262); +lean_ctor_set(x_266, 1, x_265); +x_12 = x_266; +x_13 = x_263; goto block_22; } +else +{ +lean_object* x_267; lean_object* x_268; +x_267 = lean_ctor_get(x_261, 0); +lean_inc(x_267); +x_268 = lean_ctor_get(x_261, 1); +lean_inc(x_268); +lean_dec(x_261); +x_29 = x_267; +x_30 = x_268; +goto block_103; +} +} } } else { -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -lean_dec(x_105); +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +lean_dec(x_106); lean_inc(x_3); -x_151 = l_Lean_indentExpr(x_3); -x_152 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__2; -x_153 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_153, 0, x_152); -lean_ctor_set(x_153, 1, x_151); -x_154 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; -x_155 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_154); +x_269 = l_Lean_indentExpr(x_3); +x_270 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___closed__2; +x_271 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_271, 0, x_270); +lean_ctor_set(x_271, 1, x_269); +x_272 = l___private_Lean_Elab_App_0__Lean_Elab_Term_mkProjAndCheck___closed__8; +x_273 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_273, 0, x_271); +lean_ctor_set(x_273, 1, x_272); lean_inc(x_5); -x_156 = l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1(x_155, x_5, x_6, x_7, x_8, x_9, x_10, x_104); -x_157 = lean_ctor_get(x_156, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_156, 1); -lean_inc(x_158); -lean_dec(x_156); -x_29 = x_157; -x_30 = x_158; -goto block_102; +x_274 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_273, x_5, x_6, x_7, x_8, x_9, x_10, x_105); +x_275 = lean_ctor_get(x_274, 0); +lean_inc(x_275); +x_276 = lean_ctor_get(x_274, 1); +lean_inc(x_276); +lean_dec(x_274); +x_29 = x_275; +x_30 = x_276; +goto block_103; } } else { -uint8_t x_159; +uint8_t x_277; lean_dec(x_28); lean_dec(x_26); -x_159 = !lean_is_exclusive(x_103); -if (x_159 == 0) +x_277 = !lean_is_exclusive(x_104); +if (x_277 == 0) { -lean_object* x_160; lean_object* x_161; uint8_t x_162; -x_160 = lean_ctor_get(x_103, 0); -x_161 = lean_ctor_get(x_103, 1); -x_162 = l_Lean_Exception_isInterrupt(x_160); -if (x_162 == 0) +lean_object* x_278; lean_object* x_279; uint8_t x_280; +x_278 = lean_ctor_get(x_104, 0); +x_279 = lean_ctor_get(x_104, 1); +x_280 = l_Lean_Exception_isInterrupt(x_278); +if (x_280 == 0) { -uint8_t x_163; -x_163 = l_Lean_Exception_isRuntime(x_160); -if (x_163 == 0) +uint8_t x_281; +x_281 = l_Lean_Exception_isRuntime(x_278); +if (x_281 == 0) { -if (lean_obj_tag(x_160) == 0) +if (lean_obj_tag(x_278) == 0) { -uint8_t x_164; lean_object* x_165; -lean_free_object(x_103); -x_164 = 0; +uint8_t x_282; lean_object* x_283; +lean_free_object(x_104); +x_282 = 0; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_165 = l_Lean_Meta_unfoldDefinition_x3f(x_24, x_164, x_7, x_8, x_9, x_10, x_161); -if (lean_obj_tag(x_165) == 0) +x_283 = l_Lean_Meta_unfoldDefinition_x3f(x_24, x_282, x_7, x_8, x_9, x_10, x_279); +if (lean_obj_tag(x_283) == 0) { -lean_object* x_166; -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -if (lean_obj_tag(x_166) == 0) +lean_object* x_284; +x_284 = lean_ctor_get(x_283, 0); +lean_inc(x_284); +if (lean_obj_tag(x_284) == 0) { -uint8_t x_167; +uint8_t x_285; lean_dec(x_3); lean_dec(x_1); -x_167 = !lean_is_exclusive(x_165); -if (x_167 == 0) +x_285 = !lean_is_exclusive(x_283); +if (x_285 == 0) { -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; -x_168 = lean_ctor_get(x_165, 1); -x_169 = lean_ctor_get(x_165, 0); -lean_dec(x_169); -x_170 = lean_array_get_size(x_4); -x_171 = lean_unsigned_to_nat(0u); -x_172 = lean_nat_dec_lt(x_171, x_170); -if (x_172 == 0) +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; uint8_t x_290; +x_286 = lean_ctor_get(x_283, 1); +x_287 = lean_ctor_get(x_283, 0); +lean_dec(x_287); +x_288 = lean_array_get_size(x_4); +x_289 = lean_unsigned_to_nat(0u); +x_290 = lean_nat_dec_lt(x_289, x_288); +if (x_290 == 0) { -lean_dec(x_170); +lean_dec(x_288); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55445,17 +55960,17 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_ctor_set_tag(x_165, 1); -lean_ctor_set(x_165, 0, x_160); -return x_165; +lean_ctor_set_tag(x_283, 1); +lean_ctor_set(x_283, 0, x_278); +return x_283; } else { -uint8_t x_173; -x_173 = lean_nat_dec_le(x_170, x_170); -if (x_173 == 0) +uint8_t x_291; +x_291 = lean_nat_dec_le(x_288, x_288); +if (x_291 == 0) { -lean_dec(x_170); +lean_dec(x_288); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55463,71 +55978,71 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_ctor_set_tag(x_165, 1); -lean_ctor_set(x_165, 0, x_160); -return x_165; +lean_ctor_set_tag(x_283, 1); +lean_ctor_set(x_283, 0, x_278); +return x_283; } else { -size_t x_174; size_t x_175; lean_object* x_176; lean_object* x_177; -lean_free_object(x_165); -x_174 = 0; -x_175 = lean_usize_of_nat(x_170); -lean_dec(x_170); -x_176 = lean_box(0); -x_177 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_174, x_175, x_176, x_5, x_6, x_7, x_8, x_9, x_10, x_168); +size_t x_292; size_t x_293; lean_object* x_294; lean_object* x_295; +lean_free_object(x_283); +x_292 = 0; +x_293 = lean_usize_of_nat(x_288); +lean_dec(x_288); +x_294 = lean_box(0); +x_295 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_292, x_293, x_294, x_5, x_6, x_7, x_8, x_9, x_10, x_286); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_obj_tag(x_177) == 0) +if (lean_obj_tag(x_295) == 0) { -uint8_t x_178; -x_178 = !lean_is_exclusive(x_177); -if (x_178 == 0) +uint8_t x_296; +x_296 = !lean_is_exclusive(x_295); +if (x_296 == 0) { -lean_object* x_179; -x_179 = lean_ctor_get(x_177, 0); -lean_dec(x_179); -lean_ctor_set_tag(x_177, 1); -lean_ctor_set(x_177, 0, x_160); -return x_177; +lean_object* x_297; +x_297 = lean_ctor_get(x_295, 0); +lean_dec(x_297); +lean_ctor_set_tag(x_295, 1); +lean_ctor_set(x_295, 0, x_278); +return x_295; } else { -lean_object* x_180; lean_object* x_181; -x_180 = lean_ctor_get(x_177, 1); -lean_inc(x_180); -lean_dec(x_177); -x_181 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_181, 0, x_160); -lean_ctor_set(x_181, 1, x_180); -return x_181; +lean_object* x_298; lean_object* x_299; +x_298 = lean_ctor_get(x_295, 1); +lean_inc(x_298); +lean_dec(x_295); +x_299 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_299, 0, x_278); +lean_ctor_set(x_299, 1, x_298); +return x_299; } } else { -uint8_t x_182; -lean_dec(x_160); -x_182 = !lean_is_exclusive(x_177); -if (x_182 == 0) +uint8_t x_300; +lean_dec(x_278); +x_300 = !lean_is_exclusive(x_295); +if (x_300 == 0) { -return x_177; +return x_295; } else { -lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_183 = lean_ctor_get(x_177, 0); -x_184 = lean_ctor_get(x_177, 1); -lean_inc(x_184); -lean_inc(x_183); -lean_dec(x_177); -x_185 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_185, 0, x_183); -lean_ctor_set(x_185, 1, x_184); -return x_185; +lean_object* x_301; lean_object* x_302; lean_object* x_303; +x_301 = lean_ctor_get(x_295, 0); +x_302 = lean_ctor_get(x_295, 1); +lean_inc(x_302); +lean_inc(x_301); +lean_dec(x_295); +x_303 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_303, 0, x_301); +lean_ctor_set(x_303, 1, x_302); +return x_303; } } } @@ -55535,17 +56050,17 @@ return x_185; } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; uint8_t x_189; -x_186 = lean_ctor_get(x_165, 1); -lean_inc(x_186); -lean_dec(x_165); -x_187 = lean_array_get_size(x_4); -x_188 = lean_unsigned_to_nat(0u); -x_189 = lean_nat_dec_lt(x_188, x_187); -if (x_189 == 0) +lean_object* x_304; lean_object* x_305; lean_object* x_306; uint8_t x_307; +x_304 = lean_ctor_get(x_283, 1); +lean_inc(x_304); +lean_dec(x_283); +x_305 = lean_array_get_size(x_4); +x_306 = lean_unsigned_to_nat(0u); +x_307 = lean_nat_dec_lt(x_306, x_305); +if (x_307 == 0) { -lean_object* x_190; -lean_dec(x_187); +lean_object* x_308; +lean_dec(x_305); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55553,19 +56068,19 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_190 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_190, 0, x_160); -lean_ctor_set(x_190, 1, x_186); -return x_190; +x_308 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_308, 0, x_278); +lean_ctor_set(x_308, 1, x_304); +return x_308; } else { -uint8_t x_191; -x_191 = lean_nat_dec_le(x_187, x_187); -if (x_191 == 0) +uint8_t x_309; +x_309 = lean_nat_dec_le(x_305, x_305); +if (x_309 == 0) { -lean_object* x_192; -lean_dec(x_187); +lean_object* x_310; +lean_dec(x_305); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55573,72 +56088,72 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_192 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_192, 0, x_160); -lean_ctor_set(x_192, 1, x_186); -return x_192; +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_278); +lean_ctor_set(x_310, 1, x_304); +return x_310; } else { -size_t x_193; size_t x_194; lean_object* x_195; lean_object* x_196; -x_193 = 0; -x_194 = lean_usize_of_nat(x_187); -lean_dec(x_187); -x_195 = lean_box(0); -x_196 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_193, x_194, x_195, x_5, x_6, x_7, x_8, x_9, x_10, x_186); +size_t x_311; size_t x_312; lean_object* x_313; lean_object* x_314; +x_311 = 0; +x_312 = lean_usize_of_nat(x_305); +lean_dec(x_305); +x_313 = lean_box(0); +x_314 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_311, x_312, x_313, x_5, x_6, x_7, x_8, x_9, x_10, x_304); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_obj_tag(x_196) == 0) +if (lean_obj_tag(x_314) == 0) { -lean_object* x_197; lean_object* x_198; lean_object* x_199; -x_197 = lean_ctor_get(x_196, 1); -lean_inc(x_197); -if (lean_is_exclusive(x_196)) { - lean_ctor_release(x_196, 0); - lean_ctor_release(x_196, 1); - x_198 = x_196; +lean_object* x_315; lean_object* x_316; lean_object* x_317; +x_315 = lean_ctor_get(x_314, 1); +lean_inc(x_315); +if (lean_is_exclusive(x_314)) { + lean_ctor_release(x_314, 0); + lean_ctor_release(x_314, 1); + x_316 = x_314; } else { - lean_dec_ref(x_196); - x_198 = lean_box(0); + lean_dec_ref(x_314); + x_316 = lean_box(0); } -if (lean_is_scalar(x_198)) { - x_199 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_316)) { + x_317 = lean_alloc_ctor(1, 2, 0); } else { - x_199 = x_198; - lean_ctor_set_tag(x_199, 1); + x_317 = x_316; + lean_ctor_set_tag(x_317, 1); } -lean_ctor_set(x_199, 0, x_160); -lean_ctor_set(x_199, 1, x_197); -return x_199; +lean_ctor_set(x_317, 0, x_278); +lean_ctor_set(x_317, 1, x_315); +return x_317; } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; -lean_dec(x_160); -x_200 = lean_ctor_get(x_196, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_196, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_196)) { - lean_ctor_release(x_196, 0); - lean_ctor_release(x_196, 1); - x_202 = x_196; +lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; +lean_dec(x_278); +x_318 = lean_ctor_get(x_314, 0); +lean_inc(x_318); +x_319 = lean_ctor_get(x_314, 1); +lean_inc(x_319); +if (lean_is_exclusive(x_314)) { + lean_ctor_release(x_314, 0); + lean_ctor_release(x_314, 1); + x_320 = x_314; } else { - lean_dec_ref(x_196); - x_202 = lean_box(0); + lean_dec_ref(x_314); + x_320 = lean_box(0); } -if (lean_is_scalar(x_202)) { - x_203 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_320)) { + x_321 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_202; + x_321 = x_320; } -lean_ctor_set(x_203, 0, x_200); -lean_ctor_set(x_203, 1, x_201); -return x_203; +lean_ctor_set(x_321, 0, x_318); +lean_ctor_set(x_321, 1, x_319); +return x_321; } } } @@ -55646,119 +56161,119 @@ return x_203; } else { -lean_object* x_204; lean_object* x_205; lean_object* x_206; uint8_t x_207; -x_204 = lean_ctor_get(x_165, 1); -lean_inc(x_204); -lean_dec(x_165); -x_205 = lean_ctor_get(x_166, 0); -lean_inc(x_205); -lean_dec(x_166); -lean_inc(x_160); -x_206 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__1), 12, 4); -lean_closure_set(x_206, 0, x_4); -lean_closure_set(x_206, 1, x_160); -lean_closure_set(x_206, 2, x_1); -lean_closure_set(x_206, 3, x_3); -x_207 = !lean_is_exclusive(x_160); -if (x_207 == 0) -{ -lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_208 = lean_ctor_get(x_160, 1); -lean_dec(x_208); -x_209 = lean_ctor_get(x_160, 0); -lean_dec(x_209); -x_210 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_205, x_206, x_5, x_6, x_7, x_8, x_9, x_10, x_204); -if (lean_obj_tag(x_210) == 0) -{ -lean_object* x_211; lean_object* x_212; lean_object* x_213; -x_211 = lean_ctor_get(x_210, 0); -lean_inc(x_211); -x_212 = lean_ctor_get(x_210, 1); -lean_inc(x_212); -lean_dec(x_210); -x_213 = lean_box(0); -lean_ctor_set(x_160, 1, x_213); -lean_ctor_set(x_160, 0, x_211); -x_12 = x_160; -x_13 = x_212; +lean_object* x_322; lean_object* x_323; lean_object* x_324; uint8_t x_325; +x_322 = lean_ctor_get(x_283, 1); +lean_inc(x_322); +lean_dec(x_283); +x_323 = lean_ctor_get(x_284, 0); +lean_inc(x_323); +lean_dec(x_284); +lean_inc(x_278); +x_324 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__1), 12, 4); +lean_closure_set(x_324, 0, x_4); +lean_closure_set(x_324, 1, x_278); +lean_closure_set(x_324, 2, x_1); +lean_closure_set(x_324, 3, x_3); +x_325 = !lean_is_exclusive(x_278); +if (x_325 == 0) +{ +lean_object* x_326; lean_object* x_327; lean_object* x_328; +x_326 = lean_ctor_get(x_278, 1); +lean_dec(x_326); +x_327 = lean_ctor_get(x_278, 0); +lean_dec(x_327); +x_328 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_323, x_324, x_5, x_6, x_7, x_8, x_9, x_10, x_322); +if (lean_obj_tag(x_328) == 0) +{ +lean_object* x_329; lean_object* x_330; lean_object* x_331; +x_329 = lean_ctor_get(x_328, 0); +lean_inc(x_329); +x_330 = lean_ctor_get(x_328, 1); +lean_inc(x_330); +lean_dec(x_328); +x_331 = lean_box(0); +lean_ctor_set(x_278, 1, x_331); +lean_ctor_set(x_278, 0, x_329); +x_12 = x_278; +x_13 = x_330; goto block_22; } else { -uint8_t x_214; -lean_free_object(x_160); -x_214 = !lean_is_exclusive(x_210); -if (x_214 == 0) +uint8_t x_332; +lean_free_object(x_278); +x_332 = !lean_is_exclusive(x_328); +if (x_332 == 0) { -return x_210; +return x_328; } else { -lean_object* x_215; lean_object* x_216; lean_object* x_217; -x_215 = lean_ctor_get(x_210, 0); -x_216 = lean_ctor_get(x_210, 1); -lean_inc(x_216); -lean_inc(x_215); -lean_dec(x_210); -x_217 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_217, 0, x_215); -lean_ctor_set(x_217, 1, x_216); -return x_217; +lean_object* x_333; lean_object* x_334; lean_object* x_335; +x_333 = lean_ctor_get(x_328, 0); +x_334 = lean_ctor_get(x_328, 1); +lean_inc(x_334); +lean_inc(x_333); +lean_dec(x_328); +x_335 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_335, 0, x_333); +lean_ctor_set(x_335, 1, x_334); +return x_335; } } } else { -lean_object* x_218; -lean_dec(x_160); -x_218 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_205, x_206, x_5, x_6, x_7, x_8, x_9, x_10, x_204); -if (lean_obj_tag(x_218) == 0) +lean_object* x_336; +lean_dec(x_278); +x_336 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_323, x_324, x_5, x_6, x_7, x_8, x_9, x_10, x_322); +if (lean_obj_tag(x_336) == 0) { -lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; -x_219 = lean_ctor_get(x_218, 0); -lean_inc(x_219); -x_220 = lean_ctor_get(x_218, 1); -lean_inc(x_220); -lean_dec(x_218); -x_221 = lean_box(0); -x_222 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_222, 0, x_219); -lean_ctor_set(x_222, 1, x_221); -x_12 = x_222; -x_13 = x_220; +lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; +x_337 = lean_ctor_get(x_336, 0); +lean_inc(x_337); +x_338 = lean_ctor_get(x_336, 1); +lean_inc(x_338); +lean_dec(x_336); +x_339 = lean_box(0); +x_340 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_340, 0, x_337); +lean_ctor_set(x_340, 1, x_339); +x_12 = x_340; +x_13 = x_338; goto block_22; } else { -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_223 = lean_ctor_get(x_218, 0); -lean_inc(x_223); -x_224 = lean_ctor_get(x_218, 1); -lean_inc(x_224); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_225 = x_218; +lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; +x_341 = lean_ctor_get(x_336, 0); +lean_inc(x_341); +x_342 = lean_ctor_get(x_336, 1); +lean_inc(x_342); +if (lean_is_exclusive(x_336)) { + lean_ctor_release(x_336, 0); + lean_ctor_release(x_336, 1); + x_343 = x_336; } else { - lean_dec_ref(x_218); - x_225 = lean_box(0); + lean_dec_ref(x_336); + x_343 = lean_box(0); } -if (lean_is_scalar(x_225)) { - x_226 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_343)) { + x_344 = lean_alloc_ctor(1, 2, 0); } else { - x_226 = x_225; + x_344 = x_343; } -lean_ctor_set(x_226, 0, x_223); -lean_ctor_set(x_226, 1, x_224); -return x_226; +lean_ctor_set(x_344, 0, x_341); +lean_ctor_set(x_344, 1, x_342); +return x_344; } } } } else { -uint8_t x_227; -lean_dec(x_160); +uint8_t x_345; +lean_dec(x_278); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55768,23 +56283,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_227 = !lean_is_exclusive(x_165); -if (x_227 == 0) +x_345 = !lean_is_exclusive(x_283); +if (x_345 == 0) { -return x_165; +return x_283; } else { -lean_object* x_228; lean_object* x_229; lean_object* x_230; -x_228 = lean_ctor_get(x_165, 0); -x_229 = lean_ctor_get(x_165, 1); -lean_inc(x_229); -lean_inc(x_228); -lean_dec(x_165); -x_230 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_230, 0, x_228); -lean_ctor_set(x_230, 1, x_229); -return x_230; +lean_object* x_346; lean_object* x_347; lean_object* x_348; +x_346 = lean_ctor_get(x_283, 0); +x_347 = lean_ctor_get(x_283, 1); +lean_inc(x_347); +lean_inc(x_346); +lean_dec(x_283); +x_348 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_348, 0, x_346); +lean_ctor_set(x_348, 1, x_347); +return x_348; } } } @@ -55800,7 +56315,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -return x_103; +return x_104; } } else @@ -55815,7 +56330,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -return x_103; +return x_104; } } else @@ -55830,60 +56345,60 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -return x_103; +return x_104; } } else { -lean_object* x_231; lean_object* x_232; uint8_t x_233; -x_231 = lean_ctor_get(x_103, 0); -x_232 = lean_ctor_get(x_103, 1); -lean_inc(x_232); -lean_inc(x_231); -lean_dec(x_103); -x_233 = l_Lean_Exception_isInterrupt(x_231); -if (x_233 == 0) +lean_object* x_349; lean_object* x_350; uint8_t x_351; +x_349 = lean_ctor_get(x_104, 0); +x_350 = lean_ctor_get(x_104, 1); +lean_inc(x_350); +lean_inc(x_349); +lean_dec(x_104); +x_351 = l_Lean_Exception_isInterrupt(x_349); +if (x_351 == 0) { -uint8_t x_234; -x_234 = l_Lean_Exception_isRuntime(x_231); -if (x_234 == 0) +uint8_t x_352; +x_352 = l_Lean_Exception_isRuntime(x_349); +if (x_352 == 0) { -if (lean_obj_tag(x_231) == 0) +if (lean_obj_tag(x_349) == 0) { -uint8_t x_235; lean_object* x_236; -x_235 = 0; +uint8_t x_353; lean_object* x_354; +x_353 = 0; lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_236 = l_Lean_Meta_unfoldDefinition_x3f(x_24, x_235, x_7, x_8, x_9, x_10, x_232); -if (lean_obj_tag(x_236) == 0) +x_354 = l_Lean_Meta_unfoldDefinition_x3f(x_24, x_353, x_7, x_8, x_9, x_10, x_350); +if (lean_obj_tag(x_354) == 0) { -lean_object* x_237; -x_237 = lean_ctor_get(x_236, 0); -lean_inc(x_237); -if (lean_obj_tag(x_237) == 0) +lean_object* x_355; +x_355 = lean_ctor_get(x_354, 0); +lean_inc(x_355); +if (lean_obj_tag(x_355) == 0) { -lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; uint8_t x_242; +lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; uint8_t x_360; lean_dec(x_3); lean_dec(x_1); -x_238 = lean_ctor_get(x_236, 1); -lean_inc(x_238); -if (lean_is_exclusive(x_236)) { - lean_ctor_release(x_236, 0); - lean_ctor_release(x_236, 1); - x_239 = x_236; -} else { - lean_dec_ref(x_236); - x_239 = lean_box(0); -} -x_240 = lean_array_get_size(x_4); -x_241 = lean_unsigned_to_nat(0u); -x_242 = lean_nat_dec_lt(x_241, x_240); -if (x_242 == 0) -{ -lean_object* x_243; -lean_dec(x_240); +x_356 = lean_ctor_get(x_354, 1); +lean_inc(x_356); +if (lean_is_exclusive(x_354)) { + lean_ctor_release(x_354, 0); + lean_ctor_release(x_354, 1); + x_357 = x_354; +} else { + lean_dec_ref(x_354); + x_357 = lean_box(0); +} +x_358 = lean_array_get_size(x_4); +x_359 = lean_unsigned_to_nat(0u); +x_360 = lean_nat_dec_lt(x_359, x_358); +if (x_360 == 0) +{ +lean_object* x_361; +lean_dec(x_358); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55891,24 +56406,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_is_scalar(x_239)) { - x_243 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_357)) { + x_361 = lean_alloc_ctor(1, 2, 0); } else { - x_243 = x_239; - lean_ctor_set_tag(x_243, 1); + x_361 = x_357; + lean_ctor_set_tag(x_361, 1); } -lean_ctor_set(x_243, 0, x_231); -lean_ctor_set(x_243, 1, x_238); -return x_243; +lean_ctor_set(x_361, 0, x_349); +lean_ctor_set(x_361, 1, x_356); +return x_361; } else { -uint8_t x_244; -x_244 = lean_nat_dec_le(x_240, x_240); -if (x_244 == 0) +uint8_t x_362; +x_362 = lean_nat_dec_le(x_358, x_358); +if (x_362 == 0) { -lean_object* x_245; -lean_dec(x_240); +lean_object* x_363; +lean_dec(x_358); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -55916,157 +56431,157 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_is_scalar(x_239)) { - x_245 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_357)) { + x_363 = lean_alloc_ctor(1, 2, 0); } else { - x_245 = x_239; - lean_ctor_set_tag(x_245, 1); + x_363 = x_357; + lean_ctor_set_tag(x_363, 1); } -lean_ctor_set(x_245, 0, x_231); -lean_ctor_set(x_245, 1, x_238); -return x_245; +lean_ctor_set(x_363, 0, x_349); +lean_ctor_set(x_363, 1, x_356); +return x_363; } else { -size_t x_246; size_t x_247; lean_object* x_248; lean_object* x_249; -lean_dec(x_239); -x_246 = 0; -x_247 = lean_usize_of_nat(x_240); -lean_dec(x_240); -x_248 = lean_box(0); -x_249 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_246, x_247, x_248, x_5, x_6, x_7, x_8, x_9, x_10, x_238); +size_t x_364; size_t x_365; lean_object* x_366; lean_object* x_367; +lean_dec(x_357); +x_364 = 0; +x_365 = lean_usize_of_nat(x_358); +lean_dec(x_358); +x_366 = lean_box(0); +x_367 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_resolveLValLoop___spec__1(x_4, x_364, x_365, x_366, x_5, x_6, x_7, x_8, x_9, x_10, x_356); lean_dec(x_10); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -if (lean_obj_tag(x_249) == 0) +if (lean_obj_tag(x_367) == 0) { -lean_object* x_250; lean_object* x_251; lean_object* x_252; -x_250 = lean_ctor_get(x_249, 1); -lean_inc(x_250); -if (lean_is_exclusive(x_249)) { - lean_ctor_release(x_249, 0); - lean_ctor_release(x_249, 1); - x_251 = x_249; +lean_object* x_368; lean_object* x_369; lean_object* x_370; +x_368 = lean_ctor_get(x_367, 1); +lean_inc(x_368); +if (lean_is_exclusive(x_367)) { + lean_ctor_release(x_367, 0); + lean_ctor_release(x_367, 1); + x_369 = x_367; } else { - lean_dec_ref(x_249); - x_251 = lean_box(0); + lean_dec_ref(x_367); + x_369 = lean_box(0); } -if (lean_is_scalar(x_251)) { - x_252 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_369)) { + x_370 = lean_alloc_ctor(1, 2, 0); } else { - x_252 = x_251; - lean_ctor_set_tag(x_252, 1); + x_370 = x_369; + lean_ctor_set_tag(x_370, 1); } -lean_ctor_set(x_252, 0, x_231); -lean_ctor_set(x_252, 1, x_250); -return x_252; +lean_ctor_set(x_370, 0, x_349); +lean_ctor_set(x_370, 1, x_368); +return x_370; } else { -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -lean_dec(x_231); -x_253 = lean_ctor_get(x_249, 0); -lean_inc(x_253); -x_254 = lean_ctor_get(x_249, 1); -lean_inc(x_254); -if (lean_is_exclusive(x_249)) { - lean_ctor_release(x_249, 0); - lean_ctor_release(x_249, 1); - x_255 = x_249; +lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; +lean_dec(x_349); +x_371 = lean_ctor_get(x_367, 0); +lean_inc(x_371); +x_372 = lean_ctor_get(x_367, 1); +lean_inc(x_372); +if (lean_is_exclusive(x_367)) { + lean_ctor_release(x_367, 0); + lean_ctor_release(x_367, 1); + x_373 = x_367; } else { - lean_dec_ref(x_249); - x_255 = lean_box(0); + lean_dec_ref(x_367); + x_373 = lean_box(0); } -if (lean_is_scalar(x_255)) { - x_256 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_373)) { + x_374 = lean_alloc_ctor(1, 2, 0); } else { - x_256 = x_255; + x_374 = x_373; } -lean_ctor_set(x_256, 0, x_253); -lean_ctor_set(x_256, 1, x_254); -return x_256; +lean_ctor_set(x_374, 0, x_371); +lean_ctor_set(x_374, 1, x_372); +return x_374; } } } } else { -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; -x_257 = lean_ctor_get(x_236, 1); -lean_inc(x_257); -lean_dec(x_236); -x_258 = lean_ctor_get(x_237, 0); -lean_inc(x_258); -lean_dec(x_237); -lean_inc(x_231); -x_259 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__1), 12, 4); -lean_closure_set(x_259, 0, x_4); -lean_closure_set(x_259, 1, x_231); -lean_closure_set(x_259, 2, x_1); -lean_closure_set(x_259, 3, x_3); -if (lean_is_exclusive(x_231)) { - lean_ctor_release(x_231, 0); - lean_ctor_release(x_231, 1); - x_260 = x_231; -} else { - lean_dec_ref(x_231); - x_260 = lean_box(0); +lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; +x_375 = lean_ctor_get(x_354, 1); +lean_inc(x_375); +lean_dec(x_354); +x_376 = lean_ctor_get(x_355, 0); +lean_inc(x_376); +lean_dec(x_355); +lean_inc(x_349); +x_377 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__1), 12, 4); +lean_closure_set(x_377, 0, x_4); +lean_closure_set(x_377, 1, x_349); +lean_closure_set(x_377, 2, x_1); +lean_closure_set(x_377, 3, x_3); +if (lean_is_exclusive(x_349)) { + lean_ctor_release(x_349, 0); + lean_ctor_release(x_349, 1); + x_378 = x_349; +} else { + lean_dec_ref(x_349); + x_378 = lean_box(0); } -x_261 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_258, x_259, x_5, x_6, x_7, x_8, x_9, x_10, x_257); -if (lean_obj_tag(x_261) == 0) +x_379 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_withForallBody___rarg(x_376, x_377, x_5, x_6, x_7, x_8, x_9, x_10, x_375); +if (lean_obj_tag(x_379) == 0) { -lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; -x_262 = lean_ctor_get(x_261, 0); -lean_inc(x_262); -x_263 = lean_ctor_get(x_261, 1); -lean_inc(x_263); -lean_dec(x_261); -x_264 = lean_box(0); -if (lean_is_scalar(x_260)) { - x_265 = lean_alloc_ctor(0, 2, 0); +lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; +x_380 = lean_ctor_get(x_379, 0); +lean_inc(x_380); +x_381 = lean_ctor_get(x_379, 1); +lean_inc(x_381); +lean_dec(x_379); +x_382 = lean_box(0); +if (lean_is_scalar(x_378)) { + x_383 = lean_alloc_ctor(0, 2, 0); } else { - x_265 = x_260; + x_383 = x_378; } -lean_ctor_set(x_265, 0, x_262); -lean_ctor_set(x_265, 1, x_264); -x_12 = x_265; -x_13 = x_263; +lean_ctor_set(x_383, 0, x_380); +lean_ctor_set(x_383, 1, x_382); +x_12 = x_383; +x_13 = x_381; goto block_22; } else { -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; -lean_dec(x_260); -x_266 = lean_ctor_get(x_261, 0); -lean_inc(x_266); -x_267 = lean_ctor_get(x_261, 1); -lean_inc(x_267); -if (lean_is_exclusive(x_261)) { - lean_ctor_release(x_261, 0); - lean_ctor_release(x_261, 1); - x_268 = x_261; +lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; +lean_dec(x_378); +x_384 = lean_ctor_get(x_379, 0); +lean_inc(x_384); +x_385 = lean_ctor_get(x_379, 1); +lean_inc(x_385); +if (lean_is_exclusive(x_379)) { + lean_ctor_release(x_379, 0); + lean_ctor_release(x_379, 1); + x_386 = x_379; } else { - lean_dec_ref(x_261); - x_268 = lean_box(0); + lean_dec_ref(x_379); + x_386 = lean_box(0); } -if (lean_is_scalar(x_268)) { - x_269 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_386)) { + x_387 = lean_alloc_ctor(1, 2, 0); } else { - x_269 = x_268; + x_387 = x_386; } -lean_ctor_set(x_269, 0, x_266); -lean_ctor_set(x_269, 1, x_267); -return x_269; +lean_ctor_set(x_387, 0, x_384); +lean_ctor_set(x_387, 1, x_385); +return x_387; } } } else { -lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; -lean_dec(x_231); +lean_object* x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; +lean_dec(x_349); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -56076,31 +56591,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_270 = lean_ctor_get(x_236, 0); -lean_inc(x_270); -x_271 = lean_ctor_get(x_236, 1); -lean_inc(x_271); -if (lean_is_exclusive(x_236)) { - lean_ctor_release(x_236, 0); - lean_ctor_release(x_236, 1); - x_272 = x_236; +x_388 = lean_ctor_get(x_354, 0); +lean_inc(x_388); +x_389 = lean_ctor_get(x_354, 1); +lean_inc(x_389); +if (lean_is_exclusive(x_354)) { + lean_ctor_release(x_354, 0); + lean_ctor_release(x_354, 1); + x_390 = x_354; } else { - lean_dec_ref(x_236); - x_272 = lean_box(0); + lean_dec_ref(x_354); + x_390 = lean_box(0); } -if (lean_is_scalar(x_272)) { - x_273 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_390)) { + x_391 = lean_alloc_ctor(1, 2, 0); } else { - x_273 = x_272; + x_391 = x_390; } -lean_ctor_set(x_273, 0, x_270); -lean_ctor_set(x_273, 1, x_271); -return x_273; +lean_ctor_set(x_391, 0, x_388); +lean_ctor_set(x_391, 1, x_389); +return x_391; } } else { -lean_object* x_274; +lean_object* x_392; lean_dec(x_24); lean_dec(x_10); lean_dec(x_9); @@ -56111,15 +56626,15 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_274 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_274, 0, x_231); -lean_ctor_set(x_274, 1, x_232); -return x_274; +x_392 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_392, 0, x_349); +lean_ctor_set(x_392, 1, x_350); +return x_392; } } else { -lean_object* x_275; +lean_object* x_393; lean_dec(x_24); lean_dec(x_10); lean_dec(x_9); @@ -56130,15 +56645,15 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_275 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_275, 0, x_231); -lean_ctor_set(x_275, 1, x_232); -return x_275; +x_393 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_393, 0, x_349); +lean_ctor_set(x_393, 1, x_350); +return x_393; } } else { -lean_object* x_276; +lean_object* x_394; lean_dec(x_24); lean_dec(x_10); lean_dec(x_9); @@ -56149,10 +56664,10 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_276 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_276, 0, x_231); -lean_ctor_set(x_276, 1, x_232); -return x_276; +x_394 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_394, 0, x_349); +lean_ctor_set(x_394, 1, x_350); +return x_394; } } } @@ -56208,7 +56723,7 @@ return x_21; } } } -block_102: +block_103: { uint8_t x_31; x_31 = l_Lean_Exception_isInterrupt(x_29); @@ -56218,6 +56733,8 @@ uint8_t x_32; x_32 = l_Lean_Exception_isRuntime(x_29); if (x_32 == 0) { +if (lean_obj_tag(x_29) == 0) +{ uint8_t x_33; lean_object* x_34; lean_dec(x_26); x_33 = 0; @@ -56647,21 +57164,30 @@ lean_ctor_set(x_101, 1, x_30); return x_101; } } -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_102; +lean_dec(x_24); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_10; +lean_dec(x_1); +if (lean_is_scalar(x_26)) { + x_102 = lean_alloc_ctor(1, 2, 0); +} else { + x_102 = x_26; + lean_ctor_set_tag(x_102, 1); +} +lean_ctor_set(x_102, 0, x_29); +lean_ctor_set(x_102, 1, x_30); +return x_102; +} +} } } LEAN_EXPORT lean_object* l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -56710,7 +57236,7 @@ x_11 = lean_ctor_get(x_10, 1); lean_inc(x_11); lean_dec(x_10); x_12 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName___closed__2; -x_13 = l_Lean_throwError___at_Lean_Elab_Term_mkAuxName___spec__1(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_11); +x_13 = l_Lean_throwError___at_Lean_Elab_Term_mkCoe___spec__1(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_11); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -58536,129 +59062,82 @@ lean_inc(x_5); x_232 = l___private_Lean_Elab_App_0__Lean_Elab_Term_resolveDotName(x_131, x_5, x_10, x_11, x_12, x_13, x_14, x_15, x_231); if (lean_obj_tag(x_232) == 0) { -lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; x_233 = lean_ctor_get(x_232, 0); lean_inc(x_233); x_234 = lean_ctor_get(x_232, 1); lean_inc(x_234); lean_dec(x_232); x_235 = lean_box(0); -lean_inc(x_14); -lean_inc(x_10); -x_236 = l_Lean_Elab_Term_mkConst(x_233, x_235, x_10, x_11, x_12, x_13, x_14, x_15, x_234); -if (lean_obj_tag(x_236) == 0) -{ -lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -x_237 = lean_ctor_get(x_236, 0); -lean_inc(x_237); -x_238 = lean_ctor_get(x_236, 1); -lean_inc(x_238); -lean_dec(x_236); -x_239 = lean_box(0); -x_240 = lean_box(x_6); -x_241 = lean_box(x_7); -x_242 = lean_box(x_8); -x_243 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__2___boxed), 17, 10); -lean_closure_set(x_243, 0, x_1); -lean_closure_set(x_243, 1, x_237); -lean_closure_set(x_243, 2, x_5); -lean_closure_set(x_243, 3, x_239); -lean_closure_set(x_243, 4, x_3); -lean_closure_set(x_243, 5, x_4); -lean_closure_set(x_243, 6, x_240); -lean_closure_set(x_243, 7, x_241); -lean_closure_set(x_243, 8, x_2); -lean_closure_set(x_243, 9, x_242); -x_244 = l_Lean_Elab_Term_observing___rarg(x_243, x_10, x_11, x_12, x_13, x_14, x_15, x_238); -if (lean_obj_tag(x_244) == 0) -{ -uint8_t x_245; -x_245 = !lean_is_exclusive(x_244); -if (x_245 == 0) -{ -lean_object* x_246; lean_object* x_247; -x_246 = lean_ctor_get(x_244, 0); -x_247 = lean_array_push(x_9, x_246); -lean_ctor_set(x_244, 0, x_247); -return x_244; -} -else -{ -lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; -x_248 = lean_ctor_get(x_244, 0); -x_249 = lean_ctor_get(x_244, 1); -lean_inc(x_249); -lean_inc(x_248); -lean_dec(x_244); -x_250 = lean_array_push(x_9, x_248); -x_251 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_251, 0, x_250); -lean_ctor_set(x_251, 1, x_249); -return x_251; -} -} -else -{ -uint8_t x_252; -lean_dec(x_9); -x_252 = !lean_is_exclusive(x_244); -if (x_252 == 0) -{ -return x_244; +x_236 = lean_box(x_6); +x_237 = lean_box(x_7); +x_238 = lean_box(x_8); +x_239 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__2___boxed), 17, 10); +lean_closure_set(x_239, 0, x_1); +lean_closure_set(x_239, 1, x_233); +lean_closure_set(x_239, 2, x_5); +lean_closure_set(x_239, 3, x_235); +lean_closure_set(x_239, 4, x_3); +lean_closure_set(x_239, 5, x_4); +lean_closure_set(x_239, 6, x_236); +lean_closure_set(x_239, 7, x_237); +lean_closure_set(x_239, 8, x_2); +lean_closure_set(x_239, 9, x_238); +x_240 = l_Lean_Elab_Term_observing___rarg(x_239, x_10, x_11, x_12, x_13, x_14, x_15, x_234); +if (lean_obj_tag(x_240) == 0) +{ +uint8_t x_241; +x_241 = !lean_is_exclusive(x_240); +if (x_241 == 0) +{ +lean_object* x_242; lean_object* x_243; +x_242 = lean_ctor_get(x_240, 0); +x_243 = lean_array_push(x_9, x_242); +lean_ctor_set(x_240, 0, x_243); +return x_240; } else { -lean_object* x_253; lean_object* x_254; lean_object* x_255; -x_253 = lean_ctor_get(x_244, 0); -x_254 = lean_ctor_get(x_244, 1); -lean_inc(x_254); -lean_inc(x_253); -lean_dec(x_244); -x_255 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_255, 0, x_253); -lean_ctor_set(x_255, 1, x_254); -return x_255; -} +lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; +x_244 = lean_ctor_get(x_240, 0); +x_245 = lean_ctor_get(x_240, 1); +lean_inc(x_245); +lean_inc(x_244); +lean_dec(x_240); +x_246 = lean_array_push(x_9, x_244); +x_247 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_247, 0, x_246); +lean_ctor_set(x_247, 1, x_245); +return x_247; } } else { -uint8_t x_256; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_248; lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_256 = !lean_is_exclusive(x_236); -if (x_256 == 0) +x_248 = !lean_is_exclusive(x_240); +if (x_248 == 0) { -return x_236; +return x_240; } else { -lean_object* x_257; lean_object* x_258; lean_object* x_259; -x_257 = lean_ctor_get(x_236, 0); -x_258 = lean_ctor_get(x_236, 1); -lean_inc(x_258); -lean_inc(x_257); -lean_dec(x_236); -x_259 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_259, 0, x_257); -lean_ctor_set(x_259, 1, x_258); -return x_259; +lean_object* x_249; lean_object* x_250; lean_object* x_251; +x_249 = lean_ctor_get(x_240, 0); +x_250 = lean_ctor_get(x_240, 1); +lean_inc(x_250); +lean_inc(x_249); +lean_dec(x_240); +x_251 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_251, 0, x_249); +lean_ctor_set(x_251, 1, x_250); +return x_251; } } } else { -uint8_t x_260; +uint8_t x_252; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -58671,23 +59150,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_260 = !lean_is_exclusive(x_232); -if (x_260 == 0) +x_252 = !lean_is_exclusive(x_232); +if (x_252 == 0) { return x_232; } else { -lean_object* x_261; lean_object* x_262; lean_object* x_263; -x_261 = lean_ctor_get(x_232, 0); -x_262 = lean_ctor_get(x_232, 1); -lean_inc(x_262); -lean_inc(x_261); +lean_object* x_253; lean_object* x_254; lean_object* x_255; +x_253 = lean_ctor_get(x_232, 0); +x_254 = lean_ctor_get(x_232, 1); +lean_inc(x_254); +lean_inc(x_253); lean_dec(x_232); -x_263 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_263, 0, x_261); -lean_ctor_set(x_263, 1, x_262); -return x_263; +x_255 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_255, 0, x_253); +lean_ctor_set(x_255, 1, x_254); +return x_255; } } } @@ -58695,269 +59174,269 @@ return x_263; } else { -lean_object* x_264; lean_object* x_265; +lean_object* x_256; lean_object* x_257; lean_dec(x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_264 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__18; -x_265 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_264, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_256 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__18; +x_257 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_256, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -return x_265; +return x_257; } } else { -lean_object* x_266; lean_object* x_267; uint8_t x_268; -x_266 = lean_unsigned_to_nat(0u); -x_267 = l_Lean_Syntax_getArg(x_1, x_266); -lean_inc(x_267); -x_268 = l_Lean_Syntax_isOfKind(x_267, x_28); -if (x_268 == 0) +lean_object* x_258; lean_object* x_259; uint8_t x_260; +x_258 = lean_unsigned_to_nat(0u); +x_259 = l_Lean_Syntax_getArg(x_1, x_258); +lean_inc(x_259); +x_260 = l_Lean_Syntax_isOfKind(x_259, x_28); +if (x_260 == 0) { -uint8_t x_269; uint8_t x_270; -lean_dec(x_267); -x_269 = l_List_isEmpty___rarg(x_2); +uint8_t x_261; uint8_t x_262; +lean_dec(x_259); +x_261 = l_List_isEmpty___rarg(x_2); if (x_8 == 0) { -uint8_t x_361; -x_361 = 1; -x_270 = x_361; -goto block_360; +uint8_t x_353; +x_353 = 1; +x_262 = x_353; +goto block_352; +} +else +{ +uint8_t x_354; +x_354 = 0; +x_262 = x_354; +goto block_352; +} +block_352: +{ +if (x_261 == 0) +{ +lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; +x_263 = lean_box(0); +x_264 = lean_box(x_262); +x_265 = lean_box(x_6); +x_266 = lean_box(x_7); +x_267 = lean_box(x_8); +x_268 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_268, 0, x_1); +lean_closure_set(x_268, 1, x_263); +lean_closure_set(x_268, 2, x_264); +lean_closure_set(x_268, 3, x_3); +lean_closure_set(x_268, 4, x_4); +lean_closure_set(x_268, 5, x_5); +lean_closure_set(x_268, 6, x_265); +lean_closure_set(x_268, 7, x_266); +lean_closure_set(x_268, 8, x_2); +lean_closure_set(x_268, 9, x_267); +x_269 = l_Lean_Elab_Term_observing___rarg(x_268, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_269) == 0) +{ +uint8_t x_270; +x_270 = !lean_is_exclusive(x_269); +if (x_270 == 0) +{ +lean_object* x_271; lean_object* x_272; +x_271 = lean_ctor_get(x_269, 0); +x_272 = lean_array_push(x_9, x_271); +lean_ctor_set(x_269, 0, x_272); +return x_269; } else { -uint8_t x_362; -x_362 = 0; -x_270 = x_362; -goto block_360; -} -block_360: -{ -if (x_269 == 0) -{ -lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -x_271 = lean_box(0); -x_272 = lean_box(x_270); -x_273 = lean_box(x_6); -x_274 = lean_box(x_7); -x_275 = lean_box(x_8); -x_276 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_276, 0, x_1); -lean_closure_set(x_276, 1, x_271); -lean_closure_set(x_276, 2, x_272); -lean_closure_set(x_276, 3, x_3); -lean_closure_set(x_276, 4, x_4); -lean_closure_set(x_276, 5, x_5); -lean_closure_set(x_276, 6, x_273); -lean_closure_set(x_276, 7, x_274); -lean_closure_set(x_276, 8, x_2); -lean_closure_set(x_276, 9, x_275); -x_277 = l_Lean_Elab_Term_observing___rarg(x_276, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_277) == 0) -{ -uint8_t x_278; -x_278 = !lean_is_exclusive(x_277); -if (x_278 == 0) -{ -lean_object* x_279; lean_object* x_280; -x_279 = lean_ctor_get(x_277, 0); -x_280 = lean_array_push(x_9, x_279); -lean_ctor_set(x_277, 0, x_280); -return x_277; -} -else -{ -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; -x_281 = lean_ctor_get(x_277, 0); -x_282 = lean_ctor_get(x_277, 1); -lean_inc(x_282); -lean_inc(x_281); -lean_dec(x_277); -x_283 = lean_array_push(x_9, x_281); -x_284 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_284, 0, x_283); -lean_ctor_set(x_284, 1, x_282); -return x_284; +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_273 = lean_ctor_get(x_269, 0); +x_274 = lean_ctor_get(x_269, 1); +lean_inc(x_274); +lean_inc(x_273); +lean_dec(x_269); +x_275 = lean_array_push(x_9, x_273); +x_276 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_276, 0, x_275); +lean_ctor_set(x_276, 1, x_274); +return x_276; } } else { -uint8_t x_285; +uint8_t x_277; lean_dec(x_9); -x_285 = !lean_is_exclusive(x_277); -if (x_285 == 0) +x_277 = !lean_is_exclusive(x_269); +if (x_277 == 0) { -return x_277; +return x_269; } else { -lean_object* x_286; lean_object* x_287; lean_object* x_288; -x_286 = lean_ctor_get(x_277, 0); -x_287 = lean_ctor_get(x_277, 1); -lean_inc(x_287); -lean_inc(x_286); -lean_dec(x_277); -x_288 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_288, 0, x_286); -lean_ctor_set(x_288, 1, x_287); -return x_288; +lean_object* x_278; lean_object* x_279; lean_object* x_280; +x_278 = lean_ctor_get(x_269, 0); +x_279 = lean_ctor_get(x_269, 1); +lean_inc(x_279); +lean_inc(x_278); +lean_dec(x_269); +x_280 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_280, 0, x_278); +lean_ctor_set(x_280, 1, x_279); +return x_280; } } } else { +uint8_t x_281; +x_281 = l_Array_isEmpty___rarg(x_3); +if (x_281 == 0) +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +x_282 = lean_box(0); +x_283 = lean_box(x_262); +x_284 = lean_box(x_6); +x_285 = lean_box(x_7); +x_286 = lean_box(x_8); +x_287 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_287, 0, x_1); +lean_closure_set(x_287, 1, x_282); +lean_closure_set(x_287, 2, x_283); +lean_closure_set(x_287, 3, x_3); +lean_closure_set(x_287, 4, x_4); +lean_closure_set(x_287, 5, x_5); +lean_closure_set(x_287, 6, x_284); +lean_closure_set(x_287, 7, x_285); +lean_closure_set(x_287, 8, x_2); +lean_closure_set(x_287, 9, x_286); +x_288 = l_Lean_Elab_Term_observing___rarg(x_287, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_288) == 0) +{ uint8_t x_289; -x_289 = l_Array_isEmpty___rarg(x_3); +x_289 = !lean_is_exclusive(x_288); if (x_289 == 0) { -lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; -x_290 = lean_box(0); -x_291 = lean_box(x_270); -x_292 = lean_box(x_6); -x_293 = lean_box(x_7); -x_294 = lean_box(x_8); -x_295 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_295, 0, x_1); -lean_closure_set(x_295, 1, x_290); -lean_closure_set(x_295, 2, x_291); -lean_closure_set(x_295, 3, x_3); -lean_closure_set(x_295, 4, x_4); -lean_closure_set(x_295, 5, x_5); -lean_closure_set(x_295, 6, x_292); -lean_closure_set(x_295, 7, x_293); -lean_closure_set(x_295, 8, x_2); -lean_closure_set(x_295, 9, x_294); -x_296 = l_Lean_Elab_Term_observing___rarg(x_295, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_296) == 0) -{ -uint8_t x_297; -x_297 = !lean_is_exclusive(x_296); -if (x_297 == 0) -{ -lean_object* x_298; lean_object* x_299; -x_298 = lean_ctor_get(x_296, 0); -x_299 = lean_array_push(x_9, x_298); -lean_ctor_set(x_296, 0, x_299); -return x_296; +lean_object* x_290; lean_object* x_291; +x_290 = lean_ctor_get(x_288, 0); +x_291 = lean_array_push(x_9, x_290); +lean_ctor_set(x_288, 0, x_291); +return x_288; } else { -lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; -x_300 = lean_ctor_get(x_296, 0); -x_301 = lean_ctor_get(x_296, 1); -lean_inc(x_301); -lean_inc(x_300); -lean_dec(x_296); -x_302 = lean_array_push(x_9, x_300); -x_303 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_303, 0, x_302); -lean_ctor_set(x_303, 1, x_301); -return x_303; +lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; +x_292 = lean_ctor_get(x_288, 0); +x_293 = lean_ctor_get(x_288, 1); +lean_inc(x_293); +lean_inc(x_292); +lean_dec(x_288); +x_294 = lean_array_push(x_9, x_292); +x_295 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_295, 0, x_294); +lean_ctor_set(x_295, 1, x_293); +return x_295; } } else { -uint8_t x_304; +uint8_t x_296; lean_dec(x_9); -x_304 = !lean_is_exclusive(x_296); -if (x_304 == 0) +x_296 = !lean_is_exclusive(x_288); +if (x_296 == 0) { -return x_296; +return x_288; } else { -lean_object* x_305; lean_object* x_306; lean_object* x_307; -x_305 = lean_ctor_get(x_296, 0); -x_306 = lean_ctor_get(x_296, 1); -lean_inc(x_306); -lean_inc(x_305); -lean_dec(x_296); -x_307 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_307, 0, x_305); -lean_ctor_set(x_307, 1, x_306); -return x_307; +lean_object* x_297; lean_object* x_298; lean_object* x_299; +x_297 = lean_ctor_get(x_288, 0); +x_298 = lean_ctor_get(x_288, 1); +lean_inc(x_298); +lean_inc(x_297); +lean_dec(x_288); +x_299 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_299, 0, x_297); +lean_ctor_set(x_299, 1, x_298); +return x_299; } } } else { +uint8_t x_300; +x_300 = l_Array_isEmpty___rarg(x_4); +if (x_300 == 0) +{ +lean_object* x_301; lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; +x_301 = lean_box(0); +x_302 = lean_box(x_262); +x_303 = lean_box(x_6); +x_304 = lean_box(x_7); +x_305 = lean_box(x_8); +x_306 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_306, 0, x_1); +lean_closure_set(x_306, 1, x_301); +lean_closure_set(x_306, 2, x_302); +lean_closure_set(x_306, 3, x_3); +lean_closure_set(x_306, 4, x_4); +lean_closure_set(x_306, 5, x_5); +lean_closure_set(x_306, 6, x_303); +lean_closure_set(x_306, 7, x_304); +lean_closure_set(x_306, 8, x_2); +lean_closure_set(x_306, 9, x_305); +x_307 = l_Lean_Elab_Term_observing___rarg(x_306, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_307) == 0) +{ uint8_t x_308; -x_308 = l_Array_isEmpty___rarg(x_4); +x_308 = !lean_is_exclusive(x_307); if (x_308 == 0) { -lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; -x_309 = lean_box(0); -x_310 = lean_box(x_270); -x_311 = lean_box(x_6); -x_312 = lean_box(x_7); -x_313 = lean_box(x_8); -x_314 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_314, 0, x_1); -lean_closure_set(x_314, 1, x_309); -lean_closure_set(x_314, 2, x_310); -lean_closure_set(x_314, 3, x_3); -lean_closure_set(x_314, 4, x_4); -lean_closure_set(x_314, 5, x_5); -lean_closure_set(x_314, 6, x_311); -lean_closure_set(x_314, 7, x_312); -lean_closure_set(x_314, 8, x_2); -lean_closure_set(x_314, 9, x_313); -x_315 = l_Lean_Elab_Term_observing___rarg(x_314, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_315) == 0) -{ -uint8_t x_316; -x_316 = !lean_is_exclusive(x_315); -if (x_316 == 0) -{ -lean_object* x_317; lean_object* x_318; -x_317 = lean_ctor_get(x_315, 0); -x_318 = lean_array_push(x_9, x_317); -lean_ctor_set(x_315, 0, x_318); -return x_315; -} -else -{ -lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; -x_319 = lean_ctor_get(x_315, 0); -x_320 = lean_ctor_get(x_315, 1); -lean_inc(x_320); -lean_inc(x_319); -lean_dec(x_315); -x_321 = lean_array_push(x_9, x_319); -x_322 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_322, 0, x_321); -lean_ctor_set(x_322, 1, x_320); -return x_322; +lean_object* x_309; lean_object* x_310; +x_309 = lean_ctor_get(x_307, 0); +x_310 = lean_array_push(x_9, x_309); +lean_ctor_set(x_307, 0, x_310); +return x_307; +} +else +{ +lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_311 = lean_ctor_get(x_307, 0); +x_312 = lean_ctor_get(x_307, 1); +lean_inc(x_312); +lean_inc(x_311); +lean_dec(x_307); +x_313 = lean_array_push(x_9, x_311); +x_314 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_314, 0, x_313); +lean_ctor_set(x_314, 1, x_312); +return x_314; } } else { -uint8_t x_323; +uint8_t x_315; lean_dec(x_9); -x_323 = !lean_is_exclusive(x_315); -if (x_323 == 0) +x_315 = !lean_is_exclusive(x_307); +if (x_315 == 0) { -return x_315; +return x_307; } else { -lean_object* x_324; lean_object* x_325; lean_object* x_326; -x_324 = lean_ctor_get(x_315, 0); -x_325 = lean_ctor_get(x_315, 1); -lean_inc(x_325); -lean_inc(x_324); -lean_dec(x_315); -x_326 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_326, 0, x_324); -lean_ctor_set(x_326, 1, x_325); -return x_326; +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_307, 0); +x_317 = lean_ctor_get(x_307, 1); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_307); +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } @@ -58968,129 +59447,129 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; -x_327 = 1; -x_328 = lean_box(x_327); -x_329 = lean_box(x_327); -x_330 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_330, 0, x_1); -lean_closure_set(x_330, 1, x_5); -lean_closure_set(x_330, 2, x_328); -lean_closure_set(x_330, 3, x_329); -x_331 = l_Lean_Elab_Term_observing___rarg(x_330, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_331) == 0) +uint8_t x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; +x_319 = 1; +x_320 = lean_box(x_319); +x_321 = lean_box(x_319); +x_322 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_322, 0, x_1); +lean_closure_set(x_322, 1, x_5); +lean_closure_set(x_322, 2, x_320); +lean_closure_set(x_322, 3, x_321); +x_323 = l_Lean_Elab_Term_observing___rarg(x_322, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_323) == 0) { -uint8_t x_332; -x_332 = !lean_is_exclusive(x_331); -if (x_332 == 0) +uint8_t x_324; +x_324 = !lean_is_exclusive(x_323); +if (x_324 == 0) { -lean_object* x_333; lean_object* x_334; -x_333 = lean_ctor_get(x_331, 0); -x_334 = lean_array_push(x_9, x_333); -lean_ctor_set(x_331, 0, x_334); -return x_331; +lean_object* x_325; lean_object* x_326; +x_325 = lean_ctor_get(x_323, 0); +x_326 = lean_array_push(x_9, x_325); +lean_ctor_set(x_323, 0, x_326); +return x_323; } else { -lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; -x_335 = lean_ctor_get(x_331, 0); -x_336 = lean_ctor_get(x_331, 1); -lean_inc(x_336); -lean_inc(x_335); -lean_dec(x_331); -x_337 = lean_array_push(x_9, x_335); -x_338 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_338, 0, x_337); -lean_ctor_set(x_338, 1, x_336); -return x_338; +lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; +x_327 = lean_ctor_get(x_323, 0); +x_328 = lean_ctor_get(x_323, 1); +lean_inc(x_328); +lean_inc(x_327); +lean_dec(x_323); +x_329 = lean_array_push(x_9, x_327); +x_330 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_330, 0, x_329); +lean_ctor_set(x_330, 1, x_328); +return x_330; } } else { -uint8_t x_339; +uint8_t x_331; lean_dec(x_9); -x_339 = !lean_is_exclusive(x_331); -if (x_339 == 0) +x_331 = !lean_is_exclusive(x_323); +if (x_331 == 0) { -return x_331; +return x_323; } else { -lean_object* x_340; lean_object* x_341; lean_object* x_342; -x_340 = lean_ctor_get(x_331, 0); -x_341 = lean_ctor_get(x_331, 1); -lean_inc(x_341); -lean_inc(x_340); -lean_dec(x_331); -x_342 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_342, 0, x_340); -lean_ctor_set(x_342, 1, x_341); -return x_342; -} -} -} -else -{ -lean_object* x_343; uint8_t x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; -x_343 = lean_box(0); -x_344 = 1; -x_345 = lean_box(x_270); -x_346 = lean_box(x_344); -x_347 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_347, 0, x_1); -lean_closure_set(x_347, 1, x_5); -lean_closure_set(x_347, 2, x_345); -lean_closure_set(x_347, 3, x_346); -lean_closure_set(x_347, 4, x_343); -x_348 = l_Lean_Elab_Term_observing___rarg(x_347, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_348) == 0) -{ -uint8_t x_349; -x_349 = !lean_is_exclusive(x_348); -if (x_349 == 0) -{ -lean_object* x_350; lean_object* x_351; -x_350 = lean_ctor_get(x_348, 0); -x_351 = lean_array_push(x_9, x_350); -lean_ctor_set(x_348, 0, x_351); -return x_348; +lean_object* x_332; lean_object* x_333; lean_object* x_334; +x_332 = lean_ctor_get(x_323, 0); +x_333 = lean_ctor_get(x_323, 1); +lean_inc(x_333); +lean_inc(x_332); +lean_dec(x_323); +x_334 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_334, 0, x_332); +lean_ctor_set(x_334, 1, x_333); +return x_334; +} +} } else { -lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; -x_352 = lean_ctor_get(x_348, 0); -x_353 = lean_ctor_get(x_348, 1); -lean_inc(x_353); -lean_inc(x_352); -lean_dec(x_348); -x_354 = lean_array_push(x_9, x_352); -x_355 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_355, 0, x_354); -lean_ctor_set(x_355, 1, x_353); -return x_355; +lean_object* x_335; uint8_t x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; +x_335 = lean_box(0); +x_336 = 1; +x_337 = lean_box(x_262); +x_338 = lean_box(x_336); +x_339 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_339, 0, x_1); +lean_closure_set(x_339, 1, x_5); +lean_closure_set(x_339, 2, x_337); +lean_closure_set(x_339, 3, x_338); +lean_closure_set(x_339, 4, x_335); +x_340 = l_Lean_Elab_Term_observing___rarg(x_339, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_340) == 0) +{ +uint8_t x_341; +x_341 = !lean_is_exclusive(x_340); +if (x_341 == 0) +{ +lean_object* x_342; lean_object* x_343; +x_342 = lean_ctor_get(x_340, 0); +x_343 = lean_array_push(x_9, x_342); +lean_ctor_set(x_340, 0, x_343); +return x_340; +} +else +{ +lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; +x_344 = lean_ctor_get(x_340, 0); +x_345 = lean_ctor_get(x_340, 1); +lean_inc(x_345); +lean_inc(x_344); +lean_dec(x_340); +x_346 = lean_array_push(x_9, x_344); +x_347 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_347, 0, x_346); +lean_ctor_set(x_347, 1, x_345); +return x_347; } } else { -uint8_t x_356; +uint8_t x_348; lean_dec(x_9); -x_356 = !lean_is_exclusive(x_348); -if (x_356 == 0) +x_348 = !lean_is_exclusive(x_340); +if (x_348 == 0) { -return x_348; +return x_340; } else { -lean_object* x_357; lean_object* x_358; lean_object* x_359; -x_357 = lean_ctor_get(x_348, 0); -x_358 = lean_ctor_get(x_348, 1); -lean_inc(x_358); -lean_inc(x_357); -lean_dec(x_348); -x_359 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_359, 0, x_357); -lean_ctor_set(x_359, 1, x_358); -return x_359; +lean_object* x_349; lean_object* x_350; lean_object* x_351; +x_349 = lean_ctor_get(x_340, 0); +x_350 = lean_ctor_get(x_340, 1); +lean_inc(x_350); +lean_inc(x_349); +lean_dec(x_340); +x_351 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_351, 0, x_349); +lean_ctor_set(x_351, 1, x_350); +return x_351; } } } @@ -59101,31 +59580,31 @@ return x_359; } else { -lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; -x_363 = lean_unsigned_to_nat(2u); -x_364 = l_Lean_Syntax_getArg(x_1, x_363); +lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; +x_355 = lean_unsigned_to_nat(2u); +x_356 = l_Lean_Syntax_getArg(x_1, x_355); lean_dec(x_1); -x_365 = l_Lean_Syntax_getArgs(x_364); -lean_dec(x_364); -x_366 = l_Lean_Syntax_TSepArray_getElems___rarg(x_365); -lean_dec(x_365); -x_367 = l_Lean_Elab_Term_elabExplicitUnivs(x_366, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_366); -if (lean_obj_tag(x_367) == 0) -{ -lean_object* x_368; lean_object* x_369; lean_object* x_370; -x_368 = lean_ctor_get(x_367, 0); -lean_inc(x_368); -x_369 = lean_ctor_get(x_367, 1); -lean_inc(x_369); -lean_dec(x_367); -x_370 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId(x_267, x_368, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_369); -return x_370; -} -else -{ -uint8_t x_371; -lean_dec(x_267); +x_357 = l_Lean_Syntax_getArgs(x_356); +lean_dec(x_356); +x_358 = l_Lean_Syntax_TSepArray_getElems___rarg(x_357); +lean_dec(x_357); +x_359 = l_Lean_Elab_Term_elabExplicitUnivs(x_358, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_358); +if (lean_obj_tag(x_359) == 0) +{ +lean_object* x_360; lean_object* x_361; lean_object* x_362; +x_360 = lean_ctor_get(x_359, 0); +lean_inc(x_360); +x_361 = lean_ctor_get(x_359, 1); +lean_inc(x_361); +lean_dec(x_359); +x_362 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId(x_259, x_360, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_361); +return x_362; +} +else +{ +uint8_t x_363; +lean_dec(x_259); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -59137,23 +59616,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_371 = !lean_is_exclusive(x_367); -if (x_371 == 0) +x_363 = !lean_is_exclusive(x_359); +if (x_363 == 0) { -return x_367; +return x_359; } else { -lean_object* x_372; lean_object* x_373; lean_object* x_374; -x_372 = lean_ctor_get(x_367, 0); -x_373 = lean_ctor_get(x_367, 1); -lean_inc(x_373); -lean_inc(x_372); -lean_dec(x_367); -x_374 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_374, 0, x_372); -lean_ctor_set(x_374, 1, x_373); -return x_374; +lean_object* x_364; lean_object* x_365; lean_object* x_366; +x_364 = lean_ctor_get(x_359, 0); +x_365 = lean_ctor_get(x_359, 1); +lean_inc(x_365); +lean_inc(x_364); +lean_dec(x_359); +x_366 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_366, 0, x_364); +lean_ctor_set(x_366, 1, x_365); +return x_366; } } } @@ -59161,257 +59640,257 @@ return x_374; } else { -lean_object* x_375; lean_object* x_376; -x_375 = lean_box(0); -x_376 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId(x_1, x_375, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -return x_376; +lean_object* x_367; lean_object* x_368; +x_367 = lean_box(0); +x_368 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFnId(x_1, x_367, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_368; } } else { -lean_object* x_377; lean_object* x_378; lean_object* x_379; uint8_t x_380; -x_377 = lean_unsigned_to_nat(0u); -x_378 = l_Lean_Syntax_getArg(x_1, x_377); -x_379 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; -x_380 = l_Lean_Syntax_isOfKind(x_378, x_379); -if (x_380 == 0) +lean_object* x_369; lean_object* x_370; lean_object* x_371; uint8_t x_372; +x_369 = lean_unsigned_to_nat(0u); +x_370 = l_Lean_Syntax_getArg(x_1, x_369); +x_371 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; +x_372 = l_Lean_Syntax_isOfKind(x_370, x_371); +if (x_372 == 0) { -uint8_t x_381; uint8_t x_382; -x_381 = l_List_isEmpty___rarg(x_2); +uint8_t x_373; uint8_t x_374; +x_373 = l_List_isEmpty___rarg(x_2); if (x_8 == 0) { -uint8_t x_473; -x_473 = 1; -x_382 = x_473; -goto block_472; +uint8_t x_465; +x_465 = 1; +x_374 = x_465; +goto block_464; } else { -uint8_t x_474; -x_474 = 0; -x_382 = x_474; -goto block_472; +uint8_t x_466; +x_466 = 0; +x_374 = x_466; +goto block_464; } -block_472: -{ -if (x_381 == 0) +block_464: { -lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; lean_object* x_389; -x_383 = lean_box(0); -x_384 = lean_box(x_382); -x_385 = lean_box(x_6); -x_386 = lean_box(x_7); -x_387 = lean_box(x_8); -x_388 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_388, 0, x_1); -lean_closure_set(x_388, 1, x_383); -lean_closure_set(x_388, 2, x_384); -lean_closure_set(x_388, 3, x_3); -lean_closure_set(x_388, 4, x_4); -lean_closure_set(x_388, 5, x_5); -lean_closure_set(x_388, 6, x_385); -lean_closure_set(x_388, 7, x_386); -lean_closure_set(x_388, 8, x_2); -lean_closure_set(x_388, 9, x_387); -x_389 = l_Lean_Elab_Term_observing___rarg(x_388, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_389) == 0) +if (x_373 == 0) { -uint8_t x_390; -x_390 = !lean_is_exclusive(x_389); -if (x_390 == 0) +lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; +x_375 = lean_box(0); +x_376 = lean_box(x_374); +x_377 = lean_box(x_6); +x_378 = lean_box(x_7); +x_379 = lean_box(x_8); +x_380 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_380, 0, x_1); +lean_closure_set(x_380, 1, x_375); +lean_closure_set(x_380, 2, x_376); +lean_closure_set(x_380, 3, x_3); +lean_closure_set(x_380, 4, x_4); +lean_closure_set(x_380, 5, x_5); +lean_closure_set(x_380, 6, x_377); +lean_closure_set(x_380, 7, x_378); +lean_closure_set(x_380, 8, x_2); +lean_closure_set(x_380, 9, x_379); +x_381 = l_Lean_Elab_Term_observing___rarg(x_380, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_381) == 0) +{ +uint8_t x_382; +x_382 = !lean_is_exclusive(x_381); +if (x_382 == 0) +{ +lean_object* x_383; lean_object* x_384; +x_383 = lean_ctor_get(x_381, 0); +x_384 = lean_array_push(x_9, x_383); +lean_ctor_set(x_381, 0, x_384); +return x_381; +} +else +{ +lean_object* x_385; lean_object* x_386; lean_object* x_387; lean_object* x_388; +x_385 = lean_ctor_get(x_381, 0); +x_386 = lean_ctor_get(x_381, 1); +lean_inc(x_386); +lean_inc(x_385); +lean_dec(x_381); +x_387 = lean_array_push(x_9, x_385); +x_388 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_388, 0, x_387); +lean_ctor_set(x_388, 1, x_386); +return x_388; +} +} +else +{ +uint8_t x_389; +lean_dec(x_9); +x_389 = !lean_is_exclusive(x_381); +if (x_389 == 0) { -lean_object* x_391; lean_object* x_392; -x_391 = lean_ctor_get(x_389, 0); -x_392 = lean_array_push(x_9, x_391); -lean_ctor_set(x_389, 0, x_392); -return x_389; +return x_381; } else { -lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; -x_393 = lean_ctor_get(x_389, 0); -x_394 = lean_ctor_get(x_389, 1); -lean_inc(x_394); -lean_inc(x_393); -lean_dec(x_389); -x_395 = lean_array_push(x_9, x_393); -x_396 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_396, 0, x_395); -lean_ctor_set(x_396, 1, x_394); -return x_396; +lean_object* x_390; lean_object* x_391; lean_object* x_392; +x_390 = lean_ctor_get(x_381, 0); +x_391 = lean_ctor_get(x_381, 1); +lean_inc(x_391); +lean_inc(x_390); +lean_dec(x_381); +x_392 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_392, 0, x_390); +lean_ctor_set(x_392, 1, x_391); +return x_392; +} } } else { -uint8_t x_397; -lean_dec(x_9); -x_397 = !lean_is_exclusive(x_389); -if (x_397 == 0) +uint8_t x_393; +x_393 = l_Array_isEmpty___rarg(x_3); +if (x_393 == 0) { -return x_389; -} -else +lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; +x_394 = lean_box(0); +x_395 = lean_box(x_374); +x_396 = lean_box(x_6); +x_397 = lean_box(x_7); +x_398 = lean_box(x_8); +x_399 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_399, 0, x_1); +lean_closure_set(x_399, 1, x_394); +lean_closure_set(x_399, 2, x_395); +lean_closure_set(x_399, 3, x_3); +lean_closure_set(x_399, 4, x_4); +lean_closure_set(x_399, 5, x_5); +lean_closure_set(x_399, 6, x_396); +lean_closure_set(x_399, 7, x_397); +lean_closure_set(x_399, 8, x_2); +lean_closure_set(x_399, 9, x_398); +x_400 = l_Lean_Elab_Term_observing___rarg(x_399, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_400) == 0) { -lean_object* x_398; lean_object* x_399; lean_object* x_400; -x_398 = lean_ctor_get(x_389, 0); -x_399 = lean_ctor_get(x_389, 1); -lean_inc(x_399); -lean_inc(x_398); -lean_dec(x_389); -x_400 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_400, 0, x_398); -lean_ctor_set(x_400, 1, x_399); +uint8_t x_401; +x_401 = !lean_is_exclusive(x_400); +if (x_401 == 0) +{ +lean_object* x_402; lean_object* x_403; +x_402 = lean_ctor_get(x_400, 0); +x_403 = lean_array_push(x_9, x_402); +lean_ctor_set(x_400, 0, x_403); return x_400; } +else +{ +lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; +x_404 = lean_ctor_get(x_400, 0); +x_405 = lean_ctor_get(x_400, 1); +lean_inc(x_405); +lean_inc(x_404); +lean_dec(x_400); +x_406 = lean_array_push(x_9, x_404); +x_407 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_407, 0, x_406); +lean_ctor_set(x_407, 1, x_405); +return x_407; } } else { -uint8_t x_401; -x_401 = l_Array_isEmpty___rarg(x_3); -if (x_401 == 0) -{ -lean_object* x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; -x_402 = lean_box(0); -x_403 = lean_box(x_382); -x_404 = lean_box(x_6); -x_405 = lean_box(x_7); -x_406 = lean_box(x_8); -x_407 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_407, 0, x_1); -lean_closure_set(x_407, 1, x_402); -lean_closure_set(x_407, 2, x_403); -lean_closure_set(x_407, 3, x_3); -lean_closure_set(x_407, 4, x_4); -lean_closure_set(x_407, 5, x_5); -lean_closure_set(x_407, 6, x_404); -lean_closure_set(x_407, 7, x_405); -lean_closure_set(x_407, 8, x_2); -lean_closure_set(x_407, 9, x_406); -x_408 = l_Lean_Elab_Term_observing___rarg(x_407, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_408) == 0) -{ -uint8_t x_409; -x_409 = !lean_is_exclusive(x_408); -if (x_409 == 0) -{ -lean_object* x_410; lean_object* x_411; -x_410 = lean_ctor_get(x_408, 0); -x_411 = lean_array_push(x_9, x_410); -lean_ctor_set(x_408, 0, x_411); -return x_408; -} -else -{ -lean_object* x_412; lean_object* x_413; lean_object* x_414; lean_object* x_415; -x_412 = lean_ctor_get(x_408, 0); -x_413 = lean_ctor_get(x_408, 1); -lean_inc(x_413); -lean_inc(x_412); -lean_dec(x_408); -x_414 = lean_array_push(x_9, x_412); -x_415 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_415, 0, x_414); -lean_ctor_set(x_415, 1, x_413); -return x_415; -} -} -else -{ -uint8_t x_416; +uint8_t x_408; lean_dec(x_9); -x_416 = !lean_is_exclusive(x_408); -if (x_416 == 0) +x_408 = !lean_is_exclusive(x_400); +if (x_408 == 0) { -return x_408; +return x_400; } else { -lean_object* x_417; lean_object* x_418; lean_object* x_419; -x_417 = lean_ctor_get(x_408, 0); -x_418 = lean_ctor_get(x_408, 1); -lean_inc(x_418); -lean_inc(x_417); -lean_dec(x_408); -x_419 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_419, 0, x_417); -lean_ctor_set(x_419, 1, x_418); -return x_419; +lean_object* x_409; lean_object* x_410; lean_object* x_411; +x_409 = lean_ctor_get(x_400, 0); +x_410 = lean_ctor_get(x_400, 1); +lean_inc(x_410); +lean_inc(x_409); +lean_dec(x_400); +x_411 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_411, 0, x_409); +lean_ctor_set(x_411, 1, x_410); +return x_411; } } } else { +uint8_t x_412; +x_412 = l_Array_isEmpty___rarg(x_4); +if (x_412 == 0) +{ +lean_object* x_413; lean_object* x_414; lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; +x_413 = lean_box(0); +x_414 = lean_box(x_374); +x_415 = lean_box(x_6); +x_416 = lean_box(x_7); +x_417 = lean_box(x_8); +x_418 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_418, 0, x_1); +lean_closure_set(x_418, 1, x_413); +lean_closure_set(x_418, 2, x_414); +lean_closure_set(x_418, 3, x_3); +lean_closure_set(x_418, 4, x_4); +lean_closure_set(x_418, 5, x_5); +lean_closure_set(x_418, 6, x_415); +lean_closure_set(x_418, 7, x_416); +lean_closure_set(x_418, 8, x_2); +lean_closure_set(x_418, 9, x_417); +x_419 = l_Lean_Elab_Term_observing___rarg(x_418, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_419) == 0) +{ uint8_t x_420; -x_420 = l_Array_isEmpty___rarg(x_4); +x_420 = !lean_is_exclusive(x_419); if (x_420 == 0) { -lean_object* x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; lean_object* x_427; -x_421 = lean_box(0); -x_422 = lean_box(x_382); -x_423 = lean_box(x_6); -x_424 = lean_box(x_7); -x_425 = lean_box(x_8); -x_426 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_426, 0, x_1); -lean_closure_set(x_426, 1, x_421); -lean_closure_set(x_426, 2, x_422); -lean_closure_set(x_426, 3, x_3); -lean_closure_set(x_426, 4, x_4); -lean_closure_set(x_426, 5, x_5); -lean_closure_set(x_426, 6, x_423); -lean_closure_set(x_426, 7, x_424); -lean_closure_set(x_426, 8, x_2); -lean_closure_set(x_426, 9, x_425); -x_427 = l_Lean_Elab_Term_observing___rarg(x_426, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_427) == 0) -{ -uint8_t x_428; -x_428 = !lean_is_exclusive(x_427); -if (x_428 == 0) -{ -lean_object* x_429; lean_object* x_430; -x_429 = lean_ctor_get(x_427, 0); -x_430 = lean_array_push(x_9, x_429); -lean_ctor_set(x_427, 0, x_430); -return x_427; -} -else -{ -lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; -x_431 = lean_ctor_get(x_427, 0); -x_432 = lean_ctor_get(x_427, 1); -lean_inc(x_432); -lean_inc(x_431); -lean_dec(x_427); -x_433 = lean_array_push(x_9, x_431); -x_434 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_434, 0, x_433); -lean_ctor_set(x_434, 1, x_432); -return x_434; -} -} -else -{ -uint8_t x_435; +lean_object* x_421; lean_object* x_422; +x_421 = lean_ctor_get(x_419, 0); +x_422 = lean_array_push(x_9, x_421); +lean_ctor_set(x_419, 0, x_422); +return x_419; +} +else +{ +lean_object* x_423; lean_object* x_424; lean_object* x_425; lean_object* x_426; +x_423 = lean_ctor_get(x_419, 0); +x_424 = lean_ctor_get(x_419, 1); +lean_inc(x_424); +lean_inc(x_423); +lean_dec(x_419); +x_425 = lean_array_push(x_9, x_423); +x_426 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_426, 0, x_425); +lean_ctor_set(x_426, 1, x_424); +return x_426; +} +} +else +{ +uint8_t x_427; lean_dec(x_9); -x_435 = !lean_is_exclusive(x_427); -if (x_435 == 0) +x_427 = !lean_is_exclusive(x_419); +if (x_427 == 0) { -return x_427; +return x_419; } else { -lean_object* x_436; lean_object* x_437; lean_object* x_438; -x_436 = lean_ctor_get(x_427, 0); -x_437 = lean_ctor_get(x_427, 1); -lean_inc(x_437); -lean_inc(x_436); -lean_dec(x_427); -x_438 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_438, 0, x_436); -lean_ctor_set(x_438, 1, x_437); -return x_438; +lean_object* x_428; lean_object* x_429; lean_object* x_430; +x_428 = lean_ctor_get(x_419, 0); +x_429 = lean_ctor_get(x_419, 1); +lean_inc(x_429); +lean_inc(x_428); +lean_dec(x_419); +x_430 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_430, 0, x_428); +lean_ctor_set(x_430, 1, x_429); +return x_430; } } } @@ -59422,129 +59901,129 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; lean_object* x_443; -x_439 = 1; -x_440 = lean_box(x_439); -x_441 = lean_box(x_439); -x_442 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_442, 0, x_1); -lean_closure_set(x_442, 1, x_5); -lean_closure_set(x_442, 2, x_440); -lean_closure_set(x_442, 3, x_441); -x_443 = l_Lean_Elab_Term_observing___rarg(x_442, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_443) == 0) +uint8_t x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; lean_object* x_435; +x_431 = 1; +x_432 = lean_box(x_431); +x_433 = lean_box(x_431); +x_434 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_434, 0, x_1); +lean_closure_set(x_434, 1, x_5); +lean_closure_set(x_434, 2, x_432); +lean_closure_set(x_434, 3, x_433); +x_435 = l_Lean_Elab_Term_observing___rarg(x_434, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_435) == 0) { -uint8_t x_444; -x_444 = !lean_is_exclusive(x_443); -if (x_444 == 0) +uint8_t x_436; +x_436 = !lean_is_exclusive(x_435); +if (x_436 == 0) { -lean_object* x_445; lean_object* x_446; -x_445 = lean_ctor_get(x_443, 0); -x_446 = lean_array_push(x_9, x_445); -lean_ctor_set(x_443, 0, x_446); -return x_443; +lean_object* x_437; lean_object* x_438; +x_437 = lean_ctor_get(x_435, 0); +x_438 = lean_array_push(x_9, x_437); +lean_ctor_set(x_435, 0, x_438); +return x_435; } else { -lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; -x_447 = lean_ctor_get(x_443, 0); -x_448 = lean_ctor_get(x_443, 1); -lean_inc(x_448); -lean_inc(x_447); -lean_dec(x_443); -x_449 = lean_array_push(x_9, x_447); -x_450 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_450, 0, x_449); -lean_ctor_set(x_450, 1, x_448); -return x_450; +lean_object* x_439; lean_object* x_440; lean_object* x_441; lean_object* x_442; +x_439 = lean_ctor_get(x_435, 0); +x_440 = lean_ctor_get(x_435, 1); +lean_inc(x_440); +lean_inc(x_439); +lean_dec(x_435); +x_441 = lean_array_push(x_9, x_439); +x_442 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_442, 0, x_441); +lean_ctor_set(x_442, 1, x_440); +return x_442; } } else { -uint8_t x_451; +uint8_t x_443; lean_dec(x_9); -x_451 = !lean_is_exclusive(x_443); -if (x_451 == 0) +x_443 = !lean_is_exclusive(x_435); +if (x_443 == 0) { -return x_443; +return x_435; } else { -lean_object* x_452; lean_object* x_453; lean_object* x_454; -x_452 = lean_ctor_get(x_443, 0); -x_453 = lean_ctor_get(x_443, 1); -lean_inc(x_453); -lean_inc(x_452); -lean_dec(x_443); -x_454 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_454, 0, x_452); -lean_ctor_set(x_454, 1, x_453); -return x_454; +lean_object* x_444; lean_object* x_445; lean_object* x_446; +x_444 = lean_ctor_get(x_435, 0); +x_445 = lean_ctor_get(x_435, 1); +lean_inc(x_445); +lean_inc(x_444); +lean_dec(x_435); +x_446 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_446, 0, x_444); +lean_ctor_set(x_446, 1, x_445); +return x_446; } } } else { -lean_object* x_455; uint8_t x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; -x_455 = lean_box(0); -x_456 = 1; -x_457 = lean_box(x_382); -x_458 = lean_box(x_456); -x_459 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_459, 0, x_1); -lean_closure_set(x_459, 1, x_5); -lean_closure_set(x_459, 2, x_457); -lean_closure_set(x_459, 3, x_458); -lean_closure_set(x_459, 4, x_455); -x_460 = l_Lean_Elab_Term_observing___rarg(x_459, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_460) == 0) +lean_object* x_447; uint8_t x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; +x_447 = lean_box(0); +x_448 = 1; +x_449 = lean_box(x_374); +x_450 = lean_box(x_448); +x_451 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_451, 0, x_1); +lean_closure_set(x_451, 1, x_5); +lean_closure_set(x_451, 2, x_449); +lean_closure_set(x_451, 3, x_450); +lean_closure_set(x_451, 4, x_447); +x_452 = l_Lean_Elab_Term_observing___rarg(x_451, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_452) == 0) { -uint8_t x_461; -x_461 = !lean_is_exclusive(x_460); -if (x_461 == 0) +uint8_t x_453; +x_453 = !lean_is_exclusive(x_452); +if (x_453 == 0) { -lean_object* x_462; lean_object* x_463; -x_462 = lean_ctor_get(x_460, 0); -x_463 = lean_array_push(x_9, x_462); -lean_ctor_set(x_460, 0, x_463); -return x_460; +lean_object* x_454; lean_object* x_455; +x_454 = lean_ctor_get(x_452, 0); +x_455 = lean_array_push(x_9, x_454); +lean_ctor_set(x_452, 0, x_455); +return x_452; } else { -lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; -x_464 = lean_ctor_get(x_460, 0); -x_465 = lean_ctor_get(x_460, 1); -lean_inc(x_465); -lean_inc(x_464); -lean_dec(x_460); -x_466 = lean_array_push(x_9, x_464); -x_467 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_467, 0, x_466); -lean_ctor_set(x_467, 1, x_465); -return x_467; +lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; +x_456 = lean_ctor_get(x_452, 0); +x_457 = lean_ctor_get(x_452, 1); +lean_inc(x_457); +lean_inc(x_456); +lean_dec(x_452); +x_458 = lean_array_push(x_9, x_456); +x_459 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_459, 0, x_458); +lean_ctor_set(x_459, 1, x_457); +return x_459; } } else { -uint8_t x_468; +uint8_t x_460; lean_dec(x_9); -x_468 = !lean_is_exclusive(x_460); -if (x_468 == 0) +x_460 = !lean_is_exclusive(x_452); +if (x_460 == 0) { -return x_460; +return x_452; } else { -lean_object* x_469; lean_object* x_470; lean_object* x_471; -x_469 = lean_ctor_get(x_460, 0); -x_470 = lean_ctor_get(x_460, 1); -lean_inc(x_470); -lean_inc(x_469); -lean_dec(x_460); -x_471 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_471, 0, x_469); -lean_ctor_set(x_471, 1, x_470); -return x_471; +lean_object* x_461; lean_object* x_462; lean_object* x_463; +x_461 = lean_ctor_get(x_452, 0); +x_462 = lean_ctor_get(x_452, 1); +lean_inc(x_462); +lean_inc(x_461); +lean_dec(x_452); +x_463 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_463, 0, x_461); +lean_ctor_set(x_463, 1, x_462); +return x_463; } } } @@ -59555,248 +60034,845 @@ return x_471; } else { -lean_object* x_475; lean_object* x_476; uint8_t x_477; -x_475 = lean_unsigned_to_nat(2u); -x_476 = l_Lean_Syntax_getArg(x_1, x_475); -x_477 = l_Lean_Syntax_matchesNull(x_476, x_377); -if (x_477 == 0) +lean_object* x_467; lean_object* x_468; uint8_t x_469; +x_467 = lean_unsigned_to_nat(2u); +x_468 = l_Lean_Syntax_getArg(x_1, x_467); +x_469 = l_Lean_Syntax_matchesNull(x_468, x_369); +if (x_469 == 0) { -uint8_t x_478; uint8_t x_479; -x_478 = l_List_isEmpty___rarg(x_2); +uint8_t x_470; uint8_t x_471; +x_470 = l_List_isEmpty___rarg(x_2); if (x_8 == 0) { -uint8_t x_570; -x_570 = 1; -x_479 = x_570; -goto block_569; +uint8_t x_562; +x_562 = 1; +x_471 = x_562; +goto block_561; } else { -uint8_t x_571; -x_571 = 0; -x_479 = x_571; -goto block_569; +uint8_t x_563; +x_563 = 0; +x_471 = x_563; +goto block_561; } -block_569: +block_561: { -if (x_478 == 0) +if (x_470 == 0) { -lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; lean_object* x_486; -x_480 = lean_box(0); -x_481 = lean_box(x_479); -x_482 = lean_box(x_6); -x_483 = lean_box(x_7); -x_484 = lean_box(x_8); -x_485 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_485, 0, x_1); -lean_closure_set(x_485, 1, x_480); -lean_closure_set(x_485, 2, x_481); -lean_closure_set(x_485, 3, x_3); -lean_closure_set(x_485, 4, x_4); -lean_closure_set(x_485, 5, x_5); -lean_closure_set(x_485, 6, x_482); -lean_closure_set(x_485, 7, x_483); -lean_closure_set(x_485, 8, x_2); -lean_closure_set(x_485, 9, x_484); -x_486 = l_Lean_Elab_Term_observing___rarg(x_485, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_486) == 0) +lean_object* x_472; lean_object* x_473; lean_object* x_474; lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; +x_472 = lean_box(0); +x_473 = lean_box(x_471); +x_474 = lean_box(x_6); +x_475 = lean_box(x_7); +x_476 = lean_box(x_8); +x_477 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_477, 0, x_1); +lean_closure_set(x_477, 1, x_472); +lean_closure_set(x_477, 2, x_473); +lean_closure_set(x_477, 3, x_3); +lean_closure_set(x_477, 4, x_4); +lean_closure_set(x_477, 5, x_5); +lean_closure_set(x_477, 6, x_474); +lean_closure_set(x_477, 7, x_475); +lean_closure_set(x_477, 8, x_2); +lean_closure_set(x_477, 9, x_476); +x_478 = l_Lean_Elab_Term_observing___rarg(x_477, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_478) == 0) { -uint8_t x_487; -x_487 = !lean_is_exclusive(x_486); -if (x_487 == 0) +uint8_t x_479; +x_479 = !lean_is_exclusive(x_478); +if (x_479 == 0) { -lean_object* x_488; lean_object* x_489; -x_488 = lean_ctor_get(x_486, 0); -x_489 = lean_array_push(x_9, x_488); -lean_ctor_set(x_486, 0, x_489); -return x_486; +lean_object* x_480; lean_object* x_481; +x_480 = lean_ctor_get(x_478, 0); +x_481 = lean_array_push(x_9, x_480); +lean_ctor_set(x_478, 0, x_481); +return x_478; } else { -lean_object* x_490; lean_object* x_491; lean_object* x_492; lean_object* x_493; -x_490 = lean_ctor_get(x_486, 0); -x_491 = lean_ctor_get(x_486, 1); -lean_inc(x_491); -lean_inc(x_490); -lean_dec(x_486); -x_492 = lean_array_push(x_9, x_490); -x_493 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_493, 0, x_492); -lean_ctor_set(x_493, 1, x_491); -return x_493; +lean_object* x_482; lean_object* x_483; lean_object* x_484; lean_object* x_485; +x_482 = lean_ctor_get(x_478, 0); +x_483 = lean_ctor_get(x_478, 1); +lean_inc(x_483); +lean_inc(x_482); +lean_dec(x_478); +x_484 = lean_array_push(x_9, x_482); +x_485 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_485, 0, x_484); +lean_ctor_set(x_485, 1, x_483); +return x_485; } } else { -uint8_t x_494; +uint8_t x_486; lean_dec(x_9); -x_494 = !lean_is_exclusive(x_486); -if (x_494 == 0) +x_486 = !lean_is_exclusive(x_478); +if (x_486 == 0) { -return x_486; +return x_478; } else { -lean_object* x_495; lean_object* x_496; lean_object* x_497; -x_495 = lean_ctor_get(x_486, 0); -x_496 = lean_ctor_get(x_486, 1); -lean_inc(x_496); -lean_inc(x_495); -lean_dec(x_486); -x_497 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_497, 0, x_495); -lean_ctor_set(x_497, 1, x_496); -return x_497; +lean_object* x_487; lean_object* x_488; lean_object* x_489; +x_487 = lean_ctor_get(x_478, 0); +x_488 = lean_ctor_get(x_478, 1); +lean_inc(x_488); +lean_inc(x_487); +lean_dec(x_478); +x_489 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_489, 0, x_487); +lean_ctor_set(x_489, 1, x_488); +return x_489; } } } else { +uint8_t x_490; +x_490 = l_Array_isEmpty___rarg(x_3); +if (x_490 == 0) +{ +lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; lean_object* x_497; +x_491 = lean_box(0); +x_492 = lean_box(x_471); +x_493 = lean_box(x_6); +x_494 = lean_box(x_7); +x_495 = lean_box(x_8); +x_496 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_496, 0, x_1); +lean_closure_set(x_496, 1, x_491); +lean_closure_set(x_496, 2, x_492); +lean_closure_set(x_496, 3, x_3); +lean_closure_set(x_496, 4, x_4); +lean_closure_set(x_496, 5, x_5); +lean_closure_set(x_496, 6, x_493); +lean_closure_set(x_496, 7, x_494); +lean_closure_set(x_496, 8, x_2); +lean_closure_set(x_496, 9, x_495); +x_497 = l_Lean_Elab_Term_observing___rarg(x_496, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_497) == 0) +{ uint8_t x_498; -x_498 = l_Array_isEmpty___rarg(x_3); +x_498 = !lean_is_exclusive(x_497); if (x_498 == 0) { -lean_object* x_499; lean_object* x_500; lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; -x_499 = lean_box(0); -x_500 = lean_box(x_479); -x_501 = lean_box(x_6); -x_502 = lean_box(x_7); -x_503 = lean_box(x_8); -x_504 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_504, 0, x_1); -lean_closure_set(x_504, 1, x_499); -lean_closure_set(x_504, 2, x_500); -lean_closure_set(x_504, 3, x_3); -lean_closure_set(x_504, 4, x_4); -lean_closure_set(x_504, 5, x_5); -lean_closure_set(x_504, 6, x_501); -lean_closure_set(x_504, 7, x_502); -lean_closure_set(x_504, 8, x_2); -lean_closure_set(x_504, 9, x_503); -x_505 = l_Lean_Elab_Term_observing___rarg(x_504, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_505) == 0) -{ -uint8_t x_506; -x_506 = !lean_is_exclusive(x_505); -if (x_506 == 0) -{ -lean_object* x_507; lean_object* x_508; -x_507 = lean_ctor_get(x_505, 0); -x_508 = lean_array_push(x_9, x_507); -lean_ctor_set(x_505, 0, x_508); -return x_505; -} -else -{ -lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; -x_509 = lean_ctor_get(x_505, 0); -x_510 = lean_ctor_get(x_505, 1); -lean_inc(x_510); -lean_inc(x_509); -lean_dec(x_505); -x_511 = lean_array_push(x_9, x_509); -x_512 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_512, 0, x_511); -lean_ctor_set(x_512, 1, x_510); -return x_512; -} -} -else -{ -uint8_t x_513; +lean_object* x_499; lean_object* x_500; +x_499 = lean_ctor_get(x_497, 0); +x_500 = lean_array_push(x_9, x_499); +lean_ctor_set(x_497, 0, x_500); +return x_497; +} +else +{ +lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; +x_501 = lean_ctor_get(x_497, 0); +x_502 = lean_ctor_get(x_497, 1); +lean_inc(x_502); +lean_inc(x_501); +lean_dec(x_497); +x_503 = lean_array_push(x_9, x_501); +x_504 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_504, 0, x_503); +lean_ctor_set(x_504, 1, x_502); +return x_504; +} +} +else +{ +uint8_t x_505; lean_dec(x_9); -x_513 = !lean_is_exclusive(x_505); -if (x_513 == 0) +x_505 = !lean_is_exclusive(x_497); +if (x_505 == 0) { -return x_505; +return x_497; } else { -lean_object* x_514; lean_object* x_515; lean_object* x_516; -x_514 = lean_ctor_get(x_505, 0); -x_515 = lean_ctor_get(x_505, 1); -lean_inc(x_515); -lean_inc(x_514); -lean_dec(x_505); -x_516 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_516, 0, x_514); -lean_ctor_set(x_516, 1, x_515); -return x_516; +lean_object* x_506; lean_object* x_507; lean_object* x_508; +x_506 = lean_ctor_get(x_497, 0); +x_507 = lean_ctor_get(x_497, 1); +lean_inc(x_507); +lean_inc(x_506); +lean_dec(x_497); +x_508 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_508, 0, x_506); +lean_ctor_set(x_508, 1, x_507); +return x_508; } } } else { +uint8_t x_509; +x_509 = l_Array_isEmpty___rarg(x_4); +if (x_509 == 0) +{ +lean_object* x_510; lean_object* x_511; lean_object* x_512; lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_516; +x_510 = lean_box(0); +x_511 = lean_box(x_471); +x_512 = lean_box(x_6); +x_513 = lean_box(x_7); +x_514 = lean_box(x_8); +x_515 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_515, 0, x_1); +lean_closure_set(x_515, 1, x_510); +lean_closure_set(x_515, 2, x_511); +lean_closure_set(x_515, 3, x_3); +lean_closure_set(x_515, 4, x_4); +lean_closure_set(x_515, 5, x_5); +lean_closure_set(x_515, 6, x_512); +lean_closure_set(x_515, 7, x_513); +lean_closure_set(x_515, 8, x_2); +lean_closure_set(x_515, 9, x_514); +x_516 = l_Lean_Elab_Term_observing___rarg(x_515, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_516) == 0) +{ uint8_t x_517; -x_517 = l_Array_isEmpty___rarg(x_4); +x_517 = !lean_is_exclusive(x_516); if (x_517 == 0) { -lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; lean_object* x_524; -x_518 = lean_box(0); -x_519 = lean_box(x_479); -x_520 = lean_box(x_6); -x_521 = lean_box(x_7); -x_522 = lean_box(x_8); -x_523 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_523, 0, x_1); -lean_closure_set(x_523, 1, x_518); -lean_closure_set(x_523, 2, x_519); -lean_closure_set(x_523, 3, x_3); -lean_closure_set(x_523, 4, x_4); -lean_closure_set(x_523, 5, x_5); -lean_closure_set(x_523, 6, x_520); -lean_closure_set(x_523, 7, x_521); -lean_closure_set(x_523, 8, x_2); -lean_closure_set(x_523, 9, x_522); -x_524 = l_Lean_Elab_Term_observing___rarg(x_523, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_524) == 0) -{ -uint8_t x_525; -x_525 = !lean_is_exclusive(x_524); -if (x_525 == 0) -{ -lean_object* x_526; lean_object* x_527; -x_526 = lean_ctor_get(x_524, 0); -x_527 = lean_array_push(x_9, x_526); -lean_ctor_set(x_524, 0, x_527); -return x_524; -} -else -{ -lean_object* x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; -x_528 = lean_ctor_get(x_524, 0); -x_529 = lean_ctor_get(x_524, 1); -lean_inc(x_529); -lean_inc(x_528); -lean_dec(x_524); -x_530 = lean_array_push(x_9, x_528); -x_531 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_531, 0, x_530); -lean_ctor_set(x_531, 1, x_529); -return x_531; -} -} -else -{ -uint8_t x_532; +lean_object* x_518; lean_object* x_519; +x_518 = lean_ctor_get(x_516, 0); +x_519 = lean_array_push(x_9, x_518); +lean_ctor_set(x_516, 0, x_519); +return x_516; +} +else +{ +lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_object* x_523; +x_520 = lean_ctor_get(x_516, 0); +x_521 = lean_ctor_get(x_516, 1); +lean_inc(x_521); +lean_inc(x_520); +lean_dec(x_516); +x_522 = lean_array_push(x_9, x_520); +x_523 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_523, 0, x_522); +lean_ctor_set(x_523, 1, x_521); +return x_523; +} +} +else +{ +uint8_t x_524; lean_dec(x_9); -x_532 = !lean_is_exclusive(x_524); -if (x_532 == 0) +x_524 = !lean_is_exclusive(x_516); +if (x_524 == 0) { -return x_524; +return x_516; +} +else +{ +lean_object* x_525; lean_object* x_526; lean_object* x_527; +x_525 = lean_ctor_get(x_516, 0); +x_526 = lean_ctor_get(x_516, 1); +lean_inc(x_526); +lean_inc(x_525); +lean_dec(x_516); +x_527 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_527, 0, x_525); +lean_ctor_set(x_527, 1, x_526); +return x_527; +} +} +} +else +{ +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +if (x_8 == 0) +{ +uint8_t x_528; lean_object* x_529; lean_object* x_530; lean_object* x_531; lean_object* x_532; +x_528 = 1; +x_529 = lean_box(x_528); +x_530 = lean_box(x_528); +x_531 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_531, 0, x_1); +lean_closure_set(x_531, 1, x_5); +lean_closure_set(x_531, 2, x_529); +lean_closure_set(x_531, 3, x_530); +x_532 = l_Lean_Elab_Term_observing___rarg(x_531, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_532) == 0) +{ +uint8_t x_533; +x_533 = !lean_is_exclusive(x_532); +if (x_533 == 0) +{ +lean_object* x_534; lean_object* x_535; +x_534 = lean_ctor_get(x_532, 0); +x_535 = lean_array_push(x_9, x_534); +lean_ctor_set(x_532, 0, x_535); +return x_532; +} +else +{ +lean_object* x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; +x_536 = lean_ctor_get(x_532, 0); +x_537 = lean_ctor_get(x_532, 1); +lean_inc(x_537); +lean_inc(x_536); +lean_dec(x_532); +x_538 = lean_array_push(x_9, x_536); +x_539 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_539, 0, x_538); +lean_ctor_set(x_539, 1, x_537); +return x_539; +} +} +else +{ +uint8_t x_540; +lean_dec(x_9); +x_540 = !lean_is_exclusive(x_532); +if (x_540 == 0) +{ +return x_532; +} +else +{ +lean_object* x_541; lean_object* x_542; lean_object* x_543; +x_541 = lean_ctor_get(x_532, 0); +x_542 = lean_ctor_get(x_532, 1); +lean_inc(x_542); +lean_inc(x_541); +lean_dec(x_532); +x_543 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_543, 0, x_541); +lean_ctor_set(x_543, 1, x_542); +return x_543; +} +} +} +else +{ +lean_object* x_544; uint8_t x_545; lean_object* x_546; lean_object* x_547; lean_object* x_548; lean_object* x_549; +x_544 = lean_box(0); +x_545 = 1; +x_546 = lean_box(x_471); +x_547 = lean_box(x_545); +x_548 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_548, 0, x_1); +lean_closure_set(x_548, 1, x_5); +lean_closure_set(x_548, 2, x_546); +lean_closure_set(x_548, 3, x_547); +lean_closure_set(x_548, 4, x_544); +x_549 = l_Lean_Elab_Term_observing___rarg(x_548, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_549) == 0) +{ +uint8_t x_550; +x_550 = !lean_is_exclusive(x_549); +if (x_550 == 0) +{ +lean_object* x_551; lean_object* x_552; +x_551 = lean_ctor_get(x_549, 0); +x_552 = lean_array_push(x_9, x_551); +lean_ctor_set(x_549, 0, x_552); +return x_549; +} +else +{ +lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; +x_553 = lean_ctor_get(x_549, 0); +x_554 = lean_ctor_get(x_549, 1); +lean_inc(x_554); +lean_inc(x_553); +lean_dec(x_549); +x_555 = lean_array_push(x_9, x_553); +x_556 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_556, 0, x_555); +lean_ctor_set(x_556, 1, x_554); +return x_556; +} +} +else +{ +uint8_t x_557; +lean_dec(x_9); +x_557 = !lean_is_exclusive(x_549); +if (x_557 == 0) +{ +return x_549; +} +else +{ +lean_object* x_558; lean_object* x_559; lean_object* x_560; +x_558 = lean_ctor_get(x_549, 0); +x_559 = lean_ctor_get(x_549, 1); +lean_inc(x_559); +lean_inc(x_558); +lean_dec(x_549); +x_560 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_560, 0, x_558); +lean_ctor_set(x_560, 1, x_559); +return x_560; +} +} +} +} +} +} +} +} +else +{ +lean_object* x_564; lean_object* x_565; +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_564 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__20; +x_565 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_564, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_565; +} +} +} +} +else +{ +lean_object* x_566; lean_object* x_567; uint8_t x_568; +x_566 = lean_unsigned_to_nat(1u); +x_567 = l_Lean_Syntax_getArg(x_1, x_566); +lean_inc(x_567); +x_568 = l_Lean_Syntax_isOfKind(x_567, x_20); +if (x_568 == 0) +{ +lean_object* x_569; uint8_t x_570; +lean_dec(x_1); +x_569 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; +lean_inc(x_567); +x_570 = l_Lean_Syntax_isOfKind(x_567, x_569); +if (x_570 == 0) +{ +lean_object* x_571; uint8_t x_572; +x_571 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__14; +lean_inc(x_567); +x_572 = l_Lean_Syntax_isOfKind(x_567, x_571); +if (x_572 == 0) +{ +lean_object* x_573; +lean_dec(x_567); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_573 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); +return x_573; +} +else +{ +lean_object* x_574; lean_object* x_575; uint8_t x_576; +x_574 = lean_unsigned_to_nat(0u); +x_575 = l_Lean_Syntax_getArg(x_567, x_574); +x_576 = l_Lean_Syntax_isOfKind(x_575, x_569); +if (x_576 == 0) +{ +lean_object* x_577; +lean_dec(x_567); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_577 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); +return x_577; +} +else +{ +uint8_t x_578; +x_578 = 1; +x_1 = x_567; +x_6 = x_578; +goto _start; +} +} +} +else +{ +uint8_t x_580; +x_580 = 1; +x_1 = x_567; +x_6 = x_580; +goto _start; +} +} +else +{ +lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; uint8_t x_587; +x_582 = lean_unsigned_to_nat(0u); +x_583 = l_Lean_Syntax_getArg(x_567, x_582); +x_584 = lean_unsigned_to_nat(2u); +x_585 = l_Lean_Syntax_getArg(x_567, x_584); +lean_dec(x_567); +x_586 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; +lean_inc(x_585); +x_587 = l_Lean_Syntax_isOfKind(x_585, x_586); +if (x_587 == 0) +{ +lean_object* x_588; uint8_t x_589; +x_588 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; +lean_inc(x_585); +x_589 = l_Lean_Syntax_isOfKind(x_585, x_588); +if (x_589 == 0) +{ +lean_object* x_590; +lean_dec(x_585); +lean_dec(x_583); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_590 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); +return x_590; +} +else +{ +lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; lean_object* x_595; uint8_t x_596; +x_591 = lean_box(0); +x_592 = l_Lean_Syntax_identComponents(x_585, x_591); +x_593 = lean_box(0); +x_594 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__3(x_1, x_592, x_593); +x_595 = l_List_appendTR___rarg(x_594, x_2); +x_596 = 1; +x_1 = x_583; +x_2 = x_595; +x_6 = x_596; +goto _start; +} +} +else +{ +lean_object* x_598; +lean_dec(x_1); +x_598 = l_Lean_Syntax_isFieldIdx_x3f(x_585); +if (lean_obj_tag(x_598) == 0) +{ +lean_object* x_599; lean_object* x_600; +lean_dec(x_585); +lean_dec(x_583); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_599 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; +x_600 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_599, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +return x_600; +} +else +{ +lean_object* x_601; lean_object* x_602; lean_object* x_603; uint8_t x_604; +x_601 = lean_ctor_get(x_598, 0); +lean_inc(x_601); +lean_dec(x_598); +x_602 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_602, 0, x_585); +lean_ctor_set(x_602, 1, x_601); +x_603 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_603, 0, x_602); +lean_ctor_set(x_603, 1, x_2); +x_604 = 1; +x_1 = x_583; +x_2 = x_603; +x_6 = x_604; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_606; lean_object* x_607; lean_object* x_608; lean_object* x_609; lean_object* x_610; uint8_t x_611; +x_606 = lean_unsigned_to_nat(0u); +x_607 = l_Lean_Syntax_getArg(x_1, x_606); +x_608 = lean_unsigned_to_nat(2u); +x_609 = l_Lean_Syntax_getArg(x_1, x_608); +x_610 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; +lean_inc(x_609); +x_611 = l_Lean_Syntax_isOfKind(x_609, x_610); +if (x_611 == 0) +{ +lean_object* x_612; uint8_t x_613; +x_612 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; +lean_inc(x_609); +x_613 = l_Lean_Syntax_isOfKind(x_609, x_612); +if (x_613 == 0) +{ +uint8_t x_614; uint8_t x_615; +lean_dec(x_609); +lean_dec(x_607); +x_614 = l_List_isEmpty___rarg(x_2); +if (x_8 == 0) +{ +uint8_t x_706; +x_706 = 1; +x_615 = x_706; +goto block_705; +} +else +{ +uint8_t x_707; +x_707 = 0; +x_615 = x_707; +goto block_705; +} +block_705: +{ +if (x_614 == 0) +{ +lean_object* x_616; lean_object* x_617; lean_object* x_618; lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; +x_616 = lean_box(0); +x_617 = lean_box(x_615); +x_618 = lean_box(x_6); +x_619 = lean_box(x_7); +x_620 = lean_box(x_8); +x_621 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_621, 0, x_1); +lean_closure_set(x_621, 1, x_616); +lean_closure_set(x_621, 2, x_617); +lean_closure_set(x_621, 3, x_3); +lean_closure_set(x_621, 4, x_4); +lean_closure_set(x_621, 5, x_5); +lean_closure_set(x_621, 6, x_618); +lean_closure_set(x_621, 7, x_619); +lean_closure_set(x_621, 8, x_2); +lean_closure_set(x_621, 9, x_620); +x_622 = l_Lean_Elab_Term_observing___rarg(x_621, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_622) == 0) +{ +uint8_t x_623; +x_623 = !lean_is_exclusive(x_622); +if (x_623 == 0) +{ +lean_object* x_624; lean_object* x_625; +x_624 = lean_ctor_get(x_622, 0); +x_625 = lean_array_push(x_9, x_624); +lean_ctor_set(x_622, 0, x_625); +return x_622; +} +else +{ +lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; +x_626 = lean_ctor_get(x_622, 0); +x_627 = lean_ctor_get(x_622, 1); +lean_inc(x_627); +lean_inc(x_626); +lean_dec(x_622); +x_628 = lean_array_push(x_9, x_626); +x_629 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_629, 0, x_628); +lean_ctor_set(x_629, 1, x_627); +return x_629; +} +} +else +{ +uint8_t x_630; +lean_dec(x_9); +x_630 = !lean_is_exclusive(x_622); +if (x_630 == 0) +{ +return x_622; +} +else +{ +lean_object* x_631; lean_object* x_632; lean_object* x_633; +x_631 = lean_ctor_get(x_622, 0); +x_632 = lean_ctor_get(x_622, 1); +lean_inc(x_632); +lean_inc(x_631); +lean_dec(x_622); +x_633 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_633, 0, x_631); +lean_ctor_set(x_633, 1, x_632); +return x_633; +} +} +} +else +{ +uint8_t x_634; +x_634 = l_Array_isEmpty___rarg(x_3); +if (x_634 == 0) +{ +lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_638; lean_object* x_639; lean_object* x_640; lean_object* x_641; +x_635 = lean_box(0); +x_636 = lean_box(x_615); +x_637 = lean_box(x_6); +x_638 = lean_box(x_7); +x_639 = lean_box(x_8); +x_640 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_640, 0, x_1); +lean_closure_set(x_640, 1, x_635); +lean_closure_set(x_640, 2, x_636); +lean_closure_set(x_640, 3, x_3); +lean_closure_set(x_640, 4, x_4); +lean_closure_set(x_640, 5, x_5); +lean_closure_set(x_640, 6, x_637); +lean_closure_set(x_640, 7, x_638); +lean_closure_set(x_640, 8, x_2); +lean_closure_set(x_640, 9, x_639); +x_641 = l_Lean_Elab_Term_observing___rarg(x_640, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_641) == 0) +{ +uint8_t x_642; +x_642 = !lean_is_exclusive(x_641); +if (x_642 == 0) +{ +lean_object* x_643; lean_object* x_644; +x_643 = lean_ctor_get(x_641, 0); +x_644 = lean_array_push(x_9, x_643); +lean_ctor_set(x_641, 0, x_644); +return x_641; +} +else +{ +lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; +x_645 = lean_ctor_get(x_641, 0); +x_646 = lean_ctor_get(x_641, 1); +lean_inc(x_646); +lean_inc(x_645); +lean_dec(x_641); +x_647 = lean_array_push(x_9, x_645); +x_648 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_648, 0, x_647); +lean_ctor_set(x_648, 1, x_646); +return x_648; +} +} +else +{ +uint8_t x_649; +lean_dec(x_9); +x_649 = !lean_is_exclusive(x_641); +if (x_649 == 0) +{ +return x_641; +} +else +{ +lean_object* x_650; lean_object* x_651; lean_object* x_652; +x_650 = lean_ctor_get(x_641, 0); +x_651 = lean_ctor_get(x_641, 1); +lean_inc(x_651); +lean_inc(x_650); +lean_dec(x_641); +x_652 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_652, 0, x_650); +lean_ctor_set(x_652, 1, x_651); +return x_652; +} +} +} +else +{ +uint8_t x_653; +x_653 = l_Array_isEmpty___rarg(x_4); +if (x_653 == 0) +{ +lean_object* x_654; lean_object* x_655; lean_object* x_656; lean_object* x_657; lean_object* x_658; lean_object* x_659; lean_object* x_660; +x_654 = lean_box(0); +x_655 = lean_box(x_615); +x_656 = lean_box(x_6); +x_657 = lean_box(x_7); +x_658 = lean_box(x_8); +x_659 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_659, 0, x_1); +lean_closure_set(x_659, 1, x_654); +lean_closure_set(x_659, 2, x_655); +lean_closure_set(x_659, 3, x_3); +lean_closure_set(x_659, 4, x_4); +lean_closure_set(x_659, 5, x_5); +lean_closure_set(x_659, 6, x_656); +lean_closure_set(x_659, 7, x_657); +lean_closure_set(x_659, 8, x_2); +lean_closure_set(x_659, 9, x_658); +x_660 = l_Lean_Elab_Term_observing___rarg(x_659, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_660) == 0) +{ +uint8_t x_661; +x_661 = !lean_is_exclusive(x_660); +if (x_661 == 0) +{ +lean_object* x_662; lean_object* x_663; +x_662 = lean_ctor_get(x_660, 0); +x_663 = lean_array_push(x_9, x_662); +lean_ctor_set(x_660, 0, x_663); +return x_660; +} +else +{ +lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; +x_664 = lean_ctor_get(x_660, 0); +x_665 = lean_ctor_get(x_660, 1); +lean_inc(x_665); +lean_inc(x_664); +lean_dec(x_660); +x_666 = lean_array_push(x_9, x_664); +x_667 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_667, 0, x_666); +lean_ctor_set(x_667, 1, x_665); +return x_667; +} +} +else +{ +uint8_t x_668; +lean_dec(x_9); +x_668 = !lean_is_exclusive(x_660); +if (x_668 == 0) +{ +return x_660; } else { -lean_object* x_533; lean_object* x_534; lean_object* x_535; -x_533 = lean_ctor_get(x_524, 0); -x_534 = lean_ctor_get(x_524, 1); -lean_inc(x_534); -lean_inc(x_533); -lean_dec(x_524); -x_535 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_535, 0, x_533); -lean_ctor_set(x_535, 1, x_534); -return x_535; +lean_object* x_669; lean_object* x_670; lean_object* x_671; +x_669 = lean_ctor_get(x_660, 0); +x_670 = lean_ctor_get(x_660, 1); +lean_inc(x_670); +lean_inc(x_669); +lean_dec(x_660); +x_671 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_671, 0, x_669); +lean_ctor_set(x_671, 1, x_670); +return x_671; } } } @@ -59807,593 +60883,383 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_536; lean_object* x_537; lean_object* x_538; lean_object* x_539; lean_object* x_540; -x_536 = 1; -x_537 = lean_box(x_536); -x_538 = lean_box(x_536); -x_539 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_539, 0, x_1); -lean_closure_set(x_539, 1, x_5); -lean_closure_set(x_539, 2, x_537); -lean_closure_set(x_539, 3, x_538); -x_540 = l_Lean_Elab_Term_observing___rarg(x_539, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_540) == 0) +uint8_t x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; lean_object* x_676; +x_672 = 1; +x_673 = lean_box(x_672); +x_674 = lean_box(x_672); +x_675 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_675, 0, x_1); +lean_closure_set(x_675, 1, x_5); +lean_closure_set(x_675, 2, x_673); +lean_closure_set(x_675, 3, x_674); +x_676 = l_Lean_Elab_Term_observing___rarg(x_675, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_676) == 0) { -uint8_t x_541; -x_541 = !lean_is_exclusive(x_540); -if (x_541 == 0) +uint8_t x_677; +x_677 = !lean_is_exclusive(x_676); +if (x_677 == 0) { -lean_object* x_542; lean_object* x_543; -x_542 = lean_ctor_get(x_540, 0); -x_543 = lean_array_push(x_9, x_542); -lean_ctor_set(x_540, 0, x_543); -return x_540; +lean_object* x_678; lean_object* x_679; +x_678 = lean_ctor_get(x_676, 0); +x_679 = lean_array_push(x_9, x_678); +lean_ctor_set(x_676, 0, x_679); +return x_676; } else { -lean_object* x_544; lean_object* x_545; lean_object* x_546; lean_object* x_547; -x_544 = lean_ctor_get(x_540, 0); -x_545 = lean_ctor_get(x_540, 1); -lean_inc(x_545); -lean_inc(x_544); -lean_dec(x_540); -x_546 = lean_array_push(x_9, x_544); -x_547 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_547, 0, x_546); -lean_ctor_set(x_547, 1, x_545); -return x_547; +lean_object* x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; +x_680 = lean_ctor_get(x_676, 0); +x_681 = lean_ctor_get(x_676, 1); +lean_inc(x_681); +lean_inc(x_680); +lean_dec(x_676); +x_682 = lean_array_push(x_9, x_680); +x_683 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_683, 0, x_682); +lean_ctor_set(x_683, 1, x_681); +return x_683; } } else { -uint8_t x_548; +uint8_t x_684; lean_dec(x_9); -x_548 = !lean_is_exclusive(x_540); -if (x_548 == 0) +x_684 = !lean_is_exclusive(x_676); +if (x_684 == 0) { -return x_540; +return x_676; } else { -lean_object* x_549; lean_object* x_550; lean_object* x_551; -x_549 = lean_ctor_get(x_540, 0); -x_550 = lean_ctor_get(x_540, 1); -lean_inc(x_550); -lean_inc(x_549); -lean_dec(x_540); -x_551 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_551, 0, x_549); -lean_ctor_set(x_551, 1, x_550); -return x_551; +lean_object* x_685; lean_object* x_686; lean_object* x_687; +x_685 = lean_ctor_get(x_676, 0); +x_686 = lean_ctor_get(x_676, 1); +lean_inc(x_686); +lean_inc(x_685); +lean_dec(x_676); +x_687 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_687, 0, x_685); +lean_ctor_set(x_687, 1, x_686); +return x_687; } } } else { -lean_object* x_552; uint8_t x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; lean_object* x_557; -x_552 = lean_box(0); -x_553 = 1; -x_554 = lean_box(x_479); -x_555 = lean_box(x_553); -x_556 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_556, 0, x_1); -lean_closure_set(x_556, 1, x_5); -lean_closure_set(x_556, 2, x_554); -lean_closure_set(x_556, 3, x_555); -lean_closure_set(x_556, 4, x_552); -x_557 = l_Lean_Elab_Term_observing___rarg(x_556, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_557) == 0) +lean_object* x_688; uint8_t x_689; lean_object* x_690; lean_object* x_691; lean_object* x_692; lean_object* x_693; +x_688 = lean_box(0); +x_689 = 1; +x_690 = lean_box(x_615); +x_691 = lean_box(x_689); +x_692 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_692, 0, x_1); +lean_closure_set(x_692, 1, x_5); +lean_closure_set(x_692, 2, x_690); +lean_closure_set(x_692, 3, x_691); +lean_closure_set(x_692, 4, x_688); +x_693 = l_Lean_Elab_Term_observing___rarg(x_692, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_693) == 0) { -uint8_t x_558; -x_558 = !lean_is_exclusive(x_557); -if (x_558 == 0) +uint8_t x_694; +x_694 = !lean_is_exclusive(x_693); +if (x_694 == 0) { -lean_object* x_559; lean_object* x_560; -x_559 = lean_ctor_get(x_557, 0); -x_560 = lean_array_push(x_9, x_559); -lean_ctor_set(x_557, 0, x_560); -return x_557; +lean_object* x_695; lean_object* x_696; +x_695 = lean_ctor_get(x_693, 0); +x_696 = lean_array_push(x_9, x_695); +lean_ctor_set(x_693, 0, x_696); +return x_693; } else { -lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; -x_561 = lean_ctor_get(x_557, 0); -x_562 = lean_ctor_get(x_557, 1); -lean_inc(x_562); -lean_inc(x_561); -lean_dec(x_557); -x_563 = lean_array_push(x_9, x_561); -x_564 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_564, 0, x_563); -lean_ctor_set(x_564, 1, x_562); -return x_564; +lean_object* x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; +x_697 = lean_ctor_get(x_693, 0); +x_698 = lean_ctor_get(x_693, 1); +lean_inc(x_698); +lean_inc(x_697); +lean_dec(x_693); +x_699 = lean_array_push(x_9, x_697); +x_700 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_700, 0, x_699); +lean_ctor_set(x_700, 1, x_698); +return x_700; } } else { -uint8_t x_565; +uint8_t x_701; lean_dec(x_9); -x_565 = !lean_is_exclusive(x_557); -if (x_565 == 0) +x_701 = !lean_is_exclusive(x_693); +if (x_701 == 0) { -return x_557; +return x_693; } else { -lean_object* x_566; lean_object* x_567; lean_object* x_568; -x_566 = lean_ctor_get(x_557, 0); -x_567 = lean_ctor_get(x_557, 1); -lean_inc(x_567); -lean_inc(x_566); -lean_dec(x_557); -x_568 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_568, 0, x_566); -lean_ctor_set(x_568, 1, x_567); -return x_568; -} -} -} -} +lean_object* x_702; lean_object* x_703; lean_object* x_704; +x_702 = lean_ctor_get(x_693, 0); +x_703 = lean_ctor_get(x_693, 1); +lean_inc(x_703); +lean_inc(x_702); +lean_dec(x_693); +x_704 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_704, 0, x_702); +lean_ctor_set(x_704, 1, x_703); +return x_704; } } } } -else -{ -lean_object* x_572; lean_object* x_573; -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_572 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__20; -x_573 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_572, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_573; } } } } else { -lean_object* x_574; lean_object* x_575; uint8_t x_576; -x_574 = lean_unsigned_to_nat(1u); -x_575 = l_Lean_Syntax_getArg(x_1, x_574); -lean_inc(x_575); -x_576 = l_Lean_Syntax_isOfKind(x_575, x_20); -if (x_576 == 0) +lean_object* x_708; lean_object* x_709; uint8_t x_710; +x_708 = lean_unsigned_to_nat(3u); +x_709 = l_Lean_Syntax_getArg(x_1, x_708); +x_710 = l_Lean_Syntax_matchesNull(x_709, x_606); +if (x_710 == 0) { -lean_object* x_577; uint8_t x_578; -lean_dec(x_1); -x_577 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; -lean_inc(x_575); -x_578 = l_Lean_Syntax_isOfKind(x_575, x_577); -if (x_578 == 0) -{ -lean_object* x_579; uint8_t x_580; -x_579 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__14; -lean_inc(x_575); -x_580 = l_Lean_Syntax_isOfKind(x_575, x_579); -if (x_580 == 0) -{ -lean_object* x_581; -lean_dec(x_575); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_581 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); -return x_581; -} -else -{ -lean_object* x_582; lean_object* x_583; uint8_t x_584; -x_582 = lean_unsigned_to_nat(0u); -x_583 = l_Lean_Syntax_getArg(x_575, x_582); -x_584 = l_Lean_Syntax_isOfKind(x_583, x_577); -if (x_584 == 0) +uint8_t x_711; uint8_t x_712; +lean_dec(x_609); +lean_dec(x_607); +x_711 = l_List_isEmpty___rarg(x_2); +if (x_8 == 0) { -lean_object* x_585; -lean_dec(x_575); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_585 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); -return x_585; +uint8_t x_803; +x_803 = 1; +x_712 = x_803; +goto block_802; } else { -uint8_t x_586; -x_586 = 1; -x_1 = x_575; -x_6 = x_586; -goto _start; -} +uint8_t x_804; +x_804 = 0; +x_712 = x_804; +goto block_802; } -} -else +block_802: { -uint8_t x_588; -x_588 = 1; -x_1 = x_575; -x_6 = x_588; -goto _start; -} -} -else +if (x_711 == 0) { -lean_object* x_590; lean_object* x_591; lean_object* x_592; lean_object* x_593; lean_object* x_594; uint8_t x_595; -x_590 = lean_unsigned_to_nat(0u); -x_591 = l_Lean_Syntax_getArg(x_575, x_590); -x_592 = lean_unsigned_to_nat(2u); -x_593 = l_Lean_Syntax_getArg(x_575, x_592); -lean_dec(x_575); -x_594 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; -lean_inc(x_593); -x_595 = l_Lean_Syntax_isOfKind(x_593, x_594); -if (x_595 == 0) +lean_object* x_713; lean_object* x_714; lean_object* x_715; lean_object* x_716; lean_object* x_717; lean_object* x_718; lean_object* x_719; +x_713 = lean_box(0); +x_714 = lean_box(x_712); +x_715 = lean_box(x_6); +x_716 = lean_box(x_7); +x_717 = lean_box(x_8); +x_718 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_718, 0, x_1); +lean_closure_set(x_718, 1, x_713); +lean_closure_set(x_718, 2, x_714); +lean_closure_set(x_718, 3, x_3); +lean_closure_set(x_718, 4, x_4); +lean_closure_set(x_718, 5, x_5); +lean_closure_set(x_718, 6, x_715); +lean_closure_set(x_718, 7, x_716); +lean_closure_set(x_718, 8, x_2); +lean_closure_set(x_718, 9, x_717); +x_719 = l_Lean_Elab_Term_observing___rarg(x_718, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_719) == 0) { -lean_object* x_596; uint8_t x_597; -x_596 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; -lean_inc(x_593); -x_597 = l_Lean_Syntax_isOfKind(x_593, x_596); -if (x_597 == 0) +uint8_t x_720; +x_720 = !lean_is_exclusive(x_719); +if (x_720 == 0) { -lean_object* x_598; -lean_dec(x_593); -lean_dec(x_591); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_598 = l_Lean_Elab_throwUnsupportedSyntax___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__2___rarg(x_16); -return x_598; +lean_object* x_721; lean_object* x_722; +x_721 = lean_ctor_get(x_719, 0); +x_722 = lean_array_push(x_9, x_721); +lean_ctor_set(x_719, 0, x_722); +return x_719; } else { -lean_object* x_599; lean_object* x_600; lean_object* x_601; lean_object* x_602; lean_object* x_603; uint8_t x_604; -x_599 = lean_box(0); -x_600 = l_Lean_Syntax_identComponents(x_593, x_599); -x_601 = lean_box(0); -x_602 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__3(x_1, x_600, x_601); -x_603 = l_List_appendTR___rarg(x_602, x_2); -x_604 = 1; -x_1 = x_591; -x_2 = x_603; -x_6 = x_604; -goto _start; +lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; +x_723 = lean_ctor_get(x_719, 0); +x_724 = lean_ctor_get(x_719, 1); +lean_inc(x_724); +lean_inc(x_723); +lean_dec(x_719); +x_725 = lean_array_push(x_9, x_723); +x_726 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_726, 0, x_725); +lean_ctor_set(x_726, 1, x_724); +return x_726; } } else { -lean_object* x_606; -lean_dec(x_1); -x_606 = l_Lean_Syntax_isFieldIdx_x3f(x_593); -if (lean_obj_tag(x_606) == 0) -{ -lean_object* x_607; lean_object* x_608; -lean_dec(x_593); -lean_dec(x_591); +uint8_t x_727; lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_607 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; -x_608 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_607, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -return x_608; +x_727 = !lean_is_exclusive(x_719); +if (x_727 == 0) +{ +return x_719; } else { -lean_object* x_609; lean_object* x_610; lean_object* x_611; uint8_t x_612; -x_609 = lean_ctor_get(x_606, 0); -lean_inc(x_609); -lean_dec(x_606); -x_610 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_610, 0, x_593); -lean_ctor_set(x_610, 1, x_609); -x_611 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_611, 0, x_610); -lean_ctor_set(x_611, 1, x_2); -x_612 = 1; -x_1 = x_591; -x_2 = x_611; -x_6 = x_612; -goto _start; +lean_object* x_728; lean_object* x_729; lean_object* x_730; +x_728 = lean_ctor_get(x_719, 0); +x_729 = lean_ctor_get(x_719, 1); +lean_inc(x_729); +lean_inc(x_728); +lean_dec(x_719); +x_730 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_730, 0, x_728); +lean_ctor_set(x_730, 1, x_729); +return x_730; } } } -} -} -else -{ -lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_618; uint8_t x_619; -x_614 = lean_unsigned_to_nat(0u); -x_615 = l_Lean_Syntax_getArg(x_1, x_614); -x_616 = lean_unsigned_to_nat(2u); -x_617 = l_Lean_Syntax_getArg(x_1, x_616); -x_618 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; -lean_inc(x_617); -x_619 = l_Lean_Syntax_isOfKind(x_617, x_618); -if (x_619 == 0) -{ -lean_object* x_620; uint8_t x_621; -x_620 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; -lean_inc(x_617); -x_621 = l_Lean_Syntax_isOfKind(x_617, x_620); -if (x_621 == 0) -{ -uint8_t x_622; uint8_t x_623; -lean_dec(x_617); -lean_dec(x_615); -x_622 = l_List_isEmpty___rarg(x_2); -if (x_8 == 0) -{ -uint8_t x_714; -x_714 = 1; -x_623 = x_714; -goto block_713; -} else { -uint8_t x_715; -x_715 = 0; -x_623 = x_715; -goto block_713; -} -block_713: -{ -if (x_622 == 0) +uint8_t x_731; +x_731 = l_Array_isEmpty___rarg(x_3); +if (x_731 == 0) { -lean_object* x_624; lean_object* x_625; lean_object* x_626; lean_object* x_627; lean_object* x_628; lean_object* x_629; lean_object* x_630; -x_624 = lean_box(0); -x_625 = lean_box(x_623); -x_626 = lean_box(x_6); -x_627 = lean_box(x_7); -x_628 = lean_box(x_8); -x_629 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_629, 0, x_1); -lean_closure_set(x_629, 1, x_624); -lean_closure_set(x_629, 2, x_625); -lean_closure_set(x_629, 3, x_3); -lean_closure_set(x_629, 4, x_4); -lean_closure_set(x_629, 5, x_5); -lean_closure_set(x_629, 6, x_626); -lean_closure_set(x_629, 7, x_627); -lean_closure_set(x_629, 8, x_2); -lean_closure_set(x_629, 9, x_628); -x_630 = l_Lean_Elab_Term_observing___rarg(x_629, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_630) == 0) +lean_object* x_732; lean_object* x_733; lean_object* x_734; lean_object* x_735; lean_object* x_736; lean_object* x_737; lean_object* x_738; +x_732 = lean_box(0); +x_733 = lean_box(x_712); +x_734 = lean_box(x_6); +x_735 = lean_box(x_7); +x_736 = lean_box(x_8); +x_737 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_737, 0, x_1); +lean_closure_set(x_737, 1, x_732); +lean_closure_set(x_737, 2, x_733); +lean_closure_set(x_737, 3, x_3); +lean_closure_set(x_737, 4, x_4); +lean_closure_set(x_737, 5, x_5); +lean_closure_set(x_737, 6, x_734); +lean_closure_set(x_737, 7, x_735); +lean_closure_set(x_737, 8, x_2); +lean_closure_set(x_737, 9, x_736); +x_738 = l_Lean_Elab_Term_observing___rarg(x_737, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_738) == 0) { -uint8_t x_631; -x_631 = !lean_is_exclusive(x_630); -if (x_631 == 0) +uint8_t x_739; +x_739 = !lean_is_exclusive(x_738); +if (x_739 == 0) { -lean_object* x_632; lean_object* x_633; -x_632 = lean_ctor_get(x_630, 0); -x_633 = lean_array_push(x_9, x_632); -lean_ctor_set(x_630, 0, x_633); -return x_630; +lean_object* x_740; lean_object* x_741; +x_740 = lean_ctor_get(x_738, 0); +x_741 = lean_array_push(x_9, x_740); +lean_ctor_set(x_738, 0, x_741); +return x_738; } else { -lean_object* x_634; lean_object* x_635; lean_object* x_636; lean_object* x_637; -x_634 = lean_ctor_get(x_630, 0); -x_635 = lean_ctor_get(x_630, 1); -lean_inc(x_635); -lean_inc(x_634); -lean_dec(x_630); -x_636 = lean_array_push(x_9, x_634); -x_637 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_637, 0, x_636); -lean_ctor_set(x_637, 1, x_635); -return x_637; +lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; +x_742 = lean_ctor_get(x_738, 0); +x_743 = lean_ctor_get(x_738, 1); +lean_inc(x_743); +lean_inc(x_742); +lean_dec(x_738); +x_744 = lean_array_push(x_9, x_742); +x_745 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_745, 0, x_744); +lean_ctor_set(x_745, 1, x_743); +return x_745; } } else { -uint8_t x_638; +uint8_t x_746; lean_dec(x_9); -x_638 = !lean_is_exclusive(x_630); -if (x_638 == 0) +x_746 = !lean_is_exclusive(x_738); +if (x_746 == 0) { -return x_630; +return x_738; } else { -lean_object* x_639; lean_object* x_640; lean_object* x_641; -x_639 = lean_ctor_get(x_630, 0); -x_640 = lean_ctor_get(x_630, 1); -lean_inc(x_640); -lean_inc(x_639); -lean_dec(x_630); -x_641 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_641, 0, x_639); -lean_ctor_set(x_641, 1, x_640); -return x_641; +lean_object* x_747; lean_object* x_748; lean_object* x_749; +x_747 = lean_ctor_get(x_738, 0); +x_748 = lean_ctor_get(x_738, 1); +lean_inc(x_748); +lean_inc(x_747); +lean_dec(x_738); +x_749 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_749, 0, x_747); +lean_ctor_set(x_749, 1, x_748); +return x_749; } } } else { -uint8_t x_642; -x_642 = l_Array_isEmpty___rarg(x_3); -if (x_642 == 0) +uint8_t x_750; +x_750 = l_Array_isEmpty___rarg(x_4); +if (x_750 == 0) { -lean_object* x_643; lean_object* x_644; lean_object* x_645; lean_object* x_646; lean_object* x_647; lean_object* x_648; lean_object* x_649; -x_643 = lean_box(0); -x_644 = lean_box(x_623); -x_645 = lean_box(x_6); -x_646 = lean_box(x_7); -x_647 = lean_box(x_8); -x_648 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_648, 0, x_1); -lean_closure_set(x_648, 1, x_643); -lean_closure_set(x_648, 2, x_644); -lean_closure_set(x_648, 3, x_3); -lean_closure_set(x_648, 4, x_4); -lean_closure_set(x_648, 5, x_5); -lean_closure_set(x_648, 6, x_645); -lean_closure_set(x_648, 7, x_646); -lean_closure_set(x_648, 8, x_2); -lean_closure_set(x_648, 9, x_647); -x_649 = l_Lean_Elab_Term_observing___rarg(x_648, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_649) == 0) -{ -uint8_t x_650; -x_650 = !lean_is_exclusive(x_649); -if (x_650 == 0) -{ -lean_object* x_651; lean_object* x_652; -x_651 = lean_ctor_get(x_649, 0); -x_652 = lean_array_push(x_9, x_651); -lean_ctor_set(x_649, 0, x_652); -return x_649; -} -else -{ -lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; -x_653 = lean_ctor_get(x_649, 0); -x_654 = lean_ctor_get(x_649, 1); -lean_inc(x_654); -lean_inc(x_653); -lean_dec(x_649); -x_655 = lean_array_push(x_9, x_653); -x_656 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_656, 0, x_655); -lean_ctor_set(x_656, 1, x_654); -return x_656; -} -} -else -{ -uint8_t x_657; -lean_dec(x_9); -x_657 = !lean_is_exclusive(x_649); -if (x_657 == 0) +lean_object* x_751; lean_object* x_752; lean_object* x_753; lean_object* x_754; lean_object* x_755; lean_object* x_756; lean_object* x_757; +x_751 = lean_box(0); +x_752 = lean_box(x_712); +x_753 = lean_box(x_6); +x_754 = lean_box(x_7); +x_755 = lean_box(x_8); +x_756 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_756, 0, x_1); +lean_closure_set(x_756, 1, x_751); +lean_closure_set(x_756, 2, x_752); +lean_closure_set(x_756, 3, x_3); +lean_closure_set(x_756, 4, x_4); +lean_closure_set(x_756, 5, x_5); +lean_closure_set(x_756, 6, x_753); +lean_closure_set(x_756, 7, x_754); +lean_closure_set(x_756, 8, x_2); +lean_closure_set(x_756, 9, x_755); +x_757 = l_Lean_Elab_Term_observing___rarg(x_756, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_757) == 0) { -return x_649; +uint8_t x_758; +x_758 = !lean_is_exclusive(x_757); +if (x_758 == 0) +{ +lean_object* x_759; lean_object* x_760; +x_759 = lean_ctor_get(x_757, 0); +x_760 = lean_array_push(x_9, x_759); +lean_ctor_set(x_757, 0, x_760); +return x_757; } else { -lean_object* x_658; lean_object* x_659; lean_object* x_660; -x_658 = lean_ctor_get(x_649, 0); -x_659 = lean_ctor_get(x_649, 1); -lean_inc(x_659); -lean_inc(x_658); -lean_dec(x_649); -x_660 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_660, 0, x_658); -lean_ctor_set(x_660, 1, x_659); -return x_660; -} +lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; +x_761 = lean_ctor_get(x_757, 0); +x_762 = lean_ctor_get(x_757, 1); +lean_inc(x_762); +lean_inc(x_761); +lean_dec(x_757); +x_763 = lean_array_push(x_9, x_761); +x_764 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_764, 0, x_763); +lean_ctor_set(x_764, 1, x_762); +return x_764; } } else { -uint8_t x_661; -x_661 = l_Array_isEmpty___rarg(x_4); -if (x_661 == 0) -{ -lean_object* x_662; lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; lean_object* x_668; -x_662 = lean_box(0); -x_663 = lean_box(x_623); -x_664 = lean_box(x_6); -x_665 = lean_box(x_7); -x_666 = lean_box(x_8); -x_667 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_667, 0, x_1); -lean_closure_set(x_667, 1, x_662); -lean_closure_set(x_667, 2, x_663); -lean_closure_set(x_667, 3, x_3); -lean_closure_set(x_667, 4, x_4); -lean_closure_set(x_667, 5, x_5); -lean_closure_set(x_667, 6, x_664); -lean_closure_set(x_667, 7, x_665); -lean_closure_set(x_667, 8, x_2); -lean_closure_set(x_667, 9, x_666); -x_668 = l_Lean_Elab_Term_observing___rarg(x_667, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_668) == 0) -{ -uint8_t x_669; -x_669 = !lean_is_exclusive(x_668); -if (x_669 == 0) -{ -lean_object* x_670; lean_object* x_671; -x_670 = lean_ctor_get(x_668, 0); -x_671 = lean_array_push(x_9, x_670); -lean_ctor_set(x_668, 0, x_671); -return x_668; -} -else -{ -lean_object* x_672; lean_object* x_673; lean_object* x_674; lean_object* x_675; -x_672 = lean_ctor_get(x_668, 0); -x_673 = lean_ctor_get(x_668, 1); -lean_inc(x_673); -lean_inc(x_672); -lean_dec(x_668); -x_674 = lean_array_push(x_9, x_672); -x_675 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_675, 0, x_674); -lean_ctor_set(x_675, 1, x_673); -return x_675; -} -} -else -{ -uint8_t x_676; +uint8_t x_765; lean_dec(x_9); -x_676 = !lean_is_exclusive(x_668); -if (x_676 == 0) +x_765 = !lean_is_exclusive(x_757); +if (x_765 == 0) { -return x_668; +return x_757; } else { -lean_object* x_677; lean_object* x_678; lean_object* x_679; -x_677 = lean_ctor_get(x_668, 0); -x_678 = lean_ctor_get(x_668, 1); -lean_inc(x_678); -lean_inc(x_677); -lean_dec(x_668); -x_679 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_679, 0, x_677); -lean_ctor_set(x_679, 1, x_678); -return x_679; +lean_object* x_766; lean_object* x_767; lean_object* x_768; +x_766 = lean_ctor_get(x_757, 0); +x_767 = lean_ctor_get(x_757, 1); +lean_inc(x_767); +lean_inc(x_766); +lean_dec(x_757); +x_768 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_768, 0, x_766); +lean_ctor_set(x_768, 1, x_767); +return x_768; } } } @@ -60404,129 +61270,129 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_680; lean_object* x_681; lean_object* x_682; lean_object* x_683; lean_object* x_684; -x_680 = 1; -x_681 = lean_box(x_680); -x_682 = lean_box(x_680); -x_683 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_683, 0, x_1); -lean_closure_set(x_683, 1, x_5); -lean_closure_set(x_683, 2, x_681); -lean_closure_set(x_683, 3, x_682); -x_684 = l_Lean_Elab_Term_observing___rarg(x_683, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_684) == 0) +uint8_t x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; lean_object* x_773; +x_769 = 1; +x_770 = lean_box(x_769); +x_771 = lean_box(x_769); +x_772 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_772, 0, x_1); +lean_closure_set(x_772, 1, x_5); +lean_closure_set(x_772, 2, x_770); +lean_closure_set(x_772, 3, x_771); +x_773 = l_Lean_Elab_Term_observing___rarg(x_772, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_773) == 0) { -uint8_t x_685; -x_685 = !lean_is_exclusive(x_684); -if (x_685 == 0) +uint8_t x_774; +x_774 = !lean_is_exclusive(x_773); +if (x_774 == 0) { -lean_object* x_686; lean_object* x_687; -x_686 = lean_ctor_get(x_684, 0); -x_687 = lean_array_push(x_9, x_686); -lean_ctor_set(x_684, 0, x_687); -return x_684; +lean_object* x_775; lean_object* x_776; +x_775 = lean_ctor_get(x_773, 0); +x_776 = lean_array_push(x_9, x_775); +lean_ctor_set(x_773, 0, x_776); +return x_773; } else { -lean_object* x_688; lean_object* x_689; lean_object* x_690; lean_object* x_691; -x_688 = lean_ctor_get(x_684, 0); -x_689 = lean_ctor_get(x_684, 1); -lean_inc(x_689); -lean_inc(x_688); -lean_dec(x_684); -x_690 = lean_array_push(x_9, x_688); -x_691 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_691, 0, x_690); -lean_ctor_set(x_691, 1, x_689); -return x_691; +lean_object* x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; +x_777 = lean_ctor_get(x_773, 0); +x_778 = lean_ctor_get(x_773, 1); +lean_inc(x_778); +lean_inc(x_777); +lean_dec(x_773); +x_779 = lean_array_push(x_9, x_777); +x_780 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_780, 0, x_779); +lean_ctor_set(x_780, 1, x_778); +return x_780; } } else { -uint8_t x_692; +uint8_t x_781; lean_dec(x_9); -x_692 = !lean_is_exclusive(x_684); -if (x_692 == 0) +x_781 = !lean_is_exclusive(x_773); +if (x_781 == 0) { -return x_684; +return x_773; } else { -lean_object* x_693; lean_object* x_694; lean_object* x_695; -x_693 = lean_ctor_get(x_684, 0); -x_694 = lean_ctor_get(x_684, 1); -lean_inc(x_694); -lean_inc(x_693); -lean_dec(x_684); -x_695 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_695, 0, x_693); -lean_ctor_set(x_695, 1, x_694); -return x_695; +lean_object* x_782; lean_object* x_783; lean_object* x_784; +x_782 = lean_ctor_get(x_773, 0); +x_783 = lean_ctor_get(x_773, 1); +lean_inc(x_783); +lean_inc(x_782); +lean_dec(x_773); +x_784 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_784, 0, x_782); +lean_ctor_set(x_784, 1, x_783); +return x_784; } } } else { -lean_object* x_696; uint8_t x_697; lean_object* x_698; lean_object* x_699; lean_object* x_700; lean_object* x_701; -x_696 = lean_box(0); -x_697 = 1; -x_698 = lean_box(x_623); -x_699 = lean_box(x_697); -x_700 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_700, 0, x_1); -lean_closure_set(x_700, 1, x_5); -lean_closure_set(x_700, 2, x_698); -lean_closure_set(x_700, 3, x_699); -lean_closure_set(x_700, 4, x_696); -x_701 = l_Lean_Elab_Term_observing___rarg(x_700, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_701) == 0) +lean_object* x_785; uint8_t x_786; lean_object* x_787; lean_object* x_788; lean_object* x_789; lean_object* x_790; +x_785 = lean_box(0); +x_786 = 1; +x_787 = lean_box(x_712); +x_788 = lean_box(x_786); +x_789 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_789, 0, x_1); +lean_closure_set(x_789, 1, x_5); +lean_closure_set(x_789, 2, x_787); +lean_closure_set(x_789, 3, x_788); +lean_closure_set(x_789, 4, x_785); +x_790 = l_Lean_Elab_Term_observing___rarg(x_789, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_790) == 0) { -uint8_t x_702; -x_702 = !lean_is_exclusive(x_701); -if (x_702 == 0) +uint8_t x_791; +x_791 = !lean_is_exclusive(x_790); +if (x_791 == 0) { -lean_object* x_703; lean_object* x_704; -x_703 = lean_ctor_get(x_701, 0); -x_704 = lean_array_push(x_9, x_703); -lean_ctor_set(x_701, 0, x_704); -return x_701; +lean_object* x_792; lean_object* x_793; +x_792 = lean_ctor_get(x_790, 0); +x_793 = lean_array_push(x_9, x_792); +lean_ctor_set(x_790, 0, x_793); +return x_790; } else { -lean_object* x_705; lean_object* x_706; lean_object* x_707; lean_object* x_708; -x_705 = lean_ctor_get(x_701, 0); -x_706 = lean_ctor_get(x_701, 1); -lean_inc(x_706); -lean_inc(x_705); -lean_dec(x_701); -x_707 = lean_array_push(x_9, x_705); -x_708 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_708, 0, x_707); -lean_ctor_set(x_708, 1, x_706); -return x_708; +lean_object* x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; +x_794 = lean_ctor_get(x_790, 0); +x_795 = lean_ctor_get(x_790, 1); +lean_inc(x_795); +lean_inc(x_794); +lean_dec(x_790); +x_796 = lean_array_push(x_9, x_794); +x_797 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_797, 0, x_796); +lean_ctor_set(x_797, 1, x_795); +return x_797; } } else { -uint8_t x_709; +uint8_t x_798; lean_dec(x_9); -x_709 = !lean_is_exclusive(x_701); -if (x_709 == 0) +x_798 = !lean_is_exclusive(x_790); +if (x_798 == 0) { -return x_701; +return x_790; } else { -lean_object* x_710; lean_object* x_711; lean_object* x_712; -x_710 = lean_ctor_get(x_701, 0); -x_711 = lean_ctor_get(x_701, 1); -lean_inc(x_711); -lean_inc(x_710); -lean_dec(x_701); -x_712 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_712, 0, x_710); -lean_ctor_set(x_712, 1, x_711); -return x_712; +lean_object* x_799; lean_object* x_800; lean_object* x_801; +x_799 = lean_ctor_get(x_790, 0); +x_800 = lean_ctor_get(x_790, 1); +lean_inc(x_800); +lean_inc(x_799); +lean_dec(x_790); +x_801 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_801, 0, x_799); +lean_ctor_set(x_801, 1, x_800); +return x_801; } } } @@ -60537,651 +61403,264 @@ return x_712; } else { -lean_object* x_716; lean_object* x_717; uint8_t x_718; -x_716 = lean_unsigned_to_nat(3u); -x_717 = l_Lean_Syntax_getArg(x_1, x_716); -x_718 = l_Lean_Syntax_matchesNull(x_717, x_614); -if (x_718 == 0) -{ -uint8_t x_719; uint8_t x_720; -lean_dec(x_617); -lean_dec(x_615); -x_719 = l_List_isEmpty___rarg(x_2); -if (x_8 == 0) -{ -uint8_t x_811; -x_811 = 1; -x_720 = x_811; -goto block_810; -} -else -{ -uint8_t x_812; -x_812 = 0; -x_720 = x_812; -goto block_810; -} -block_810: -{ -if (x_719 == 0) -{ -lean_object* x_721; lean_object* x_722; lean_object* x_723; lean_object* x_724; lean_object* x_725; lean_object* x_726; lean_object* x_727; -x_721 = lean_box(0); -x_722 = lean_box(x_720); -x_723 = lean_box(x_6); -x_724 = lean_box(x_7); -x_725 = lean_box(x_8); -x_726 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_726, 0, x_1); -lean_closure_set(x_726, 1, x_721); -lean_closure_set(x_726, 2, x_722); -lean_closure_set(x_726, 3, x_3); -lean_closure_set(x_726, 4, x_4); -lean_closure_set(x_726, 5, x_5); -lean_closure_set(x_726, 6, x_723); -lean_closure_set(x_726, 7, x_724); -lean_closure_set(x_726, 8, x_2); -lean_closure_set(x_726, 9, x_725); -x_727 = l_Lean_Elab_Term_observing___rarg(x_726, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_727) == 0) -{ -uint8_t x_728; -x_728 = !lean_is_exclusive(x_727); -if (x_728 == 0) -{ -lean_object* x_729; lean_object* x_730; -x_729 = lean_ctor_get(x_727, 0); -x_730 = lean_array_push(x_9, x_729); -lean_ctor_set(x_727, 0, x_730); -return x_727; -} -else -{ -lean_object* x_731; lean_object* x_732; lean_object* x_733; lean_object* x_734; -x_731 = lean_ctor_get(x_727, 0); -x_732 = lean_ctor_get(x_727, 1); -lean_inc(x_732); -lean_inc(x_731); -lean_dec(x_727); -x_733 = lean_array_push(x_9, x_731); -x_734 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_734, 0, x_733); -lean_ctor_set(x_734, 1, x_732); -return x_734; -} -} -else -{ -uint8_t x_735; -lean_dec(x_9); -x_735 = !lean_is_exclusive(x_727); -if (x_735 == 0) -{ -return x_727; -} -else -{ -lean_object* x_736; lean_object* x_737; lean_object* x_738; -x_736 = lean_ctor_get(x_727, 0); -x_737 = lean_ctor_get(x_727, 1); -lean_inc(x_737); -lean_inc(x_736); -lean_dec(x_727); -x_738 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_738, 0, x_736); -lean_ctor_set(x_738, 1, x_737); -return x_738; -} -} -} -else -{ -uint8_t x_739; -x_739 = l_Array_isEmpty___rarg(x_3); -if (x_739 == 0) -{ -lean_object* x_740; lean_object* x_741; lean_object* x_742; lean_object* x_743; lean_object* x_744; lean_object* x_745; lean_object* x_746; -x_740 = lean_box(0); -x_741 = lean_box(x_720); -x_742 = lean_box(x_6); -x_743 = lean_box(x_7); -x_744 = lean_box(x_8); -x_745 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_745, 0, x_1); -lean_closure_set(x_745, 1, x_740); -lean_closure_set(x_745, 2, x_741); -lean_closure_set(x_745, 3, x_3); -lean_closure_set(x_745, 4, x_4); -lean_closure_set(x_745, 5, x_5); -lean_closure_set(x_745, 6, x_742); -lean_closure_set(x_745, 7, x_743); -lean_closure_set(x_745, 8, x_2); -lean_closure_set(x_745, 9, x_744); -x_746 = l_Lean_Elab_Term_observing___rarg(x_745, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_746) == 0) -{ -uint8_t x_747; -x_747 = !lean_is_exclusive(x_746); -if (x_747 == 0) -{ -lean_object* x_748; lean_object* x_749; -x_748 = lean_ctor_get(x_746, 0); -x_749 = lean_array_push(x_9, x_748); -lean_ctor_set(x_746, 0, x_749); -return x_746; -} -else -{ -lean_object* x_750; lean_object* x_751; lean_object* x_752; lean_object* x_753; -x_750 = lean_ctor_get(x_746, 0); -x_751 = lean_ctor_get(x_746, 1); -lean_inc(x_751); -lean_inc(x_750); -lean_dec(x_746); -x_752 = lean_array_push(x_9, x_750); -x_753 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_753, 0, x_752); -lean_ctor_set(x_753, 1, x_751); -return x_753; -} -} -else -{ -uint8_t x_754; -lean_dec(x_9); -x_754 = !lean_is_exclusive(x_746); -if (x_754 == 0) -{ -return x_746; -} -else -{ -lean_object* x_755; lean_object* x_756; lean_object* x_757; -x_755 = lean_ctor_get(x_746, 0); -x_756 = lean_ctor_get(x_746, 1); -lean_inc(x_756); -lean_inc(x_755); -lean_dec(x_746); -x_757 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_757, 0, x_755); -lean_ctor_set(x_757, 1, x_756); -return x_757; -} +lean_object* x_805; lean_object* x_806; lean_object* x_807; lean_object* x_808; lean_object* x_809; +x_805 = lean_box(0); +x_806 = l_Lean_Syntax_identComponents(x_609, x_805); +x_807 = lean_box(0); +x_808 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__4(x_1, x_806, x_807); +x_809 = l_List_appendTR___rarg(x_808, x_2); +x_1 = x_607; +x_2 = x_809; +goto _start; } } -else -{ -uint8_t x_758; -x_758 = l_Array_isEmpty___rarg(x_4); -if (x_758 == 0) -{ -lean_object* x_759; lean_object* x_760; lean_object* x_761; lean_object* x_762; lean_object* x_763; lean_object* x_764; lean_object* x_765; -x_759 = lean_box(0); -x_760 = lean_box(x_720); -x_761 = lean_box(x_6); -x_762 = lean_box(x_7); -x_763 = lean_box(x_8); -x_764 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_764, 0, x_1); -lean_closure_set(x_764, 1, x_759); -lean_closure_set(x_764, 2, x_760); -lean_closure_set(x_764, 3, x_3); -lean_closure_set(x_764, 4, x_4); -lean_closure_set(x_764, 5, x_5); -lean_closure_set(x_764, 6, x_761); -lean_closure_set(x_764, 7, x_762); -lean_closure_set(x_764, 8, x_2); -lean_closure_set(x_764, 9, x_763); -x_765 = l_Lean_Elab_Term_observing___rarg(x_764, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_765) == 0) -{ -uint8_t x_766; -x_766 = !lean_is_exclusive(x_765); -if (x_766 == 0) -{ -lean_object* x_767; lean_object* x_768; -x_767 = lean_ctor_get(x_765, 0); -x_768 = lean_array_push(x_9, x_767); -lean_ctor_set(x_765, 0, x_768); -return x_765; -} -else -{ -lean_object* x_769; lean_object* x_770; lean_object* x_771; lean_object* x_772; -x_769 = lean_ctor_get(x_765, 0); -x_770 = lean_ctor_get(x_765, 1); -lean_inc(x_770); -lean_inc(x_769); -lean_dec(x_765); -x_771 = lean_array_push(x_9, x_769); -x_772 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_772, 0, x_771); -lean_ctor_set(x_772, 1, x_770); -return x_772; -} -} -else -{ -uint8_t x_773; -lean_dec(x_9); -x_773 = !lean_is_exclusive(x_765); -if (x_773 == 0) -{ -return x_765; } else { -lean_object* x_774; lean_object* x_775; lean_object* x_776; -x_774 = lean_ctor_get(x_765, 0); -x_775 = lean_ctor_get(x_765, 1); -lean_inc(x_775); -lean_inc(x_774); -lean_dec(x_765); -x_776 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_776, 0, x_774); -lean_ctor_set(x_776, 1, x_775); -return x_776; -} -} -} -else +lean_object* x_811; lean_object* x_812; uint8_t x_813; +x_811 = lean_unsigned_to_nat(3u); +x_812 = l_Lean_Syntax_getArg(x_1, x_811); +x_813 = l_Lean_Syntax_matchesNull(x_812, x_606); +if (x_813 == 0) { -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); +uint8_t x_814; uint8_t x_815; +lean_dec(x_609); +lean_dec(x_607); +x_814 = l_List_isEmpty___rarg(x_2); if (x_8 == 0) { -uint8_t x_777; lean_object* x_778; lean_object* x_779; lean_object* x_780; lean_object* x_781; -x_777 = 1; -x_778 = lean_box(x_777); -x_779 = lean_box(x_777); -x_780 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_780, 0, x_1); -lean_closure_set(x_780, 1, x_5); -lean_closure_set(x_780, 2, x_778); -lean_closure_set(x_780, 3, x_779); -x_781 = l_Lean_Elab_Term_observing___rarg(x_780, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_781) == 0) -{ -uint8_t x_782; -x_782 = !lean_is_exclusive(x_781); -if (x_782 == 0) -{ -lean_object* x_783; lean_object* x_784; -x_783 = lean_ctor_get(x_781, 0); -x_784 = lean_array_push(x_9, x_783); -lean_ctor_set(x_781, 0, x_784); -return x_781; +uint8_t x_906; +x_906 = 1; +x_815 = x_906; +goto block_905; } else { -lean_object* x_785; lean_object* x_786; lean_object* x_787; lean_object* x_788; -x_785 = lean_ctor_get(x_781, 0); -x_786 = lean_ctor_get(x_781, 1); -lean_inc(x_786); -lean_inc(x_785); -lean_dec(x_781); -x_787 = lean_array_push(x_9, x_785); -x_788 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_788, 0, x_787); -lean_ctor_set(x_788, 1, x_786); -return x_788; +uint8_t x_907; +x_907 = 0; +x_815 = x_907; +goto block_905; } -} -else +block_905: { -uint8_t x_789; -lean_dec(x_9); -x_789 = !lean_is_exclusive(x_781); -if (x_789 == 0) -{ -return x_781; -} -else +if (x_814 == 0) { -lean_object* x_790; lean_object* x_791; lean_object* x_792; -x_790 = lean_ctor_get(x_781, 0); -x_791 = lean_ctor_get(x_781, 1); -lean_inc(x_791); -lean_inc(x_790); -lean_dec(x_781); -x_792 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_792, 0, x_790); -lean_ctor_set(x_792, 1, x_791); -return x_792; -} -} -} -else +lean_object* x_816; lean_object* x_817; lean_object* x_818; lean_object* x_819; lean_object* x_820; lean_object* x_821; lean_object* x_822; +x_816 = lean_box(0); +x_817 = lean_box(x_815); +x_818 = lean_box(x_6); +x_819 = lean_box(x_7); +x_820 = lean_box(x_8); +x_821 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_821, 0, x_1); +lean_closure_set(x_821, 1, x_816); +lean_closure_set(x_821, 2, x_817); +lean_closure_set(x_821, 3, x_3); +lean_closure_set(x_821, 4, x_4); +lean_closure_set(x_821, 5, x_5); +lean_closure_set(x_821, 6, x_818); +lean_closure_set(x_821, 7, x_819); +lean_closure_set(x_821, 8, x_2); +lean_closure_set(x_821, 9, x_820); +x_822 = l_Lean_Elab_Term_observing___rarg(x_821, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_822) == 0) { -lean_object* x_793; uint8_t x_794; lean_object* x_795; lean_object* x_796; lean_object* x_797; lean_object* x_798; -x_793 = lean_box(0); -x_794 = 1; -x_795 = lean_box(x_720); -x_796 = lean_box(x_794); -x_797 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_797, 0, x_1); -lean_closure_set(x_797, 1, x_5); -lean_closure_set(x_797, 2, x_795); -lean_closure_set(x_797, 3, x_796); -lean_closure_set(x_797, 4, x_793); -x_798 = l_Lean_Elab_Term_observing___rarg(x_797, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_798) == 0) +uint8_t x_823; +x_823 = !lean_is_exclusive(x_822); +if (x_823 == 0) { -uint8_t x_799; -x_799 = !lean_is_exclusive(x_798); -if (x_799 == 0) -{ -lean_object* x_800; lean_object* x_801; -x_800 = lean_ctor_get(x_798, 0); -x_801 = lean_array_push(x_9, x_800); -lean_ctor_set(x_798, 0, x_801); -return x_798; +lean_object* x_824; lean_object* x_825; +x_824 = lean_ctor_get(x_822, 0); +x_825 = lean_array_push(x_9, x_824); +lean_ctor_set(x_822, 0, x_825); +return x_822; } else { -lean_object* x_802; lean_object* x_803; lean_object* x_804; lean_object* x_805; -x_802 = lean_ctor_get(x_798, 0); -x_803 = lean_ctor_get(x_798, 1); -lean_inc(x_803); -lean_inc(x_802); -lean_dec(x_798); -x_804 = lean_array_push(x_9, x_802); -x_805 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_805, 0, x_804); -lean_ctor_set(x_805, 1, x_803); -return x_805; +lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; +x_826 = lean_ctor_get(x_822, 0); +x_827 = lean_ctor_get(x_822, 1); +lean_inc(x_827); +lean_inc(x_826); +lean_dec(x_822); +x_828 = lean_array_push(x_9, x_826); +x_829 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_829, 0, x_828); +lean_ctor_set(x_829, 1, x_827); +return x_829; } } else { -uint8_t x_806; +uint8_t x_830; lean_dec(x_9); -x_806 = !lean_is_exclusive(x_798); -if (x_806 == 0) -{ -return x_798; -} -else +x_830 = !lean_is_exclusive(x_822); +if (x_830 == 0) { -lean_object* x_807; lean_object* x_808; lean_object* x_809; -x_807 = lean_ctor_get(x_798, 0); -x_808 = lean_ctor_get(x_798, 1); -lean_inc(x_808); -lean_inc(x_807); -lean_dec(x_798); -x_809 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_809, 0, x_807); -lean_ctor_set(x_809, 1, x_808); -return x_809; -} -} -} -} -} -} -} +return x_822; } else { -lean_object* x_813; lean_object* x_814; lean_object* x_815; lean_object* x_816; lean_object* x_817; -x_813 = lean_box(0); -x_814 = l_Lean_Syntax_identComponents(x_617, x_813); -x_815 = lean_box(0); -x_816 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__4(x_1, x_814, x_815); -x_817 = l_List_appendTR___rarg(x_816, x_2); -x_1 = x_615; -x_2 = x_817; -goto _start; +lean_object* x_831; lean_object* x_832; lean_object* x_833; +x_831 = lean_ctor_get(x_822, 0); +x_832 = lean_ctor_get(x_822, 1); +lean_inc(x_832); +lean_inc(x_831); +lean_dec(x_822); +x_833 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_833, 0, x_831); +lean_ctor_set(x_833, 1, x_832); +return x_833; } } } else { -lean_object* x_819; lean_object* x_820; uint8_t x_821; -x_819 = lean_unsigned_to_nat(3u); -x_820 = l_Lean_Syntax_getArg(x_1, x_819); -x_821 = l_Lean_Syntax_matchesNull(x_820, x_614); -if (x_821 == 0) -{ -uint8_t x_822; uint8_t x_823; -lean_dec(x_617); -lean_dec(x_615); -x_822 = l_List_isEmpty___rarg(x_2); -if (x_8 == 0) -{ -uint8_t x_914; -x_914 = 1; -x_823 = x_914; -goto block_913; -} -else -{ -uint8_t x_915; -x_915 = 0; -x_823 = x_915; -goto block_913; -} -block_913: +uint8_t x_834; +x_834 = l_Array_isEmpty___rarg(x_3); +if (x_834 == 0) { -if (x_822 == 0) +lean_object* x_835; lean_object* x_836; lean_object* x_837; lean_object* x_838; lean_object* x_839; lean_object* x_840; lean_object* x_841; +x_835 = lean_box(0); +x_836 = lean_box(x_815); +x_837 = lean_box(x_6); +x_838 = lean_box(x_7); +x_839 = lean_box(x_8); +x_840 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_840, 0, x_1); +lean_closure_set(x_840, 1, x_835); +lean_closure_set(x_840, 2, x_836); +lean_closure_set(x_840, 3, x_3); +lean_closure_set(x_840, 4, x_4); +lean_closure_set(x_840, 5, x_5); +lean_closure_set(x_840, 6, x_837); +lean_closure_set(x_840, 7, x_838); +lean_closure_set(x_840, 8, x_2); +lean_closure_set(x_840, 9, x_839); +x_841 = l_Lean_Elab_Term_observing___rarg(x_840, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_841) == 0) { -lean_object* x_824; lean_object* x_825; lean_object* x_826; lean_object* x_827; lean_object* x_828; lean_object* x_829; lean_object* x_830; -x_824 = lean_box(0); -x_825 = lean_box(x_823); -x_826 = lean_box(x_6); -x_827 = lean_box(x_7); -x_828 = lean_box(x_8); -x_829 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_829, 0, x_1); -lean_closure_set(x_829, 1, x_824); -lean_closure_set(x_829, 2, x_825); -lean_closure_set(x_829, 3, x_3); -lean_closure_set(x_829, 4, x_4); -lean_closure_set(x_829, 5, x_5); -lean_closure_set(x_829, 6, x_826); -lean_closure_set(x_829, 7, x_827); -lean_closure_set(x_829, 8, x_2); -lean_closure_set(x_829, 9, x_828); -x_830 = l_Lean_Elab_Term_observing___rarg(x_829, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_830) == 0) -{ -uint8_t x_831; -x_831 = !lean_is_exclusive(x_830); -if (x_831 == 0) +uint8_t x_842; +x_842 = !lean_is_exclusive(x_841); +if (x_842 == 0) { -lean_object* x_832; lean_object* x_833; -x_832 = lean_ctor_get(x_830, 0); -x_833 = lean_array_push(x_9, x_832); -lean_ctor_set(x_830, 0, x_833); -return x_830; +lean_object* x_843; lean_object* x_844; +x_843 = lean_ctor_get(x_841, 0); +x_844 = lean_array_push(x_9, x_843); +lean_ctor_set(x_841, 0, x_844); +return x_841; } else { -lean_object* x_834; lean_object* x_835; lean_object* x_836; lean_object* x_837; -x_834 = lean_ctor_get(x_830, 0); -x_835 = lean_ctor_get(x_830, 1); -lean_inc(x_835); -lean_inc(x_834); -lean_dec(x_830); -x_836 = lean_array_push(x_9, x_834); -x_837 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_837, 0, x_836); -lean_ctor_set(x_837, 1, x_835); -return x_837; +lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; +x_845 = lean_ctor_get(x_841, 0); +x_846 = lean_ctor_get(x_841, 1); +lean_inc(x_846); +lean_inc(x_845); +lean_dec(x_841); +x_847 = lean_array_push(x_9, x_845); +x_848 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_848, 0, x_847); +lean_ctor_set(x_848, 1, x_846); +return x_848; } } else { -uint8_t x_838; +uint8_t x_849; lean_dec(x_9); -x_838 = !lean_is_exclusive(x_830); -if (x_838 == 0) +x_849 = !lean_is_exclusive(x_841); +if (x_849 == 0) { -return x_830; +return x_841; } else { -lean_object* x_839; lean_object* x_840; lean_object* x_841; -x_839 = lean_ctor_get(x_830, 0); -x_840 = lean_ctor_get(x_830, 1); -lean_inc(x_840); -lean_inc(x_839); -lean_dec(x_830); -x_841 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_841, 0, x_839); -lean_ctor_set(x_841, 1, x_840); -return x_841; +lean_object* x_850; lean_object* x_851; lean_object* x_852; +x_850 = lean_ctor_get(x_841, 0); +x_851 = lean_ctor_get(x_841, 1); +lean_inc(x_851); +lean_inc(x_850); +lean_dec(x_841); +x_852 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_852, 0, x_850); +lean_ctor_set(x_852, 1, x_851); +return x_852; } } } else { -uint8_t x_842; -x_842 = l_Array_isEmpty___rarg(x_3); -if (x_842 == 0) +uint8_t x_853; +x_853 = l_Array_isEmpty___rarg(x_4); +if (x_853 == 0) { -lean_object* x_843; lean_object* x_844; lean_object* x_845; lean_object* x_846; lean_object* x_847; lean_object* x_848; lean_object* x_849; -x_843 = lean_box(0); -x_844 = lean_box(x_823); -x_845 = lean_box(x_6); -x_846 = lean_box(x_7); -x_847 = lean_box(x_8); -x_848 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_848, 0, x_1); -lean_closure_set(x_848, 1, x_843); -lean_closure_set(x_848, 2, x_844); -lean_closure_set(x_848, 3, x_3); -lean_closure_set(x_848, 4, x_4); -lean_closure_set(x_848, 5, x_5); -lean_closure_set(x_848, 6, x_845); -lean_closure_set(x_848, 7, x_846); -lean_closure_set(x_848, 8, x_2); -lean_closure_set(x_848, 9, x_847); -x_849 = l_Lean_Elab_Term_observing___rarg(x_848, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_849) == 0) -{ -uint8_t x_850; -x_850 = !lean_is_exclusive(x_849); -if (x_850 == 0) -{ -lean_object* x_851; lean_object* x_852; -x_851 = lean_ctor_get(x_849, 0); -x_852 = lean_array_push(x_9, x_851); -lean_ctor_set(x_849, 0, x_852); -return x_849; -} -else -{ -lean_object* x_853; lean_object* x_854; lean_object* x_855; lean_object* x_856; -x_853 = lean_ctor_get(x_849, 0); -x_854 = lean_ctor_get(x_849, 1); -lean_inc(x_854); -lean_inc(x_853); -lean_dec(x_849); -x_855 = lean_array_push(x_9, x_853); -x_856 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_856, 0, x_855); -lean_ctor_set(x_856, 1, x_854); -return x_856; -} -} -else -{ -uint8_t x_857; -lean_dec(x_9); -x_857 = !lean_is_exclusive(x_849); -if (x_857 == 0) +lean_object* x_854; lean_object* x_855; lean_object* x_856; lean_object* x_857; lean_object* x_858; lean_object* x_859; lean_object* x_860; +x_854 = lean_box(0); +x_855 = lean_box(x_815); +x_856 = lean_box(x_6); +x_857 = lean_box(x_7); +x_858 = lean_box(x_8); +x_859 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_859, 0, x_1); +lean_closure_set(x_859, 1, x_854); +lean_closure_set(x_859, 2, x_855); +lean_closure_set(x_859, 3, x_3); +lean_closure_set(x_859, 4, x_4); +lean_closure_set(x_859, 5, x_5); +lean_closure_set(x_859, 6, x_856); +lean_closure_set(x_859, 7, x_857); +lean_closure_set(x_859, 8, x_2); +lean_closure_set(x_859, 9, x_858); +x_860 = l_Lean_Elab_Term_observing___rarg(x_859, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_860) == 0) { -return x_849; -} -else +uint8_t x_861; +x_861 = !lean_is_exclusive(x_860); +if (x_861 == 0) { -lean_object* x_858; lean_object* x_859; lean_object* x_860; -x_858 = lean_ctor_get(x_849, 0); -x_859 = lean_ctor_get(x_849, 1); -lean_inc(x_859); -lean_inc(x_858); -lean_dec(x_849); -x_860 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_860, 0, x_858); -lean_ctor_set(x_860, 1, x_859); +lean_object* x_862; lean_object* x_863; +x_862 = lean_ctor_get(x_860, 0); +x_863 = lean_array_push(x_9, x_862); +lean_ctor_set(x_860, 0, x_863); return x_860; } +else +{ +lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; +x_864 = lean_ctor_get(x_860, 0); +x_865 = lean_ctor_get(x_860, 1); +lean_inc(x_865); +lean_inc(x_864); +lean_dec(x_860); +x_866 = lean_array_push(x_9, x_864); +x_867 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_867, 0, x_866); +lean_ctor_set(x_867, 1, x_865); +return x_867; } } else { -uint8_t x_861; -x_861 = l_Array_isEmpty___rarg(x_4); -if (x_861 == 0) -{ -lean_object* x_862; lean_object* x_863; lean_object* x_864; lean_object* x_865; lean_object* x_866; lean_object* x_867; lean_object* x_868; -x_862 = lean_box(0); -x_863 = lean_box(x_823); -x_864 = lean_box(x_6); -x_865 = lean_box(x_7); -x_866 = lean_box(x_8); -x_867 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_867, 0, x_1); -lean_closure_set(x_867, 1, x_862); -lean_closure_set(x_867, 2, x_863); -lean_closure_set(x_867, 3, x_3); -lean_closure_set(x_867, 4, x_4); -lean_closure_set(x_867, 5, x_5); -lean_closure_set(x_867, 6, x_864); -lean_closure_set(x_867, 7, x_865); -lean_closure_set(x_867, 8, x_2); -lean_closure_set(x_867, 9, x_866); -x_868 = l_Lean_Elab_Term_observing___rarg(x_867, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_868) == 0) -{ -uint8_t x_869; -x_869 = !lean_is_exclusive(x_868); -if (x_869 == 0) -{ -lean_object* x_870; lean_object* x_871; -x_870 = lean_ctor_get(x_868, 0); -x_871 = lean_array_push(x_9, x_870); -lean_ctor_set(x_868, 0, x_871); -return x_868; -} -else -{ -lean_object* x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; -x_872 = lean_ctor_get(x_868, 0); -x_873 = lean_ctor_get(x_868, 1); -lean_inc(x_873); -lean_inc(x_872); -lean_dec(x_868); -x_874 = lean_array_push(x_9, x_872); -x_875 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_875, 0, x_874); -lean_ctor_set(x_875, 1, x_873); -return x_875; -} -} -else -{ -uint8_t x_876; +uint8_t x_868; lean_dec(x_9); -x_876 = !lean_is_exclusive(x_868); -if (x_876 == 0) +x_868 = !lean_is_exclusive(x_860); +if (x_868 == 0) { -return x_868; +return x_860; } else { -lean_object* x_877; lean_object* x_878; lean_object* x_879; -x_877 = lean_ctor_get(x_868, 0); -x_878 = lean_ctor_get(x_868, 1); -lean_inc(x_878); -lean_inc(x_877); -lean_dec(x_868); -x_879 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_879, 0, x_877); -lean_ctor_set(x_879, 1, x_878); -return x_879; +lean_object* x_869; lean_object* x_870; lean_object* x_871; +x_869 = lean_ctor_get(x_860, 0); +x_870 = lean_ctor_get(x_860, 1); +lean_inc(x_870); +lean_inc(x_869); +lean_dec(x_860); +x_871 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_871, 0, x_869); +lean_ctor_set(x_871, 1, x_870); +return x_871; } } } @@ -61192,129 +61671,129 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; lean_object* x_884; -x_880 = 1; -x_881 = lean_box(x_880); -x_882 = lean_box(x_880); -x_883 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_883, 0, x_1); -lean_closure_set(x_883, 1, x_5); -lean_closure_set(x_883, 2, x_881); -lean_closure_set(x_883, 3, x_882); -x_884 = l_Lean_Elab_Term_observing___rarg(x_883, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_884) == 0) +uint8_t x_872; lean_object* x_873; lean_object* x_874; lean_object* x_875; lean_object* x_876; +x_872 = 1; +x_873 = lean_box(x_872); +x_874 = lean_box(x_872); +x_875 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_875, 0, x_1); +lean_closure_set(x_875, 1, x_5); +lean_closure_set(x_875, 2, x_873); +lean_closure_set(x_875, 3, x_874); +x_876 = l_Lean_Elab_Term_observing___rarg(x_875, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_876) == 0) { -uint8_t x_885; -x_885 = !lean_is_exclusive(x_884); -if (x_885 == 0) +uint8_t x_877; +x_877 = !lean_is_exclusive(x_876); +if (x_877 == 0) { -lean_object* x_886; lean_object* x_887; -x_886 = lean_ctor_get(x_884, 0); -x_887 = lean_array_push(x_9, x_886); -lean_ctor_set(x_884, 0, x_887); -return x_884; +lean_object* x_878; lean_object* x_879; +x_878 = lean_ctor_get(x_876, 0); +x_879 = lean_array_push(x_9, x_878); +lean_ctor_set(x_876, 0, x_879); +return x_876; } else { -lean_object* x_888; lean_object* x_889; lean_object* x_890; lean_object* x_891; -x_888 = lean_ctor_get(x_884, 0); -x_889 = lean_ctor_get(x_884, 1); -lean_inc(x_889); -lean_inc(x_888); -lean_dec(x_884); -x_890 = lean_array_push(x_9, x_888); -x_891 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_891, 0, x_890); -lean_ctor_set(x_891, 1, x_889); -return x_891; +lean_object* x_880; lean_object* x_881; lean_object* x_882; lean_object* x_883; +x_880 = lean_ctor_get(x_876, 0); +x_881 = lean_ctor_get(x_876, 1); +lean_inc(x_881); +lean_inc(x_880); +lean_dec(x_876); +x_882 = lean_array_push(x_9, x_880); +x_883 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_883, 0, x_882); +lean_ctor_set(x_883, 1, x_881); +return x_883; } } else { -uint8_t x_892; +uint8_t x_884; lean_dec(x_9); -x_892 = !lean_is_exclusive(x_884); -if (x_892 == 0) +x_884 = !lean_is_exclusive(x_876); +if (x_884 == 0) { -return x_884; +return x_876; } else { -lean_object* x_893; lean_object* x_894; lean_object* x_895; -x_893 = lean_ctor_get(x_884, 0); -x_894 = lean_ctor_get(x_884, 1); -lean_inc(x_894); -lean_inc(x_893); -lean_dec(x_884); -x_895 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_895, 0, x_893); -lean_ctor_set(x_895, 1, x_894); -return x_895; +lean_object* x_885; lean_object* x_886; lean_object* x_887; +x_885 = lean_ctor_get(x_876, 0); +x_886 = lean_ctor_get(x_876, 1); +lean_inc(x_886); +lean_inc(x_885); +lean_dec(x_876); +x_887 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_887, 0, x_885); +lean_ctor_set(x_887, 1, x_886); +return x_887; } } } else { -lean_object* x_896; uint8_t x_897; lean_object* x_898; lean_object* x_899; lean_object* x_900; lean_object* x_901; -x_896 = lean_box(0); -x_897 = 1; -x_898 = lean_box(x_823); -x_899 = lean_box(x_897); -x_900 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_900, 0, x_1); -lean_closure_set(x_900, 1, x_5); -lean_closure_set(x_900, 2, x_898); -lean_closure_set(x_900, 3, x_899); -lean_closure_set(x_900, 4, x_896); -x_901 = l_Lean_Elab_Term_observing___rarg(x_900, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_901) == 0) +lean_object* x_888; uint8_t x_889; lean_object* x_890; lean_object* x_891; lean_object* x_892; lean_object* x_893; +x_888 = lean_box(0); +x_889 = 1; +x_890 = lean_box(x_815); +x_891 = lean_box(x_889); +x_892 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_892, 0, x_1); +lean_closure_set(x_892, 1, x_5); +lean_closure_set(x_892, 2, x_890); +lean_closure_set(x_892, 3, x_891); +lean_closure_set(x_892, 4, x_888); +x_893 = l_Lean_Elab_Term_observing___rarg(x_892, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_893) == 0) { -uint8_t x_902; -x_902 = !lean_is_exclusive(x_901); -if (x_902 == 0) +uint8_t x_894; +x_894 = !lean_is_exclusive(x_893); +if (x_894 == 0) { -lean_object* x_903; lean_object* x_904; -x_903 = lean_ctor_get(x_901, 0); -x_904 = lean_array_push(x_9, x_903); -lean_ctor_set(x_901, 0, x_904); -return x_901; +lean_object* x_895; lean_object* x_896; +x_895 = lean_ctor_get(x_893, 0); +x_896 = lean_array_push(x_9, x_895); +lean_ctor_set(x_893, 0, x_896); +return x_893; } else { -lean_object* x_905; lean_object* x_906; lean_object* x_907; lean_object* x_908; -x_905 = lean_ctor_get(x_901, 0); -x_906 = lean_ctor_get(x_901, 1); -lean_inc(x_906); -lean_inc(x_905); -lean_dec(x_901); -x_907 = lean_array_push(x_9, x_905); -x_908 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_908, 0, x_907); -lean_ctor_set(x_908, 1, x_906); -return x_908; +lean_object* x_897; lean_object* x_898; lean_object* x_899; lean_object* x_900; +x_897 = lean_ctor_get(x_893, 0); +x_898 = lean_ctor_get(x_893, 1); +lean_inc(x_898); +lean_inc(x_897); +lean_dec(x_893); +x_899 = lean_array_push(x_9, x_897); +x_900 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_900, 0, x_899); +lean_ctor_set(x_900, 1, x_898); +return x_900; } } else { -uint8_t x_909; +uint8_t x_901; lean_dec(x_9); -x_909 = !lean_is_exclusive(x_901); -if (x_909 == 0) +x_901 = !lean_is_exclusive(x_893); +if (x_901 == 0) { -return x_901; +return x_893; } else { -lean_object* x_910; lean_object* x_911; lean_object* x_912; -x_910 = lean_ctor_get(x_901, 0); -x_911 = lean_ctor_get(x_901, 1); -lean_inc(x_911); -lean_inc(x_910); -lean_dec(x_901); -x_912 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_912, 0, x_910); -lean_ctor_set(x_912, 1, x_911); -return x_912; +lean_object* x_902; lean_object* x_903; lean_object* x_904; +x_902 = lean_ctor_get(x_893, 0); +x_903 = lean_ctor_get(x_893, 1); +lean_inc(x_903); +lean_inc(x_902); +lean_dec(x_893); +x_904 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_904, 0, x_902); +lean_ctor_set(x_904, 1, x_903); +return x_904; } } } @@ -61325,42 +61804,42 @@ return x_912; } else { -lean_object* x_916; +lean_object* x_908; lean_dec(x_1); -x_916 = l_Lean_Syntax_isFieldIdx_x3f(x_617); -if (lean_obj_tag(x_916) == 0) +x_908 = l_Lean_Syntax_isFieldIdx_x3f(x_609); +if (lean_obj_tag(x_908) == 0) { -lean_object* x_917; lean_object* x_918; -lean_dec(x_617); -lean_dec(x_615); +lean_object* x_909; lean_object* x_910; +lean_dec(x_609); +lean_dec(x_607); lean_dec(x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_917 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; -x_918 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_917, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_909 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; +x_910 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_909, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -return x_918; +return x_910; } else { -lean_object* x_919; lean_object* x_920; lean_object* x_921; -x_919 = lean_ctor_get(x_916, 0); -lean_inc(x_919); -lean_dec(x_916); -x_920 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_920, 0, x_617); -lean_ctor_set(x_920, 1, x_919); -x_921 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_921, 0, x_920); -lean_ctor_set(x_921, 1, x_2); -x_1 = x_615; -x_2 = x_921; +lean_object* x_911; lean_object* x_912; lean_object* x_913; +x_911 = lean_ctor_get(x_908, 0); +lean_inc(x_911); +lean_dec(x_908); +x_912 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_912, 0, x_609); +lean_ctor_set(x_912, 1, x_911); +x_913 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_913, 0, x_912); +lean_ctor_set(x_913, 1, x_2); +x_1 = x_607; +x_2 = x_913; goto _start; } } @@ -61369,260 +61848,260 @@ goto _start; } else { -lean_object* x_923; lean_object* x_924; lean_object* x_925; lean_object* x_926; lean_object* x_927; uint8_t x_928; -x_923 = lean_unsigned_to_nat(0u); -x_924 = l_Lean_Syntax_getArg(x_1, x_923); -x_925 = lean_unsigned_to_nat(2u); -x_926 = l_Lean_Syntax_getArg(x_1, x_925); -x_927 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; -lean_inc(x_926); -x_928 = l_Lean_Syntax_isOfKind(x_926, x_927); -if (x_928 == 0) +lean_object* x_915; lean_object* x_916; lean_object* x_917; lean_object* x_918; lean_object* x_919; uint8_t x_920; +x_915 = lean_unsigned_to_nat(0u); +x_916 = l_Lean_Syntax_getArg(x_1, x_915); +x_917 = lean_unsigned_to_nat(2u); +x_918 = l_Lean_Syntax_getArg(x_1, x_917); +x_919 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__22; +lean_inc(x_918); +x_920 = l_Lean_Syntax_isOfKind(x_918, x_919); +if (x_920 == 0) { -lean_object* x_929; uint8_t x_930; -x_929 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; -lean_inc(x_926); -x_930 = l_Lean_Syntax_isOfKind(x_926, x_929); -if (x_930 == 0) +lean_object* x_921; uint8_t x_922; +x_921 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__12; +lean_inc(x_918); +x_922 = l_Lean_Syntax_isOfKind(x_918, x_921); +if (x_922 == 0) { -uint8_t x_931; uint8_t x_932; -lean_dec(x_926); -lean_dec(x_924); -x_931 = l_List_isEmpty___rarg(x_2); +uint8_t x_923; uint8_t x_924; +lean_dec(x_918); +lean_dec(x_916); +x_923 = l_List_isEmpty___rarg(x_2); if (x_8 == 0) { -uint8_t x_1023; -x_1023 = 1; -x_932 = x_1023; -goto block_1022; +uint8_t x_1015; +x_1015 = 1; +x_924 = x_1015; +goto block_1014; } else { -uint8_t x_1024; -x_1024 = 0; -x_932 = x_1024; -goto block_1022; +uint8_t x_1016; +x_1016 = 0; +x_924 = x_1016; +goto block_1014; } -block_1022: +block_1014: { -if (x_931 == 0) +if (x_923 == 0) { -lean_object* x_933; lean_object* x_934; lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; lean_object* x_939; -x_933 = lean_box(0); -x_934 = lean_box(x_932); -x_935 = lean_box(x_6); -x_936 = lean_box(x_7); -x_937 = lean_box(x_8); -x_938 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_938, 0, x_1); -lean_closure_set(x_938, 1, x_933); -lean_closure_set(x_938, 2, x_934); -lean_closure_set(x_938, 3, x_3); -lean_closure_set(x_938, 4, x_4); -lean_closure_set(x_938, 5, x_5); -lean_closure_set(x_938, 6, x_935); -lean_closure_set(x_938, 7, x_936); -lean_closure_set(x_938, 8, x_2); -lean_closure_set(x_938, 9, x_937); -x_939 = l_Lean_Elab_Term_observing___rarg(x_938, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_939) == 0) +lean_object* x_925; lean_object* x_926; lean_object* x_927; lean_object* x_928; lean_object* x_929; lean_object* x_930; lean_object* x_931; +x_925 = lean_box(0); +x_926 = lean_box(x_924); +x_927 = lean_box(x_6); +x_928 = lean_box(x_7); +x_929 = lean_box(x_8); +x_930 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_930, 0, x_1); +lean_closure_set(x_930, 1, x_925); +lean_closure_set(x_930, 2, x_926); +lean_closure_set(x_930, 3, x_3); +lean_closure_set(x_930, 4, x_4); +lean_closure_set(x_930, 5, x_5); +lean_closure_set(x_930, 6, x_927); +lean_closure_set(x_930, 7, x_928); +lean_closure_set(x_930, 8, x_2); +lean_closure_set(x_930, 9, x_929); +x_931 = l_Lean_Elab_Term_observing___rarg(x_930, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_931) == 0) { -uint8_t x_940; -x_940 = !lean_is_exclusive(x_939); -if (x_940 == 0) +uint8_t x_932; +x_932 = !lean_is_exclusive(x_931); +if (x_932 == 0) { -lean_object* x_941; lean_object* x_942; -x_941 = lean_ctor_get(x_939, 0); -x_942 = lean_array_push(x_9, x_941); -lean_ctor_set(x_939, 0, x_942); -return x_939; +lean_object* x_933; lean_object* x_934; +x_933 = lean_ctor_get(x_931, 0); +x_934 = lean_array_push(x_9, x_933); +lean_ctor_set(x_931, 0, x_934); +return x_931; } else { -lean_object* x_943; lean_object* x_944; lean_object* x_945; lean_object* x_946; -x_943 = lean_ctor_get(x_939, 0); -x_944 = lean_ctor_get(x_939, 1); -lean_inc(x_944); -lean_inc(x_943); -lean_dec(x_939); -x_945 = lean_array_push(x_9, x_943); -x_946 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_946, 0, x_945); -lean_ctor_set(x_946, 1, x_944); -return x_946; +lean_object* x_935; lean_object* x_936; lean_object* x_937; lean_object* x_938; +x_935 = lean_ctor_get(x_931, 0); +x_936 = lean_ctor_get(x_931, 1); +lean_inc(x_936); +lean_inc(x_935); +lean_dec(x_931); +x_937 = lean_array_push(x_9, x_935); +x_938 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_938, 0, x_937); +lean_ctor_set(x_938, 1, x_936); +return x_938; } } else { -uint8_t x_947; +uint8_t x_939; lean_dec(x_9); -x_947 = !lean_is_exclusive(x_939); -if (x_947 == 0) +x_939 = !lean_is_exclusive(x_931); +if (x_939 == 0) { -return x_939; +return x_931; } else { -lean_object* x_948; lean_object* x_949; lean_object* x_950; -x_948 = lean_ctor_get(x_939, 0); -x_949 = lean_ctor_get(x_939, 1); -lean_inc(x_949); -lean_inc(x_948); -lean_dec(x_939); -x_950 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_950, 0, x_948); -lean_ctor_set(x_950, 1, x_949); -return x_950; +lean_object* x_940; lean_object* x_941; lean_object* x_942; +x_940 = lean_ctor_get(x_931, 0); +x_941 = lean_ctor_get(x_931, 1); +lean_inc(x_941); +lean_inc(x_940); +lean_dec(x_931); +x_942 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_942, 0, x_940); +lean_ctor_set(x_942, 1, x_941); +return x_942; } } } else { +uint8_t x_943; +x_943 = l_Array_isEmpty___rarg(x_3); +if (x_943 == 0) +{ +lean_object* x_944; lean_object* x_945; lean_object* x_946; lean_object* x_947; lean_object* x_948; lean_object* x_949; lean_object* x_950; +x_944 = lean_box(0); +x_945 = lean_box(x_924); +x_946 = lean_box(x_6); +x_947 = lean_box(x_7); +x_948 = lean_box(x_8); +x_949 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_949, 0, x_1); +lean_closure_set(x_949, 1, x_944); +lean_closure_set(x_949, 2, x_945); +lean_closure_set(x_949, 3, x_3); +lean_closure_set(x_949, 4, x_4); +lean_closure_set(x_949, 5, x_5); +lean_closure_set(x_949, 6, x_946); +lean_closure_set(x_949, 7, x_947); +lean_closure_set(x_949, 8, x_2); +lean_closure_set(x_949, 9, x_948); +x_950 = l_Lean_Elab_Term_observing___rarg(x_949, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_950) == 0) +{ uint8_t x_951; -x_951 = l_Array_isEmpty___rarg(x_3); +x_951 = !lean_is_exclusive(x_950); if (x_951 == 0) { -lean_object* x_952; lean_object* x_953; lean_object* x_954; lean_object* x_955; lean_object* x_956; lean_object* x_957; lean_object* x_958; -x_952 = lean_box(0); -x_953 = lean_box(x_932); -x_954 = lean_box(x_6); -x_955 = lean_box(x_7); -x_956 = lean_box(x_8); -x_957 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_957, 0, x_1); -lean_closure_set(x_957, 1, x_952); -lean_closure_set(x_957, 2, x_953); -lean_closure_set(x_957, 3, x_3); -lean_closure_set(x_957, 4, x_4); -lean_closure_set(x_957, 5, x_5); -lean_closure_set(x_957, 6, x_954); -lean_closure_set(x_957, 7, x_955); -lean_closure_set(x_957, 8, x_2); -lean_closure_set(x_957, 9, x_956); -x_958 = l_Lean_Elab_Term_observing___rarg(x_957, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_958) == 0) -{ -uint8_t x_959; -x_959 = !lean_is_exclusive(x_958); -if (x_959 == 0) -{ -lean_object* x_960; lean_object* x_961; -x_960 = lean_ctor_get(x_958, 0); -x_961 = lean_array_push(x_9, x_960); -lean_ctor_set(x_958, 0, x_961); -return x_958; -} -else -{ -lean_object* x_962; lean_object* x_963; lean_object* x_964; lean_object* x_965; -x_962 = lean_ctor_get(x_958, 0); -x_963 = lean_ctor_get(x_958, 1); -lean_inc(x_963); -lean_inc(x_962); -lean_dec(x_958); -x_964 = lean_array_push(x_9, x_962); -x_965 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_965, 0, x_964); -lean_ctor_set(x_965, 1, x_963); -return x_965; -} -} -else -{ -uint8_t x_966; +lean_object* x_952; lean_object* x_953; +x_952 = lean_ctor_get(x_950, 0); +x_953 = lean_array_push(x_9, x_952); +lean_ctor_set(x_950, 0, x_953); +return x_950; +} +else +{ +lean_object* x_954; lean_object* x_955; lean_object* x_956; lean_object* x_957; +x_954 = lean_ctor_get(x_950, 0); +x_955 = lean_ctor_get(x_950, 1); +lean_inc(x_955); +lean_inc(x_954); +lean_dec(x_950); +x_956 = lean_array_push(x_9, x_954); +x_957 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_957, 0, x_956); +lean_ctor_set(x_957, 1, x_955); +return x_957; +} +} +else +{ +uint8_t x_958; lean_dec(x_9); -x_966 = !lean_is_exclusive(x_958); -if (x_966 == 0) +x_958 = !lean_is_exclusive(x_950); +if (x_958 == 0) { -return x_958; +return x_950; } else { -lean_object* x_967; lean_object* x_968; lean_object* x_969; -x_967 = lean_ctor_get(x_958, 0); -x_968 = lean_ctor_get(x_958, 1); -lean_inc(x_968); -lean_inc(x_967); -lean_dec(x_958); -x_969 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_969, 0, x_967); -lean_ctor_set(x_969, 1, x_968); -return x_969; +lean_object* x_959; lean_object* x_960; lean_object* x_961; +x_959 = lean_ctor_get(x_950, 0); +x_960 = lean_ctor_get(x_950, 1); +lean_inc(x_960); +lean_inc(x_959); +lean_dec(x_950); +x_961 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_961, 0, x_959); +lean_ctor_set(x_961, 1, x_960); +return x_961; } } } else { +uint8_t x_962; +x_962 = l_Array_isEmpty___rarg(x_4); +if (x_962 == 0) +{ +lean_object* x_963; lean_object* x_964; lean_object* x_965; lean_object* x_966; lean_object* x_967; lean_object* x_968; lean_object* x_969; +x_963 = lean_box(0); +x_964 = lean_box(x_924); +x_965 = lean_box(x_6); +x_966 = lean_box(x_7); +x_967 = lean_box(x_8); +x_968 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); +lean_closure_set(x_968, 0, x_1); +lean_closure_set(x_968, 1, x_963); +lean_closure_set(x_968, 2, x_964); +lean_closure_set(x_968, 3, x_3); +lean_closure_set(x_968, 4, x_4); +lean_closure_set(x_968, 5, x_5); +lean_closure_set(x_968, 6, x_965); +lean_closure_set(x_968, 7, x_966); +lean_closure_set(x_968, 8, x_2); +lean_closure_set(x_968, 9, x_967); +x_969 = l_Lean_Elab_Term_observing___rarg(x_968, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_969) == 0) +{ uint8_t x_970; -x_970 = l_Array_isEmpty___rarg(x_4); +x_970 = !lean_is_exclusive(x_969); if (x_970 == 0) { -lean_object* x_971; lean_object* x_972; lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; lean_object* x_977; -x_971 = lean_box(0); -x_972 = lean_box(x_932); -x_973 = lean_box(x_6); -x_974 = lean_box(x_7); -x_975 = lean_box(x_8); -x_976 = lean_alloc_closure((void*)(l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___lambda__1___boxed), 17, 10); -lean_closure_set(x_976, 0, x_1); -lean_closure_set(x_976, 1, x_971); -lean_closure_set(x_976, 2, x_972); -lean_closure_set(x_976, 3, x_3); -lean_closure_set(x_976, 4, x_4); -lean_closure_set(x_976, 5, x_5); -lean_closure_set(x_976, 6, x_973); -lean_closure_set(x_976, 7, x_974); -lean_closure_set(x_976, 8, x_2); -lean_closure_set(x_976, 9, x_975); -x_977 = l_Lean_Elab_Term_observing___rarg(x_976, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_977) == 0) -{ -uint8_t x_978; -x_978 = !lean_is_exclusive(x_977); -if (x_978 == 0) -{ -lean_object* x_979; lean_object* x_980; -x_979 = lean_ctor_get(x_977, 0); -x_980 = lean_array_push(x_9, x_979); -lean_ctor_set(x_977, 0, x_980); -return x_977; -} -else -{ -lean_object* x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; -x_981 = lean_ctor_get(x_977, 0); -x_982 = lean_ctor_get(x_977, 1); -lean_inc(x_982); -lean_inc(x_981); -lean_dec(x_977); -x_983 = lean_array_push(x_9, x_981); -x_984 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_984, 0, x_983); -lean_ctor_set(x_984, 1, x_982); -return x_984; -} -} -else -{ -uint8_t x_985; +lean_object* x_971; lean_object* x_972; +x_971 = lean_ctor_get(x_969, 0); +x_972 = lean_array_push(x_9, x_971); +lean_ctor_set(x_969, 0, x_972); +return x_969; +} +else +{ +lean_object* x_973; lean_object* x_974; lean_object* x_975; lean_object* x_976; +x_973 = lean_ctor_get(x_969, 0); +x_974 = lean_ctor_get(x_969, 1); +lean_inc(x_974); +lean_inc(x_973); +lean_dec(x_969); +x_975 = lean_array_push(x_9, x_973); +x_976 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_976, 0, x_975); +lean_ctor_set(x_976, 1, x_974); +return x_976; +} +} +else +{ +uint8_t x_977; lean_dec(x_9); -x_985 = !lean_is_exclusive(x_977); -if (x_985 == 0) +x_977 = !lean_is_exclusive(x_969); +if (x_977 == 0) { -return x_977; +return x_969; } else { -lean_object* x_986; lean_object* x_987; lean_object* x_988; -x_986 = lean_ctor_get(x_977, 0); -x_987 = lean_ctor_get(x_977, 1); -lean_inc(x_987); -lean_inc(x_986); -lean_dec(x_977); -x_988 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_988, 0, x_986); -lean_ctor_set(x_988, 1, x_987); -return x_988; +lean_object* x_978; lean_object* x_979; lean_object* x_980; +x_978 = lean_ctor_get(x_969, 0); +x_979 = lean_ctor_get(x_969, 1); +lean_inc(x_979); +lean_inc(x_978); +lean_dec(x_969); +x_980 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_980, 0, x_978); +lean_ctor_set(x_980, 1, x_979); +return x_980; } } } @@ -61633,129 +62112,129 @@ lean_dec(x_3); lean_dec(x_2); if (x_8 == 0) { -uint8_t x_989; lean_object* x_990; lean_object* x_991; lean_object* x_992; lean_object* x_993; -x_989 = 1; -x_990 = lean_box(x_989); -x_991 = lean_box(x_989); -x_992 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); -lean_closure_set(x_992, 0, x_1); -lean_closure_set(x_992, 1, x_5); -lean_closure_set(x_992, 2, x_990); -lean_closure_set(x_992, 3, x_991); -x_993 = l_Lean_Elab_Term_observing___rarg(x_992, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_993) == 0) +uint8_t x_981; lean_object* x_982; lean_object* x_983; lean_object* x_984; lean_object* x_985; +x_981 = 1; +x_982 = lean_box(x_981); +x_983 = lean_box(x_981); +x_984 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTerm___boxed), 11, 4); +lean_closure_set(x_984, 0, x_1); +lean_closure_set(x_984, 1, x_5); +lean_closure_set(x_984, 2, x_982); +lean_closure_set(x_984, 3, x_983); +x_985 = l_Lean_Elab_Term_observing___rarg(x_984, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_985) == 0) { -uint8_t x_994; -x_994 = !lean_is_exclusive(x_993); -if (x_994 == 0) +uint8_t x_986; +x_986 = !lean_is_exclusive(x_985); +if (x_986 == 0) { -lean_object* x_995; lean_object* x_996; -x_995 = lean_ctor_get(x_993, 0); -x_996 = lean_array_push(x_9, x_995); -lean_ctor_set(x_993, 0, x_996); -return x_993; +lean_object* x_987; lean_object* x_988; +x_987 = lean_ctor_get(x_985, 0); +x_988 = lean_array_push(x_9, x_987); +lean_ctor_set(x_985, 0, x_988); +return x_985; } else { -lean_object* x_997; lean_object* x_998; lean_object* x_999; lean_object* x_1000; -x_997 = lean_ctor_get(x_993, 0); -x_998 = lean_ctor_get(x_993, 1); -lean_inc(x_998); -lean_inc(x_997); -lean_dec(x_993); -x_999 = lean_array_push(x_9, x_997); -x_1000 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1000, 0, x_999); -lean_ctor_set(x_1000, 1, x_998); -return x_1000; +lean_object* x_989; lean_object* x_990; lean_object* x_991; lean_object* x_992; +x_989 = lean_ctor_get(x_985, 0); +x_990 = lean_ctor_get(x_985, 1); +lean_inc(x_990); +lean_inc(x_989); +lean_dec(x_985); +x_991 = lean_array_push(x_9, x_989); +x_992 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_992, 0, x_991); +lean_ctor_set(x_992, 1, x_990); +return x_992; } } else { -uint8_t x_1001; +uint8_t x_993; lean_dec(x_9); -x_1001 = !lean_is_exclusive(x_993); -if (x_1001 == 0) +x_993 = !lean_is_exclusive(x_985); +if (x_993 == 0) { -return x_993; +return x_985; } else { -lean_object* x_1002; lean_object* x_1003; lean_object* x_1004; -x_1002 = lean_ctor_get(x_993, 0); -x_1003 = lean_ctor_get(x_993, 1); -lean_inc(x_1003); -lean_inc(x_1002); -lean_dec(x_993); -x_1004 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1004, 0, x_1002); -lean_ctor_set(x_1004, 1, x_1003); -return x_1004; +lean_object* x_994; lean_object* x_995; lean_object* x_996; +x_994 = lean_ctor_get(x_985, 0); +x_995 = lean_ctor_get(x_985, 1); +lean_inc(x_995); +lean_inc(x_994); +lean_dec(x_985); +x_996 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_996, 0, x_994); +lean_ctor_set(x_996, 1, x_995); +return x_996; } } } else { -lean_object* x_1005; uint8_t x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; lean_object* x_1010; -x_1005 = lean_box(0); -x_1006 = 1; -x_1007 = lean_box(x_932); -x_1008 = lean_box(x_1006); -x_1009 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); -lean_closure_set(x_1009, 0, x_1); -lean_closure_set(x_1009, 1, x_5); -lean_closure_set(x_1009, 2, x_1007); -lean_closure_set(x_1009, 3, x_1008); -lean_closure_set(x_1009, 4, x_1005); -x_1010 = l_Lean_Elab_Term_observing___rarg(x_1009, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_1010) == 0) +lean_object* x_997; uint8_t x_998; lean_object* x_999; lean_object* x_1000; lean_object* x_1001; lean_object* x_1002; +x_997 = lean_box(0); +x_998 = 1; +x_999 = lean_box(x_924); +x_1000 = lean_box(x_998); +x_1001 = lean_alloc_closure((void*)(l_Lean_Elab_Term_elabTermEnsuringType___boxed), 12, 5); +lean_closure_set(x_1001, 0, x_1); +lean_closure_set(x_1001, 1, x_5); +lean_closure_set(x_1001, 2, x_999); +lean_closure_set(x_1001, 3, x_1000); +lean_closure_set(x_1001, 4, x_997); +x_1002 = l_Lean_Elab_Term_observing___rarg(x_1001, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_1002) == 0) { -uint8_t x_1011; -x_1011 = !lean_is_exclusive(x_1010); -if (x_1011 == 0) +uint8_t x_1003; +x_1003 = !lean_is_exclusive(x_1002); +if (x_1003 == 0) { -lean_object* x_1012; lean_object* x_1013; -x_1012 = lean_ctor_get(x_1010, 0); -x_1013 = lean_array_push(x_9, x_1012); -lean_ctor_set(x_1010, 0, x_1013); -return x_1010; +lean_object* x_1004; lean_object* x_1005; +x_1004 = lean_ctor_get(x_1002, 0); +x_1005 = lean_array_push(x_9, x_1004); +lean_ctor_set(x_1002, 0, x_1005); +return x_1002; } else { -lean_object* x_1014; lean_object* x_1015; lean_object* x_1016; lean_object* x_1017; -x_1014 = lean_ctor_get(x_1010, 0); -x_1015 = lean_ctor_get(x_1010, 1); -lean_inc(x_1015); -lean_inc(x_1014); -lean_dec(x_1010); -x_1016 = lean_array_push(x_9, x_1014); -x_1017 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1017, 0, x_1016); -lean_ctor_set(x_1017, 1, x_1015); -return x_1017; +lean_object* x_1006; lean_object* x_1007; lean_object* x_1008; lean_object* x_1009; +x_1006 = lean_ctor_get(x_1002, 0); +x_1007 = lean_ctor_get(x_1002, 1); +lean_inc(x_1007); +lean_inc(x_1006); +lean_dec(x_1002); +x_1008 = lean_array_push(x_9, x_1006); +x_1009 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1009, 0, x_1008); +lean_ctor_set(x_1009, 1, x_1007); +return x_1009; } } else { -uint8_t x_1018; +uint8_t x_1010; lean_dec(x_9); -x_1018 = !lean_is_exclusive(x_1010); -if (x_1018 == 0) +x_1010 = !lean_is_exclusive(x_1002); +if (x_1010 == 0) { -return x_1010; +return x_1002; } else { -lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; -x_1019 = lean_ctor_get(x_1010, 0); -x_1020 = lean_ctor_get(x_1010, 1); -lean_inc(x_1020); -lean_inc(x_1019); -lean_dec(x_1010); -x_1021 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1021, 0, x_1019); -lean_ctor_set(x_1021, 1, x_1020); -return x_1021; +lean_object* x_1011; lean_object* x_1012; lean_object* x_1013; +x_1011 = lean_ctor_get(x_1002, 0); +x_1012 = lean_ctor_get(x_1002, 1); +lean_inc(x_1012); +lean_inc(x_1011); +lean_dec(x_1002); +x_1013 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1013, 0, x_1011); +lean_ctor_set(x_1013, 1, x_1012); +return x_1013; } } } @@ -61766,55 +62245,55 @@ return x_1021; } else { -lean_object* x_1025; lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; lean_object* x_1029; -x_1025 = lean_box(0); -x_1026 = l_Lean_Syntax_identComponents(x_926, x_1025); -x_1027 = lean_box(0); -x_1028 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__5(x_1, x_1026, x_1027); -x_1029 = l_List_appendTR___rarg(x_1028, x_2); -x_1 = x_924; -x_2 = x_1029; +lean_object* x_1017; lean_object* x_1018; lean_object* x_1019; lean_object* x_1020; lean_object* x_1021; +x_1017 = lean_box(0); +x_1018 = l_Lean_Syntax_identComponents(x_918, x_1017); +x_1019 = lean_box(0); +x_1020 = l_List_mapTR_loop___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__5(x_1, x_1018, x_1019); +x_1021 = l_List_appendTR___rarg(x_1020, x_2); +x_1 = x_916; +x_2 = x_1021; goto _start; } } else { -lean_object* x_1031; +lean_object* x_1023; lean_dec(x_1); -x_1031 = l_Lean_Syntax_isFieldIdx_x3f(x_926); -if (lean_obj_tag(x_1031) == 0) +x_1023 = l_Lean_Syntax_isFieldIdx_x3f(x_918); +if (lean_obj_tag(x_1023) == 0) { -lean_object* x_1032; lean_object* x_1033; -lean_dec(x_926); -lean_dec(x_924); +lean_object* x_1024; lean_object* x_1025; +lean_dec(x_918); +lean_dec(x_916); lean_dec(x_9); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_1032 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; -x_1033 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_1032, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_1024 = l___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___closed__24; +x_1025 = l_Lean_throwError___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__1(x_1024, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -return x_1033; -} -else -{ -lean_object* x_1034; lean_object* x_1035; lean_object* x_1036; -x_1034 = lean_ctor_get(x_1031, 0); -lean_inc(x_1034); -lean_dec(x_1031); -x_1035 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1035, 0, x_926); -lean_ctor_set(x_1035, 1, x_1034); -x_1036 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_1036, 0, x_1035); -lean_ctor_set(x_1036, 1, x_2); -x_1 = x_924; -x_2 = x_1036; +return x_1025; +} +else +{ +lean_object* x_1026; lean_object* x_1027; lean_object* x_1028; +x_1026 = lean_ctor_get(x_1023, 0); +lean_inc(x_1026); +lean_dec(x_1023); +x_1027 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1027, 0, x_918); +lean_ctor_set(x_1027, 1, x_1026); +x_1028 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_1028, 0, x_1027); +lean_ctor_set(x_1028, 1, x_2); +x_1 = x_916; +x_2 = x_1028; goto _start; } } @@ -61822,17 +62301,17 @@ goto _start; } else { -lean_object* x_1038; lean_object* x_1039; lean_object* x_1040; uint8_t x_1041; -x_1038 = l_Lean_Syntax_getArgs(x_1); +lean_object* x_1030; lean_object* x_1031; lean_object* x_1032; uint8_t x_1033; +x_1030 = l_Lean_Syntax_getArgs(x_1); lean_dec(x_1); -x_1039 = lean_array_get_size(x_1038); -x_1040 = lean_unsigned_to_nat(0u); -x_1041 = lean_nat_dec_lt(x_1040, x_1039); -if (x_1041 == 0) -{ -lean_object* x_1042; -lean_dec(x_1039); -lean_dec(x_1038); +x_1031 = lean_array_get_size(x_1030); +x_1032 = lean_unsigned_to_nat(0u); +x_1033 = lean_nat_dec_lt(x_1032, x_1031); +if (x_1033 == 0) +{ +lean_object* x_1034; +lean_dec(x_1031); +lean_dec(x_1030); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -61843,27 +62322,27 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_1042 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1042, 0, x_9); -lean_ctor_set(x_1042, 1, x_16); -return x_1042; +x_1034 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1034, 0, x_9); +lean_ctor_set(x_1034, 1, x_16); +return x_1034; } else { -uint8_t x_1043; -x_1043 = !lean_is_exclusive(x_10); -if (x_1043 == 0) +uint8_t x_1035; +x_1035 = !lean_is_exclusive(x_10); +if (x_1035 == 0) { -uint8_t x_1044; uint8_t x_1045; -x_1044 = 0; -lean_ctor_set_uint8(x_10, sizeof(void*)*9 + 1, x_1044); -x_1045 = lean_nat_dec_le(x_1039, x_1039); -if (x_1045 == 0) +uint8_t x_1036; uint8_t x_1037; +x_1036 = 0; +lean_ctor_set_uint8(x_10, sizeof(void*)*9 + 1, x_1036); +x_1037 = lean_nat_dec_le(x_1031, x_1031); +if (x_1037 == 0) { -lean_object* x_1046; +lean_object* x_1038; lean_dec(x_10); -lean_dec(x_1039); -lean_dec(x_1038); +lean_dec(x_1031); +lean_dec(x_1030); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -61873,83 +62352,83 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_1046 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1046, 0, x_9); -lean_ctor_set(x_1046, 1, x_16); -return x_1046; -} -else -{ -size_t x_1047; size_t x_1048; lean_object* x_1049; -x_1047 = 0; -x_1048 = lean_usize_of_nat(x_1039); -lean_dec(x_1039); -x_1049 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_1038, x_1047, x_1048, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_1038); -return x_1049; -} -} -else -{ -lean_object* x_1050; lean_object* x_1051; lean_object* x_1052; uint8_t x_1053; uint8_t x_1054; lean_object* x_1055; lean_object* x_1056; lean_object* x_1057; lean_object* x_1058; uint8_t x_1059; uint8_t x_1060; uint8_t x_1061; uint8_t x_1062; uint8_t x_1063; lean_object* x_1064; lean_object* x_1065; uint8_t x_1066; uint8_t x_1067; uint8_t x_1068; uint8_t x_1069; lean_object* x_1070; uint8_t x_1071; -x_1050 = lean_ctor_get(x_10, 0); -x_1051 = lean_ctor_get(x_10, 1); -x_1052 = lean_ctor_get(x_10, 2); -x_1053 = lean_ctor_get_uint8(x_10, sizeof(void*)*9); -x_1054 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 2); -x_1055 = lean_ctor_get(x_10, 3); -x_1056 = lean_ctor_get(x_10, 4); -x_1057 = lean_ctor_get(x_10, 5); -x_1058 = lean_ctor_get(x_10, 6); -x_1059 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 3); -x_1060 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 4); -x_1061 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 5); -x_1062 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 6); -x_1063 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 7); -x_1064 = lean_ctor_get(x_10, 7); -x_1065 = lean_ctor_get(x_10, 8); -x_1066 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 8); -x_1067 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 9); -x_1068 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 10); -lean_inc(x_1065); -lean_inc(x_1064); -lean_inc(x_1058); +x_1038 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1038, 0, x_9); +lean_ctor_set(x_1038, 1, x_16); +return x_1038; +} +else +{ +size_t x_1039; size_t x_1040; lean_object* x_1041; +x_1039 = 0; +x_1040 = lean_usize_of_nat(x_1031); +lean_dec(x_1031); +x_1041 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_1030, x_1039, x_1040, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_1030); +return x_1041; +} +} +else +{ +lean_object* x_1042; lean_object* x_1043; lean_object* x_1044; uint8_t x_1045; uint8_t x_1046; lean_object* x_1047; lean_object* x_1048; lean_object* x_1049; lean_object* x_1050; uint8_t x_1051; uint8_t x_1052; uint8_t x_1053; uint8_t x_1054; uint8_t x_1055; lean_object* x_1056; lean_object* x_1057; uint8_t x_1058; uint8_t x_1059; uint8_t x_1060; uint8_t x_1061; lean_object* x_1062; uint8_t x_1063; +x_1042 = lean_ctor_get(x_10, 0); +x_1043 = lean_ctor_get(x_10, 1); +x_1044 = lean_ctor_get(x_10, 2); +x_1045 = lean_ctor_get_uint8(x_10, sizeof(void*)*9); +x_1046 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 2); +x_1047 = lean_ctor_get(x_10, 3); +x_1048 = lean_ctor_get(x_10, 4); +x_1049 = lean_ctor_get(x_10, 5); +x_1050 = lean_ctor_get(x_10, 6); +x_1051 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 3); +x_1052 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 4); +x_1053 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 5); +x_1054 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 6); +x_1055 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 7); +x_1056 = lean_ctor_get(x_10, 7); +x_1057 = lean_ctor_get(x_10, 8); +x_1058 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 8); +x_1059 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 9); +x_1060 = lean_ctor_get_uint8(x_10, sizeof(void*)*9 + 10); lean_inc(x_1057); lean_inc(x_1056); -lean_inc(x_1055); -lean_inc(x_1052); -lean_inc(x_1051); lean_inc(x_1050); +lean_inc(x_1049); +lean_inc(x_1048); +lean_inc(x_1047); +lean_inc(x_1044); +lean_inc(x_1043); +lean_inc(x_1042); lean_dec(x_10); -x_1069 = 0; -x_1070 = lean_alloc_ctor(0, 9, 11); -lean_ctor_set(x_1070, 0, x_1050); -lean_ctor_set(x_1070, 1, x_1051); -lean_ctor_set(x_1070, 2, x_1052); -lean_ctor_set(x_1070, 3, x_1055); -lean_ctor_set(x_1070, 4, x_1056); -lean_ctor_set(x_1070, 5, x_1057); -lean_ctor_set(x_1070, 6, x_1058); -lean_ctor_set(x_1070, 7, x_1064); -lean_ctor_set(x_1070, 8, x_1065); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9, x_1053); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 1, x_1069); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 2, x_1054); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 3, x_1059); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 4, x_1060); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 5, x_1061); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 6, x_1062); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 7, x_1063); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 8, x_1066); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 9, x_1067); -lean_ctor_set_uint8(x_1070, sizeof(void*)*9 + 10, x_1068); -x_1071 = lean_nat_dec_le(x_1039, x_1039); -if (x_1071 == 0) -{ -lean_object* x_1072; -lean_dec(x_1070); -lean_dec(x_1039); -lean_dec(x_1038); +x_1061 = 0; +x_1062 = lean_alloc_ctor(0, 9, 11); +lean_ctor_set(x_1062, 0, x_1042); +lean_ctor_set(x_1062, 1, x_1043); +lean_ctor_set(x_1062, 2, x_1044); +lean_ctor_set(x_1062, 3, x_1047); +lean_ctor_set(x_1062, 4, x_1048); +lean_ctor_set(x_1062, 5, x_1049); +lean_ctor_set(x_1062, 6, x_1050); +lean_ctor_set(x_1062, 7, x_1056); +lean_ctor_set(x_1062, 8, x_1057); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9, x_1045); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 1, x_1061); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 2, x_1046); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 3, x_1051); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 4, x_1052); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 5, x_1053); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 6, x_1054); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 7, x_1055); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 8, x_1058); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 9, x_1059); +lean_ctor_set_uint8(x_1062, sizeof(void*)*9 + 10, x_1060); +x_1063 = lean_nat_dec_le(x_1031, x_1031); +if (x_1063 == 0) +{ +lean_object* x_1064; +lean_dec(x_1062); +lean_dec(x_1031); +lean_dec(x_1030); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -61959,20 +62438,20 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_1072 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_1072, 0, x_9); -lean_ctor_set(x_1072, 1, x_16); -return x_1072; +x_1064 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_1064, 0, x_9); +lean_ctor_set(x_1064, 1, x_16); +return x_1064; } else { -size_t x_1073; size_t x_1074; lean_object* x_1075; -x_1073 = 0; -x_1074 = lean_usize_of_nat(x_1039); -lean_dec(x_1039); -x_1075 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_1038, x_1073, x_1074, x_9, x_1070, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_1038); -return x_1075; +size_t x_1065; size_t x_1066; lean_object* x_1067; +x_1065 = 0; +x_1066 = lean_usize_of_nat(x_1031); +lean_dec(x_1031); +x_1067 = l_Array_foldlMUnsafe_fold___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppFn___spec__6(x_2, x_3, x_4, x_5, x_6, x_7, x_1030, x_1065, x_1066, x_9, x_1062, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_1030); +return x_1067; } } } @@ -63294,7 +63773,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__8; x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(1629u); +x_3 = lean_unsigned_to_nat(1632u); x_4 = lean_unsigned_to_nat(57u); x_5 = l_Lean_Elab_Term_elabAppArgs_elabAsElim_x3f___lambda__1___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -63366,7 +63845,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__8; x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_mergeFailures___spec__2___closed__1; -x_3 = lean_unsigned_to_nat(1630u); +x_3 = lean_unsigned_to_nat(1633u); x_4 = lean_unsigned_to_nat(84u); x_5 = l_Lean_Elab_Term_elabAppArgs_elabAsElim_x3f___lambda__1___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -65336,7 +65815,7 @@ static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0_ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Elab_Term_ElabElim_finalize___lambda__9___closed__8; x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Elab_App_0__Lean_Elab_Term_elabAppAux___spec__5___closed__1; -x_3 = lean_unsigned_to_nat(1654u); +x_3 = lean_unsigned_to_nat(1657u); x_4 = lean_unsigned_to_nat(21u); x_5 = l_Lean_Elab_Term_elabAppArgs_elabAsElim_x3f___lambda__1___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -68083,7 +68562,7 @@ x_4 = l_Lean_addBuiltinDeclarationRanges(x_2, x_3, x_1); return x_4; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -68093,7 +68572,7 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -68103,27 +68582,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2; x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_4____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3; x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_4____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5() { _start: { lean_object* x_1; @@ -68131,17 +68610,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7() { _start: { lean_object* x_1; @@ -68149,37 +68628,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8; x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_4____closed__3; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9; x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_4____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11() { _start: { lean_object* x_1; @@ -68187,17 +68666,17 @@ x_1 = lean_mk_string_unchecked("App", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13() { _start: { lean_object* x_1; @@ -68205,33 +68684,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13; +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15() { +static lean_object* _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14; -x_2 = lean_unsigned_to_nat(24880u); +x_1 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14; +x_2 = lean_unsigned_to_nat(24906u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1; +x_2 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1; x_3 = 0; -x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15; +x_4 = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -69368,37 +69847,37 @@ lean_mark_persistent(l___regBuiltin_Lean_Elab_Term_elabProj_declRange__1___close if (builtin) {res = l___regBuiltin_Lean_Elab_Term_elabProj_declRange__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__1); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__2); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__3); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__4); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__5); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__6); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__7); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__8); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__9); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__10); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__11); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__12); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__13); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__14); -l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15(); -lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880____closed__15); -if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24880_(lean_io_mk_world()); +}l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__1); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__2); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__3); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__4); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__5); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__6); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__7); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__8); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__9); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__10); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__11); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__12); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__13); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__14); +l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15 = _init_l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15(); +lean_mark_persistent(l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906____closed__15); +if (builtin) {res = l_Lean_Elab_Term_initFn____x40_Lean_Elab_App___hyg_24906_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Import.c b/stage0/stdlib/Lean/Elab/Import.c index 7e6ca2489e66..e63b9ec665c8 100644 --- a/stage0/stdlib/Lean/Elab/Import.c +++ b/stage0/stdlib/Lean/Elab/Import.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.Import -// Imports: Lean.Parser.Module Lean.Data.Json +// Imports: Lean.Parser.Module Lean.Util.Paths #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,6 +14,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_IO_println___at_Lean_Elab_printImports___spec__1(lean_object*, lean_object*); +lean_object* l_Lean_initSrcSearchPath(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_headerToImports___boxed(lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_processHeader___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -27,6 +28,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_processHeader(lean_object*, lean_object*, l static lean_object* l_Lean_Elab_headerToImports___closed__2; lean_object* lean_string_push(lean_object*, uint32_t); lean_object* l_Lean_MessageData_ofFormat(lean_object*); +LEAN_EXPORT lean_object* lean_print_import_srcs(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_mkInputContext(lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImports___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* l_IO_print___at_IO_println___spec__1(lean_object*, lean_object*); @@ -35,6 +37,7 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_headerToImports___closed__1; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l_Lean_Elab_headerToImports___closed__4; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImports___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_processHeader___closed__1; @@ -44,10 +47,12 @@ lean_object* l_Lean_findOLean(lean_object*, lean_object*); static lean_object* l_Lean_Elab_headerToImports___closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_parseImports(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); size_t lean_usize_add(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +lean_object* l_Lean_findLean(lean_object*, lean_object*, lean_object*); lean_object* lean_io_error_to_string(lean_object*); static lean_object* l_Lean_Elab_headerToImports___closed__5; lean_object* l_Lean_Parser_parseHeader(lean_object*, lean_object*); @@ -1082,8 +1087,250 @@ lean_dec(x_1); return x_10; } } +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_6, x_5); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_1); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_7); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +lean_dec(x_7); +x_11 = lean_array_uget(x_4, x_6); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +lean_dec(x_11); +lean_inc(x_1); +x_13 = l_Lean_findLean(x_1, x_12, x_8); +lean_dec(x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_IO_println___at_Lean_Elab_printImports___spec__1(x_14, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; size_t x_18; size_t x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = 1; +x_19 = lean_usize_add(x_6, x_18); +x_20 = lean_box(0); +x_6 = x_19; +x_7 = x_20; +x_8 = x_17; +goto _start; +} +else +{ +uint8_t x_22; +lean_dec(x_1); +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +return x_16; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_16, 0); +x_24 = lean_ctor_get(x_16, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_16); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +} +else +{ +uint8_t x_26; +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_13); +if (x_26 == 0) +{ +return x_13; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_13, 0); +x_28 = lean_ctor_get(x_13, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_13); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +} +LEAN_EXPORT lean_object* lean_print_import_srcs(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_box(0); +x_5 = l_Lean_initSrcSearchPath(x_4, x_3); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = l_Lean_Elab_parseImports(x_1, x_2, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_box(0); +x_13 = lean_array_size(x_11); +x_14 = 0; +x_15 = lean_box(0); +x_16 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1(x_6, x_11, x_12, x_11, x_13, x_14, x_15, x_10); +lean_dec(x_11); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +lean_ctor_set(x_16, 0, x_15); +return x_16; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) +{ +return x_16; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_16); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +else +{ +uint8_t x_25; +lean_dec(x_6); +x_25 = !lean_is_exclusive(x_8); +if (x_25 == 0) +{ +return x_8; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_8, 0); +x_27 = lean_ctor_get(x_8, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_8); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +else +{ +uint8_t x_29; +lean_dec(x_2); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_5); +if (x_29 == 0) +{ +return x_5; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_5, 0); +x_31 = lean_ctor_get(x_5, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_5); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_10 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_printImportSrcs___spec__1(x_1, x_2, x_3, x_4, x_9, x_10, x_7, x_8); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} lean_object* initialize_Lean_Parser_Module(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_Data_Json(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Util_Paths(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_Import(uint8_t builtin, lean_object* w) { lean_object * res; @@ -1092,7 +1339,7 @@ _G_initialized = true; res = initialize_Lean_Parser_Module(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Lean_Data_Json(builtin, lean_io_mk_world()); +res = initialize_Lean_Util_Paths(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); l_Lean_Elab_headerToImports___closed__1 = _init_l_Lean_Elab_headerToImports___closed__1(); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Attr.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Attr.c index 5ffb3c45fb00..fcb33277724a 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Attr.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Attr.c @@ -13,11 +13,9 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__2___closed__1; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_56____closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__14; @@ -31,9 +29,11 @@ lean_object* l_Lean_getConstInfo___at_Lean_Compiler_initFn____x40_Lean_Compiler_ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__13; lean_object* l___private_Lean_Elab_Tactic_Config_0__Lean_Elab_Tactic_elabConfig(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6; lean_object* l_Lean_ConstantInfo_type(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___closed__4; lean_object* l_Lean_indentD(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2; uint8_t l_Lean_Exception_isInterrupt(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__24; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1___closed__1; @@ -45,29 +45,29 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig lean_object* l_Lean_replaceRef(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__16; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_intToBitVecExt; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__7; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__7; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__15; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740_(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_56____closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4; uint8_t lean_string_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6; lean_object* l_Lean_Exception_toMessageData(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_addBVNormalizeProcBuiltinAttr(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__2; lean_object* l_Lean_Level_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_107____closed__4; uint8_t l_Lean_Expr_hasSyntheticSorry(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_Tactic_getConfigItems(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -78,52 +78,55 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_evalUnsafe____x40_Lean_ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_714_(lean_object*); lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Option_register___at_Lean_initFn____x40_Lean_Util_Trace___hyg_1552____spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2; lean_object* l_Lean_declareBuiltin(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__11; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__9; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__22; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__12; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getKind(lean_object*); lean_object* l_Lean_Elab_getBetterRef(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__19; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5; lean_object* l_Lean_Meta_DiscrTree_empty(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_56____closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_714____closed__4; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__13; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_addMacroStack___at_Lean_Elab_Term_instAddErrorMessageContextTermElabM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__18; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__20; lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__11; lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_evalUnsafe____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_145____boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766_(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__25; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__19; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_107_(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__9; lean_object* l___private_Lean_Elab_Tactic_Config_0__Lean_Elab_Tactic_mkConfigItemViews(lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801_(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1___closed__5; uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -134,8 +137,11 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__1; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__4; lean_object* l_Lean_Meta_Simp_registerSimprocAttr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2; lean_object* l_Lean_Meta_registerSimpAttr(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__1; @@ -143,14 +149,15 @@ uint8_t l_Lean_Environment_contains(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__1___closed__3; lean_object* l_Lean_MessageData_ofExpr(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3; lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__26; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201_(lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_714____closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__27; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7; lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Elab_Term_synthesizeInstMVarCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_evalUnsafe____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_145_(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -159,14 +166,13 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_107____closed__6; lean_object* l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__3; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_isNone(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_addBVNormalizeProcBuiltinAttr___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_107____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__1; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__3; @@ -188,9 +194,12 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab lean_object* l_Lean_Meta_evalExpr_x27___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__5; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__15; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -198,15 +207,13 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_sat_solver; uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__4___closed__1; static lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_evalUnsafe____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_145____closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1; lean_object* l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__18; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__17; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig___lambda__2___closed__2; uint8_t l_Array_isEmpty___rarg(lean_object*); @@ -1484,7 +1491,7 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lea _start: { lean_object* x_1; -x_1 = l_Lean_Meta_DiscrTree_empty(lean_box(0)); +x_1 = lean_mk_string_unchecked("int_toBitVec", 12, 12); return x_1; } } @@ -1492,7 +1499,66 @@ static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lea _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__1; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("intToBitVecExt", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__10; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__12; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("simp theorems used to convert UIntX/IntX statements into BitVec ones", 68, 68); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4; +x_5 = l_Lean_Meta_registerSimpAttr(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_DiscrTree_empty(lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1; x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; x_3 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_3, 0, x_1); @@ -1502,11 +1568,11 @@ lean_ctor_set(x_3, 3, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2; x_3 = lean_st_mk_ref(x_2, x_1); x_4 = !lean_is_exclusive(x_3); if (x_4 == 0) @@ -1528,7 +1594,7 @@ return x_7; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1() { _start: { lean_object* x_1; @@ -1536,17 +1602,17 @@ x_1 = lean_mk_string_unchecked("bv_normalize_proc", 17, 17); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3() { _start: { lean_object* x_1; @@ -1554,17 +1620,17 @@ x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3; x_2 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5() { _start: { lean_object* x_1; @@ -1572,7 +1638,7 @@ x_1 = lean_mk_string_unchecked("bvNormalizeSimprocExt", 21, 21); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; @@ -1581,12 +1647,12 @@ x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDeci x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__2; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__10; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__12; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7() { _start: { lean_object* x_1; @@ -1594,14 +1660,14 @@ x_1 = lean_mk_string_unchecked("simprocs used by bv_normalize", 29, 29); return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6; x_6 = l_Lean_Meta_Simp_registerSimprocAttr(x_2, x_3, x_4, x_5, x_1); return x_6; } @@ -2047,6 +2113,8 @@ else { uint8_t x_107; lean_dec(x_8); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); x_107 = !lean_is_exclusive(x_10); @@ -2089,6 +2157,8 @@ goto block_99; else { uint8_t x_114; +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); x_114 = !lean_is_exclusive(x_10); @@ -2170,6 +2240,8 @@ lean_dec(x_3); lean_dec(x_1); x_26 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_27 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_26, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_28 = !lean_is_exclusive(x_27); if (x_28 == 0) { @@ -2204,6 +2276,8 @@ lean_dec(x_3); lean_dec(x_1); x_34 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_35 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_34, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_36 = !lean_is_exclusive(x_35); if (x_36 == 0) { @@ -2237,6 +2311,8 @@ lean_dec(x_3); lean_dec(x_1); x_42 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_43 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_42, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_44 = !lean_is_exclusive(x_43); if (x_44 == 0) { @@ -2269,6 +2345,8 @@ lean_dec(x_3); lean_dec(x_1); x_50 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_51 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_50, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_52 = !lean_is_exclusive(x_51); if (x_52 == 0) { @@ -2317,6 +2395,8 @@ lean_dec(x_3); lean_dec(x_1); x_63 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_64 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_63, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_65 = !lean_is_exclusive(x_64); if (x_65 == 0) { @@ -2348,6 +2428,8 @@ lean_dec(x_3); lean_dec(x_1); x_69 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_70 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_69, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_71 = !lean_is_exclusive(x_70); if (x_71 == 0) { @@ -2378,6 +2460,8 @@ lean_dec(x_3); lean_dec(x_1); x_75 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_76 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_75, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_77 = !lean_is_exclusive(x_76); if (x_77 == 0) { @@ -2407,6 +2491,8 @@ lean_dec(x_3); lean_dec(x_1); x_81 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_82 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_81, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_83 = !lean_is_exclusive(x_82); if (x_83 == 0) { @@ -2435,6 +2521,8 @@ lean_dec(x_3); lean_dec(x_1); x_87 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_88 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_87, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_89 = !lean_is_exclusive(x_88); if (x_89 == 0) { @@ -2463,6 +2551,8 @@ lean_dec(x_3); lean_dec(x_1); x_93 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__2; x_94 = l_Lean_throwError___at___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___spec__1(x_93, x_4, x_5, x_13); +lean_dec(x_5); +lean_dec(x_4); x_95 = !lean_is_exclusive(x_94); if (x_95 == 0) { @@ -2502,8 +2592,6 @@ uint8_t x_8; lean_object* x_9; x_8 = lean_unbox(x_3); lean_dec(x_3); x_9 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___lambda__1(x_1, x_2, x_8, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); return x_9; } } @@ -2512,8 +2600,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__ { lean_object* x_7; x_7 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); return x_7; } @@ -2522,7 +2608,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_addBVNormalizeProc _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3; x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_5, x_1, x_2, x_3, x_4); return x_6; } @@ -2537,7 +2623,7 @@ x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_addBVNormalizeProcBuiltinAttr(x_1, x_ return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1() { _start: { lean_object* x_1; @@ -2545,7 +2631,7 @@ x_1 = lean_mk_string_unchecked("addBVNormalizeProcBuiltinAttr", 29, 29); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; @@ -2554,21 +2640,21 @@ x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDeci x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__2; x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__10; x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__12; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; -x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2; +x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2; x_8 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin(x_1, x_2, x_7, x_4, x_5, x_6); return x_8; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1() { _start: { lean_object* x_1; @@ -2576,35 +2662,35 @@ x_1 = lean_mk_string_unchecked("Not implemented yet, [-builtin_bv_normalize_proc return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2; x_6 = l_Lean_throwError___at_Lean_Attribute_Builtin_ensureNoArgs___spec__2(x_5, x_2, x_3, x_4); return x_6; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_7____closed__26; -x_2 = lean_unsigned_to_nat(1175u); +x_2 = lean_unsigned_to_nat(1201u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2() { _start: { lean_object* x_1; @@ -2612,17 +2698,17 @@ x_1 = lean_mk_string_unchecked("bvNormalizeProcBuiltinAttr", 26, 26); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4() { _start: { lean_object* x_1; @@ -2630,13 +2716,13 @@ x_1 = lean_mk_string_unchecked("Builtin bv_normalize simproc", 28, 28); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -2646,29 +2732,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___boxed), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___boxed), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -2676,33 +2762,31 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2(x_1, x_2, x_3, x_4); +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2(x_1, x_2, x_3, x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); @@ -2858,26 +2942,41 @@ lean_dec_ref(res); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740____closed__5); if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_740_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; +l_Lean_Elab_Tactic_BVDecide_Frontend_intToBitVecExt = lean_io_result_get_value(res); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_intToBitVecExt); +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766____closed__2); +if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_766_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef); lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775____closed__7); -if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_775_(lean_io_mk_world()); +}l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801____closed__7); +if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_801_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt); @@ -2938,31 +3037,31 @@ l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide lean_mark_persistent(l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__18); l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__19 = _init_l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__19(); lean_mark_persistent(l___private_Lean_Elab_Tactic_BVDecide_Frontend_Attr_0__Lean_Elab_Tactic_BVDecide_Frontend_addBuiltin___closed__19); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____lambda__2___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175____closed__8); -if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1175_(lean_io_mk_world()); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201____closed__8); +if (builtin) {res = l_Lean_Elab_Tactic_BVDecide_Frontend_initFn____x40_Lean_Elab_Tactic_BVDecide_Frontend_Attr___hyg_1201_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVCheck.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVCheck.c index 825a3dbf8c2e..71a32bc61d5e 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVCheck.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVCheck.c @@ -59,7 +59,6 @@ static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_ev lean_object* l_System_FilePath_parent(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_lratChecker___closed__3; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_getSrcDir___closed__3; -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(lean_object*); lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_bvUnsat___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_bvCheck___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -77,6 +76,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_evalBvCheck___c static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_lratChecker___closed__4; lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_TacticContext_new(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_evalBvCheck___lambda__1___closed__5; +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_evalBvCheck___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_BVCheck_evalBvCheck__1___closed__4; lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1456,7 +1456,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_13; } else @@ -1483,7 +1483,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_20 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_20; } else @@ -1509,7 +1509,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_25 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_25 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_25; } else diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide.c index 4b8b63bc9da7..a2e25c3b22d8 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVDecide.c @@ -352,7 +352,6 @@ static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_evalBvTrace(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_reflectBV___lambda__1___closed__10; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__15___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBoolExpr_go___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__9___closed__6; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_instToExprBoolExpr_go___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__9___closed__29; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_bvUnsat___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -494,6 +493,7 @@ LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Fro static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_LratCert_toReflectionProof___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__8___lambda__3___closed__3; LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___spec__6___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_reconstructCounterExample___spec__8___closed__3; +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_evalBvTrace__1___closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_closeWithBVReflection___spec__10___at_Lean_Elab_Tactic_BVDecide_Frontend_closeWithBVReflection___spec__11(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_lratBitblaster___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -23975,7 +23975,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_13; } else @@ -23999,7 +23999,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_18 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_18 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_18; } else diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVTrace.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVTrace.c index 7f3a59ccb795..ac16b5c1d86e 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVTrace.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/BVTrace.c @@ -58,7 +58,6 @@ lean_object* l_Lean_Elab_Term_getDeclName_x3f(lean_object*, lean_object*, lean_o static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_getLratFileName___closed__4; static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace__1___closed__1; lean_object* l_Std_Tactic_BVDecide_LRAT_loadLRATProof(lean_object*, lean_object*); -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_getLratFileName___closed__1; lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -78,6 +77,7 @@ static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace___c static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace___lambda__2___closed__2; static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace__1___closed__7; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace___closed__2; +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_BVDecide_LRAT_trim_go___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_BVTrace_evalBvTrace___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -611,7 +611,7 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_13; } else @@ -638,7 +638,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_20 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_20 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_20; } else diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize.c index 9b023f704a1a..f88f18e924e4 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize.c +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize -// Imports: Lean.Meta.AppBuilder Lean.Meta.Tactic.AC.Main Lean.Elab.Tactic.Simp Lean.Elab.Tactic.FalseOrByContra Lean.Elab.Tactic.BVDecide.Frontend.Attr Std.Tactic.BVDecide.Normalize Std.Tactic.BVDecide.Syntax +// Imports: Lean.Elab.Tactic.FalseOrByContra Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Simproc Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Rewrite Lean.Elab.Tactic.BVDecide.Frontend.Normalize.AndFlatten Lean.Elab.Tactic.BVDecide.Frontend.Normalize.EmbeddedConstraint Lean.Elab.Tactic.BVDecide.Frontend.Normalize.AC #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,17715 +14,2110 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5; -lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -static lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Simp_Result_getProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023_(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_mkNatLit(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351_(lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_mk_empty_array_with_capacity(lean_object*); -lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5; -extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeExt; -static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3; -lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_mkLt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1; +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3; double lean_float_div(double, double); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1; -lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; -size_t lean_uint64_to_usize(uint64_t); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387_(lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass(lean_object*); -uint8_t l_Lean_Expr_isApp(lean_object*); -lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2; extern lean_object* l_Lean_Elab_Tactic_tacticElabAttribute; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2; -lean_object* lean_array_push(lean_object*, lean_object*); -lean_object* l_Lean_Meta_simpGoal(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1; -lean_object* lean_mk_array(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1; -static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952_(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_getMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821_(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2; uint8_t lean_float_decLt(double, double); -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2; -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2; +static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass; lean_object* lean_io_get_num_heartbeats(lean_object*); uint8_t l_Lean_Syntax_isOfKind(lean_object*, lean_object*); -lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); extern lean_object* l_Lean_trace_profiler_useHeartbeats; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12; -lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6; -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1___boxed(lean_object*); -lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6; -lean_object* l_Lean_Level_ofNat(lean_object*); -LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1; +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6; +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__4; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3; lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3; -size_t lean_usize_of_nat(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6; -lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; -static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2; -uint8_t l_instDecidableNot___rarg(uint8_t); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6; lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2; -lean_object* l_BitVec_neg(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Meta_processPostponed___spec__2___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Meta_sevalSimpExtension; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6; -uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Simp_SimprocExtension_getSimprocs(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_nat_div(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass; lean_object* l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Meta_processPostponed___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_elabBVDecideConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10; static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; -lean_object* l_Lean_Meta_getBitVecValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_BitVec_ofNat(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; -lean_object* l_Lean_Meta_AC_acNfHypMeta(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1; -lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); -lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657_(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -lean_object* l_Lean_Meta_mkDecideProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10; -lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7; -lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9; +lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_mono_nanos_now(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11; -lean_object* l_Lean_Meta_Simp_getSEvalSimprocs___rarg(lean_object*, lean_object*); -uint64_t l_Lean_Expr_hash(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7; -static lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508_(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12; -lean_object* l_BitVec_add(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1; -lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1; -uint8_t lean_name_eq(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -lean_object* l_Lean_Meta_Simp_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_trace_profiler_threshold; lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); -static lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3; -static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7; -static lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline(lean_object*); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Meta_simpGlobalConfig; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8; static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14; -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -lean_object* l_Lean_Meta_SimpExtension_getTheorems(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6; double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083_(lean_object*); -lean_object* l_Lean_LocalDecl_userName(lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662_(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact___boxed(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; -lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389_(lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_constLevels_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1; -lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -lean_object* lean_nat_pow(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12; -lean_object* l_Lean_Meta_Simp_registerBuiltinSimproc(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085_(lean_object*); -uint8_t lean_nat_dec_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349_(lean_object*); -lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; -uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9; -lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15; -lean_object* lean_nat_log2(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3; -uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4; -uint64_t lean_uint64_xor(uint64_t, uint64_t); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2; -lean_object* lean_nat_mul(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_sub(size_t, size_t); -lean_object* lean_array_mk(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1; -lean_object* l_Lean_MVarId_tryClearMany(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1; -size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Expr_fvar___override(lean_object*); -size_t lean_array_size(lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6; +lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7; +lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2; extern lean_object* l_Lean_trace_profiler; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1; -static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -lean_object* lean_string_append(lean_object*, lean_object*); +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_array_get_size(lean_object*); -lean_object* l_Lean_LocalDecl_toExpr(lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1; -extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3; -uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5; -uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8; LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11; -lean_object* lean_nat_add(lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2; -lean_object* l_Lean_MVarId_assertHypotheses(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5; -lean_object* l_Lean_Meta_SimpTheoremsArray_addTheorem(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4; -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2; -lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5; lean_object* l_Lean_Elab_Tactic_replaceMainGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9; -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -lean_object* lean_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_falseOrByContra(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -size_t lean_usize_land(size_t, size_t); -LEAN_EXPORT uint8_t l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021_(lean_object*); double lean_float_sub(double, double); -static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823_(lean_object*); -static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3; -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Bool", 4, 4); -return x_1; +lean_object* x_10; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_9); +return x_10; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1___boxed), 9, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4() { -_start: +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1; +x_13 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 4); +if (x_13 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); -return x_1; -} +lean_object* x_14; lean_object* x_15; +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_12, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_15; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass; +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_2); +x_18 = l_List_appendTR___rarg(x_3, x_17); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_12, x_18, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_20; +} } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} +uint8_t x_12; +x_12 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2(x_1, x_2, x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_14; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("cond_neg", 8, 8); -return x_1; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass; +lean_inc(x_2); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_2); +x_17 = l_List_appendTR___rarg(x_3, x_16); +x_18 = lean_box(0); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_19; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8() { +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("cond_pos", 8, 8); -return x_1; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2; +x_3 = l_List_appendTR___rarg(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_14; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_3); -x_14 = lean_simp(x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -x_19 = l_Lean_Expr_cleanupAnnotations(x_18); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_21 = l_Lean_Expr_isConstOf(x_19, x_20); -if (x_21 == 0) -{ -lean_object* x_22; uint8_t x_23; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; -x_23 = l_Lean_Expr_isConstOf(x_19, x_22); -lean_dec(x_19); -if (x_23 == 0) -{ -lean_object* x_24; -lean_dec(x_16); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_14, 0, x_24); -return x_14; -} -else -{ -lean_object* x_25; -lean_free_object(x_14); -x_25 = l_Lean_Meta_Simp_Result_getProof(x_16, x_9, x_10, x_11, x_12, x_17); -if (lean_obj_tag(x_25) == 0) -{ -uint8_t x_26; -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; -x_27 = lean_ctor_get(x_25, 0); -x_28 = l_Lean_Expr_constLevels_x21(x_1); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; -x_30 = l_Lean_Expr_const___override(x_29, x_28); -lean_inc(x_5); -x_31 = l_Lean_mkApp4(x_30, x_2, x_3, x_4, x_5); -x_32 = l_Lean_Expr_app___override(x_31, x_27); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_32); -x_34 = 1; -x_35 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_35, 0, x_5); -lean_ctor_set(x_35, 1, x_33); -lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_34); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_25, 0, x_36); -return x_25; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_37 = lean_ctor_get(x_25, 0); -x_38 = lean_ctor_get(x_25, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_25); -x_39 = l_Lean_Expr_constLevels_x21(x_1); -x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; -x_41 = l_Lean_Expr_const___override(x_40, x_39); -lean_inc(x_5); -x_42 = l_Lean_mkApp4(x_41, x_2, x_3, x_4, x_5); -x_43 = l_Lean_Expr_app___override(x_42, x_37); -x_44 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_44, 0, x_43); -x_45 = 1; -x_46 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_46, 0, x_5); -lean_ctor_set(x_46, 1, x_44); -lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_45); -x_47 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_47, 0, x_46); -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_38); -return x_48; -} -} -else -{ -uint8_t x_49; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_49 = !lean_is_exclusive(x_25); -if (x_49 == 0) -{ -return x_25; -} -else +lean_object* x_8; uint8_t x_9; +x_8 = lean_box(0); +x_9 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); +if (x_9 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_25, 0); -x_51 = lean_ctor_get(x_25, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_25); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} -} -} +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1; +x_11 = lean_box(0); +lean_inc(x_1); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3(x_1, x_8, x_10, x_11, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_12; } else { -lean_object* x_53; -lean_dec(x_19); -lean_free_object(x_14); -x_53 = l_Lean_Meta_Simp_Result_getProof(x_16, x_9, x_10, x_11, x_12, x_17); -if (lean_obj_tag(x_53) == 0) -{ -uint8_t x_54; -x_54 = !lean_is_exclusive(x_53); -if (x_54 == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; -x_55 = lean_ctor_get(x_53, 0); -x_56 = l_Lean_Expr_constLevels_x21(x_1); -x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; -x_58 = l_Lean_Expr_const___override(x_57, x_56); -lean_inc(x_4); -x_59 = l_Lean_mkApp4(x_58, x_2, x_3, x_4, x_5); -x_60 = l_Lean_Expr_app___override(x_59, x_55); -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_60); -x_62 = 1; -x_63 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_63, 0, x_4); -lean_ctor_set(x_63, 1, x_61); -lean_ctor_set_uint8(x_63, sizeof(void*)*2, x_62); -x_64 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_53, 0, x_64); -return x_53; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3; +x_14 = lean_box(0); +lean_inc(x_1); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3(x_1, x_8, x_13, x_14, x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_15; } -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_65 = lean_ctor_get(x_53, 0); -x_66 = lean_ctor_get(x_53, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_53); -x_67 = l_Lean_Expr_constLevels_x21(x_1); -x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; -x_69 = l_Lean_Expr_const___override(x_68, x_67); -lean_inc(x_4); -x_70 = l_Lean_mkApp4(x_69, x_2, x_3, x_4, x_5); -x_71 = l_Lean_Expr_app___override(x_70, x_65); -x_72 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_72, 0, x_71); -x_73 = 1; -x_74 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_74, 0, x_4); -lean_ctor_set(x_74, 1, x_72); -lean_ctor_set_uint8(x_74, sizeof(void*)*2, x_73); -x_75 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_75, 0, x_74); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_66); -return x_76; } } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_77; +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_77 = !lean_is_exclusive(x_53); -if (x_77 == 0) -{ -return x_53; -} -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_53, 0); -x_79 = lean_ctor_get(x_53, 1); -lean_inc(x_79); -lean_inc(x_78); -lean_dec(x_53); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -return x_80; -} -} +return x_10; } } -else -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_81 = lean_ctor_get(x_14, 0); -x_82 = lean_ctor_get(x_14, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_14); -x_83 = lean_ctor_get(x_81, 0); -lean_inc(x_83); -x_84 = l_Lean_Expr_cleanupAnnotations(x_83); -x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_86 = l_Lean_Expr_isConstOf(x_84, x_85); -if (x_86 == 0) -{ -lean_object* x_87; uint8_t x_88; -x_87 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; -x_88 = l_Lean_Expr_isConstOf(x_84, x_87); -lean_dec(x_84); -if (x_88 == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_89; lean_object* x_90; -lean_dec(x_81); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_5); +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_89 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_82); -return x_90; -} -else -{ -lean_object* x_91; -x_91 = l_Lean_Meta_Simp_Result_getProof(x_81, x_9, x_10, x_11, x_12, x_82); -if (lean_obj_tag(x_91) == 0) -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_94 = x_91; -} else { - lean_dec_ref(x_91); - x_94 = lean_box(0); -} -x_95 = l_Lean_Expr_constLevels_x21(x_1); -x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; -x_97 = l_Lean_Expr_const___override(x_96, x_95); -lean_inc(x_5); -x_98 = l_Lean_mkApp4(x_97, x_2, x_3, x_4, x_5); -x_99 = l_Lean_Expr_app___override(x_98, x_92); -x_100 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_100, 0, x_99); -x_101 = 1; -x_102 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_102, 0, x_5); -lean_ctor_set(x_102, 1, x_100); -lean_ctor_set_uint8(x_102, sizeof(void*)*2, x_101); -x_103 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_103, 0, x_102); -if (lean_is_scalar(x_94)) { - x_104 = lean_alloc_ctor(0, 2, 0); -} else { - x_104 = x_94; +lean_dec(x_1); +return x_12; } -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_93); -return x_104; } -else +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -lean_dec(x_5); +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_105 = lean_ctor_get(x_91, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_91, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_107 = x_91; -} else { - lean_dec_ref(x_91); - x_107 = lean_box(0); -} -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(1, 2, 0); -} else { - x_108 = x_107; -} -lean_ctor_set(x_108, 0, x_105); -lean_ctor_set(x_108, 1, x_106); -return x_108; -} +lean_dec(x_1); +return x_12; } } -else -{ -lean_object* x_109; -lean_dec(x_84); -x_109 = l_Lean_Meta_Simp_Result_getProof(x_81, x_9, x_10, x_11, x_12, x_82); -if (lean_obj_tag(x_109) == 0) +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_110 = lean_ctor_get(x_109, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_109, 1); -lean_inc(x_111); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_112 = x_109; -} else { - lean_dec_ref(x_109); - x_112 = lean_box(0); -} -x_113 = l_Lean_Expr_constLevels_x21(x_1); -x_114 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; -x_115 = l_Lean_Expr_const___override(x_114, x_113); +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); lean_inc(x_4); -x_116 = l_Lean_mkApp4(x_115, x_2, x_3, x_4, x_5); -x_117 = l_Lean_Expr_app___override(x_116, x_110); -x_118 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_118, 0, x_117); -x_119 = 1; -x_120 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_120, 0, x_4); -lean_ctor_set(x_120, 1, x_118); -lean_ctor_set_uint8(x_120, sizeof(void*)*2, x_119); -x_121 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_121, 0, x_120); -if (lean_is_scalar(x_112)) { - x_122 = lean_alloc_ctor(0, 2, 0); -} else { - x_122 = x_112; -} -lean_ctor_set(x_122, 0, x_121); -lean_ctor_set(x_122, 1, x_111); -return x_122; -} -else +lean_inc(x_3); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline(x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_123 = lean_ctor_get(x_109, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_109, 1); -lean_inc(x_124); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_125 = x_109; -} else { - lean_dec_ref(x_109); - x_125 = lean_box(0); -} -if (lean_is_scalar(x_125)) { - x_126 = lean_alloc_ctor(1, 2, 0); -} else { - x_126 = x_125; -} -lean_ctor_set(x_126, 0, x_123); -lean_ctor_set(x_126, 1, x_124); -return x_126; -} -} -} +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_11, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_13; } else { -uint8_t x_127; -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +uint8_t x_14; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_127 = !lean_is_exclusive(x_14); -if (x_127 == 0) +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) { -return x_14; +return x_10; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; -x_128 = lean_ctor_get(x_14, 0); -x_129 = lean_ctor_get(x_14, 1); -lean_inc(x_129); -lean_inc(x_128); -lean_dec(x_14); -x_130 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_130, 0, x_128); -lean_ctor_set(x_130, 1, x_129); -return x_130; -} -} +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_9); -return x_11; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed), 13, 0); +x_1 = lean_mk_string_unchecked("Meta", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed), 9, 0); +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("cond", 4, 4); +x_1 = lean_mk_string_unchecked("bv", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5() { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Running preprocessing pipeline on:\n", 35, 35); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6() { +_start: { -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7() { +_start: { -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8() { +_start: { -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) +lean_object* x_9; lean_object* x_10; +x_9 = lean_box(0); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_10 = l_Lean_MVarId_falseOrByContra(x_1, x_9, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_10) == 0) { -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; +lean_object* x_11; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_10, 0); +lean_dec(x_13); +lean_ctor_set(x_10, 0, x_9); +return x_10; +} +else +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_10, 1); +lean_inc(x_14); +lean_dec(x_10); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_9); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} } else { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = l_Lean_Expr_appArg(x_22, lean_box(0)); -x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_28 = l_Lean_Expr_isApp(x_27); -if (x_28 == 0) +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_dec(x_10); +x_17 = !lean_is_exclusive(x_11); +if (x_17 == 0) { -lean_object* x_29; lean_object* x_30; -lean_dec(x_27); -lean_dec(x_26); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_18 = lean_ctor_get(x_11, 0); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4; +x_20 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_16); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_unbox(x_21); lean_dec(x_21); -lean_dec(x_16); -x_29 = lean_box(0); -x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_30; +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +lean_free_object(x_11); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = lean_box(0); +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_18, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_23); +return x_25; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); -x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; -x_34 = l_Lean_Expr_isConstOf(x_32, x_33); -if (x_34 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) { -lean_object* x_35; lean_object* x_36; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_27 = lean_ctor_get(x_20, 1); +x_28 = lean_ctor_get(x_20, 0); +lean_dec(x_28); +lean_inc(x_18); +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6; +lean_ctor_set_tag(x_20, 7); +lean_ctor_set(x_20, 1, x_11); +lean_ctor_set(x_20, 0, x_29); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_20); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_19, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_27); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_35 = lean_box(0); -x_36 = lean_apply_9(x_11, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_36; +x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_18, x_33, x_2, x_3, x_4, x_5, x_6, x_7, x_34); +lean_dec(x_33); +return x_35; } else { -lean_object* x_37; -x_37 = lean_apply_13(x_10, x_32, x_31, x_26, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_37; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_36 = lean_ctor_get(x_20, 1); +lean_inc(x_36); +lean_dec(x_20); +lean_inc(x_18); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_11); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_19, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_36); +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_18, x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_43); +lean_dec(x_42); +return x_44; } } } +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_45 = lean_ctor_get(x_11, 0); +lean_inc(x_45); +lean_dec(x_11); +x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4; +x_47 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_46, x_2, x_3, x_4, x_5, x_6, x_7, x_16); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_unbox(x_48); +lean_dec(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_47, 1); +lean_inc(x_50); +lean_dec(x_47); +x_51 = lean_box(0); +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_45, x_51, x_2, x_3, x_4, x_5, x_6, x_7, x_50); +return x_52; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_53 = lean_ctor_get(x_47, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_54 = x_47; +} else { + lean_dec_ref(x_47); + x_54 = lean_box(0); } +lean_inc(x_45); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_45); +x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6; +if (lean_is_scalar(x_54)) { + x_57 = lean_alloc_ctor(7, 2, 0); +} else { + x_57 = x_54; + lean_ctor_set_tag(x_57, 7); } +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_55); +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8; +x_59 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +x_60 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_46, x_59, x_2, x_3, x_4, x_5, x_6, x_7, x_53); +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +lean_dec(x_60); +x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_45, x_61, x_2, x_3, x_4, x_5, x_6, x_7, x_62); +lean_dec(x_61); +return x_63; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_1); -return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); +uint8_t x_64; lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); +x_64 = !lean_is_exclusive(x_10); +if (x_64 == 0) +{ return x_10; } -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); -return x_1; +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_10, 0); +x_66 = lean_ctor_get(x_10, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_10); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Elab", 4, 4); -return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Tactic", 6, 6); -return x_1; +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_2); +return x_10; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4() { +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); -return x_1; +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_6); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_6); +return x_10; +} } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5() { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Frontend", 8, 8); -return x_1; +lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_inc(x_9); +x_12 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Meta_processPostponed___spec__3(x_1, x_5, x_2, x_3, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); +lean_dec(x_12); +x_14 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_4, x_7, x_8, x_9, x_10, x_13); +lean_dec(x_9); +return x_14; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6() { +static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Normalize", 9, 9); -return x_1; +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); +return x_3; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7() { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, double x_8, double x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("reduceCond", 10, 10); -return x_1; +if (x_7 == 0) +{ +double x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___closed__1; +x_17 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_3); +lean_ctor_set_float(x_17, sizeof(void*)*2, x_16); +lean_ctor_set_float(x_17, sizeof(void*)*2 + 8, x_16); +lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 16, x_2); +x_18 = lean_box(0); +x_19 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_17, x_18, x_11, x_12, x_13, x_14, x_15); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_20, 0, x_1); +lean_ctor_set(x_20, 1, x_3); +lean_ctor_set_float(x_20, sizeof(void*)*2, x_8); +lean_ctor_set_float(x_20, sizeof(void*)*2 + 8, x_9); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 16, x_2); +x_21 = lean_box(0); +x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_20, x_21, x_11, x_12, x_13, x_14, x_15); +return x_22; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8() { +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 53, 53); +return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9() { +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; -x_2 = lean_unsigned_to_nat(4u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10() { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, double x_7, double x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = lean_box(3); -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13() { -_start: +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 5); +lean_inc(x_16); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_5); +x_17 = lean_apply_6(x_9, x_5, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_18, x_11, x_12, x_13, x_14, x_19); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_5); +return x_20; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2; +x_23 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_22, x_11, x_12, x_13, x_14, x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_5); +return x_23; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14; -x_2 = lean_array_mk(x_1); -return x_2; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16() { +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond), 9, 0); +x_1 = l_Lean_trace_profiler_useHeartbeats; return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2() { +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2() { _start: { lean_object* x_1; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; +x_1 = l_Lean_trace_profiler; return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8; -x_4 = 0; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1() { +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("BEq", 3, 3); +x_1 = l_Lean_trace_profiler_threshold; return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2() { +static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("beq", 3, 3); -return x_1; +lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; +x_1 = lean_unsigned_to_nat(1000u); +x_2 = 0; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Float_ofScientific(x_1, x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3() { +static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; +x_1 = lean_unsigned_to_nat(1000000000u); +x_2 = 0; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Float_ofScientific(x_1, x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4() { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Eq", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5() { -_start: +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Meta_processPostponed___spec__2___rarg(x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1; +x_18 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_17); +if (x_18 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6() { -_start: +lean_object* x_19; lean_object* x_20; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_113 = lean_io_mono_nanos_now(x_16); +x_114 = lean_ctor_get(x_113, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_113, 1); +lean_inc(x_115); +lean_dec(x_113); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_116 = lean_apply_5(x_7, x_9, x_10, x_11, x_12, x_115); +if (lean_obj_tag(x_116) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = l_Lean_Level_ofNat(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7() { -_start: +uint8_t x_117; +x_117 = !lean_is_exclusive(x_116); +if (x_117 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8() { -_start: +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; +x_118 = lean_ctor_get(x_116, 0); +x_119 = lean_ctor_get(x_116, 1); +x_120 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_120, 0, x_118); +x_121 = lean_io_mono_nanos_now(x_119); +x_122 = !lean_is_exclusive(x_121); +if (x_122 == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} +lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; double x_127; double x_128; double x_129; double x_130; double x_131; lean_object* x_132; lean_object* x_133; +x_123 = lean_ctor_get(x_121, 0); +x_124 = lean_ctor_get(x_121, 1); +x_125 = 0; +x_126 = lean_unsigned_to_nat(0u); +x_127 = l_Float_ofScientific(x_114, x_125, x_126); +lean_dec(x_114); +x_128 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_129 = lean_float_div(x_127, x_128); +x_130 = l_Float_ofScientific(x_123, x_125, x_126); +lean_dec(x_123); +x_131 = lean_float_div(x_130, x_128); +x_132 = lean_box_float(x_129); +x_133 = lean_box_float(x_131); +lean_ctor_set(x_121, 1, x_133); +lean_ctor_set(x_121, 0, x_132); +lean_ctor_set(x_116, 1, x_121); +lean_ctor_set(x_116, 0, x_120); +x_19 = x_116; +x_20 = x_124; +goto block_112; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_134; lean_object* x_135; uint8_t x_136; lean_object* x_137; double x_138; double x_139; double x_140; double x_141; double x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_134 = lean_ctor_get(x_121, 0); +x_135 = lean_ctor_get(x_121, 1); +lean_inc(x_135); +lean_inc(x_134); +lean_dec(x_121); +x_136 = 0; +x_137 = lean_unsigned_to_nat(0u); +x_138 = l_Float_ofScientific(x_114, x_136, x_137); +lean_dec(x_114); +x_139 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_140 = lean_float_div(x_138, x_139); +x_141 = l_Float_ofScientific(x_134, x_136, x_137); +lean_dec(x_134); +x_142 = lean_float_div(x_141, x_139); +x_143 = lean_box_float(x_140); +x_144 = lean_box_float(x_142); +x_145 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_145, 0, x_143); +lean_ctor_set(x_145, 1, x_144); +lean_ctor_set(x_116, 1, x_145); +lean_ctor_set(x_116, 0, x_120); +x_19 = x_116; +x_20 = x_135; +goto block_112; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; uint8_t x_153; lean_object* x_154; double x_155; double x_156; double x_157; double x_158; double x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_146 = lean_ctor_get(x_116, 0); +x_147 = lean_ctor_get(x_116, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_116); +x_148 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_148, 0, x_146); +x_149 = lean_io_mono_nanos_now(x_147); +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_149, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_149)) { + lean_ctor_release(x_149, 0); + lean_ctor_release(x_149, 1); + x_152 = x_149; +} else { + lean_dec_ref(x_149); + x_152 = lean_box(0); } +x_153 = 0; +x_154 = lean_unsigned_to_nat(0u); +x_155 = l_Float_ofScientific(x_114, x_153, x_154); +lean_dec(x_114); +x_156 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_157 = lean_float_div(x_155, x_156); +x_158 = l_Float_ofScientific(x_150, x_153, x_154); +lean_dec(x_150); +x_159 = lean_float_div(x_158, x_156); +x_160 = lean_box_float(x_157); +x_161 = lean_box_float(x_159); +if (lean_is_scalar(x_152)) { + x_162 = lean_alloc_ctor(0, 2, 0); +} else { + x_162 = x_152; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_ctor_set(x_162, 0, x_160); +lean_ctor_set(x_162, 1, x_161); +x_163 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_163, 0, x_148); +lean_ctor_set(x_163, 1, x_162); +x_19 = x_163; +x_20 = x_151; +goto block_112; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Std", 3, 3); -return x_1; -} +uint8_t x_164; +x_164 = !lean_is_exclusive(x_116); +if (x_164 == 0) +{ +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; +x_165 = lean_ctor_get(x_116, 0); +x_166 = lean_ctor_get(x_116, 1); +x_167 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_167, 0, x_165); +x_168 = lean_io_mono_nanos_now(x_166); +x_169 = !lean_is_exclusive(x_168); +if (x_169 == 0) +{ +lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; double x_174; double x_175; double x_176; double x_177; double x_178; lean_object* x_179; lean_object* x_180; +x_170 = lean_ctor_get(x_168, 0); +x_171 = lean_ctor_get(x_168, 1); +x_172 = 0; +x_173 = lean_unsigned_to_nat(0u); +x_174 = l_Float_ofScientific(x_114, x_172, x_173); +lean_dec(x_114); +x_175 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_176 = lean_float_div(x_174, x_175); +x_177 = l_Float_ofScientific(x_170, x_172, x_173); +lean_dec(x_170); +x_178 = lean_float_div(x_177, x_175); +x_179 = lean_box_float(x_176); +x_180 = lean_box_float(x_178); +lean_ctor_set(x_168, 1, x_180); +lean_ctor_set(x_168, 0, x_179); +lean_ctor_set_tag(x_116, 0); +lean_ctor_set(x_116, 1, x_168); +lean_ctor_set(x_116, 0, x_167); +x_19 = x_116; +x_20 = x_171; +goto block_112; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_to_beq", 9, 9); -return x_1; +lean_object* x_181; lean_object* x_182; uint8_t x_183; lean_object* x_184; double x_185; double x_186; double x_187; double x_188; double x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +x_181 = lean_ctor_get(x_168, 0); +x_182 = lean_ctor_get(x_168, 1); +lean_inc(x_182); +lean_inc(x_181); +lean_dec(x_168); +x_183 = 0; +x_184 = lean_unsigned_to_nat(0u); +x_185 = l_Float_ofScientific(x_114, x_183, x_184); +lean_dec(x_114); +x_186 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_187 = lean_float_div(x_185, x_186); +x_188 = l_Float_ofScientific(x_181, x_183, x_184); +lean_dec(x_181); +x_189 = lean_float_div(x_188, x_186); +x_190 = lean_box_float(x_187); +x_191 = lean_box_float(x_189); +x_192 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_192, 0, x_190); +lean_ctor_set(x_192, 1, x_191); +lean_ctor_set_tag(x_116, 0); +lean_ctor_set(x_116, 1, x_192); +lean_ctor_set(x_116, 0, x_167); +x_19 = x_116; +x_20 = x_182; +goto block_112; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; +lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; uint8_t x_200; lean_object* x_201; double x_202; double x_203; double x_204; double x_205; double x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; +x_193 = lean_ctor_get(x_116, 0); +x_194 = lean_ctor_get(x_116, 1); +lean_inc(x_194); +lean_inc(x_193); +lean_dec(x_116); +x_195 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_195, 0, x_193); +x_196 = lean_io_mono_nanos_now(x_194); +x_197 = lean_ctor_get(x_196, 0); +lean_inc(x_197); +x_198 = lean_ctor_get(x_196, 1); +lean_inc(x_198); +if (lean_is_exclusive(x_196)) { + lean_ctor_release(x_196, 0); + lean_ctor_release(x_196, 1); + x_199 = x_196; +} else { + lean_dec_ref(x_196); + x_199 = lean_box(0); } +x_200 = 0; +x_201 = lean_unsigned_to_nat(0u); +x_202 = l_Float_ofScientific(x_114, x_200, x_201); +lean_dec(x_114); +x_203 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5; +x_204 = lean_float_div(x_202, x_203); +x_205 = l_Float_ofScientific(x_197, x_200, x_201); +lean_dec(x_197); +x_206 = lean_float_div(x_205, x_203); +x_207 = lean_box_float(x_204); +x_208 = lean_box_float(x_206); +if (lean_is_scalar(x_199)) { + x_209 = lean_alloc_ctor(0, 2, 0); +} else { + x_209 = x_199; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; +lean_ctor_set(x_209, 0, x_207); +lean_ctor_set(x_209, 1, x_208); +x_210 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_210, 0, x_195); +lean_ctor_set(x_210, 1, x_209); +x_19 = x_210; +x_20 = x_198; +goto block_112; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +block_112: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_12 = lean_box(0); -lean_inc(x_1); -x_13 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_12); -lean_inc(x_2); -x_14 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_13); -x_15 = lean_array_mk(x_14); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3; -x_17 = l_Lean_Meta_mkAppM(x_16, x_15, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; uint8_t x_27; +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +x_22 = lean_ctor_get(x_19, 0); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2; +x_26 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_25); +if (x_26 == 0) { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +if (x_6 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_19 = lean_ctor_get(x_17, 0); -x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; -x_23 = l_Lean_mkApp3(x_20, x_21, x_19, x_22); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; -x_25 = l_Lean_mkAppB(x_24, x_2, x_1); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -x_27 = 1; -x_28 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_28, 0, x_23); -lean_ctor_set(x_28, 1, x_26); -lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_27); -x_29 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_17, 0, x_29); -return x_17; +uint8_t x_92; +x_92 = 0; +x_27 = x_92; +goto block_91; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_30 = lean_ctor_get(x_17, 0); -x_31 = lean_ctor_get(x_17, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_17); -x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; -x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; -x_35 = l_Lean_mkApp3(x_32, x_33, x_30, x_34); -x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; -x_37 = l_Lean_mkAppB(x_36, x_2, x_1); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_37); -x_39 = 1; -x_40 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_40, 0, x_35); -lean_ctor_set(x_40, 1, x_38); -lean_ctor_set_uint8(x_40, sizeof(void*)*2, x_39); -x_41 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_41, 0, x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_31); -return x_42; +lean_object* x_93; double x_94; double x_95; lean_object* x_96; +x_93 = lean_box(0); +x_94 = lean_unbox_float(x_23); +lean_dec(x_23); +x_95 = lean_unbox_float(x_24); +lean_dec(x_24); +x_96 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_94, x_95, x_5, x_93, x_9, x_10, x_11, x_12, x_20); +return x_96; } } else { -uint8_t x_43; -lean_dec(x_2); -lean_dec(x_1); -x_43 = !lean_is_exclusive(x_17); -if (x_43 == 0) +if (x_6 == 0) { -return x_17; +double x_97; double x_98; double x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; double x_104; double x_105; double x_106; uint8_t x_107; +x_97 = lean_unbox_float(x_24); +x_98 = lean_unbox_float(x_23); +x_99 = lean_float_sub(x_97, x_98); +x_100 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3; +x_101 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_100); +x_102 = 0; +x_103 = lean_unsigned_to_nat(0u); +x_104 = l_Float_ofScientific(x_101, x_102, x_103); +lean_dec(x_101); +x_105 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__4; +x_106 = lean_float_div(x_104, x_105); +x_107 = lean_float_decLt(x_106, x_99); +x_27 = x_107; +goto block_91; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_17, 0); -x_45 = lean_ctor_get(x_17, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_17); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; -} -} +lean_object* x_108; double x_109; double x_110; lean_object* x_111; +x_108 = lean_box(0); +x_109 = lean_unbox_float(x_23); +lean_dec(x_23); +x_110 = lean_unbox_float(x_24); +lean_dec(x_24); +x_111 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_109, x_110, x_5, x_108, x_9, x_10, x_11, x_12, x_20); +return x_111; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +block_91: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -lean_inc(x_2); -x_11 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_15 = l_Lean_Expr_cleanupAnnotations(x_12); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_17 = l_Lean_Expr_isConstOf(x_15, x_16); -lean_dec(x_15); -if (x_17 == 0) +if (x_27 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(x_2, x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +lean_dec(x_24); +lean_dec(x_23); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_19; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_dec(x_2); -lean_dec(x_1); -x_20 = lean_box(0); -x_21 = lean_apply_9(x_14, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_21; -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2), 10, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +x_28 = lean_st_ref_take(x_12, x_20); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_29, 3); +lean_inc(x_30); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = !lean_is_exclusive(x_29); +if (x_32 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) +lean_object* x_33; uint8_t x_34; +x_33 = lean_ctor_get(x_29, 3); +lean_dec(x_33); +x_34 = !lean_is_exclusive(x_30); +if (x_34 == 0) { -lean_object* x_14; lean_object* x_15; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_30, 0); +x_36 = l_Lean_PersistentArray_append___rarg(x_15, x_35); +lean_dec(x_35); +lean_ctor_set(x_30, 0, x_36); +x_37 = lean_st_ref_set(x_12, x_29, x_31); +x_38 = lean_ctor_get(x_37, 1); +lean_inc(x_38); +lean_dec(x_37); +x_39 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_22, x_9, x_10, x_11, x_12, x_38); lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_22); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; +return x_39; } else { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_39, 0); +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_39); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} } else { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_28 = l_Lean_Expr_isConstOf(x_26, x_27); -lean_dec(x_26); -if (x_28 == 0) +uint8_t x_44; +x_44 = !lean_is_exclusive(x_39); +if (x_44 == 0) { -lean_object* x_29; lean_object* x_30; -lean_dec(x_21); -lean_dec(x_16); -x_29 = lean_box(0); -x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_30; +return x_39; } else { -lean_object* x_31; -x_31 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_31; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_39, 0); +x_46 = lean_ctor_get(x_39, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_39); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } +else +{ +uint64_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_48 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); +x_49 = lean_ctor_get(x_30, 0); +lean_inc(x_49); +lean_dec(x_30); +x_50 = l_Lean_PersistentArray_append___rarg(x_15, x_49); +lean_dec(x_49); +x_51 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set_uint64(x_51, sizeof(void*)*1, x_48); +lean_ctor_set(x_29, 3, x_51); +x_52 = lean_st_ref_set(x_12, x_29, x_31); +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +lean_dec(x_52); +x_54 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_22, x_9, x_10, x_11, x_12, x_53); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_22); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_57 = x_54; +} else { + lean_dec_ref(x_54); + x_57 = lean_box(0); } +if (lean_is_scalar(x_57)) { + x_58 = lean_alloc_ctor(0, 2, 0); +} else { + x_58 = x_57; } +lean_ctor_set(x_58, 0, x_55); +lean_ctor_set(x_58, 1, x_56); +return x_58; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_12; -} +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_59 = lean_ctor_get(x_54, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_54, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_61 = x_54; +} else { + lean_dec_ref(x_54); + x_61 = lean_box(0); } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("eqToBEq", 7, 7); -return x_1; +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(1, 2, 0); +} else { + x_62 = x_61; } +lean_ctor_set(x_62, 0, x_59); +lean_ctor_set(x_62, 1, x_60); +return x_62; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_2 = lean_unsigned_to_nat(3u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint64_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_63 = lean_ctor_get(x_29, 0); +x_64 = lean_ctor_get(x_29, 1); +x_65 = lean_ctor_get(x_29, 2); +x_66 = lean_ctor_get(x_29, 4); +x_67 = lean_ctor_get(x_29, 5); +x_68 = lean_ctor_get(x_29, 6); +x_69 = lean_ctor_get(x_29, 7); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_29); +x_70 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); +x_71 = lean_ctor_get(x_30, 0); +lean_inc(x_71); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + x_72 = x_30; +} else { + lean_dec_ref(x_30); + x_72 = lean_box(0); } +x_73 = l_Lean_PersistentArray_append___rarg(x_15, x_71); +lean_dec(x_71); +if (lean_is_scalar(x_72)) { + x_74 = lean_alloc_ctor(0, 1, 8); +} else { + x_74 = x_72; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4() { -_start: +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set_uint64(x_74, sizeof(void*)*1, x_70); +x_75 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_75, 0, x_63); +lean_ctor_set(x_75, 1, x_64); +lean_ctor_set(x_75, 2, x_65); +lean_ctor_set(x_75, 3, x_74); +lean_ctor_set(x_75, 4, x_66); +lean_ctor_set(x_75, 5, x_67); +lean_ctor_set(x_75, 6, x_68); +lean_ctor_set(x_75, 7, x_69); +x_76 = lean_st_ref_set(x_12, x_75, x_31); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_22, x_9, x_10, x_11, x_12, x_77); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_22); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_81 = x_78; +} else { + lean_dec_ref(x_78); + x_81 = lean_box(0); } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +if (lean_is_scalar(x_81)) { + x_82 = lean_alloc_ctor(0, 2, 0); +} else { + x_82 = x_81; } +lean_ctor_set(x_82, 0, x_79); +lean_ctor_set(x_82, 1, x_80); +return x_82; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_83 = lean_ctor_get(x_78, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_78, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_85 = x_78; +} else { + lean_dec_ref(x_78); + x_85 = lean_box(0); } +if (lean_is_scalar(x_85)) { + x_86 = lean_alloc_ctor(1, 2, 0); +} else { + x_86 = x_85; } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6; -x_2 = lean_array_mk(x_1); -return x_2; +lean_ctor_set(x_86, 0, x_83); +lean_ctor_set(x_86, 1, x_84); +return x_86; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8() { -_start: +} +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq), 9, 0); -return x_1; +lean_object* x_87; double x_88; double x_89; lean_object* x_90; +x_87 = lean_box(0); +x_88 = lean_unbox_float(x_23); +lean_dec(x_23); +x_89 = lean_unbox_float(x_24); +lean_dec(x_24); +x_90 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_88, x_89, x_5, x_87, x_9, x_10, x_11, x_12, x_20); +return x_90; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("BitVec", 6, 6); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("and_ones", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +else { -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); +lean_object* x_211; lean_object* x_212; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +x_303 = lean_io_get_num_heartbeats(x_16); +x_304 = lean_ctor_get(x_303, 0); +lean_inc(x_304); +x_305 = lean_ctor_get(x_303, 1); +lean_inc(x_305); +lean_dec(x_303); lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_306 = lean_apply_5(x_7, x_9, x_10, x_11, x_12, x_305); +if (lean_obj_tag(x_306) == 0) { -uint8_t x_13; -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +uint8_t x_307; +x_307 = !lean_is_exclusive(x_306); +if (x_307 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_15); -return x_11; +lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; uint8_t x_312; +x_308 = lean_ctor_get(x_306, 0); +x_309 = lean_ctor_get(x_306, 1); +x_310 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_310, 0, x_308); +x_311 = lean_io_get_num_heartbeats(x_309); +x_312 = !lean_is_exclusive(x_311); +if (x_312 == 0) +{ +lean_object* x_313; lean_object* x_314; uint8_t x_315; lean_object* x_316; double x_317; double x_318; lean_object* x_319; lean_object* x_320; +x_313 = lean_ctor_get(x_311, 0); +x_314 = lean_ctor_get(x_311, 1); +x_315 = 0; +x_316 = lean_unsigned_to_nat(0u); +x_317 = l_Float_ofScientific(x_304, x_315, x_316); +lean_dec(x_304); +x_318 = l_Float_ofScientific(x_313, x_315, x_316); +lean_dec(x_313); +x_319 = lean_box_float(x_317); +x_320 = lean_box_float(x_318); +lean_ctor_set(x_311, 1, x_320); +lean_ctor_set(x_311, 0, x_319); +lean_ctor_set(x_306, 1, x_311); +lean_ctor_set(x_306, 0, x_310); +x_211 = x_306; +x_212 = x_314; +goto block_302; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_321; lean_object* x_322; uint8_t x_323; lean_object* x_324; double x_325; double x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; +x_321 = lean_ctor_get(x_311, 0); +x_322 = lean_ctor_get(x_311, 1); +lean_inc(x_322); +lean_inc(x_321); +lean_dec(x_311); +x_323 = 0; +x_324 = lean_unsigned_to_nat(0u); +x_325 = l_Float_ofScientific(x_304, x_323, x_324); +lean_dec(x_304); +x_326 = l_Float_ofScientific(x_321, x_323, x_324); +lean_dec(x_321); +x_327 = lean_box_float(x_325); +x_328 = lean_box_float(x_326); +x_329 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_329, 0, x_327); +lean_ctor_set(x_329, 1, x_328); +lean_ctor_set(x_306, 1, x_329); +lean_ctor_set(x_306, 0, x_310); +x_211 = x_306; +x_212 = x_322; +goto block_302; } } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_11); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_21 = lean_ctor_get(x_12, 0); -x_22 = lean_ctor_get(x_11, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_unsigned_to_nat(1u); -x_26 = l_BitVec_ofNat(x_23, x_25); -x_27 = l_BitVec_neg(x_23, x_26); -lean_dec(x_26); -x_28 = lean_nat_dec_eq(x_24, x_27); -lean_dec(x_27); -lean_dec(x_24); -if (x_28 == 0) -{ -lean_object* x_29; -lean_dec(x_23); -lean_free_object(x_12); -lean_dec(x_1); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_29); -return x_11; +lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; uint8_t x_337; lean_object* x_338; double x_339; double x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; +x_330 = lean_ctor_get(x_306, 0); +x_331 = lean_ctor_get(x_306, 1); +lean_inc(x_331); +lean_inc(x_330); +lean_dec(x_306); +x_332 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_332, 0, x_330); +x_333 = lean_io_get_num_heartbeats(x_331); +x_334 = lean_ctor_get(x_333, 0); +lean_inc(x_334); +x_335 = lean_ctor_get(x_333, 1); +lean_inc(x_335); +if (lean_is_exclusive(x_333)) { + lean_ctor_release(x_333, 0); + lean_ctor_release(x_333, 1); + x_336 = x_333; +} else { + lean_dec_ref(x_333); + x_336 = lean_box(0); } -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; -x_30 = l_Lean_mkNatLit(x_23); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; -lean_inc(x_1); -x_32 = l_Lean_mkAppB(x_31, x_30, x_1); -lean_ctor_set(x_12, 0, x_32); -x_33 = 1; -x_34 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_34, 0, x_1); -lean_ctor_set(x_34, 1, x_12); -lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_11, 0, x_35); -return x_11; +x_337 = 0; +x_338 = lean_unsigned_to_nat(0u); +x_339 = l_Float_ofScientific(x_304, x_337, x_338); +lean_dec(x_304); +x_340 = l_Float_ofScientific(x_334, x_337, x_338); +lean_dec(x_334); +x_341 = lean_box_float(x_339); +x_342 = lean_box_float(x_340); +if (lean_is_scalar(x_336)) { + x_343 = lean_alloc_ctor(0, 2, 0); +} else { + x_343 = x_336; +} +lean_ctor_set(x_343, 0, x_341); +lean_ctor_set(x_343, 1, x_342); +x_344 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_344, 0, x_332); +lean_ctor_set(x_344, 1, x_343); +x_211 = x_344; +x_212 = x_335; +goto block_302; } } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_36 = lean_ctor_get(x_12, 0); -x_37 = lean_ctor_get(x_11, 1); -lean_inc(x_37); -lean_dec(x_11); -x_38 = lean_ctor_get(x_36, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_36, 1); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_unsigned_to_nat(1u); -x_41 = l_BitVec_ofNat(x_38, x_40); -x_42 = l_BitVec_neg(x_38, x_41); -lean_dec(x_41); -x_43 = lean_nat_dec_eq(x_39, x_42); -lean_dec(x_42); -lean_dec(x_39); -if (x_43 == 0) +uint8_t x_345; +x_345 = !lean_is_exclusive(x_306); +if (x_345 == 0) { -lean_object* x_44; lean_object* x_45; -lean_dec(x_38); -lean_free_object(x_12); -lean_dec(x_1); -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_37); -return x_45; -} -else +lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; uint8_t x_350; +x_346 = lean_ctor_get(x_306, 0); +x_347 = lean_ctor_get(x_306, 1); +x_348 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_348, 0, x_346); +x_349 = lean_io_get_num_heartbeats(x_347); +x_350 = !lean_is_exclusive(x_349); +if (x_350 == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_46 = l_Lean_mkNatLit(x_38); -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; -lean_inc(x_1); -x_48 = l_Lean_mkAppB(x_47, x_46, x_1); -lean_ctor_set(x_12, 0, x_48); -x_49 = 1; -x_50 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_50, 0, x_1); -lean_ctor_set(x_50, 1, x_12); -lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_49); -x_51 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_51, 0, x_50); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_37); -return x_52; -} -} +lean_object* x_351; lean_object* x_352; uint8_t x_353; lean_object* x_354; double x_355; double x_356; lean_object* x_357; lean_object* x_358; +x_351 = lean_ctor_get(x_349, 0); +x_352 = lean_ctor_get(x_349, 1); +x_353 = 0; +x_354 = lean_unsigned_to_nat(0u); +x_355 = l_Float_ofScientific(x_304, x_353, x_354); +lean_dec(x_304); +x_356 = l_Float_ofScientific(x_351, x_353, x_354); +lean_dec(x_351); +x_357 = lean_box_float(x_355); +x_358 = lean_box_float(x_356); +lean_ctor_set(x_349, 1, x_358); +lean_ctor_set(x_349, 0, x_357); +lean_ctor_set_tag(x_306, 0); +lean_ctor_set(x_306, 1, x_349); +lean_ctor_set(x_306, 0, x_348); +x_211 = x_306; +x_212 = x_352; +goto block_302; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_53 = lean_ctor_get(x_12, 0); -lean_inc(x_53); -lean_dec(x_12); -x_54 = lean_ctor_get(x_11, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_55 = x_11; -} else { - lean_dec_ref(x_11); - x_55 = lean_box(0); -} -x_56 = lean_ctor_get(x_53, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_53, 1); -lean_inc(x_57); -lean_dec(x_53); -x_58 = lean_unsigned_to_nat(1u); -x_59 = l_BitVec_ofNat(x_56, x_58); -x_60 = l_BitVec_neg(x_56, x_59); -lean_dec(x_59); -x_61 = lean_nat_dec_eq(x_57, x_60); -lean_dec(x_60); -lean_dec(x_57); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; -lean_dec(x_56); -lean_dec(x_1); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_55)) { - x_63 = lean_alloc_ctor(0, 2, 0); -} else { - x_63 = x_55; +lean_object* x_359; lean_object* x_360; uint8_t x_361; lean_object* x_362; double x_363; double x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; +x_359 = lean_ctor_get(x_349, 0); +x_360 = lean_ctor_get(x_349, 1); +lean_inc(x_360); +lean_inc(x_359); +lean_dec(x_349); +x_361 = 0; +x_362 = lean_unsigned_to_nat(0u); +x_363 = l_Float_ofScientific(x_304, x_361, x_362); +lean_dec(x_304); +x_364 = l_Float_ofScientific(x_359, x_361, x_362); +lean_dec(x_359); +x_365 = lean_box_float(x_363); +x_366 = lean_box_float(x_364); +x_367 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_367, 0, x_365); +lean_ctor_set(x_367, 1, x_366); +lean_ctor_set_tag(x_306, 0); +lean_ctor_set(x_306, 1, x_367); +lean_ctor_set(x_306, 0, x_348); +x_211 = x_306; +x_212 = x_360; +goto block_302; } -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_54); -return x_63; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_64 = l_Lean_mkNatLit(x_56); -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; -lean_inc(x_1); -x_66 = l_Lean_mkAppB(x_65, x_64, x_1); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = 1; -x_69 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_69, 0, x_1); -lean_ctor_set(x_69, 1, x_67); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_68); -x_70 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_70, 0, x_69); -if (lean_is_scalar(x_55)) { - x_71 = lean_alloc_ctor(0, 2, 0); -} else { - x_71 = x_55; -} -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_54); -return x_71; -} -} -} -} -else -{ -uint8_t x_72; -lean_dec(x_1); -x_72 = !lean_is_exclusive(x_11); -if (x_72 == 0) -{ -return x_11; -} -else -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_11, 0); -x_74 = lean_ctor_get(x_11, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_11); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -return x_75; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed), 10, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HAnd", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hAnd", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_43; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_11; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("andOnes", 7, 7); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; -x_2 = lean_unsigned_to_nat(6u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4; -x_2 = lean_unsigned_to_nat(1u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ones_and", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -lean_dec(x_2); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; -} -} -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_11); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_21 = lean_ctor_get(x_12, 0); -x_22 = lean_ctor_get(x_11, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_unsigned_to_nat(1u); -x_26 = l_BitVec_ofNat(x_23, x_25); -x_27 = l_BitVec_neg(x_23, x_26); -lean_dec(x_26); -x_28 = lean_nat_dec_eq(x_24, x_27); -lean_dec(x_27); -lean_dec(x_24); -if (x_28 == 0) -{ -lean_object* x_29; -lean_dec(x_23); -lean_free_object(x_12); -lean_dec(x_2); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_29); -return x_11; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; -x_30 = l_Lean_mkNatLit(x_23); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; -lean_inc(x_2); -x_32 = l_Lean_mkAppB(x_31, x_30, x_2); -lean_ctor_set(x_12, 0, x_32); -x_33 = 1; -x_34 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_34, 0, x_2); -lean_ctor_set(x_34, 1, x_12); -lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_33); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_11, 0, x_35); -return x_11; -} -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_36 = lean_ctor_get(x_12, 0); -x_37 = lean_ctor_get(x_11, 1); -lean_inc(x_37); -lean_dec(x_11); -x_38 = lean_ctor_get(x_36, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_36, 1); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_unsigned_to_nat(1u); -x_41 = l_BitVec_ofNat(x_38, x_40); -x_42 = l_BitVec_neg(x_38, x_41); -lean_dec(x_41); -x_43 = lean_nat_dec_eq(x_39, x_42); -lean_dec(x_42); -lean_dec(x_39); -if (x_43 == 0) -{ -lean_object* x_44; lean_object* x_45; -lean_dec(x_38); -lean_free_object(x_12); -lean_dec(x_2); -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_37); -return x_45; -} -else -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_46 = l_Lean_mkNatLit(x_38); -x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; -lean_inc(x_2); -x_48 = l_Lean_mkAppB(x_47, x_46, x_2); -lean_ctor_set(x_12, 0, x_48); -x_49 = 1; -x_50 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_50, 0, x_2); -lean_ctor_set(x_50, 1, x_12); -lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_49); -x_51 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_51, 0, x_50); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_37); -return x_52; -} -} -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_53 = lean_ctor_get(x_12, 0); -lean_inc(x_53); -lean_dec(x_12); -x_54 = lean_ctor_get(x_11, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_55 = x_11; -} else { - lean_dec_ref(x_11); - x_55 = lean_box(0); -} -x_56 = lean_ctor_get(x_53, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_53, 1); -lean_inc(x_57); -lean_dec(x_53); -x_58 = lean_unsigned_to_nat(1u); -x_59 = l_BitVec_ofNat(x_56, x_58); -x_60 = l_BitVec_neg(x_56, x_59); -lean_dec(x_59); -x_61 = lean_nat_dec_eq(x_57, x_60); -lean_dec(x_60); -lean_dec(x_57); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; -lean_dec(x_56); -lean_dec(x_2); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_55)) { - x_63 = lean_alloc_ctor(0, 2, 0); -} else { - x_63 = x_55; -} -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_54); -return x_63; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_64 = l_Lean_mkNatLit(x_56); -x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; -lean_inc(x_2); -x_66 = l_Lean_mkAppB(x_65, x_64, x_2); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = 1; -x_69 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_69, 0, x_2); -lean_ctor_set(x_69, 1, x_67); -lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_68); -x_70 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_70, 0, x_69); -if (lean_is_scalar(x_55)) { - x_71 = lean_alloc_ctor(0, 2, 0); -} else { - x_71 = x_55; -} -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_54); -return x_71; -} -} -} -} -else -{ -uint8_t x_72; -lean_dec(x_2); -x_72 = !lean_is_exclusive(x_11); -if (x_72 == 0) -{ -return x_11; -} -else -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_11, 0); -x_74 = lean_ctor_get(x_11, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_11); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -return x_75; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed), 10, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_43; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_11; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("onesAnd", 7, 7); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("max_ult'", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -lean_dec(x_2); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; -} -} -else -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_11); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_21 = lean_ctor_get(x_12, 0); -x_22 = lean_ctor_get(x_11, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = lean_unsigned_to_nat(1u); -x_26 = l_BitVec_ofNat(x_23, x_25); -x_27 = l_BitVec_neg(x_23, x_26); -lean_dec(x_26); -x_28 = lean_nat_dec_eq(x_24, x_27); -lean_dec(x_27); -lean_dec(x_24); -if (x_28 == 0) -{ -lean_object* x_29; -lean_dec(x_23); -lean_free_object(x_12); -lean_dec(x_2); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_29); -return x_11; -} -else -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; -x_30 = l_Lean_mkNatLit(x_23); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; -x_32 = l_Lean_mkAppB(x_31, x_30, x_2); -lean_ctor_set(x_12, 0, x_32); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; -x_34 = 1; -x_35 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_12); -lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_34); -x_36 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_11, 0, x_36); -return x_11; -} -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_37 = lean_ctor_get(x_12, 0); -x_38 = lean_ctor_get(x_11, 1); -lean_inc(x_38); -lean_dec(x_11); -x_39 = lean_ctor_get(x_37, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_37, 1); -lean_inc(x_40); -lean_dec(x_37); -x_41 = lean_unsigned_to_nat(1u); -x_42 = l_BitVec_ofNat(x_39, x_41); -x_43 = l_BitVec_neg(x_39, x_42); -lean_dec(x_42); -x_44 = lean_nat_dec_eq(x_40, x_43); -lean_dec(x_43); -lean_dec(x_40); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; -lean_dec(x_39); -lean_free_object(x_12); -lean_dec(x_2); -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_38); -return x_46; -} -else -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_47 = l_Lean_mkNatLit(x_39); -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; -x_49 = l_Lean_mkAppB(x_48, x_47, x_2); -lean_ctor_set(x_12, 0, x_49); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; -x_51 = 1; -x_52 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_12); -lean_ctor_set_uint8(x_52, sizeof(void*)*2, x_51); -x_53 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_53, 0, x_52); -x_54 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_38); -return x_54; -} -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; -x_55 = lean_ctor_get(x_12, 0); -lean_inc(x_55); -lean_dec(x_12); -x_56 = lean_ctor_get(x_11, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_11)) { - lean_ctor_release(x_11, 0); - lean_ctor_release(x_11, 1); - x_57 = x_11; -} else { - lean_dec_ref(x_11); - x_57 = lean_box(0); -} -x_58 = lean_ctor_get(x_55, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_55, 1); -lean_inc(x_59); -lean_dec(x_55); -x_60 = lean_unsigned_to_nat(1u); -x_61 = l_BitVec_ofNat(x_58, x_60); -x_62 = l_BitVec_neg(x_58, x_61); -lean_dec(x_61); -x_63 = lean_nat_dec_eq(x_59, x_62); -lean_dec(x_62); -lean_dec(x_59); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; -lean_dec(x_58); -lean_dec(x_2); -x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_57)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_57; -} -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_56); -return x_65; -} -else -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_66 = l_Lean_mkNatLit(x_58); -x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; -x_68 = l_Lean_mkAppB(x_67, x_66, x_2); -x_69 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_69, 0, x_68); -x_70 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; -x_71 = 1; -x_72 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_69); -lean_ctor_set_uint8(x_72, sizeof(void*)*2, x_71); -x_73 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_73, 0, x_72); -if (lean_is_scalar(x_57)) { - x_74 = lean_alloc_ctor(0, 2, 0); -} else { - x_74 = x_57; -} -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set(x_74, 1, x_56); -return x_74; -} -} -} -} -else -{ -uint8_t x_75; -lean_dec(x_2); -x_75 = !lean_is_exclusive(x_11); -if (x_75 == 0) -{ -return x_11; -} -else -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_11, 0); -x_77 = lean_ctor_get(x_11, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_11); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed), 10, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ult", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; -x_28 = l_Lean_Expr_isConstOf(x_26, x_27); -lean_dec(x_26); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; -lean_dec(x_21); -lean_dec(x_16); -x_29 = lean_box(0); -x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_30; -} -else -{ -lean_object* x_31; -x_31 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_31; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_11; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("maxUlt", 6, 6); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; -x_2 = lean_unsigned_to_nat(3u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("neg_eq_not_add", 14, 14); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Complement", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("complement", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HAdd", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hAdd", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ofNat", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_11 = l_Lean_Meta_getNatValue_x3f(x_2, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_11, 0, x_15); -return x_11; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; -} -} -else -{ -lean_object* x_19; uint8_t x_20; -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_dec(x_11); -x_20 = !lean_is_exclusive(x_12); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_22 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_19); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_box(0); -lean_inc(x_21); -x_26 = l_Lean_mkNatLit(x_21); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; -lean_inc(x_1); -lean_inc(x_26); -x_28 = l_Lean_mkAppB(x_27, x_26, x_1); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_1); -lean_ctor_set(x_29, 1, x_25); -x_30 = lean_array_mk(x_29); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_32 = l_Lean_Meta_mkAppM(x_31, x_30, x_6, x_7, x_8, x_9, x_24); -if (lean_obj_tag(x_32) == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -lean_dec(x_32); -x_35 = lean_unsigned_to_nat(1u); -x_36 = l_BitVec_ofNat(x_21, x_35); -lean_dec(x_21); -x_37 = l_Lean_mkNatLit(x_36); -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; -x_39 = l_Lean_mkAppB(x_38, x_26, x_37); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_25); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_33); -lean_ctor_set(x_41, 1, x_40); -x_42 = lean_array_mk(x_41); -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_44 = l_Lean_Meta_mkAppM(x_43, x_42, x_6, x_7, x_8, x_9, x_34); -if (lean_obj_tag(x_44) == 0) -{ -uint8_t x_45; -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) -{ -lean_object* x_46; uint8_t x_47; lean_object* x_48; lean_object* x_49; -x_46 = lean_ctor_get(x_44, 0); -lean_ctor_set(x_12, 0, x_28); -x_47 = 1; -x_48 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_12); -lean_ctor_set_uint8(x_48, sizeof(void*)*2, x_47); -x_49 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_44, 0, x_49); -return x_44; -} -else -{ -lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_50 = lean_ctor_get(x_44, 0); -x_51 = lean_ctor_get(x_44, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_44); -lean_ctor_set(x_12, 0, x_28); -x_52 = 1; -x_53 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_53, 0, x_50); -lean_ctor_set(x_53, 1, x_12); -lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_52); -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_53); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_51); -return x_55; -} -} -else -{ -uint8_t x_56; -lean_dec(x_28); -lean_free_object(x_12); -x_56 = !lean_is_exclusive(x_44); -if (x_56 == 0) -{ -return x_44; -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_44, 0); -x_58 = lean_ctor_get(x_44, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_44); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -return x_59; -} -} -} -else -{ -uint8_t x_60; -lean_dec(x_28); -lean_dec(x_26); -lean_free_object(x_12); -lean_dec(x_21); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_60 = !lean_is_exclusive(x_32); -if (x_60 == 0) -{ -return x_32; -} -else -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_32, 0); -x_62 = lean_ctor_get(x_32, 1); -lean_inc(x_62); -lean_inc(x_61); -lean_dec(x_32); -x_63 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_63, 0, x_61); -lean_ctor_set(x_63, 1, x_62); -return x_63; -} -} -} -else -{ -uint8_t x_64; -lean_dec(x_23); -lean_free_object(x_12); -lean_dec(x_21); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_64 = !lean_is_exclusive(x_22); -if (x_64 == 0) -{ -lean_object* x_65; lean_object* x_66; -x_65 = lean_ctor_get(x_22, 0); -lean_dec(x_65); -x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_22, 0, x_66); -return x_22; -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_22, 1); -lean_inc(x_67); -lean_dec(x_22); -x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_67); -return x_69; -} -} -} -else -{ -uint8_t x_70; -lean_free_object(x_12); -lean_dec(x_21); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_70 = !lean_is_exclusive(x_22); -if (x_70 == 0) -{ -return x_22; -} -else -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_22, 0); -x_72 = lean_ctor_get(x_22, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_22); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; -} -} -} -else -{ -lean_object* x_74; lean_object* x_75; -x_74 = lean_ctor_get(x_12, 0); -lean_inc(x_74); -lean_dec(x_12); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_75 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_19); -if (lean_obj_tag(x_75) == 0) -{ -lean_object* x_76; -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -if (lean_obj_tag(x_76) == 0) -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_77 = lean_ctor_get(x_75, 1); -lean_inc(x_77); -lean_dec(x_75); -x_78 = lean_box(0); -lean_inc(x_74); -x_79 = l_Lean_mkNatLit(x_74); -x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; -lean_inc(x_1); -lean_inc(x_79); -x_81 = l_Lean_mkAppB(x_80, x_79, x_1); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_1); -lean_ctor_set(x_82, 1, x_78); -x_83 = lean_array_mk(x_82); -x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_85 = l_Lean_Meta_mkAppM(x_84, x_83, x_6, x_7, x_8, x_9, x_77); -if (lean_obj_tag(x_85) == 0) -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_85, 1); -lean_inc(x_87); -lean_dec(x_85); -x_88 = lean_unsigned_to_nat(1u); -x_89 = l_BitVec_ofNat(x_74, x_88); -lean_dec(x_74); -x_90 = l_Lean_mkNatLit(x_89); -x_91 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; -x_92 = l_Lean_mkAppB(x_91, x_79, x_90); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_78); -x_94 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_94, 0, x_86); -lean_ctor_set(x_94, 1, x_93); -x_95 = lean_array_mk(x_94); -x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_97 = l_Lean_Meta_mkAppM(x_96, x_95, x_6, x_7, x_8, x_9, x_87); -if (lean_obj_tag(x_97) == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_98 = lean_ctor_get(x_97, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_97, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_100 = x_97; -} else { - lean_dec_ref(x_97); - x_100 = lean_box(0); -} -x_101 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_101, 0, x_81); -x_102 = 1; -x_103 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_103, 0, x_98); -lean_ctor_set(x_103, 1, x_101); -lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_102); -x_104 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_104, 0, x_103); -if (lean_is_scalar(x_100)) { - x_105 = lean_alloc_ctor(0, 2, 0); -} else { - x_105 = x_100; -} -lean_ctor_set(x_105, 0, x_104); -lean_ctor_set(x_105, 1, x_99); -return x_105; -} -else -{ -lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -lean_dec(x_81); -x_106 = lean_ctor_get(x_97, 0); -lean_inc(x_106); -x_107 = lean_ctor_get(x_97, 1); -lean_inc(x_107); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_108 = x_97; -} else { - lean_dec_ref(x_97); - x_108 = lean_box(0); -} -if (lean_is_scalar(x_108)) { - x_109 = lean_alloc_ctor(1, 2, 0); -} else { - x_109 = x_108; -} -lean_ctor_set(x_109, 0, x_106); -lean_ctor_set(x_109, 1, x_107); -return x_109; -} -} -else -{ -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -lean_dec(x_81); -lean_dec(x_79); -lean_dec(x_74); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -x_110 = lean_ctor_get(x_85, 0); -lean_inc(x_110); -x_111 = lean_ctor_get(x_85, 1); -lean_inc(x_111); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_112 = x_85; -} else { - lean_dec_ref(x_85); - x_112 = lean_box(0); -} -if (lean_is_scalar(x_112)) { - x_113 = lean_alloc_ctor(1, 2, 0); -} else { - x_113 = x_112; -} -lean_ctor_set(x_113, 0, x_110); -lean_ctor_set(x_113, 1, x_111); -return x_113; -} -} -else -{ -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -lean_dec(x_76); -lean_dec(x_74); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_114 = lean_ctor_get(x_75, 1); -lean_inc(x_114); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_115 = x_75; -} else { - lean_dec_ref(x_75); - x_115 = lean_box(0); -} -x_116 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_115)) { - x_117 = lean_alloc_ctor(0, 2, 0); -} else { - x_117 = x_115; -} -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_117, 1, x_114); -return x_117; -} -} -else -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -lean_dec(x_74); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_118 = lean_ctor_get(x_75, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_75, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_120 = x_75; -} else { - lean_dec_ref(x_75); - x_120 = lean_box(0); -} -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); -} else { - x_121 = x_120; -} -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_119); -return x_121; -} -} -} -} -else -{ -uint8_t x_122; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_122 = !lean_is_exclusive(x_11); -if (x_122 == 0) -{ -return x_11; -} -else -{ -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_11, 0); -x_124 = lean_ctor_get(x_11, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_11); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4; -x_19 = l_Lean_Expr_isConstOf(x_17, x_18); -lean_dec(x_17); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; -lean_dec(x_16); -lean_dec(x_2); -x_20 = lean_box(0); -x_21 = lean_apply_9(x_11, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_21; -} -else -{ -lean_object* x_22; -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_16); -return x_22; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2), 10, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Neg", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("neg", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; uint8_t x_22; -x_21 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_22 = l_Lean_Expr_isApp(x_21); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; -lean_dec(x_21); -lean_dec(x_16); -x_23 = lean_box(0); -x_24 = lean_apply_9(x_11, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_24; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_25 = l_Lean_Expr_appArg(x_21, lean_box(0)); -x_26 = l_Lean_Expr_appFnCleanup(x_21, lean_box(0)); -x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; -x_28 = l_Lean_Expr_isConstOf(x_26, x_27); -lean_dec(x_26); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; -lean_dec(x_25); -lean_dec(x_16); -x_29 = lean_box(0); -x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_30; -} -else -{ -lean_object* x_31; -x_31 = lean_apply_10(x_10, x_25, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_31; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; -x_2 = lean_unsigned_to_nat(3u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("add_const_right", 15, 15); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("add_const_left", 14, 14); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_1); -x_12 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_14 = !lean_is_exclusive(x_12); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 0); -lean_dec(x_15); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_12, 0, x_16); -return x_12; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_dec(x_12); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; -} -} -else -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_13); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_13, 0); -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); -lean_dec(x_12); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_21, 0); -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_26 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_29 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -if (lean_obj_tag(x_30) == 0) -{ -uint8_t x_31; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_29); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_33); -return x_29; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_29, 1); -lean_inc(x_34); -lean_dec(x_29); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -return x_36; -} -} -else -{ -uint8_t x_37; -x_37 = !lean_is_exclusive(x_30); -if (x_37 == 0) -{ -uint8_t x_38; -x_38 = !lean_is_exclusive(x_29); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_39 = lean_ctor_get(x_30, 0); -x_40 = lean_ctor_get(x_29, 1); -x_41 = lean_ctor_get(x_29, 0); -lean_dec(x_41); -x_42 = !lean_is_exclusive(x_39); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_43 = lean_ctor_get(x_39, 0); -x_44 = lean_ctor_get(x_39, 1); -x_45 = lean_nat_dec_eq(x_24, x_43); -lean_dec(x_43); -if (x_45 == 0) -{ -lean_object* x_46; -lean_free_object(x_39); -lean_dec(x_44); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_46); -return x_29; -} -else -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_free_object(x_29); -x_47 = l_BitVec_add(x_24, x_25, x_44); -lean_dec(x_44); -lean_dec(x_25); -x_48 = lean_box(0); -x_49 = l_Lean_mkNatLit(x_24); -x_50 = l_Lean_mkNatLit(x_47); -x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_49); -x_52 = l_Lean_mkAppB(x_51, x_49, x_50); -lean_inc(x_2); -lean_ctor_set_tag(x_39, 1); -lean_ctor_set(x_39, 1, x_48); -lean_ctor_set(x_39, 0, x_2); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_39); -lean_ctor_set(x_21, 0, x_52); -x_53 = lean_array_mk(x_21); -x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_55 = l_Lean_Meta_mkAppM(x_54, x_53, x_7, x_8, x_9, x_10, x_40); -if (lean_obj_tag(x_55) == 0) -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_57 = lean_ctor_get(x_55, 0); -x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_59 = l_Lean_mkApp4(x_58, x_49, x_1, x_2, x_3); -lean_ctor_set(x_30, 0, x_59); -x_60 = 1; -x_61 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_30); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_60); -lean_ctor_set(x_13, 0, x_61); -lean_ctor_set(x_55, 0, x_13); -return x_55; -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; -x_62 = lean_ctor_get(x_55, 0); -x_63 = lean_ctor_get(x_55, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_55); -x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_65 = l_Lean_mkApp4(x_64, x_49, x_1, x_2, x_3); -lean_ctor_set(x_30, 0, x_65); -x_66 = 1; -x_67 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_67, 0, x_62); -lean_ctor_set(x_67, 1, x_30); -lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); -lean_ctor_set(x_13, 0, x_67); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_13); -lean_ctor_set(x_68, 1, x_63); -return x_68; -} -} -else -{ -uint8_t x_69; -lean_dec(x_49); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_69 = !lean_is_exclusive(x_55); -if (x_69 == 0) -{ -return x_55; -} -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_55, 0); -x_71 = lean_ctor_get(x_55, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_55); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; -} -} -} -} -else -{ -lean_object* x_73; lean_object* x_74; uint8_t x_75; -x_73 = lean_ctor_get(x_39, 0); -x_74 = lean_ctor_get(x_39, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_39); -x_75 = lean_nat_dec_eq(x_24, x_73); -lean_dec(x_73); -if (x_75 == 0) -{ -lean_object* x_76; -lean_dec(x_74); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_76 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_76); -return x_29; -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -lean_free_object(x_29); -x_77 = l_BitVec_add(x_24, x_25, x_74); -lean_dec(x_74); -lean_dec(x_25); -x_78 = lean_box(0); -x_79 = l_Lean_mkNatLit(x_24); -x_80 = l_Lean_mkNatLit(x_77); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_79); -x_82 = l_Lean_mkAppB(x_81, x_79, x_80); -lean_inc(x_2); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_2); -lean_ctor_set(x_83, 1, x_78); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_83); -lean_ctor_set(x_21, 0, x_82); -x_84 = lean_array_mk(x_21); -x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_86 = l_Lean_Meta_mkAppM(x_85, x_84, x_7, x_8, x_9, x_10, x_40); -if (lean_obj_tag(x_86) == 0) -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_89 = x_86; -} else { - lean_dec_ref(x_86); - x_89 = lean_box(0); -} -x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_91 = l_Lean_mkApp4(x_90, x_79, x_1, x_2, x_3); -lean_ctor_set(x_30, 0, x_91); -x_92 = 1; -x_93 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_93, 0, x_87); -lean_ctor_set(x_93, 1, x_30); -lean_ctor_set_uint8(x_93, sizeof(void*)*2, x_92); -lean_ctor_set(x_13, 0, x_93); -if (lean_is_scalar(x_89)) { - x_94 = lean_alloc_ctor(0, 2, 0); -} else { - x_94 = x_89; -} -lean_ctor_set(x_94, 0, x_13); -lean_ctor_set(x_94, 1, x_88); -return x_94; -} -else -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -lean_dec(x_79); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_95 = lean_ctor_get(x_86, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_86, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_97 = x_86; -} else { - lean_dec_ref(x_86); - x_97 = lean_box(0); -} -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(1, 2, 0); -} else { - x_98 = x_97; -} -lean_ctor_set(x_98, 0, x_95); -lean_ctor_set(x_98, 1, x_96); -return x_98; -} -} -} -} -else -{ -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_99 = lean_ctor_get(x_30, 0); -x_100 = lean_ctor_get(x_29, 1); -lean_inc(x_100); -lean_dec(x_29); -x_101 = lean_ctor_get(x_99, 0); -lean_inc(x_101); -x_102 = lean_ctor_get(x_99, 1); -lean_inc(x_102); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_103 = x_99; -} else { - lean_dec_ref(x_99); - x_103 = lean_box(0); -} -x_104 = lean_nat_dec_eq(x_24, x_101); -lean_dec(x_101); -if (x_104 == 0) -{ -lean_object* x_105; lean_object* x_106; -lean_dec(x_103); -lean_dec(x_102); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_100); -return x_106; -} -else -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_107 = l_BitVec_add(x_24, x_25, x_102); -lean_dec(x_102); -lean_dec(x_25); -x_108 = lean_box(0); -x_109 = l_Lean_mkNatLit(x_24); -x_110 = l_Lean_mkNatLit(x_107); -x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_109); -x_112 = l_Lean_mkAppB(x_111, x_109, x_110); -lean_inc(x_2); -if (lean_is_scalar(x_103)) { - x_113 = lean_alloc_ctor(1, 2, 0); -} else { - x_113 = x_103; - lean_ctor_set_tag(x_113, 1); -} -lean_ctor_set(x_113, 0, x_2); -lean_ctor_set(x_113, 1, x_108); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_113); -lean_ctor_set(x_21, 0, x_112); -x_114 = lean_array_mk(x_21); -x_115 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_116 = l_Lean_Meta_mkAppM(x_115, x_114, x_7, x_8, x_9, x_10, x_100); -if (lean_obj_tag(x_116) == 0) -{ -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_116, 1); -lean_inc(x_118); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_119 = x_116; -} else { - lean_dec_ref(x_116); - x_119 = lean_box(0); -} -x_120 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_121 = l_Lean_mkApp4(x_120, x_109, x_1, x_2, x_3); -lean_ctor_set(x_30, 0, x_121); -x_122 = 1; -x_123 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_123, 0, x_117); -lean_ctor_set(x_123, 1, x_30); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_122); -lean_ctor_set(x_13, 0, x_123); -if (lean_is_scalar(x_119)) { - x_124 = lean_alloc_ctor(0, 2, 0); -} else { - x_124 = x_119; -} -lean_ctor_set(x_124, 0, x_13); -lean_ctor_set(x_124, 1, x_118); -return x_124; -} -else -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -lean_dec(x_109); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_125 = lean_ctor_get(x_116, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_116, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_127 = x_116; -} else { - lean_dec_ref(x_116); - x_127 = lean_box(0); -} -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); -} else { - x_128 = x_127; -} -lean_ctor_set(x_128, 0, x_125); -lean_ctor_set(x_128, 1, x_126); -return x_128; -} -} -} -} -else -{ -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; -x_129 = lean_ctor_get(x_30, 0); -lean_inc(x_129); -lean_dec(x_30); -x_130 = lean_ctor_get(x_29, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_29)) { - lean_ctor_release(x_29, 0); - lean_ctor_release(x_29, 1); - x_131 = x_29; -} else { - lean_dec_ref(x_29); - x_131 = lean_box(0); -} -x_132 = lean_ctor_get(x_129, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_129, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_129)) { - lean_ctor_release(x_129, 0); - lean_ctor_release(x_129, 1); - x_134 = x_129; -} else { - lean_dec_ref(x_129); - x_134 = lean_box(0); -} -x_135 = lean_nat_dec_eq(x_24, x_132); -lean_dec(x_132); -if (x_135 == 0) -{ -lean_object* x_136; lean_object* x_137; -lean_dec(x_134); -lean_dec(x_133); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_136 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_131)) { - x_137 = lean_alloc_ctor(0, 2, 0); -} else { - x_137 = x_131; -} -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_130); -return x_137; -} -else -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -lean_dec(x_131); -x_138 = l_BitVec_add(x_24, x_25, x_133); -lean_dec(x_133); -lean_dec(x_25); -x_139 = lean_box(0); -x_140 = l_Lean_mkNatLit(x_24); -x_141 = l_Lean_mkNatLit(x_138); -x_142 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_140); -x_143 = l_Lean_mkAppB(x_142, x_140, x_141); -lean_inc(x_2); -if (lean_is_scalar(x_134)) { - x_144 = lean_alloc_ctor(1, 2, 0); -} else { - x_144 = x_134; - lean_ctor_set_tag(x_144, 1); -} -lean_ctor_set(x_144, 0, x_2); -lean_ctor_set(x_144, 1, x_139); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_144); -lean_ctor_set(x_21, 0, x_143); -x_145 = lean_array_mk(x_21); -x_146 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_147 = l_Lean_Meta_mkAppM(x_146, x_145, x_7, x_8, x_9, x_10, x_130); -if (lean_obj_tag(x_147) == 0) -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_147, 1); -lean_inc(x_149); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_150 = x_147; -} else { - lean_dec_ref(x_147); - x_150 = lean_box(0); -} -x_151 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_152 = l_Lean_mkApp4(x_151, x_140, x_1, x_2, x_3); -x_153 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_153, 0, x_152); -x_154 = 1; -x_155 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_155, 0, x_148); -lean_ctor_set(x_155, 1, x_153); -lean_ctor_set_uint8(x_155, sizeof(void*)*2, x_154); -lean_ctor_set(x_13, 0, x_155); -if (lean_is_scalar(x_150)) { - x_156 = lean_alloc_ctor(0, 2, 0); -} else { - x_156 = x_150; -} -lean_ctor_set(x_156, 0, x_13); -lean_ctor_set(x_156, 1, x_149); -return x_156; -} -else -{ -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; -lean_dec(x_140); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_157 = lean_ctor_get(x_147, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_147, 1); -lean_inc(x_158); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_159 = x_147; -} else { - lean_dec_ref(x_147); - x_159 = lean_box(0); -} -if (lean_is_scalar(x_159)) { - x_160 = lean_alloc_ctor(1, 2, 0); -} else { - x_160 = x_159; -} -lean_ctor_set(x_160, 0, x_157); -lean_ctor_set(x_160, 1, x_158); -return x_160; -} -} -} -} -} -else -{ -uint8_t x_161; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_161 = !lean_is_exclusive(x_29); -if (x_161 == 0) -{ -return x_29; -} -else -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; -x_162 = lean_ctor_get(x_29, 0); -x_163 = lean_ctor_get(x_29, 1); -lean_inc(x_163); -lean_inc(x_162); -lean_dec(x_29); -x_164 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set(x_164, 1, x_163); -return x_164; -} -} -} -else -{ -uint8_t x_165; -x_165 = !lean_is_exclusive(x_27); -if (x_165 == 0) -{ -uint8_t x_166; -x_166 = !lean_is_exclusive(x_26); -if (x_166 == 0) -{ -lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; -x_167 = lean_ctor_get(x_27, 0); -x_168 = lean_ctor_get(x_26, 1); -x_169 = lean_ctor_get(x_26, 0); -lean_dec(x_169); -x_170 = !lean_is_exclusive(x_167); -if (x_170 == 0) -{ -lean_object* x_171; lean_object* x_172; uint8_t x_173; -x_171 = lean_ctor_get(x_167, 0); -x_172 = lean_ctor_get(x_167, 1); -x_173 = lean_nat_dec_eq(x_24, x_171); -lean_dec(x_171); -if (x_173 == 0) -{ -lean_object* x_174; -lean_free_object(x_167); -lean_dec(x_172); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_174 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_26, 0, x_174); -return x_26; -} -else -{ -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -lean_free_object(x_26); -x_175 = l_BitVec_add(x_24, x_25, x_172); -lean_dec(x_172); -lean_dec(x_25); -x_176 = lean_box(0); -x_177 = l_Lean_mkNatLit(x_24); -x_178 = l_Lean_mkNatLit(x_175); -x_179 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_177); -x_180 = l_Lean_mkAppB(x_179, x_177, x_178); -lean_inc(x_3); -lean_ctor_set_tag(x_167, 1); -lean_ctor_set(x_167, 1, x_176); -lean_ctor_set(x_167, 0, x_3); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_167); -lean_ctor_set(x_21, 0, x_180); -x_181 = lean_array_mk(x_21); -x_182 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_183 = l_Lean_Meta_mkAppM(x_182, x_181, x_7, x_8, x_9, x_10, x_168); -if (lean_obj_tag(x_183) == 0) -{ -uint8_t x_184; -x_184 = !lean_is_exclusive(x_183); -if (x_184 == 0) -{ -lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; lean_object* x_189; -x_185 = lean_ctor_get(x_183, 0); -x_186 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_187 = l_Lean_mkApp4(x_186, x_177, x_1, x_2, x_3); -lean_ctor_set(x_27, 0, x_187); -x_188 = 1; -x_189 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_189, 0, x_185); -lean_ctor_set(x_189, 1, x_27); -lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_188); -lean_ctor_set(x_13, 0, x_189); -lean_ctor_set(x_183, 0, x_13); -return x_183; -} -else -{ -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; lean_object* x_195; lean_object* x_196; -x_190 = lean_ctor_get(x_183, 0); -x_191 = lean_ctor_get(x_183, 1); -lean_inc(x_191); -lean_inc(x_190); -lean_dec(x_183); -x_192 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_193 = l_Lean_mkApp4(x_192, x_177, x_1, x_2, x_3); -lean_ctor_set(x_27, 0, x_193); -x_194 = 1; -x_195 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_195, 0, x_190); -lean_ctor_set(x_195, 1, x_27); -lean_ctor_set_uint8(x_195, sizeof(void*)*2, x_194); -lean_ctor_set(x_13, 0, x_195); -x_196 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_196, 0, x_13); -lean_ctor_set(x_196, 1, x_191); -return x_196; -} -} -else -{ -uint8_t x_197; -lean_dec(x_177); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_197 = !lean_is_exclusive(x_183); -if (x_197 == 0) -{ -return x_183; -} -else -{ -lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_198 = lean_ctor_get(x_183, 0); -x_199 = lean_ctor_get(x_183, 1); -lean_inc(x_199); -lean_inc(x_198); -lean_dec(x_183); -x_200 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_200, 0, x_198); -lean_ctor_set(x_200, 1, x_199); -return x_200; -} -} -} -} -else -{ -lean_object* x_201; lean_object* x_202; uint8_t x_203; -x_201 = lean_ctor_get(x_167, 0); -x_202 = lean_ctor_get(x_167, 1); -lean_inc(x_202); -lean_inc(x_201); -lean_dec(x_167); -x_203 = lean_nat_dec_eq(x_24, x_201); -lean_dec(x_201); -if (x_203 == 0) -{ -lean_object* x_204; -lean_dec(x_202); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_204 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_26, 0, x_204); -return x_26; -} -else -{ -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -lean_free_object(x_26); -x_205 = l_BitVec_add(x_24, x_25, x_202); -lean_dec(x_202); -lean_dec(x_25); -x_206 = lean_box(0); -x_207 = l_Lean_mkNatLit(x_24); -x_208 = l_Lean_mkNatLit(x_205); -x_209 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_207); -x_210 = l_Lean_mkAppB(x_209, x_207, x_208); -lean_inc(x_3); -x_211 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_211, 0, x_3); -lean_ctor_set(x_211, 1, x_206); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_211); -lean_ctor_set(x_21, 0, x_210); -x_212 = lean_array_mk(x_21); -x_213 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_214 = l_Lean_Meta_mkAppM(x_213, x_212, x_7, x_8, x_9, x_10, x_168); -if (lean_obj_tag(x_214) == 0) -{ -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; lean_object* x_221; lean_object* x_222; -x_215 = lean_ctor_get(x_214, 0); -lean_inc(x_215); -x_216 = lean_ctor_get(x_214, 1); -lean_inc(x_216); -if (lean_is_exclusive(x_214)) { - lean_ctor_release(x_214, 0); - lean_ctor_release(x_214, 1); - x_217 = x_214; -} else { - lean_dec_ref(x_214); - x_217 = lean_box(0); -} -x_218 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_219 = l_Lean_mkApp4(x_218, x_207, x_1, x_2, x_3); -lean_ctor_set(x_27, 0, x_219); -x_220 = 1; -x_221 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_221, 0, x_215); -lean_ctor_set(x_221, 1, x_27); -lean_ctor_set_uint8(x_221, sizeof(void*)*2, x_220); -lean_ctor_set(x_13, 0, x_221); -if (lean_is_scalar(x_217)) { - x_222 = lean_alloc_ctor(0, 2, 0); -} else { - x_222 = x_217; -} -lean_ctor_set(x_222, 0, x_13); -lean_ctor_set(x_222, 1, x_216); -return x_222; -} -else -{ -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -lean_dec(x_207); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_223 = lean_ctor_get(x_214, 0); -lean_inc(x_223); -x_224 = lean_ctor_get(x_214, 1); -lean_inc(x_224); -if (lean_is_exclusive(x_214)) { - lean_ctor_release(x_214, 0); - lean_ctor_release(x_214, 1); - x_225 = x_214; -} else { - lean_dec_ref(x_214); - x_225 = lean_box(0); -} -if (lean_is_scalar(x_225)) { - x_226 = lean_alloc_ctor(1, 2, 0); -} else { - x_226 = x_225; -} -lean_ctor_set(x_226, 0, x_223); -lean_ctor_set(x_226, 1, x_224); -return x_226; -} -} -} -} -else -{ -lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; uint8_t x_232; -x_227 = lean_ctor_get(x_27, 0); -x_228 = lean_ctor_get(x_26, 1); -lean_inc(x_228); -lean_dec(x_26); -x_229 = lean_ctor_get(x_227, 0); -lean_inc(x_229); -x_230 = lean_ctor_get(x_227, 1); -lean_inc(x_230); -if (lean_is_exclusive(x_227)) { - lean_ctor_release(x_227, 0); - lean_ctor_release(x_227, 1); - x_231 = x_227; -} else { - lean_dec_ref(x_227); - x_231 = lean_box(0); -} -x_232 = lean_nat_dec_eq(x_24, x_229); -lean_dec(x_229); -if (x_232 == 0) -{ -lean_object* x_233; lean_object* x_234; -lean_dec(x_231); -lean_dec(x_230); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_233 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_234 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_234, 0, x_233); -lean_ctor_set(x_234, 1, x_228); -return x_234; -} -else -{ -lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -x_235 = l_BitVec_add(x_24, x_25, x_230); -lean_dec(x_230); -lean_dec(x_25); -x_236 = lean_box(0); -x_237 = l_Lean_mkNatLit(x_24); -x_238 = l_Lean_mkNatLit(x_235); -x_239 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_237); -x_240 = l_Lean_mkAppB(x_239, x_237, x_238); -lean_inc(x_3); -if (lean_is_scalar(x_231)) { - x_241 = lean_alloc_ctor(1, 2, 0); -} else { - x_241 = x_231; - lean_ctor_set_tag(x_241, 1); -} -lean_ctor_set(x_241, 0, x_3); -lean_ctor_set(x_241, 1, x_236); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_241); -lean_ctor_set(x_21, 0, x_240); -x_242 = lean_array_mk(x_21); -x_243 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_244 = l_Lean_Meta_mkAppM(x_243, x_242, x_7, x_8, x_9, x_10, x_228); -if (lean_obj_tag(x_244) == 0) -{ -lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; uint8_t x_250; lean_object* x_251; lean_object* x_252; -x_245 = lean_ctor_get(x_244, 0); -lean_inc(x_245); -x_246 = lean_ctor_get(x_244, 1); -lean_inc(x_246); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - lean_ctor_release(x_244, 1); - x_247 = x_244; -} else { - lean_dec_ref(x_244); - x_247 = lean_box(0); -} -x_248 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_249 = l_Lean_mkApp4(x_248, x_237, x_1, x_2, x_3); -lean_ctor_set(x_27, 0, x_249); -x_250 = 1; -x_251 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_251, 0, x_245); -lean_ctor_set(x_251, 1, x_27); -lean_ctor_set_uint8(x_251, sizeof(void*)*2, x_250); -lean_ctor_set(x_13, 0, x_251); -if (lean_is_scalar(x_247)) { - x_252 = lean_alloc_ctor(0, 2, 0); -} else { - x_252 = x_247; -} -lean_ctor_set(x_252, 0, x_13); -lean_ctor_set(x_252, 1, x_246); -return x_252; -} -else -{ -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -lean_dec(x_237); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_253 = lean_ctor_get(x_244, 0); -lean_inc(x_253); -x_254 = lean_ctor_get(x_244, 1); -lean_inc(x_254); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - lean_ctor_release(x_244, 1); - x_255 = x_244; -} else { - lean_dec_ref(x_244); - x_255 = lean_box(0); -} -if (lean_is_scalar(x_255)) { - x_256 = lean_alloc_ctor(1, 2, 0); -} else { - x_256 = x_255; -} -lean_ctor_set(x_256, 0, x_253); -lean_ctor_set(x_256, 1, x_254); -return x_256; -} -} -} -} -else -{ -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; uint8_t x_263; -x_257 = lean_ctor_get(x_27, 0); -lean_inc(x_257); -lean_dec(x_27); -x_258 = lean_ctor_get(x_26, 1); -lean_inc(x_258); -if (lean_is_exclusive(x_26)) { - lean_ctor_release(x_26, 0); - lean_ctor_release(x_26, 1); - x_259 = x_26; -} else { - lean_dec_ref(x_26); - x_259 = lean_box(0); -} -x_260 = lean_ctor_get(x_257, 0); -lean_inc(x_260); -x_261 = lean_ctor_get(x_257, 1); -lean_inc(x_261); -if (lean_is_exclusive(x_257)) { - lean_ctor_release(x_257, 0); - lean_ctor_release(x_257, 1); - x_262 = x_257; -} else { - lean_dec_ref(x_257); - x_262 = lean_box(0); -} -x_263 = lean_nat_dec_eq(x_24, x_260); -lean_dec(x_260); -if (x_263 == 0) -{ -lean_object* x_264; lean_object* x_265; -lean_dec(x_262); -lean_dec(x_261); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_264 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_259)) { - x_265 = lean_alloc_ctor(0, 2, 0); -} else { - x_265 = x_259; -} -lean_ctor_set(x_265, 0, x_264); -lean_ctor_set(x_265, 1, x_258); -return x_265; -} -else -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; -lean_dec(x_259); -x_266 = l_BitVec_add(x_24, x_25, x_261); -lean_dec(x_261); -lean_dec(x_25); -x_267 = lean_box(0); -x_268 = l_Lean_mkNatLit(x_24); -x_269 = l_Lean_mkNatLit(x_266); -x_270 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_268); -x_271 = l_Lean_mkAppB(x_270, x_268, x_269); -lean_inc(x_3); -if (lean_is_scalar(x_262)) { - x_272 = lean_alloc_ctor(1, 2, 0); -} else { - x_272 = x_262; - lean_ctor_set_tag(x_272, 1); -} -lean_ctor_set(x_272, 0, x_3); -lean_ctor_set(x_272, 1, x_267); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_272); -lean_ctor_set(x_21, 0, x_271); -x_273 = lean_array_mk(x_21); -x_274 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_275 = l_Lean_Meta_mkAppM(x_274, x_273, x_7, x_8, x_9, x_10, x_258); -if (lean_obj_tag(x_275) == 0) -{ -lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; uint8_t x_282; lean_object* x_283; lean_object* x_284; -x_276 = lean_ctor_get(x_275, 0); -lean_inc(x_276); -x_277 = lean_ctor_get(x_275, 1); -lean_inc(x_277); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_278 = x_275; -} else { - lean_dec_ref(x_275); - x_278 = lean_box(0); -} -x_279 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_280 = l_Lean_mkApp4(x_279, x_268, x_1, x_2, x_3); -x_281 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_281, 0, x_280); -x_282 = 1; -x_283 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_283, 0, x_276); -lean_ctor_set(x_283, 1, x_281); -lean_ctor_set_uint8(x_283, sizeof(void*)*2, x_282); -lean_ctor_set(x_13, 0, x_283); -if (lean_is_scalar(x_278)) { - x_284 = lean_alloc_ctor(0, 2, 0); -} else { - x_284 = x_278; -} -lean_ctor_set(x_284, 0, x_13); -lean_ctor_set(x_284, 1, x_277); -return x_284; -} -else -{ -lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; -lean_dec(x_268); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_285 = lean_ctor_get(x_275, 0); -lean_inc(x_285); -x_286 = lean_ctor_get(x_275, 1); -lean_inc(x_286); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_287 = x_275; -} else { - lean_dec_ref(x_275); - x_287 = lean_box(0); -} -if (lean_is_scalar(x_287)) { - x_288 = lean_alloc_ctor(1, 2, 0); -} else { - x_288 = x_287; -} -lean_ctor_set(x_288, 0, x_285); -lean_ctor_set(x_288, 1, x_286); -return x_288; -} -} -} -} -} -else -{ -uint8_t x_289; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_289 = !lean_is_exclusive(x_26); -if (x_289 == 0) -{ -return x_26; -} -else -{ -lean_object* x_290; lean_object* x_291; lean_object* x_292; -x_290 = lean_ctor_get(x_26, 0); -x_291 = lean_ctor_get(x_26, 1); -lean_inc(x_291); -lean_inc(x_290); -lean_dec(x_26); -x_292 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_292, 0, x_290); -lean_ctor_set(x_292, 1, x_291); -return x_292; -} -} -} -else -{ -lean_object* x_293; lean_object* x_294; lean_object* x_295; -x_293 = lean_ctor_get(x_21, 0); -x_294 = lean_ctor_get(x_21, 1); -lean_inc(x_294); -lean_inc(x_293); -lean_dec(x_21); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_295 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); -if (lean_obj_tag(x_295) == 0) -{ -lean_object* x_296; -x_296 = lean_ctor_get(x_295, 0); -lean_inc(x_296); -if (lean_obj_tag(x_296) == 0) -{ -lean_object* x_297; lean_object* x_298; -x_297 = lean_ctor_get(x_295, 1); -lean_inc(x_297); -lean_dec(x_295); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_298 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_297); -if (lean_obj_tag(x_298) == 0) -{ -lean_object* x_299; -x_299 = lean_ctor_get(x_298, 0); -lean_inc(x_299); -if (lean_obj_tag(x_299) == 0) -{ -lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_300 = lean_ctor_get(x_298, 1); -lean_inc(x_300); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_301 = x_298; -} else { - lean_dec_ref(x_298); - x_301 = lean_box(0); -} -x_302 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_301)) { - x_303 = lean_alloc_ctor(0, 2, 0); -} else { - x_303 = x_301; -} -lean_ctor_set(x_303, 0, x_302); -lean_ctor_set(x_303, 1, x_300); -return x_303; -} -else -{ -lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; uint8_t x_311; -x_304 = lean_ctor_get(x_299, 0); -lean_inc(x_304); -if (lean_is_exclusive(x_299)) { - lean_ctor_release(x_299, 0); - x_305 = x_299; -} else { - lean_dec_ref(x_299); - x_305 = lean_box(0); -} -x_306 = lean_ctor_get(x_298, 1); -lean_inc(x_306); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_307 = x_298; -} else { - lean_dec_ref(x_298); - x_307 = lean_box(0); -} -x_308 = lean_ctor_get(x_304, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_304, 1); -lean_inc(x_309); -if (lean_is_exclusive(x_304)) { - lean_ctor_release(x_304, 0); - lean_ctor_release(x_304, 1); - x_310 = x_304; -} else { - lean_dec_ref(x_304); - x_310 = lean_box(0); -} -x_311 = lean_nat_dec_eq(x_293, x_308); -lean_dec(x_308); -if (x_311 == 0) -{ -lean_object* x_312; lean_object* x_313; -lean_dec(x_310); -lean_dec(x_309); -lean_dec(x_305); -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_312 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_307)) { - x_313 = lean_alloc_ctor(0, 2, 0); -} else { - x_313 = x_307; -} -lean_ctor_set(x_313, 0, x_312); -lean_ctor_set(x_313, 1, x_306); -return x_313; -} -else -{ -lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; -lean_dec(x_307); -x_314 = l_BitVec_add(x_293, x_294, x_309); -lean_dec(x_309); -lean_dec(x_294); -x_315 = lean_box(0); -x_316 = l_Lean_mkNatLit(x_293); -x_317 = l_Lean_mkNatLit(x_314); -x_318 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_316); -x_319 = l_Lean_mkAppB(x_318, x_316, x_317); -lean_inc(x_2); -if (lean_is_scalar(x_310)) { - x_320 = lean_alloc_ctor(1, 2, 0); -} else { - x_320 = x_310; - lean_ctor_set_tag(x_320, 1); -} -lean_ctor_set(x_320, 0, x_2); -lean_ctor_set(x_320, 1, x_315); -x_321 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_321, 0, x_319); -lean_ctor_set(x_321, 1, x_320); -x_322 = lean_array_mk(x_321); -x_323 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_324 = l_Lean_Meta_mkAppM(x_323, x_322, x_7, x_8, x_9, x_10, x_306); -if (lean_obj_tag(x_324) == 0) -{ -lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; uint8_t x_331; lean_object* x_332; lean_object* x_333; -x_325 = lean_ctor_get(x_324, 0); -lean_inc(x_325); -x_326 = lean_ctor_get(x_324, 1); -lean_inc(x_326); -if (lean_is_exclusive(x_324)) { - lean_ctor_release(x_324, 0); - lean_ctor_release(x_324, 1); - x_327 = x_324; -} else { - lean_dec_ref(x_324); - x_327 = lean_box(0); -} -x_328 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_329 = l_Lean_mkApp4(x_328, x_316, x_1, x_2, x_3); -if (lean_is_scalar(x_305)) { - x_330 = lean_alloc_ctor(1, 1, 0); -} else { - x_330 = x_305; -} -lean_ctor_set(x_330, 0, x_329); -x_331 = 1; -x_332 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_332, 0, x_325); -lean_ctor_set(x_332, 1, x_330); -lean_ctor_set_uint8(x_332, sizeof(void*)*2, x_331); -lean_ctor_set(x_13, 0, x_332); -if (lean_is_scalar(x_327)) { - x_333 = lean_alloc_ctor(0, 2, 0); -} else { - x_333 = x_327; -} -lean_ctor_set(x_333, 0, x_13); -lean_ctor_set(x_333, 1, x_326); -return x_333; -} -else -{ -lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; -lean_dec(x_316); -lean_dec(x_305); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_334 = lean_ctor_get(x_324, 0); -lean_inc(x_334); -x_335 = lean_ctor_get(x_324, 1); -lean_inc(x_335); -if (lean_is_exclusive(x_324)) { - lean_ctor_release(x_324, 0); - lean_ctor_release(x_324, 1); - x_336 = x_324; -} else { - lean_dec_ref(x_324); - x_336 = lean_box(0); -} -if (lean_is_scalar(x_336)) { - x_337 = lean_alloc_ctor(1, 2, 0); -} else { - x_337 = x_336; -} -lean_ctor_set(x_337, 0, x_334); -lean_ctor_set(x_337, 1, x_335); -return x_337; -} -} -} -} -else -{ -lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_338 = lean_ctor_get(x_298, 0); -lean_inc(x_338); -x_339 = lean_ctor_get(x_298, 1); -lean_inc(x_339); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_340 = x_298; -} else { - lean_dec_ref(x_298); - x_340 = lean_box(0); -} -if (lean_is_scalar(x_340)) { - x_341 = lean_alloc_ctor(1, 2, 0); -} else { - x_341 = x_340; -} -lean_ctor_set(x_341, 0, x_338); -lean_ctor_set(x_341, 1, x_339); -return x_341; -} -} -else -{ -lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; -x_342 = lean_ctor_get(x_296, 0); -lean_inc(x_342); -if (lean_is_exclusive(x_296)) { - lean_ctor_release(x_296, 0); - x_343 = x_296; -} else { - lean_dec_ref(x_296); - x_343 = lean_box(0); -} -x_344 = lean_ctor_get(x_295, 1); -lean_inc(x_344); -if (lean_is_exclusive(x_295)) { - lean_ctor_release(x_295, 0); - lean_ctor_release(x_295, 1); - x_345 = x_295; -} else { - lean_dec_ref(x_295); - x_345 = lean_box(0); -} -x_346 = lean_ctor_get(x_342, 0); -lean_inc(x_346); -x_347 = lean_ctor_get(x_342, 1); -lean_inc(x_347); -if (lean_is_exclusive(x_342)) { - lean_ctor_release(x_342, 0); - lean_ctor_release(x_342, 1); - x_348 = x_342; -} else { - lean_dec_ref(x_342); - x_348 = lean_box(0); -} -x_349 = lean_nat_dec_eq(x_293, x_346); -lean_dec(x_346); -if (x_349 == 0) -{ -lean_object* x_350; lean_object* x_351; -lean_dec(x_348); -lean_dec(x_347); -lean_dec(x_343); -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_350 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_345)) { - x_351 = lean_alloc_ctor(0, 2, 0); -} else { - x_351 = x_345; -} -lean_ctor_set(x_351, 0, x_350); -lean_ctor_set(x_351, 1, x_344); -return x_351; -} -else -{ -lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; -lean_dec(x_345); -x_352 = l_BitVec_add(x_293, x_294, x_347); -lean_dec(x_347); -lean_dec(x_294); -x_353 = lean_box(0); -x_354 = l_Lean_mkNatLit(x_293); -x_355 = l_Lean_mkNatLit(x_352); -x_356 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_354); -x_357 = l_Lean_mkAppB(x_356, x_354, x_355); -lean_inc(x_3); -if (lean_is_scalar(x_348)) { - x_358 = lean_alloc_ctor(1, 2, 0); -} else { - x_358 = x_348; - lean_ctor_set_tag(x_358, 1); -} -lean_ctor_set(x_358, 0, x_3); -lean_ctor_set(x_358, 1, x_353); -x_359 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_359, 0, x_357); -lean_ctor_set(x_359, 1, x_358); -x_360 = lean_array_mk(x_359); -x_361 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_362 = l_Lean_Meta_mkAppM(x_361, x_360, x_7, x_8, x_9, x_10, x_344); -if (lean_obj_tag(x_362) == 0) -{ -lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; uint8_t x_369; lean_object* x_370; lean_object* x_371; -x_363 = lean_ctor_get(x_362, 0); -lean_inc(x_363); -x_364 = lean_ctor_get(x_362, 1); -lean_inc(x_364); -if (lean_is_exclusive(x_362)) { - lean_ctor_release(x_362, 0); - lean_ctor_release(x_362, 1); - x_365 = x_362; -} else { - lean_dec_ref(x_362); - x_365 = lean_box(0); -} -x_366 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_367 = l_Lean_mkApp4(x_366, x_354, x_1, x_2, x_3); -if (lean_is_scalar(x_343)) { - x_368 = lean_alloc_ctor(1, 1, 0); -} else { - x_368 = x_343; -} -lean_ctor_set(x_368, 0, x_367); -x_369 = 1; -x_370 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_370, 0, x_363); -lean_ctor_set(x_370, 1, x_368); -lean_ctor_set_uint8(x_370, sizeof(void*)*2, x_369); -lean_ctor_set(x_13, 0, x_370); -if (lean_is_scalar(x_365)) { - x_371 = lean_alloc_ctor(0, 2, 0); -} else { - x_371 = x_365; -} -lean_ctor_set(x_371, 0, x_13); -lean_ctor_set(x_371, 1, x_364); -return x_371; -} -else -{ -lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; -lean_dec(x_354); -lean_dec(x_343); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_372 = lean_ctor_get(x_362, 0); -lean_inc(x_372); -x_373 = lean_ctor_get(x_362, 1); -lean_inc(x_373); -if (lean_is_exclusive(x_362)) { - lean_ctor_release(x_362, 0); - lean_ctor_release(x_362, 1); - x_374 = x_362; -} else { - lean_dec_ref(x_362); - x_374 = lean_box(0); -} -if (lean_is_scalar(x_374)) { - x_375 = lean_alloc_ctor(1, 2, 0); -} else { - x_375 = x_374; -} -lean_ctor_set(x_375, 0, x_372); -lean_ctor_set(x_375, 1, x_373); -return x_375; -} -} -} -} -else -{ -lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_376 = lean_ctor_get(x_295, 0); -lean_inc(x_376); -x_377 = lean_ctor_get(x_295, 1); -lean_inc(x_377); -if (lean_is_exclusive(x_295)) { - lean_ctor_release(x_295, 0); - lean_ctor_release(x_295, 1); - x_378 = x_295; -} else { - lean_dec_ref(x_295); - x_378 = lean_box(0); -} -if (lean_is_scalar(x_378)) { - x_379 = lean_alloc_ctor(1, 2, 0); -} else { - x_379 = x_378; -} -lean_ctor_set(x_379, 0, x_376); -lean_ctor_set(x_379, 1, x_377); -return x_379; -} -} -} -else -{ -lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; -x_380 = lean_ctor_get(x_13, 0); -lean_inc(x_380); -lean_dec(x_13); -x_381 = lean_ctor_get(x_12, 1); -lean_inc(x_381); -lean_dec(x_12); -x_382 = lean_ctor_get(x_380, 0); -lean_inc(x_382); -x_383 = lean_ctor_get(x_380, 1); -lean_inc(x_383); -if (lean_is_exclusive(x_380)) { - lean_ctor_release(x_380, 0); - lean_ctor_release(x_380, 1); - x_384 = x_380; -} else { - lean_dec_ref(x_380); - x_384 = lean_box(0); -} -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_385 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_381); -if (lean_obj_tag(x_385) == 0) -{ -lean_object* x_386; -x_386 = lean_ctor_get(x_385, 0); -lean_inc(x_386); -if (lean_obj_tag(x_386) == 0) -{ -lean_object* x_387; lean_object* x_388; -x_387 = lean_ctor_get(x_385, 1); -lean_inc(x_387); -lean_dec(x_385); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_388 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_387); -if (lean_obj_tag(x_388) == 0) -{ -lean_object* x_389; -x_389 = lean_ctor_get(x_388, 0); -lean_inc(x_389); -if (lean_obj_tag(x_389) == 0) -{ -lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_390 = lean_ctor_get(x_388, 1); -lean_inc(x_390); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_391 = x_388; -} else { - lean_dec_ref(x_388); - x_391 = lean_box(0); -} -x_392 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_391)) { - x_393 = lean_alloc_ctor(0, 2, 0); -} else { - x_393 = x_391; -} -lean_ctor_set(x_393, 0, x_392); -lean_ctor_set(x_393, 1, x_390); -return x_393; -} -else -{ -lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; uint8_t x_401; -x_394 = lean_ctor_get(x_389, 0); -lean_inc(x_394); -if (lean_is_exclusive(x_389)) { - lean_ctor_release(x_389, 0); - x_395 = x_389; -} else { - lean_dec_ref(x_389); - x_395 = lean_box(0); -} -x_396 = lean_ctor_get(x_388, 1); -lean_inc(x_396); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_397 = x_388; -} else { - lean_dec_ref(x_388); - x_397 = lean_box(0); -} -x_398 = lean_ctor_get(x_394, 0); -lean_inc(x_398); -x_399 = lean_ctor_get(x_394, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_394)) { - lean_ctor_release(x_394, 0); - lean_ctor_release(x_394, 1); - x_400 = x_394; -} else { - lean_dec_ref(x_394); - x_400 = lean_box(0); -} -x_401 = lean_nat_dec_eq(x_382, x_398); -lean_dec(x_398); -if (x_401 == 0) -{ -lean_object* x_402; lean_object* x_403; -lean_dec(x_400); -lean_dec(x_399); -lean_dec(x_395); -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_402 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_397)) { - x_403 = lean_alloc_ctor(0, 2, 0); -} else { - x_403 = x_397; -} -lean_ctor_set(x_403, 0, x_402); -lean_ctor_set(x_403, 1, x_396); -return x_403; -} -else -{ -lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; -lean_dec(x_397); -x_404 = l_BitVec_add(x_382, x_383, x_399); -lean_dec(x_399); -lean_dec(x_383); -x_405 = lean_box(0); -x_406 = l_Lean_mkNatLit(x_382); -x_407 = l_Lean_mkNatLit(x_404); -x_408 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_406); -x_409 = l_Lean_mkAppB(x_408, x_406, x_407); -lean_inc(x_2); -if (lean_is_scalar(x_400)) { - x_410 = lean_alloc_ctor(1, 2, 0); -} else { - x_410 = x_400; - lean_ctor_set_tag(x_410, 1); -} -lean_ctor_set(x_410, 0, x_2); -lean_ctor_set(x_410, 1, x_405); -if (lean_is_scalar(x_384)) { - x_411 = lean_alloc_ctor(1, 2, 0); -} else { - x_411 = x_384; - lean_ctor_set_tag(x_411, 1); -} -lean_ctor_set(x_411, 0, x_409); -lean_ctor_set(x_411, 1, x_410); -x_412 = lean_array_mk(x_411); -x_413 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_414 = l_Lean_Meta_mkAppM(x_413, x_412, x_7, x_8, x_9, x_10, x_396); -if (lean_obj_tag(x_414) == 0) -{ -lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; -x_415 = lean_ctor_get(x_414, 0); -lean_inc(x_415); -x_416 = lean_ctor_get(x_414, 1); -lean_inc(x_416); -if (lean_is_exclusive(x_414)) { - lean_ctor_release(x_414, 0); - lean_ctor_release(x_414, 1); - x_417 = x_414; -} else { - lean_dec_ref(x_414); - x_417 = lean_box(0); -} -x_418 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; -x_419 = l_Lean_mkApp4(x_418, x_406, x_1, x_2, x_3); -if (lean_is_scalar(x_395)) { - x_420 = lean_alloc_ctor(1, 1, 0); -} else { - x_420 = x_395; -} -lean_ctor_set(x_420, 0, x_419); -x_421 = 1; -x_422 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_422, 0, x_415); -lean_ctor_set(x_422, 1, x_420); -lean_ctor_set_uint8(x_422, sizeof(void*)*2, x_421); -x_423 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_423, 0, x_422); -if (lean_is_scalar(x_417)) { - x_424 = lean_alloc_ctor(0, 2, 0); -} else { - x_424 = x_417; -} -lean_ctor_set(x_424, 0, x_423); -lean_ctor_set(x_424, 1, x_416); -return x_424; -} -else -{ -lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; -lean_dec(x_406); -lean_dec(x_395); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_425 = lean_ctor_get(x_414, 0); -lean_inc(x_425); -x_426 = lean_ctor_get(x_414, 1); -lean_inc(x_426); -if (lean_is_exclusive(x_414)) { - lean_ctor_release(x_414, 0); - lean_ctor_release(x_414, 1); - x_427 = x_414; -} else { - lean_dec_ref(x_414); - x_427 = lean_box(0); -} -if (lean_is_scalar(x_427)) { - x_428 = lean_alloc_ctor(1, 2, 0); -} else { - x_428 = x_427; -} -lean_ctor_set(x_428, 0, x_425); -lean_ctor_set(x_428, 1, x_426); -return x_428; -} -} -} -} -else -{ -lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_429 = lean_ctor_get(x_388, 0); -lean_inc(x_429); -x_430 = lean_ctor_get(x_388, 1); -lean_inc(x_430); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_431 = x_388; -} else { - lean_dec_ref(x_388); - x_431 = lean_box(0); -} -if (lean_is_scalar(x_431)) { - x_432 = lean_alloc_ctor(1, 2, 0); -} else { - x_432 = x_431; -} -lean_ctor_set(x_432, 0, x_429); -lean_ctor_set(x_432, 1, x_430); -return x_432; -} -} -else -{ -lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; uint8_t x_440; -x_433 = lean_ctor_get(x_386, 0); -lean_inc(x_433); -if (lean_is_exclusive(x_386)) { - lean_ctor_release(x_386, 0); - x_434 = x_386; -} else { - lean_dec_ref(x_386); - x_434 = lean_box(0); -} -x_435 = lean_ctor_get(x_385, 1); -lean_inc(x_435); -if (lean_is_exclusive(x_385)) { - lean_ctor_release(x_385, 0); - lean_ctor_release(x_385, 1); - x_436 = x_385; -} else { - lean_dec_ref(x_385); - x_436 = lean_box(0); -} -x_437 = lean_ctor_get(x_433, 0); -lean_inc(x_437); -x_438 = lean_ctor_get(x_433, 1); -lean_inc(x_438); -if (lean_is_exclusive(x_433)) { - lean_ctor_release(x_433, 0); - lean_ctor_release(x_433, 1); - x_439 = x_433; -} else { - lean_dec_ref(x_433); - x_439 = lean_box(0); -} -x_440 = lean_nat_dec_eq(x_382, x_437); -lean_dec(x_437); -if (x_440 == 0) -{ -lean_object* x_441; lean_object* x_442; -lean_dec(x_439); -lean_dec(x_438); -lean_dec(x_434); -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_441 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_436)) { - x_442 = lean_alloc_ctor(0, 2, 0); -} else { - x_442 = x_436; -} -lean_ctor_set(x_442, 0, x_441); -lean_ctor_set(x_442, 1, x_435); -return x_442; -} -else -{ -lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; -lean_dec(x_436); -x_443 = l_BitVec_add(x_382, x_383, x_438); -lean_dec(x_438); -lean_dec(x_383); -x_444 = lean_box(0); -x_445 = l_Lean_mkNatLit(x_382); -x_446 = l_Lean_mkNatLit(x_443); -x_447 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_445); -x_448 = l_Lean_mkAppB(x_447, x_445, x_446); -lean_inc(x_3); -if (lean_is_scalar(x_439)) { - x_449 = lean_alloc_ctor(1, 2, 0); -} else { - x_449 = x_439; - lean_ctor_set_tag(x_449, 1); -} -lean_ctor_set(x_449, 0, x_3); -lean_ctor_set(x_449, 1, x_444); -if (lean_is_scalar(x_384)) { - x_450 = lean_alloc_ctor(1, 2, 0); -} else { - x_450 = x_384; - lean_ctor_set_tag(x_450, 1); -} -lean_ctor_set(x_450, 0, x_448); -lean_ctor_set(x_450, 1, x_449); -x_451 = lean_array_mk(x_450); -x_452 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_453 = l_Lean_Meta_mkAppM(x_452, x_451, x_7, x_8, x_9, x_10, x_435); -if (lean_obj_tag(x_453) == 0) -{ -lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; uint8_t x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; -x_454 = lean_ctor_get(x_453, 0); -lean_inc(x_454); -x_455 = lean_ctor_get(x_453, 1); -lean_inc(x_455); -if (lean_is_exclusive(x_453)) { - lean_ctor_release(x_453, 0); - lean_ctor_release(x_453, 1); - x_456 = x_453; -} else { - lean_dec_ref(x_453); - x_456 = lean_box(0); -} -x_457 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; -x_458 = l_Lean_mkApp4(x_457, x_445, x_1, x_2, x_3); -if (lean_is_scalar(x_434)) { - x_459 = lean_alloc_ctor(1, 1, 0); -} else { - x_459 = x_434; -} -lean_ctor_set(x_459, 0, x_458); -x_460 = 1; -x_461 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_461, 0, x_454); -lean_ctor_set(x_461, 1, x_459); -lean_ctor_set_uint8(x_461, sizeof(void*)*2, x_460); -x_462 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_462, 0, x_461); -if (lean_is_scalar(x_456)) { - x_463 = lean_alloc_ctor(0, 2, 0); -} else { - x_463 = x_456; -} -lean_ctor_set(x_463, 0, x_462); -lean_ctor_set(x_463, 1, x_455); -return x_463; -} -else -{ -lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; -lean_dec(x_445); -lean_dec(x_434); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_464 = lean_ctor_get(x_453, 0); -lean_inc(x_464); -x_465 = lean_ctor_get(x_453, 1); -lean_inc(x_465); -if (lean_is_exclusive(x_453)) { - lean_ctor_release(x_453, 0); - lean_ctor_release(x_453, 1); - x_466 = x_453; -} else { - lean_dec_ref(x_453); - x_466 = lean_box(0); -} -if (lean_is_scalar(x_466)) { - x_467 = lean_alloc_ctor(1, 2, 0); -} else { - x_467 = x_466; -} -lean_ctor_set(x_467, 0, x_464); -lean_ctor_set(x_467, 1, x_465); -return x_467; -} -} -} -} -else -{ -lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_468 = lean_ctor_get(x_385, 0); -lean_inc(x_468); -x_469 = lean_ctor_get(x_385, 1); -lean_inc(x_469); -if (lean_is_exclusive(x_385)) { - lean_ctor_release(x_385, 0); - lean_ctor_release(x_385, 1); - x_470 = x_385; -} else { - lean_dec_ref(x_385); - x_470 = lean_box(0); -} -if (lean_is_scalar(x_470)) { - x_471 = lean_alloc_ctor(1, 2, 0); -} else { - x_471 = x_470; -} -lean_ctor_set(x_471, 0, x_468); -lean_ctor_set(x_471, 1, x_469); -return x_471; -} -} -} -} -else -{ -uint8_t x_472; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_472 = !lean_is_exclusive(x_12); -if (x_472 == 0) -{ -return x_12; -} -else -{ -lean_object* x_473; lean_object* x_474; lean_object* x_475; -x_473 = lean_ctor_get(x_12, 0); -x_474 = lean_ctor_get(x_12, 1); -lean_inc(x_474); -lean_inc(x_473); -lean_dec(x_12); -x_475 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_475, 0, x_473); -lean_ctor_set(x_475, 1, x_474); -return x_475; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_2); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -lean_dec(x_1); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_1); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_1); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_1); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_1); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_1); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_1); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(x_1, x_21, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_43; -} -} -} -} -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2), 10, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_43; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_12; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("bv_add_const", 12, 12); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_2 = lean_unsigned_to_nat(6u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("add_const_right'", 16, 16); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("add_const_left'", 15, 15); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_1); -x_12 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) -{ -lean_object* x_13; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_14 = !lean_is_exclusive(x_12); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 0); -lean_dec(x_15); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_12, 0, x_16); -return x_12; -} -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_dec(x_12); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; -} -} -else -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_13); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_13, 0); -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); -lean_dec(x_12); -x_23 = !lean_is_exclusive(x_21); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_21, 0); -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_26 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_29 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -if (lean_obj_tag(x_30) == 0) -{ -uint8_t x_31; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_31 = !lean_is_exclusive(x_29); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_33); -return x_29; -} -else -{ -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_29, 1); -lean_inc(x_34); -lean_dec(x_29); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -return x_36; -} -} -else -{ -uint8_t x_37; -x_37 = !lean_is_exclusive(x_30); -if (x_37 == 0) -{ -uint8_t x_38; -x_38 = !lean_is_exclusive(x_29); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_39 = lean_ctor_get(x_30, 0); -x_40 = lean_ctor_get(x_29, 1); -x_41 = lean_ctor_get(x_29, 0); -lean_dec(x_41); -x_42 = !lean_is_exclusive(x_39); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_43 = lean_ctor_get(x_39, 0); -x_44 = lean_ctor_get(x_39, 1); -x_45 = lean_nat_dec_eq(x_24, x_43); -lean_dec(x_43); -if (x_45 == 0) -{ -lean_object* x_46; -lean_free_object(x_39); -lean_dec(x_44); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_46); -return x_29; -} -else -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_free_object(x_29); -x_47 = l_BitVec_add(x_24, x_25, x_44); -lean_dec(x_44); -lean_dec(x_25); -x_48 = lean_box(0); -x_49 = l_Lean_mkNatLit(x_24); -x_50 = l_Lean_mkNatLit(x_47); -x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_49); -x_52 = l_Lean_mkAppB(x_51, x_49, x_50); -lean_inc(x_2); -lean_ctor_set_tag(x_39, 1); -lean_ctor_set(x_39, 1, x_48); -lean_ctor_set(x_39, 0, x_2); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_39); -lean_ctor_set(x_21, 0, x_52); -x_53 = lean_array_mk(x_21); -x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_55 = l_Lean_Meta_mkAppM(x_54, x_53, x_7, x_8, x_9, x_10, x_40); -if (lean_obj_tag(x_55) == 0) -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; -x_57 = lean_ctor_get(x_55, 0); -x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_59 = l_Lean_mkApp4(x_58, x_49, x_2, x_3, x_1); -lean_ctor_set(x_30, 0, x_59); -x_60 = 1; -x_61 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_61, 0, x_57); -lean_ctor_set(x_61, 1, x_30); -lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_60); -lean_ctor_set(x_13, 0, x_61); -lean_ctor_set(x_55, 0, x_13); -return x_55; -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; -x_62 = lean_ctor_get(x_55, 0); -x_63 = lean_ctor_get(x_55, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_55); -x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_65 = l_Lean_mkApp4(x_64, x_49, x_2, x_3, x_1); -lean_ctor_set(x_30, 0, x_65); -x_66 = 1; -x_67 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_67, 0, x_62); -lean_ctor_set(x_67, 1, x_30); -lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); -lean_ctor_set(x_13, 0, x_67); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_13); -lean_ctor_set(x_68, 1, x_63); -return x_68; -} -} -else -{ -uint8_t x_69; -lean_dec(x_49); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_69 = !lean_is_exclusive(x_55); -if (x_69 == 0) -{ -return x_55; -} -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_55, 0); -x_71 = lean_ctor_get(x_55, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_55); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; -} -} -} -} -else -{ -lean_object* x_73; lean_object* x_74; uint8_t x_75; -x_73 = lean_ctor_get(x_39, 0); -x_74 = lean_ctor_get(x_39, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_39); -x_75 = lean_nat_dec_eq(x_24, x_73); -lean_dec(x_73); -if (x_75 == 0) -{ -lean_object* x_76; -lean_dec(x_74); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_76 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_29, 0, x_76); -return x_29; -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -lean_free_object(x_29); -x_77 = l_BitVec_add(x_24, x_25, x_74); -lean_dec(x_74); -lean_dec(x_25); -x_78 = lean_box(0); -x_79 = l_Lean_mkNatLit(x_24); -x_80 = l_Lean_mkNatLit(x_77); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_79); -x_82 = l_Lean_mkAppB(x_81, x_79, x_80); -lean_inc(x_2); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_2); -lean_ctor_set(x_83, 1, x_78); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_83); -lean_ctor_set(x_21, 0, x_82); -x_84 = lean_array_mk(x_21); -x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_86 = l_Lean_Meta_mkAppM(x_85, x_84, x_7, x_8, x_9, x_10, x_40); -if (lean_obj_tag(x_86) == 0) -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_89 = x_86; -} else { - lean_dec_ref(x_86); - x_89 = lean_box(0); -} -x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_91 = l_Lean_mkApp4(x_90, x_79, x_2, x_3, x_1); -lean_ctor_set(x_30, 0, x_91); -x_92 = 1; -x_93 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_93, 0, x_87); -lean_ctor_set(x_93, 1, x_30); -lean_ctor_set_uint8(x_93, sizeof(void*)*2, x_92); -lean_ctor_set(x_13, 0, x_93); -if (lean_is_scalar(x_89)) { - x_94 = lean_alloc_ctor(0, 2, 0); -} else { - x_94 = x_89; -} -lean_ctor_set(x_94, 0, x_13); -lean_ctor_set(x_94, 1, x_88); -return x_94; -} -else -{ -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -lean_dec(x_79); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_95 = lean_ctor_get(x_86, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_86, 1); -lean_inc(x_96); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_97 = x_86; -} else { - lean_dec_ref(x_86); - x_97 = lean_box(0); -} -if (lean_is_scalar(x_97)) { - x_98 = lean_alloc_ctor(1, 2, 0); -} else { - x_98 = x_97; -} -lean_ctor_set(x_98, 0, x_95); -lean_ctor_set(x_98, 1, x_96); -return x_98; -} -} -} -} -else -{ -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; -x_99 = lean_ctor_get(x_30, 0); -x_100 = lean_ctor_get(x_29, 1); -lean_inc(x_100); -lean_dec(x_29); -x_101 = lean_ctor_get(x_99, 0); -lean_inc(x_101); -x_102 = lean_ctor_get(x_99, 1); -lean_inc(x_102); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_103 = x_99; -} else { - lean_dec_ref(x_99); - x_103 = lean_box(0); -} -x_104 = lean_nat_dec_eq(x_24, x_101); -lean_dec(x_101); -if (x_104 == 0) -{ -lean_object* x_105; lean_object* x_106; -lean_dec(x_103); -lean_dec(x_102); -lean_free_object(x_30); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_106 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_100); -return x_106; -} -else -{ -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_107 = l_BitVec_add(x_24, x_25, x_102); -lean_dec(x_102); -lean_dec(x_25); -x_108 = lean_box(0); -x_109 = l_Lean_mkNatLit(x_24); -x_110 = l_Lean_mkNatLit(x_107); -x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_109); -x_112 = l_Lean_mkAppB(x_111, x_109, x_110); -lean_inc(x_2); -if (lean_is_scalar(x_103)) { - x_113 = lean_alloc_ctor(1, 2, 0); -} else { - x_113 = x_103; - lean_ctor_set_tag(x_113, 1); -} -lean_ctor_set(x_113, 0, x_2); -lean_ctor_set(x_113, 1, x_108); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_113); -lean_ctor_set(x_21, 0, x_112); -x_114 = lean_array_mk(x_21); -x_115 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_116 = l_Lean_Meta_mkAppM(x_115, x_114, x_7, x_8, x_9, x_10, x_100); -if (lean_obj_tag(x_116) == 0) -{ -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_116, 1); -lean_inc(x_118); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_119 = x_116; -} else { - lean_dec_ref(x_116); - x_119 = lean_box(0); -} -x_120 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_121 = l_Lean_mkApp4(x_120, x_109, x_2, x_3, x_1); -lean_ctor_set(x_30, 0, x_121); -x_122 = 1; -x_123 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_123, 0, x_117); -lean_ctor_set(x_123, 1, x_30); -lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_122); -lean_ctor_set(x_13, 0, x_123); -if (lean_is_scalar(x_119)) { - x_124 = lean_alloc_ctor(0, 2, 0); -} else { - x_124 = x_119; -} -lean_ctor_set(x_124, 0, x_13); -lean_ctor_set(x_124, 1, x_118); -return x_124; -} -else -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -lean_dec(x_109); -lean_free_object(x_30); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_125 = lean_ctor_get(x_116, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_116, 1); -lean_inc(x_126); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_127 = x_116; -} else { - lean_dec_ref(x_116); - x_127 = lean_box(0); -} -if (lean_is_scalar(x_127)) { - x_128 = lean_alloc_ctor(1, 2, 0); -} else { - x_128 = x_127; -} -lean_ctor_set(x_128, 0, x_125); -lean_ctor_set(x_128, 1, x_126); -return x_128; -} -} -} -} -else -{ -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; -x_129 = lean_ctor_get(x_30, 0); -lean_inc(x_129); -lean_dec(x_30); -x_130 = lean_ctor_get(x_29, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_29)) { - lean_ctor_release(x_29, 0); - lean_ctor_release(x_29, 1); - x_131 = x_29; -} else { - lean_dec_ref(x_29); - x_131 = lean_box(0); -} -x_132 = lean_ctor_get(x_129, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_129, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_129)) { - lean_ctor_release(x_129, 0); - lean_ctor_release(x_129, 1); - x_134 = x_129; -} else { - lean_dec_ref(x_129); - x_134 = lean_box(0); -} -x_135 = lean_nat_dec_eq(x_24, x_132); -lean_dec(x_132); -if (x_135 == 0) -{ -lean_object* x_136; lean_object* x_137; -lean_dec(x_134); -lean_dec(x_133); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_136 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_131)) { - x_137 = lean_alloc_ctor(0, 2, 0); -} else { - x_137 = x_131; -} -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set(x_137, 1, x_130); -return x_137; -} -else -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -lean_dec(x_131); -x_138 = l_BitVec_add(x_24, x_25, x_133); -lean_dec(x_133); -lean_dec(x_25); -x_139 = lean_box(0); -x_140 = l_Lean_mkNatLit(x_24); -x_141 = l_Lean_mkNatLit(x_138); -x_142 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_140); -x_143 = l_Lean_mkAppB(x_142, x_140, x_141); -lean_inc(x_2); -if (lean_is_scalar(x_134)) { - x_144 = lean_alloc_ctor(1, 2, 0); -} else { - x_144 = x_134; - lean_ctor_set_tag(x_144, 1); -} -lean_ctor_set(x_144, 0, x_2); -lean_ctor_set(x_144, 1, x_139); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_144); -lean_ctor_set(x_21, 0, x_143); -x_145 = lean_array_mk(x_21); -x_146 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_147 = l_Lean_Meta_mkAppM(x_146, x_145, x_7, x_8, x_9, x_10, x_130); -if (lean_obj_tag(x_147) == 0) -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; -x_148 = lean_ctor_get(x_147, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_147, 1); -lean_inc(x_149); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_150 = x_147; -} else { - lean_dec_ref(x_147); - x_150 = lean_box(0); -} -x_151 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_152 = l_Lean_mkApp4(x_151, x_140, x_2, x_3, x_1); -x_153 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_153, 0, x_152); -x_154 = 1; -x_155 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_155, 0, x_148); -lean_ctor_set(x_155, 1, x_153); -lean_ctor_set_uint8(x_155, sizeof(void*)*2, x_154); -lean_ctor_set(x_13, 0, x_155); -if (lean_is_scalar(x_150)) { - x_156 = lean_alloc_ctor(0, 2, 0); -} else { - x_156 = x_150; -} -lean_ctor_set(x_156, 0, x_13); -lean_ctor_set(x_156, 1, x_149); -return x_156; -} -else -{ -lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; -lean_dec(x_140); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_157 = lean_ctor_get(x_147, 0); -lean_inc(x_157); -x_158 = lean_ctor_get(x_147, 1); -lean_inc(x_158); -if (lean_is_exclusive(x_147)) { - lean_ctor_release(x_147, 0); - lean_ctor_release(x_147, 1); - x_159 = x_147; -} else { - lean_dec_ref(x_147); - x_159 = lean_box(0); -} -if (lean_is_scalar(x_159)) { - x_160 = lean_alloc_ctor(1, 2, 0); -} else { - x_160 = x_159; -} -lean_ctor_set(x_160, 0, x_157); -lean_ctor_set(x_160, 1, x_158); -return x_160; -} -} -} -} -} -else -{ -uint8_t x_161; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_161 = !lean_is_exclusive(x_29); -if (x_161 == 0) -{ -return x_29; -} -else -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; -x_162 = lean_ctor_get(x_29, 0); -x_163 = lean_ctor_get(x_29, 1); -lean_inc(x_163); -lean_inc(x_162); -lean_dec(x_29); -x_164 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set(x_164, 1, x_163); -return x_164; -} -} -} -else -{ -uint8_t x_165; -x_165 = !lean_is_exclusive(x_27); -if (x_165 == 0) -{ -uint8_t x_166; -x_166 = !lean_is_exclusive(x_26); -if (x_166 == 0) -{ -lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; -x_167 = lean_ctor_get(x_27, 0); -x_168 = lean_ctor_get(x_26, 1); -x_169 = lean_ctor_get(x_26, 0); -lean_dec(x_169); -x_170 = !lean_is_exclusive(x_167); -if (x_170 == 0) -{ -lean_object* x_171; lean_object* x_172; uint8_t x_173; -x_171 = lean_ctor_get(x_167, 0); -x_172 = lean_ctor_get(x_167, 1); -x_173 = lean_nat_dec_eq(x_24, x_171); -lean_dec(x_171); -if (x_173 == 0) -{ -lean_object* x_174; -lean_free_object(x_167); -lean_dec(x_172); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_174 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_26, 0, x_174); -return x_26; -} -else -{ -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -lean_free_object(x_26); -x_175 = l_BitVec_add(x_24, x_25, x_172); -lean_dec(x_172); -lean_dec(x_25); -x_176 = lean_box(0); -x_177 = l_Lean_mkNatLit(x_24); -x_178 = l_Lean_mkNatLit(x_175); -x_179 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_177); -x_180 = l_Lean_mkAppB(x_179, x_177, x_178); -lean_inc(x_3); -lean_ctor_set_tag(x_167, 1); -lean_ctor_set(x_167, 1, x_176); -lean_ctor_set(x_167, 0, x_3); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_167); -lean_ctor_set(x_21, 0, x_180); -x_181 = lean_array_mk(x_21); -x_182 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_183 = l_Lean_Meta_mkAppM(x_182, x_181, x_7, x_8, x_9, x_10, x_168); -if (lean_obj_tag(x_183) == 0) -{ -uint8_t x_184; -x_184 = !lean_is_exclusive(x_183); -if (x_184 == 0) -{ -lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; lean_object* x_189; -x_185 = lean_ctor_get(x_183, 0); -x_186 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_187 = l_Lean_mkApp4(x_186, x_177, x_2, x_3, x_1); -lean_ctor_set(x_27, 0, x_187); -x_188 = 1; -x_189 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_189, 0, x_185); -lean_ctor_set(x_189, 1, x_27); -lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_188); -lean_ctor_set(x_13, 0, x_189); -lean_ctor_set(x_183, 0, x_13); -return x_183; -} -else -{ -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; lean_object* x_195; lean_object* x_196; -x_190 = lean_ctor_get(x_183, 0); -x_191 = lean_ctor_get(x_183, 1); -lean_inc(x_191); -lean_inc(x_190); -lean_dec(x_183); -x_192 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_193 = l_Lean_mkApp4(x_192, x_177, x_2, x_3, x_1); -lean_ctor_set(x_27, 0, x_193); -x_194 = 1; -x_195 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_195, 0, x_190); -lean_ctor_set(x_195, 1, x_27); -lean_ctor_set_uint8(x_195, sizeof(void*)*2, x_194); -lean_ctor_set(x_13, 0, x_195); -x_196 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_196, 0, x_13); -lean_ctor_set(x_196, 1, x_191); -return x_196; -} -} -else -{ -uint8_t x_197; -lean_dec(x_177); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_197 = !lean_is_exclusive(x_183); -if (x_197 == 0) -{ -return x_183; -} -else -{ -lean_object* x_198; lean_object* x_199; lean_object* x_200; -x_198 = lean_ctor_get(x_183, 0); -x_199 = lean_ctor_get(x_183, 1); -lean_inc(x_199); -lean_inc(x_198); -lean_dec(x_183); -x_200 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_200, 0, x_198); -lean_ctor_set(x_200, 1, x_199); -return x_200; -} -} -} -} -else -{ -lean_object* x_201; lean_object* x_202; uint8_t x_203; -x_201 = lean_ctor_get(x_167, 0); -x_202 = lean_ctor_get(x_167, 1); -lean_inc(x_202); -lean_inc(x_201); -lean_dec(x_167); -x_203 = lean_nat_dec_eq(x_24, x_201); -lean_dec(x_201); -if (x_203 == 0) -{ -lean_object* x_204; -lean_dec(x_202); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_204 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_26, 0, x_204); -return x_26; -} -else -{ -lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; -lean_free_object(x_26); -x_205 = l_BitVec_add(x_24, x_25, x_202); -lean_dec(x_202); -lean_dec(x_25); -x_206 = lean_box(0); -x_207 = l_Lean_mkNatLit(x_24); -x_208 = l_Lean_mkNatLit(x_205); -x_209 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_207); -x_210 = l_Lean_mkAppB(x_209, x_207, x_208); -lean_inc(x_3); -x_211 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_211, 0, x_3); -lean_ctor_set(x_211, 1, x_206); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_211); -lean_ctor_set(x_21, 0, x_210); -x_212 = lean_array_mk(x_21); -x_213 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_214 = l_Lean_Meta_mkAppM(x_213, x_212, x_7, x_8, x_9, x_10, x_168); -if (lean_obj_tag(x_214) == 0) -{ -lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; lean_object* x_221; lean_object* x_222; -x_215 = lean_ctor_get(x_214, 0); -lean_inc(x_215); -x_216 = lean_ctor_get(x_214, 1); -lean_inc(x_216); -if (lean_is_exclusive(x_214)) { - lean_ctor_release(x_214, 0); - lean_ctor_release(x_214, 1); - x_217 = x_214; -} else { - lean_dec_ref(x_214); - x_217 = lean_box(0); -} -x_218 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_219 = l_Lean_mkApp4(x_218, x_207, x_2, x_3, x_1); -lean_ctor_set(x_27, 0, x_219); -x_220 = 1; -x_221 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_221, 0, x_215); -lean_ctor_set(x_221, 1, x_27); -lean_ctor_set_uint8(x_221, sizeof(void*)*2, x_220); -lean_ctor_set(x_13, 0, x_221); -if (lean_is_scalar(x_217)) { - x_222 = lean_alloc_ctor(0, 2, 0); -} else { - x_222 = x_217; -} -lean_ctor_set(x_222, 0, x_13); -lean_ctor_set(x_222, 1, x_216); -return x_222; -} -else -{ -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -lean_dec(x_207); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_223 = lean_ctor_get(x_214, 0); -lean_inc(x_223); -x_224 = lean_ctor_get(x_214, 1); -lean_inc(x_224); -if (lean_is_exclusive(x_214)) { - lean_ctor_release(x_214, 0); - lean_ctor_release(x_214, 1); - x_225 = x_214; -} else { - lean_dec_ref(x_214); - x_225 = lean_box(0); -} -if (lean_is_scalar(x_225)) { - x_226 = lean_alloc_ctor(1, 2, 0); -} else { - x_226 = x_225; -} -lean_ctor_set(x_226, 0, x_223); -lean_ctor_set(x_226, 1, x_224); -return x_226; -} -} -} -} -else -{ -lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; uint8_t x_232; -x_227 = lean_ctor_get(x_27, 0); -x_228 = lean_ctor_get(x_26, 1); -lean_inc(x_228); -lean_dec(x_26); -x_229 = lean_ctor_get(x_227, 0); -lean_inc(x_229); -x_230 = lean_ctor_get(x_227, 1); -lean_inc(x_230); -if (lean_is_exclusive(x_227)) { - lean_ctor_release(x_227, 0); - lean_ctor_release(x_227, 1); - x_231 = x_227; -} else { - lean_dec_ref(x_227); - x_231 = lean_box(0); -} -x_232 = lean_nat_dec_eq(x_24, x_229); -lean_dec(x_229); -if (x_232 == 0) -{ -lean_object* x_233; lean_object* x_234; -lean_dec(x_231); -lean_dec(x_230); -lean_free_object(x_27); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_233 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_234 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_234, 0, x_233); -lean_ctor_set(x_234, 1, x_228); -return x_234; -} -else -{ -lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -x_235 = l_BitVec_add(x_24, x_25, x_230); -lean_dec(x_230); -lean_dec(x_25); -x_236 = lean_box(0); -x_237 = l_Lean_mkNatLit(x_24); -x_238 = l_Lean_mkNatLit(x_235); -x_239 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_237); -x_240 = l_Lean_mkAppB(x_239, x_237, x_238); -lean_inc(x_3); -if (lean_is_scalar(x_231)) { - x_241 = lean_alloc_ctor(1, 2, 0); -} else { - x_241 = x_231; - lean_ctor_set_tag(x_241, 1); -} -lean_ctor_set(x_241, 0, x_3); -lean_ctor_set(x_241, 1, x_236); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_241); -lean_ctor_set(x_21, 0, x_240); -x_242 = lean_array_mk(x_21); -x_243 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_244 = l_Lean_Meta_mkAppM(x_243, x_242, x_7, x_8, x_9, x_10, x_228); -if (lean_obj_tag(x_244) == 0) -{ -lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; uint8_t x_250; lean_object* x_251; lean_object* x_252; -x_245 = lean_ctor_get(x_244, 0); -lean_inc(x_245); -x_246 = lean_ctor_get(x_244, 1); -lean_inc(x_246); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - lean_ctor_release(x_244, 1); - x_247 = x_244; -} else { - lean_dec_ref(x_244); - x_247 = lean_box(0); -} -x_248 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_249 = l_Lean_mkApp4(x_248, x_237, x_2, x_3, x_1); -lean_ctor_set(x_27, 0, x_249); -x_250 = 1; -x_251 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_251, 0, x_245); -lean_ctor_set(x_251, 1, x_27); -lean_ctor_set_uint8(x_251, sizeof(void*)*2, x_250); -lean_ctor_set(x_13, 0, x_251); -if (lean_is_scalar(x_247)) { - x_252 = lean_alloc_ctor(0, 2, 0); -} else { - x_252 = x_247; -} -lean_ctor_set(x_252, 0, x_13); -lean_ctor_set(x_252, 1, x_246); -return x_252; -} -else -{ -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -lean_dec(x_237); -lean_free_object(x_27); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_253 = lean_ctor_get(x_244, 0); -lean_inc(x_253); -x_254 = lean_ctor_get(x_244, 1); -lean_inc(x_254); -if (lean_is_exclusive(x_244)) { - lean_ctor_release(x_244, 0); - lean_ctor_release(x_244, 1); - x_255 = x_244; -} else { - lean_dec_ref(x_244); - x_255 = lean_box(0); -} -if (lean_is_scalar(x_255)) { - x_256 = lean_alloc_ctor(1, 2, 0); -} else { - x_256 = x_255; -} -lean_ctor_set(x_256, 0, x_253); -lean_ctor_set(x_256, 1, x_254); -return x_256; -} -} -} -} -else -{ -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; uint8_t x_263; -x_257 = lean_ctor_get(x_27, 0); -lean_inc(x_257); -lean_dec(x_27); -x_258 = lean_ctor_get(x_26, 1); -lean_inc(x_258); -if (lean_is_exclusive(x_26)) { - lean_ctor_release(x_26, 0); - lean_ctor_release(x_26, 1); - x_259 = x_26; -} else { - lean_dec_ref(x_26); - x_259 = lean_box(0); -} -x_260 = lean_ctor_get(x_257, 0); -lean_inc(x_260); -x_261 = lean_ctor_get(x_257, 1); -lean_inc(x_261); -if (lean_is_exclusive(x_257)) { - lean_ctor_release(x_257, 0); - lean_ctor_release(x_257, 1); - x_262 = x_257; -} else { - lean_dec_ref(x_257); - x_262 = lean_box(0); -} -x_263 = lean_nat_dec_eq(x_24, x_260); -lean_dec(x_260); -if (x_263 == 0) -{ -lean_object* x_264; lean_object* x_265; -lean_dec(x_262); -lean_dec(x_261); -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_264 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_259)) { - x_265 = lean_alloc_ctor(0, 2, 0); -} else { - x_265 = x_259; -} -lean_ctor_set(x_265, 0, x_264); -lean_ctor_set(x_265, 1, x_258); -return x_265; -} -else -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; -lean_dec(x_259); -x_266 = l_BitVec_add(x_24, x_25, x_261); -lean_dec(x_261); -lean_dec(x_25); -x_267 = lean_box(0); -x_268 = l_Lean_mkNatLit(x_24); -x_269 = l_Lean_mkNatLit(x_266); -x_270 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_268); -x_271 = l_Lean_mkAppB(x_270, x_268, x_269); -lean_inc(x_3); -if (lean_is_scalar(x_262)) { - x_272 = lean_alloc_ctor(1, 2, 0); -} else { - x_272 = x_262; - lean_ctor_set_tag(x_272, 1); -} -lean_ctor_set(x_272, 0, x_3); -lean_ctor_set(x_272, 1, x_267); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_272); -lean_ctor_set(x_21, 0, x_271); -x_273 = lean_array_mk(x_21); -x_274 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_275 = l_Lean_Meta_mkAppM(x_274, x_273, x_7, x_8, x_9, x_10, x_258); -if (lean_obj_tag(x_275) == 0) -{ -lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; uint8_t x_282; lean_object* x_283; lean_object* x_284; -x_276 = lean_ctor_get(x_275, 0); -lean_inc(x_276); -x_277 = lean_ctor_get(x_275, 1); -lean_inc(x_277); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_278 = x_275; -} else { - lean_dec_ref(x_275); - x_278 = lean_box(0); -} -x_279 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_280 = l_Lean_mkApp4(x_279, x_268, x_2, x_3, x_1); -x_281 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_281, 0, x_280); -x_282 = 1; -x_283 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_283, 0, x_276); -lean_ctor_set(x_283, 1, x_281); -lean_ctor_set_uint8(x_283, sizeof(void*)*2, x_282); -lean_ctor_set(x_13, 0, x_283); -if (lean_is_scalar(x_278)) { - x_284 = lean_alloc_ctor(0, 2, 0); -} else { - x_284 = x_278; -} -lean_ctor_set(x_284, 0, x_13); -lean_ctor_set(x_284, 1, x_277); -return x_284; -} -else -{ -lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; -lean_dec(x_268); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_285 = lean_ctor_get(x_275, 0); -lean_inc(x_285); -x_286 = lean_ctor_get(x_275, 1); -lean_inc(x_286); -if (lean_is_exclusive(x_275)) { - lean_ctor_release(x_275, 0); - lean_ctor_release(x_275, 1); - x_287 = x_275; -} else { - lean_dec_ref(x_275); - x_287 = lean_box(0); -} -if (lean_is_scalar(x_287)) { - x_288 = lean_alloc_ctor(1, 2, 0); -} else { - x_288 = x_287; -} -lean_ctor_set(x_288, 0, x_285); -lean_ctor_set(x_288, 1, x_286); -return x_288; -} -} -} -} -} -else -{ -uint8_t x_289; -lean_free_object(x_21); -lean_dec(x_25); -lean_dec(x_24); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_289 = !lean_is_exclusive(x_26); -if (x_289 == 0) -{ -return x_26; -} -else -{ -lean_object* x_290; lean_object* x_291; lean_object* x_292; -x_290 = lean_ctor_get(x_26, 0); -x_291 = lean_ctor_get(x_26, 1); -lean_inc(x_291); -lean_inc(x_290); -lean_dec(x_26); -x_292 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_292, 0, x_290); -lean_ctor_set(x_292, 1, x_291); -return x_292; -} -} -} -else -{ -lean_object* x_293; lean_object* x_294; lean_object* x_295; -x_293 = lean_ctor_get(x_21, 0); -x_294 = lean_ctor_get(x_21, 1); -lean_inc(x_294); -lean_inc(x_293); -lean_dec(x_21); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_295 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); -if (lean_obj_tag(x_295) == 0) -{ -lean_object* x_296; -x_296 = lean_ctor_get(x_295, 0); -lean_inc(x_296); -if (lean_obj_tag(x_296) == 0) -{ -lean_object* x_297; lean_object* x_298; -x_297 = lean_ctor_get(x_295, 1); -lean_inc(x_297); -lean_dec(x_295); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_298 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_297); -if (lean_obj_tag(x_298) == 0) -{ -lean_object* x_299; -x_299 = lean_ctor_get(x_298, 0); -lean_inc(x_299); -if (lean_obj_tag(x_299) == 0) -{ -lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_300 = lean_ctor_get(x_298, 1); -lean_inc(x_300); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_301 = x_298; -} else { - lean_dec_ref(x_298); - x_301 = lean_box(0); -} -x_302 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_301)) { - x_303 = lean_alloc_ctor(0, 2, 0); -} else { - x_303 = x_301; -} -lean_ctor_set(x_303, 0, x_302); -lean_ctor_set(x_303, 1, x_300); -return x_303; -} -else -{ -lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; uint8_t x_311; -x_304 = lean_ctor_get(x_299, 0); -lean_inc(x_304); -if (lean_is_exclusive(x_299)) { - lean_ctor_release(x_299, 0); - x_305 = x_299; -} else { - lean_dec_ref(x_299); - x_305 = lean_box(0); -} -x_306 = lean_ctor_get(x_298, 1); -lean_inc(x_306); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_307 = x_298; -} else { - lean_dec_ref(x_298); - x_307 = lean_box(0); -} -x_308 = lean_ctor_get(x_304, 0); -lean_inc(x_308); -x_309 = lean_ctor_get(x_304, 1); -lean_inc(x_309); -if (lean_is_exclusive(x_304)) { - lean_ctor_release(x_304, 0); - lean_ctor_release(x_304, 1); - x_310 = x_304; -} else { - lean_dec_ref(x_304); - x_310 = lean_box(0); -} -x_311 = lean_nat_dec_eq(x_293, x_308); -lean_dec(x_308); -if (x_311 == 0) -{ -lean_object* x_312; lean_object* x_313; -lean_dec(x_310); -lean_dec(x_309); -lean_dec(x_305); -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_312 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_307)) { - x_313 = lean_alloc_ctor(0, 2, 0); -} else { - x_313 = x_307; -} -lean_ctor_set(x_313, 0, x_312); -lean_ctor_set(x_313, 1, x_306); -return x_313; -} -else -{ -lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; -lean_dec(x_307); -x_314 = l_BitVec_add(x_293, x_294, x_309); -lean_dec(x_309); -lean_dec(x_294); -x_315 = lean_box(0); -x_316 = l_Lean_mkNatLit(x_293); -x_317 = l_Lean_mkNatLit(x_314); -x_318 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_316); -x_319 = l_Lean_mkAppB(x_318, x_316, x_317); -lean_inc(x_2); -if (lean_is_scalar(x_310)) { - x_320 = lean_alloc_ctor(1, 2, 0); -} else { - x_320 = x_310; - lean_ctor_set_tag(x_320, 1); -} -lean_ctor_set(x_320, 0, x_2); -lean_ctor_set(x_320, 1, x_315); -x_321 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_321, 0, x_319); -lean_ctor_set(x_321, 1, x_320); -x_322 = lean_array_mk(x_321); -x_323 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_324 = l_Lean_Meta_mkAppM(x_323, x_322, x_7, x_8, x_9, x_10, x_306); -if (lean_obj_tag(x_324) == 0) -{ -lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; uint8_t x_331; lean_object* x_332; lean_object* x_333; -x_325 = lean_ctor_get(x_324, 0); -lean_inc(x_325); -x_326 = lean_ctor_get(x_324, 1); -lean_inc(x_326); -if (lean_is_exclusive(x_324)) { - lean_ctor_release(x_324, 0); - lean_ctor_release(x_324, 1); - x_327 = x_324; -} else { - lean_dec_ref(x_324); - x_327 = lean_box(0); -} -x_328 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_329 = l_Lean_mkApp4(x_328, x_316, x_2, x_3, x_1); -if (lean_is_scalar(x_305)) { - x_330 = lean_alloc_ctor(1, 1, 0); -} else { - x_330 = x_305; -} -lean_ctor_set(x_330, 0, x_329); -x_331 = 1; -x_332 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_332, 0, x_325); -lean_ctor_set(x_332, 1, x_330); -lean_ctor_set_uint8(x_332, sizeof(void*)*2, x_331); -lean_ctor_set(x_13, 0, x_332); -if (lean_is_scalar(x_327)) { - x_333 = lean_alloc_ctor(0, 2, 0); -} else { - x_333 = x_327; -} -lean_ctor_set(x_333, 0, x_13); -lean_ctor_set(x_333, 1, x_326); -return x_333; -} -else -{ -lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; -lean_dec(x_316); -lean_dec(x_305); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_334 = lean_ctor_get(x_324, 0); -lean_inc(x_334); -x_335 = lean_ctor_get(x_324, 1); -lean_inc(x_335); -if (lean_is_exclusive(x_324)) { - lean_ctor_release(x_324, 0); - lean_ctor_release(x_324, 1); - x_336 = x_324; -} else { - lean_dec_ref(x_324); - x_336 = lean_box(0); -} -if (lean_is_scalar(x_336)) { - x_337 = lean_alloc_ctor(1, 2, 0); -} else { - x_337 = x_336; -} -lean_ctor_set(x_337, 0, x_334); -lean_ctor_set(x_337, 1, x_335); -return x_337; -} -} -} -} -else -{ -lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_338 = lean_ctor_get(x_298, 0); -lean_inc(x_338); -x_339 = lean_ctor_get(x_298, 1); -lean_inc(x_339); -if (lean_is_exclusive(x_298)) { - lean_ctor_release(x_298, 0); - lean_ctor_release(x_298, 1); - x_340 = x_298; -} else { - lean_dec_ref(x_298); - x_340 = lean_box(0); -} -if (lean_is_scalar(x_340)) { - x_341 = lean_alloc_ctor(1, 2, 0); -} else { - x_341 = x_340; -} -lean_ctor_set(x_341, 0, x_338); -lean_ctor_set(x_341, 1, x_339); -return x_341; -} -} -else -{ -lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; -x_342 = lean_ctor_get(x_296, 0); -lean_inc(x_342); -if (lean_is_exclusive(x_296)) { - lean_ctor_release(x_296, 0); - x_343 = x_296; -} else { - lean_dec_ref(x_296); - x_343 = lean_box(0); -} -x_344 = lean_ctor_get(x_295, 1); -lean_inc(x_344); -if (lean_is_exclusive(x_295)) { - lean_ctor_release(x_295, 0); - lean_ctor_release(x_295, 1); - x_345 = x_295; -} else { - lean_dec_ref(x_295); - x_345 = lean_box(0); -} -x_346 = lean_ctor_get(x_342, 0); -lean_inc(x_346); -x_347 = lean_ctor_get(x_342, 1); -lean_inc(x_347); -if (lean_is_exclusive(x_342)) { - lean_ctor_release(x_342, 0); - lean_ctor_release(x_342, 1); - x_348 = x_342; -} else { - lean_dec_ref(x_342); - x_348 = lean_box(0); -} -x_349 = lean_nat_dec_eq(x_293, x_346); -lean_dec(x_346); -if (x_349 == 0) -{ -lean_object* x_350; lean_object* x_351; -lean_dec(x_348); -lean_dec(x_347); -lean_dec(x_343); -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_350 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_345)) { - x_351 = lean_alloc_ctor(0, 2, 0); -} else { - x_351 = x_345; -} -lean_ctor_set(x_351, 0, x_350); -lean_ctor_set(x_351, 1, x_344); -return x_351; -} -else -{ -lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; -lean_dec(x_345); -x_352 = l_BitVec_add(x_293, x_294, x_347); -lean_dec(x_347); -lean_dec(x_294); -x_353 = lean_box(0); -x_354 = l_Lean_mkNatLit(x_293); -x_355 = l_Lean_mkNatLit(x_352); -x_356 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_354); -x_357 = l_Lean_mkAppB(x_356, x_354, x_355); -lean_inc(x_3); -if (lean_is_scalar(x_348)) { - x_358 = lean_alloc_ctor(1, 2, 0); -} else { - x_358 = x_348; - lean_ctor_set_tag(x_358, 1); -} -lean_ctor_set(x_358, 0, x_3); -lean_ctor_set(x_358, 1, x_353); -x_359 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_359, 0, x_357); -lean_ctor_set(x_359, 1, x_358); -x_360 = lean_array_mk(x_359); -x_361 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_362 = l_Lean_Meta_mkAppM(x_361, x_360, x_7, x_8, x_9, x_10, x_344); -if (lean_obj_tag(x_362) == 0) -{ -lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; uint8_t x_369; lean_object* x_370; lean_object* x_371; -x_363 = lean_ctor_get(x_362, 0); -lean_inc(x_363); -x_364 = lean_ctor_get(x_362, 1); -lean_inc(x_364); -if (lean_is_exclusive(x_362)) { - lean_ctor_release(x_362, 0); - lean_ctor_release(x_362, 1); - x_365 = x_362; -} else { - lean_dec_ref(x_362); - x_365 = lean_box(0); -} -x_366 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_367 = l_Lean_mkApp4(x_366, x_354, x_2, x_3, x_1); -if (lean_is_scalar(x_343)) { - x_368 = lean_alloc_ctor(1, 1, 0); -} else { - x_368 = x_343; -} -lean_ctor_set(x_368, 0, x_367); -x_369 = 1; -x_370 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_370, 0, x_363); -lean_ctor_set(x_370, 1, x_368); -lean_ctor_set_uint8(x_370, sizeof(void*)*2, x_369); -lean_ctor_set(x_13, 0, x_370); -if (lean_is_scalar(x_365)) { - x_371 = lean_alloc_ctor(0, 2, 0); -} else { - x_371 = x_365; -} -lean_ctor_set(x_371, 0, x_13); -lean_ctor_set(x_371, 1, x_364); -return x_371; -} -else -{ -lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; -lean_dec(x_354); -lean_dec(x_343); -lean_free_object(x_13); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_372 = lean_ctor_get(x_362, 0); -lean_inc(x_372); -x_373 = lean_ctor_get(x_362, 1); -lean_inc(x_373); -if (lean_is_exclusive(x_362)) { - lean_ctor_release(x_362, 0); - lean_ctor_release(x_362, 1); - x_374 = x_362; -} else { - lean_dec_ref(x_362); - x_374 = lean_box(0); -} -if (lean_is_scalar(x_374)) { - x_375 = lean_alloc_ctor(1, 2, 0); -} else { - x_375 = x_374; -} -lean_ctor_set(x_375, 0, x_372); -lean_ctor_set(x_375, 1, x_373); -return x_375; -} -} -} -} -else -{ -lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; -lean_dec(x_294); -lean_dec(x_293); -lean_free_object(x_13); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_376 = lean_ctor_get(x_295, 0); -lean_inc(x_376); -x_377 = lean_ctor_get(x_295, 1); -lean_inc(x_377); -if (lean_is_exclusive(x_295)) { - lean_ctor_release(x_295, 0); - lean_ctor_release(x_295, 1); - x_378 = x_295; -} else { - lean_dec_ref(x_295); - x_378 = lean_box(0); -} -if (lean_is_scalar(x_378)) { - x_379 = lean_alloc_ctor(1, 2, 0); -} else { - x_379 = x_378; -} -lean_ctor_set(x_379, 0, x_376); -lean_ctor_set(x_379, 1, x_377); -return x_379; -} -} -} -else -{ -lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; -x_380 = lean_ctor_get(x_13, 0); -lean_inc(x_380); -lean_dec(x_13); -x_381 = lean_ctor_get(x_12, 1); -lean_inc(x_381); -lean_dec(x_12); -x_382 = lean_ctor_get(x_380, 0); -lean_inc(x_382); -x_383 = lean_ctor_get(x_380, 1); -lean_inc(x_383); -if (lean_is_exclusive(x_380)) { - lean_ctor_release(x_380, 0); - lean_ctor_release(x_380, 1); - x_384 = x_380; -} else { - lean_dec_ref(x_380); - x_384 = lean_box(0); -} -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); -x_385 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_381); -if (lean_obj_tag(x_385) == 0) -{ -lean_object* x_386; -x_386 = lean_ctor_get(x_385, 0); -lean_inc(x_386); -if (lean_obj_tag(x_386) == 0) -{ -lean_object* x_387; lean_object* x_388; -x_387 = lean_ctor_get(x_385, 1); -lean_inc(x_387); -lean_dec(x_385); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_3); -x_388 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_387); -if (lean_obj_tag(x_388) == 0) -{ -lean_object* x_389; -x_389 = lean_ctor_get(x_388, 0); -lean_inc(x_389); -if (lean_obj_tag(x_389) == 0) -{ -lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_390 = lean_ctor_get(x_388, 1); -lean_inc(x_390); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_391 = x_388; -} else { - lean_dec_ref(x_388); - x_391 = lean_box(0); -} -x_392 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_391)) { - x_393 = lean_alloc_ctor(0, 2, 0); -} else { - x_393 = x_391; -} -lean_ctor_set(x_393, 0, x_392); -lean_ctor_set(x_393, 1, x_390); -return x_393; -} -else -{ -lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; uint8_t x_401; -x_394 = lean_ctor_get(x_389, 0); -lean_inc(x_394); -if (lean_is_exclusive(x_389)) { - lean_ctor_release(x_389, 0); - x_395 = x_389; -} else { - lean_dec_ref(x_389); - x_395 = lean_box(0); -} -x_396 = lean_ctor_get(x_388, 1); -lean_inc(x_396); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_397 = x_388; -} else { - lean_dec_ref(x_388); - x_397 = lean_box(0); -} -x_398 = lean_ctor_get(x_394, 0); -lean_inc(x_398); -x_399 = lean_ctor_get(x_394, 1); -lean_inc(x_399); -if (lean_is_exclusive(x_394)) { - lean_ctor_release(x_394, 0); - lean_ctor_release(x_394, 1); - x_400 = x_394; -} else { - lean_dec_ref(x_394); - x_400 = lean_box(0); -} -x_401 = lean_nat_dec_eq(x_382, x_398); -lean_dec(x_398); -if (x_401 == 0) -{ -lean_object* x_402; lean_object* x_403; -lean_dec(x_400); -lean_dec(x_399); -lean_dec(x_395); -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_402 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_397)) { - x_403 = lean_alloc_ctor(0, 2, 0); -} else { - x_403 = x_397; -} -lean_ctor_set(x_403, 0, x_402); -lean_ctor_set(x_403, 1, x_396); -return x_403; -} -else -{ -lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; -lean_dec(x_397); -x_404 = l_BitVec_add(x_382, x_383, x_399); -lean_dec(x_399); -lean_dec(x_383); -x_405 = lean_box(0); -x_406 = l_Lean_mkNatLit(x_382); -x_407 = l_Lean_mkNatLit(x_404); -x_408 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_406); -x_409 = l_Lean_mkAppB(x_408, x_406, x_407); -lean_inc(x_2); -if (lean_is_scalar(x_400)) { - x_410 = lean_alloc_ctor(1, 2, 0); -} else { - x_410 = x_400; - lean_ctor_set_tag(x_410, 1); -} -lean_ctor_set(x_410, 0, x_2); -lean_ctor_set(x_410, 1, x_405); -if (lean_is_scalar(x_384)) { - x_411 = lean_alloc_ctor(1, 2, 0); -} else { - x_411 = x_384; - lean_ctor_set_tag(x_411, 1); -} -lean_ctor_set(x_411, 0, x_409); -lean_ctor_set(x_411, 1, x_410); -x_412 = lean_array_mk(x_411); -x_413 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_414 = l_Lean_Meta_mkAppM(x_413, x_412, x_7, x_8, x_9, x_10, x_396); -if (lean_obj_tag(x_414) == 0) -{ -lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; -x_415 = lean_ctor_get(x_414, 0); -lean_inc(x_415); -x_416 = lean_ctor_get(x_414, 1); -lean_inc(x_416); -if (lean_is_exclusive(x_414)) { - lean_ctor_release(x_414, 0); - lean_ctor_release(x_414, 1); - x_417 = x_414; -} else { - lean_dec_ref(x_414); - x_417 = lean_box(0); -} -x_418 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; -x_419 = l_Lean_mkApp4(x_418, x_406, x_2, x_3, x_1); -if (lean_is_scalar(x_395)) { - x_420 = lean_alloc_ctor(1, 1, 0); -} else { - x_420 = x_395; -} -lean_ctor_set(x_420, 0, x_419); -x_421 = 1; -x_422 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_422, 0, x_415); -lean_ctor_set(x_422, 1, x_420); -lean_ctor_set_uint8(x_422, sizeof(void*)*2, x_421); -x_423 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_423, 0, x_422); -if (lean_is_scalar(x_417)) { - x_424 = lean_alloc_ctor(0, 2, 0); -} else { - x_424 = x_417; -} -lean_ctor_set(x_424, 0, x_423); -lean_ctor_set(x_424, 1, x_416); -return x_424; -} -else -{ -lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; -lean_dec(x_406); -lean_dec(x_395); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_425 = lean_ctor_get(x_414, 0); -lean_inc(x_425); -x_426 = lean_ctor_get(x_414, 1); -lean_inc(x_426); -if (lean_is_exclusive(x_414)) { - lean_ctor_release(x_414, 0); - lean_ctor_release(x_414, 1); - x_427 = x_414; -} else { - lean_dec_ref(x_414); - x_427 = lean_box(0); -} -if (lean_is_scalar(x_427)) { - x_428 = lean_alloc_ctor(1, 2, 0); -} else { - x_428 = x_427; -} -lean_ctor_set(x_428, 0, x_425); -lean_ctor_set(x_428, 1, x_426); -return x_428; -} -} -} -} -else -{ -lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_429 = lean_ctor_get(x_388, 0); -lean_inc(x_429); -x_430 = lean_ctor_get(x_388, 1); -lean_inc(x_430); -if (lean_is_exclusive(x_388)) { - lean_ctor_release(x_388, 0); - lean_ctor_release(x_388, 1); - x_431 = x_388; -} else { - lean_dec_ref(x_388); - x_431 = lean_box(0); -} -if (lean_is_scalar(x_431)) { - x_432 = lean_alloc_ctor(1, 2, 0); -} else { - x_432 = x_431; -} -lean_ctor_set(x_432, 0, x_429); -lean_ctor_set(x_432, 1, x_430); -return x_432; -} -} -else -{ -lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; uint8_t x_440; -x_433 = lean_ctor_get(x_386, 0); -lean_inc(x_433); -if (lean_is_exclusive(x_386)) { - lean_ctor_release(x_386, 0); - x_434 = x_386; -} else { - lean_dec_ref(x_386); - x_434 = lean_box(0); -} -x_435 = lean_ctor_get(x_385, 1); -lean_inc(x_435); -if (lean_is_exclusive(x_385)) { - lean_ctor_release(x_385, 0); - lean_ctor_release(x_385, 1); - x_436 = x_385; -} else { - lean_dec_ref(x_385); - x_436 = lean_box(0); -} -x_437 = lean_ctor_get(x_433, 0); -lean_inc(x_437); -x_438 = lean_ctor_get(x_433, 1); -lean_inc(x_438); -if (lean_is_exclusive(x_433)) { - lean_ctor_release(x_433, 0); - lean_ctor_release(x_433, 1); - x_439 = x_433; -} else { - lean_dec_ref(x_433); - x_439 = lean_box(0); -} -x_440 = lean_nat_dec_eq(x_382, x_437); -lean_dec(x_437); -if (x_440 == 0) -{ -lean_object* x_441; lean_object* x_442; -lean_dec(x_439); -lean_dec(x_438); -lean_dec(x_434); -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_441 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -if (lean_is_scalar(x_436)) { - x_442 = lean_alloc_ctor(0, 2, 0); -} else { - x_442 = x_436; -} -lean_ctor_set(x_442, 0, x_441); -lean_ctor_set(x_442, 1, x_435); -return x_442; -} -else -{ -lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; -lean_dec(x_436); -x_443 = l_BitVec_add(x_382, x_383, x_438); -lean_dec(x_438); -lean_dec(x_383); -x_444 = lean_box(0); -x_445 = l_Lean_mkNatLit(x_382); -x_446 = l_Lean_mkNatLit(x_443); -x_447 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; -lean_inc(x_445); -x_448 = l_Lean_mkAppB(x_447, x_445, x_446); -lean_inc(x_3); -if (lean_is_scalar(x_439)) { - x_449 = lean_alloc_ctor(1, 2, 0); -} else { - x_449 = x_439; - lean_ctor_set_tag(x_449, 1); -} -lean_ctor_set(x_449, 0, x_3); -lean_ctor_set(x_449, 1, x_444); -if (lean_is_scalar(x_384)) { - x_450 = lean_alloc_ctor(1, 2, 0); -} else { - x_450 = x_384; - lean_ctor_set_tag(x_450, 1); -} -lean_ctor_set(x_450, 0, x_448); -lean_ctor_set(x_450, 1, x_449); -x_451 = lean_array_mk(x_450); -x_452 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_453 = l_Lean_Meta_mkAppM(x_452, x_451, x_7, x_8, x_9, x_10, x_435); -if (lean_obj_tag(x_453) == 0) -{ -lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; uint8_t x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; -x_454 = lean_ctor_get(x_453, 0); -lean_inc(x_454); -x_455 = lean_ctor_get(x_453, 1); -lean_inc(x_455); -if (lean_is_exclusive(x_453)) { - lean_ctor_release(x_453, 0); - lean_ctor_release(x_453, 1); - x_456 = x_453; -} else { - lean_dec_ref(x_453); - x_456 = lean_box(0); -} -x_457 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; -x_458 = l_Lean_mkApp4(x_457, x_445, x_2, x_3, x_1); -if (lean_is_scalar(x_434)) { - x_459 = lean_alloc_ctor(1, 1, 0); -} else { - x_459 = x_434; -} -lean_ctor_set(x_459, 0, x_458); -x_460 = 1; -x_461 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_461, 0, x_454); -lean_ctor_set(x_461, 1, x_459); -lean_ctor_set_uint8(x_461, sizeof(void*)*2, x_460); -x_462 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_462, 0, x_461); -if (lean_is_scalar(x_456)) { - x_463 = lean_alloc_ctor(0, 2, 0); -} else { - x_463 = x_456; -} -lean_ctor_set(x_463, 0, x_462); -lean_ctor_set(x_463, 1, x_455); -return x_463; -} -else -{ -lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; -lean_dec(x_445); -lean_dec(x_434); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_464 = lean_ctor_get(x_453, 0); -lean_inc(x_464); -x_465 = lean_ctor_get(x_453, 1); -lean_inc(x_465); -if (lean_is_exclusive(x_453)) { - lean_ctor_release(x_453, 0); - lean_ctor_release(x_453, 1); - x_466 = x_453; -} else { - lean_dec_ref(x_453); - x_466 = lean_box(0); -} -if (lean_is_scalar(x_466)) { - x_467 = lean_alloc_ctor(1, 2, 0); -} else { - x_467 = x_466; -} -lean_ctor_set(x_467, 0, x_464); -lean_ctor_set(x_467, 1, x_465); -return x_467; -} -} -} -} -else -{ -lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; -lean_dec(x_384); -lean_dec(x_383); -lean_dec(x_382); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_468 = lean_ctor_get(x_385, 0); -lean_inc(x_468); -x_469 = lean_ctor_get(x_385, 1); -lean_inc(x_469); -if (lean_is_exclusive(x_385)) { - lean_ctor_release(x_385, 0); - lean_ctor_release(x_385, 1); - x_470 = x_385; -} else { - lean_dec_ref(x_385); - x_470 = lean_box(0); -} -if (lean_is_scalar(x_470)) { - x_471 = lean_alloc_ctor(1, 2, 0); -} else { - x_471 = x_470; -} -lean_ctor_set(x_471, 0, x_468); -lean_ctor_set(x_471, 1, x_469); -return x_471; -} -} -} -} -else -{ -uint8_t x_472; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_472 = !lean_is_exclusive(x_12); -if (x_472 == 0) -{ -return x_12; -} -else -{ -lean_object* x_473; lean_object* x_474; lean_object* x_475; -x_473 = lean_ctor_get(x_12, 0); -x_474 = lean_ctor_get(x_12, 1); -lean_inc(x_474); -lean_inc(x_473); -lean_dec(x_12); -x_475 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_475, 0, x_473); -lean_ctor_set(x_475, 1, x_474); -return x_475; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -lean_dec(x_2); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_2); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_2); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_2); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_2); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_2); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -lean_dec(x_2); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(x_2, x_21, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_43; -} -} -} -} -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2), 10, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; uint8_t x_27; -x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_27 = l_Lean_Expr_isApp(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_28 = lean_box(0); -x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_29; -} -else -{ -lean_object* x_30; uint8_t x_31; -x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); -x_31 = l_Lean_Expr_isApp(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -lean_dec(x_30); -lean_dec(x_21); -lean_dec(x_16); -x_32 = lean_box(0); -x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_33; -} -else -{ -lean_object* x_34; uint8_t x_35; -x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); -x_35 = l_Lean_Expr_isApp(x_34); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; -lean_dec(x_34); -lean_dec(x_21); -lean_dec(x_16); -x_36 = lean_box(0); -x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_37; -} -else -{ -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_21); -lean_dec(x_16); -x_41 = lean_box(0); -x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_42; -} -else -{ -lean_object* x_43; -x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_43; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_12; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("bv_add_const'", 13, 13); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(lean_object* x_1) { -_start: -{ -lean_object* x_2; uint8_t x_3; uint8_t x_4; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_nat_dec_eq(x_1, x_2); -x_4 = l_instDecidableNot___rarg(x_3); -if (x_4 == 0) -{ -lean_object* x_5; -x_5 = lean_box(0); -return x_5; -} -else -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_nat_log2(x_1); -x_7 = lean_unsigned_to_nat(2u); -x_8 = lean_nat_pow(x_7, x_6); -x_9 = lean_nat_dec_eq(x_8, x_1); -lean_dec(x_8); -if (x_9 == 0) -{ -lean_object* x_10; -lean_dec(x_6); -x_10 = lean_box(0); -return x_10; -} -else -{ -lean_object* x_11; -x_11 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_11, 0, x_6); -return x_11; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact___boxed(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_1); -lean_dec(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HPow", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hPow", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_box(0); -x_9 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_9, 0, x_2); -lean_ctor_set(x_9, 1, x_8); -x_10 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_array_mk(x_10); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3; -x_13 = l_Lean_Meta_mkAppM(x_12, x_11, x_3, x_4, x_5, x_6, x_7); -return x_13; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HShiftRight", 11, 11); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hShiftRight", 11, 11); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(2u); -x_2 = l_Lean_mkNatLit(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("udiv_ofNat_eq_of_lt", 19, 19); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_14 = l_Lean_mkNatLit(x_1); -x_15 = lean_box(0); -lean_inc(x_14); -x_16 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -lean_inc(x_2); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_2); -lean_ctor_set(x_17, 1, x_16); -x_18 = lean_array_mk(x_17); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_20 = l_Lean_Meta_mkAppM(x_19, x_18, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_14); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(x_23, x_14, x_9, x_10, x_11, x_12, x_22); -if (lean_obj_tag(x_24) == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l_Lean_mkNatLit(x_3); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_27); -x_28 = l_Lean_Meta_mkEq(x_25, x_27, x_9, x_10, x_11, x_12, x_26); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_31 = l_Lean_Meta_mkDecideProof(x_29, x_9, x_10, x_11, x_12, x_30); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = l_Lean_mkNatLit(x_4); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_34); -lean_inc(x_14); -x_35 = l_Lean_Meta_mkLt(x_14, x_34, x_9, x_10, x_11, x_12, x_33); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l_Lean_Meta_mkDecideProof(x_36, x_9, x_10, x_11, x_12, x_37); -if (lean_obj_tag(x_38) == 0) -{ -uint8_t x_39; -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; -x_40 = lean_ctor_get(x_38, 0); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_15); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_32); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_14); -lean_ctor_set(x_43, 1, x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_27); -lean_ctor_set(x_44, 1, x_43); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_2); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_34); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_array_mk(x_46); -x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; -x_49 = l_Lean_mkAppN(x_48, x_47); -lean_dec(x_47); -x_50 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_50, 0, x_49); -x_51 = 1; -x_52 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_52, 0, x_21); -lean_ctor_set(x_52, 1, x_50); -lean_ctor_set_uint8(x_52, sizeof(void*)*2, x_51); -x_53 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_38, 0, x_53); -return x_38; -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_54 = lean_ctor_get(x_38, 0); -x_55 = lean_ctor_get(x_38, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_38); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_15); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_32); -lean_ctor_set(x_57, 1, x_56); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_14); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_27); -lean_ctor_set(x_59, 1, x_58); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_2); -lean_ctor_set(x_60, 1, x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_34); -lean_ctor_set(x_61, 1, x_60); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; -x_64 = l_Lean_mkAppN(x_63, x_62); -lean_dec(x_62); -x_65 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_65, 0, x_64); -x_66 = 1; -x_67 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_67, 0, x_21); -lean_ctor_set(x_67, 1, x_65); -lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); -x_68 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_68, 0, x_67); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_55); -return x_69; -} -} -else -{ -uint8_t x_70; -lean_dec(x_34); -lean_dec(x_32); -lean_dec(x_27); -lean_dec(x_21); -lean_dec(x_14); -lean_dec(x_2); -x_70 = !lean_is_exclusive(x_38); -if (x_70 == 0) -{ -return x_38; -} -else -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_38, 0); -x_72 = lean_ctor_get(x_38, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_38); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; -} -} -} -else -{ -uint8_t x_74; -lean_dec(x_34); -lean_dec(x_32); -lean_dec(x_27); -lean_dec(x_21); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_2); -x_74 = !lean_is_exclusive(x_35); -if (x_74 == 0) -{ -return x_35; -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_35, 0); -x_76 = lean_ctor_get(x_35, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_35); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; -} -} -} -else -{ -uint8_t x_78; -lean_dec(x_27); -lean_dec(x_21); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_4); -lean_dec(x_2); -x_78 = !lean_is_exclusive(x_31); -if (x_78 == 0) -{ -return x_31; -} -else -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_31, 0); -x_80 = lean_ctor_get(x_31, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_31); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -return x_81; -} -} -} -else -{ -uint8_t x_82; -lean_dec(x_27); -lean_dec(x_21); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_4); -lean_dec(x_2); -x_82 = !lean_is_exclusive(x_28); -if (x_82 == 0) -{ -return x_28; -} -else -{ -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_28, 0); -x_84 = lean_ctor_get(x_28, 1); -lean_inc(x_84); -lean_inc(x_83); -lean_dec(x_28); -x_85 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -return x_85; -} -} -} -else -{ -uint8_t x_86; -lean_dec(x_21); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_86 = !lean_is_exclusive(x_24); -if (x_86 == 0) -{ -return x_24; -} -else -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_24, 0); -x_88 = lean_ctor_get(x_24, 1); -lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_24); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; -} -} -} -else -{ -uint8_t x_90; -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_90 = !lean_is_exclusive(x_20); -if (x_90 == 0) -{ -return x_20; -} -else -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_20, 0); -x_92 = lean_ctor_get(x_20, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_20); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -return x_93; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_15 = l_Lean_Meta_getBitVecValue_x3f(x_6, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -if (lean_obj_tag(x_16) == 0) -{ -uint8_t x_17; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_17 = !lean_is_exclusive(x_15); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_15, 0); -lean_dec(x_18); -x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_15, 0, x_19); -return x_15; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_15, 1); -lean_inc(x_20); -lean_dec(x_15); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; -} -} -else -{ -lean_object* x_23; uint8_t x_24; -x_23 = lean_ctor_get(x_16, 0); -lean_inc(x_23); -lean_dec(x_16); -x_24 = !lean_is_exclusive(x_15); -if (x_24 == 0) -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_15, 1); -x_26 = lean_ctor_get(x_15, 0); -lean_dec(x_26); -x_27 = lean_ctor_get(x_23, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_23, 1); -lean_inc(x_28); -lean_dec(x_23); -x_29 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_15, 0, x_30); -return x_15; -} -else -{ -lean_object* x_31; uint8_t x_32; -x_31 = lean_ctor_get(x_29, 0); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_nat_dec_le(x_27, x_31); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; -lean_free_object(x_15); -x_33 = lean_box(0); -x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_31, x_5, x_28, x_27, x_33, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); -return x_34; -} -else -{ -lean_object* x_35; -lean_dec(x_31); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -lean_ctor_set(x_15, 0, x_35); -return x_15; -} -} -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_15, 1); -lean_inc(x_36); -lean_dec(x_15); -x_37 = lean_ctor_get(x_23, 0); -lean_inc(x_37); -x_38 = lean_ctor_get(x_23, 1); -lean_inc(x_38); -lean_dec(x_23); -x_39 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_38); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_36); -return x_41; -} -else -{ -lean_object* x_42; uint8_t x_43; -x_42 = lean_ctor_get(x_39, 0); -lean_inc(x_42); -lean_dec(x_39); -x_43 = lean_nat_dec_le(x_37, x_42); -if (x_43 == 0) -{ -lean_object* x_44; lean_object* x_45; -x_44 = lean_box(0); -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_42, x_5, x_38, x_37, x_44, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_36); -return x_45; -} -else -{ -lean_object* x_46; lean_object* x_47; -lean_dec(x_42); -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_36); -return x_47; -} -} -} -} -} -else -{ -uint8_t x_48; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_5); -x_48 = !lean_is_exclusive(x_15); -if (x_48 == 0) -{ -return x_15; -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_15, 0); -x_50 = lean_ctor_get(x_15, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_15); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed), 14, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("HDiv", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("hDiv", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Expr_isApp(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -lean_dec(x_12); -x_14 = lean_box(0); -x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); -x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); -x_18 = l_Lean_Expr_isApp(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; -lean_dec(x_17); -lean_dec(x_16); -x_19 = lean_box(0); -x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_16); -x_24 = lean_box(0); -x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = l_Lean_Expr_appArg(x_22, lean_box(0)); -x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_28 = l_Lean_Expr_isApp(x_27); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; -lean_dec(x_27); -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_29 = lean_box(0); -x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_30; -} -else -{ -lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); -x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); -x_33 = l_Lean_Expr_isApp(x_32); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_34 = lean_box(0); -x_35 = lean_apply_9(x_11, x_34, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_35; -} -else -{ -lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_36 = l_Lean_Expr_appArg(x_32, lean_box(0)); -x_37 = l_Lean_Expr_appFnCleanup(x_32, lean_box(0)); -x_38 = l_Lean_Expr_isApp(x_37); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; -lean_dec(x_37); -lean_dec(x_36); -lean_dec(x_31); -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_39 = lean_box(0); -x_40 = lean_apply_9(x_11, x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_40; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_41 = l_Lean_Expr_appArg(x_37, lean_box(0)); -x_42 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; -x_44 = l_Lean_Expr_isConstOf(x_42, x_43); -lean_dec(x_42); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; -lean_dec(x_41); -lean_dec(x_36); -lean_dec(x_31); -lean_dec(x_26); -lean_dec(x_21); -lean_dec(x_16); -x_45 = lean_box(0); -x_46 = lean_apply_9(x_11, x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_46; -} -else -{ -lean_object* x_47; -x_47 = lean_apply_14(x_10, x_41, x_36, x_31, x_26, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -return x_47; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_15; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("bv_udiv_of_two_pow", 18, 18); -return x_1; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1; -x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -return x_8; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; -x_2 = lean_unsigned_to_nat(6u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; -x_2 = lean_unsigned_to_nat(2u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(3); -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14; -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow), 9, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16; -x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); -return x_5; -} -} -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510_(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2; -x_4 = 1; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1; -x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); -return x_6; -} -} -LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_1, 0); -lean_inc(x_7); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; -} -else -{ -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_6); -return x_10; -} -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; -lean_inc(x_9); -x_12 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Meta_processPostponed___spec__3(x_1, x_5, x_2, x_3, x_7, x_8, x_9, x_10, x_11); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_4, x_7, x_8, x_9, x_10, x_13); -lean_dec(x_9); -return x_14; -} -} -static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; double x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = 0; -x_3 = l_Float_ofScientific(x_1, x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, double x_8, double x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -if (x_7 == 0) -{ -double x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___closed__1; -x_17 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_3); -lean_ctor_set_float(x_17, sizeof(void*)*2, x_16); -lean_ctor_set_float(x_17, sizeof(void*)*2 + 8, x_16); -lean_ctor_set_uint8(x_17, sizeof(void*)*2 + 16, x_2); -x_18 = lean_box(0); -x_19 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_17, x_18, x_11, x_12, x_13, x_14, x_15); -return x_19; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_20, 0, x_1); -lean_ctor_set(x_20, 1, x_3); -lean_ctor_set_float(x_20, sizeof(void*)*2, x_8); -lean_ctor_set_float(x_20, sizeof(void*)*2 + 8, x_9); -lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 16, x_2); -x_21 = lean_box(0); -x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_20, x_21, x_11, x_12, x_13, x_14, x_15); -return x_22; -} -} -} -static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 53, 53); -return x_1; -} -} -static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, double x_7, double x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_13, 5); -lean_inc(x_16); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_5); -x_17 = lean_apply_6(x_9, x_5, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_18, x_11, x_12, x_13, x_14, x_19); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_5); -return x_20; -} -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2; -x_23 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_16, x_5, x_6, x_7, x_8, x_22, x_11, x_12, x_13, x_14, x_21); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_5); -return x_23; -} -} -} -static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_trace_profiler_useHeartbeats; -return x_1; -} -} -static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_trace_profiler; -return x_1; -} -} -static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_trace_profiler_threshold; -return x_1; -} -} -static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__4() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; -x_1 = lean_unsigned_to_nat(1000u); -x_2 = 0; -x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Float_ofScientific(x_1, x_2, x_3); -return x_4; -} -} -static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; -x_1 = lean_unsigned_to_nat(1000000000u); -x_2 = 0; -x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Float_ofScientific(x_1, x_2, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Meta_processPostponed___spec__2___rarg(x_12, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1; -x_18 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_113 = lean_io_mono_nanos_now(x_16); -x_114 = lean_ctor_get(x_113, 0); -lean_inc(x_114); -x_115 = lean_ctor_get(x_113, 1); -lean_inc(x_115); -lean_dec(x_113); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_116 = lean_apply_5(x_7, x_9, x_10, x_11, x_12, x_115); -if (lean_obj_tag(x_116) == 0) -{ -uint8_t x_117; -x_117 = !lean_is_exclusive(x_116); -if (x_117 == 0) -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; -x_118 = lean_ctor_get(x_116, 0); -x_119 = lean_ctor_get(x_116, 1); -x_120 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_120, 0, x_118); -x_121 = lean_io_mono_nanos_now(x_119); -x_122 = !lean_is_exclusive(x_121); -if (x_122 == 0) -{ -lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; double x_127; double x_128; double x_129; double x_130; double x_131; lean_object* x_132; lean_object* x_133; -x_123 = lean_ctor_get(x_121, 0); -x_124 = lean_ctor_get(x_121, 1); -x_125 = 0; -x_126 = lean_unsigned_to_nat(0u); -x_127 = l_Float_ofScientific(x_114, x_125, x_126); -lean_dec(x_114); -x_128 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_129 = lean_float_div(x_127, x_128); -x_130 = l_Float_ofScientific(x_123, x_125, x_126); -lean_dec(x_123); -x_131 = lean_float_div(x_130, x_128); -x_132 = lean_box_float(x_129); -x_133 = lean_box_float(x_131); -lean_ctor_set(x_121, 1, x_133); -lean_ctor_set(x_121, 0, x_132); -lean_ctor_set(x_116, 1, x_121); -lean_ctor_set(x_116, 0, x_120); -x_19 = x_116; -x_20 = x_124; -goto block_112; -} -else -{ -lean_object* x_134; lean_object* x_135; uint8_t x_136; lean_object* x_137; double x_138; double x_139; double x_140; double x_141; double x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_134 = lean_ctor_get(x_121, 0); -x_135 = lean_ctor_get(x_121, 1); -lean_inc(x_135); -lean_inc(x_134); -lean_dec(x_121); -x_136 = 0; -x_137 = lean_unsigned_to_nat(0u); -x_138 = l_Float_ofScientific(x_114, x_136, x_137); -lean_dec(x_114); -x_139 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_140 = lean_float_div(x_138, x_139); -x_141 = l_Float_ofScientific(x_134, x_136, x_137); -lean_dec(x_134); -x_142 = lean_float_div(x_141, x_139); -x_143 = lean_box_float(x_140); -x_144 = lean_box_float(x_142); -x_145 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -lean_ctor_set(x_116, 1, x_145); -lean_ctor_set(x_116, 0, x_120); -x_19 = x_116; -x_20 = x_135; -goto block_112; -} -} -else -{ -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; uint8_t x_153; lean_object* x_154; double x_155; double x_156; double x_157; double x_158; double x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; -x_146 = lean_ctor_get(x_116, 0); -x_147 = lean_ctor_get(x_116, 1); -lean_inc(x_147); -lean_inc(x_146); -lean_dec(x_116); -x_148 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_148, 0, x_146); -x_149 = lean_io_mono_nanos_now(x_147); -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_149, 1); -lean_inc(x_151); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_152 = x_149; -} else { - lean_dec_ref(x_149); - x_152 = lean_box(0); -} -x_153 = 0; -x_154 = lean_unsigned_to_nat(0u); -x_155 = l_Float_ofScientific(x_114, x_153, x_154); -lean_dec(x_114); -x_156 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_157 = lean_float_div(x_155, x_156); -x_158 = l_Float_ofScientific(x_150, x_153, x_154); -lean_dec(x_150); -x_159 = lean_float_div(x_158, x_156); -x_160 = lean_box_float(x_157); -x_161 = lean_box_float(x_159); -if (lean_is_scalar(x_152)) { - x_162 = lean_alloc_ctor(0, 2, 0); -} else { - x_162 = x_152; -} -lean_ctor_set(x_162, 0, x_160); -lean_ctor_set(x_162, 1, x_161); -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_148); -lean_ctor_set(x_163, 1, x_162); -x_19 = x_163; -x_20 = x_151; -goto block_112; -} -} -else -{ -uint8_t x_164; -x_164 = !lean_is_exclusive(x_116); -if (x_164 == 0) -{ -lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; -x_165 = lean_ctor_get(x_116, 0); -x_166 = lean_ctor_get(x_116, 1); -x_167 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_167, 0, x_165); -x_168 = lean_io_mono_nanos_now(x_166); -x_169 = !lean_is_exclusive(x_168); -if (x_169 == 0) -{ -lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; double x_174; double x_175; double x_176; double x_177; double x_178; lean_object* x_179; lean_object* x_180; -x_170 = lean_ctor_get(x_168, 0); -x_171 = lean_ctor_get(x_168, 1); -x_172 = 0; -x_173 = lean_unsigned_to_nat(0u); -x_174 = l_Float_ofScientific(x_114, x_172, x_173); -lean_dec(x_114); -x_175 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_176 = lean_float_div(x_174, x_175); -x_177 = l_Float_ofScientific(x_170, x_172, x_173); -lean_dec(x_170); -x_178 = lean_float_div(x_177, x_175); -x_179 = lean_box_float(x_176); -x_180 = lean_box_float(x_178); -lean_ctor_set(x_168, 1, x_180); -lean_ctor_set(x_168, 0, x_179); -lean_ctor_set_tag(x_116, 0); -lean_ctor_set(x_116, 1, x_168); -lean_ctor_set(x_116, 0, x_167); -x_19 = x_116; -x_20 = x_171; -goto block_112; -} -else -{ -lean_object* x_181; lean_object* x_182; uint8_t x_183; lean_object* x_184; double x_185; double x_186; double x_187; double x_188; double x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_181 = lean_ctor_get(x_168, 0); -x_182 = lean_ctor_get(x_168, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_168); -x_183 = 0; -x_184 = lean_unsigned_to_nat(0u); -x_185 = l_Float_ofScientific(x_114, x_183, x_184); -lean_dec(x_114); -x_186 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_187 = lean_float_div(x_185, x_186); -x_188 = l_Float_ofScientific(x_181, x_183, x_184); -lean_dec(x_181); -x_189 = lean_float_div(x_188, x_186); -x_190 = lean_box_float(x_187); -x_191 = lean_box_float(x_189); -x_192 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_192, 0, x_190); -lean_ctor_set(x_192, 1, x_191); -lean_ctor_set_tag(x_116, 0); -lean_ctor_set(x_116, 1, x_192); -lean_ctor_set(x_116, 0, x_167); -x_19 = x_116; -x_20 = x_182; -goto block_112; -} -} -else -{ -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; uint8_t x_200; lean_object* x_201; double x_202; double x_203; double x_204; double x_205; double x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_193 = lean_ctor_get(x_116, 0); -x_194 = lean_ctor_get(x_116, 1); -lean_inc(x_194); -lean_inc(x_193); -lean_dec(x_116); -x_195 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_195, 0, x_193); -x_196 = lean_io_mono_nanos_now(x_194); -x_197 = lean_ctor_get(x_196, 0); -lean_inc(x_197); -x_198 = lean_ctor_get(x_196, 1); -lean_inc(x_198); -if (lean_is_exclusive(x_196)) { - lean_ctor_release(x_196, 0); - lean_ctor_release(x_196, 1); - x_199 = x_196; -} else { - lean_dec_ref(x_196); - x_199 = lean_box(0); -} -x_200 = 0; -x_201 = lean_unsigned_to_nat(0u); -x_202 = l_Float_ofScientific(x_114, x_200, x_201); -lean_dec(x_114); -x_203 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5; -x_204 = lean_float_div(x_202, x_203); -x_205 = l_Float_ofScientific(x_197, x_200, x_201); -lean_dec(x_197); -x_206 = lean_float_div(x_205, x_203); -x_207 = lean_box_float(x_204); -x_208 = lean_box_float(x_206); -if (lean_is_scalar(x_199)) { - x_209 = lean_alloc_ctor(0, 2, 0); -} else { - x_209 = x_199; -} -lean_ctor_set(x_209, 0, x_207); -lean_ctor_set(x_209, 1, x_208); -x_210 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_210, 0, x_195); -lean_ctor_set(x_210, 1, x_209); -x_19 = x_210; -x_20 = x_198; -goto block_112; -} -} -block_112: -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; uint8_t x_27; -x_21 = lean_ctor_get(x_19, 1); -lean_inc(x_21); -x_22 = lean_ctor_get(x_19, 0); -lean_inc(x_22); -lean_dec(x_19); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2; -x_26 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_25); -if (x_26 == 0) -{ -if (x_6 == 0) -{ -uint8_t x_92; -x_92 = 0; -x_27 = x_92; -goto block_91; -} -else -{ -lean_object* x_93; double x_94; double x_95; lean_object* x_96; -x_93 = lean_box(0); -x_94 = lean_unbox_float(x_23); -lean_dec(x_23); -x_95 = lean_unbox_float(x_24); -lean_dec(x_24); -x_96 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_94, x_95, x_5, x_93, x_9, x_10, x_11, x_12, x_20); -return x_96; -} -} -else -{ -if (x_6 == 0) -{ -double x_97; double x_98; double x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; double x_104; double x_105; double x_106; uint8_t x_107; -x_97 = lean_unbox_float(x_24); -x_98 = lean_unbox_float(x_23); -x_99 = lean_float_sub(x_97, x_98); -x_100 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3; -x_101 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_100); -x_102 = 0; -x_103 = lean_unsigned_to_nat(0u); -x_104 = l_Float_ofScientific(x_101, x_102, x_103); -lean_dec(x_101); -x_105 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__4; -x_106 = lean_float_div(x_104, x_105); -x_107 = lean_float_decLt(x_106, x_99); -x_27 = x_107; -goto block_91; -} -else -{ -lean_object* x_108; double x_109; double x_110; lean_object* x_111; -x_108 = lean_box(0); -x_109 = lean_unbox_float(x_23); -lean_dec(x_23); -x_110 = lean_unbox_float(x_24); -lean_dec(x_24); -x_111 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_109, x_110, x_5, x_108, x_9, x_10, x_11, x_12, x_20); -return x_111; -} -} -block_91: -{ -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -lean_dec(x_24); -lean_dec(x_23); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_28 = lean_st_ref_take(x_12, x_20); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_29, 3); -lean_inc(x_30); -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = !lean_is_exclusive(x_29); -if (x_32 == 0) -{ -lean_object* x_33; uint8_t x_34; -x_33 = lean_ctor_get(x_29, 3); -lean_dec(x_33); -x_34 = !lean_is_exclusive(x_30); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_35 = lean_ctor_get(x_30, 0); -x_36 = l_Lean_PersistentArray_append___rarg(x_15, x_35); -lean_dec(x_35); -lean_ctor_set(x_30, 0, x_36); -x_37 = lean_st_ref_set(x_12, x_29, x_31); -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); -x_39 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_22, x_9, x_10, x_11, x_12, x_38); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_22); -if (lean_obj_tag(x_39) == 0) -{ -uint8_t x_40; -x_40 = !lean_is_exclusive(x_39); -if (x_40 == 0) -{ -return x_39; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_39, 0); -x_42 = lean_ctor_get(x_39, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_39); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; -} -} -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_39); -if (x_44 == 0) -{ -return x_39; -} -else -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_39, 0); -x_46 = lean_ctor_get(x_39, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_39); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -} -else -{ -uint64_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_48 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); -x_49 = lean_ctor_get(x_30, 0); -lean_inc(x_49); -lean_dec(x_30); -x_50 = l_Lean_PersistentArray_append___rarg(x_15, x_49); -lean_dec(x_49); -x_51 = lean_alloc_ctor(0, 1, 8); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set_uint64(x_51, sizeof(void*)*1, x_48); -lean_ctor_set(x_29, 3, x_51); -x_52 = lean_st_ref_set(x_12, x_29, x_31); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_22, x_9, x_10, x_11, x_12, x_53); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_22); -if (lean_obj_tag(x_54) == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_57 = x_54; -} else { - lean_dec_ref(x_54); - x_57 = lean_box(0); -} -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(0, 2, 0); -} else { - x_58 = x_57; -} -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_59 = lean_ctor_get(x_54, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_54, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_61 = x_54; -} else { - lean_dec_ref(x_54); - x_61 = lean_box(0); -} -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); -} else { - x_62 = x_61; -} -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; -} -} -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint64_t x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_63 = lean_ctor_get(x_29, 0); -x_64 = lean_ctor_get(x_29, 1); -x_65 = lean_ctor_get(x_29, 2); -x_66 = lean_ctor_get(x_29, 4); -x_67 = lean_ctor_get(x_29, 5); -x_68 = lean_ctor_get(x_29, 6); -x_69 = lean_ctor_get(x_29, 7); -lean_inc(x_69); -lean_inc(x_68); -lean_inc(x_67); -lean_inc(x_66); -lean_inc(x_65); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_29); -x_70 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); -x_71 = lean_ctor_get(x_30, 0); -lean_inc(x_71); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - x_72 = x_30; -} else { - lean_dec_ref(x_30); - x_72 = lean_box(0); -} -x_73 = l_Lean_PersistentArray_append___rarg(x_15, x_71); -lean_dec(x_71); -if (lean_is_scalar(x_72)) { - x_74 = lean_alloc_ctor(0, 1, 8); -} else { - x_74 = x_72; -} -lean_ctor_set(x_74, 0, x_73); -lean_ctor_set_uint64(x_74, sizeof(void*)*1, x_70); -x_75 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_75, 0, x_63); -lean_ctor_set(x_75, 1, x_64); -lean_ctor_set(x_75, 2, x_65); -lean_ctor_set(x_75, 3, x_74); -lean_ctor_set(x_75, 4, x_66); -lean_ctor_set(x_75, 5, x_67); -lean_ctor_set(x_75, 6, x_68); -lean_ctor_set(x_75, 7, x_69); -x_76 = lean_st_ref_set(x_12, x_75, x_31); -x_77 = lean_ctor_get(x_76, 1); -lean_inc(x_77); -lean_dec(x_76); -x_78 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_22, x_9, x_10, x_11, x_12, x_77); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_22); -if (lean_obj_tag(x_78) == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_81 = x_78; -} else { - lean_dec_ref(x_78); - x_81 = lean_box(0); -} -if (lean_is_scalar(x_81)) { - x_82 = lean_alloc_ctor(0, 2, 0); -} else { - x_82 = x_81; -} -lean_ctor_set(x_82, 0, x_79); -lean_ctor_set(x_82, 1, x_80); -return x_82; -} -else -{ -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_83 = lean_ctor_get(x_78, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_78, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_85 = x_78; -} else { - lean_dec_ref(x_78); - x_85 = lean_box(0); -} -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(1, 2, 0); -} else { - x_86 = x_85; -} -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_84); -return x_86; -} -} -} -else -{ -lean_object* x_87; double x_88; double x_89; lean_object* x_90; -x_87 = lean_box(0); -x_88 = lean_unbox_float(x_23); -lean_dec(x_23); -x_89 = lean_unbox_float(x_24); -lean_dec(x_24); -x_90 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_22, x_26, x_88, x_89, x_5, x_87, x_9, x_10, x_11, x_12, x_20); -return x_90; -} -} -} -} -else -{ -lean_object* x_211; lean_object* x_212; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; -x_303 = lean_io_get_num_heartbeats(x_16); -x_304 = lean_ctor_get(x_303, 0); -lean_inc(x_304); -x_305 = lean_ctor_get(x_303, 1); -lean_inc(x_305); -lean_dec(x_303); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -x_306 = lean_apply_5(x_7, x_9, x_10, x_11, x_12, x_305); -if (lean_obj_tag(x_306) == 0) -{ -uint8_t x_307; -x_307 = !lean_is_exclusive(x_306); -if (x_307 == 0) -{ -lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; uint8_t x_312; -x_308 = lean_ctor_get(x_306, 0); -x_309 = lean_ctor_get(x_306, 1); -x_310 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_310, 0, x_308); -x_311 = lean_io_get_num_heartbeats(x_309); -x_312 = !lean_is_exclusive(x_311); -if (x_312 == 0) -{ -lean_object* x_313; lean_object* x_314; uint8_t x_315; lean_object* x_316; double x_317; double x_318; lean_object* x_319; lean_object* x_320; -x_313 = lean_ctor_get(x_311, 0); -x_314 = lean_ctor_get(x_311, 1); -x_315 = 0; -x_316 = lean_unsigned_to_nat(0u); -x_317 = l_Float_ofScientific(x_304, x_315, x_316); -lean_dec(x_304); -x_318 = l_Float_ofScientific(x_313, x_315, x_316); -lean_dec(x_313); -x_319 = lean_box_float(x_317); -x_320 = lean_box_float(x_318); -lean_ctor_set(x_311, 1, x_320); -lean_ctor_set(x_311, 0, x_319); -lean_ctor_set(x_306, 1, x_311); -lean_ctor_set(x_306, 0, x_310); -x_211 = x_306; -x_212 = x_314; -goto block_302; -} -else -{ -lean_object* x_321; lean_object* x_322; uint8_t x_323; lean_object* x_324; double x_325; double x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; -x_321 = lean_ctor_get(x_311, 0); -x_322 = lean_ctor_get(x_311, 1); -lean_inc(x_322); -lean_inc(x_321); -lean_dec(x_311); -x_323 = 0; -x_324 = lean_unsigned_to_nat(0u); -x_325 = l_Float_ofScientific(x_304, x_323, x_324); -lean_dec(x_304); -x_326 = l_Float_ofScientific(x_321, x_323, x_324); -lean_dec(x_321); -x_327 = lean_box_float(x_325); -x_328 = lean_box_float(x_326); -x_329 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_329, 0, x_327); -lean_ctor_set(x_329, 1, x_328); -lean_ctor_set(x_306, 1, x_329); -lean_ctor_set(x_306, 0, x_310); -x_211 = x_306; -x_212 = x_322; -goto block_302; -} -} -else -{ -lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; uint8_t x_337; lean_object* x_338; double x_339; double x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; -x_330 = lean_ctor_get(x_306, 0); -x_331 = lean_ctor_get(x_306, 1); -lean_inc(x_331); -lean_inc(x_330); -lean_dec(x_306); -x_332 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_332, 0, x_330); -x_333 = lean_io_get_num_heartbeats(x_331); -x_334 = lean_ctor_get(x_333, 0); -lean_inc(x_334); -x_335 = lean_ctor_get(x_333, 1); -lean_inc(x_335); -if (lean_is_exclusive(x_333)) { - lean_ctor_release(x_333, 0); - lean_ctor_release(x_333, 1); - x_336 = x_333; -} else { - lean_dec_ref(x_333); - x_336 = lean_box(0); -} -x_337 = 0; -x_338 = lean_unsigned_to_nat(0u); -x_339 = l_Float_ofScientific(x_304, x_337, x_338); -lean_dec(x_304); -x_340 = l_Float_ofScientific(x_334, x_337, x_338); -lean_dec(x_334); -x_341 = lean_box_float(x_339); -x_342 = lean_box_float(x_340); -if (lean_is_scalar(x_336)) { - x_343 = lean_alloc_ctor(0, 2, 0); -} else { - x_343 = x_336; -} -lean_ctor_set(x_343, 0, x_341); -lean_ctor_set(x_343, 1, x_342); -x_344 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_344, 0, x_332); -lean_ctor_set(x_344, 1, x_343); -x_211 = x_344; -x_212 = x_335; -goto block_302; -} -} -else -{ -uint8_t x_345; -x_345 = !lean_is_exclusive(x_306); -if (x_345 == 0) -{ -lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; uint8_t x_350; -x_346 = lean_ctor_get(x_306, 0); -x_347 = lean_ctor_get(x_306, 1); -x_348 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_348, 0, x_346); -x_349 = lean_io_get_num_heartbeats(x_347); -x_350 = !lean_is_exclusive(x_349); -if (x_350 == 0) -{ -lean_object* x_351; lean_object* x_352; uint8_t x_353; lean_object* x_354; double x_355; double x_356; lean_object* x_357; lean_object* x_358; -x_351 = lean_ctor_get(x_349, 0); -x_352 = lean_ctor_get(x_349, 1); -x_353 = 0; -x_354 = lean_unsigned_to_nat(0u); -x_355 = l_Float_ofScientific(x_304, x_353, x_354); -lean_dec(x_304); -x_356 = l_Float_ofScientific(x_351, x_353, x_354); -lean_dec(x_351); -x_357 = lean_box_float(x_355); -x_358 = lean_box_float(x_356); -lean_ctor_set(x_349, 1, x_358); -lean_ctor_set(x_349, 0, x_357); -lean_ctor_set_tag(x_306, 0); -lean_ctor_set(x_306, 1, x_349); -lean_ctor_set(x_306, 0, x_348); -x_211 = x_306; -x_212 = x_352; -goto block_302; -} -else -{ -lean_object* x_359; lean_object* x_360; uint8_t x_361; lean_object* x_362; double x_363; double x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; -x_359 = lean_ctor_get(x_349, 0); -x_360 = lean_ctor_get(x_349, 1); -lean_inc(x_360); -lean_inc(x_359); -lean_dec(x_349); -x_361 = 0; -x_362 = lean_unsigned_to_nat(0u); -x_363 = l_Float_ofScientific(x_304, x_361, x_362); -lean_dec(x_304); -x_364 = l_Float_ofScientific(x_359, x_361, x_362); -lean_dec(x_359); -x_365 = lean_box_float(x_363); -x_366 = lean_box_float(x_364); -x_367 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_367, 0, x_365); -lean_ctor_set(x_367, 1, x_366); -lean_ctor_set_tag(x_306, 0); -lean_ctor_set(x_306, 1, x_367); -lean_ctor_set(x_306, 0, x_348); -x_211 = x_306; -x_212 = x_360; -goto block_302; -} -} -else -{ -lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; uint8_t x_375; lean_object* x_376; double x_377; double x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; -x_368 = lean_ctor_get(x_306, 0); -x_369 = lean_ctor_get(x_306, 1); -lean_inc(x_369); -lean_inc(x_368); -lean_dec(x_306); -x_370 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_370, 0, x_368); -x_371 = lean_io_get_num_heartbeats(x_369); -x_372 = lean_ctor_get(x_371, 0); -lean_inc(x_372); -x_373 = lean_ctor_get(x_371, 1); -lean_inc(x_373); -if (lean_is_exclusive(x_371)) { - lean_ctor_release(x_371, 0); - lean_ctor_release(x_371, 1); - x_374 = x_371; -} else { - lean_dec_ref(x_371); - x_374 = lean_box(0); -} -x_375 = 0; -x_376 = lean_unsigned_to_nat(0u); -x_377 = l_Float_ofScientific(x_304, x_375, x_376); -lean_dec(x_304); -x_378 = l_Float_ofScientific(x_372, x_375, x_376); -lean_dec(x_372); -x_379 = lean_box_float(x_377); -x_380 = lean_box_float(x_378); -if (lean_is_scalar(x_374)) { - x_381 = lean_alloc_ctor(0, 2, 0); -} else { - x_381 = x_374; -} -lean_ctor_set(x_381, 0, x_379); -lean_ctor_set(x_381, 1, x_380); -x_382 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_382, 0, x_370); -lean_ctor_set(x_382, 1, x_381); -x_211 = x_382; -x_212 = x_373; -goto block_302; -} -} -block_302: -{ -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; uint8_t x_218; uint8_t x_219; -x_213 = lean_ctor_get(x_211, 1); -lean_inc(x_213); -x_214 = lean_ctor_get(x_211, 0); -lean_inc(x_214); -lean_dec(x_211); -x_215 = lean_ctor_get(x_213, 0); -lean_inc(x_215); -x_216 = lean_ctor_get(x_213, 1); -lean_inc(x_216); -lean_dec(x_213); -x_217 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2; -x_218 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_217); -if (x_218 == 0) -{ -if (x_6 == 0) -{ -uint8_t x_284; -x_284 = 0; -x_219 = x_284; -goto block_283; -} -else -{ -lean_object* x_285; double x_286; double x_287; lean_object* x_288; -x_285 = lean_box(0); -x_286 = lean_unbox_float(x_215); -lean_dec(x_215); -x_287 = lean_unbox_float(x_216); -lean_dec(x_216); -x_288 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_286, x_287, x_5, x_285, x_9, x_10, x_11, x_12, x_212); -return x_288; -} -} -else -{ -if (x_6 == 0) -{ -double x_289; double x_290; double x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; double x_296; uint8_t x_297; -x_289 = lean_unbox_float(x_216); -x_290 = lean_unbox_float(x_215); -x_291 = lean_float_sub(x_289, x_290); -x_292 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3; -x_293 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_292); -x_294 = 0; -x_295 = lean_unsigned_to_nat(0u); -x_296 = l_Float_ofScientific(x_293, x_294, x_295); -lean_dec(x_293); -x_297 = lean_float_decLt(x_296, x_291); -x_219 = x_297; -goto block_283; -} -else -{ -lean_object* x_298; double x_299; double x_300; lean_object* x_301; -x_298 = lean_box(0); -x_299 = lean_unbox_float(x_215); -lean_dec(x_215); -x_300 = lean_unbox_float(x_216); -lean_dec(x_216); -x_301 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_299, x_300, x_5, x_298, x_9, x_10, x_11, x_12, x_212); -return x_301; -} -} -block_283: -{ -if (x_219 == 0) -{ -lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; -lean_dec(x_216); -lean_dec(x_215); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -x_220 = lean_st_ref_take(x_12, x_212); -x_221 = lean_ctor_get(x_220, 0); -lean_inc(x_221); -x_222 = lean_ctor_get(x_221, 3); -lean_inc(x_222); -x_223 = lean_ctor_get(x_220, 1); -lean_inc(x_223); -lean_dec(x_220); -x_224 = !lean_is_exclusive(x_221); -if (x_224 == 0) -{ -lean_object* x_225; uint8_t x_226; -x_225 = lean_ctor_get(x_221, 3); -lean_dec(x_225); -x_226 = !lean_is_exclusive(x_222); -if (x_226 == 0) -{ -lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_227 = lean_ctor_get(x_222, 0); -x_228 = l_Lean_PersistentArray_append___rarg(x_15, x_227); -lean_dec(x_227); -lean_ctor_set(x_222, 0, x_228); -x_229 = lean_st_ref_set(x_12, x_221, x_223); -x_230 = lean_ctor_get(x_229, 1); -lean_inc(x_230); -lean_dec(x_229); -x_231 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_214, x_9, x_10, x_11, x_12, x_230); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_214); -if (lean_obj_tag(x_231) == 0) -{ -uint8_t x_232; -x_232 = !lean_is_exclusive(x_231); -if (x_232 == 0) -{ -return x_231; -} -else -{ -lean_object* x_233; lean_object* x_234; lean_object* x_235; -x_233 = lean_ctor_get(x_231, 0); -x_234 = lean_ctor_get(x_231, 1); -lean_inc(x_234); -lean_inc(x_233); -lean_dec(x_231); -x_235 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_235, 0, x_233); -lean_ctor_set(x_235, 1, x_234); -return x_235; -} -} -else -{ -uint8_t x_236; -x_236 = !lean_is_exclusive(x_231); -if (x_236 == 0) -{ -return x_231; -} -else -{ -lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_237 = lean_ctor_get(x_231, 0); -x_238 = lean_ctor_get(x_231, 1); -lean_inc(x_238); -lean_inc(x_237); -lean_dec(x_231); -x_239 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_239, 0, x_237); -lean_ctor_set(x_239, 1, x_238); -return x_239; -} -} -} -else -{ -uint64_t x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_240 = lean_ctor_get_uint64(x_222, sizeof(void*)*1); -x_241 = lean_ctor_get(x_222, 0); -lean_inc(x_241); -lean_dec(x_222); -x_242 = l_Lean_PersistentArray_append___rarg(x_15, x_241); -lean_dec(x_241); -x_243 = lean_alloc_ctor(0, 1, 8); -lean_ctor_set(x_243, 0, x_242); -lean_ctor_set_uint64(x_243, sizeof(void*)*1, x_240); -lean_ctor_set(x_221, 3, x_243); -x_244 = lean_st_ref_set(x_12, x_221, x_223); -x_245 = lean_ctor_get(x_244, 1); -lean_inc(x_245); -lean_dec(x_244); -x_246 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_214, x_9, x_10, x_11, x_12, x_245); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_214); -if (lean_obj_tag(x_246) == 0) -{ -lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_247 = lean_ctor_get(x_246, 0); -lean_inc(x_247); -x_248 = lean_ctor_get(x_246, 1); -lean_inc(x_248); -if (lean_is_exclusive(x_246)) { - lean_ctor_release(x_246, 0); - lean_ctor_release(x_246, 1); - x_249 = x_246; -} else { - lean_dec_ref(x_246); - x_249 = lean_box(0); -} -if (lean_is_scalar(x_249)) { - x_250 = lean_alloc_ctor(0, 2, 0); -} else { - x_250 = x_249; -} -lean_ctor_set(x_250, 0, x_247); -lean_ctor_set(x_250, 1, x_248); -return x_250; -} -else -{ -lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; -x_251 = lean_ctor_get(x_246, 0); -lean_inc(x_251); -x_252 = lean_ctor_get(x_246, 1); -lean_inc(x_252); -if (lean_is_exclusive(x_246)) { - lean_ctor_release(x_246, 0); - lean_ctor_release(x_246, 1); - x_253 = x_246; -} else { - lean_dec_ref(x_246); - x_253 = lean_box(0); -} -if (lean_is_scalar(x_253)) { - x_254 = lean_alloc_ctor(1, 2, 0); -} else { - x_254 = x_253; -} -lean_ctor_set(x_254, 0, x_251); -lean_ctor_set(x_254, 1, x_252); -return x_254; -} -} -} -else -{ -lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; uint64_t x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; -x_255 = lean_ctor_get(x_221, 0); -x_256 = lean_ctor_get(x_221, 1); -x_257 = lean_ctor_get(x_221, 2); -x_258 = lean_ctor_get(x_221, 4); -x_259 = lean_ctor_get(x_221, 5); -x_260 = lean_ctor_get(x_221, 6); -x_261 = lean_ctor_get(x_221, 7); -lean_inc(x_261); -lean_inc(x_260); -lean_inc(x_259); -lean_inc(x_258); -lean_inc(x_257); -lean_inc(x_256); -lean_inc(x_255); -lean_dec(x_221); -x_262 = lean_ctor_get_uint64(x_222, sizeof(void*)*1); -x_263 = lean_ctor_get(x_222, 0); -lean_inc(x_263); -if (lean_is_exclusive(x_222)) { - lean_ctor_release(x_222, 0); - x_264 = x_222; -} else { - lean_dec_ref(x_222); - x_264 = lean_box(0); -} -x_265 = l_Lean_PersistentArray_append___rarg(x_15, x_263); -lean_dec(x_263); -if (lean_is_scalar(x_264)) { - x_266 = lean_alloc_ctor(0, 1, 8); -} else { - x_266 = x_264; -} -lean_ctor_set(x_266, 0, x_265); -lean_ctor_set_uint64(x_266, sizeof(void*)*1, x_262); -x_267 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_267, 0, x_255); -lean_ctor_set(x_267, 1, x_256); -lean_ctor_set(x_267, 2, x_257); -lean_ctor_set(x_267, 3, x_266); -lean_ctor_set(x_267, 4, x_258); -lean_ctor_set(x_267, 5, x_259); -lean_ctor_set(x_267, 6, x_260); -lean_ctor_set(x_267, 7, x_261); -x_268 = lean_st_ref_set(x_12, x_267, x_223); -x_269 = lean_ctor_get(x_268, 1); -lean_inc(x_269); -lean_dec(x_268); -x_270 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_214, x_9, x_10, x_11, x_12, x_269); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_214); -if (lean_obj_tag(x_270) == 0) -{ -lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; -x_271 = lean_ctor_get(x_270, 0); -lean_inc(x_271); -x_272 = lean_ctor_get(x_270, 1); -lean_inc(x_272); -if (lean_is_exclusive(x_270)) { - lean_ctor_release(x_270, 0); - lean_ctor_release(x_270, 1); - x_273 = x_270; -} else { - lean_dec_ref(x_270); - x_273 = lean_box(0); -} -if (lean_is_scalar(x_273)) { - x_274 = lean_alloc_ctor(0, 2, 0); -} else { - x_274 = x_273; -} -lean_ctor_set(x_274, 0, x_271); -lean_ctor_set(x_274, 1, x_272); -return x_274; -} -else -{ -lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; -x_275 = lean_ctor_get(x_270, 0); -lean_inc(x_275); -x_276 = lean_ctor_get(x_270, 1); -lean_inc(x_276); -if (lean_is_exclusive(x_270)) { - lean_ctor_release(x_270, 0); - lean_ctor_release(x_270, 1); - x_277 = x_270; -} else { - lean_dec_ref(x_270); - x_277 = lean_box(0); -} -if (lean_is_scalar(x_277)) { - x_278 = lean_alloc_ctor(1, 2, 0); -} else { - x_278 = x_277; -} -lean_ctor_set(x_278, 0, x_275); -lean_ctor_set(x_278, 1, x_276); -return x_278; -} -} -} -else -{ -lean_object* x_279; double x_280; double x_281; lean_object* x_282; -x_279 = lean_box(0); -x_280 = lean_unbox_float(x_215); -lean_dec(x_215); -x_281 = lean_unbox_float(x_216); -lean_dec(x_216); -x_282 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_280, x_281, x_5, x_279, x_9, x_10, x_11, x_12, x_212); -return x_282; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = lean_ctor_get(x_8, 2); -lean_inc(x_11); -lean_inc(x_1); -x_12 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_unbox(x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2; -x_17 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_16); -if (x_17 == 0) -{ -lean_object* x_18; -lean_dec(x_13); -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_18 = lean_apply_5(x_3, x_6, x_7, x_8, x_9, x_15); -if (lean_obj_tag(x_18) == 0) -{ -uint8_t x_19; -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) -{ -return x_18; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_18, 0); -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_18); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; -} -} -else -{ -uint8_t x_23; -x_23 = !lean_is_exclusive(x_18); -if (x_23 == 0) -{ -return x_18; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_18, 0); -x_25 = lean_ctor_get(x_18, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_18); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; -} -} -} -else -{ -lean_object* x_27; uint8_t x_28; lean_object* x_29; -x_27 = lean_box(0); -x_28 = lean_unbox(x_13); -lean_dec(x_13); -x_29 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4(x_11, x_1, x_4, x_5, x_2, x_28, x_3, x_27, x_6, x_7, x_8, x_9, x_15); -lean_dec(x_11); -return x_29; -} -} -else -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_12, 1); -lean_inc(x_30); -lean_dec(x_12); -x_31 = lean_box(0); -x_32 = lean_unbox(x_13); -lean_dec(x_13); -x_33 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4(x_11, x_1, x_4, x_5, x_2, x_32, x_3, x_31, x_6, x_7, x_8, x_9, x_30); -lean_dec(x_11); -return x_33; -} -} -} -LEAN_EXPORT uint8_t l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1(lean_object* x_1) { -_start: -{ -uint8_t x_2; -x_2 = 0; -return x_2; -} -} -static lean_object* _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1___boxed), 1, 0); -return x_1; -} -} -static lean_object* _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Running pass: ", 14, 14); -return x_1; -} -} -static lean_object* _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -lean_dec(x_1); -x_9 = 1; -x_10 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1; -x_11 = l_Lean_Name_toString(x_8, x_9, x_10); -x_12 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2; -x_13 = lean_string_append(x_12, x_11); -lean_dec(x_11); -x_14 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3; -x_15 = lean_string_append(x_13, x_14); -x_16 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_16, 0, x_15); -x_17 = l_Lean_MessageData_ofFormat(x_16); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_7); -return x_18; -} -} -static lean_object* _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("bv", 2, 2); -return x_1; -} -} -static lean_object* _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_8; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -return x_8; -} -else -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_9; lean_object* x_10; -x_9 = lean_ctor_get(x_2, 1); -lean_inc(x_9); -lean_dec(x_2); -x_10 = lean_box(0); -x_1 = x_10; -x_2 = x_9; -goto _start; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_12 = lean_ctor_get(x_2, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_2, 1); -lean_inc(x_13); -lean_dec(x_2); -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -lean_dec(x_1); -lean_inc(x_12); -x_15 = lean_alloc_closure((void*)(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___boxed), 7, 1); -lean_closure_set(x_15, 0, x_12); -x_16 = lean_ctor_get(x_12, 1); -lean_inc(x_16); -lean_dec(x_12); -x_17 = lean_apply_1(x_16, x_14); -x_18 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2; -x_19 = 1; -x_20 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_21 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(x_18, x_15, x_17, x_19, x_20, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_1 = x_22; -x_2 = x_13; -x_7 = x_23; -goto _start; -} -else -{ -uint8_t x_25; -lean_dec(x_13); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_25 = !lean_is_exclusive(x_21); -if (x_25 == 0) -{ -return x_21; -} -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_21, 0); -x_27 = lean_ctor_get(x_21, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_21); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; -x_8 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_8, 0, x_1); -x_9 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_9, 0, x_8); -lean_ctor_set(x_9, 1, x_7); -return x_9; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Meta", 4, 4); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Rerunning pipeline on:\n", 23, 23); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Pipeline reached a fixpoint", 27, 27); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; -lean_inc(x_2); -x_8 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_8, 0, x_2); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_1); -x_9 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3(x_8, x_1, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_9, 0); -lean_dec(x_12); -x_13 = lean_box(0); -lean_ctor_set(x_9, 0, x_13); -return x_9; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_dec(x_9); -x_15 = lean_box(0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; -} -} -else -{ -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_9, 1); -lean_inc(x_17); -lean_dec(x_9); -x_18 = !lean_is_exclusive(x_10); -if (x_18 == 0) -{ -lean_object* x_19; uint8_t x_20; -x_19 = lean_ctor_get(x_10, 0); -x_20 = lean_name_eq(x_2, x_19); -lean_dec(x_2); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_22 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_21, x_3, x_4, x_5, x_6, x_17); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_unbox(x_23); -lean_dec(x_23); -if (x_24 == 0) -{ -lean_object* x_25; -lean_free_object(x_10); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_2 = x_19; -x_7 = x_25; -goto _start; -} -else -{ -uint8_t x_27; -x_27 = !lean_is_exclusive(x_22); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_28 = lean_ctor_get(x_22, 1); -x_29 = lean_ctor_get(x_22, 0); -lean_dec(x_29); -lean_inc(x_19); -x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4; -lean_ctor_set_tag(x_22, 7); -lean_ctor_set(x_22, 1, x_10); -lean_ctor_set(x_22, 0, x_30); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_22); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_21, x_32, x_3, x_4, x_5, x_6, x_28); -x_34 = lean_ctor_get(x_33, 1); -lean_inc(x_34); -lean_dec(x_33); -x_2 = x_19; -x_7 = x_34; -goto _start; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_36 = lean_ctor_get(x_22, 1); -lean_inc(x_36); -lean_dec(x_22); -lean_inc(x_19); -x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4; -x_38 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set(x_38, 1, x_10); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_40 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -x_41 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_21, x_40, x_3, x_4, x_5, x_6, x_36); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -x_2 = x_19; -x_7 = x_42; -goto _start; -} -} -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -lean_free_object(x_10); -lean_dec(x_1); -x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_45 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_44, x_3, x_4, x_5, x_6, x_17); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_unbox(x_46); -lean_dec(x_46); -if (x_47 == 0) -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_45, 1); -lean_inc(x_48); -lean_dec(x_45); -x_49 = lean_box(0); -x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_19, x_49, x_3, x_4, x_5, x_6, x_48); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_50; -} -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_51 = lean_ctor_get(x_45, 1); -lean_inc(x_51); -lean_dec(x_45); -x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7; -x_53 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_44, x_52, x_3, x_4, x_5, x_6, x_51); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_19, x_54, x_3, x_4, x_5, x_6, x_55); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_54); -return x_56; -} -} -} -else -{ -lean_object* x_57; uint8_t x_58; -x_57 = lean_ctor_get(x_10, 0); -lean_inc(x_57); -lean_dec(x_10); -x_58 = lean_name_eq(x_2, x_57); -lean_dec(x_2); -if (x_58 == 0) -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_60 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_59, x_3, x_4, x_5, x_6, x_17); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_unbox(x_61); -lean_dec(x_61); -if (x_62 == 0) -{ -lean_object* x_63; -x_63 = lean_ctor_get(x_60, 1); -lean_inc(x_63); -lean_dec(x_60); -x_2 = x_57; -x_7 = x_63; -goto _start; -} -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_65 = lean_ctor_get(x_60, 1); -lean_inc(x_65); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_66 = x_60; -} else { - lean_dec_ref(x_60); - x_66 = lean_box(0); -} -lean_inc(x_57); -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_57); -x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4; -if (lean_is_scalar(x_66)) { - x_69 = lean_alloc_ctor(7, 2, 0); -} else { - x_69 = x_66; - lean_ctor_set_tag(x_69, 7); -} -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_67); -x_70 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_71 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -x_72 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_59, x_71, x_3, x_4, x_5, x_6, x_65); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -lean_dec(x_72); -x_2 = x_57; -x_7 = x_73; -goto _start; -} -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; uint8_t x_78; -lean_dec(x_1); -x_75 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_76 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_75, x_3, x_4, x_5, x_6, x_17); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_unbox(x_77); -lean_dec(x_77); -if (x_78 == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_76, 1); -lean_inc(x_79); -lean_dec(x_76); -x_80 = lean_box(0); -x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_57, x_80, x_3, x_4, x_5, x_6, x_79); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_81; -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_82 = lean_ctor_get(x_76, 1); -lean_inc(x_82); -lean_dec(x_76); -x_83 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7; -x_84 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_75, x_83, x_3, x_4, x_5, x_6, x_82); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_57, x_85, x_3, x_4, x_5, x_6, x_86); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_85); -return x_87; -} -} -} -} -} -else -{ -uint8_t x_88; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_88 = !lean_is_exclusive(x_9); -if (x_88 == 0) -{ -return x_9; -} -else -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_9, 0); -x_90 = lean_ctor_get(x_9, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_9); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; -} -} -} -} -LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; uint8_t x_17; double x_18; double x_19; lean_object* x_20; -x_16 = lean_unbox(x_2); -lean_dec(x_2); -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox_float(x_8); -lean_dec(x_8); -x_19 = lean_unbox_float(x_9); -lean_dec(x_9); -x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2(x_1, x_16, x_3, x_4, x_5, x_6, x_17, x_18, x_19, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_6); -return x_20; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; uint8_t x_17; double x_18; double x_19; lean_object* x_20; -x_16 = lean_unbox(x_2); -lean_dec(x_2); -x_17 = lean_unbox(x_6); -lean_dec(x_6); -x_18 = lean_unbox_float(x_7); -lean_dec(x_7); -x_19 = lean_unbox_float(x_8); -lean_dec(x_8); -x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3(x_1, x_16, x_3, x_4, x_5, x_17, x_18, x_19, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_10); -return x_20; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -uint8_t x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_unbox(x_3); -lean_dec(x_3); -x_15 = lean_unbox(x_6); -lean_dec(x_6); -x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4(x_1, x_2, x_14, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_8); -lean_dec(x_1); -return x_16; -} -} -LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; lean_object* x_12; -x_11 = lean_unbox(x_4); -lean_dec(x_4); -x_12 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1___boxed(lean_object* x_1) { -_start: -{ -uint8_t x_2; lean_object* x_3; -x_2 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__1(x_1); -lean_dec(x_1); -x_3 = lean_box(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_8; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeExt; -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt; -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Meta_sevalSimpExtension; -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5; -x_2 = lean_unsigned_to_nat(0u); -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(32u); -x_2 = lean_mk_empty_array_with_capacity(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9() { -_start: -{ -size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = 5; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7; -x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); -lean_ctor_set(x_5, 0, x_2); -lean_ctor_set(x_5, 1, x_3); -lean_ctor_set(x_5, 2, x_4); -lean_ctor_set(x_5, 3, x_4); -lean_ctor_set_usize(x_5, 4, x_1); -return x_5; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9; -x_3 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_1); -lean_ctor_set(x_3, 2, x_1); -lean_ctor_set(x_3, 3, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1; -x_9 = l_Lean_Meta_SimpExtension_getTheorems(x_8, x_5, x_6, x_7); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2; -x_13 = l_Lean_Meta_Simp_SimprocExtension_getSimprocs(x_12, x_5, x_6, x_11); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3; -x_17 = l_Lean_Meta_SimpExtension_getTheorems(x_16, x_5, x_6, x_15); -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -x_21 = l_Lean_Meta_Simp_getSEvalSimprocs___rarg(x_6, x_20); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_21, 0); -x_24 = lean_ctor_get(x_21, 1); -x_25 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_6, x_24); -x_26 = !lean_is_exclusive(x_25); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; uint8_t x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_27 = lean_ctor_get(x_25, 0); -x_28 = lean_ctor_get(x_25, 1); -x_29 = lean_unsigned_to_nat(2u); -x_30 = 0; -x_31 = 1; -x_32 = 0; -x_33 = lean_alloc_ctor(0, 2, 19); -lean_ctor_set(x_33, 0, x_1); -lean_ctor_set(x_33, 1, x_29); -lean_ctor_set_uint8(x_33, sizeof(void*)*2, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 1, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 2, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 3, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 4, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 5, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 6, x_32); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 7, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 8, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 9, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 10, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 11, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 12, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 13, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 14, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 15, x_30); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 16, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 17, x_31); -lean_ctor_set_uint8(x_33, sizeof(void*)*2 + 18, x_31); -x_34 = lean_box(0); -lean_ctor_set_tag(x_25, 1); -lean_ctor_set(x_25, 1, x_34); -lean_ctor_set(x_25, 0, x_19); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_25); -lean_ctor_set(x_21, 0, x_10); -x_35 = lean_array_mk(x_21); -x_36 = l_Lean_Meta_Simp_mkContext(x_33, x_35, x_27, x_3, x_4, x_5, x_6, x_28); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_36, 0); -x_39 = lean_ctor_get(x_36, 1); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_40 = l_Lean_MVarId_getNondepPropHyps(x_2, x_3, x_4, x_5, x_6, x_39); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -lean_ctor_set_tag(x_36, 1); -lean_ctor_set(x_36, 1, x_34); -lean_ctor_set(x_36, 0, x_23); -lean_ctor_set_tag(x_17, 1); -lean_ctor_set(x_17, 1, x_36); -lean_ctor_set(x_17, 0, x_14); -x_43 = lean_array_mk(x_17); -x_44 = lean_box(0); -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_46 = l_Lean_Meta_simpGoal(x_2, x_38, x_43, x_44, x_31, x_41, x_45, x_3, x_4, x_5, x_6, x_42); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -lean_dec(x_47); -if (lean_obj_tag(x_48) == 0) -{ -uint8_t x_49; -x_49 = !lean_is_exclusive(x_46); -if (x_49 == 0) -{ -lean_object* x_50; -x_50 = lean_ctor_get(x_46, 0); -lean_dec(x_50); -lean_ctor_set(x_46, 0, x_44); -return x_46; -} -else -{ -lean_object* x_51; lean_object* x_52; -x_51 = lean_ctor_get(x_46, 1); -lean_inc(x_51); -lean_dec(x_46); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_44); -lean_ctor_set(x_52, 1, x_51); -return x_52; -} -} -else -{ -uint8_t x_53; -x_53 = !lean_is_exclusive(x_48); -if (x_53 == 0) -{ -uint8_t x_54; -x_54 = !lean_is_exclusive(x_46); -if (x_54 == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_48, 0); -x_56 = lean_ctor_get(x_46, 0); -lean_dec(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -lean_ctor_set(x_48, 0, x_57); -lean_ctor_set(x_46, 0, x_48); -return x_46; -} -else -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_58 = lean_ctor_get(x_48, 0); -x_59 = lean_ctor_get(x_46, 1); -lean_inc(x_59); -lean_dec(x_46); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -lean_ctor_set(x_48, 0, x_60); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_48); -lean_ctor_set(x_61, 1, x_59); -return x_61; -} -} -else -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_62 = lean_ctor_get(x_48, 0); -lean_inc(x_62); -lean_dec(x_48); -x_63 = lean_ctor_get(x_46, 1); -lean_inc(x_63); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_64 = x_46; -} else { - lean_dec_ref(x_46); - x_64 = lean_box(0); -} -x_65 = lean_ctor_get(x_62, 1); -lean_inc(x_65); -lean_dec(x_62); -x_66 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_66, 0, x_65); -if (lean_is_scalar(x_64)) { - x_67 = lean_alloc_ctor(0, 2, 0); -} else { - x_67 = x_64; -} -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_63); -return x_67; -} -} -} -else -{ -uint8_t x_68; -x_68 = !lean_is_exclusive(x_46); -if (x_68 == 0) -{ -return x_46; -} -else -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_46, 0); -x_70 = lean_ctor_get(x_46, 1); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_46); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -return x_71; -} -} -} -else -{ -uint8_t x_72; -lean_free_object(x_36); -lean_dec(x_38); -lean_dec(x_23); -lean_free_object(x_17); -lean_dec(x_14); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_72 = !lean_is_exclusive(x_40); -if (x_72 == 0) -{ -return x_40; -} -else -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_40, 0); -x_74 = lean_ctor_get(x_40, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_40); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -return x_75; -} -} -} -else -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_36, 0); -x_77 = lean_ctor_get(x_36, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_36); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_78 = l_Lean_MVarId_getNondepPropHyps(x_2, x_3, x_4, x_5, x_6, x_77); -if (lean_obj_tag(x_78) == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_79 = lean_ctor_get(x_78, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_78, 1); -lean_inc(x_80); -lean_dec(x_78); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_23); -lean_ctor_set(x_81, 1, x_34); -lean_ctor_set_tag(x_17, 1); -lean_ctor_set(x_17, 1, x_81); -lean_ctor_set(x_17, 0, x_14); -x_82 = lean_array_mk(x_17); -x_83 = lean_box(0); -x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_85 = l_Lean_Meta_simpGoal(x_2, x_76, x_82, x_83, x_31, x_79, x_84, x_3, x_4, x_5, x_6, x_80); -if (lean_obj_tag(x_85) == 0) -{ -lean_object* x_86; lean_object* x_87; -x_86 = lean_ctor_get(x_85, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -lean_dec(x_86); -if (lean_obj_tag(x_87) == 0) -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_85, 1); -lean_inc(x_88); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_89 = x_85; -} else { - lean_dec_ref(x_85); - x_89 = lean_box(0); -} -if (lean_is_scalar(x_89)) { - x_90 = lean_alloc_ctor(0, 2, 0); -} else { - x_90 = x_89; -} -lean_ctor_set(x_90, 0, x_83); -lean_ctor_set(x_90, 1, x_88); -return x_90; -} -else -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_91 = lean_ctor_get(x_87, 0); -lean_inc(x_91); -if (lean_is_exclusive(x_87)) { - lean_ctor_release(x_87, 0); - x_92 = x_87; -} else { - lean_dec_ref(x_87); - x_92 = lean_box(0); -} -x_93 = lean_ctor_get(x_85, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_94 = x_85; -} else { - lean_dec_ref(x_85); - x_94 = lean_box(0); -} -x_95 = lean_ctor_get(x_91, 1); -lean_inc(x_95); -lean_dec(x_91); -if (lean_is_scalar(x_92)) { - x_96 = lean_alloc_ctor(1, 1, 0); -} else { - x_96 = x_92; -} -lean_ctor_set(x_96, 0, x_95); -if (lean_is_scalar(x_94)) { - x_97 = lean_alloc_ctor(0, 2, 0); -} else { - x_97 = x_94; -} -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_93); -return x_97; -} -} -else -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_98 = lean_ctor_get(x_85, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_85, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_100 = x_85; -} else { - lean_dec_ref(x_85); - x_100 = lean_box(0); -} -if (lean_is_scalar(x_100)) { - x_101 = lean_alloc_ctor(1, 2, 0); -} else { - x_101 = x_100; -} -lean_ctor_set(x_101, 0, x_98); -lean_ctor_set(x_101, 1, x_99); -return x_101; -} -} -else -{ -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -lean_dec(x_76); -lean_dec(x_23); -lean_free_object(x_17); -lean_dec(x_14); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_102 = lean_ctor_get(x_78, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_78, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_104 = x_78; -} else { - lean_dec_ref(x_78); - x_104 = lean_box(0); -} -if (lean_is_scalar(x_104)) { - x_105 = lean_alloc_ctor(1, 2, 0); -} else { - x_105 = x_104; -} -lean_ctor_set(x_105, 0, x_102); -lean_ctor_set(x_105, 1, x_103); -return x_105; -} -} -} -else -{ -lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; uint8_t x_110; uint8_t x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_106 = lean_ctor_get(x_25, 0); -x_107 = lean_ctor_get(x_25, 1); -lean_inc(x_107); -lean_inc(x_106); -lean_dec(x_25); -x_108 = lean_unsigned_to_nat(2u); -x_109 = 0; -x_110 = 1; -x_111 = 0; -x_112 = lean_alloc_ctor(0, 2, 19); -lean_ctor_set(x_112, 0, x_1); -lean_ctor_set(x_112, 1, x_108); -lean_ctor_set_uint8(x_112, sizeof(void*)*2, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 1, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 2, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 3, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 4, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 5, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 6, x_111); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 7, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 8, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 9, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 10, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 11, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 12, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 13, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 14, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 15, x_109); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 16, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 17, x_110); -lean_ctor_set_uint8(x_112, sizeof(void*)*2 + 18, x_110); -x_113 = lean_box(0); -x_114 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_114, 0, x_19); -lean_ctor_set(x_114, 1, x_113); -lean_ctor_set_tag(x_21, 1); -lean_ctor_set(x_21, 1, x_114); -lean_ctor_set(x_21, 0, x_10); -x_115 = lean_array_mk(x_21); -x_116 = l_Lean_Meta_Simp_mkContext(x_112, x_115, x_106, x_3, x_4, x_5, x_6, x_107); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -x_118 = lean_ctor_get(x_116, 1); -lean_inc(x_118); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_119 = x_116; -} else { - lean_dec_ref(x_116); - x_119 = lean_box(0); -} -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_120 = l_Lean_MVarId_getNondepPropHyps(x_2, x_3, x_4, x_5, x_6, x_118); -if (lean_obj_tag(x_120) == 0) -{ -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_121 = lean_ctor_get(x_120, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -lean_dec(x_120); -if (lean_is_scalar(x_119)) { - x_123 = lean_alloc_ctor(1, 2, 0); -} else { - x_123 = x_119; - lean_ctor_set_tag(x_123, 1); -} -lean_ctor_set(x_123, 0, x_23); -lean_ctor_set(x_123, 1, x_113); -lean_ctor_set_tag(x_17, 1); -lean_ctor_set(x_17, 1, x_123); -lean_ctor_set(x_17, 0, x_14); -x_124 = lean_array_mk(x_17); -x_125 = lean_box(0); -x_126 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_127 = l_Lean_Meta_simpGoal(x_2, x_117, x_124, x_125, x_110, x_121, x_126, x_3, x_4, x_5, x_6, x_122); -if (lean_obj_tag(x_127) == 0) -{ -lean_object* x_128; lean_object* x_129; -x_128 = lean_ctor_get(x_127, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -lean_dec(x_128); -if (lean_obj_tag(x_129) == 0) -{ -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_127, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_131 = x_127; -} else { - lean_dec_ref(x_127); - x_131 = lean_box(0); -} -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(0, 2, 0); -} else { - x_132 = x_131; -} -lean_ctor_set(x_132, 0, x_125); -lean_ctor_set(x_132, 1, x_130); -return x_132; -} -else -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_133 = lean_ctor_get(x_129, 0); -lean_inc(x_133); -if (lean_is_exclusive(x_129)) { - lean_ctor_release(x_129, 0); - x_134 = x_129; -} else { - lean_dec_ref(x_129); - x_134 = lean_box(0); -} -x_135 = lean_ctor_get(x_127, 1); -lean_inc(x_135); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_136 = x_127; -} else { - lean_dec_ref(x_127); - x_136 = lean_box(0); -} -x_137 = lean_ctor_get(x_133, 1); -lean_inc(x_137); -lean_dec(x_133); -if (lean_is_scalar(x_134)) { - x_138 = lean_alloc_ctor(1, 1, 0); -} else { - x_138 = x_134; -} -lean_ctor_set(x_138, 0, x_137); -if (lean_is_scalar(x_136)) { - x_139 = lean_alloc_ctor(0, 2, 0); -} else { - x_139 = x_136; -} -lean_ctor_set(x_139, 0, x_138); -lean_ctor_set(x_139, 1, x_135); -return x_139; -} -} -else -{ -lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_140 = lean_ctor_get(x_127, 0); -lean_inc(x_140); -x_141 = lean_ctor_get(x_127, 1); -lean_inc(x_141); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_142 = x_127; -} else { - lean_dec_ref(x_127); - x_142 = lean_box(0); -} -if (lean_is_scalar(x_142)) { - x_143 = lean_alloc_ctor(1, 2, 0); -} else { - x_143 = x_142; -} -lean_ctor_set(x_143, 0, x_140); -lean_ctor_set(x_143, 1, x_141); -return x_143; -} -} -else -{ -lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -lean_dec(x_119); -lean_dec(x_117); -lean_dec(x_23); -lean_free_object(x_17); -lean_dec(x_14); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_144 = lean_ctor_get(x_120, 0); -lean_inc(x_144); -x_145 = lean_ctor_get(x_120, 1); -lean_inc(x_145); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_146 = x_120; -} else { - lean_dec_ref(x_120); - x_146 = lean_box(0); -} -if (lean_is_scalar(x_146)) { - x_147 = lean_alloc_ctor(1, 2, 0); -} else { - x_147 = x_146; -} -lean_ctor_set(x_147, 0, x_144); -lean_ctor_set(x_147, 1, x_145); -return x_147; -} -} -} -else -{ -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; uint8_t x_155; uint8_t x_156; uint8_t x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; -x_148 = lean_ctor_get(x_21, 0); -x_149 = lean_ctor_get(x_21, 1); -lean_inc(x_149); -lean_inc(x_148); -lean_dec(x_21); -x_150 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_6, x_149); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_150, 1); -lean_inc(x_152); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - lean_ctor_release(x_150, 1); - x_153 = x_150; -} else { - lean_dec_ref(x_150); - x_153 = lean_box(0); -} -x_154 = lean_unsigned_to_nat(2u); -x_155 = 0; -x_156 = 1; -x_157 = 0; -x_158 = lean_alloc_ctor(0, 2, 19); -lean_ctor_set(x_158, 0, x_1); -lean_ctor_set(x_158, 1, x_154); -lean_ctor_set_uint8(x_158, sizeof(void*)*2, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 1, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 2, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 3, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 4, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 5, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 6, x_157); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 7, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 8, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 9, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 10, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 11, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 12, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 13, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 14, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 15, x_155); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 16, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 17, x_156); -lean_ctor_set_uint8(x_158, sizeof(void*)*2 + 18, x_156); -x_159 = lean_box(0); -if (lean_is_scalar(x_153)) { - x_160 = lean_alloc_ctor(1, 2, 0); -} else { - x_160 = x_153; - lean_ctor_set_tag(x_160, 1); -} -lean_ctor_set(x_160, 0, x_19); -lean_ctor_set(x_160, 1, x_159); -x_161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_161, 0, x_10); -lean_ctor_set(x_161, 1, x_160); -x_162 = lean_array_mk(x_161); -x_163 = l_Lean_Meta_Simp_mkContext(x_158, x_162, x_151, x_3, x_4, x_5, x_6, x_152); -x_164 = lean_ctor_get(x_163, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_163, 1); -lean_inc(x_165); -if (lean_is_exclusive(x_163)) { - lean_ctor_release(x_163, 0); - lean_ctor_release(x_163, 1); - x_166 = x_163; -} else { - lean_dec_ref(x_163); - x_166 = lean_box(0); -} -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_167 = l_Lean_MVarId_getNondepPropHyps(x_2, x_3, x_4, x_5, x_6, x_165); -if (lean_obj_tag(x_167) == 0) -{ -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -lean_dec(x_167); -if (lean_is_scalar(x_166)) { - x_170 = lean_alloc_ctor(1, 2, 0); -} else { - x_170 = x_166; - lean_ctor_set_tag(x_170, 1); -} -lean_ctor_set(x_170, 0, x_148); -lean_ctor_set(x_170, 1, x_159); -lean_ctor_set_tag(x_17, 1); -lean_ctor_set(x_17, 1, x_170); -lean_ctor_set(x_17, 0, x_14); -x_171 = lean_array_mk(x_17); -x_172 = lean_box(0); -x_173 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_174 = l_Lean_Meta_simpGoal(x_2, x_164, x_171, x_172, x_156, x_168, x_173, x_3, x_4, x_5, x_6, x_169); -if (lean_obj_tag(x_174) == 0) -{ -lean_object* x_175; lean_object* x_176; -x_175 = lean_ctor_get(x_174, 0); -lean_inc(x_175); -x_176 = lean_ctor_get(x_175, 0); -lean_inc(x_176); -lean_dec(x_175); -if (lean_obj_tag(x_176) == 0) -{ -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_174, 1); -lean_inc(x_177); -if (lean_is_exclusive(x_174)) { - lean_ctor_release(x_174, 0); - lean_ctor_release(x_174, 1); - x_178 = x_174; -} else { - lean_dec_ref(x_174); - x_178 = lean_box(0); -} -if (lean_is_scalar(x_178)) { - x_179 = lean_alloc_ctor(0, 2, 0); -} else { - x_179 = x_178; -} -lean_ctor_set(x_179, 0, x_172); -lean_ctor_set(x_179, 1, x_177); -return x_179; -} -else -{ -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; -x_180 = lean_ctor_get(x_176, 0); -lean_inc(x_180); -if (lean_is_exclusive(x_176)) { - lean_ctor_release(x_176, 0); - x_181 = x_176; -} else { - lean_dec_ref(x_176); - x_181 = lean_box(0); -} -x_182 = lean_ctor_get(x_174, 1); -lean_inc(x_182); -if (lean_is_exclusive(x_174)) { - lean_ctor_release(x_174, 0); - lean_ctor_release(x_174, 1); - x_183 = x_174; -} else { - lean_dec_ref(x_174); - x_183 = lean_box(0); -} -x_184 = lean_ctor_get(x_180, 1); -lean_inc(x_184); -lean_dec(x_180); -if (lean_is_scalar(x_181)) { - x_185 = lean_alloc_ctor(1, 1, 0); -} else { - x_185 = x_181; -} -lean_ctor_set(x_185, 0, x_184); -if (lean_is_scalar(x_183)) { - x_186 = lean_alloc_ctor(0, 2, 0); -} else { - x_186 = x_183; -} -lean_ctor_set(x_186, 0, x_185); -lean_ctor_set(x_186, 1, x_182); -return x_186; -} -} -else -{ -lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; -x_187 = lean_ctor_get(x_174, 0); -lean_inc(x_187); -x_188 = lean_ctor_get(x_174, 1); -lean_inc(x_188); -if (lean_is_exclusive(x_174)) { - lean_ctor_release(x_174, 0); - lean_ctor_release(x_174, 1); - x_189 = x_174; -} else { - lean_dec_ref(x_174); - x_189 = lean_box(0); -} -if (lean_is_scalar(x_189)) { - x_190 = lean_alloc_ctor(1, 2, 0); -} else { - x_190 = x_189; -} -lean_ctor_set(x_190, 0, x_187); -lean_ctor_set(x_190, 1, x_188); -return x_190; -} -} -else -{ -lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; -lean_dec(x_166); -lean_dec(x_164); -lean_dec(x_148); -lean_free_object(x_17); -lean_dec(x_14); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_191 = lean_ctor_get(x_167, 0); -lean_inc(x_191); -x_192 = lean_ctor_get(x_167, 1); -lean_inc(x_192); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_193 = x_167; -} else { - lean_dec_ref(x_167); - x_193 = lean_box(0); -} -if (lean_is_scalar(x_193)) { - x_194 = lean_alloc_ctor(1, 2, 0); -} else { - x_194 = x_193; -} -lean_ctor_set(x_194, 0, x_191); -lean_ctor_set(x_194, 1, x_192); -return x_194; -} -} -} -else -{ -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; uint8_t x_207; uint8_t x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; -x_195 = lean_ctor_get(x_17, 0); -x_196 = lean_ctor_get(x_17, 1); -lean_inc(x_196); -lean_inc(x_195); -lean_dec(x_17); -x_197 = l_Lean_Meta_Simp_getSEvalSimprocs___rarg(x_6, x_196); -x_198 = lean_ctor_get(x_197, 0); -lean_inc(x_198); -x_199 = lean_ctor_get(x_197, 1); -lean_inc(x_199); -if (lean_is_exclusive(x_197)) { - lean_ctor_release(x_197, 0); - lean_ctor_release(x_197, 1); - x_200 = x_197; -} else { - lean_dec_ref(x_197); - x_200 = lean_box(0); -} -x_201 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_6, x_199); -x_202 = lean_ctor_get(x_201, 0); -lean_inc(x_202); -x_203 = lean_ctor_get(x_201, 1); -lean_inc(x_203); -if (lean_is_exclusive(x_201)) { - lean_ctor_release(x_201, 0); - lean_ctor_release(x_201, 1); - x_204 = x_201; -} else { - lean_dec_ref(x_201); - x_204 = lean_box(0); -} -x_205 = lean_unsigned_to_nat(2u); -x_206 = 0; -x_207 = 1; -x_208 = 0; -x_209 = lean_alloc_ctor(0, 2, 19); -lean_ctor_set(x_209, 0, x_1); -lean_ctor_set(x_209, 1, x_205); -lean_ctor_set_uint8(x_209, sizeof(void*)*2, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 1, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 2, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 3, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 4, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 5, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 6, x_208); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 7, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 8, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 9, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 10, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 11, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 12, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 13, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 14, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 15, x_206); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 16, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 17, x_207); -lean_ctor_set_uint8(x_209, sizeof(void*)*2 + 18, x_207); -x_210 = lean_box(0); -if (lean_is_scalar(x_204)) { - x_211 = lean_alloc_ctor(1, 2, 0); -} else { - x_211 = x_204; - lean_ctor_set_tag(x_211, 1); -} -lean_ctor_set(x_211, 0, x_195); -lean_ctor_set(x_211, 1, x_210); -if (lean_is_scalar(x_200)) { - x_212 = lean_alloc_ctor(1, 2, 0); -} else { - x_212 = x_200; - lean_ctor_set_tag(x_212, 1); -} -lean_ctor_set(x_212, 0, x_10); -lean_ctor_set(x_212, 1, x_211); -x_213 = lean_array_mk(x_212); -x_214 = l_Lean_Meta_Simp_mkContext(x_209, x_213, x_202, x_3, x_4, x_5, x_6, x_203); -x_215 = lean_ctor_get(x_214, 0); -lean_inc(x_215); -x_216 = lean_ctor_get(x_214, 1); -lean_inc(x_216); -if (lean_is_exclusive(x_214)) { - lean_ctor_release(x_214, 0); - lean_ctor_release(x_214, 1); - x_217 = x_214; -} else { - lean_dec_ref(x_214); - x_217 = lean_box(0); -} -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_218 = l_Lean_MVarId_getNondepPropHyps(x_2, x_3, x_4, x_5, x_6, x_216); -if (lean_obj_tag(x_218) == 0) -{ -lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_219 = lean_ctor_get(x_218, 0); -lean_inc(x_219); -x_220 = lean_ctor_get(x_218, 1); -lean_inc(x_220); -lean_dec(x_218); -if (lean_is_scalar(x_217)) { - x_221 = lean_alloc_ctor(1, 2, 0); -} else { - x_221 = x_217; - lean_ctor_set_tag(x_221, 1); -} -lean_ctor_set(x_221, 0, x_198); -lean_ctor_set(x_221, 1, x_210); -x_222 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_222, 0, x_14); -lean_ctor_set(x_222, 1, x_221); -x_223 = lean_array_mk(x_222); -x_224 = lean_box(0); -x_225 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_226 = l_Lean_Meta_simpGoal(x_2, x_215, x_223, x_224, x_207, x_219, x_225, x_3, x_4, x_5, x_6, x_220); -if (lean_obj_tag(x_226) == 0) -{ -lean_object* x_227; lean_object* x_228; -x_227 = lean_ctor_get(x_226, 0); -lean_inc(x_227); -x_228 = lean_ctor_get(x_227, 0); -lean_inc(x_228); -lean_dec(x_227); -if (lean_obj_tag(x_228) == 0) -{ -lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_229 = lean_ctor_get(x_226, 1); -lean_inc(x_229); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_230 = x_226; -} else { - lean_dec_ref(x_226); - x_230 = lean_box(0); -} -if (lean_is_scalar(x_230)) { - x_231 = lean_alloc_ctor(0, 2, 0); -} else { - x_231 = x_230; -} -lean_ctor_set(x_231, 0, x_224); -lean_ctor_set(x_231, 1, x_229); -return x_231; -} -else -{ -lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; -x_232 = lean_ctor_get(x_228, 0); -lean_inc(x_232); -if (lean_is_exclusive(x_228)) { - lean_ctor_release(x_228, 0); - x_233 = x_228; -} else { - lean_dec_ref(x_228); - x_233 = lean_box(0); -} -x_234 = lean_ctor_get(x_226, 1); -lean_inc(x_234); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_235 = x_226; -} else { - lean_dec_ref(x_226); - x_235 = lean_box(0); -} -x_236 = lean_ctor_get(x_232, 1); -lean_inc(x_236); -lean_dec(x_232); -if (lean_is_scalar(x_233)) { - x_237 = lean_alloc_ctor(1, 1, 0); -} else { - x_237 = x_233; -} -lean_ctor_set(x_237, 0, x_236); -if (lean_is_scalar(x_235)) { - x_238 = lean_alloc_ctor(0, 2, 0); -} else { - x_238 = x_235; -} -lean_ctor_set(x_238, 0, x_237); -lean_ctor_set(x_238, 1, x_234); -return x_238; -} -} -else -{ -lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; -x_239 = lean_ctor_get(x_226, 0); -lean_inc(x_239); -x_240 = lean_ctor_get(x_226, 1); -lean_inc(x_240); -if (lean_is_exclusive(x_226)) { - lean_ctor_release(x_226, 0); - lean_ctor_release(x_226, 1); - x_241 = x_226; -} else { - lean_dec_ref(x_226); - x_241 = lean_box(0); -} -if (lean_is_scalar(x_241)) { - x_242 = lean_alloc_ctor(1, 2, 0); -} else { - x_242 = x_241; -} -lean_ctor_set(x_242, 0, x_239); -lean_ctor_set(x_242, 1, x_240); -return x_242; -} -} -else -{ -lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; -lean_dec(x_217); -lean_dec(x_215); -lean_dec(x_198); -lean_dec(x_14); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_243 = lean_ctor_get(x_218, 0); -lean_inc(x_243); -x_244 = lean_ctor_get(x_218, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_245 = x_218; -} else { - lean_dec_ref(x_218); - x_245 = lean_box(0); -} -if (lean_is_scalar(x_245)) { - x_246 = lean_alloc_ctor(1, 2, 0); -} else { - x_246 = x_245; -} -lean_ctor_set(x_246, 0, x_243); -lean_ctor_set(x_246, 1, x_244); -return x_246; -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("rewriteRules", 12, 12); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1), 7, 1); -lean_closure_set(x_2, 0, x_1); -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2; -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); -lean_ctor_set(x_4, 1, x_2); -return x_4; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1; -x_3 = l_Lean_Expr_const___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("and_left", 8, 8); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("and_right", 9, 9); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6; -x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); -return x_7; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2; -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; -lean_inc(x_2); -x_14 = l_Lean_mkApp3(x_11, x_12, x_2, x_13); -x_15 = lean_ctor_get(x_1, 2); -lean_inc(x_15); -lean_dec(x_1); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5; -lean_inc(x_15); -lean_inc(x_3); -lean_inc(x_2); -x_17 = l_Lean_mkApp3(x_16, x_2, x_3, x_15); -x_18 = 0; -x_19 = 0; -lean_inc(x_10); -x_20 = lean_alloc_ctor(0, 3, 2); -lean_ctor_set(x_20, 0, x_10); -lean_ctor_set(x_20, 1, x_14); -lean_ctor_set(x_20, 2, x_17); -lean_ctor_set_uint8(x_20, sizeof(void*)*3, x_18); -lean_ctor_set_uint8(x_20, sizeof(void*)*3 + 1, x_19); -lean_inc(x_3); -x_21 = l_Lean_mkApp3(x_11, x_12, x_3, x_13); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8; -x_23 = l_Lean_mkApp3(x_22, x_2, x_3, x_15); -x_24 = lean_alloc_ctor(0, 3, 2); -lean_ctor_set(x_24, 0, x_10); -lean_ctor_set(x_24, 1, x_21); -lean_ctor_set(x_24, 2, x_23); -lean_ctor_set_uint8(x_24, sizeof(void*)*3, x_18); -lean_ctor_set_uint8(x_24, sizeof(void*)*3 + 1, x_19); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_20); -lean_ctor_set(x_25, 1, x_24); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_9); -return x_27; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_8, 0, x_7); -lean_ctor_set(x_8, 1, x_6); -return x_8; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2___boxed), 6, 0); -return x_1; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; -x_14 = l_Lean_Expr_isConstOf(x_12, x_13); -lean_dec(x_12); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_15 = lean_box(0); -x_16 = lean_apply_6(x_11, x_15, x_6, x_7, x_8, x_9, x_10); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_box(0); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1(x_2, x_3, x_4, x_17, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_18; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1; -x_12 = l_Lean_Expr_cleanupAnnotations(x_1); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_14 = l_Lean_Expr_isConstOf(x_12, x_13); -lean_dec(x_12); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_15 = lean_box(0); -x_16 = lean_apply_6(x_11, x_15, x_6, x_7, x_8, x_9, x_10); -return x_16; -} -else -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_box(0); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3(x_2, x_3, x_4, x_5, x_17, x_6, x_7, x_8, x_9, x_10); -return x_18; -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("and", 3, 3); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1; -x_11 = l_Lean_Expr_cleanupAnnotations(x_3); -x_12 = l_Lean_Expr_isApp(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; -lean_dec(x_11); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_13 = lean_box(0); -x_14 = lean_apply_6(x_10, x_13, x_5, x_6, x_7, x_8, x_9); -return x_14; -} -else -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_15 = l_Lean_Expr_appArg(x_11, lean_box(0)); -x_16 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); -x_17 = l_Lean_Expr_isApp(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_18 = lean_box(0); -x_19 = lean_apply_6(x_10, x_18, x_5, x_6, x_7, x_8, x_9); -return x_19; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = l_Lean_Expr_appArg(x_16, lean_box(0)); -x_21 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); -x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2; -x_23 = l_Lean_Expr_isConstOf(x_21, x_22); -lean_dec(x_21); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -lean_dec(x_20); -lean_dec(x_15); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_24 = lean_box(0); -x_25 = lean_apply_6(x_10, x_24, x_5, x_6, x_7, x_8, x_9); -return x_25; -} -else -{ -lean_object* x_26; -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__4(x_4, x_2, x_1, x_20, x_15, x_5, x_6, x_7, x_8, x_9); -return x_26; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_7 = lean_ctor_get(x_1, 1); -lean_inc(x_7); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1; -x_9 = l_Lean_Expr_cleanupAnnotations(x_7); -x_10 = l_Lean_Expr_isApp(x_9); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; -lean_dec(x_9); -lean_dec(x_1); -x_11 = lean_box(0); -x_12 = lean_apply_6(x_8, x_11, x_2, x_3, x_4, x_5, x_6); -return x_12; -} -else -{ -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Expr_appArg(x_9, lean_box(0)); -x_14 = l_Lean_Expr_appFnCleanup(x_9, lean_box(0)); -x_15 = l_Lean_Expr_isApp(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_1); -x_16 = lean_box(0); -x_17 = lean_apply_6(x_8, x_16, x_2, x_3, x_4, x_5, x_6); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = l_Lean_Expr_appArg(x_14, lean_box(0)); -x_19 = l_Lean_Expr_appFnCleanup(x_14, lean_box(0)); -x_20 = l_Lean_Expr_isApp(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_13); -lean_dec(x_1); -x_21 = lean_box(0); -x_22 = lean_apply_6(x_8, x_21, x_2, x_3, x_4, x_5, x_6); -return x_22; -} -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = l_Lean_Expr_appArg(x_19, lean_box(0)); -x_24 = l_Lean_Expr_appFnCleanup(x_19, lean_box(0)); -x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_26 = l_Lean_Expr_isConstOf(x_24, x_25); -lean_dec(x_24); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; -lean_dec(x_23); -lean_dec(x_18); -lean_dec(x_13); -lean_dec(x_1); -x_27 = lean_box(0); -x_28 = lean_apply_6(x_8, x_27, x_2, x_3, x_4, x_5, x_6); -return x_28; -} -else -{ -lean_object* x_29; -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5(x_1, x_23, x_18, x_13, x_2, x_3, x_4, x_5, x_6); -return x_29; -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_5); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit(x_1, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -if (x_3 == 0) -{ -uint8_t x_11; -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_9, 0); -lean_dec(x_12); -x_13 = lean_array_push(x_2, x_1); -lean_ctor_set(x_9, 0, x_13); -return x_9; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_9, 1); -lean_inc(x_14); -lean_dec(x_9); -x_15 = lean_array_push(x_2, x_1); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_15); -lean_ctor_set(x_16, 1, x_14); -return x_16; -} -} -else -{ -uint8_t x_17; -lean_dec(x_1); -x_17 = !lean_is_exclusive(x_9); -if (x_17 == 0) -{ -lean_object* x_18; -x_18 = lean_ctor_get(x_9, 0); -lean_dec(x_18); -lean_ctor_set(x_9, 0, x_2); -return x_9; -} -else -{ -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_9, 1); -lean_inc(x_19); -lean_dec(x_9); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_2); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -} -else -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; -lean_dec(x_1); -x_21 = lean_ctor_get(x_10, 0); -lean_inc(x_21); -lean_dec(x_10); -x_22 = lean_ctor_get(x_9, 1); -lean_inc(x_22); -lean_dec(x_9); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -x_25 = 0; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_26 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(x_23, x_2, x_25, x_4, x_5, x_6, x_7, x_22); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_1 = x_24; -x_2 = x_27; -x_3 = x_25; -x_8 = x_28; -goto _start; -} -else -{ -uint8_t x_30; -lean_dec(x_24); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) -{ -return x_26; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; -} -} -} -} -else -{ -uint8_t x_34; -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_9); -if (x_34 == 0) -{ -return x_9; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_9, 0); -x_36 = lean_ctor_get(x_9, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_9); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -uint8_t x_9; lean_object* x_10; -x_9 = lean_unbox(x_3); -lean_dec(x_3); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_5, x_4); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_6); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -else -{ -lean_object* x_14; uint8_t x_15; -x_14 = lean_array_uget(x_3, x_5); -x_15 = !lean_is_exclusive(x_6); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_6, 0); -x_17 = lean_ctor_get(x_6, 1); -lean_inc(x_7); -lean_inc(x_14); -x_18 = l_Lean_FVarId_getDecl(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_7); -lean_inc(x_14); -x_21 = l_Lean_FVarId_getType(x_14, x_7, x_8, x_9, x_10, x_20); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = l_Lean_LocalDecl_userName(x_19); -lean_dec(x_19); -lean_inc(x_14); -x_25 = l_Lean_Expr_fvar___override(x_14); -x_26 = 0; -x_27 = 0; -x_28 = lean_alloc_ctor(0, 3, 2); -lean_ctor_set(x_28, 0, x_24); -lean_ctor_set(x_28, 1, x_22); -lean_ctor_set(x_28, 2, x_25); -lean_ctor_set_uint8(x_28, sizeof(void*)*3, x_26); -lean_ctor_set_uint8(x_28, sizeof(void*)*3 + 1, x_27); -x_29 = lean_array_get_size(x_16); -x_30 = 1; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(x_28, x_16, x_30, x_7, x_8, x_9, x_10, x_23); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = lean_array_get_size(x_32); -x_35 = lean_nat_dec_lt(x_29, x_34); -lean_dec(x_34); -lean_dec(x_29); -if (x_35 == 0) -{ -size_t x_36; size_t x_37; -lean_dec(x_14); -lean_ctor_set(x_6, 0, x_32); -x_36 = 1; -x_37 = lean_usize_add(x_5, x_36); -x_5 = x_37; -x_11 = x_33; -goto _start; -} -else -{ -lean_object* x_39; size_t x_40; size_t x_41; -x_39 = lean_array_push(x_17, x_14); -lean_ctor_set(x_6, 1, x_39); -lean_ctor_set(x_6, 0, x_32); -x_40 = 1; -x_41 = lean_usize_add(x_5, x_40); -x_5 = x_41; -x_11 = x_33; -goto _start; -} -} -else -{ -uint8_t x_43; -lean_dec(x_29); -lean_free_object(x_6); -lean_dec(x_17); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_43 = !lean_is_exclusive(x_31); -if (x_43 == 0) -{ -return x_31; -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_31, 0); -x_45 = lean_ctor_get(x_31, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_31); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; -} -} -} -else -{ -uint8_t x_47; -lean_dec(x_19); -lean_free_object(x_6); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_47 = !lean_is_exclusive(x_21); -if (x_47 == 0) -{ -return x_21; -} -else -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_21, 0); -x_49 = lean_ctor_get(x_21, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_21); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; -} -} -} -else -{ -uint8_t x_51; -lean_free_object(x_6); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_51 = !lean_is_exclusive(x_18); -if (x_51 == 0) -{ -return x_18; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_18, 0); -x_53 = lean_ctor_get(x_18, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_18); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; -} -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_6, 0); -x_56 = lean_ctor_get(x_6, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_6); -lean_inc(x_7); -lean_inc(x_14); -x_57 = l_Lean_FVarId_getDecl(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -lean_inc(x_7); -lean_inc(x_14); -x_60 = l_Lean_FVarId_getType(x_14, x_7, x_8, x_9, x_10, x_59); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_63 = l_Lean_LocalDecl_userName(x_58); -lean_dec(x_58); -lean_inc(x_14); -x_64 = l_Lean_Expr_fvar___override(x_14); -x_65 = 0; -x_66 = 0; -x_67 = lean_alloc_ctor(0, 3, 2); -lean_ctor_set(x_67, 0, x_63); -lean_ctor_set(x_67, 1, x_61); -lean_ctor_set(x_67, 2, x_64); -lean_ctor_set_uint8(x_67, sizeof(void*)*3, x_65); -lean_ctor_set_uint8(x_67, sizeof(void*)*3 + 1, x_66); -x_68 = lean_array_get_size(x_55); -x_69 = 1; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_70 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_splitAnds(x_67, x_55, x_69, x_7, x_8, x_9, x_10, x_62); -if (lean_obj_tag(x_70) == 0) -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; -x_71 = lean_ctor_get(x_70, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_70, 1); -lean_inc(x_72); -lean_dec(x_70); -x_73 = lean_array_get_size(x_71); -x_74 = lean_nat_dec_lt(x_68, x_73); -lean_dec(x_73); -lean_dec(x_68); -if (x_74 == 0) -{ -lean_object* x_75; size_t x_76; size_t x_77; -lean_dec(x_14); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_71); -lean_ctor_set(x_75, 1, x_56); -x_76 = 1; -x_77 = lean_usize_add(x_5, x_76); -x_5 = x_77; -x_6 = x_75; -x_11 = x_72; -goto _start; -} -else -{ -lean_object* x_79; lean_object* x_80; size_t x_81; size_t x_82; -x_79 = lean_array_push(x_56, x_14); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_71); -lean_ctor_set(x_80, 1, x_79); -x_81 = 1; -x_82 = lean_usize_add(x_5, x_81); -x_5 = x_82; -x_6 = x_80; -x_11 = x_72; -goto _start; -} -} -else -{ -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -lean_dec(x_68); -lean_dec(x_56); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_84 = lean_ctor_get(x_70, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_70, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_86 = x_70; -} else { - lean_dec_ref(x_70); - x_86 = lean_box(0); -} -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); -} else { - x_87 = x_86; -} -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; -} -} -else -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_58); -lean_dec(x_56); -lean_dec(x_55); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_88 = lean_ctor_get(x_60, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_60, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_90 = x_60; -} else { - lean_dec_ref(x_60); - x_90 = lean_box(0); -} -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 2, 0); -} else { - x_91 = x_90; -} -lean_ctor_set(x_91, 0, x_88); -lean_ctor_set(x_91, 1, x_89); -return x_91; -} -} -else -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -lean_dec(x_56); -lean_dec(x_55); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_92 = lean_ctor_get(x_57, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_57, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_94 = x_57; -} else { - lean_dec_ref(x_57); - x_94 = lean_box(0); -} -if (lean_is_scalar(x_94)) { - x_95 = lean_alloc_ctor(1, 2, 0); -} else { - x_95 = x_94; -} -lean_ctor_set(x_95, 0, x_92); -lean_ctor_set(x_95, 1, x_93); -return x_95; -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1; -x_2 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_7 = l_Lean_MVarId_getNondepPropHyps(x_1, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_7) == 0) -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_box(0); -x_11 = lean_array_size(x_8); -x_12 = 0; -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1(x_8, x_10, x_8, x_11, x_12, x_13, x_2, x_3, x_4, x_5, x_9); -lean_dec(x_8); -if (lean_obj_tag(x_14) == 0) -{ -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_16, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_dec(x_16); -x_20 = lean_array_get_size(x_18); -x_21 = lean_unsigned_to_nat(0u); -x_22 = lean_nat_dec_eq(x_20, x_21); -lean_dec(x_20); -if (x_22 == 0) -{ -lean_object* x_23; -lean_free_object(x_14); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_23 = l_Lean_MVarId_assertHypotheses(x_1, x_18, x_2, x_3, x_4, x_5, x_17); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l_Lean_MVarId_tryClearMany(x_26, x_19, x_2, x_3, x_4, x_5, x_25); -lean_dec(x_19); -if (lean_obj_tag(x_27) == 0) -{ -uint8_t x_28; -x_28 = !lean_is_exclusive(x_27); -if (x_28 == 0) -{ -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_27, 0); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_27, 0, x_30); -return x_27; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_31 = lean_ctor_get(x_27, 0); -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_27); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_31); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -return x_34; -} -} -else -{ -uint8_t x_35; -x_35 = !lean_is_exclusive(x_27); -if (x_35 == 0) -{ -return x_27; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_27, 0); -x_37 = lean_ctor_get(x_27, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_27); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -} -else -{ -uint8_t x_39; -lean_dec(x_19); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_39 = !lean_is_exclusive(x_23); -if (x_39 == 0) -{ -return x_23; -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_23, 0); -x_41 = lean_ctor_get(x_23, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_23); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; -} -} -} -else -{ -lean_object* x_43; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_43 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_43, 0, x_1); -lean_ctor_set(x_14, 0, x_43); -return x_14; -} -} -else -{ -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_44 = lean_ctor_get(x_14, 0); -x_45 = lean_ctor_get(x_14, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_14); -x_46 = lean_ctor_get(x_44, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_44, 1); -lean_inc(x_47); -lean_dec(x_44); -x_48 = lean_array_get_size(x_46); -x_49 = lean_unsigned_to_nat(0u); -x_50 = lean_nat_dec_eq(x_48, x_49); -lean_dec(x_48); -if (x_50 == 0) -{ -lean_object* x_51; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_51 = l_Lean_MVarId_assertHypotheses(x_1, x_46, x_2, x_3, x_4, x_5, x_45); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = l_Lean_MVarId_tryClearMany(x_54, x_47, x_2, x_3, x_4, x_5, x_53); -lean_dec(x_47); -if (lean_obj_tag(x_55) == 0) -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_58 = x_55; -} else { - lean_dec_ref(x_55); - x_58 = lean_box(0); -} -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_56); -if (lean_is_scalar(x_58)) { - x_60 = lean_alloc_ctor(0, 2, 0); -} else { - x_60 = x_58; -} -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_57); -return x_60; -} -else -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_61 = lean_ctor_get(x_55, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_55, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_55)) { - lean_ctor_release(x_55, 0); - lean_ctor_release(x_55, 1); - x_63 = x_55; -} else { - lean_dec_ref(x_55); - x_63 = lean_box(0); -} -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; -} -} -else -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -lean_dec(x_47); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_65 = lean_ctor_get(x_51, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_51, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_67 = x_51; -} else { - lean_dec_ref(x_51); - x_67 = lean_box(0); -} -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; -} -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; -} -} -else -{ -lean_object* x_69; lean_object* x_70; -lean_dec(x_47); -lean_dec(x_46); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_69 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_69, 0, x_1); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_45); -return x_70; -} -} -} -else -{ -uint8_t x_71; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_71 = !lean_is_exclusive(x_14); -if (x_71 == 0) -{ -return x_14; -} -else -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_14, 0); -x_73 = lean_ctor_get(x_14, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_14); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; -} -} -} -else -{ -uint8_t x_75; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_75 = !lean_is_exclusive(x_7); -if (x_75 == 0) -{ -return x_7; -} -else -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_7, 0); -x_77 = lean_ctor_get(x_7, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_7); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; -lean_inc(x_1); -x_7 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1), 6, 1); -lean_closure_set(x_7, 0, x_1); -x_8 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_1, x_7, x_2, x_3, x_4, x_5, x_6); -return x_8; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("andFlattening", 13, 13); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1), 6, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___spec__1(x_1, x_2, x_3, x_12, x_13, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint64_t x_43; uint64_t x_44; uint64_t x_45; uint64_t x_46; uint64_t x_47; uint64_t x_48; uint64_t x_49; size_t x_50; size_t x_51; size_t x_52; size_t x_53; size_t x_54; lean_object* x_55; uint8_t x_56; -x_40 = lean_ctor_get(x_4, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_4, 1); -lean_inc(x_41); -x_42 = lean_array_get_size(x_41); -x_43 = l_Lean_Expr_hash(x_5); -x_44 = 32; -x_45 = lean_uint64_shift_right(x_43, x_44); -x_46 = lean_uint64_xor(x_43, x_45); -x_47 = 16; -x_48 = lean_uint64_shift_right(x_46, x_47); -x_49 = lean_uint64_xor(x_46, x_48); -x_50 = lean_uint64_to_usize(x_49); -x_51 = lean_usize_of_nat(x_42); -lean_dec(x_42); -x_52 = 1; -x_53 = lean_usize_sub(x_51, x_52); -x_54 = lean_usize_land(x_50, x_53); -x_55 = lean_array_uget(x_41, x_54); -x_56 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_5, x_55); -if (x_56 == 0) -{ -uint8_t x_57; -x_57 = !lean_is_exclusive(x_4); -if (x_57 == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_58 = lean_ctor_get(x_4, 1); -lean_dec(x_58); -x_59 = lean_ctor_get(x_4, 0); -lean_dec(x_59); -x_60 = lean_unsigned_to_nat(1u); -x_61 = lean_nat_add(x_40, x_60); -lean_dec(x_40); -x_62 = lean_box(0); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_5); -lean_ctor_set(x_63, 1, x_62); -lean_ctor_set(x_63, 2, x_55); -x_64 = lean_array_uset(x_41, x_54, x_63); -x_65 = lean_unsigned_to_nat(4u); -x_66 = lean_nat_mul(x_61, x_65); -x_67 = lean_unsigned_to_nat(3u); -x_68 = lean_nat_div(x_66, x_67); -lean_dec(x_66); -x_69 = lean_array_get_size(x_64); -x_70 = lean_nat_dec_le(x_68, x_69); -lean_dec(x_69); -lean_dec(x_68); -if (x_70 == 0) -{ -lean_object* x_71; -x_71 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_64); -lean_ctor_set(x_4, 1, x_71); -lean_ctor_set(x_4, 0, x_61); -x_12 = x_4; -goto block_39; -} -else -{ -lean_ctor_set(x_4, 1, x_64); -lean_ctor_set(x_4, 0, x_61); -x_12 = x_4; -goto block_39; -} -} -else -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; uint8_t x_82; -lean_dec(x_4); -x_72 = lean_unsigned_to_nat(1u); -x_73 = lean_nat_add(x_40, x_72); -lean_dec(x_40); -x_74 = lean_box(0); -x_75 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_75, 0, x_5); -lean_ctor_set(x_75, 1, x_74); -lean_ctor_set(x_75, 2, x_55); -x_76 = lean_array_uset(x_41, x_54, x_75); -x_77 = lean_unsigned_to_nat(4u); -x_78 = lean_nat_mul(x_73, x_77); -x_79 = lean_unsigned_to_nat(3u); -x_80 = lean_nat_div(x_78, x_79); -lean_dec(x_78); -x_81 = lean_array_get_size(x_76); -x_82 = lean_nat_dec_le(x_80, x_81); -lean_dec(x_81); -lean_dec(x_80); -if (x_82 == 0) -{ -lean_object* x_83; lean_object* x_84; -x_83 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_76); -x_84 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_84, 0, x_73); -lean_ctor_set(x_84, 1, x_83); -x_12 = x_84; -goto block_39; -} -else -{ -lean_object* x_85; -x_85 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_85, 0, x_73); -lean_ctor_set(x_85, 1, x_76); -x_12 = x_85; -goto block_39; -} -} -} -else -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -lean_dec(x_55); -lean_dec(x_41); -lean_dec(x_40); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_5); -x_86 = lean_array_push(x_3, x_1); -x_87 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_87, 0, x_2); -lean_ctor_set(x_87, 1, x_4); -x_88 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -x_89 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_89, 0, x_88); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_11); -return x_90; -} -block_39: -{ -lean_object* x_13; -lean_inc(x_7); -lean_inc(x_1); -x_13 = l_Lean_FVarId_getDecl(x_1, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_LocalDecl_toExpr(x_14); -lean_dec(x_14); -x_17 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_17, 0, x_1); -x_18 = l_Lean_Meta_simpGlobalConfig; -x_19 = l_Lean_Meta_SimpTheoremsArray_addTheorem(x_2, x_17, x_16, x_18, x_7, x_8, x_9, x_10, x_15); -if (lean_obj_tag(x_19) == 0) -{ -uint8_t x_20; -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_12); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_3); -lean_ctor_set(x_23, 1, x_22); -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_19, 0, x_24); -return x_19; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_25 = lean_ctor_get(x_19, 0); -x_26 = lean_ctor_get(x_19, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_19); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_12); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_3); -lean_ctor_set(x_28, 1, x_27); -x_29 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_29, 0, x_28); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_26); -return x_30; -} -} -else -{ -uint8_t x_31; -lean_dec(x_12); -lean_dec(x_3); -x_31 = !lean_is_exclusive(x_19); -if (x_31 == 0) -{ -return x_19; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_19, 0); -x_33 = lean_ctor_get(x_19, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_19); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} -} -} -else -{ -uint8_t x_35; -lean_dec(x_12); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_35 = !lean_is_exclusive(x_13); -if (x_35 == 0) -{ -return x_13; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_13, 0); -x_37 = lean_ctor_get(x_13, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_13); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_1); -lean_ctor_set(x_10, 1, x_2); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_3); -lean_ctor_set(x_11, 1, x_10); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_9); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Expr_cleanupAnnotations(x_1); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; -x_15 = l_Lean_Expr_isConstOf(x_13, x_14); -lean_dec(x_13); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_6); -lean_dec(x_2); -x_16 = lean_box(0); -x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_3, x_5, x_4, x_16, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1(x_2, x_3, x_4, x_5, x_6, x_18, x_8, x_9, x_10, x_11, x_12); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_13 = l_Lean_Expr_cleanupAnnotations(x_7); -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; -x_15 = l_Lean_Expr_isConstOf(x_13, x_14); -lean_dec(x_13); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_16 = lean_box(0); -x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_2, x_4, x_3, x_16, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -return x_17; -} -else -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_box(0); -x_19 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3(x_5, x_1, x_2, x_3, x_4, x_6, x_18, x_8, x_9, x_10, x_11, x_12); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -uint8_t x_12; -x_12 = lean_usize_dec_lt(x_5, x_4); -if (x_12 == 0) -{ -lean_object* x_13; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_6); -lean_ctor_set(x_13, 1, x_11); -return x_13; -} -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_14 = lean_array_uget(x_3, x_5); -x_24 = lean_ctor_get(x_6, 1); -lean_inc(x_24); -x_25 = lean_ctor_get(x_6, 0); -lean_inc(x_25); -lean_dec(x_6); -x_26 = lean_ctor_get(x_24, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -lean_inc(x_7); -lean_inc(x_14); -x_28 = l_Lean_FVarId_getType(x_14, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_Expr_cleanupAnnotations(x_29); -x_32 = l_Lean_Expr_isApp(x_31); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -lean_dec(x_31); -lean_dec(x_14); -x_33 = lean_box(0); -x_34 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_26, x_27, x_25, x_33, x_7, x_8, x_9, x_10, x_30); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_15 = x_35; -x_16 = x_36; -goto block_23; -} -else -{ -lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = l_Lean_Expr_appArg(x_31, lean_box(0)); -x_38 = l_Lean_Expr_appFnCleanup(x_31, lean_box(0)); -x_39 = l_Lean_Expr_isApp(x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_dec(x_38); -lean_dec(x_37); -lean_dec(x_14); -x_40 = lean_box(0); -x_41 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_26, x_27, x_25, x_40, x_7, x_8, x_9, x_10, x_30); -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); -x_15 = x_42; -x_16 = x_43; -goto block_23; -} -else -{ -lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_44 = l_Lean_Expr_appArg(x_38, lean_box(0)); -x_45 = l_Lean_Expr_appFnCleanup(x_38, lean_box(0)); -x_46 = l_Lean_Expr_isApp(x_45); -if (x_46 == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -lean_dec(x_45); -lean_dec(x_44); -lean_dec(x_37); -lean_dec(x_14); -x_47 = lean_box(0); -x_48 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_26, x_27, x_25, x_47, x_7, x_8, x_9, x_10, x_30); -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -x_15 = x_49; -x_16 = x_50; -goto block_23; -} -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_51 = l_Lean_Expr_appArg(x_45, lean_box(0)); -x_52 = l_Lean_Expr_appFnCleanup(x_45, lean_box(0)); -x_53 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; -x_54 = l_Lean_Expr_isConstOf(x_52, x_53); -lean_dec(x_52); -if (x_54 == 0) -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_51); -lean_dec(x_44); -lean_dec(x_37); -lean_dec(x_14); -x_55 = lean_box(0); -x_56 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_26, x_27, x_25, x_55, x_7, x_8, x_9, x_10, x_30); -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_15 = x_57; -x_16 = x_58; -goto block_23; -} -else -{ -lean_object* x_59; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_59 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__4(x_14, x_26, x_25, x_27, x_51, x_44, x_37, x_7, x_8, x_9, x_10, x_30); -if (lean_obj_tag(x_59) == 0) -{ -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_15 = x_60; -x_16 = x_61; -goto block_23; -} -else -{ -uint8_t x_62; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_62 = !lean_is_exclusive(x_59); -if (x_62 == 0) -{ -return x_59; -} -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_59, 0); -x_64 = lean_ctor_get(x_59, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_59); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; -} -} -} -} -} -} -} -else -{ -uint8_t x_66; -lean_dec(x_27); -lean_dec(x_26); -lean_dec(x_25); -lean_dec(x_14); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_66 = !lean_is_exclusive(x_28); -if (x_66 == 0) -{ -return x_28; -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_28, 0); -x_68 = lean_ctor_get(x_28, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_28); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; -} -} -block_23: -{ -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_17; lean_object* x_18; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_17 = lean_ctor_get(x_15, 0); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; -} -else -{ -lean_object* x_19; size_t x_20; size_t x_21; -x_19 = lean_ctor_get(x_15, 0); -lean_inc(x_19); -lean_dec(x_15); -x_20 = 1; -x_21 = lean_usize_add(x_5, x_20); -x_5 = x_21; -x_6 = x_19; -x_11 = x_16; -goto _start; -} -} -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(10u); -x_2 = lean_unsigned_to_nat(1u); -x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1; -x_3 = lean_mk_array(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_1); -x_8 = l_Lean_MVarId_getNondepPropHyps(x_1, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_8) == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_8, 1); -lean_inc(x_10); -lean_dec(x_8); -x_11 = lean_box(0); -x_12 = lean_array_size(x_9); -x_13 = 0; -x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5; -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1(x_9, x_11, x_9, x_12, x_13, x_14, x_3, x_4, x_5, x_6, x_10); -lean_dec(x_9); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = lean_ctor_get(x_16, 0); -lean_inc(x_19); -lean_dec(x_16); -x_20 = lean_ctor_get(x_17, 0); -lean_inc(x_20); -lean_dec(x_17); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_21 = l_Lean_MVarId_tryClearMany(x_1, x_19, x_3, x_4, x_5, x_6, x_18); -lean_dec(x_19); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_6, x_23); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_unsigned_to_nat(2u); -x_28 = 0; -x_29 = 1; -x_30 = 0; -x_31 = lean_alloc_ctor(0, 2, 19); -lean_ctor_set(x_31, 0, x_2); -lean_ctor_set(x_31, 1, x_27); -lean_ctor_set_uint8(x_31, sizeof(void*)*2, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 1, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 2, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 3, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 4, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 5, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 6, x_30); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 7, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 8, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 9, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 10, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 11, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 12, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 13, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 14, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 15, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 16, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 17, x_29); -lean_ctor_set_uint8(x_31, sizeof(void*)*2 + 18, x_29); -x_32 = l_Lean_Meta_Simp_mkContext(x_31, x_20, x_25, x_3, x_4, x_5, x_6, x_26); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -lean_dec(x_32); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_22); -x_35 = l_Lean_MVarId_getNondepPropHyps(x_22, x_3, x_4, x_5, x_6, x_34); -if (lean_obj_tag(x_35) == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_box(0); -x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1; -x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11; -x_41 = l_Lean_Meta_simpGoal(x_22, x_33, x_39, x_38, x_29, x_36, x_40, x_3, x_4, x_5, x_6, x_37); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -lean_dec(x_42); -if (lean_obj_tag(x_43) == 0) -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_41); -if (x_44 == 0) -{ -lean_object* x_45; -x_45 = lean_ctor_get(x_41, 0); -lean_dec(x_45); -lean_ctor_set(x_41, 0, x_38); -return x_41; -} -else -{ -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_41, 1); -lean_inc(x_46); -lean_dec(x_41); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_38); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -else -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_43); -if (x_48 == 0) -{ -uint8_t x_49; -x_49 = !lean_is_exclusive(x_41); -if (x_49 == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_43, 0); -x_51 = lean_ctor_get(x_41, 0); -lean_dec(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -lean_ctor_set(x_43, 0, x_52); -lean_ctor_set(x_41, 0, x_43); -return x_41; -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_53 = lean_ctor_get(x_43, 0); -x_54 = lean_ctor_get(x_41, 1); -lean_inc(x_54); -lean_dec(x_41); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -lean_ctor_set(x_43, 0, x_55); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_43); -lean_ctor_set(x_56, 1, x_54); -return x_56; -} -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_57 = lean_ctor_get(x_43, 0); -lean_inc(x_57); -lean_dec(x_43); -x_58 = lean_ctor_get(x_41, 1); -lean_inc(x_58); -if (lean_is_exclusive(x_41)) { - lean_ctor_release(x_41, 0); - lean_ctor_release(x_41, 1); - x_59 = x_41; +lean_object* x_368; lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; lean_object* x_374; uint8_t x_375; lean_object* x_376; double x_377; double x_378; lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_382; +x_368 = lean_ctor_get(x_306, 0); +x_369 = lean_ctor_get(x_306, 1); +lean_inc(x_369); +lean_inc(x_368); +lean_dec(x_306); +x_370 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_370, 0, x_368); +x_371 = lean_io_get_num_heartbeats(x_369); +x_372 = lean_ctor_get(x_371, 0); +lean_inc(x_372); +x_373 = lean_ctor_get(x_371, 1); +lean_inc(x_373); +if (lean_is_exclusive(x_371)) { + lean_ctor_release(x_371, 0); + lean_ctor_release(x_371, 1); + x_374 = x_371; } else { - lean_dec_ref(x_41); - x_59 = lean_box(0); + lean_dec_ref(x_371); + x_374 = lean_box(0); } -x_60 = lean_ctor_get(x_57, 1); -lean_inc(x_60); -lean_dec(x_57); -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_60); -if (lean_is_scalar(x_59)) { - x_62 = lean_alloc_ctor(0, 2, 0); +x_375 = 0; +x_376 = lean_unsigned_to_nat(0u); +x_377 = l_Float_ofScientific(x_304, x_375, x_376); +lean_dec(x_304); +x_378 = l_Float_ofScientific(x_372, x_375, x_376); +lean_dec(x_372); +x_379 = lean_box_float(x_377); +x_380 = lean_box_float(x_378); +if (lean_is_scalar(x_374)) { + x_381 = lean_alloc_ctor(0, 2, 0); } else { - x_62 = x_59; -} -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_58); -return x_62; -} -} -} -else -{ -uint8_t x_63; -x_63 = !lean_is_exclusive(x_41); -if (x_63 == 0) -{ -return x_41; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_41, 0); -x_65 = lean_ctor_get(x_41, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_41); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; -} -} -} -else -{ -uint8_t x_67; -lean_dec(x_33); -lean_dec(x_22); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_67 = !lean_is_exclusive(x_35); -if (x_67 == 0) -{ -return x_35; -} -else -{ -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_35, 0); -x_69 = lean_ctor_get(x_35, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_35); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -return x_70; -} -} -} -else -{ -uint8_t x_71; -lean_dec(x_20); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_71 = !lean_is_exclusive(x_21); -if (x_71 == 0) -{ -return x_21; -} -else -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_21, 0); -x_73 = lean_ctor_get(x_21, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_21); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; -} -} -} -else -{ -uint8_t x_75; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_75 = !lean_is_exclusive(x_15); -if (x_75 == 0) -{ -return x_15; -} -else -{ -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_15, 0); -x_77 = lean_ctor_get(x_15, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_15); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -else -{ -uint8_t x_79; -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_79 = !lean_is_exclusive(x_8); -if (x_79 == 0) -{ -return x_8; -} -else -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_8, 0); -x_81 = lean_ctor_get(x_8, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_8); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -return x_82; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; lean_object* x_9; -lean_inc(x_2); -x_8 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1), 7, 2); -lean_closure_set(x_8, 0, x_2); -lean_closure_set(x_8, 1, x_1); -x_9 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_2, x_8, x_3, x_4, x_5, x_6, x_7); -return x_9; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("embeddedConstraintSubsitution", 29, 29); -return x_1; -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass(lean_object* x_1) { -_start: -{ -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1), 7, 1); -lean_closure_set(x_2, 0, x_1); -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2; -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); -lean_ctor_set(x_4, 1, x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -size_t x_12; size_t x_13; lean_object* x_14; -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___spec__1(x_1, x_2, x_3, x_12, x_13, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_14; -} -} -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; -x_13 = lean_usize_dec_lt(x_6, x_5); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_7); -lean_ctor_set(x_14, 1, x_12); -return x_14; -} -else -{ -lean_object* x_15; uint8_t x_16; -x_15 = lean_array_uget(x_4, x_6); -x_16 = !lean_is_exclusive(x_7); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_7, 1); -x_18 = lean_ctor_get(x_7, 0); -lean_dec(x_18); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_17); -x_19 = l_Lean_Meta_AC_acNfHypMeta(x_17, x_15, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -if (lean_obj_tag(x_20) == 0) -{ -uint8_t x_21; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -x_21 = !lean_is_exclusive(x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_19, 0); -lean_dec(x_22); -x_23 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1; -lean_ctor_set(x_7, 0, x_23); -lean_ctor_set(x_19, 0, x_7); -return x_19; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_dec(x_19); -x_25 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1; -lean_ctor_set(x_7, 0, x_25); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_7); -lean_ctor_set(x_26, 1, x_24); -return x_26; -} + x_381 = x_374; } -else -{ -lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; -lean_dec(x_17); -x_27 = lean_ctor_get(x_19, 1); -lean_inc(x_27); -lean_dec(x_19); -x_28 = lean_ctor_get(x_20, 0); -lean_inc(x_28); -lean_dec(x_20); -lean_inc(x_3); -lean_ctor_set(x_7, 1, x_28); -lean_ctor_set(x_7, 0, x_3); -x_29 = 1; -x_30 = lean_usize_add(x_6, x_29); -x_6 = x_30; -x_12 = x_27; -goto _start; +lean_ctor_set(x_381, 0, x_379); +lean_ctor_set(x_381, 1, x_380); +x_382 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_382, 0, x_370); +lean_ctor_set(x_382, 1, x_381); +x_211 = x_382; +x_212 = x_373; +goto block_302; } } -else +block_302: { -uint8_t x_32; -lean_free_object(x_7); -lean_dec(x_17); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -x_32 = !lean_is_exclusive(x_19); -if (x_32 == 0) +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; uint8_t x_218; uint8_t x_219; +x_213 = lean_ctor_get(x_211, 1); +lean_inc(x_213); +x_214 = lean_ctor_get(x_211, 0); +lean_inc(x_214); +lean_dec(x_211); +x_215 = lean_ctor_get(x_213, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_213, 1); +lean_inc(x_216); +lean_dec(x_213); +x_217 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2; +x_218 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_217); +if (x_218 == 0) { -return x_19; +if (x_6 == 0) +{ +uint8_t x_284; +x_284 = 0; +x_219 = x_284; +goto block_283; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_19, 0); -x_34 = lean_ctor_get(x_19, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_19); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} +lean_object* x_285; double x_286; double x_287; lean_object* x_288; +x_285 = lean_box(0); +x_286 = lean_unbox_float(x_215); +lean_dec(x_215); +x_287 = lean_unbox_float(x_216); +lean_dec(x_216); +x_288 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_286, x_287, x_5, x_285, x_9, x_10, x_11, x_12, x_212); +return x_288; } } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_7, 1); -lean_inc(x_36); -lean_dec(x_7); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_36); -x_37 = l_Lean_Meta_AC_acNfHypMeta(x_36, x_15, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_37) == 0) -{ -lean_object* x_38; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -if (lean_obj_tag(x_38) == 0) +if (x_6 == 0) { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_40 = x_37; -} else { - lean_dec_ref(x_37); - x_40 = lean_box(0); -} -x_41 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1; -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_36); -if (lean_is_scalar(x_40)) { - x_43 = lean_alloc_ctor(0, 2, 0); -} else { - x_43 = x_40; -} -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_39); -return x_43; +double x_289; double x_290; double x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; double x_296; uint8_t x_297; +x_289 = lean_unbox_float(x_216); +x_290 = lean_unbox_float(x_215); +x_291 = lean_float_sub(x_289, x_290); +x_292 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3; +x_293 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_292); +x_294 = 0; +x_295 = lean_unsigned_to_nat(0u); +x_296 = l_Float_ofScientific(x_293, x_294, x_295); +lean_dec(x_293); +x_297 = lean_float_decLt(x_296, x_291); +x_219 = x_297; +goto block_283; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; size_t x_48; -lean_dec(x_36); -x_44 = lean_ctor_get(x_37, 1); -lean_inc(x_44); -lean_dec(x_37); -x_45 = lean_ctor_get(x_38, 0); -lean_inc(x_45); -lean_dec(x_38); -lean_inc(x_3); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_3); -lean_ctor_set(x_46, 1, x_45); -x_47 = 1; -x_48 = lean_usize_add(x_6, x_47); -x_6 = x_48; -x_7 = x_46; -x_12 = x_44; -goto _start; +lean_object* x_298; double x_299; double x_300; lean_object* x_301; +x_298 = lean_box(0); +x_299 = lean_unbox_float(x_215); +lean_dec(x_215); +x_300 = lean_unbox_float(x_216); +lean_dec(x_216); +x_301 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_299, x_300, x_5, x_298, x_9, x_10, x_11, x_12, x_212); +return x_301; } } -else +block_283: { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -lean_dec(x_36); +if (x_219 == 0) +{ +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; +lean_dec(x_216); +lean_dec(x_215); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_220 = lean_st_ref_take(x_12, x_212); +x_221 = lean_ctor_get(x_220, 0); +lean_inc(x_221); +x_222 = lean_ctor_get(x_221, 3); +lean_inc(x_222); +x_223 = lean_ctor_get(x_220, 1); +lean_inc(x_223); +lean_dec(x_220); +x_224 = !lean_is_exclusive(x_221); +if (x_224 == 0) +{ +lean_object* x_225; uint8_t x_226; +x_225 = lean_ctor_get(x_221, 3); +lean_dec(x_225); +x_226 = !lean_is_exclusive(x_222); +if (x_226 == 0) +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; +x_227 = lean_ctor_get(x_222, 0); +x_228 = l_Lean_PersistentArray_append___rarg(x_15, x_227); +lean_dec(x_227); +lean_ctor_set(x_222, 0, x_228); +x_229 = lean_st_ref_set(x_12, x_221, x_223); +x_230 = lean_ctor_get(x_229, 1); +lean_inc(x_230); +lean_dec(x_229); +x_231 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_214, x_9, x_10, x_11, x_12, x_230); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_3); -x_50 = lean_ctor_get(x_37, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_37, 1); -lean_inc(x_51); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_52 = x_37; -} else { - lean_dec_ref(x_37); - x_52 = lean_box(0); -} -if (lean_is_scalar(x_52)) { - x_53 = lean_alloc_ctor(1, 2, 0); -} else { - x_53 = x_52; -} -lean_ctor_set(x_53, 0, x_50); -lean_ctor_set(x_53, 1, x_51); -return x_53; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_7 = l_Lean_MVarId_getNondepPropHyps(x_1, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_7) == 0) +lean_dec(x_214); +if (lean_obj_tag(x_231) == 0) { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; -x_8 = lean_ctor_get(x_7, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_7, 1); -lean_inc(x_9); -lean_dec(x_7); -x_10 = lean_box(0); -x_11 = lean_box(0); -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_1); -x_13 = lean_array_size(x_8); -x_14 = 0; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1(x_8, x_10, x_11, x_8, x_13, x_14, x_12, x_2, x_3, x_4, x_5, x_9); -lean_dec(x_8); -if (lean_obj_tag(x_15) == 0) +uint8_t x_232; +x_232 = !lean_is_exclusive(x_231); +if (x_232 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -if (lean_obj_tag(x_17) == 0) +return x_231; +} +else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_dec(x_16); -x_20 = lean_box(0); -x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_19, x_20, x_2, x_3, x_4, x_5, x_18); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_21; +lean_object* x_233; lean_object* x_234; lean_object* x_235; +x_233 = lean_ctor_get(x_231, 0); +x_234 = lean_ctor_get(x_231, 1); +lean_inc(x_234); +lean_inc(x_233); +lean_dec(x_231); +x_235 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_235, 0, x_233); +lean_ctor_set(x_235, 1, x_234); +return x_235; +} } else { -uint8_t x_22; -lean_dec(x_16); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_22 = !lean_is_exclusive(x_15); -if (x_22 == 0) +uint8_t x_236; +x_236 = !lean_is_exclusive(x_231); +if (x_236 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_15, 0); -lean_dec(x_23); -x_24 = lean_ctor_get(x_17, 0); -lean_inc(x_24); -lean_dec(x_17); -lean_ctor_set(x_15, 0, x_24); -return x_15; +return x_231; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_15, 1); -lean_inc(x_25); -lean_dec(x_15); -x_26 = lean_ctor_get(x_17, 0); -lean_inc(x_26); -lean_dec(x_17); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_25); -return x_27; +lean_object* x_237; lean_object* x_238; lean_object* x_239; +x_237 = lean_ctor_get(x_231, 0); +x_238 = lean_ctor_get(x_231, 1); +lean_inc(x_238); +lean_inc(x_237); +lean_dec(x_231); +x_239 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_239, 0, x_237); +lean_ctor_set(x_239, 1, x_238); +return x_239; } } } else { -uint8_t x_28; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_28 = !lean_is_exclusive(x_15); -if (x_28 == 0) -{ -return x_15; -} -else +uint64_t x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; +x_240 = lean_ctor_get_uint64(x_222, sizeof(void*)*1); +x_241 = lean_ctor_get(x_222, 0); +lean_inc(x_241); +lean_dec(x_222); +x_242 = l_Lean_PersistentArray_append___rarg(x_15, x_241); +lean_dec(x_241); +x_243 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_243, 0, x_242); +lean_ctor_set_uint64(x_243, sizeof(void*)*1, x_240); +lean_ctor_set(x_221, 3, x_243); +x_244 = lean_st_ref_set(x_12, x_221, x_223); +x_245 = lean_ctor_get(x_244, 1); +lean_inc(x_245); +lean_dec(x_244); +x_246 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_214, x_9, x_10, x_11, x_12, x_245); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_214); +if (lean_obj_tag(x_246) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_15, 0); -x_30 = lean_ctor_get(x_15, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_15); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; +x_247 = lean_ctor_get(x_246, 0); +lean_inc(x_247); +x_248 = lean_ctor_get(x_246, 1); +lean_inc(x_248); +if (lean_is_exclusive(x_246)) { + lean_ctor_release(x_246, 0); + lean_ctor_release(x_246, 1); + x_249 = x_246; +} else { + lean_dec_ref(x_246); + x_249 = lean_box(0); } +if (lean_is_scalar(x_249)) { + x_250 = lean_alloc_ctor(0, 2, 0); +} else { + x_250 = x_249; } +lean_ctor_set(x_250, 0, x_247); +lean_ctor_set(x_250, 1, x_248); +return x_250; } else { -uint8_t x_32; -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_32 = !lean_is_exclusive(x_7); -if (x_32 == 0) -{ -return x_7; +lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; +x_251 = lean_ctor_get(x_246, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_246, 1); +lean_inc(x_252); +if (lean_is_exclusive(x_246)) { + lean_ctor_release(x_246, 0); + lean_ctor_release(x_246, 1); + x_253 = x_246; +} else { + lean_dec_ref(x_246); + x_253 = lean_box(0); } -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_7, 0); -x_34 = lean_ctor_get(x_7, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_7); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +if (lean_is_scalar(x_253)) { + x_254 = lean_alloc_ctor(1, 2, 0); +} else { + x_254 = x_253; } +lean_ctor_set(x_254, 0, x_251); +lean_ctor_set(x_254, 1, x_252); +return x_254; } } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("ac_nf", 5, 5); -return x_1; +lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; uint64_t x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; +x_255 = lean_ctor_get(x_221, 0); +x_256 = lean_ctor_get(x_221, 1); +x_257 = lean_ctor_get(x_221, 2); +x_258 = lean_ctor_get(x_221, 4); +x_259 = lean_ctor_get(x_221, 5); +x_260 = lean_ctor_get(x_221, 6); +x_261 = lean_ctor_get(x_221, 7); +lean_inc(x_261); +lean_inc(x_260); +lean_inc(x_259); +lean_inc(x_258); +lean_inc(x_257); +lean_inc(x_256); +lean_inc(x_255); +lean_dec(x_221); +x_262 = lean_ctor_get_uint64(x_222, sizeof(void*)*1); +x_263 = lean_ctor_get(x_222, 0); +lean_inc(x_263); +if (lean_is_exclusive(x_222)) { + lean_ctor_release(x_222, 0); + x_264 = x_222; +} else { + lean_dec_ref(x_222); + x_264 = lean_box(0); } +x_265 = l_Lean_PersistentArray_append___rarg(x_15, x_263); +lean_dec(x_263); +if (lean_is_scalar(x_264)) { + x_266 = lean_alloc_ctor(0, 1, 8); +} else { + x_266 = x_264; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2() { -_start: +lean_ctor_set(x_266, 0, x_265); +lean_ctor_set_uint64(x_266, sizeof(void*)*1, x_262); +x_267 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_267, 0, x_255); +lean_ctor_set(x_267, 1, x_256); +lean_ctor_set(x_267, 2, x_257); +lean_ctor_set(x_267, 3, x_266); +lean_ctor_set(x_267, 4, x_258); +lean_ctor_set(x_267, 5, x_259); +lean_ctor_set(x_267, 6, x_260); +lean_ctor_set(x_267, 7, x_261); +x_268 = lean_st_ref_set(x_12, x_267, x_223); +x_269 = lean_ctor_get(x_268, 1); +lean_inc(x_269); +lean_dec(x_268); +x_270 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_214, x_9, x_10, x_11, x_12, x_269); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_214); +if (lean_obj_tag(x_270) == 0) { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} +lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; +x_271 = lean_ctor_get(x_270, 0); +lean_inc(x_271); +x_272 = lean_ctor_get(x_270, 1); +lean_inc(x_272); +if (lean_is_exclusive(x_270)) { + lean_ctor_release(x_270, 0); + lean_ctor_release(x_270, 1); + x_273 = x_270; +} else { + lean_dec_ref(x_270); + x_273 = lean_box(0); } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1), 6, 0); -return x_1; +if (lean_is_scalar(x_273)) { + x_274 = lean_alloc_ctor(0, 2, 0); +} else { + x_274 = x_273; } +lean_ctor_set(x_274, 0, x_271); +lean_ctor_set(x_274, 1, x_272); +return x_274; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3; -x_3 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; +lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; +x_275 = lean_ctor_get(x_270, 0); +lean_inc(x_275); +x_276 = lean_ctor_get(x_270, 1); +lean_inc(x_276); +if (lean_is_exclusive(x_270)) { + lean_ctor_release(x_270, 0); + lean_ctor_release(x_270, 1); + x_277 = x_270; +} else { + lean_dec_ref(x_270); + x_277 = lean_box(0); } +if (lean_is_scalar(x_277)) { + x_278 = lean_alloc_ctor(1, 2, 0); +} else { + x_278 = x_277; } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass() { -_start: -{ -lean_object* x_1; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4; -return x_1; +lean_ctor_set(x_278, 0, x_275); +lean_ctor_set(x_278, 1, x_276); +return x_278; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +} +else { -size_t x_13; size_t x_14; lean_object* x_15; -x_13 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_14 = lean_unbox_usize(x_6); -lean_dec(x_6); -x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_4); -lean_dec(x_2); -lean_dec(x_1); -return x_15; +lean_object* x_279; double x_280; double x_281; lean_object* x_282; +x_279 = lean_box(0); +x_280 = lean_unbox_float(x_215); +lean_dec(x_215); +x_281 = lean_unbox_float(x_216); +lean_dec(x_216); +x_282 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_2, x_3, x_4, x_15, x_214, x_218, x_280, x_281, x_5, x_279, x_9, x_10, x_11, x_12, x_212); +return x_282; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_inc(x_1); -return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1___boxed), 2, 0); -return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_6; uint8_t x_7; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1; -x_7 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 4); -if (x_7 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_8, 2); +lean_inc(x_11); +lean_inc(x_1); +x_12 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_unbox(x_13); +if (x_14 == 0) { -lean_object* x_8; lean_object* x_9; -lean_dec(x_3); -lean_dec(x_2); -x_8 = lean_box(0); -x_9 = lean_apply_2(x_6, x_4, x_8); -return x_9; -} -else +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2; +x_17 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_16); +if (x_17 == 0) { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass(x_2); -x_11 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_11, 0, x_10); -lean_ctor_set(x_11, 1, x_3); -x_12 = l_List_appendTR___rarg(x_4, x_11); -x_13 = lean_box(0); -x_14 = lean_apply_2(x_6, x_12, x_13); -return x_14; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +lean_object* x_18; +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_18 = lean_apply_5(x_3, x_6, x_7, x_8, x_9, x_15); +if (lean_obj_tag(x_18) == 0) { -uint8_t x_6; -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 3); -if (x_6 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2(x_1, x_2, x_3, x_4, x_7); -return x_8; +return x_18; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass; -lean_inc(x_3); -x_10 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_10, 0, x_9); -lean_ctor_set(x_10, 1, x_3); -x_11 = l_List_appendTR___rarg(x_4, x_10); -x_12 = lean_box(0); -x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2(x_1, x_2, x_3, x_11, x_12); -return x_13; -} -} -} -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_18); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_2 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -lean_inc(x_2); -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass(x_2); -x_4 = lean_box(0); -x_5 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_5, 0, x_3); -lean_ctor_set(x_5, 1, x_4); -x_6 = lean_ctor_get_uint8(x_1, sizeof(void*)*2 + 2); -if (x_6 == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_18); +if (x_23 == 0) { -lean_object* x_7; lean_object* x_8; -x_7 = lean_box(0); -x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3(x_1, x_2, x_4, x_5, x_7); -lean_dec(x_1); -return x_8; +return x_18; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1; -x_10 = l_List_appendTR___rarg(x_5, x_9); -x_11 = lean_box(0); -x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3(x_1, x_2, x_4, x_10, x_11); -lean_dec(x_1); -return x_12; -} -} +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_18, 0); +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_18); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -lean_dec(x_1); -return x_6; +lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_27 = lean_box(0); +x_28 = lean_unbox(x_13); +lean_dec(x_13); +x_29 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4(x_11, x_1, x_4, x_5, x_2, x_28, x_3, x_27, x_6, x_7, x_8, x_9, x_15); +lean_dec(x_11); +return x_29; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: +else { -lean_object* x_6; -x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__3(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_5); -lean_dec(x_1); -return x_6; +lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_12, 1); +lean_inc(x_30); +lean_dec(x_12); +x_31 = lean_box(0); +x_32 = lean_unbox(x_13); +lean_dec(x_13); +x_33 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4(x_11, x_1, x_4, x_5, x_2, x_32, x_3, x_31, x_6, x_7, x_8, x_9, x_30); +lean_dec(x_11); +return x_33; +} } } static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Normalizing goal", 16, 16); +x_1 = lean_mk_string_unchecked("Preprocessing goal", 18, 18); return x_1; } } @@ -17756,278 +2151,128 @@ lean_ctor_set(x_8, 1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1() { _start: { -lean_object* x_9; lean_object* x_10; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline(x_1); -x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_9, x_2, x_4, x_5, x_6, x_7, x_8); -return x_10; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Running preprocessing pipeline on:\n", 35, 35); +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go), 8, 1); +lean_closure_set(x_8, 0, x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run___rarg), 8, 3); +lean_closure_set(x_9, 0, x_2); +lean_closure_set(x_9, 1, x_1); +lean_closure_set(x_9, 2, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2; +x_12 = 1; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7; +x_14 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1(x_10, x_11, x_9, x_12, x_13, x_3, x_4, x_5, x_6, x_7); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_9; -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_2); -x_9 = l_Lean_MVarId_falseOrByContra(x_1, x_2, x_4, x_5, x_6, x_7, x_8); -if (lean_obj_tag(x_9) == 0) -{ -lean_object* x_10; -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -if (lean_obj_tag(x_10) == 0) -{ -uint8_t x_11; -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_7; +x_7 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_11 = !lean_is_exclusive(x_9); -if (x_11 == 0) -{ -lean_object* x_12; -x_12 = lean_ctor_get(x_9, 0); -lean_dec(x_12); -lean_ctor_set(x_9, 0, x_2); -return x_9; -} -else -{ -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_9, 1); -lean_inc(x_13); -lean_dec(x_9); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_13); -return x_14; -} -} -else -{ -lean_object* x_15; uint8_t x_16; lean_dec(x_2); -x_15 = lean_ctor_get(x_9, 1); -lean_inc(x_15); -lean_dec(x_9); -x_16 = !lean_is_exclusive(x_10); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_17 = lean_ctor_get(x_10, 0); -x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_19 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_18, x_4, x_5, x_6, x_7, x_15); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_unbox(x_20); -lean_dec(x_20); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_free_object(x_10); -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); -lean_dec(x_19); -x_23 = lean_box(0); -x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_3, x_17, x_23, x_4, x_5, x_6, x_7, x_22); -return x_24; -} -else -{ -uint8_t x_25; -x_25 = !lean_is_exclusive(x_19); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_26 = lean_ctor_get(x_19, 1); -x_27 = lean_ctor_get(x_19, 0); -lean_dec(x_27); -lean_inc(x_17); -x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2; -lean_ctor_set_tag(x_19, 7); -lean_ctor_set(x_19, 1, x_10); -lean_ctor_set(x_19, 0, x_28); -x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_19); -lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_18, x_30, x_4, x_5, x_6, x_7, x_26); -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_3, x_17, x_32, x_4, x_5, x_6, x_7, x_33); -lean_dec(x_32); -return x_34; -} -else -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_35 = lean_ctor_get(x_19, 1); -lean_inc(x_35); -lean_dec(x_19); -lean_inc(x_17); -x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2; -x_37 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_10); -x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_39 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -x_40 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_18, x_39, x_4, x_5, x_6, x_7, x_35); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_3, x_17, x_41, x_4, x_5, x_6, x_7, x_42); -lean_dec(x_41); -return x_43; -} +lean_dec(x_1); +return x_7; } } -else +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_44 = lean_ctor_get(x_10, 0); -lean_inc(x_44); +lean_object* x_12; +x_12 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); -x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2; -x_46 = l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(x_45, x_4, x_5, x_6, x_7, x_15); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_unbox(x_47); -lean_dec(x_47); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_dec(x_46); -x_50 = lean_box(0); -x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_3, x_44, x_50, x_4, x_5, x_6, x_7, x_49); -return x_51; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_52 = lean_ctor_get(x_46, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_53 = x_46; -} else { - lean_dec_ref(x_46); - x_53 = lean_box(0); -} -lean_inc(x_44); -x_54 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_54, 0, x_44); -x_55 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2; -if (lean_is_scalar(x_53)) { - x_56 = lean_alloc_ctor(7, 2, 0); -} else { - x_56 = x_53; - lean_ctor_set_tag(x_56, 7); -} -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_54); -x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5; -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -x_59 = l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(x_45, x_58, x_4, x_5, x_6, x_7, x_52); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_3, x_44, x_60, x_4, x_5, x_6, x_7, x_61); -lean_dec(x_60); -return x_62; -} -} -} -} -else -{ -uint8_t x_63; +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_63 = !lean_is_exclusive(x_9); -if (x_63 == 0) -{ -return x_9; +return x_12; } -else +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_9, 0); -x_65 = lean_ctor_get(x_9, 1); -lean_inc(x_65); -lean_inc(x_64); +uint8_t x_16; uint8_t x_17; double x_18; double x_19; lean_object* x_20; +x_16 = lean_unbox(x_2); +lean_dec(x_2); +x_17 = lean_unbox(x_7); +lean_dec(x_7); +x_18 = lean_unbox_float(x_8); +lean_dec(x_8); +x_19 = lean_unbox_float(x_9); lean_dec(x_9); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2(x_1, x_16, x_3, x_4, x_5, x_6, x_17, x_18, x_19, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +return x_20; } } +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; uint8_t x_17; double x_18; double x_19; lean_object* x_20; +x_16 = lean_unbox(x_2); +lean_dec(x_2); +x_17 = lean_unbox(x_6); +lean_dec(x_6); +x_18 = lean_unbox_float(x_7); +lean_dec(x_7); +x_19 = lean_unbox_float(x_8); +lean_dec(x_8); +x_20 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3(x_1, x_16, x_3, x_4, x_5, x_17, x_18, x_19, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_10); +return x_20; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1() { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___boxed), 6, 0); -return x_1; +uint8_t x_14; uint8_t x_15; lean_object* x_16; +x_14 = lean_unbox(x_3); +lean_dec(x_3); +x_15 = lean_unbox(x_6); +lean_dec(x_6); +x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4(x_1, x_2, x_14, x_4, x_5, x_15, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_1); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_8 = lean_box(0); -x_9 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3), 8, 3); -lean_closure_set(x_9, 0, x_1); -lean_closure_set(x_9, 1, x_8); -lean_closure_set(x_9, 2, x_2); -x_10 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1; -x_12 = 1; -x_13 = l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3; -x_14 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(x_10, x_11, x_9, x_12, x_13, x_3, x_4, x_5, x_6, x_7); -return x_14; +uint8_t x_11; lean_object* x_12; +x_11 = lean_unbox(x_4); +lean_dec(x_4); +x_12 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; } } LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -18043,16 +2288,15 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1() { _start: { -lean_object* x_9; -x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -return x_9; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2() { _start: { lean_object* x_1; @@ -18060,7 +2304,7 @@ x_1 = lean_mk_string_unchecked("Parser", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3() { _start: { lean_object* x_1; @@ -18068,19 +2312,19 @@ x_1 = lean_mk_string_unchecked("bvNormalize", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5() { _start: { lean_object* x_1; @@ -18088,14 +2332,14 @@ x_1 = lean_mk_string_unchecked("optConfig", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5() { +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; } @@ -18104,7 +2348,7 @@ LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNo _start: { lean_object* x_11; uint8_t x_12; -x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4; lean_inc(x_1); x_12 = l_Lean_Syntax_isOfKind(x_1, x_11); if (x_12 == 0) @@ -18117,7 +2361,7 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_13 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_13; } else @@ -18126,7 +2370,7 @@ lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; x_14 = lean_unsigned_to_nat(1u); x_15 = l_Lean_Syntax_getArg(x_1, x_14); lean_dec(x_1); -x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5; +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6; lean_inc(x_15); x_17 = l_Lean_Syntax_isOfKind(x_15, x_16); if (x_17 == 0) @@ -18139,7 +2383,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_18 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_MVarId_elabFalseOrByContra___spec__1___rarg(x_10); +x_18 = l_Lean_Elab_throwUnsupportedSyntax___at_Lean_Elab_Tactic_evalExact___spec__1___rarg(x_10); return x_18; } else @@ -18323,26 +2567,58 @@ static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Norm _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("evalBVNormalize", 15, 15); +x_1 = lean_mk_string_unchecked("Elab", 4, 4); return x_1; } } static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Frontend", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Normalize", 9, 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("evalBVNormalize", 15, 15); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6() { +_start: +{ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2; -x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5; -x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6; -x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5; x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); return x_8; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7() { _start: { lean_object* x_1; @@ -18350,7 +2626,7 @@ x_1 = l_Lean_Elab_Tactic_tacticElabAttribute; return x_1; } } -static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4() { +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8() { _start: { lean_object* x_1; @@ -18362,640 +2638,94 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Norma _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3; -x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__3; -x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2; -x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8; x_6 = l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(x_2, x_3, x_4, x_5, x_1); return x_6; } } -lean_object* initialize_Lean_Meta_AppBuilder(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_Meta_Tactic_AC_Main(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_Elab_Tactic_Simp(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Elab_Tactic_FalseOrByContra(uint8_t builtin, lean_object*); -lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(uint8_t builtin, lean_object*); -lean_object* initialize_Std_Tactic_BVDecide_Normalize(uint8_t builtin, lean_object*); -lean_object* initialize_Std_Tactic_BVDecide_Syntax(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Rewrite(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AndFlatten(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_EmbeddedConstraint(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AC(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; -res = initialize_Lean_Meta_AppBuilder(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Lean_Meta_Tactic_AC_Main(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Lean_Elab_Tactic_Simp(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); res = initialize_Lean_Elab_Tactic_FalseOrByContra(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Std_Tactic_BVDecide_Normalize(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -res = initialize_Std_Tactic_BVDecide_Syntax(builtin, lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__8); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__9); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__10); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__11); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__12); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__13); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__14); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__15); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349____closed__16); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_349_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351____closed__2); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_351_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655____closed__8); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_655_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_657_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__8); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__9); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__10); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__11); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021____closed__12); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1021_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1023_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387____closed__3); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1387_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1389_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660____closed__6); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1660_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_1662_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083____closed__6); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2083_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2085_(lean_io_mk_world()); -if (lean_io_result_is_error(res)) return res; -lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__8); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__9); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__10); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__11); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__12); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952____closed__13); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2952_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_2954_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__8); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__9); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__10); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__11); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__12); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__13); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__14); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821____closed__15); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3821_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Rewrite(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_3823_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AndFlatten(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__1); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__2); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__3); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__4); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__5); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__6); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__7); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__8); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__9); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__10); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__11); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__12); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__13); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__14); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__15); -l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508____closed__16); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4508_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_EmbeddedConstraint(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize___hyg_4510_(lean_io_mk_world()); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AC(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__2___closed__1(); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__1); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__3___closed__2); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__1); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__2); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3(); -lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__3); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__4 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__4(); -l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__4___closed__5(); -l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1 = _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1(); -lean_mark_persistent(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__1); -l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2 = _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2(); -lean_mark_persistent(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__2); -l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3 = _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3(); -lean_mark_persistent(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___lambda__2___closed__3); -l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1 = _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1(); -lean_mark_persistent(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__1); -l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2 = _init_l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2(); -lean_mark_persistent(l_List_foldlM___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__3___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__9); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__10); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___elambda__1___closed__11); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_rewriteRulesPass___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__6); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__7); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__1___closed__8); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__3___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass_trySplit___lambda__5___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___elambda__1___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_andFlatteningPass); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___elambda__1___lambda__1___closed__5); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_embeddedConstraintPass___closed__2); -l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___elambda__1___spec__1___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__2); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass___closed__4); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_acNormalizePass); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___lambda__2___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_passPipeline___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_passPipeline___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize_go___closed__8); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__2___closed__1(); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__1); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__3___closed__2); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__1); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__2); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__3); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__4 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__4(); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___spec__1___lambda__4___closed__5(); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__2(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__2); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__3(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__1___closed__3); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__1); -l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___lambda__3___closed__2); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bvNormalize___closed__2); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__1); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__2(); @@ -19006,6 +2736,8 @@ l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4 = _in lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__4); l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5(); lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize___closed__6); l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__1); l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__2(); @@ -19014,6 +2746,14 @@ l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1__ lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__3); l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4(); lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1___closed__8); if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_evalBVNormalize__1(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AC.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AC.c new file mode 100644 index 000000000000..62a4fda75af8 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AC.c @@ -0,0 +1,548 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.AC +// Imports: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic Lean.Meta.Tactic.AC.Main +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_AC_acNfHypMeta(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uget(lean_object*, size_t); +size_t lean_array_size(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_lt(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3; +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = lean_usize_dec_lt(x_6, x_5); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_7); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +else +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_uget(x_4, x_6); +x_18 = !lean_is_exclusive(x_7); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_7, 1); +x_20 = lean_ctor_get(x_7, 0); +lean_dec(x_20); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_19); +x_21 = l_Lean_Meta_AC_acNfHypMeta(x_19, x_17, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 0); +lean_dec(x_24); +x_25 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1; +lean_ctor_set(x_7, 0, x_25); +lean_ctor_set(x_21, 0, x_7); +return x_21; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_21, 1); +lean_inc(x_26); +lean_dec(x_21); +x_27 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1; +lean_ctor_set(x_7, 0, x_27); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_7); +lean_ctor_set(x_28, 1, x_26); +return x_28; +} +} +else +{ +lean_object* x_29; lean_object* x_30; size_t x_31; size_t x_32; +lean_dec(x_19); +x_29 = lean_ctor_get(x_21, 1); +lean_inc(x_29); +lean_dec(x_21); +x_30 = lean_ctor_get(x_22, 0); +lean_inc(x_30); +lean_dec(x_22); +lean_inc(x_3); +lean_ctor_set(x_7, 1, x_30); +lean_ctor_set(x_7, 0, x_3); +x_31 = 1; +x_32 = lean_usize_add(x_6, x_31); +x_6 = x_32; +x_14 = x_29; +goto _start; +} +} +else +{ +uint8_t x_34; +lean_free_object(x_7); +lean_dec(x_19); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +x_34 = !lean_is_exclusive(x_21); +if (x_34 == 0) +{ +return x_21; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_21, 0); +x_36 = lean_ctor_get(x_21, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_21); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_7, 1); +lean_inc(x_38); +lean_dec(x_7); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_38); +x_39 = l_Lean_Meta_AC_acNfHypMeta(x_38, x_17, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_39) == 0) +{ +lean_object* x_40; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_42 = x_39; +} else { + lean_dec_ref(x_39); + x_42 = lean_box(0); +} +x_43 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1; +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_38); +if (lean_is_scalar(x_42)) { + x_45 = lean_alloc_ctor(0, 2, 0); +} else { + x_45 = x_42; +} +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_41); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; size_t x_49; size_t x_50; +lean_dec(x_38); +x_46 = lean_ctor_get(x_39, 1); +lean_inc(x_46); +lean_dec(x_39); +x_47 = lean_ctor_get(x_40, 0); +lean_inc(x_47); +lean_dec(x_40); +lean_inc(x_3); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_3); +lean_ctor_set(x_48, 1, x_47); +x_49 = 1; +x_50 = lean_usize_add(x_6, x_49); +x_6 = x_50; +x_7 = x_48; +x_14 = x_46; +goto _start; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_dec(x_38); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_3); +x_52 = lean_ctor_get(x_39, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_39, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_54 = x_39; +} else { + lean_dec_ref(x_39); + x_54 = lean_box(0); +} +if (lean_is_scalar(x_54)) { + x_55 = lean_alloc_ctor(1, 2, 0); +} else { + x_55 = x_54; +} +lean_ctor_set(x_55, 0, x_52); +lean_ctor_set(x_55, 1, x_53); +return x_55; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_9 = l_Lean_MVarId_getNondepPropHyps(x_1, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_box(0); +x_13 = lean_box(0); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_1); +x_15 = lean_array_size(x_10); +x_16 = 0; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1(x_10, x_12, x_13, x_10, x_15, x_16, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_11); +lean_dec(x_10); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1(x_21, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_20); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_23; +} +else +{ +uint8_t x_24; +lean_dec(x_18); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_17, 0); +lean_dec(x_25); +x_26 = lean_ctor_get(x_19, 0); +lean_inc(x_26); +lean_dec(x_19); +lean_ctor_set(x_17, 0, x_26); +return x_17; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_17, 1); +lean_inc(x_27); +lean_dec(x_17); +x_28 = lean_ctor_get(x_19, 0); +lean_inc(x_28); +lean_dec(x_19); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; +} +} +} +else +{ +uint8_t x_30; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_30 = !lean_is_exclusive(x_17); +if (x_30 == 0) +{ +return x_17; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_17, 0); +x_32 = lean_ctor_get(x_17, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_17); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +} +else +{ +uint8_t x_34; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_9); +if (x_34 == 0) +{ +return x_9; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_9, 0); +x_36 = lean_ctor_get(x_9, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_9); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ac_nf", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +size_t x_15; size_t x_16; lean_object* x_17; +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1(x_1, x_2, x_3, x_4, x_15, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_AC_Main(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AC(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_AC_Main(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___elambda__1___spec__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_acNormalizePass); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AndFlatten.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AndFlatten.c new file mode 100644 index 000000000000..b3fe072d49b8 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/AndFlatten.c @@ -0,0 +1,2797 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.AndFlatten +// Imports: Std.Tactic.BVDecide.Normalize.Bool Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic Lean.Meta.Tactic.Assert +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +size_t lean_uint64_to_usize(uint64_t); +uint8_t l_Lean_Expr_isApp(lean_object*); +uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17; +lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2; +lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4; +lean_object* l_Lean_Level_ofNat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1; +size_t lean_usize_of_nat(lean_object*); +lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10; +lean_object* lean_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_shift_right(uint64_t, uint64_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); +lean_object* lean_nat_div(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19; +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15; +lean_object* lean_st_mk_ref(lean_object*, lean_object*); +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t l_Lean_Expr_hash(lean_object*); +lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_LocalDecl_userName(lean_object*); +lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processFVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +uint64_t lean_uint64_xor(uint64_t, uint64_t); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2; +lean_object* lean_nat_mul(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16; +size_t lean_usize_sub(size_t, size_t); +lean_object* lean_array_mk(lean_object*); +lean_object* l_Lean_MVarId_tryClearMany(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_add(size_t, size_t); +lean_object* lean_array_uget(lean_object*, size_t); +lean_object* l_Lean_Expr_fvar___override(lean_object*); +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get_size(lean_object*); +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3; +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8; +lean_object* l_Lean_MVarId_assertHypotheses(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3; +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14; +size_t lean_usize_land(size_t, size_t); +uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Eq", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = l_Lean_Level_ofNat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Bool", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Std", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Normalize", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("and_left", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("and_right", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14; +x_4 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11; +lean_inc(x_1); +x_15 = l_Lean_mkApp3(x_12, x_13, x_1, x_14); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18; +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_17 = l_Lean_mkApp3(x_16, x_1, x_2, x_3); +x_18 = 0; +x_19 = 0; +lean_inc(x_4); +x_20 = lean_alloc_ctor(0, 3, 2); +lean_ctor_set(x_20, 0, x_4); +lean_ctor_set(x_20, 1, x_15); +lean_ctor_set(x_20, 2, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*3, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*3 + 1, x_19); +lean_inc(x_2); +x_21 = l_Lean_mkApp3(x_12, x_13, x_2, x_14); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21; +x_23 = l_Lean_mkApp3(x_22, x_1, x_2, x_3); +x_24 = lean_alloc_ctor(0, 3, 2); +lean_ctor_set(x_24, 0, x_4); +lean_ctor_set(x_24, 1, x_21); +lean_ctor_set(x_24, 2, x_23); +lean_ctor_set_uint8(x_24, sizeof(void*)*3, x_18); +lean_ctor_set_uint8(x_24, sizeof(void*)*3 + 1, x_19); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_20); +lean_ctor_set(x_25, 1, x_24); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_11); +return x_27; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2___boxed), 7, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1; +x_13 = l_Lean_Expr_cleanupAnnotations(x_1); +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10; +x_15 = l_Lean_Expr_isConstOf(x_13, x_14); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_16 = lean_box(0); +x_17 = lean_apply_7(x_12, x_16, x_6, x_7, x_8, x_9, x_10, x_11); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1(x_4, x_5, x_2, x_3, x_18, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_19; +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("and", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1; +x_12 = l_Lean_Expr_cleanupAnnotations(x_3); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_apply_7(x_11, x_14, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_box(0); +x_20 = lean_apply_7(x_11, x_19, x_5, x_6, x_7, x_8, x_9, x_10); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2; +x_24 = l_Lean_Expr_isConstOf(x_22, x_23); +lean_dec(x_22); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_25 = lean_box(0); +x_26 = lean_apply_7(x_11, x_25, x_5, x_6, x_7, x_8, x_9, x_10); +return x_26; +} +else +{ +lean_object* x_27; +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3(x_4, x_1, x_2, x_21, x_16, x_5, x_6, x_7, x_8, x_9, x_10); +return x_27; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_1, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_1, 2); +lean_inc(x_10); +lean_dec(x_1); +x_11 = lean_st_ref_get(x_2, x_7); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 2); +lean_inc(x_13); +lean_dec(x_12); +x_14 = !lean_is_exclusive(x_11); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; lean_object* x_31; uint8_t x_32; +x_15 = lean_ctor_get(x_11, 1); +x_16 = lean_ctor_get(x_11, 0); +lean_dec(x_16); +x_17 = lean_ctor_get(x_13, 1); +lean_inc(x_17); +lean_dec(x_13); +x_18 = lean_array_get_size(x_17); +x_19 = l_Lean_Expr_hash(x_9); +x_20 = 32; +x_21 = lean_uint64_shift_right(x_19, x_20); +x_22 = lean_uint64_xor(x_19, x_21); +x_23 = 16; +x_24 = lean_uint64_shift_right(x_22, x_23); +x_25 = lean_uint64_xor(x_22, x_24); +x_26 = lean_uint64_to_usize(x_25); +x_27 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_28 = 1; +x_29 = lean_usize_sub(x_27, x_28); +x_30 = lean_usize_land(x_26, x_29); +x_31 = lean_array_uget(x_17, x_30); +lean_dec(x_17); +x_32 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_31); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; +lean_free_object(x_11); +x_56 = lean_st_ref_take(x_2, x_15); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_57, 2); +lean_inc(x_58); +x_59 = lean_ctor_get(x_56, 1); +lean_inc(x_59); +lean_dec(x_56); +x_60 = !lean_is_exclusive(x_57); +if (x_60 == 0) +{ +lean_object* x_61; uint8_t x_62; +x_61 = lean_ctor_get(x_57, 2); +lean_dec(x_61); +x_62 = !lean_is_exclusive(x_58); +if (x_62 == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; size_t x_66; size_t x_67; size_t x_68; lean_object* x_69; uint8_t x_70; +x_63 = lean_ctor_get(x_58, 0); +x_64 = lean_ctor_get(x_58, 1); +x_65 = lean_array_get_size(x_64); +x_66 = lean_usize_of_nat(x_65); +lean_dec(x_65); +x_67 = lean_usize_sub(x_66, x_28); +x_68 = lean_usize_land(x_26, x_67); +x_69 = lean_array_uget(x_64, x_68); +x_70 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_69); +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; +x_71 = lean_unsigned_to_nat(1u); +x_72 = lean_nat_add(x_63, x_71); +lean_dec(x_63); +x_73 = lean_box(0); +lean_inc(x_9); +x_74 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_74, 0, x_9); +lean_ctor_set(x_74, 1, x_73); +lean_ctor_set(x_74, 2, x_69); +x_75 = lean_array_uset(x_64, x_68, x_74); +x_76 = lean_unsigned_to_nat(4u); +x_77 = lean_nat_mul(x_72, x_76); +x_78 = lean_unsigned_to_nat(3u); +x_79 = lean_nat_div(x_77, x_78); +lean_dec(x_77); +x_80 = lean_array_get_size(x_75); +x_81 = lean_nat_dec_le(x_79, x_80); +lean_dec(x_80); +lean_dec(x_79); +if (x_81 == 0) +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_75); +lean_ctor_set(x_58, 1, x_82); +lean_ctor_set(x_58, 0, x_72); +x_83 = lean_st_ref_set(x_2, x_57, x_59); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +x_33 = x_84; +goto block_55; +} +else +{ +lean_object* x_85; lean_object* x_86; +lean_ctor_set(x_58, 1, x_75); +lean_ctor_set(x_58, 0, x_72); +x_85 = lean_st_ref_set(x_2, x_57, x_59); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_33 = x_86; +goto block_55; +} +} +else +{ +lean_object* x_87; lean_object* x_88; +lean_dec(x_69); +x_87 = lean_st_ref_set(x_2, x_57, x_59); +x_88 = lean_ctor_get(x_87, 1); +lean_inc(x_88); +lean_dec(x_87); +x_33 = x_88; +goto block_55; +} +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; size_t x_92; size_t x_93; size_t x_94; lean_object* x_95; uint8_t x_96; +x_89 = lean_ctor_get(x_58, 0); +x_90 = lean_ctor_get(x_58, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_58); +x_91 = lean_array_get_size(x_90); +x_92 = lean_usize_of_nat(x_91); +lean_dec(x_91); +x_93 = lean_usize_sub(x_92, x_28); +x_94 = lean_usize_land(x_26, x_93); +x_95 = lean_array_uget(x_90, x_94); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_95); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; +x_97 = lean_unsigned_to_nat(1u); +x_98 = lean_nat_add(x_89, x_97); +lean_dec(x_89); +x_99 = lean_box(0); +lean_inc(x_9); +x_100 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_100, 0, x_9); +lean_ctor_set(x_100, 1, x_99); +lean_ctor_set(x_100, 2, x_95); +x_101 = lean_array_uset(x_90, x_94, x_100); +x_102 = lean_unsigned_to_nat(4u); +x_103 = lean_nat_mul(x_98, x_102); +x_104 = lean_unsigned_to_nat(3u); +x_105 = lean_nat_div(x_103, x_104); +lean_dec(x_103); +x_106 = lean_array_get_size(x_101); +x_107 = lean_nat_dec_le(x_105, x_106); +lean_dec(x_106); +lean_dec(x_105); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_108 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_101); +x_109 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_98); +lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_57, 2, x_109); +x_110 = lean_st_ref_set(x_2, x_57, x_59); +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +lean_dec(x_110); +x_33 = x_111; +goto block_55; +} +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_98); +lean_ctor_set(x_112, 1, x_101); +lean_ctor_set(x_57, 2, x_112); +x_113 = lean_st_ref_set(x_2, x_57, x_59); +x_114 = lean_ctor_get(x_113, 1); +lean_inc(x_114); +lean_dec(x_113); +x_33 = x_114; +goto block_55; +} +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_95); +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_89); +lean_ctor_set(x_115, 1, x_90); +lean_ctor_set(x_57, 2, x_115); +x_116 = lean_st_ref_set(x_2, x_57, x_59); +x_117 = lean_ctor_get(x_116, 1); +lean_inc(x_117); +lean_dec(x_116); +x_33 = x_117; +goto block_55; +} +} +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; size_t x_124; size_t x_125; size_t x_126; lean_object* x_127; uint8_t x_128; +x_118 = lean_ctor_get(x_57, 0); +x_119 = lean_ctor_get(x_57, 1); +lean_inc(x_119); +lean_inc(x_118); +lean_dec(x_57); +x_120 = lean_ctor_get(x_58, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_58, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_122 = x_58; +} else { + lean_dec_ref(x_58); + x_122 = lean_box(0); +} +x_123 = lean_array_get_size(x_121); +x_124 = lean_usize_of_nat(x_123); +lean_dec(x_123); +x_125 = lean_usize_sub(x_124, x_28); +x_126 = lean_usize_land(x_26, x_125); +x_127 = lean_array_uget(x_121, x_126); +x_128 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_127); +if (x_128 == 0) +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_139; +x_129 = lean_unsigned_to_nat(1u); +x_130 = lean_nat_add(x_120, x_129); +lean_dec(x_120); +x_131 = lean_box(0); +lean_inc(x_9); +x_132 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_132, 0, x_9); +lean_ctor_set(x_132, 1, x_131); +lean_ctor_set(x_132, 2, x_127); +x_133 = lean_array_uset(x_121, x_126, x_132); +x_134 = lean_unsigned_to_nat(4u); +x_135 = lean_nat_mul(x_130, x_134); +x_136 = lean_unsigned_to_nat(3u); +x_137 = lean_nat_div(x_135, x_136); +lean_dec(x_135); +x_138 = lean_array_get_size(x_133); +x_139 = lean_nat_dec_le(x_137, x_138); +lean_dec(x_138); +lean_dec(x_137); +if (x_139 == 0) +{ +lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_140 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_133); +if (lean_is_scalar(x_122)) { + x_141 = lean_alloc_ctor(0, 2, 0); +} else { + x_141 = x_122; +} +lean_ctor_set(x_141, 0, x_130); +lean_ctor_set(x_141, 1, x_140); +x_142 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_142, 0, x_118); +lean_ctor_set(x_142, 1, x_119); +lean_ctor_set(x_142, 2, x_141); +x_143 = lean_st_ref_set(x_2, x_142, x_59); +x_144 = lean_ctor_get(x_143, 1); +lean_inc(x_144); +lean_dec(x_143); +x_33 = x_144; +goto block_55; +} +else +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +if (lean_is_scalar(x_122)) { + x_145 = lean_alloc_ctor(0, 2, 0); +} else { + x_145 = x_122; +} +lean_ctor_set(x_145, 0, x_130); +lean_ctor_set(x_145, 1, x_133); +x_146 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_146, 0, x_118); +lean_ctor_set(x_146, 1, x_119); +lean_ctor_set(x_146, 2, x_145); +x_147 = lean_st_ref_set(x_2, x_146, x_59); +x_148 = lean_ctor_get(x_147, 1); +lean_inc(x_148); +lean_dec(x_147); +x_33 = x_148; +goto block_55; +} +} +else +{ +lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +lean_dec(x_127); +if (lean_is_scalar(x_122)) { + x_149 = lean_alloc_ctor(0, 2, 0); +} else { + x_149 = x_122; +} +lean_ctor_set(x_149, 0, x_120); +lean_ctor_set(x_149, 1, x_121); +x_150 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_150, 0, x_118); +lean_ctor_set(x_150, 1, x_119); +lean_ctor_set(x_150, 2, x_149); +x_151 = lean_st_ref_set(x_2, x_150, x_59); +x_152 = lean_ctor_get(x_151, 1); +lean_inc(x_152); +lean_dec(x_151); +x_33 = x_152; +goto block_55; +} +} +block_55: +{ +lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1; +x_35 = l_Lean_Expr_cleanupAnnotations(x_9); +x_36 = l_Lean_Expr_isApp(x_35); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +lean_dec(x_35); +lean_dec(x_10); +lean_dec(x_8); +x_37 = lean_box(0); +x_38 = lean_apply_7(x_34, x_37, x_2, x_3, x_4, x_5, x_6, x_33); +return x_38; +} +else +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = l_Lean_Expr_appArg(x_35, lean_box(0)); +x_40 = l_Lean_Expr_appFnCleanup(x_35, lean_box(0)); +x_41 = l_Lean_Expr_isApp(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_10); +lean_dec(x_8); +x_42 = lean_box(0); +x_43 = lean_apply_7(x_34, x_42, x_2, x_3, x_4, x_5, x_6, x_33); +return x_43; +} +else +{ +lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_44 = l_Lean_Expr_appArg(x_40, lean_box(0)); +x_45 = l_Lean_Expr_appFnCleanup(x_40, lean_box(0)); +x_46 = l_Lean_Expr_isApp(x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_45); +lean_dec(x_44); +lean_dec(x_39); +lean_dec(x_10); +lean_dec(x_8); +x_47 = lean_box(0); +x_48 = lean_apply_7(x_34, x_47, x_2, x_3, x_4, x_5, x_6, x_33); +return x_48; +} +else +{ +lean_object* x_49; lean_object* x_50; uint8_t x_51; +x_49 = l_Lean_Expr_appFnCleanup(x_45, lean_box(0)); +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2; +x_51 = l_Lean_Expr_isConstOf(x_49, x_50); +lean_dec(x_49); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; +lean_dec(x_44); +lean_dec(x_39); +lean_dec(x_10); +lean_dec(x_8); +x_52 = lean_box(0); +x_53 = lean_apply_7(x_34, x_52, x_2, x_3, x_4, x_5, x_6, x_33); +return x_53; +} +else +{ +lean_object* x_54; +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4(x_10, x_8, x_44, x_39, x_2, x_3, x_4, x_5, x_6, x_33); +return x_54; +} +} +} +} +} +} +else +{ +lean_object* x_153; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_153 = lean_box(0); +lean_ctor_set(x_11, 0, x_153); +return x_11; +} +} +else +{ +lean_object* x_154; lean_object* x_155; lean_object* x_156; uint64_t x_157; uint64_t x_158; uint64_t x_159; uint64_t x_160; uint64_t x_161; uint64_t x_162; uint64_t x_163; size_t x_164; size_t x_165; size_t x_166; size_t x_167; size_t x_168; lean_object* x_169; uint8_t x_170; +x_154 = lean_ctor_get(x_11, 1); +lean_inc(x_154); +lean_dec(x_11); +x_155 = lean_ctor_get(x_13, 1); +lean_inc(x_155); +lean_dec(x_13); +x_156 = lean_array_get_size(x_155); +x_157 = l_Lean_Expr_hash(x_9); +x_158 = 32; +x_159 = lean_uint64_shift_right(x_157, x_158); +x_160 = lean_uint64_xor(x_157, x_159); +x_161 = 16; +x_162 = lean_uint64_shift_right(x_160, x_161); +x_163 = lean_uint64_xor(x_160, x_162); +x_164 = lean_uint64_to_usize(x_163); +x_165 = lean_usize_of_nat(x_156); +lean_dec(x_156); +x_166 = 1; +x_167 = lean_usize_sub(x_165, x_166); +x_168 = lean_usize_land(x_164, x_167); +x_169 = lean_array_uget(x_155, x_168); +lean_dec(x_155); +x_170 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_169); +lean_dec(x_169); +if (x_170 == 0) +{ +lean_object* x_171; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; size_t x_205; size_t x_206; size_t x_207; lean_object* x_208; uint8_t x_209; +x_194 = lean_st_ref_take(x_2, x_154); +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_ctor_get(x_195, 2); +lean_inc(x_196); +x_197 = lean_ctor_get(x_194, 1); +lean_inc(x_197); +lean_dec(x_194); +x_198 = lean_ctor_get(x_195, 0); +lean_inc(x_198); +x_199 = lean_ctor_get(x_195, 1); +lean_inc(x_199); +if (lean_is_exclusive(x_195)) { + lean_ctor_release(x_195, 0); + lean_ctor_release(x_195, 1); + lean_ctor_release(x_195, 2); + x_200 = x_195; +} else { + lean_dec_ref(x_195); + x_200 = lean_box(0); +} +x_201 = lean_ctor_get(x_196, 0); +lean_inc(x_201); +x_202 = lean_ctor_get(x_196, 1); +lean_inc(x_202); +if (lean_is_exclusive(x_196)) { + lean_ctor_release(x_196, 0); + lean_ctor_release(x_196, 1); + x_203 = x_196; +} else { + lean_dec_ref(x_196); + x_203 = lean_box(0); +} +x_204 = lean_array_get_size(x_202); +x_205 = lean_usize_of_nat(x_204); +lean_dec(x_204); +x_206 = lean_usize_sub(x_205, x_166); +x_207 = lean_usize_land(x_164, x_206); +x_208 = lean_array_uget(x_202, x_207); +x_209 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_208); +if (x_209 == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; +x_210 = lean_unsigned_to_nat(1u); +x_211 = lean_nat_add(x_201, x_210); +lean_dec(x_201); +x_212 = lean_box(0); +lean_inc(x_9); +x_213 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_213, 0, x_9); +lean_ctor_set(x_213, 1, x_212); +lean_ctor_set(x_213, 2, x_208); +x_214 = lean_array_uset(x_202, x_207, x_213); +x_215 = lean_unsigned_to_nat(4u); +x_216 = lean_nat_mul(x_211, x_215); +x_217 = lean_unsigned_to_nat(3u); +x_218 = lean_nat_div(x_216, x_217); +lean_dec(x_216); +x_219 = lean_array_get_size(x_214); +x_220 = lean_nat_dec_le(x_218, x_219); +lean_dec(x_219); +lean_dec(x_218); +if (x_220 == 0) +{ +lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; +x_221 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_214); +if (lean_is_scalar(x_203)) { + x_222 = lean_alloc_ctor(0, 2, 0); +} else { + x_222 = x_203; +} +lean_ctor_set(x_222, 0, x_211); +lean_ctor_set(x_222, 1, x_221); +if (lean_is_scalar(x_200)) { + x_223 = lean_alloc_ctor(0, 3, 0); +} else { + x_223 = x_200; +} +lean_ctor_set(x_223, 0, x_198); +lean_ctor_set(x_223, 1, x_199); +lean_ctor_set(x_223, 2, x_222); +x_224 = lean_st_ref_set(x_2, x_223, x_197); +x_225 = lean_ctor_get(x_224, 1); +lean_inc(x_225); +lean_dec(x_224); +x_171 = x_225; +goto block_193; +} +else +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +if (lean_is_scalar(x_203)) { + x_226 = lean_alloc_ctor(0, 2, 0); +} else { + x_226 = x_203; +} +lean_ctor_set(x_226, 0, x_211); +lean_ctor_set(x_226, 1, x_214); +if (lean_is_scalar(x_200)) { + x_227 = lean_alloc_ctor(0, 3, 0); +} else { + x_227 = x_200; +} +lean_ctor_set(x_227, 0, x_198); +lean_ctor_set(x_227, 1, x_199); +lean_ctor_set(x_227, 2, x_226); +x_228 = lean_st_ref_set(x_2, x_227, x_197); +x_229 = lean_ctor_get(x_228, 1); +lean_inc(x_229); +lean_dec(x_228); +x_171 = x_229; +goto block_193; +} +} +else +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; +lean_dec(x_208); +if (lean_is_scalar(x_203)) { + x_230 = lean_alloc_ctor(0, 2, 0); +} else { + x_230 = x_203; +} +lean_ctor_set(x_230, 0, x_201); +lean_ctor_set(x_230, 1, x_202); +if (lean_is_scalar(x_200)) { + x_231 = lean_alloc_ctor(0, 3, 0); +} else { + x_231 = x_200; +} +lean_ctor_set(x_231, 0, x_198); +lean_ctor_set(x_231, 1, x_199); +lean_ctor_set(x_231, 2, x_230); +x_232 = lean_st_ref_set(x_2, x_231, x_197); +x_233 = lean_ctor_get(x_232, 1); +lean_inc(x_233); +lean_dec(x_232); +x_171 = x_233; +goto block_193; +} +block_193: +{ +lean_object* x_172; lean_object* x_173; uint8_t x_174; +x_172 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1; +x_173 = l_Lean_Expr_cleanupAnnotations(x_9); +x_174 = l_Lean_Expr_isApp(x_173); +if (x_174 == 0) +{ +lean_object* x_175; lean_object* x_176; +lean_dec(x_173); +lean_dec(x_10); +lean_dec(x_8); +x_175 = lean_box(0); +x_176 = lean_apply_7(x_172, x_175, x_2, x_3, x_4, x_5, x_6, x_171); +return x_176; +} +else +{ +lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_177 = l_Lean_Expr_appArg(x_173, lean_box(0)); +x_178 = l_Lean_Expr_appFnCleanup(x_173, lean_box(0)); +x_179 = l_Lean_Expr_isApp(x_178); +if (x_179 == 0) +{ +lean_object* x_180; lean_object* x_181; +lean_dec(x_178); +lean_dec(x_177); +lean_dec(x_10); +lean_dec(x_8); +x_180 = lean_box(0); +x_181 = lean_apply_7(x_172, x_180, x_2, x_3, x_4, x_5, x_6, x_171); +return x_181; +} +else +{ +lean_object* x_182; lean_object* x_183; uint8_t x_184; +x_182 = l_Lean_Expr_appArg(x_178, lean_box(0)); +x_183 = l_Lean_Expr_appFnCleanup(x_178, lean_box(0)); +x_184 = l_Lean_Expr_isApp(x_183); +if (x_184 == 0) +{ +lean_object* x_185; lean_object* x_186; +lean_dec(x_183); +lean_dec(x_182); +lean_dec(x_177); +lean_dec(x_10); +lean_dec(x_8); +x_185 = lean_box(0); +x_186 = lean_apply_7(x_172, x_185, x_2, x_3, x_4, x_5, x_6, x_171); +return x_186; +} +else +{ +lean_object* x_187; lean_object* x_188; uint8_t x_189; +x_187 = l_Lean_Expr_appFnCleanup(x_183, lean_box(0)); +x_188 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2; +x_189 = l_Lean_Expr_isConstOf(x_187, x_188); +lean_dec(x_187); +if (x_189 == 0) +{ +lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_dec(x_177); +lean_dec(x_10); +lean_dec(x_8); +x_190 = lean_box(0); +x_191 = lean_apply_7(x_172, x_190, x_2, x_3, x_4, x_5, x_6, x_171); +return x_191; +} +else +{ +lean_object* x_192; +x_192 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4(x_10, x_8, x_182, x_177, x_2, x_3, x_4, x_5, x_6, x_171); +return x_192; +} +} +} +} +} +} +else +{ +lean_object* x_234; lean_object* x_235; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_234 = lean_box(0); +x_235 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_235, 0, x_234); +lean_ctor_set(x_235, 1, x_154); +return x_235; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; +} +else +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_1); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_11); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit(x_11, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_free_object(x_1); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_st_ref_take(x_2, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_array_push(x_20, x_11); +lean_ctor_set(x_17, 1, x_21); +x_22 = lean_st_ref_set(x_2, x_17, x_18); +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_1 = x_12; +x_7 = x_23; +goto _start; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_25 = lean_ctor_get(x_17, 0); +x_26 = lean_ctor_get(x_17, 1); +x_27 = lean_ctor_get(x_17, 2); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_17); +x_28 = lean_array_push(x_26, x_11); +x_29 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_29, 0, x_25); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set(x_29, 2, x_27); +x_30 = lean_st_ref_set(x_2, x_29, x_18); +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_1 = x_12; +x_7 = x_31; +goto _start; +} +} +else +{ +lean_object* x_33; lean_object* x_34; uint8_t x_35; +lean_dec(x_11); +x_33 = lean_ctor_get(x_14, 0); +lean_inc(x_33); +lean_dec(x_14); +x_34 = lean_ctor_get(x_13, 1); +lean_inc(x_34); +lean_dec(x_13); +x_35 = !lean_is_exclusive(x_33); +if (x_35 == 0) +{ +lean_object* x_36; +x_36 = lean_ctor_get(x_33, 1); +lean_ctor_set(x_1, 0, x_36); +lean_ctor_set_tag(x_33, 1); +lean_ctor_set(x_33, 1, x_1); +x_1 = x_33; +x_7 = x_34; +goto _start; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_33, 0); +x_39 = lean_ctor_get(x_33, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_33); +lean_ctor_set(x_1, 0, x_39); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_1); +x_1 = x_40; +x_7 = x_34; +goto _start; +} +} +} +else +{ +uint8_t x_42; +lean_free_object(x_1); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_42 = !lean_is_exclusive(x_13); +if (x_42 == 0) +{ +return x_13; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_13, 0); +x_44 = lean_ctor_get(x_13, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_13); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_1, 0); +x_47 = lean_ctor_get(x_1, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_46); +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit(x_46, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +if (lean_obj_tag(x_49) == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_st_ref_take(x_2, x_50); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_51, 1); +lean_inc(x_53); +lean_dec(x_51); +x_54 = lean_ctor_get(x_52, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_52, 1); +lean_inc(x_55); +x_56 = lean_ctor_get(x_52, 2); +lean_inc(x_56); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + lean_ctor_release(x_52, 2); + x_57 = x_52; +} else { + lean_dec_ref(x_52); + x_57 = lean_box(0); +} +x_58 = lean_array_push(x_55, x_46); +if (lean_is_scalar(x_57)) { + x_59 = lean_alloc_ctor(0, 3, 0); +} else { + x_59 = x_57; +} +lean_ctor_set(x_59, 0, x_54); +lean_ctor_set(x_59, 1, x_58); +lean_ctor_set(x_59, 2, x_56); +x_60 = lean_st_ref_set(x_2, x_59, x_53); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_1 = x_47; +x_7 = x_61; +goto _start; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +lean_dec(x_46); +x_63 = lean_ctor_get(x_49, 0); +lean_inc(x_63); +lean_dec(x_49); +x_64 = lean_ctor_get(x_48, 1); +lean_inc(x_64); +lean_dec(x_48); +x_65 = lean_ctor_get(x_63, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_67 = x_63; +} else { + lean_dec_ref(x_63); + x_67 = lean_box(0); +} +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_47); +if (lean_is_scalar(x_67)) { + x_69 = lean_alloc_ctor(1, 2, 0); +} else { + x_69 = x_67; + lean_ctor_set_tag(x_69, 1); +} +lean_ctor_set(x_69, 0, x_65); +lean_ctor_set(x_69, 1, x_68); +x_1 = x_69; +x_7 = x_64; +goto _start; +} +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_71 = lean_ctor_get(x_48, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_48, 1); +lean_inc(x_72); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_73 = x_48; +} else { + lean_dec_ref(x_48); + x_73 = lean_box(0); +} +if (lean_is_scalar(x_73)) { + x_74 = lean_alloc_ctor(1, 2, 0); +} else { + x_74 = x_73; +} +lean_ctor_set(x_74, 0, x_71); +lean_ctor_set(x_74, 1, x_72); +return x_74; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processFVar(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_3); +lean_inc(x_1); +x_8 = l_Lean_FVarId_getType(x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 2); +lean_inc(x_13); +lean_dec(x_12); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_array_get_size(x_15); +x_17 = l_Lean_Expr_hash(x_9); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +lean_dec(x_15); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_9, x_29); +lean_dec(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +lean_inc(x_3); +lean_inc(x_1); +x_31 = l_Lean_FVarId_getDecl(x_1, x_3, x_4, x_5, x_6, x_14); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_LocalDecl_userName(x_32); +lean_dec(x_32); +lean_inc(x_1); +x_35 = l_Lean_Expr_fvar___override(x_1); +x_36 = 0; +x_37 = 0; +x_38 = lean_alloc_ctor(0, 3, 2); +lean_ctor_set(x_38, 0, x_34); +lean_ctor_set(x_38, 1, x_9); +lean_ctor_set(x_38, 2, x_35); +lean_ctor_set_uint8(x_38, sizeof(void*)*3, x_36); +lean_ctor_set_uint8(x_38, sizeof(void*)*3 + 1, x_37); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit(x_38, x_2, x_3, x_4, x_5, x_6, x_33); +if (lean_obj_tag(x_39) == 0) +{ +lean_object* x_40; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +if (lean_obj_tag(x_40) == 0) +{ +uint8_t x_41; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_39); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_39, 0); +lean_dec(x_42); +x_43 = lean_box(0); +lean_ctor_set(x_39, 0, x_43); +return x_39; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_39, 1); +lean_inc(x_44); +lean_dec(x_39); +x_45 = lean_box(0); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_44); +return x_46; +} +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +x_47 = lean_ctor_get(x_40, 0); +lean_inc(x_47); +lean_dec(x_40); +x_48 = lean_ctor_get(x_39, 1); +lean_inc(x_48); +lean_dec(x_39); +x_49 = lean_ctor_get(x_47, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_47, 1); +lean_inc(x_50); +lean_dec(x_47); +x_51 = lean_st_ref_take(x_2, x_48); +x_52 = !lean_is_exclusive(x_51); +if (x_52 == 0) +{ +lean_object* x_53; uint8_t x_54; +x_53 = lean_ctor_get(x_51, 0); +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; +x_55 = lean_ctor_get(x_51, 1); +x_56 = lean_ctor_get(x_53, 0); +x_57 = lean_array_push(x_56, x_1); +lean_ctor_set(x_53, 0, x_57); +x_58 = lean_st_ref_set(x_2, x_53, x_55); +x_59 = !lean_is_exclusive(x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_60 = lean_ctor_get(x_58, 1); +x_61 = lean_ctor_get(x_58, 0); +lean_dec(x_61); +x_62 = lean_box(0); +lean_ctor_set_tag(x_58, 1); +lean_ctor_set(x_58, 1, x_62); +lean_ctor_set(x_58, 0, x_50); +lean_ctor_set_tag(x_51, 1); +lean_ctor_set(x_51, 1, x_58); +lean_ctor_set(x_51, 0, x_49); +x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(x_51, x_2, x_3, x_4, x_5, x_6, x_60); +return x_63; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_64 = lean_ctor_get(x_58, 1); +lean_inc(x_64); +lean_dec(x_58); +x_65 = lean_box(0); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_50); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set_tag(x_51, 1); +lean_ctor_set(x_51, 1, x_66); +lean_ctor_set(x_51, 0, x_49); +x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(x_51, x_2, x_3, x_4, x_5, x_6, x_64); +return x_67; +} +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_68 = lean_ctor_get(x_51, 1); +x_69 = lean_ctor_get(x_53, 0); +x_70 = lean_ctor_get(x_53, 1); +x_71 = lean_ctor_get(x_53, 2); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_53); +x_72 = lean_array_push(x_69, x_1); +x_73 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +lean_ctor_set(x_73, 2, x_71); +x_74 = lean_st_ref_set(x_2, x_73, x_68); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_76 = x_74; +} else { + lean_dec_ref(x_74); + x_76 = lean_box(0); +} +x_77 = lean_box(0); +if (lean_is_scalar(x_76)) { + x_78 = lean_alloc_ctor(1, 2, 0); +} else { + x_78 = x_76; + lean_ctor_set_tag(x_78, 1); +} +lean_ctor_set(x_78, 0, x_50); +lean_ctor_set(x_78, 1, x_77); +lean_ctor_set_tag(x_51, 1); +lean_ctor_set(x_51, 1, x_78); +lean_ctor_set(x_51, 0, x_49); +x_79 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(x_51, x_2, x_3, x_4, x_5, x_6, x_75); +return x_79; +} +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_80 = lean_ctor_get(x_51, 0); +x_81 = lean_ctor_get(x_51, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_51); +x_82 = lean_ctor_get(x_80, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_80, 1); +lean_inc(x_83); +x_84 = lean_ctor_get(x_80, 2); +lean_inc(x_84); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + lean_ctor_release(x_80, 2); + x_85 = x_80; +} else { + lean_dec_ref(x_80); + x_85 = lean_box(0); +} +x_86 = lean_array_push(x_82, x_1); +if (lean_is_scalar(x_85)) { + x_87 = lean_alloc_ctor(0, 3, 0); +} else { + x_87 = x_85; +} +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_83); +lean_ctor_set(x_87, 2, x_84); +x_88 = lean_st_ref_set(x_2, x_87, x_81); +x_89 = lean_ctor_get(x_88, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_88)) { + lean_ctor_release(x_88, 0); + lean_ctor_release(x_88, 1); + x_90 = x_88; +} else { + lean_dec_ref(x_88); + x_90 = lean_box(0); +} +x_91 = lean_box(0); +if (lean_is_scalar(x_90)) { + x_92 = lean_alloc_ctor(1, 2, 0); +} else { + x_92 = x_90; + lean_ctor_set_tag(x_92, 1); +} +lean_ctor_set(x_92, 0, x_50); +lean_ctor_set(x_92, 1, x_91); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_49); +lean_ctor_set(x_93, 1, x_92); +x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_splitAnds(x_93, x_2, x_3, x_4, x_5, x_6, x_89); +return x_94; +} +} +} +else +{ +uint8_t x_95; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_95 = !lean_is_exclusive(x_39); +if (x_95 == 0) +{ +return x_39; +} +else +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_39, 0); +x_97 = lean_ctor_get(x_39, 1); +lean_inc(x_97); +lean_inc(x_96); +lean_dec(x_39); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +return x_98; +} +} +} +else +{ +uint8_t x_99; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_99 = !lean_is_exclusive(x_31); +if (x_99 == 0) +{ +return x_31; +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_31, 0); +x_101 = lean_ctor_get(x_31, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_31); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; +} +} +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_103 = lean_st_ref_take(x_2, x_14); +x_104 = lean_ctor_get(x_103, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_103, 1); +lean_inc(x_105); +lean_dec(x_103); +x_106 = !lean_is_exclusive(x_104); +if (x_106 == 0) +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; +x_107 = lean_ctor_get(x_104, 0); +x_108 = lean_array_push(x_107, x_1); +lean_ctor_set(x_104, 0, x_108); +x_109 = lean_st_ref_set(x_2, x_104, x_105); +lean_dec(x_2); +x_110 = !lean_is_exclusive(x_109); +if (x_110 == 0) +{ +lean_object* x_111; lean_object* x_112; +x_111 = lean_ctor_get(x_109, 0); +lean_dec(x_111); +x_112 = lean_box(0); +lean_ctor_set(x_109, 0, x_112); +return x_109; +} +else +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_109, 1); +lean_inc(x_113); +lean_dec(x_109); +x_114 = lean_box(0); +x_115 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_113); +return x_115; +} +} +else +{ +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_116 = lean_ctor_get(x_104, 0); +x_117 = lean_ctor_get(x_104, 1); +x_118 = lean_ctor_get(x_104, 2); +lean_inc(x_118); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_104); +x_119 = lean_array_push(x_116, x_1); +x_120 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_120, 0, x_119); +lean_ctor_set(x_120, 1, x_117); +lean_ctor_set(x_120, 2, x_118); +x_121 = lean_st_ref_set(x_2, x_120, x_105); +lean_dec(x_2); +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + x_123 = x_121; +} else { + lean_dec_ref(x_121); + x_123 = lean_box(0); +} +x_124 = lean_box(0); +if (lean_is_scalar(x_123)) { + x_125 = lean_alloc_ctor(0, 2, 0); +} else { + x_125 = x_123; +} +lean_ctor_set(x_125, 0, x_124); +lean_ctor_set(x_125, 1, x_122); +return x_125; +} +} +} +else +{ +uint8_t x_126; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_126 = !lean_is_exclusive(x_8); +if (x_126 == 0) +{ +return x_8; +} +else +{ +lean_object* x_127; lean_object* x_128; lean_object* x_129; +x_127 = lean_ctor_get(x_8, 0); +x_128 = lean_ctor_get(x_8, 1); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_8); +x_129 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_129, 0, x_127); +lean_ctor_set(x_129, 1, x_128); +return x_129; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; +x_11 = lean_usize_dec_eq(x_2, x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_4); +x_12 = lean_array_uget(x_1, x_2); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processFVar(x_12, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; size_t x_16; size_t x_17; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = 1; +x_17 = lean_usize_add(x_2, x_16); +x_2 = x_17; +x_4 = x_14; +x_10 = x_15; +goto _start; +} +else +{ +uint8_t x_19; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_19 = !lean_is_exclusive(x_13); +if (x_19 == 0) +{ +return x_13; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_13, 0); +x_21 = lean_ctor_get(x_13, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_13); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +else +{ +lean_object* x_23; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_4); +lean_ctor_set(x_23, 1, x_10); +return x_23; +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_9 = lean_apply_6(x_1, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_apply_7(x_2, x_10, x_3, x_4, x_5, x_6, x_7, x_11); +return x_12; +} +else +{ +uint8_t x_13; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_13 = !lean_is_exclusive(x_9); +if (x_13 == 0) +{ +return x_9; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_9, 0); +x_15 = lean_ctor_get(x_9, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_9); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2___rarg), 8, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_apply_1(x_2, x_3); +x_10 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_9, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +return x_10; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +else +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_10); +if (x_15 == 0) +{ +return x_10; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_10, 0); +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_10); +x_18 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +return x_18; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3___rarg), 8, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; uint8_t x_10; +x_8 = lean_array_get_size(x_1); +x_9 = lean_unsigned_to_nat(0u); +x_10 = lean_nat_dec_lt(x_9, x_8); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_7); +return x_12; +} +else +{ +uint8_t x_13; +x_13 = lean_nat_dec_le(x_8, x_8); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_7); +return x_15; +} +else +{ +size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; +x_16 = 0; +x_17 = lean_usize_of_nat(x_8); +lean_dec(x_8); +x_18 = lean_box(0); +x_19 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1(x_1, x_16, x_17, x_18, x_2, x_3, x_4, x_5, x_6, x_7); +return x_19; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1___boxed), 7, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_inc(x_1); +x_8 = lean_alloc_closure((void*)(l_Lean_MVarId_getNondepPropHyps), 6, 1); +lean_closure_set(x_8, 0, x_1); +x_9 = lean_alloc_closure((void*)(l_StateRefT_x27_lift___rarg___boxed), 2, 1); +lean_closure_set(x_9, 0, x_8); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1; +x_11 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__2___rarg), 8, 2); +lean_closure_set(x_11, 0, x_9); +lean_closure_set(x_11, 1, x_10); +x_12 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__3___rarg(x_1, x_11, x_2, x_3, x_4, x_5, x_6, x_7); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_12 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_13 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___spec__1(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_1); +return x_8; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(10u); +x_2 = lean_unsigned_to_nat(1u); +x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2; +x_3 = lean_mk_array(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4; +x_3 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5; +x_10 = lean_st_mk_ref(x_9, x_8); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_11); +lean_inc(x_1); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal(x_1, x_11, x_4, x_5, x_6, x_7, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_st_ref_get(x_11, x_14); +lean_dec(x_11); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = l_Array_isEmpty___rarg(x_20); +if (x_21 == 0) +{ +lean_object* x_22; +lean_free_object(x_15); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_22 = l_Lean_MVarId_assertHypotheses(x_1, x_20, x_4, x_5, x_6, x_7, x_18); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Lean_MVarId_tryClearMany(x_25, x_19, x_4, x_5, x_6, x_7, x_24); +lean_dec(x_19); +if (lean_obj_tag(x_26) == 0) +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 0); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_26, 0, x_29); +return x_26; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_26, 0); +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_26); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_30); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; +} +} +else +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_26); +if (x_34 == 0) +{ +return x_26; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_26, 0); +x_36 = lean_ctor_get(x_26, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_26); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +uint8_t x_38; +lean_dec(x_19); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_38 = !lean_is_exclusive(x_22); +if (x_38 == 0) +{ +return x_22; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_22, 0); +x_40 = lean_ctor_get(x_22, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_22); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +lean_object* x_42; +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_1); +lean_ctor_set(x_15, 0, x_42); +return x_15; +} +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_43 = lean_ctor_get(x_15, 0); +x_44 = lean_ctor_get(x_15, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_15); +x_45 = lean_ctor_get(x_43, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_dec(x_43); +x_47 = l_Array_isEmpty___rarg(x_46); +if (x_47 == 0) +{ +lean_object* x_48; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_48 = l_Lean_MVarId_assertHypotheses(x_1, x_46, x_4, x_5, x_6, x_7, x_44); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l_Lean_MVarId_tryClearMany(x_51, x_45, x_4, x_5, x_6, x_7, x_50); +lean_dec(x_45); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_52, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_52, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_55 = x_52; +} else { + lean_dec_ref(x_52); + x_55 = lean_box(0); +} +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_53); +if (lean_is_scalar(x_55)) { + x_57 = lean_alloc_ctor(0, 2, 0); +} else { + x_57 = x_55; +} +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_54); +return x_57; +} +else +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_58 = lean_ctor_get(x_52, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_52, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_60 = x_52; +} else { + lean_dec_ref(x_52); + x_60 = lean_box(0); +} +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); +} else { + x_61 = x_60; +} +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; +} +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_45); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_62 = lean_ctor_get(x_48, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_48, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_64 = x_48; +} else { + lean_dec_ref(x_48); + x_64 = lean_box(0); +} +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(1, 2, 0); +} else { + x_65 = x_64; +} +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_63); +return x_65; +} +} +else +{ +lean_object* x_66; lean_object* x_67; +lean_dec(x_46); +lean_dec(x_45); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_66 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_66, 0, x_1); +x_67 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_44); +return x_67; +} +} +} +else +{ +uint8_t x_68; +lean_dec(x_11); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_68 = !lean_is_exclusive(x_13); +if (x_68 == 0) +{ +return x_13; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_13, 0); +x_70 = lean_ctor_get(x_13, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_13); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("andFlattening", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___boxed), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +lean_object* initialize_Std_Tactic_BVDecide_Normalize_Bool(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Assert(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_AndFlatten(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Tactic_BVDecide_Normalize_Bool(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Assert(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__13); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__14); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__15); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__16); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__17); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__18); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__19); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__20); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__1___closed__21); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__3___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_trySplit___lambda__4___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass_processGoal___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___elambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andFlatteningPass); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Basic.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Basic.c new file mode 100644 index 000000000000..2897476d7058 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Basic.c @@ -0,0 +1,5175 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic +// Imports: Lean.Meta.Basic Lean.Elab.Tactic.BVDecide.Frontend.Attr +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3; +double lean_float_div(double, double); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4; +size_t lean_uint64_to_usize(uint64_t); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); +lean_object* lean_mk_array(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___boxed(lean_object*, lean_object*); +lean_object* l_Lean_replaceRef(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_float_decLt(double, double); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1; +lean_object* lean_io_get_num_heartbeats(lean_object*); +lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_trace_profiler_useHeartbeats; +lean_object* l_Lean_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_getConfig___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(lean_object*); +size_t lean_usize_of_nat(lean_object*); +static lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1; +lean_object* lean_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_shift_right(uint64_t, uint64_t); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +lean_object* lean_nat_div(lean_object*, lean_object*); +lean_object* l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(lean_object*, lean_object*); +static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_PersistentArray_append___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run(lean_object*); +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_mk_ref(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, double, double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_io_mono_nanos_now(lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2; +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1; +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11; +uint8_t lean_name_eq(lean_object*, lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_getConfig(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); +extern lean_object* l_Lean_trace_profiler_threshold; +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static double l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofExpr(lean_object*); +lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Trace_0__Lean_addTraceNode___spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10; +double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9; +lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_xor(uint64_t, uint64_t); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2; +lean_object* lean_nat_mul(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1; +size_t lean_usize_sub(size_t, size_t); +lean_object* lean_array_mk(lean_object*); +lean_object* l_Lean_isTracingEnabledForCore(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uget(lean_object*, size_t); +static double l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4; +lean_object* l_Lean_Expr_fvar___override(lean_object*); +size_t lean_array_size(lean_object*); +extern lean_object* l_Lean_trace_profiler; +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2; +static lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3; +lean_object* lean_array_get_size(lean_object*); +uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1; +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2; +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1; +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +lean_object* l_Lean_MessageData_ofName(lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8; +size_t lean_usize_land(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +double lean_float_sub(double, double); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_getConfig(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_getConfig___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_getConfig(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_6, 2); +x_10 = l_Lean_isTracingEnabledForCore(x_1, x_9, x_8); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +return x_10; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +} +static double _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_10 = lean_ctor_get(x_7, 5); +x_11 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_5, x_6, x_7, x_8, x_9); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_st_ref_take(x_8, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 3); +lean_inc(x_16); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_18 = lean_ctor_get(x_14, 1); +x_19 = lean_ctor_get(x_14, 0); +lean_dec(x_19); +x_20 = !lean_is_exclusive(x_15); +if (x_20 == 0) +{ +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_15, 3); +lean_dec(x_21); +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +lean_object* x_23; double x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_23 = lean_ctor_get(x_16, 0); +x_24 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +x_25 = 0; +x_26 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_27 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_27, 0, x_1); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set_float(x_27, sizeof(void*)*2, x_24); +lean_ctor_set_float(x_27, sizeof(void*)*2 + 8, x_24); +lean_ctor_set_uint8(x_27, sizeof(void*)*2 + 16, x_25); +x_28 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3; +x_29 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_12); +lean_ctor_set(x_29, 2, x_28); +lean_inc(x_10); +lean_ctor_set(x_14, 1, x_29); +lean_ctor_set(x_14, 0, x_10); +x_30 = l_Lean_PersistentArray_push___rarg(x_23, x_14); +lean_ctor_set(x_16, 0, x_30); +x_31 = lean_st_ref_set(x_8, x_15, x_18); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_31, 0); +lean_dec(x_33); +x_34 = lean_box(0); +lean_ctor_set(x_31, 0, x_34); +return x_31; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_31, 1); +lean_inc(x_35); +lean_dec(x_31); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +return x_37; +} +} +else +{ +uint64_t x_38; lean_object* x_39; double x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_38 = lean_ctor_get_uint64(x_16, sizeof(void*)*1); +x_39 = lean_ctor_get(x_16, 0); +lean_inc(x_39); +lean_dec(x_16); +x_40 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +x_41 = 0; +x_42 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_43 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_43, 0, x_1); +lean_ctor_set(x_43, 1, x_42); +lean_ctor_set_float(x_43, sizeof(void*)*2, x_40); +lean_ctor_set_float(x_43, sizeof(void*)*2 + 8, x_40); +lean_ctor_set_uint8(x_43, sizeof(void*)*2 + 16, x_41); +x_44 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3; +x_45 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_12); +lean_ctor_set(x_45, 2, x_44); +lean_inc(x_10); +lean_ctor_set(x_14, 1, x_45); +lean_ctor_set(x_14, 0, x_10); +x_46 = l_Lean_PersistentArray_push___rarg(x_39, x_14); +x_47 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set_uint64(x_47, sizeof(void*)*1, x_38); +lean_ctor_set(x_15, 3, x_47); +x_48 = lean_st_ref_set(x_8, x_15, x_18); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_50 = x_48; +} else { + lean_dec_ref(x_48); + x_50 = lean_box(0); +} +x_51 = lean_box(0); +if (lean_is_scalar(x_50)) { + x_52 = lean_alloc_ctor(0, 2, 0); +} else { + x_52 = x_50; +} +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_49); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint64_t x_60; lean_object* x_61; lean_object* x_62; double x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_53 = lean_ctor_get(x_15, 0); +x_54 = lean_ctor_get(x_15, 1); +x_55 = lean_ctor_get(x_15, 2); +x_56 = lean_ctor_get(x_15, 4); +x_57 = lean_ctor_get(x_15, 5); +x_58 = lean_ctor_get(x_15, 6); +x_59 = lean_ctor_get(x_15, 7); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_15); +x_60 = lean_ctor_get_uint64(x_16, sizeof(void*)*1); +x_61 = lean_ctor_get(x_16, 0); +lean_inc(x_61); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + x_62 = x_16; +} else { + lean_dec_ref(x_16); + x_62 = lean_box(0); +} +x_63 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +x_64 = 0; +x_65 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_66 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_66, 0, x_1); +lean_ctor_set(x_66, 1, x_65); +lean_ctor_set_float(x_66, sizeof(void*)*2, x_63); +lean_ctor_set_float(x_66, sizeof(void*)*2 + 8, x_63); +lean_ctor_set_uint8(x_66, sizeof(void*)*2 + 16, x_64); +x_67 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3; +x_68 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_12); +lean_ctor_set(x_68, 2, x_67); +lean_inc(x_10); +lean_ctor_set(x_14, 1, x_68); +lean_ctor_set(x_14, 0, x_10); +x_69 = l_Lean_PersistentArray_push___rarg(x_61, x_14); +if (lean_is_scalar(x_62)) { + x_70 = lean_alloc_ctor(0, 1, 8); +} else { + x_70 = x_62; +} +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set_uint64(x_70, sizeof(void*)*1, x_60); +x_71 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_71, 0, x_53); +lean_ctor_set(x_71, 1, x_54); +lean_ctor_set(x_71, 2, x_55); +lean_ctor_set(x_71, 3, x_70); +lean_ctor_set(x_71, 4, x_56); +lean_ctor_set(x_71, 5, x_57); +lean_ctor_set(x_71, 6, x_58); +lean_ctor_set(x_71, 7, x_59); +x_72 = lean_st_ref_set(x_8, x_71, x_18); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; +} else { + lean_dec_ref(x_72); + x_74 = lean_box(0); +} +x_75 = lean_box(0); +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 2, 0); +} else { + x_76 = x_74; +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_73); +return x_76; +} +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint64_t x_86; lean_object* x_87; lean_object* x_88; double x_89; uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_77 = lean_ctor_get(x_14, 1); +lean_inc(x_77); +lean_dec(x_14); +x_78 = lean_ctor_get(x_15, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_15, 1); +lean_inc(x_79); +x_80 = lean_ctor_get(x_15, 2); +lean_inc(x_80); +x_81 = lean_ctor_get(x_15, 4); +lean_inc(x_81); +x_82 = lean_ctor_get(x_15, 5); +lean_inc(x_82); +x_83 = lean_ctor_get(x_15, 6); +lean_inc(x_83); +x_84 = lean_ctor_get(x_15, 7); +lean_inc(x_84); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + lean_ctor_release(x_15, 2); + lean_ctor_release(x_15, 3); + lean_ctor_release(x_15, 4); + lean_ctor_release(x_15, 5); + lean_ctor_release(x_15, 6); + lean_ctor_release(x_15, 7); + x_85 = x_15; +} else { + lean_dec_ref(x_15); + x_85 = lean_box(0); +} +x_86 = lean_ctor_get_uint64(x_16, sizeof(void*)*1); +x_87 = lean_ctor_get(x_16, 0); +lean_inc(x_87); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + x_88 = x_16; +} else { + lean_dec_ref(x_16); + x_88 = lean_box(0); +} +x_89 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +x_90 = 0; +x_91 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_92 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_92, 0, x_1); +lean_ctor_set(x_92, 1, x_91); +lean_ctor_set_float(x_92, sizeof(void*)*2, x_89); +lean_ctor_set_float(x_92, sizeof(void*)*2 + 8, x_89); +lean_ctor_set_uint8(x_92, sizeof(void*)*2 + 16, x_90); +x_93 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3; +x_94 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_12); +lean_ctor_set(x_94, 2, x_93); +lean_inc(x_10); +x_95 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_95, 0, x_10); +lean_ctor_set(x_95, 1, x_94); +x_96 = l_Lean_PersistentArray_push___rarg(x_87, x_95); +if (lean_is_scalar(x_88)) { + x_97 = lean_alloc_ctor(0, 1, 8); +} else { + x_97 = x_88; +} +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set_uint64(x_97, sizeof(void*)*1, x_86); +if (lean_is_scalar(x_85)) { + x_98 = lean_alloc_ctor(0, 8, 0); +} else { + x_98 = x_85; +} +lean_ctor_set(x_98, 0, x_78); +lean_ctor_set(x_98, 1, x_79); +lean_ctor_set(x_98, 2, x_80); +lean_ctor_set(x_98, 3, x_97); +lean_ctor_set(x_98, 4, x_81); +lean_ctor_set(x_98, 5, x_82); +lean_ctor_set(x_98, 6, x_83); +lean_ctor_set(x_98, 7, x_84); +x_99 = lean_st_ref_set(x_8, x_98, x_77); +x_100 = lean_ctor_get(x_99, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_101 = x_99; +} else { + lean_dec_ref(x_99); + x_101 = lean_box(0); +} +x_102 = lean_box(0); +if (lean_is_scalar(x_101)) { + x_103 = lean_alloc_ctor(0, 2, 0); +} else { + x_103 = x_101; +} +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_100); +return x_103; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Meta", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bv", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" was already rewritten\? ", 24, 24); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("false", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; uint8_t x_10; +x_9 = lean_st_ref_get(x_3, x_8); +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_ctor_get(x_9, 1); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_13, x_2, x_3, x_4, x_5, x_6, x_7, x_12); +x_15 = !lean_is_exclusive(x_11); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_11, 1); +x_17 = lean_ctor_get(x_11, 0); +lean_dec(x_17); +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; uint64_t x_26; uint64_t x_27; uint64_t x_28; size_t x_29; size_t x_30; size_t x_31; size_t x_32; size_t x_33; lean_object* x_34; uint8_t x_35; uint8_t x_36; +x_19 = lean_ctor_get(x_14, 0); +x_20 = lean_ctor_get(x_14, 1); +x_21 = lean_array_get_size(x_16); +x_22 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_23 = 32; +x_24 = lean_uint64_shift_right(x_22, x_23); +x_25 = lean_uint64_xor(x_22, x_24); +x_26 = 16; +x_27 = lean_uint64_shift_right(x_25, x_26); +x_28 = lean_uint64_xor(x_25, x_27); +x_29 = lean_uint64_to_usize(x_28); +x_30 = lean_usize_of_nat(x_21); +lean_dec(x_21); +x_31 = 1; +x_32 = lean_usize_sub(x_30, x_31); +x_33 = lean_usize_land(x_29, x_32); +x_34 = lean_array_uget(x_16, x_33); +lean_dec(x_16); +x_35 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_34); +lean_dec(x_34); +x_36 = lean_unbox(x_19); +lean_dec(x_19); +if (x_36 == 0) +{ +lean_object* x_37; +lean_free_object(x_11); +lean_free_object(x_9); +lean_dec(x_1); +x_37 = lean_box(x_35); +lean_ctor_set(x_14, 0, x_37); +return x_14; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +lean_free_object(x_14); +x_38 = l_Lean_Expr_fvar___override(x_1); +x_39 = l_Lean_MessageData_ofExpr(x_38); +x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_39); +lean_ctor_set(x_11, 0, x_40); +x_41 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7; +lean_ctor_set_tag(x_9, 7); +lean_ctor_set(x_9, 1, x_41); +if (x_35 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_9); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_40); +x_45 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_44, x_2, x_3, x_4, x_5, x_6, x_7, x_20); +x_46 = !lean_is_exclusive(x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_45, 0); +lean_dec(x_47); +x_48 = lean_box(x_35); +lean_ctor_set(x_45, 0, x_48); +return x_45; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_45, 1); +lean_inc(x_49); +lean_dec(x_45); +x_50 = lean_box(x_35); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_49); +return x_51; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_52 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_9); +lean_ctor_set(x_53, 1, x_52); +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_40); +x_55 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_54, x_2, x_3, x_4, x_5, x_6, x_7, x_20); +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; +x_57 = lean_ctor_get(x_55, 0); +lean_dec(x_57); +x_58 = lean_box(x_35); +lean_ctor_set(x_55, 0, x_58); +return x_55; +} +else +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_55, 1); +lean_inc(x_59); +lean_dec(x_55); +x_60 = lean_box(x_35); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +return x_61; +} +} +} +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; uint64_t x_68; uint64_t x_69; uint64_t x_70; uint64_t x_71; size_t x_72; size_t x_73; size_t x_74; size_t x_75; size_t x_76; lean_object* x_77; uint8_t x_78; uint8_t x_79; +x_62 = lean_ctor_get(x_14, 0); +x_63 = lean_ctor_get(x_14, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_14); +x_64 = lean_array_get_size(x_16); +x_65 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_66 = 32; +x_67 = lean_uint64_shift_right(x_65, x_66); +x_68 = lean_uint64_xor(x_65, x_67); +x_69 = 16; +x_70 = lean_uint64_shift_right(x_68, x_69); +x_71 = lean_uint64_xor(x_68, x_70); +x_72 = lean_uint64_to_usize(x_71); +x_73 = lean_usize_of_nat(x_64); +lean_dec(x_64); +x_74 = 1; +x_75 = lean_usize_sub(x_73, x_74); +x_76 = lean_usize_land(x_72, x_75); +x_77 = lean_array_uget(x_16, x_76); +lean_dec(x_16); +x_78 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_77); +lean_dec(x_77); +x_79 = lean_unbox(x_62); +lean_dec(x_62); +if (x_79 == 0) +{ +lean_object* x_80; lean_object* x_81; +lean_free_object(x_11); +lean_free_object(x_9); +lean_dec(x_1); +x_80 = lean_box(x_78); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_82 = l_Lean_Expr_fvar___override(x_1); +x_83 = l_Lean_MessageData_ofExpr(x_82); +x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_83); +lean_ctor_set(x_11, 0, x_84); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7; +lean_ctor_set_tag(x_9, 7); +lean_ctor_set(x_9, 1, x_85); +if (x_78 == 0) +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_86 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10; +x_87 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_87, 0, x_9); +lean_ctor_set(x_87, 1, x_86); +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_87); +lean_ctor_set(x_88, 1, x_84); +x_89 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_88, x_2, x_3, x_4, x_5, x_6, x_7, x_63); +x_90 = lean_ctor_get(x_89, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_91 = x_89; +} else { + lean_dec_ref(x_89); + x_91 = lean_box(0); +} +x_92 = lean_box(x_78); +if (lean_is_scalar(x_91)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_91; +} +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_90); +return x_93; +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_94 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13; +x_95 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_95, 0, x_9); +lean_ctor_set(x_95, 1, x_94); +x_96 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_84); +x_97 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_96, x_2, x_3, x_4, x_5, x_6, x_7, x_63); +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_99 = x_97; +} else { + lean_dec_ref(x_97); + x_99 = lean_box(0); +} +x_100 = lean_box(x_78); +if (lean_is_scalar(x_99)) { + x_101 = lean_alloc_ctor(0, 2, 0); +} else { + x_101 = x_99; +} +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_98); +return x_101; +} +} +} +} +else +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint64_t x_107; uint64_t x_108; uint64_t x_109; uint64_t x_110; uint64_t x_111; uint64_t x_112; uint64_t x_113; size_t x_114; size_t x_115; size_t x_116; size_t x_117; size_t x_118; lean_object* x_119; uint8_t x_120; uint8_t x_121; +x_102 = lean_ctor_get(x_11, 1); +lean_inc(x_102); +lean_dec(x_11); +x_103 = lean_ctor_get(x_14, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_14, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_14)) { + lean_ctor_release(x_14, 0); + lean_ctor_release(x_14, 1); + x_105 = x_14; +} else { + lean_dec_ref(x_14); + x_105 = lean_box(0); +} +x_106 = lean_array_get_size(x_102); +x_107 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_108 = 32; +x_109 = lean_uint64_shift_right(x_107, x_108); +x_110 = lean_uint64_xor(x_107, x_109); +x_111 = 16; +x_112 = lean_uint64_shift_right(x_110, x_111); +x_113 = lean_uint64_xor(x_110, x_112); +x_114 = lean_uint64_to_usize(x_113); +x_115 = lean_usize_of_nat(x_106); +lean_dec(x_106); +x_116 = 1; +x_117 = lean_usize_sub(x_115, x_116); +x_118 = lean_usize_land(x_114, x_117); +x_119 = lean_array_uget(x_102, x_118); +lean_dec(x_102); +x_120 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_119); +lean_dec(x_119); +x_121 = lean_unbox(x_103); +lean_dec(x_103); +if (x_121 == 0) +{ +lean_object* x_122; lean_object* x_123; +lean_free_object(x_9); +lean_dec(x_1); +x_122 = lean_box(x_120); +if (lean_is_scalar(x_105)) { + x_123 = lean_alloc_ctor(0, 2, 0); +} else { + x_123 = x_105; +} +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set(x_123, 1, x_104); +return x_123; +} +else +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_105); +x_124 = l_Lean_Expr_fvar___override(x_1); +x_125 = l_Lean_MessageData_ofExpr(x_124); +x_126 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +x_127 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_127, 1, x_125); +x_128 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7; +lean_ctor_set_tag(x_9, 7); +lean_ctor_set(x_9, 1, x_128); +lean_ctor_set(x_9, 0, x_127); +if (x_120 == 0) +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_129 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10; +x_130 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_130, 0, x_9); +lean_ctor_set(x_130, 1, x_129); +x_131 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_126); +x_132 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_131, x_2, x_3, x_4, x_5, x_6, x_7, x_104); +x_133 = lean_ctor_get(x_132, 1); +lean_inc(x_133); +if (lean_is_exclusive(x_132)) { + lean_ctor_release(x_132, 0); + lean_ctor_release(x_132, 1); + x_134 = x_132; +} else { + lean_dec_ref(x_132); + x_134 = lean_box(0); +} +x_135 = lean_box(x_120); +if (lean_is_scalar(x_134)) { + x_136 = lean_alloc_ctor(0, 2, 0); +} else { + x_136 = x_134; +} +lean_ctor_set(x_136, 0, x_135); +lean_ctor_set(x_136, 1, x_133); +return x_136; +} +else +{ +lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_137 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13; +x_138 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_138, 0, x_9); +lean_ctor_set(x_138, 1, x_137); +x_139 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_139, 1, x_126); +x_140 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_139, x_2, x_3, x_4, x_5, x_6, x_7, x_104); +x_141 = lean_ctor_get(x_140, 1); +lean_inc(x_141); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_142 = x_140; +} else { + lean_dec_ref(x_140); + x_142 = lean_box(0); +} +x_143 = lean_box(x_120); +if (lean_is_scalar(x_142)) { + x_144 = lean_alloc_ctor(0, 2, 0); +} else { + x_144 = x_142; +} +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_141); +return x_144; +} +} +} +} +else +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; uint64_t x_155; uint64_t x_156; uint64_t x_157; uint64_t x_158; uint64_t x_159; uint64_t x_160; uint64_t x_161; size_t x_162; size_t x_163; size_t x_164; size_t x_165; size_t x_166; lean_object* x_167; uint8_t x_168; uint8_t x_169; +x_145 = lean_ctor_get(x_9, 0); +x_146 = lean_ctor_get(x_9, 1); +lean_inc(x_146); +lean_inc(x_145); +lean_dec(x_9); +x_147 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_148 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_147, x_2, x_3, x_4, x_5, x_6, x_7, x_146); +x_149 = lean_ctor_get(x_145, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_145)) { + lean_ctor_release(x_145, 0); + lean_ctor_release(x_145, 1); + x_150 = x_145; +} else { + lean_dec_ref(x_145); + x_150 = lean_box(0); +} +x_151 = lean_ctor_get(x_148, 0); +lean_inc(x_151); +x_152 = lean_ctor_get(x_148, 1); +lean_inc(x_152); +if (lean_is_exclusive(x_148)) { + lean_ctor_release(x_148, 0); + lean_ctor_release(x_148, 1); + x_153 = x_148; +} else { + lean_dec_ref(x_148); + x_153 = lean_box(0); +} +x_154 = lean_array_get_size(x_149); +x_155 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_156 = 32; +x_157 = lean_uint64_shift_right(x_155, x_156); +x_158 = lean_uint64_xor(x_155, x_157); +x_159 = 16; +x_160 = lean_uint64_shift_right(x_158, x_159); +x_161 = lean_uint64_xor(x_158, x_160); +x_162 = lean_uint64_to_usize(x_161); +x_163 = lean_usize_of_nat(x_154); +lean_dec(x_154); +x_164 = 1; +x_165 = lean_usize_sub(x_163, x_164); +x_166 = lean_usize_land(x_162, x_165); +x_167 = lean_array_uget(x_149, x_166); +lean_dec(x_149); +x_168 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_167); +lean_dec(x_167); +x_169 = lean_unbox(x_151); +lean_dec(x_151); +if (x_169 == 0) +{ +lean_object* x_170; lean_object* x_171; +lean_dec(x_150); +lean_dec(x_1); +x_170 = lean_box(x_168); +if (lean_is_scalar(x_153)) { + x_171 = lean_alloc_ctor(0, 2, 0); +} else { + x_171 = x_153; +} +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_152); +return x_171; +} +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_dec(x_153); +x_172 = l_Lean_Expr_fvar___override(x_1); +x_173 = l_Lean_MessageData_ofExpr(x_172); +x_174 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +if (lean_is_scalar(x_150)) { + x_175 = lean_alloc_ctor(7, 2, 0); +} else { + x_175 = x_150; + lean_ctor_set_tag(x_175, 7); +} +lean_ctor_set(x_175, 0, x_174); +lean_ctor_set(x_175, 1, x_173); +x_176 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7; +x_177 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_177, 0, x_175); +lean_ctor_set(x_177, 1, x_176); +if (x_168 == 0) +{ +lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; +x_178 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10; +x_179 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +x_180 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_180, 0, x_179); +lean_ctor_set(x_180, 1, x_174); +x_181 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_147, x_180, x_2, x_3, x_4, x_5, x_6, x_7, x_152); +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +if (lean_is_exclusive(x_181)) { + lean_ctor_release(x_181, 0); + lean_ctor_release(x_181, 1); + x_183 = x_181; +} else { + lean_dec_ref(x_181); + x_183 = lean_box(0); +} +x_184 = lean_box(x_168); +if (lean_is_scalar(x_183)) { + x_185 = lean_alloc_ctor(0, 2, 0); +} else { + x_185 = x_183; +} +lean_ctor_set(x_185, 0, x_184); +lean_ctor_set(x_185, 1, x_182); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; +x_186 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13; +x_187 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_187, 0, x_177); +lean_ctor_set(x_187, 1, x_186); +x_188 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_188, 0, x_187); +lean_ctor_set(x_188, 1, x_174); +x_189 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_147, x_188, x_2, x_3, x_4, x_5, x_6, x_7, x_152); +x_190 = lean_ctor_get(x_189, 1); +lean_inc(x_190); +if (lean_is_exclusive(x_189)) { + lean_ctor_release(x_189, 0); + lean_ctor_release(x_189, 1); + x_191 = x_189; +} else { + lean_dec_ref(x_189); + x_191 = lean_box(0); +} +x_192 = lean_box(x_168); +if (lean_is_scalar(x_191)) { + x_193 = lean_alloc_ctor(0, 2, 0); +} else { + x_193 = x_191; +} +lean_ctor_set(x_193, 0, x_192); +lean_ctor_set(x_193, 1, x_190); +return x_193; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_1); +lean_dec(x_1); +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___lambda__1(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_st_ref_take(x_4, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_11, 0); +x_15 = lean_ctor_get(x_11, 1); +x_16 = lean_array_get_size(x_15); +x_17 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_14, x_31); +lean_dec(x_14); +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_1); +lean_ctor_set(x_34, 1, x_33); +lean_ctor_set(x_34, 2, x_29); +x_35 = lean_array_uset(x_15, x_28, x_34); +x_36 = lean_unsigned_to_nat(4u); +x_37 = lean_nat_mul(x_32, x_36); +x_38 = lean_unsigned_to_nat(3u); +x_39 = lean_nat_div(x_37, x_38); +lean_dec(x_37); +x_40 = lean_array_get_size(x_35); +x_41 = lean_nat_dec_le(x_39, x_40); +lean_dec(x_40); +lean_dec(x_39); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_35); +lean_ctor_set(x_11, 1, x_42); +lean_ctor_set(x_11, 0, x_32); +x_43 = lean_st_ref_set(x_4, x_11, x_12); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +lean_ctor_set(x_43, 0, x_33); +return x_43; +} +else +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_dec(x_43); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_33); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} +} +else +{ +lean_object* x_48; uint8_t x_49; +lean_ctor_set(x_11, 1, x_35); +lean_ctor_set(x_11, 0, x_32); +x_48 = lean_st_ref_set(x_4, x_11, x_12); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; +x_50 = lean_ctor_get(x_48, 0); +lean_dec(x_50); +lean_ctor_set(x_48, 0, x_33); +return x_48; +} +else +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_48, 1); +lean_inc(x_51); +lean_dec(x_48); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_33); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +lean_object* x_53; uint8_t x_54; +lean_dec(x_29); +lean_dec(x_1); +x_53 = lean_st_ref_set(x_4, x_11, x_12); +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_53, 0); +lean_dec(x_55); +x_56 = lean_box(0); +lean_ctor_set(x_53, 0, x_56); +return x_53; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_53, 1); +lean_inc(x_57); +lean_dec(x_53); +x_58 = lean_box(0); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_57); +return x_59; +} +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; uint64_t x_68; uint64_t x_69; size_t x_70; size_t x_71; size_t x_72; size_t x_73; size_t x_74; lean_object* x_75; uint8_t x_76; +x_60 = lean_ctor_get(x_11, 0); +x_61 = lean_ctor_get(x_11, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_11); +x_62 = lean_array_get_size(x_61); +x_63 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_64 = 32; +x_65 = lean_uint64_shift_right(x_63, x_64); +x_66 = lean_uint64_xor(x_63, x_65); +x_67 = 16; +x_68 = lean_uint64_shift_right(x_66, x_67); +x_69 = lean_uint64_xor(x_66, x_68); +x_70 = lean_uint64_to_usize(x_69); +x_71 = lean_usize_of_nat(x_62); +lean_dec(x_62); +x_72 = 1; +x_73 = lean_usize_sub(x_71, x_72); +x_74 = lean_usize_land(x_70, x_73); +x_75 = lean_array_uget(x_61, x_74); +x_76 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_75); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_77 = lean_unsigned_to_nat(1u); +x_78 = lean_nat_add(x_60, x_77); +lean_dec(x_60); +x_79 = lean_box(0); +x_80 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_80, 0, x_1); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_75); +x_81 = lean_array_uset(x_61, x_74, x_80); +x_82 = lean_unsigned_to_nat(4u); +x_83 = lean_nat_mul(x_78, x_82); +x_84 = lean_unsigned_to_nat(3u); +x_85 = lean_nat_div(x_83, x_84); +lean_dec(x_83); +x_86 = lean_array_get_size(x_81); +x_87 = lean_nat_dec_le(x_85, x_86); +lean_dec(x_86); +lean_dec(x_85); +if (x_87 == 0) +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_88 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_81); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_78); +lean_ctor_set(x_89, 1, x_88); +x_90 = lean_st_ref_set(x_4, x_89, x_12); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_92 = x_90; +} else { + lean_dec_ref(x_90); + x_92 = lean_box(0); +} +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_92; +} +lean_ctor_set(x_93, 0, x_79); +lean_ctor_set(x_93, 1, x_91); +return x_93; +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_78); +lean_ctor_set(x_94, 1, x_81); +x_95 = lean_st_ref_set(x_4, x_94, x_12); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_95)) { + lean_ctor_release(x_95, 0); + lean_ctor_release(x_95, 1); + x_97 = x_95; +} else { + lean_dec_ref(x_95); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(0, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_79); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +lean_dec(x_75); +lean_dec(x_1); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_60); +lean_ctor_set(x_99, 1, x_61); +x_100 = lean_st_ref_set(x_4, x_99, x_12); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_102 = x_100; +} else { + lean_dec_ref(x_100); + x_102 = lean_box(0); +} +x_103 = lean_box(0); +if (lean_is_scalar(x_102)) { + x_104 = lean_alloc_ctor(0, 2, 0); +} else { + x_104 = x_102; +} +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_101); +return x_104; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Adding ", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" to the rewritten set", 21, 21); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_10 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = lean_box(0); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_13); +return x_15; +} +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_10); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_17 = lean_ctor_get(x_10, 1); +x_18 = lean_ctor_get(x_10, 0); +lean_dec(x_18); +lean_inc(x_1); +x_19 = l_Lean_Expr_fvar___override(x_1); +x_20 = l_Lean_MessageData_ofExpr(x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2; +lean_ctor_set_tag(x_10, 7); +lean_ctor_set(x_10, 1, x_20); +lean_ctor_set(x_10, 0, x_21); +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4; +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_10); +lean_ctor_set(x_23, 1, x_22); +x_24 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_9, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_17); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(x_1, x_25, x_2, x_3, x_4, x_5, x_6, x_7, x_26); +lean_dec(x_25); +return x_27; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_28 = lean_ctor_get(x_10, 1); +lean_inc(x_28); +lean_dec(x_10); +lean_inc(x_1); +x_29 = l_Lean_Expr_fvar___override(x_1); +x_30 = l_Lean_MessageData_ofExpr(x_29); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_9, x_34, x_2, x_3, x_4, x_5, x_6, x_7, x_28); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(x_1, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_37); +lean_dec(x_36); +return x_38; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_9 = l_Lean_MVarId_getNondepPropHyps(x_2, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_array_get_size(x_10); +lean_dec(x_10); +x_13 = lean_unsigned_to_nat(4u); +x_14 = lean_nat_mul(x_12, x_13); +lean_dec(x_12); +x_15 = lean_unsigned_to_nat(3u); +x_16 = lean_nat_div(x_14, x_15); +lean_dec(x_14); +x_17 = lean_unsigned_to_nat(1u); +x_18 = l_Nat_nextPowerOfTwo_go(x_16, x_17, lean_box(0)); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_mk_array(x_18, x_19); +x_21 = lean_unsigned_to_nat(0u); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +x_23 = lean_st_mk_ref(x_22, x_11); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_24); +x_26 = lean_apply_7(x_3, x_1, x_24, x_4, x_5, x_6, x_7, x_25); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_st_ref_get(x_24, x_28); +lean_dec(x_24); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_dec(x_31); +lean_ctor_set(x_29, 0, x_27); +return x_29; +} +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_27); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +else +{ +uint8_t x_34; +lean_dec(x_24); +x_34 = !lean_is_exclusive(x_26); +if (x_34 == 0) +{ +return x_26; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_26, 0); +x_36 = lean_ctor_get(x_26, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_26); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +uint8_t x_38; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_38 = !lean_is_exclusive(x_9); +if (x_38 == 0) +{ +return x_9; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_9, 0); +x_40 = lean_ctor_get(x_9, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_9); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_run___rarg), 8, 0); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(32u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3() { +_start: +{ +size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = 5; +x_2 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2; +x_3 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_4); +lean_ctor_set(x_5, 3, x_4); +lean_ctor_set_usize(x_5, 4, x_1); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_3 = lean_st_ref_get(x_1, x_2); +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +x_5 = lean_ctor_get(x_3, 1); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_4, 3); +lean_inc(x_6); +lean_dec(x_4); +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_st_ref_take(x_1, x_5); +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_9, 3); +lean_inc(x_10); +x_11 = lean_ctor_get(x_8, 1); +lean_inc(x_11); +lean_dec(x_8); +x_12 = !lean_is_exclusive(x_9); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_9, 3); +lean_dec(x_13); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_10, 0); +lean_dec(x_15); +x_16 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3; +lean_ctor_set(x_10, 0, x_16); +x_17 = lean_st_ref_set(x_1, x_9, x_11); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +lean_ctor_set(x_17, 0, x_7); +return x_17; +} +else +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_7); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +else +{ +uint64_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_22 = lean_ctor_get_uint64(x_10, sizeof(void*)*1); +lean_dec(x_10); +x_23 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3; +x_24 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set_uint64(x_24, sizeof(void*)*1, x_22); +lean_ctor_set(x_9, 3, x_24); +x_25 = lean_st_ref_set(x_1, x_9, x_11); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +if (lean_is_exclusive(x_25)) { + lean_ctor_release(x_25, 0); + lean_ctor_release(x_25, 1); + x_27 = x_25; +} else { + lean_dec_ref(x_25); + x_27 = lean_box(0); +} +if (lean_is_scalar(x_27)) { + x_28 = lean_alloc_ctor(0, 2, 0); +} else { + x_28 = x_27; +} +lean_ctor_set(x_28, 0, x_7); +lean_ctor_set(x_28, 1, x_26); +return x_28; +} +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint64_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_29 = lean_ctor_get(x_9, 0); +x_30 = lean_ctor_get(x_9, 1); +x_31 = lean_ctor_get(x_9, 2); +x_32 = lean_ctor_get(x_9, 4); +x_33 = lean_ctor_get(x_9, 5); +x_34 = lean_ctor_get(x_9, 6); +x_35 = lean_ctor_get(x_9, 7); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_9); +x_36 = lean_ctor_get_uint64(x_10, sizeof(void*)*1); +if (lean_is_exclusive(x_10)) { + lean_ctor_release(x_10, 0); + x_37 = x_10; +} else { + lean_dec_ref(x_10); + x_37 = lean_box(0); +} +x_38 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3; +if (lean_is_scalar(x_37)) { + x_39 = lean_alloc_ctor(0, 1, 8); +} else { + x_39 = x_37; +} +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set_uint64(x_39, sizeof(void*)*1, x_36); +x_40 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_40, 0, x_29); +lean_ctor_set(x_40, 1, x_30); +lean_ctor_set(x_40, 2, x_31); +lean_ctor_set(x_40, 3, x_39); +lean_ctor_set(x_40, 4, x_32); +lean_ctor_set(x_40, 5, x_33); +lean_ctor_set(x_40, 6, x_34); +lean_ctor_set(x_40, 7, x_35); +x_41 = lean_st_ref_set(x_1, x_40, x_11); +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + lean_ctor_release(x_41, 1); + x_43 = x_41; +} else { + lean_dec_ref(x_41); + x_43 = lean_box(0); +} +if (lean_is_scalar(x_43)) { + x_44 = lean_alloc_ctor(0, 2, 0); +} else { + x_44 = x_43; +} +lean_ctor_set(x_44, 0, x_7); +lean_ctor_set(x_44, 1, x_42); +return x_44; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = lean_alloc_closure((void*)(l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___boxed), 2, 0); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_9); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_13 = lean_ctor_get(x_9, 5); +x_14 = l_Lean_replaceRef(x_3, x_13); +lean_dec(x_13); +lean_ctor_set(x_9, 5, x_14); +x_15 = lean_st_ref_get(x_10, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_ctor_get(x_16, 3); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lean_PersistentArray_toArray___rarg(x_19); +lean_dec(x_19); +x_21 = lean_array_size(x_20); +x_22 = 0; +x_23 = l_Array_mapMUnsafe_map___at___private_Lean_Util_Trace_0__Lean_addTraceNode___spec__1(x_21, x_22, x_20); +x_24 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_24, 0, x_2); +lean_ctor_set(x_24, 1, x_4); +lean_ctor_set(x_24, 2, x_23); +x_25 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_24, x_7, x_8, x_9, x_10, x_17); +lean_dec(x_9); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_st_ref_take(x_10, x_27); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_29, 3); +lean_inc(x_30); +x_31 = !lean_is_exclusive(x_28); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_32 = lean_ctor_get(x_28, 1); +x_33 = lean_ctor_get(x_28, 0); +lean_dec(x_33); +x_34 = !lean_is_exclusive(x_29); +if (x_34 == 0) +{ +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_29, 3); +lean_dec(x_35); +x_36 = !lean_is_exclusive(x_30); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_37 = lean_ctor_get(x_30, 0); +lean_dec(x_37); +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set(x_28, 0, x_3); +x_38 = l_Lean_PersistentArray_push___rarg(x_1, x_28); +lean_ctor_set(x_30, 0, x_38); +x_39 = lean_st_ref_set(x_10, x_29, x_32); +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_39, 0); +lean_dec(x_41); +x_42 = lean_box(0); +lean_ctor_set(x_39, 0, x_42); +return x_39; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 1); +lean_inc(x_43); +lean_dec(x_39); +x_44 = lean_box(0); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +return x_45; +} +} +else +{ +uint64_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_46 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); +lean_dec(x_30); +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set(x_28, 0, x_3); +x_47 = l_Lean_PersistentArray_push___rarg(x_1, x_28); +x_48 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set_uint64(x_48, sizeof(void*)*1, x_46); +lean_ctor_set(x_29, 3, x_48); +x_49 = lean_st_ref_set(x_10, x_29, x_32); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; +} else { + lean_dec_ref(x_49); + x_51 = lean_box(0); +} +x_52 = lean_box(0); +if (lean_is_scalar(x_51)) { + x_53 = lean_alloc_ctor(0, 2, 0); +} else { + x_53 = x_51; +} +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_50); +return x_53; +} +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_54 = lean_ctor_get(x_29, 0); +x_55 = lean_ctor_get(x_29, 1); +x_56 = lean_ctor_get(x_29, 2); +x_57 = lean_ctor_get(x_29, 4); +x_58 = lean_ctor_get(x_29, 5); +x_59 = lean_ctor_get(x_29, 6); +x_60 = lean_ctor_get(x_29, 7); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_29); +x_61 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + x_62 = x_30; +} else { + lean_dec_ref(x_30); + x_62 = lean_box(0); +} +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set(x_28, 0, x_3); +x_63 = l_Lean_PersistentArray_push___rarg(x_1, x_28); +if (lean_is_scalar(x_62)) { + x_64 = lean_alloc_ctor(0, 1, 8); +} else { + x_64 = x_62; +} +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set_uint64(x_64, sizeof(void*)*1, x_61); +x_65 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_65, 0, x_54); +lean_ctor_set(x_65, 1, x_55); +lean_ctor_set(x_65, 2, x_56); +lean_ctor_set(x_65, 3, x_64); +lean_ctor_set(x_65, 4, x_57); +lean_ctor_set(x_65, 5, x_58); +lean_ctor_set(x_65, 6, x_59); +lean_ctor_set(x_65, 7, x_60); +x_66 = lean_st_ref_set(x_10, x_65, x_32); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_68 = x_66; +} else { + lean_dec_ref(x_66); + x_68 = lean_box(0); +} +x_69 = lean_box(0); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 0); +} else { + x_70 = x_68; +} +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_67); +return x_70; +} +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint64_t x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_71 = lean_ctor_get(x_28, 1); +lean_inc(x_71); +lean_dec(x_28); +x_72 = lean_ctor_get(x_29, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_29, 1); +lean_inc(x_73); +x_74 = lean_ctor_get(x_29, 2); +lean_inc(x_74); +x_75 = lean_ctor_get(x_29, 4); +lean_inc(x_75); +x_76 = lean_ctor_get(x_29, 5); +lean_inc(x_76); +x_77 = lean_ctor_get(x_29, 6); +lean_inc(x_77); +x_78 = lean_ctor_get(x_29, 7); +lean_inc(x_78); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + lean_ctor_release(x_29, 2); + lean_ctor_release(x_29, 3); + lean_ctor_release(x_29, 4); + lean_ctor_release(x_29, 5); + lean_ctor_release(x_29, 6); + lean_ctor_release(x_29, 7); + x_79 = x_29; +} else { + lean_dec_ref(x_29); + x_79 = lean_box(0); +} +x_80 = lean_ctor_get_uint64(x_30, sizeof(void*)*1); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + x_81 = x_30; +} else { + lean_dec_ref(x_30); + x_81 = lean_box(0); +} +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_3); +lean_ctor_set(x_82, 1, x_26); +x_83 = l_Lean_PersistentArray_push___rarg(x_1, x_82); +if (lean_is_scalar(x_81)) { + x_84 = lean_alloc_ctor(0, 1, 8); +} else { + x_84 = x_81; +} +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set_uint64(x_84, sizeof(void*)*1, x_80); +if (lean_is_scalar(x_79)) { + x_85 = lean_alloc_ctor(0, 8, 0); +} else { + x_85 = x_79; +} +lean_ctor_set(x_85, 0, x_72); +lean_ctor_set(x_85, 1, x_73); +lean_ctor_set(x_85, 2, x_74); +lean_ctor_set(x_85, 3, x_84); +lean_ctor_set(x_85, 4, x_75); +lean_ctor_set(x_85, 5, x_76); +lean_ctor_set(x_85, 6, x_77); +lean_ctor_set(x_85, 7, x_78); +x_86 = lean_st_ref_set(x_10, x_85, x_71); +x_87 = lean_ctor_get(x_86, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_88 = x_86; +} else { + lean_dec_ref(x_86); + x_88 = lean_box(0); +} +x_89 = lean_box(0); +if (lean_is_scalar(x_88)) { + x_90 = lean_alloc_ctor(0, 2, 0); +} else { + x_90 = x_88; +} +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_87); +return x_90; +} +} +else +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; size_t x_113; size_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; uint64_t x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; +x_91 = lean_ctor_get(x_9, 0); +x_92 = lean_ctor_get(x_9, 1); +x_93 = lean_ctor_get(x_9, 2); +x_94 = lean_ctor_get(x_9, 3); +x_95 = lean_ctor_get(x_9, 4); +x_96 = lean_ctor_get(x_9, 5); +x_97 = lean_ctor_get(x_9, 6); +x_98 = lean_ctor_get(x_9, 7); +x_99 = lean_ctor_get(x_9, 8); +x_100 = lean_ctor_get(x_9, 9); +x_101 = lean_ctor_get(x_9, 10); +x_102 = lean_ctor_get_uint8(x_9, sizeof(void*)*12); +x_103 = lean_ctor_get(x_9, 11); +x_104 = lean_ctor_get_uint8(x_9, sizeof(void*)*12 + 1); +lean_inc(x_103); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +lean_inc(x_98); +lean_inc(x_97); +lean_inc(x_96); +lean_inc(x_95); +lean_inc(x_94); +lean_inc(x_93); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_9); +x_105 = l_Lean_replaceRef(x_3, x_96); +lean_dec(x_96); +x_106 = lean_alloc_ctor(0, 12, 2); +lean_ctor_set(x_106, 0, x_91); +lean_ctor_set(x_106, 1, x_92); +lean_ctor_set(x_106, 2, x_93); +lean_ctor_set(x_106, 3, x_94); +lean_ctor_set(x_106, 4, x_95); +lean_ctor_set(x_106, 5, x_105); +lean_ctor_set(x_106, 6, x_97); +lean_ctor_set(x_106, 7, x_98); +lean_ctor_set(x_106, 8, x_99); +lean_ctor_set(x_106, 9, x_100); +lean_ctor_set(x_106, 10, x_101); +lean_ctor_set(x_106, 11, x_103); +lean_ctor_set_uint8(x_106, sizeof(void*)*12, x_102); +lean_ctor_set_uint8(x_106, sizeof(void*)*12 + 1, x_104); +x_107 = lean_st_ref_get(x_10, x_11); +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = lean_ctor_get(x_108, 3); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +lean_dec(x_110); +x_112 = l_Lean_PersistentArray_toArray___rarg(x_111); +lean_dec(x_111); +x_113 = lean_array_size(x_112); +x_114 = 0; +x_115 = l_Array_mapMUnsafe_map___at___private_Lean_Util_Trace_0__Lean_addTraceNode___spec__1(x_113, x_114, x_112); +x_116 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_116, 0, x_2); +lean_ctor_set(x_116, 1, x_4); +lean_ctor_set(x_116, 2, x_115); +x_117 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_116, x_7, x_8, x_106, x_10, x_109); +lean_dec(x_106); +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_117, 1); +lean_inc(x_119); +lean_dec(x_117); +x_120 = lean_st_ref_take(x_10, x_119); +x_121 = lean_ctor_get(x_120, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_121, 3); +lean_inc(x_122); +x_123 = lean_ctor_get(x_120, 1); +lean_inc(x_123); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_124 = x_120; +} else { + lean_dec_ref(x_120); + x_124 = lean_box(0); +} +x_125 = lean_ctor_get(x_121, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_121, 1); +lean_inc(x_126); +x_127 = lean_ctor_get(x_121, 2); +lean_inc(x_127); +x_128 = lean_ctor_get(x_121, 4); +lean_inc(x_128); +x_129 = lean_ctor_get(x_121, 5); +lean_inc(x_129); +x_130 = lean_ctor_get(x_121, 6); +lean_inc(x_130); +x_131 = lean_ctor_get(x_121, 7); +lean_inc(x_131); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + lean_ctor_release(x_121, 2); + lean_ctor_release(x_121, 3); + lean_ctor_release(x_121, 4); + lean_ctor_release(x_121, 5); + lean_ctor_release(x_121, 6); + lean_ctor_release(x_121, 7); + x_132 = x_121; +} else { + lean_dec_ref(x_121); + x_132 = lean_box(0); +} +x_133 = lean_ctor_get_uint64(x_122, sizeof(void*)*1); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + x_134 = x_122; +} else { + lean_dec_ref(x_122); + x_134 = lean_box(0); +} +if (lean_is_scalar(x_124)) { + x_135 = lean_alloc_ctor(0, 2, 0); +} else { + x_135 = x_124; +} +lean_ctor_set(x_135, 0, x_3); +lean_ctor_set(x_135, 1, x_118); +x_136 = l_Lean_PersistentArray_push___rarg(x_1, x_135); +if (lean_is_scalar(x_134)) { + x_137 = lean_alloc_ctor(0, 1, 8); +} else { + x_137 = x_134; +} +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set_uint64(x_137, sizeof(void*)*1, x_133); +if (lean_is_scalar(x_132)) { + x_138 = lean_alloc_ctor(0, 8, 0); +} else { + x_138 = x_132; +} +lean_ctor_set(x_138, 0, x_125); +lean_ctor_set(x_138, 1, x_126); +lean_ctor_set(x_138, 2, x_127); +lean_ctor_set(x_138, 3, x_137); +lean_ctor_set(x_138, 4, x_128); +lean_ctor_set(x_138, 5, x_129); +lean_ctor_set(x_138, 6, x_130); +lean_ctor_set(x_138, 7, x_131); +x_139 = lean_st_ref_set(x_10, x_138, x_123); +x_140 = lean_ctor_get(x_139, 1); +lean_inc(x_140); +if (lean_is_exclusive(x_139)) { + lean_ctor_release(x_139, 0); + lean_ctor_release(x_139, 1); + x_141 = x_139; +} else { + lean_dec_ref(x_139); + x_141 = lean_box(0); +} +x_142 = lean_box(0); +if (lean_is_scalar(x_141)) { + x_143 = lean_alloc_ctor(0, 2, 0); +} else { + x_143 = x_141; +} +lean_ctor_set(x_143, 0, x_142); +lean_ctor_set(x_143, 1, x_140); +return x_143; +} +} +} +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_1, 0); +lean_inc(x_9); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_8); +return x_12; +} +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_inc(x_11); +x_14 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3(x_1, x_5, x_2, x_3, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_15); +lean_dec(x_11); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, double x_8, double x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: +{ +if (x_7 == 0) +{ +double x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1; +x_19 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_19, 0, x_1); +lean_ctor_set(x_19, 1, x_3); +lean_ctor_set_float(x_19, sizeof(void*)*2, x_18); +lean_ctor_set_float(x_19, sizeof(void*)*2 + 8, x_18); +lean_ctor_set_uint8(x_19, sizeof(void*)*2 + 16, x_2); +x_20 = lean_box(0); +x_21 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_19, x_20, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_21; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_22, 0, x_1); +lean_ctor_set(x_22, 1, x_3); +lean_ctor_set_float(x_22, sizeof(void*)*2, x_8); +lean_ctor_set_float(x_22, sizeof(void*)*2 + 8, x_9); +lean_ctor_set_uint8(x_22, sizeof(void*)*2 + 16, x_2); +x_23 = lean_box(0); +x_24 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1(x_4, x_5, x_10, x_6, x_22, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +return x_24; +} +} +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 53, 53); +return x_1; +} +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, double x_7, double x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +_start: +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 5); +lean_inc(x_18); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_5); +x_19 = lean_apply_8(x_9, x_5, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_18, x_5, x_6, x_7, x_8, x_20, x_11, x_12, x_13, x_14, x_15, x_16, x_21); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_5); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_19, 1); +lean_inc(x_23); +lean_dec(x_19); +x_24 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2; +x_25 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_18, x_5, x_6, x_7, x_8, x_24, x_11, x_12, x_13, x_14, x_15, x_16, x_23); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_5); +return x_25; +} +} +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_trace_profiler_useHeartbeats; +return x_1; +} +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_trace_profiler; +return x_1; +} +} +static lean_object* _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_trace_profiler_threshold; +return x_1; +} +} +static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; +x_1 = lean_unsigned_to_nat(1000u); +x_2 = 0; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Float_ofScientific(x_1, x_2, x_3); +return x_4; +} +} +static double _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5() { +_start: +{ +lean_object* x_1; uint8_t x_2; lean_object* x_3; double x_4; +x_1 = lean_unsigned_to_nat(1000000000u); +x_2 = 0; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Float_ofScientific(x_1, x_2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_16 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg(x_14, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1; +x_20 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_125 = lean_io_mono_nanos_now(x_18); +x_126 = lean_ctor_get(x_125, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_125, 1); +lean_inc(x_127); +lean_dec(x_125); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_128 = lean_apply_7(x_7, x_9, x_10, x_11, x_12, x_13, x_14, x_127); +if (lean_obj_tag(x_128) == 0) +{ +uint8_t x_129; +x_129 = !lean_is_exclusive(x_128); +if (x_129 == 0) +{ +lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; uint8_t x_134; +x_130 = lean_ctor_get(x_128, 0); +x_131 = lean_ctor_get(x_128, 1); +x_132 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_132, 0, x_130); +x_133 = lean_io_mono_nanos_now(x_131); +x_134 = !lean_is_exclusive(x_133); +if (x_134 == 0) +{ +lean_object* x_135; lean_object* x_136; uint8_t x_137; lean_object* x_138; double x_139; double x_140; double x_141; double x_142; double x_143; lean_object* x_144; lean_object* x_145; +x_135 = lean_ctor_get(x_133, 0); +x_136 = lean_ctor_get(x_133, 1); +x_137 = 0; +x_138 = lean_unsigned_to_nat(0u); +x_139 = l_Float_ofScientific(x_126, x_137, x_138); +lean_dec(x_126); +x_140 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_141 = lean_float_div(x_139, x_140); +x_142 = l_Float_ofScientific(x_135, x_137, x_138); +lean_dec(x_135); +x_143 = lean_float_div(x_142, x_140); +x_144 = lean_box_float(x_141); +x_145 = lean_box_float(x_143); +lean_ctor_set(x_133, 1, x_145); +lean_ctor_set(x_133, 0, x_144); +lean_ctor_set(x_128, 1, x_133); +lean_ctor_set(x_128, 0, x_132); +x_21 = x_128; +x_22 = x_136; +goto block_124; +} +else +{ +lean_object* x_146; lean_object* x_147; uint8_t x_148; lean_object* x_149; double x_150; double x_151; double x_152; double x_153; double x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_146 = lean_ctor_get(x_133, 0); +x_147 = lean_ctor_get(x_133, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_133); +x_148 = 0; +x_149 = lean_unsigned_to_nat(0u); +x_150 = l_Float_ofScientific(x_126, x_148, x_149); +lean_dec(x_126); +x_151 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_152 = lean_float_div(x_150, x_151); +x_153 = l_Float_ofScientific(x_146, x_148, x_149); +lean_dec(x_146); +x_154 = lean_float_div(x_153, x_151); +x_155 = lean_box_float(x_152); +x_156 = lean_box_float(x_154); +x_157 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_157, 0, x_155); +lean_ctor_set(x_157, 1, x_156); +lean_ctor_set(x_128, 1, x_157); +lean_ctor_set(x_128, 0, x_132); +x_21 = x_128; +x_22 = x_147; +goto block_124; +} +} +else +{ +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; uint8_t x_165; lean_object* x_166; double x_167; double x_168; double x_169; double x_170; double x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_158 = lean_ctor_get(x_128, 0); +x_159 = lean_ctor_get(x_128, 1); +lean_inc(x_159); +lean_inc(x_158); +lean_dec(x_128); +x_160 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_160, 0, x_158); +x_161 = lean_io_mono_nanos_now(x_159); +x_162 = lean_ctor_get(x_161, 0); +lean_inc(x_162); +x_163 = lean_ctor_get(x_161, 1); +lean_inc(x_163); +if (lean_is_exclusive(x_161)) { + lean_ctor_release(x_161, 0); + lean_ctor_release(x_161, 1); + x_164 = x_161; +} else { + lean_dec_ref(x_161); + x_164 = lean_box(0); +} +x_165 = 0; +x_166 = lean_unsigned_to_nat(0u); +x_167 = l_Float_ofScientific(x_126, x_165, x_166); +lean_dec(x_126); +x_168 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_169 = lean_float_div(x_167, x_168); +x_170 = l_Float_ofScientific(x_162, x_165, x_166); +lean_dec(x_162); +x_171 = lean_float_div(x_170, x_168); +x_172 = lean_box_float(x_169); +x_173 = lean_box_float(x_171); +if (lean_is_scalar(x_164)) { + x_174 = lean_alloc_ctor(0, 2, 0); +} else { + x_174 = x_164; +} +lean_ctor_set(x_174, 0, x_172); +lean_ctor_set(x_174, 1, x_173); +x_175 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_175, 0, x_160); +lean_ctor_set(x_175, 1, x_174); +x_21 = x_175; +x_22 = x_163; +goto block_124; +} +} +else +{ +uint8_t x_176; +x_176 = !lean_is_exclusive(x_128); +if (x_176 == 0) +{ +lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; uint8_t x_181; +x_177 = lean_ctor_get(x_128, 0); +x_178 = lean_ctor_get(x_128, 1); +x_179 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_179, 0, x_177); +x_180 = lean_io_mono_nanos_now(x_178); +x_181 = !lean_is_exclusive(x_180); +if (x_181 == 0) +{ +lean_object* x_182; lean_object* x_183; uint8_t x_184; lean_object* x_185; double x_186; double x_187; double x_188; double x_189; double x_190; lean_object* x_191; lean_object* x_192; +x_182 = lean_ctor_get(x_180, 0); +x_183 = lean_ctor_get(x_180, 1); +x_184 = 0; +x_185 = lean_unsigned_to_nat(0u); +x_186 = l_Float_ofScientific(x_126, x_184, x_185); +lean_dec(x_126); +x_187 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_188 = lean_float_div(x_186, x_187); +x_189 = l_Float_ofScientific(x_182, x_184, x_185); +lean_dec(x_182); +x_190 = lean_float_div(x_189, x_187); +x_191 = lean_box_float(x_188); +x_192 = lean_box_float(x_190); +lean_ctor_set(x_180, 1, x_192); +lean_ctor_set(x_180, 0, x_191); +lean_ctor_set_tag(x_128, 0); +lean_ctor_set(x_128, 1, x_180); +lean_ctor_set(x_128, 0, x_179); +x_21 = x_128; +x_22 = x_183; +goto block_124; +} +else +{ +lean_object* x_193; lean_object* x_194; uint8_t x_195; lean_object* x_196; double x_197; double x_198; double x_199; double x_200; double x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; +x_193 = lean_ctor_get(x_180, 0); +x_194 = lean_ctor_get(x_180, 1); +lean_inc(x_194); +lean_inc(x_193); +lean_dec(x_180); +x_195 = 0; +x_196 = lean_unsigned_to_nat(0u); +x_197 = l_Float_ofScientific(x_126, x_195, x_196); +lean_dec(x_126); +x_198 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_199 = lean_float_div(x_197, x_198); +x_200 = l_Float_ofScientific(x_193, x_195, x_196); +lean_dec(x_193); +x_201 = lean_float_div(x_200, x_198); +x_202 = lean_box_float(x_199); +x_203 = lean_box_float(x_201); +x_204 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_204, 0, x_202); +lean_ctor_set(x_204, 1, x_203); +lean_ctor_set_tag(x_128, 0); +lean_ctor_set(x_128, 1, x_204); +lean_ctor_set(x_128, 0, x_179); +x_21 = x_128; +x_22 = x_194; +goto block_124; +} +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; uint8_t x_212; lean_object* x_213; double x_214; double x_215; double x_216; double x_217; double x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; +x_205 = lean_ctor_get(x_128, 0); +x_206 = lean_ctor_get(x_128, 1); +lean_inc(x_206); +lean_inc(x_205); +lean_dec(x_128); +x_207 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_207, 0, x_205); +x_208 = lean_io_mono_nanos_now(x_206); +x_209 = lean_ctor_get(x_208, 0); +lean_inc(x_209); +x_210 = lean_ctor_get(x_208, 1); +lean_inc(x_210); +if (lean_is_exclusive(x_208)) { + lean_ctor_release(x_208, 0); + lean_ctor_release(x_208, 1); + x_211 = x_208; +} else { + lean_dec_ref(x_208); + x_211 = lean_box(0); +} +x_212 = 0; +x_213 = lean_unsigned_to_nat(0u); +x_214 = l_Float_ofScientific(x_126, x_212, x_213); +lean_dec(x_126); +x_215 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5; +x_216 = lean_float_div(x_214, x_215); +x_217 = l_Float_ofScientific(x_209, x_212, x_213); +lean_dec(x_209); +x_218 = lean_float_div(x_217, x_215); +x_219 = lean_box_float(x_216); +x_220 = lean_box_float(x_218); +if (lean_is_scalar(x_211)) { + x_221 = lean_alloc_ctor(0, 2, 0); +} else { + x_221 = x_211; +} +lean_ctor_set(x_221, 0, x_219); +lean_ctor_set(x_221, 1, x_220); +x_222 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_222, 0, x_207); +lean_ctor_set(x_222, 1, x_221); +x_21 = x_222; +x_22 = x_210; +goto block_124; +} +} +block_124: +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; uint8_t x_29; +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 0); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_23, 1); +lean_inc(x_26); +lean_dec(x_23); +x_27 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2; +x_28 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_27); +if (x_28 == 0) +{ +if (x_6 == 0) +{ +uint8_t x_94; +x_94 = 0; +x_29 = x_94; +goto block_93; +} +else +{ +lean_object* x_95; double x_96; double x_97; lean_object* x_98; +x_95 = lean_box(0); +x_96 = lean_unbox_float(x_25); +lean_dec(x_25); +x_97 = lean_unbox_float(x_26); +lean_dec(x_26); +x_98 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_24, x_28, x_96, x_97, x_5, x_95, x_9, x_10, x_11, x_12, x_13, x_14, x_22); +return x_98; +} +} +else +{ +double x_99; double x_100; double x_101; +x_99 = lean_unbox_float(x_26); +x_100 = lean_unbox_float(x_25); +x_101 = lean_float_sub(x_99, x_100); +if (x_20 == 0) +{ +if (x_6 == 0) +{ +lean_object* x_102; lean_object* x_103; uint8_t x_104; lean_object* x_105; double x_106; double x_107; double x_108; uint8_t x_109; +x_102 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3; +x_103 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_102); +x_104 = 0; +x_105 = lean_unsigned_to_nat(0u); +x_106 = l_Float_ofScientific(x_103, x_104, x_105); +lean_dec(x_103); +x_107 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4; +x_108 = lean_float_div(x_106, x_107); +x_109 = lean_float_decLt(x_108, x_101); +x_29 = x_109; +goto block_93; +} +else +{ +lean_object* x_110; double x_111; double x_112; lean_object* x_113; +x_110 = lean_box(0); +x_111 = lean_unbox_float(x_25); +lean_dec(x_25); +x_112 = lean_unbox_float(x_26); +lean_dec(x_26); +x_113 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_24, x_28, x_111, x_112, x_5, x_110, x_9, x_10, x_11, x_12, x_13, x_14, x_22); +return x_113; +} +} +else +{ +if (x_6 == 0) +{ +lean_object* x_114; lean_object* x_115; uint8_t x_116; lean_object* x_117; double x_118; uint8_t x_119; +x_114 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3; +x_115 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_114); +x_116 = 0; +x_117 = lean_unsigned_to_nat(0u); +x_118 = l_Float_ofScientific(x_115, x_116, x_117); +lean_dec(x_115); +x_119 = lean_float_decLt(x_118, x_101); +x_29 = x_119; +goto block_93; +} +else +{ +lean_object* x_120; double x_121; double x_122; lean_object* x_123; +x_120 = lean_box(0); +x_121 = lean_unbox_float(x_25); +lean_dec(x_25); +x_122 = lean_unbox_float(x_26); +lean_dec(x_26); +x_123 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_24, x_28, x_121, x_122, x_5, x_120, x_9, x_10, x_11, x_12, x_13, x_14, x_22); +return x_123; +} +} +} +block_93: +{ +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_30 = lean_st_ref_take(x_14, x_22); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_31, 3); +lean_inc(x_32); +x_33 = lean_ctor_get(x_30, 1); +lean_inc(x_33); +lean_dec(x_30); +x_34 = !lean_is_exclusive(x_31); +if (x_34 == 0) +{ +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_31, 3); +lean_dec(x_35); +x_36 = !lean_is_exclusive(x_32); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_37 = lean_ctor_get(x_32, 0); +x_38 = l_Lean_PersistentArray_append___rarg(x_17, x_37); +lean_dec(x_37); +lean_ctor_set(x_32, 0, x_38); +x_39 = lean_st_ref_set(x_14, x_31, x_33); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +lean_dec(x_39); +x_41 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_24, x_9, x_10, x_11, x_12, x_13, x_14, x_40); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_24); +if (lean_obj_tag(x_41) == 0) +{ +uint8_t x_42; +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) +{ +return x_41; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_41, 0); +x_44 = lean_ctor_get(x_41, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_41); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +else +{ +uint8_t x_46; +x_46 = !lean_is_exclusive(x_41); +if (x_46 == 0) +{ +return x_41; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_41, 0); +x_48 = lean_ctor_get(x_41, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_41); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; +} +} +} +else +{ +uint64_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_50 = lean_ctor_get_uint64(x_32, sizeof(void*)*1); +x_51 = lean_ctor_get(x_32, 0); +lean_inc(x_51); +lean_dec(x_32); +x_52 = l_Lean_PersistentArray_append___rarg(x_17, x_51); +lean_dec(x_51); +x_53 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set_uint64(x_53, sizeof(void*)*1, x_50); +lean_ctor_set(x_31, 3, x_53); +x_54 = lean_st_ref_set(x_14, x_31, x_33); +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +lean_dec(x_54); +x_56 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_24, x_9, x_10, x_11, x_12, x_13, x_14, x_55); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_24); +if (lean_obj_tag(x_56) == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_59 = x_56; +} else { + lean_dec_ref(x_56); + x_59 = lean_box(0); +} +if (lean_is_scalar(x_59)) { + x_60 = lean_alloc_ctor(0, 2, 0); +} else { + x_60 = x_59; +} +lean_ctor_set(x_60, 0, x_57); +lean_ctor_set(x_60, 1, x_58); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_61 = lean_ctor_get(x_56, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_56, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_63 = x_56; +} else { + lean_dec_ref(x_56); + x_63 = lean_box(0); +} +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 2, 0); +} else { + x_64 = x_63; +} +lean_ctor_set(x_64, 0, x_61); +lean_ctor_set(x_64, 1, x_62); +return x_64; +} +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint64_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_65 = lean_ctor_get(x_31, 0); +x_66 = lean_ctor_get(x_31, 1); +x_67 = lean_ctor_get(x_31, 2); +x_68 = lean_ctor_get(x_31, 4); +x_69 = lean_ctor_get(x_31, 5); +x_70 = lean_ctor_get(x_31, 6); +x_71 = lean_ctor_get(x_31, 7); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_31); +x_72 = lean_ctor_get_uint64(x_32, sizeof(void*)*1); +x_73 = lean_ctor_get(x_32, 0); +lean_inc(x_73); +if (lean_is_exclusive(x_32)) { + lean_ctor_release(x_32, 0); + x_74 = x_32; +} else { + lean_dec_ref(x_32); + x_74 = lean_box(0); +} +x_75 = l_Lean_PersistentArray_append___rarg(x_17, x_73); +lean_dec(x_73); +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 1, 8); +} else { + x_76 = x_74; +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set_uint64(x_76, sizeof(void*)*1, x_72); +x_77 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_77, 0, x_65); +lean_ctor_set(x_77, 1, x_66); +lean_ctor_set(x_77, 2, x_67); +lean_ctor_set(x_77, 3, x_76); +lean_ctor_set(x_77, 4, x_68); +lean_ctor_set(x_77, 5, x_69); +lean_ctor_set(x_77, 6, x_70); +lean_ctor_set(x_77, 7, x_71); +x_78 = lean_st_ref_set(x_14, x_77, x_33); +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_24, x_9, x_10, x_11, x_12, x_13, x_14, x_79); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_24); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_83 = x_80; +} else { + lean_dec_ref(x_80); + x_83 = lean_box(0); +} +if (lean_is_scalar(x_83)) { + x_84 = lean_alloc_ctor(0, 2, 0); +} else { + x_84 = x_83; +} +lean_ctor_set(x_84, 0, x_81); +lean_ctor_set(x_84, 1, x_82); +return x_84; +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_85 = lean_ctor_get(x_80, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_80, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_87 = x_80; +} else { + lean_dec_ref(x_80); + x_87 = lean_box(0); +} +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(1, 2, 0); +} else { + x_88 = x_87; +} +lean_ctor_set(x_88, 0, x_85); +lean_ctor_set(x_88, 1, x_86); +return x_88; +} +} +} +else +{ +lean_object* x_89; double x_90; double x_91; lean_object* x_92; +x_89 = lean_box(0); +x_90 = lean_unbox_float(x_25); +lean_dec(x_25); +x_91 = lean_unbox_float(x_26); +lean_dec(x_26); +x_92 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_24, x_28, x_90, x_91, x_5, x_89, x_9, x_10, x_11, x_12, x_13, x_14, x_22); +return x_92; +} +} +} +} +else +{ +lean_object* x_223; lean_object* x_224; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; +x_327 = lean_io_get_num_heartbeats(x_18); +x_328 = lean_ctor_get(x_327, 0); +lean_inc(x_328); +x_329 = lean_ctor_get(x_327, 1); +lean_inc(x_329); +lean_dec(x_327); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_330 = lean_apply_7(x_7, x_9, x_10, x_11, x_12, x_13, x_14, x_329); +if (lean_obj_tag(x_330) == 0) +{ +uint8_t x_331; +x_331 = !lean_is_exclusive(x_330); +if (x_331 == 0) +{ +lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; uint8_t x_336; +x_332 = lean_ctor_get(x_330, 0); +x_333 = lean_ctor_get(x_330, 1); +x_334 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_334, 0, x_332); +x_335 = lean_io_get_num_heartbeats(x_333); +x_336 = !lean_is_exclusive(x_335); +if (x_336 == 0) +{ +lean_object* x_337; lean_object* x_338; uint8_t x_339; lean_object* x_340; double x_341; double x_342; lean_object* x_343; lean_object* x_344; +x_337 = lean_ctor_get(x_335, 0); +x_338 = lean_ctor_get(x_335, 1); +x_339 = 0; +x_340 = lean_unsigned_to_nat(0u); +x_341 = l_Float_ofScientific(x_328, x_339, x_340); +lean_dec(x_328); +x_342 = l_Float_ofScientific(x_337, x_339, x_340); +lean_dec(x_337); +x_343 = lean_box_float(x_341); +x_344 = lean_box_float(x_342); +lean_ctor_set(x_335, 1, x_344); +lean_ctor_set(x_335, 0, x_343); +lean_ctor_set(x_330, 1, x_335); +lean_ctor_set(x_330, 0, x_334); +x_223 = x_330; +x_224 = x_338; +goto block_326; +} +else +{ +lean_object* x_345; lean_object* x_346; uint8_t x_347; lean_object* x_348; double x_349; double x_350; lean_object* x_351; lean_object* x_352; lean_object* x_353; +x_345 = lean_ctor_get(x_335, 0); +x_346 = lean_ctor_get(x_335, 1); +lean_inc(x_346); +lean_inc(x_345); +lean_dec(x_335); +x_347 = 0; +x_348 = lean_unsigned_to_nat(0u); +x_349 = l_Float_ofScientific(x_328, x_347, x_348); +lean_dec(x_328); +x_350 = l_Float_ofScientific(x_345, x_347, x_348); +lean_dec(x_345); +x_351 = lean_box_float(x_349); +x_352 = lean_box_float(x_350); +x_353 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_353, 0, x_351); +lean_ctor_set(x_353, 1, x_352); +lean_ctor_set(x_330, 1, x_353); +lean_ctor_set(x_330, 0, x_334); +x_223 = x_330; +x_224 = x_346; +goto block_326; +} +} +else +{ +lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; uint8_t x_361; lean_object* x_362; double x_363; double x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; +x_354 = lean_ctor_get(x_330, 0); +x_355 = lean_ctor_get(x_330, 1); +lean_inc(x_355); +lean_inc(x_354); +lean_dec(x_330); +x_356 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_356, 0, x_354); +x_357 = lean_io_get_num_heartbeats(x_355); +x_358 = lean_ctor_get(x_357, 0); +lean_inc(x_358); +x_359 = lean_ctor_get(x_357, 1); +lean_inc(x_359); +if (lean_is_exclusive(x_357)) { + lean_ctor_release(x_357, 0); + lean_ctor_release(x_357, 1); + x_360 = x_357; +} else { + lean_dec_ref(x_357); + x_360 = lean_box(0); +} +x_361 = 0; +x_362 = lean_unsigned_to_nat(0u); +x_363 = l_Float_ofScientific(x_328, x_361, x_362); +lean_dec(x_328); +x_364 = l_Float_ofScientific(x_358, x_361, x_362); +lean_dec(x_358); +x_365 = lean_box_float(x_363); +x_366 = lean_box_float(x_364); +if (lean_is_scalar(x_360)) { + x_367 = lean_alloc_ctor(0, 2, 0); +} else { + x_367 = x_360; +} +lean_ctor_set(x_367, 0, x_365); +lean_ctor_set(x_367, 1, x_366); +x_368 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_368, 0, x_356); +lean_ctor_set(x_368, 1, x_367); +x_223 = x_368; +x_224 = x_359; +goto block_326; +} +} +else +{ +uint8_t x_369; +x_369 = !lean_is_exclusive(x_330); +if (x_369 == 0) +{ +lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; uint8_t x_374; +x_370 = lean_ctor_get(x_330, 0); +x_371 = lean_ctor_get(x_330, 1); +x_372 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_372, 0, x_370); +x_373 = lean_io_get_num_heartbeats(x_371); +x_374 = !lean_is_exclusive(x_373); +if (x_374 == 0) +{ +lean_object* x_375; lean_object* x_376; uint8_t x_377; lean_object* x_378; double x_379; double x_380; lean_object* x_381; lean_object* x_382; +x_375 = lean_ctor_get(x_373, 0); +x_376 = lean_ctor_get(x_373, 1); +x_377 = 0; +x_378 = lean_unsigned_to_nat(0u); +x_379 = l_Float_ofScientific(x_328, x_377, x_378); +lean_dec(x_328); +x_380 = l_Float_ofScientific(x_375, x_377, x_378); +lean_dec(x_375); +x_381 = lean_box_float(x_379); +x_382 = lean_box_float(x_380); +lean_ctor_set(x_373, 1, x_382); +lean_ctor_set(x_373, 0, x_381); +lean_ctor_set_tag(x_330, 0); +lean_ctor_set(x_330, 1, x_373); +lean_ctor_set(x_330, 0, x_372); +x_223 = x_330; +x_224 = x_376; +goto block_326; +} +else +{ +lean_object* x_383; lean_object* x_384; uint8_t x_385; lean_object* x_386; double x_387; double x_388; lean_object* x_389; lean_object* x_390; lean_object* x_391; +x_383 = lean_ctor_get(x_373, 0); +x_384 = lean_ctor_get(x_373, 1); +lean_inc(x_384); +lean_inc(x_383); +lean_dec(x_373); +x_385 = 0; +x_386 = lean_unsigned_to_nat(0u); +x_387 = l_Float_ofScientific(x_328, x_385, x_386); +lean_dec(x_328); +x_388 = l_Float_ofScientific(x_383, x_385, x_386); +lean_dec(x_383); +x_389 = lean_box_float(x_387); +x_390 = lean_box_float(x_388); +x_391 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_391, 0, x_389); +lean_ctor_set(x_391, 1, x_390); +lean_ctor_set_tag(x_330, 0); +lean_ctor_set(x_330, 1, x_391); +lean_ctor_set(x_330, 0, x_372); +x_223 = x_330; +x_224 = x_384; +goto block_326; +} +} +else +{ +lean_object* x_392; lean_object* x_393; lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; uint8_t x_399; lean_object* x_400; double x_401; double x_402; lean_object* x_403; lean_object* x_404; lean_object* x_405; lean_object* x_406; +x_392 = lean_ctor_get(x_330, 0); +x_393 = lean_ctor_get(x_330, 1); +lean_inc(x_393); +lean_inc(x_392); +lean_dec(x_330); +x_394 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_394, 0, x_392); +x_395 = lean_io_get_num_heartbeats(x_393); +x_396 = lean_ctor_get(x_395, 0); +lean_inc(x_396); +x_397 = lean_ctor_get(x_395, 1); +lean_inc(x_397); +if (lean_is_exclusive(x_395)) { + lean_ctor_release(x_395, 0); + lean_ctor_release(x_395, 1); + x_398 = x_395; +} else { + lean_dec_ref(x_395); + x_398 = lean_box(0); +} +x_399 = 0; +x_400 = lean_unsigned_to_nat(0u); +x_401 = l_Float_ofScientific(x_328, x_399, x_400); +lean_dec(x_328); +x_402 = l_Float_ofScientific(x_396, x_399, x_400); +lean_dec(x_396); +x_403 = lean_box_float(x_401); +x_404 = lean_box_float(x_402); +if (lean_is_scalar(x_398)) { + x_405 = lean_alloc_ctor(0, 2, 0); +} else { + x_405 = x_398; +} +lean_ctor_set(x_405, 0, x_403); +lean_ctor_set(x_405, 1, x_404); +x_406 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_406, 0, x_394); +lean_ctor_set(x_406, 1, x_405); +x_223 = x_406; +x_224 = x_397; +goto block_326; +} +} +block_326: +{ +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; uint8_t x_230; uint8_t x_231; +x_225 = lean_ctor_get(x_223, 1); +lean_inc(x_225); +x_226 = lean_ctor_get(x_223, 0); +lean_inc(x_226); +lean_dec(x_223); +x_227 = lean_ctor_get(x_225, 0); +lean_inc(x_227); +x_228 = lean_ctor_get(x_225, 1); +lean_inc(x_228); +lean_dec(x_225); +x_229 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2; +x_230 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_229); +if (x_230 == 0) +{ +if (x_6 == 0) +{ +uint8_t x_296; +x_296 = 0; +x_231 = x_296; +goto block_295; +} +else +{ +lean_object* x_297; double x_298; double x_299; lean_object* x_300; +x_297 = lean_box(0); +x_298 = lean_unbox_float(x_227); +lean_dec(x_227); +x_299 = lean_unbox_float(x_228); +lean_dec(x_228); +x_300 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_226, x_230, x_298, x_299, x_5, x_297, x_9, x_10, x_11, x_12, x_13, x_14, x_224); +return x_300; +} +} +else +{ +double x_301; double x_302; double x_303; +x_301 = lean_unbox_float(x_228); +x_302 = lean_unbox_float(x_227); +x_303 = lean_float_sub(x_301, x_302); +if (x_20 == 0) +{ +if (x_6 == 0) +{ +lean_object* x_304; lean_object* x_305; uint8_t x_306; lean_object* x_307; double x_308; double x_309; double x_310; uint8_t x_311; +x_304 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3; +x_305 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_304); +x_306 = 0; +x_307 = lean_unsigned_to_nat(0u); +x_308 = l_Float_ofScientific(x_305, x_306, x_307); +lean_dec(x_305); +x_309 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4; +x_310 = lean_float_div(x_308, x_309); +x_311 = lean_float_decLt(x_310, x_303); +x_231 = x_311; +goto block_295; +} +else +{ +lean_object* x_312; double x_313; double x_314; lean_object* x_315; +x_312 = lean_box(0); +x_313 = lean_unbox_float(x_227); +lean_dec(x_227); +x_314 = lean_unbox_float(x_228); +lean_dec(x_228); +x_315 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_226, x_230, x_313, x_314, x_5, x_312, x_9, x_10, x_11, x_12, x_13, x_14, x_224); +return x_315; +} +} +else +{ +if (x_6 == 0) +{ +lean_object* x_316; lean_object* x_317; uint8_t x_318; lean_object* x_319; double x_320; uint8_t x_321; +x_316 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3; +x_317 = l_Lean_Option_get___at_Lean_profiler_threshold_getSecs___spec__1(x_1, x_316); +x_318 = 0; +x_319 = lean_unsigned_to_nat(0u); +x_320 = l_Float_ofScientific(x_317, x_318, x_319); +lean_dec(x_317); +x_321 = lean_float_decLt(x_320, x_303); +x_231 = x_321; +goto block_295; +} +else +{ +lean_object* x_322; double x_323; double x_324; lean_object* x_325; +x_322 = lean_box(0); +x_323 = lean_unbox_float(x_227); +lean_dec(x_227); +x_324 = lean_unbox_float(x_228); +lean_dec(x_228); +x_325 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_226, x_230, x_323, x_324, x_5, x_322, x_9, x_10, x_11, x_12, x_13, x_14, x_224); +return x_325; +} +} +} +block_295: +{ +if (x_231 == 0) +{ +lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; uint8_t x_236; +lean_dec(x_228); +lean_dec(x_227); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_232 = lean_st_ref_take(x_14, x_224); +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_233, 3); +lean_inc(x_234); +x_235 = lean_ctor_get(x_232, 1); +lean_inc(x_235); +lean_dec(x_232); +x_236 = !lean_is_exclusive(x_233); +if (x_236 == 0) +{ +lean_object* x_237; uint8_t x_238; +x_237 = lean_ctor_get(x_233, 3); +lean_dec(x_237); +x_238 = !lean_is_exclusive(x_234); +if (x_238 == 0) +{ +lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; +x_239 = lean_ctor_get(x_234, 0); +x_240 = l_Lean_PersistentArray_append___rarg(x_17, x_239); +lean_dec(x_239); +lean_ctor_set(x_234, 0, x_240); +x_241 = lean_st_ref_set(x_14, x_233, x_235); +x_242 = lean_ctor_get(x_241, 1); +lean_inc(x_242); +lean_dec(x_241); +x_243 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_226, x_9, x_10, x_11, x_12, x_13, x_14, x_242); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_226); +if (lean_obj_tag(x_243) == 0) +{ +uint8_t x_244; +x_244 = !lean_is_exclusive(x_243); +if (x_244 == 0) +{ +return x_243; +} +else +{ +lean_object* x_245; lean_object* x_246; lean_object* x_247; +x_245 = lean_ctor_get(x_243, 0); +x_246 = lean_ctor_get(x_243, 1); +lean_inc(x_246); +lean_inc(x_245); +lean_dec(x_243); +x_247 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_247, 0, x_245); +lean_ctor_set(x_247, 1, x_246); +return x_247; +} +} +else +{ +uint8_t x_248; +x_248 = !lean_is_exclusive(x_243); +if (x_248 == 0) +{ +return x_243; +} +else +{ +lean_object* x_249; lean_object* x_250; lean_object* x_251; +x_249 = lean_ctor_get(x_243, 0); +x_250 = lean_ctor_get(x_243, 1); +lean_inc(x_250); +lean_inc(x_249); +lean_dec(x_243); +x_251 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_251, 0, x_249); +lean_ctor_set(x_251, 1, x_250); +return x_251; +} +} +} +else +{ +uint64_t x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; +x_252 = lean_ctor_get_uint64(x_234, sizeof(void*)*1); +x_253 = lean_ctor_get(x_234, 0); +lean_inc(x_253); +lean_dec(x_234); +x_254 = l_Lean_PersistentArray_append___rarg(x_17, x_253); +lean_dec(x_253); +x_255 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_255, 0, x_254); +lean_ctor_set_uint64(x_255, sizeof(void*)*1, x_252); +lean_ctor_set(x_233, 3, x_255); +x_256 = lean_st_ref_set(x_14, x_233, x_235); +x_257 = lean_ctor_get(x_256, 1); +lean_inc(x_257); +lean_dec(x_256); +x_258 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_226, x_9, x_10, x_11, x_12, x_13, x_14, x_257); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_226); +if (lean_obj_tag(x_258) == 0) +{ +lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; +x_259 = lean_ctor_get(x_258, 0); +lean_inc(x_259); +x_260 = lean_ctor_get(x_258, 1); +lean_inc(x_260); +if (lean_is_exclusive(x_258)) { + lean_ctor_release(x_258, 0); + lean_ctor_release(x_258, 1); + x_261 = x_258; +} else { + lean_dec_ref(x_258); + x_261 = lean_box(0); +} +if (lean_is_scalar(x_261)) { + x_262 = lean_alloc_ctor(0, 2, 0); +} else { + x_262 = x_261; +} +lean_ctor_set(x_262, 0, x_259); +lean_ctor_set(x_262, 1, x_260); +return x_262; +} +else +{ +lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; +x_263 = lean_ctor_get(x_258, 0); +lean_inc(x_263); +x_264 = lean_ctor_get(x_258, 1); +lean_inc(x_264); +if (lean_is_exclusive(x_258)) { + lean_ctor_release(x_258, 0); + lean_ctor_release(x_258, 1); + x_265 = x_258; +} else { + lean_dec_ref(x_258); + x_265 = lean_box(0); +} +if (lean_is_scalar(x_265)) { + x_266 = lean_alloc_ctor(1, 2, 0); +} else { + x_266 = x_265; +} +lean_ctor_set(x_266, 0, x_263); +lean_ctor_set(x_266, 1, x_264); +return x_266; +} +} +} +else +{ +lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; uint64_t x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +x_267 = lean_ctor_get(x_233, 0); +x_268 = lean_ctor_get(x_233, 1); +x_269 = lean_ctor_get(x_233, 2); +x_270 = lean_ctor_get(x_233, 4); +x_271 = lean_ctor_get(x_233, 5); +x_272 = lean_ctor_get(x_233, 6); +x_273 = lean_ctor_get(x_233, 7); +lean_inc(x_273); +lean_inc(x_272); +lean_inc(x_271); +lean_inc(x_270); +lean_inc(x_269); +lean_inc(x_268); +lean_inc(x_267); +lean_dec(x_233); +x_274 = lean_ctor_get_uint64(x_234, sizeof(void*)*1); +x_275 = lean_ctor_get(x_234, 0); +lean_inc(x_275); +if (lean_is_exclusive(x_234)) { + lean_ctor_release(x_234, 0); + x_276 = x_234; +} else { + lean_dec_ref(x_234); + x_276 = lean_box(0); +} +x_277 = l_Lean_PersistentArray_append___rarg(x_17, x_275); +lean_dec(x_275); +if (lean_is_scalar(x_276)) { + x_278 = lean_alloc_ctor(0, 1, 8); +} else { + x_278 = x_276; +} +lean_ctor_set(x_278, 0, x_277); +lean_ctor_set_uint64(x_278, sizeof(void*)*1, x_274); +x_279 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_279, 0, x_267); +lean_ctor_set(x_279, 1, x_268); +lean_ctor_set(x_279, 2, x_269); +lean_ctor_set(x_279, 3, x_278); +lean_ctor_set(x_279, 4, x_270); +lean_ctor_set(x_279, 5, x_271); +lean_ctor_set(x_279, 6, x_272); +lean_ctor_set(x_279, 7, x_273); +x_280 = lean_st_ref_set(x_14, x_279, x_235); +x_281 = lean_ctor_get(x_280, 1); +lean_inc(x_281); +lean_dec(x_280); +x_282 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_226, x_9, x_10, x_11, x_12, x_13, x_14, x_281); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_226); +if (lean_obj_tag(x_282) == 0) +{ +lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; +x_283 = lean_ctor_get(x_282, 0); +lean_inc(x_283); +x_284 = lean_ctor_get(x_282, 1); +lean_inc(x_284); +if (lean_is_exclusive(x_282)) { + lean_ctor_release(x_282, 0); + lean_ctor_release(x_282, 1); + x_285 = x_282; +} else { + lean_dec_ref(x_282); + x_285 = lean_box(0); +} +if (lean_is_scalar(x_285)) { + x_286 = lean_alloc_ctor(0, 2, 0); +} else { + x_286 = x_285; +} +lean_ctor_set(x_286, 0, x_283); +lean_ctor_set(x_286, 1, x_284); +return x_286; +} +else +{ +lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; +x_287 = lean_ctor_get(x_282, 0); +lean_inc(x_287); +x_288 = lean_ctor_get(x_282, 1); +lean_inc(x_288); +if (lean_is_exclusive(x_282)) { + lean_ctor_release(x_282, 0); + lean_ctor_release(x_282, 1); + x_289 = x_282; +} else { + lean_dec_ref(x_282); + x_289 = lean_box(0); +} +if (lean_is_scalar(x_289)) { + x_290 = lean_alloc_ctor(1, 2, 0); +} else { + x_290 = x_289; +} +lean_ctor_set(x_290, 0, x_287); +lean_ctor_set(x_290, 1, x_288); +return x_290; +} +} +} +else +{ +lean_object* x_291; double x_292; double x_293; lean_object* x_294; +x_291 = lean_box(0); +x_292 = lean_unbox_float(x_227); +lean_dec(x_227); +x_293 = lean_unbox_float(x_228); +lean_dec(x_228); +x_294 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_2, x_3, x_4, x_17, x_226, x_230, x_292, x_293, x_5, x_291, x_9, x_10, x_11, x_12, x_13, x_14, x_224); +return x_294; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_10, 2); +lean_inc(x_13); +lean_inc(x_1); +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2; +x_19 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_13, x_18); +if (x_19 == 0) +{ +lean_object* x_20; +lean_dec(x_15); +lean_dec(x_13); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_20 = lean_apply_7(x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +if (lean_obj_tag(x_20) == 0) +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +return x_20; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_20); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_20); +if (x_25 == 0) +{ +return x_20; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_20, 0); +x_27 = lean_ctor_get(x_20, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_20); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} +} +else +{ +lean_object* x_29; uint8_t x_30; lean_object* x_31; +x_29 = lean_box(0); +x_30 = lean_unbox(x_15); +lean_dec(x_15); +x_31 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4(x_13, x_1, x_4, x_5, x_2, x_30, x_3, x_29, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +lean_dec(x_13); +return x_31; +} +} +else +{ +lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_14, 1); +lean_inc(x_32); +lean_dec(x_14); +x_33 = lean_box(0); +x_34 = lean_unbox(x_15); +lean_dec(x_15); +x_35 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4(x_13, x_1, x_4, x_5, x_2, x_34, x_3, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +lean_dec(x_13); +return x_35; +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Running pass: ", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" on\n", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_11 = lean_ctor_get(x_1, 0); +lean_inc(x_11); +lean_dec(x_1); +x_12 = l_Lean_MessageData_ofName(x_11); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_2); +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_10); +return x_21; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; +lean_inc(x_2); +lean_inc(x_1); +x_10 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___boxed), 10, 2); +lean_closure_set(x_10, 0, x_1); +lean_closure_set(x_10, 1, x_2); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_dec(x_1); +x_12 = lean_apply_1(x_11, x_2); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1; +x_14 = 1; +x_15 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2; +x_16 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1(x_13, x_10, x_12, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_16; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Util_Trace_0__Lean_addTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_12; +} +} +LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_MonadExcept_ofExcept___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; double x_20; double x_21; lean_object* x_22; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox(x_7); +lean_dec(x_7); +x_20 = lean_unbox_float(x_8); +lean_dec(x_8); +x_21 = lean_unbox_float(x_9); +lean_dec(x_9); +x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__2(x_1, x_18, x_3, x_4, x_5, x_6, x_19, x_20, x_21, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_6); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; double x_20; double x_21; lean_object* x_22; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox(x_6); +lean_dec(x_6); +x_20 = lean_unbox_float(x_7); +lean_dec(x_7); +x_21 = lean_unbox_float(x_8); +lean_dec(x_8); +x_22 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3(x_1, x_18, x_3, x_4, x_5, x_19, x_20, x_21, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_10); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +uint8_t x_16; uint8_t x_17; lean_object* x_18; +x_16 = lean_unbox(x_3); +lean_dec(x_3); +x_17 = lean_unbox(x_6); +lean_dec(x_6); +x_18 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4(x_1, x_2, x_16, x_4, x_5, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_8); +lean_dec(x_1); +return x_18; +} +} +LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; lean_object* x_14; +x_13 = lean_unbox(x_4); +lean_dec(x_4); +x_14 = l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1(x_1, x_2, x_3, x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_11; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_1); +x_12 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_12, 0, x_11); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_9); +return x_13; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Fixpoint iteration solved the goal", 34, 34); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_15; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_6); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = lean_ctor_get(x_5, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_5, 1); +lean_inc(x_17); +lean_dec(x_5); +x_18 = !lean_is_exclusive(x_6); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_6, 1); +x_20 = lean_ctor_get(x_6, 0); +lean_dec(x_20); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_19); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run(x_16, x_19, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +lean_free_object(x_6); +lean_dec(x_17); +lean_dec(x_3); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_25 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_24, x_8, x_9, x_10, x_11, x_12, x_13, x_23); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_unbox(x_26); +lean_dec(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_box(0); +x_30 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_19, x_29, x_8, x_9, x_10, x_11, x_12, x_13, x_28); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_31 = !lean_is_exclusive(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_30, 0); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +lean_dec(x_32); +lean_ctor_set(x_30, 0, x_33); +return x_30; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_30, 0); +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_30); +x_36 = lean_ctor_get(x_34, 0); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +return x_37; +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_38 = lean_ctor_get(x_25, 1); +lean_inc(x_38); +lean_dec(x_25); +x_39 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2; +x_40 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_24, x_39, x_8, x_9, x_10, x_11, x_12, x_13, x_38); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_19, x_41, x_8, x_9, x_10, x_11, x_12, x_13, x_42); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_41); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_43, 0); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +lean_dec(x_45); +lean_ctor_set(x_43, 0, x_46); +return x_43; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_47 = lean_ctor_get(x_43, 0); +x_48 = lean_ctor_get(x_43, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_43); +x_49 = lean_ctor_get(x_47, 0); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_48); +return x_50; +} +} +} +else +{ +lean_object* x_51; lean_object* x_52; +lean_dec(x_19); +x_51 = lean_ctor_get(x_21, 1); +lean_inc(x_51); +lean_dec(x_21); +x_52 = lean_ctor_get(x_22, 0); +lean_inc(x_52); +lean_dec(x_22); +lean_inc(x_3); +lean_ctor_set(x_6, 1, x_52); +lean_ctor_set(x_6, 0, x_3); +x_5 = x_17; +x_7 = lean_box(0); +x_14 = x_51; +goto _start; +} +} +else +{ +uint8_t x_54; +lean_free_object(x_6); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +x_54 = !lean_is_exclusive(x_21); +if (x_54 == 0) +{ +return x_21; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_21, 0); +x_56 = lean_ctor_get(x_21, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_21); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +} +else +{ +lean_object* x_58; lean_object* x_59; +x_58 = lean_ctor_get(x_6, 1); +lean_inc(x_58); +lean_dec(x_6); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_58); +x_59 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run(x_16, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +lean_dec(x_17); +lean_dec(x_3); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_63 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_62, x_8, x_9, x_10, x_11, x_12, x_13, x_61); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_unbox(x_64); +lean_dec(x_64); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +lean_dec(x_63); +x_67 = lean_box(0); +x_68 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_58, x_67, x_8, x_9, x_10, x_11, x_12, x_13, x_66); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_71 = x_68; +} else { + lean_dec_ref(x_68); + x_71 = lean_box(0); +} +x_72 = lean_ctor_get(x_69, 0); +lean_inc(x_72); +lean_dec(x_69); +if (lean_is_scalar(x_71)) { + x_73 = lean_alloc_ctor(0, 2, 0); +} else { + x_73 = x_71; +} +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; +} +else +{ +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_74 = lean_ctor_get(x_63, 1); +lean_inc(x_74); +lean_dec(x_63); +x_75 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2; +x_76 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_62, x_75, x_8, x_9, x_10, x_11, x_12, x_13, x_74); +x_77 = lean_ctor_get(x_76, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_76, 1); +lean_inc(x_78); +lean_dec(x_76); +x_79 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_58, x_77, x_8, x_9, x_10, x_11, x_12, x_13, x_78); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_77); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_82 = x_79; +} else { + lean_dec_ref(x_79); + x_82 = lean_box(0); +} +x_83 = lean_ctor_get(x_80, 0); +lean_inc(x_83); +lean_dec(x_80); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); +} else { + x_84 = x_82; +} +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; +} +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_58); +x_85 = lean_ctor_get(x_59, 1); +lean_inc(x_85); +lean_dec(x_59); +x_86 = lean_ctor_get(x_60, 0); +lean_inc(x_86); +lean_dec(x_60); +lean_inc(x_3); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_3); +lean_ctor_set(x_87, 1, x_86); +x_5 = x_17; +x_6 = x_87; +x_7 = lean_box(0); +x_14 = x_85; +goto _start; +} +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_58); +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_3); +x_89 = lean_ctor_get(x_59, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_59, 1); +lean_inc(x_90); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_91 = x_59; +} else { + lean_dec_ref(x_59); + x_91 = lean_box(0); +} +if (lean_is_scalar(x_91)) { + x_92 = lean_alloc_ctor(1, 2, 0); +} else { + x_92 = x_91; +} +lean_ctor_set(x_92, 0, x_89); +lean_ctor_set(x_92, 1, x_90); +return x_92; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Rerunning pipeline on:\n", 23, 23); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Pipeline reached a fixpoint", 27, 27); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_name_eq(x_1, x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_13, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_3, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +return x_18; +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_14); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_20 = lean_ctor_get(x_14, 1); +x_21 = lean_ctor_get(x_14, 0); +lean_dec(x_21); +lean_inc(x_2); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_2); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2; +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_22); +lean_ctor_set(x_14, 0, x_23); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_14); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_20); +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_3, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_29 = lean_ctor_get(x_14, 1); +lean_inc(x_29); +lean_dec(x_14); +lean_inc(x_2); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_2); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +x_35 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_13, x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_29); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +lean_dec(x_35); +x_37 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(x_3, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +return x_37; +} +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +lean_dec(x_3); +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4; +x_39 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_unbox(x_40); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +lean_dec(x_39); +x_43 = lean_box(0); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_2, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_42); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_44; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_39, 1); +lean_inc(x_45); +lean_dec(x_39); +x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4; +x_47 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_38, x_46, x_5, x_6, x_7, x_8, x_9, x_10, x_45); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_2, x_48, x_5, x_6, x_7, x_8, x_9, x_10, x_49); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_48); +return x_50; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_box(0); +x_11 = lean_box(0); +lean_inc(x_2); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_2); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_13 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(x_1, x_10, x_11, x_1, x_1, x_12, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_box(0); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3(x_2, x_17, x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_16); +lean_dec(x_2); +return x_19; +} +else +{ +uint8_t x_20; +lean_dec(x_14); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_13); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_13, 0); +lean_dec(x_21); +x_22 = lean_ctor_get(x_15, 0); +lean_inc(x_22); +lean_dec(x_15); +lean_ctor_set(x_13, 0, x_22); +return x_13; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_13, 1); +lean_inc(x_23); +lean_dec(x_13); +x_24 = lean_ctor_get(x_15, 0); +lean_inc(x_24); +lean_dec(x_15); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; +} +} +} +else +{ +uint8_t x_26; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_13); +if (x_26 == 0) +{ +return x_13; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_13, 0); +x_28 = lean_ctor_get(x_13, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_13); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_3); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_4); +lean_dec(x_1); +return x_12; +} +} +lean_object* initialize_Lean_Meta_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__1(); +l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__2); +l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3 = _init_l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___closed__13); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_rewriteFinished___closed__4); +l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1 = _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1(); +lean_mark_persistent(l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__1); +l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2 = _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2(); +lean_mark_persistent(l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__2); +l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3 = _init_l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3(); +lean_mark_persistent(l___private_Lean_Util_Trace_0__Lean_getResetTraces___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__2___rarg___closed__3); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__1); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__3___closed__2); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__1); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__2); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__3); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__4(); +l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5 = _init_l_Lean_withTraceNode___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___spec__1___lambda__4___closed__5(); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_run___closed__1); +l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1 = _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___lambda__1___closed__1); +l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1 = _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__1); +l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2 = _init_l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___spec__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Pass_fixpointPipeline___lambda__3___closed__4); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/EmbeddedConstraint.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/EmbeddedConstraint.c new file mode 100644 index 000000000000..eadf2b985df2 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/EmbeddedConstraint.c @@ -0,0 +1,1895 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.EmbeddedConstraint +// Imports: Std.Tactic.BVDecide.Normalize.Bool Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic Lean.Meta.Tactic.Simp +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1; +size_t lean_uint64_to_usize(uint64_t); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isApp(lean_object*); +uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* l_Lean_Meta_simpGoal(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_array(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5; +lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4; +lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3; +lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1; +size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3; +uint64_t lean_uint64_shift_right(uint64_t, uint64_t); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_nat_div(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2; +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t l_Lean_Expr_hash(lean_object*); +lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Simp_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6; +extern lean_object* l_Lean_Meta_simpGlobalConfig; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7; +uint64_t lean_uint64_xor(uint64_t, uint64_t); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_nat_mul(lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1; +size_t lean_usize_sub(size_t, size_t); +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6; +lean_object* l_Lean_MVarId_tryClearMany(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uget(lean_object*, size_t); +size_t lean_array_size(lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get_size(lean_object*); +lean_object* l_Lean_LocalDecl_toExpr(lean_object*); +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3; +lean_object* lean_nat_add(lean_object*, lean_object*); +lean_object* l_Lean_Meta_SimpTheoremsArray_addTheorem(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2(lean_object*, lean_object*); +size_t lean_usize_land(size_t, size_t); +uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_1, 1); +lean_inc(x_15); +x_16 = lean_array_get_size(x_15); +x_17 = l_Lean_Expr_hash(x_2); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_CollectFVars_visit___spec__1(x_2, x_29); +if (x_30 == 0) +{ +uint8_t x_31; +x_31 = !lean_is_exclusive(x_1); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_32 = lean_ctor_get(x_1, 1); +lean_dec(x_32); +x_33 = lean_ctor_get(x_1, 0); +lean_dec(x_33); +x_34 = lean_unsigned_to_nat(1u); +x_35 = lean_nat_add(x_14, x_34); +lean_dec(x_14); +x_36 = lean_box(0); +x_37 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_37, 0, x_2); +lean_ctor_set(x_37, 1, x_36); +lean_ctor_set(x_37, 2, x_29); +x_38 = lean_array_uset(x_15, x_28, x_37); +x_39 = lean_unsigned_to_nat(4u); +x_40 = lean_nat_mul(x_35, x_39); +x_41 = lean_unsigned_to_nat(3u); +x_42 = lean_nat_div(x_40, x_41); +lean_dec(x_40); +x_43 = lean_array_get_size(x_38); +x_44 = lean_nat_dec_le(x_42, x_43); +lean_dec(x_43); +lean_dec(x_42); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_38); +lean_ctor_set(x_1, 1, x_45); +lean_ctor_set(x_1, 0, x_35); +lean_inc(x_9); +lean_inc(x_3); +x_46 = l_Lean_FVarId_getDecl(x_3, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_49 = l_Lean_LocalDecl_toExpr(x_47); +lean_dec(x_47); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_3); +x_51 = l_Lean_Meta_simpGlobalConfig; +x_52 = l_Lean_Meta_SimpTheoremsArray_addTheorem(x_4, x_50, x_49, x_51, x_9, x_10, x_11, x_12, x_48); +if (lean_obj_tag(x_52) == 0) +{ +uint8_t x_53; +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_1); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_5); +lean_ctor_set(x_56, 1, x_55); +x_57 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_52, 0, x_57); +return x_52; +} +else +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_58 = lean_ctor_get(x_52, 0); +x_59 = lean_ctor_get(x_52, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_52); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_1); +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_5); +lean_ctor_set(x_61, 1, x_60); +x_62 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_62, 0, x_61); +x_63 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_59); +return x_63; +} +} +else +{ +uint8_t x_64; +lean_dec(x_1); +lean_dec(x_5); +x_64 = !lean_is_exclusive(x_52); +if (x_64 == 0) +{ +return x_52; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_52, 0); +x_66 = lean_ctor_get(x_52, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_52); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; +} +} +} +else +{ +uint8_t x_68; +lean_dec(x_1); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_68 = !lean_is_exclusive(x_46); +if (x_68 == 0) +{ +return x_46; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_46, 0); +x_70 = lean_ctor_get(x_46, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_46); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +else +{ +lean_object* x_72; +lean_ctor_set(x_1, 1, x_38); +lean_ctor_set(x_1, 0, x_35); +lean_inc(x_9); +lean_inc(x_3); +x_72 = l_Lean_FVarId_getDecl(x_3, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); +x_75 = l_Lean_LocalDecl_toExpr(x_73); +lean_dec(x_73); +x_76 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_76, 0, x_3); +x_77 = l_Lean_Meta_simpGlobalConfig; +x_78 = l_Lean_Meta_SimpTheoremsArray_addTheorem(x_4, x_76, x_75, x_77, x_9, x_10, x_11, x_12, x_74); +if (lean_obj_tag(x_78) == 0) +{ +uint8_t x_79; +x_79 = !lean_is_exclusive(x_78); +if (x_79 == 0) +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_78, 0); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_1); +x_82 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_82, 0, x_5); +lean_ctor_set(x_82, 1, x_81); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_78, 0, x_83); +return x_78; +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_84 = lean_ctor_get(x_78, 0); +x_85 = lean_ctor_get(x_78, 1); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_78); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_84); +lean_ctor_set(x_86, 1, x_1); +x_87 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_87, 0, x_5); +lean_ctor_set(x_87, 1, x_86); +x_88 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_88, 0, x_87); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_85); +return x_89; +} +} +else +{ +uint8_t x_90; +lean_dec(x_1); +lean_dec(x_5); +x_90 = !lean_is_exclusive(x_78); +if (x_90 == 0) +{ +return x_78; +} +else +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_78, 0); +x_92 = lean_ctor_get(x_78, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_78); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; +} +} +} +else +{ +uint8_t x_94; +lean_dec(x_1); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_94 = !lean_is_exclusive(x_72); +if (x_94 == 0) +{ +return x_72; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_72, 0); +x_96 = lean_ctor_get(x_72, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_72); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; +} +} +} +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; +lean_dec(x_1); +x_98 = lean_unsigned_to_nat(1u); +x_99 = lean_nat_add(x_14, x_98); +lean_dec(x_14); +x_100 = lean_box(0); +x_101 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_101, 0, x_2); +lean_ctor_set(x_101, 1, x_100); +lean_ctor_set(x_101, 2, x_29); +x_102 = lean_array_uset(x_15, x_28, x_101); +x_103 = lean_unsigned_to_nat(4u); +x_104 = lean_nat_mul(x_99, x_103); +x_105 = lean_unsigned_to_nat(3u); +x_106 = lean_nat_div(x_104, x_105); +lean_dec(x_104); +x_107 = lean_array_get_size(x_102); +x_108 = lean_nat_dec_le(x_106, x_107); +lean_dec(x_107); +lean_dec(x_106); +if (x_108 == 0) +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_CollectFVars_visit___spec__2(x_102); +x_110 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_110, 0, x_99); +lean_ctor_set(x_110, 1, x_109); +lean_inc(x_9); +lean_inc(x_3); +x_111 = l_Lean_FVarId_getDecl(x_3, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_112 = lean_ctor_get(x_111, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 1); +lean_inc(x_113); +lean_dec(x_111); +x_114 = l_Lean_LocalDecl_toExpr(x_112); +lean_dec(x_112); +x_115 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_115, 0, x_3); +x_116 = l_Lean_Meta_simpGlobalConfig; +x_117 = l_Lean_Meta_SimpTheoremsArray_addTheorem(x_4, x_115, x_114, x_116, x_9, x_10, x_11, x_12, x_113); +if (lean_obj_tag(x_117) == 0) +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_117, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_120 = x_117; +} else { + lean_dec_ref(x_117); + x_120 = lean_box(0); +} +x_121 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_110); +x_122 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_122, 0, x_5); +lean_ctor_set(x_122, 1, x_121); +x_123 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_123, 0, x_122); +if (lean_is_scalar(x_120)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_120; +} +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_119); +return x_124; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_110); +lean_dec(x_5); +x_125 = lean_ctor_get(x_117, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_117, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_117)) { + lean_ctor_release(x_117, 0); + lean_ctor_release(x_117, 1); + x_127 = x_117; +} else { + lean_dec_ref(x_117); + x_127 = lean_box(0); +} +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); +} else { + x_128 = x_127; +} +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; +} +} +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +lean_dec(x_110); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_129 = lean_ctor_get(x_111, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_111, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + x_131 = x_111; +} else { + lean_dec_ref(x_111); + x_131 = lean_box(0); +} +if (lean_is_scalar(x_131)) { + x_132 = lean_alloc_ctor(1, 2, 0); +} else { + x_132 = x_131; +} +lean_ctor_set(x_132, 0, x_129); +lean_ctor_set(x_132, 1, x_130); +return x_132; +} +} +else +{ +lean_object* x_133; lean_object* x_134; +x_133 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_133, 0, x_99); +lean_ctor_set(x_133, 1, x_102); +lean_inc(x_9); +lean_inc(x_3); +x_134 = l_Lean_FVarId_getDecl(x_3, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_134) == 0) +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +lean_dec(x_134); +x_137 = l_Lean_LocalDecl_toExpr(x_135); +lean_dec(x_135); +x_138 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_138, 0, x_3); +x_139 = l_Lean_Meta_simpGlobalConfig; +x_140 = l_Lean_Meta_SimpTheoremsArray_addTheorem(x_4, x_138, x_137, x_139, x_9, x_10, x_11, x_12, x_136); +if (lean_obj_tag(x_140) == 0) +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_141 = lean_ctor_get(x_140, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_140, 1); +lean_inc(x_142); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_143 = x_140; +} else { + lean_dec_ref(x_140); + x_143 = lean_box(0); +} +x_144 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_144, 0, x_141); +lean_ctor_set(x_144, 1, x_133); +x_145 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_145, 0, x_5); +lean_ctor_set(x_145, 1, x_144); +x_146 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_146, 0, x_145); +if (lean_is_scalar(x_143)) { + x_147 = lean_alloc_ctor(0, 2, 0); +} else { + x_147 = x_143; +} +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_142); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_133); +lean_dec(x_5); +x_148 = lean_ctor_get(x_140, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_140, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_140)) { + lean_ctor_release(x_140, 0); + lean_ctor_release(x_140, 1); + x_150 = x_140; +} else { + lean_dec_ref(x_140); + x_150 = lean_box(0); +} +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); +} else { + x_151 = x_150; +} +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; +} +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +lean_dec(x_133); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_152 = lean_ctor_get(x_134, 0); +lean_inc(x_152); +x_153 = lean_ctor_get(x_134, 1); +lean_inc(x_153); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_154 = x_134; +} else { + lean_dec_ref(x_134); + x_154 = lean_box(0); +} +if (lean_is_scalar(x_154)) { + x_155 = lean_alloc_ctor(1, 2, 0); +} else { + x_155 = x_154; +} +lean_ctor_set(x_155, 0, x_152); +lean_ctor_set(x_155, 1, x_153); +return x_155; +} +} +} +} +else +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_29); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +x_156 = lean_array_push(x_5, x_3); +x_157 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_157, 0, x_4); +lean_ctor_set(x_157, 1, x_1); +x_158 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_158, 0, x_156); +lean_ctor_set(x_158, 1, x_157); +x_159 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_159, 0, x_158); +x_160 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_160, 0, x_159); +lean_ctor_set(x_160, 1, x_13); +return x_160; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_2); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_11); +return x_15; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Bool", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1; +x_2 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = l_Lean_Expr_cleanupAnnotations(x_6); +x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3; +x_16 = l_Lean_Expr_isConstOf(x_14, x_15); +lean_dec(x_14); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_5); +lean_dec(x_2); +x_17 = lean_box(0); +x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_3, x_1, x_4, x_17, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_box(0); +x_20 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1(x_1, x_5, x_2, x_3, x_4, x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_20; +} +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Eq", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; +x_14 = lean_usize_dec_lt(x_5, x_4); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_6); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_16 = lean_array_uget(x_3, x_5); +x_26 = lean_ctor_get(x_6, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_6, 0); +lean_inc(x_27); +lean_dec(x_6); +x_28 = lean_ctor_get(x_26, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_26, 1); +lean_inc(x_29); +lean_dec(x_26); +lean_inc(x_9); +lean_inc(x_16); +x_30 = l_Lean_FVarId_getType(x_16, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l_Lean_Expr_cleanupAnnotations(x_31); +x_34 = l_Lean_Expr_isApp(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_33); +lean_dec(x_16); +x_35 = lean_box(0); +x_36 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_28, x_29, x_27, x_35, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_17 = x_37; +x_18 = x_38; +goto block_25; +} +else +{ +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = l_Lean_Expr_appArg(x_33, lean_box(0)); +x_40 = l_Lean_Expr_appFnCleanup(x_33, lean_box(0)); +x_41 = l_Lean_Expr_isApp(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_16); +x_42 = lean_box(0); +x_43 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_28, x_29, x_27, x_42, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_17 = x_44; +x_18 = x_45; +goto block_25; +} +else +{ +lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = l_Lean_Expr_appArg(x_40, lean_box(0)); +x_47 = l_Lean_Expr_appFnCleanup(x_40, lean_box(0)); +x_48 = l_Lean_Expr_isApp(x_47); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_47); +lean_dec(x_46); +lean_dec(x_39); +lean_dec(x_16); +x_49 = lean_box(0); +x_50 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_28, x_29, x_27, x_49, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_17 = x_51; +x_18 = x_52; +goto block_25; +} +else +{ +lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_53 = l_Lean_Expr_appFnCleanup(x_47, lean_box(0)); +x_54 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2; +x_55 = l_Lean_Expr_isConstOf(x_53, x_54); +lean_dec(x_53); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_dec(x_46); +lean_dec(x_39); +lean_dec(x_16); +x_56 = lean_box(0); +x_57 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_28, x_29, x_27, x_56, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_17 = x_58; +x_18 = x_59; +goto block_25; +} +else +{ +lean_object* x_60; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_60 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3(x_29, x_16, x_28, x_27, x_46, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +lean_dec(x_60); +x_17 = x_61; +x_18 = x_62; +goto block_25; +} +else +{ +uint8_t x_63; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_63 = !lean_is_exclusive(x_60); +if (x_63 == 0) +{ +return x_60; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_60, 0); +x_65 = lean_ctor_get(x_60, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_60); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; +} +} +} +} +} +} +} +else +{ +uint8_t x_67; +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_67 = !lean_is_exclusive(x_30); +if (x_67 == 0) +{ +return x_30; +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_30, 0); +x_69 = lean_ctor_get(x_30, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_30); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; +} +} +block_25: +{ +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +else +{ +lean_object* x_21; size_t x_22; size_t x_23; +x_21 = lean_ctor_get(x_17, 0); +lean_inc(x_21); +lean_dec(x_17); +x_22 = 1; +x_23 = lean_usize_add(x_5, x_22); +x_5 = x_23; +x_6 = x_21; +x_13 = x_18; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_10 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_apply_8(x_2, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_13; +} +else +{ +uint8_t x_14; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) +{ +return x_10; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2___rarg), 9, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_apply_2(x_2, x_3, x_4); +x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +return x_11; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_11, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_11); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3___rarg), 9, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_MVarId_getNondepPropHyps(x_1, x_4, x_5, x_6, x_7, x_8); +return x_9; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(32u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6() { +_start: +{ +size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = 5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_4); +lean_ctor_set(x_5, 3, x_4); +lean_ctor_set_usize(x_5, 4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6; +x_3 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_1); +lean_ctor_set(x_3, 3, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; uint8_t x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_12 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_ctor_get(x_5, 1); +x_16 = lean_unsigned_to_nat(2u); +x_17 = 0; +x_18 = 1; +x_19 = 0; +lean_inc(x_15); +x_20 = lean_alloc_ctor(0, 2, 19); +lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 1, x_16); +lean_ctor_set_uint8(x_20, sizeof(void*)*2, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 1, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 2, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 3, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 4, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 5, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 6, x_19); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 7, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 8, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 9, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 10, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 11, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 12, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 13, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 14, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 15, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 16, x_17); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 17, x_18); +lean_ctor_set_uint8(x_20, sizeof(void*)*2 + 18, x_18); +x_21 = l_Lean_Meta_Simp_mkContext(x_20, x_1, x_13, x_7, x_8, x_9, x_10, x_14); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_24 = l_Lean_MVarId_getNondepPropHyps(x_2, x_7, x_8, x_9, x_10, x_23); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_box(0); +x_28 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8; +x_29 = l_Lean_Meta_simpGoal(x_2, x_22, x_3, x_27, x_18, x_25, x_28, x_7, x_8, x_9, x_10, x_26); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +if (lean_obj_tag(x_31) == 0) +{ +uint8_t x_32; +x_32 = !lean_is_exclusive(x_29); +if (x_32 == 0) +{ +lean_object* x_33; +x_33 = lean_ctor_get(x_29, 0); +lean_dec(x_33); +lean_ctor_set(x_29, 0, x_27); +return x_29; +} +else +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_dec(x_29); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_27); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_31); +if (x_36 == 0) +{ +uint8_t x_37; +x_37 = !lean_is_exclusive(x_29); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_31, 0); +x_39 = lean_ctor_get(x_29, 0); +lean_dec(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +lean_ctor_set(x_31, 0, x_40); +lean_ctor_set(x_29, 0, x_31); +return x_29; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_41 = lean_ctor_get(x_31, 0); +x_42 = lean_ctor_get(x_29, 1); +lean_inc(x_42); +lean_dec(x_29); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +lean_ctor_set(x_31, 0, x_43); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_31); +lean_ctor_set(x_44, 1, x_42); +return x_44; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_31, 0); +lean_inc(x_45); +lean_dec(x_31); +x_46 = lean_ctor_get(x_29, 1); +lean_inc(x_46); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_47 = x_29; +} else { + lean_dec_ref(x_29); + x_47 = lean_box(0); +} +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +lean_dec(x_45); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +if (lean_is_scalar(x_47)) { + x_50 = lean_alloc_ctor(0, 2, 0); +} else { + x_50 = x_47; +} +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_46); +return x_50; +} +} +} +else +{ +uint8_t x_51; +x_51 = !lean_is_exclusive(x_29); +if (x_51 == 0) +{ +return x_29; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_29, 0); +x_53 = lean_ctor_get(x_29, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_29); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +} +} +else +{ +uint8_t x_55; +lean_dec(x_22); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +x_55 = !lean_is_exclusive(x_24); +if (x_55 == 0) +{ +return x_24; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_24, 0); +x_57 = lean_ctor_get(x_24, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_24); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(10u); +x_2 = lean_unsigned_to_nat(1u); +x_3 = l_Nat_nextPowerOfTwo_go(x_1, x_2, lean_box(0)); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2; +x_3 = lean_mk_array(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; size_t x_11; size_t x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_box(0); +x_11 = lean_array_size(x_2); +x_12 = 0; +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1(x_2, x_10, x_2, x_11, x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_ctor_get(x_15, 0); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_ctor_get(x_16, 0); +lean_inc(x_19); +lean_dec(x_16); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_20 = l_Lean_MVarId_tryClearMany(x_1, x_18, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_18); +if (lean_obj_tag(x_20) == 0) +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = l_Array_isEmpty___rarg(x_19); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_free_object(x_20); +x_25 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1; +x_26 = lean_box(0); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2(x_19, x_22, x_25, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_23); +return x_27; +} +else +{ +lean_object* x_28; +lean_dec(x_19); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_20, 0, x_28); +return x_20; +} +} +else +{ +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_20, 0); +x_30 = lean_ctor_get(x_20, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_20); +x_31 = l_Array_isEmpty___rarg(x_19); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1; +x_33 = lean_box(0); +x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2(x_19, x_29, x_32, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_30); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_19); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_29); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_30); +return x_36; +} +} +} +else +{ +uint8_t x_37; +lean_dec(x_19); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_37 = !lean_is_exclusive(x_20); +if (x_37 == 0) +{ +return x_20; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_20, 0); +x_39 = lean_ctor_get(x_20, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_20); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_14); +if (x_41 == 0) +{ +return x_14; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_14, 0); +x_43 = lean_ctor_get(x_14, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_14); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1___boxed), 8, 1); +lean_closure_set(x_9, 0, x_1); +lean_inc(x_1); +x_10 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___boxed), 9, 1); +lean_closure_set(x_10, 0, x_1); +x_11 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__2___rarg), 9, 2); +lean_closure_set(x_11, 0, x_9); +lean_closure_set(x_11, 1, x_10); +x_12 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__3___rarg(x_1, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("embeddedConstraintSubsitution", 29, 29); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_7); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +size_t x_14; size_t x_15; lean_object* x_16; +x_14 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_15 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_16 = l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1(x_1, x_2, x_3, x_14, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +lean_object* initialize_Std_Tactic_BVDecide_Normalize_Bool(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Simp(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_EmbeddedConstraint(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Tactic_BVDecide_Normalize_Bool(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Simp(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__2); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___lambda__3___closed__3); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___spec__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__2___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___elambda__1___lambda__3___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_embeddedConstraintPass); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Rewrite.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Rewrite.c new file mode 100644 index 000000000000..495044b7f839 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Rewrite.c @@ -0,0 +1,3691 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Rewrite +// Imports: Lean.Elab.Tactic.Simp Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Basic Lean.Elab.Tactic.BVDecide.Frontend.Attr +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeExt; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10; +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2; +size_t lean_uint64_to_usize(uint64_t); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* l_Lean_Meta_simpGoal(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1; +lean_object* l_Lean_stringToMessageData(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3; +lean_object* l_Lean_Meta_getSimpCongrTheorems___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3; +uint64_t l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(lean_object*); +size_t lean_usize_of_nat(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4; +lean_object* l_Lean_MVarId_getNondepPropHyps(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_take(lean_object*, lean_object*); +extern lean_object* l_Lean_Meta_sevalSimpExtension; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass; +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3(lean_object*); +uint64_t lean_uint64_shift_right(uint64_t, uint64_t); +lean_object* l_Lean_Meta_Simp_SimprocExtension_getSimprocs(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_nat_div(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2; +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_object* lean_st_ref_get(lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14; +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Simp_getSEvalSimprocs___rarg(lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Simp_mkContext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9; +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2(lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofExpr(lean_object*); +lean_object* l_Lean_Meta_SimpExtension_getTheorems(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4; +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9; +uint64_t lean_uint64_xor(uint64_t, uint64_t); +lean_object* lean_nat_mul(lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(lean_object*); +lean_object* l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1; +lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4; +size_t lean_usize_sub(size_t, size_t); +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8; +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7; +size_t lean_usize_add(size_t, size_t); +static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3; +lean_object* lean_array_uget(lean_object*, size_t); +lean_object* l_Lean_Expr_fvar___override(lean_object*); +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(lean_object*, lean_object*); +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10; +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5; +size_t lean_usize_land(size_t, size_t); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Array_isEmpty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___lambda__1(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(x_1); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Meta", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bv", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1; +x_2 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2; +x_3 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" was already rewritten\? ", 24, 24); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("false", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_eq(x_2, x_3); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_20; lean_object* x_21; lean_object* x_24; uint8_t x_25; +x_13 = lean_array_uget(x_1, x_2); +x_24 = lean_st_ref_get(x_6, x_11); +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_24, 0); +x_27 = lean_ctor_get(x_24, 1); +x_28 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4; +x_29 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +x_30 = !lean_is_exclusive(x_26); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_ctor_get(x_26, 1); +x_32 = lean_ctor_get(x_26, 0); +lean_dec(x_32); +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint64_t x_37; uint64_t x_38; uint64_t x_39; uint64_t x_40; uint64_t x_41; uint64_t x_42; uint64_t x_43; size_t x_44; size_t x_45; size_t x_46; size_t x_47; size_t x_48; lean_object* x_49; uint8_t x_50; uint8_t x_51; +x_34 = lean_ctor_get(x_29, 0); +x_35 = lean_ctor_get(x_29, 1); +x_36 = lean_array_get_size(x_31); +x_37 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_13); +x_38 = 32; +x_39 = lean_uint64_shift_right(x_37, x_38); +x_40 = lean_uint64_xor(x_37, x_39); +x_41 = 16; +x_42 = lean_uint64_shift_right(x_40, x_41); +x_43 = lean_uint64_xor(x_40, x_42); +x_44 = lean_uint64_to_usize(x_43); +x_45 = lean_usize_of_nat(x_36); +lean_dec(x_36); +x_46 = 1; +x_47 = lean_usize_sub(x_45, x_46); +x_48 = lean_usize_land(x_44, x_47); +x_49 = lean_array_uget(x_31, x_48); +lean_dec(x_31); +x_50 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_13, x_49); +lean_dec(x_49); +x_51 = lean_unbox(x_34); +lean_dec(x_34); +if (x_51 == 0) +{ +lean_free_object(x_29); +lean_free_object(x_26); +lean_free_object(x_24); +if (x_50 == 0) +{ +uint8_t x_52; +x_52 = 1; +x_20 = x_52; +x_21 = x_35; +goto block_23; +} +else +{ +uint8_t x_53; +x_53 = 0; +x_20 = x_53; +x_21 = x_35; +goto block_23; +} +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_inc(x_13); +x_54 = l_Lean_Expr_fvar___override(x_13); +x_55 = l_Lean_MessageData_ofExpr(x_54); +x_56 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6; +lean_ctor_set_tag(x_29, 7); +lean_ctor_set(x_29, 1, x_55); +lean_ctor_set(x_29, 0, x_56); +x_57 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8; +lean_ctor_set_tag(x_26, 7); +lean_ctor_set(x_26, 1, x_57); +lean_ctor_set(x_26, 0, x_29); +if (x_50 == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_58 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_58); +x_59 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_59, 0, x_24); +lean_ctor_set(x_59, 1, x_56); +x_60 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_59, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +x_62 = 1; +x_20 = x_62; +x_21 = x_61; +goto block_23; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; +x_63 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_63); +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_24); +lean_ctor_set(x_64, 1, x_56); +x_65 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_64, x_5, x_6, x_7, x_8, x_9, x_10, x_35); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = 0; +x_20 = x_67; +x_21 = x_66; +goto block_23; +} +} +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; uint64_t x_71; uint64_t x_72; uint64_t x_73; uint64_t x_74; uint64_t x_75; uint64_t x_76; uint64_t x_77; size_t x_78; size_t x_79; size_t x_80; size_t x_81; size_t x_82; lean_object* x_83; uint8_t x_84; uint8_t x_85; +x_68 = lean_ctor_get(x_29, 0); +x_69 = lean_ctor_get(x_29, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_29); +x_70 = lean_array_get_size(x_31); +x_71 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_13); +x_72 = 32; +x_73 = lean_uint64_shift_right(x_71, x_72); +x_74 = lean_uint64_xor(x_71, x_73); +x_75 = 16; +x_76 = lean_uint64_shift_right(x_74, x_75); +x_77 = lean_uint64_xor(x_74, x_76); +x_78 = lean_uint64_to_usize(x_77); +x_79 = lean_usize_of_nat(x_70); +lean_dec(x_70); +x_80 = 1; +x_81 = lean_usize_sub(x_79, x_80); +x_82 = lean_usize_land(x_78, x_81); +x_83 = lean_array_uget(x_31, x_82); +lean_dec(x_31); +x_84 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_13, x_83); +lean_dec(x_83); +x_85 = lean_unbox(x_68); +lean_dec(x_68); +if (x_85 == 0) +{ +lean_free_object(x_26); +lean_free_object(x_24); +if (x_84 == 0) +{ +uint8_t x_86; +x_86 = 1; +x_20 = x_86; +x_21 = x_69; +goto block_23; +} +else +{ +uint8_t x_87; +x_87 = 0; +x_20 = x_87; +x_21 = x_69; +goto block_23; +} +} +else +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_inc(x_13); +x_88 = l_Lean_Expr_fvar___override(x_13); +x_89 = l_Lean_MessageData_ofExpr(x_88); +x_90 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6; +x_91 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_89); +x_92 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8; +lean_ctor_set_tag(x_26, 7); +lean_ctor_set(x_26, 1, x_92); +lean_ctor_set(x_26, 0, x_91); +if (x_84 == 0) +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_93 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_93); +x_94 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_94, 0, x_24); +lean_ctor_set(x_94, 1, x_90); +x_95 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_94, x_5, x_6, x_7, x_8, x_9, x_10, x_69); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +lean_dec(x_95); +x_97 = 1; +x_20 = x_97; +x_21 = x_96; +goto block_23; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_98 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_98); +x_99 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_99, 0, x_24); +lean_ctor_set(x_99, 1, x_90); +x_100 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_99, x_5, x_6, x_7, x_8, x_9, x_10, x_69); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +x_102 = 0; +x_20 = x_102; +x_21 = x_101; +goto block_23; +} +} +} +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint64_t x_108; uint64_t x_109; uint64_t x_110; uint64_t x_111; uint64_t x_112; uint64_t x_113; uint64_t x_114; size_t x_115; size_t x_116; size_t x_117; size_t x_118; size_t x_119; lean_object* x_120; uint8_t x_121; uint8_t x_122; +x_103 = lean_ctor_get(x_26, 1); +lean_inc(x_103); +lean_dec(x_26); +x_104 = lean_ctor_get(x_29, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_29, 1); +lean_inc(x_105); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_106 = x_29; +} else { + lean_dec_ref(x_29); + x_106 = lean_box(0); +} +x_107 = lean_array_get_size(x_103); +x_108 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_13); +x_109 = 32; +x_110 = lean_uint64_shift_right(x_108, x_109); +x_111 = lean_uint64_xor(x_108, x_110); +x_112 = 16; +x_113 = lean_uint64_shift_right(x_111, x_112); +x_114 = lean_uint64_xor(x_111, x_113); +x_115 = lean_uint64_to_usize(x_114); +x_116 = lean_usize_of_nat(x_107); +lean_dec(x_107); +x_117 = 1; +x_118 = lean_usize_sub(x_116, x_117); +x_119 = lean_usize_land(x_115, x_118); +x_120 = lean_array_uget(x_103, x_119); +lean_dec(x_103); +x_121 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_13, x_120); +lean_dec(x_120); +x_122 = lean_unbox(x_104); +lean_dec(x_104); +if (x_122 == 0) +{ +lean_dec(x_106); +lean_free_object(x_24); +if (x_121 == 0) +{ +uint8_t x_123; +x_123 = 1; +x_20 = x_123; +x_21 = x_105; +goto block_23; +} +else +{ +uint8_t x_124; +x_124 = 0; +x_20 = x_124; +x_21 = x_105; +goto block_23; +} +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +lean_inc(x_13); +x_125 = l_Lean_Expr_fvar___override(x_13); +x_126 = l_Lean_MessageData_ofExpr(x_125); +x_127 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6; +if (lean_is_scalar(x_106)) { + x_128 = lean_alloc_ctor(7, 2, 0); +} else { + x_128 = x_106; + lean_ctor_set_tag(x_128, 7); +} +lean_ctor_set(x_128, 0, x_127); +lean_ctor_set(x_128, 1, x_126); +x_129 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8; +x_130 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +if (x_121 == 0) +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; +x_131 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_131); +lean_ctor_set(x_24, 0, x_130); +x_132 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_132, 0, x_24); +lean_ctor_set(x_132, 1, x_127); +x_133 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_132, x_5, x_6, x_7, x_8, x_9, x_10, x_105); +x_134 = lean_ctor_get(x_133, 1); +lean_inc(x_134); +lean_dec(x_133); +x_135 = 1; +x_20 = x_135; +x_21 = x_134; +goto block_23; +} +else +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; uint8_t x_140; +x_136 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_136); +lean_ctor_set(x_24, 0, x_130); +x_137 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_137, 0, x_24); +lean_ctor_set(x_137, 1, x_127); +x_138 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_28, x_137, x_5, x_6, x_7, x_8, x_9, x_10, x_105); +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +lean_dec(x_138); +x_140 = 0; +x_20 = x_140; +x_21 = x_139; +goto block_23; +} +} +} +} +else +{ +lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; uint64_t x_151; uint64_t x_152; uint64_t x_153; uint64_t x_154; uint64_t x_155; uint64_t x_156; uint64_t x_157; size_t x_158; size_t x_159; size_t x_160; size_t x_161; size_t x_162; lean_object* x_163; uint8_t x_164; uint8_t x_165; +x_141 = lean_ctor_get(x_24, 0); +x_142 = lean_ctor_get(x_24, 1); +lean_inc(x_142); +lean_inc(x_141); +lean_dec(x_24); +x_143 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4; +x_144 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_143, x_5, x_6, x_7, x_8, x_9, x_10, x_142); +x_145 = lean_ctor_get(x_141, 1); +lean_inc(x_145); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_146 = x_141; +} else { + lean_dec_ref(x_141); + x_146 = lean_box(0); +} +x_147 = lean_ctor_get(x_144, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_144, 1); +lean_inc(x_148); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_149 = x_144; +} else { + lean_dec_ref(x_144); + x_149 = lean_box(0); +} +x_150 = lean_array_get_size(x_145); +x_151 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_13); +x_152 = 32; +x_153 = lean_uint64_shift_right(x_151, x_152); +x_154 = lean_uint64_xor(x_151, x_153); +x_155 = 16; +x_156 = lean_uint64_shift_right(x_154, x_155); +x_157 = lean_uint64_xor(x_154, x_156); +x_158 = lean_uint64_to_usize(x_157); +x_159 = lean_usize_of_nat(x_150); +lean_dec(x_150); +x_160 = 1; +x_161 = lean_usize_sub(x_159, x_160); +x_162 = lean_usize_land(x_158, x_161); +x_163 = lean_array_uget(x_145, x_162); +lean_dec(x_145); +x_164 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_13, x_163); +lean_dec(x_163); +x_165 = lean_unbox(x_147); +lean_dec(x_147); +if (x_165 == 0) +{ +lean_dec(x_149); +lean_dec(x_146); +if (x_164 == 0) +{ +uint8_t x_166; +x_166 = 1; +x_20 = x_166; +x_21 = x_148; +goto block_23; +} +else +{ +uint8_t x_167; +x_167 = 0; +x_20 = x_167; +x_21 = x_148; +goto block_23; +} +} +else +{ +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_inc(x_13); +x_168 = l_Lean_Expr_fvar___override(x_13); +x_169 = l_Lean_MessageData_ofExpr(x_168); +x_170 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6; +if (lean_is_scalar(x_149)) { + x_171 = lean_alloc_ctor(7, 2, 0); +} else { + x_171 = x_149; + lean_ctor_set_tag(x_171, 7); +} +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_169); +x_172 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8; +if (lean_is_scalar(x_146)) { + x_173 = lean_alloc_ctor(7, 2, 0); +} else { + x_173 = x_146; + lean_ctor_set_tag(x_173, 7); +} +lean_ctor_set(x_173, 0, x_171); +lean_ctor_set(x_173, 1, x_172); +if (x_164 == 0) +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; uint8_t x_179; +x_174 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11; +x_175 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_175, 0, x_173); +lean_ctor_set(x_175, 1, x_174); +x_176 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_176, 0, x_175); +lean_ctor_set(x_176, 1, x_170); +x_177 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_143, x_176, x_5, x_6, x_7, x_8, x_9, x_10, x_148); +x_178 = lean_ctor_get(x_177, 1); +lean_inc(x_178); +lean_dec(x_177); +x_179 = 1; +x_20 = x_179; +x_21 = x_178; +goto block_23; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; uint8_t x_185; +x_180 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14; +x_181 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_181, 0, x_173); +lean_ctor_set(x_181, 1, x_180); +x_182 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_170); +x_183 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_143, x_182, x_5, x_6, x_7, x_8, x_9, x_10, x_148); +x_184 = lean_ctor_get(x_183, 1); +lean_inc(x_184); +lean_dec(x_183); +x_185 = 0; +x_20 = x_185; +x_21 = x_184; +goto block_23; +} +} +} +block_19: +{ +size_t x_16; size_t x_17; +x_16 = 1; +x_17 = lean_usize_add(x_2, x_16); +x_2 = x_17; +x_4 = x_14; +x_11 = x_15; +goto _start; +} +block_23: +{ +if (x_20 == 0) +{ +lean_dec(x_13); +x_14 = x_4; +x_15 = x_21; +goto block_19; +} +else +{ +lean_object* x_22; +x_22 = lean_array_push(x_4, x_13); +x_14 = x_22; +x_15 = x_21; +goto block_19; +} +} +} +else +{ +lean_object* x_186; +x_186 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_186, 0, x_4); +lean_ctor_set(x_186, 1, x_11); +return x_186; +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_10 = lean_apply_7(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_10) == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_apply_8(x_2, x_11, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_13; +} +else +{ +uint8_t x_14; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_10); +if (x_14 == 0) +{ +return x_10; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_apply_2(x_2, x_3, x_4); +x_11 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_10, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +else +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_11); +if (x_16 == 0) +{ +return x_11; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_11, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_11); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg), 9, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_MVarId_getNondepPropHyps(x_1, x_4, x_5, x_6, x_7, x_8); +return x_9; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_9); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_8); +return x_13; +} +else +{ +uint8_t x_14; +x_14 = lean_nat_dec_le(x_9, x_9); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_9); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_8); +return x_16; +} +else +{ +size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; +x_17 = 0; +x_18 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1; +x_20 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1(x_1, x_17, x_18, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_20; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___boxed), 8, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +lean_inc(x_1); +x_9 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_9, 0, x_1); +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1; +x_11 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_11, 0, x_9); +lean_closure_set(x_11, 1, x_10); +x_12 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_1, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; lean_object* x_11; +x_10 = lean_unbox(x_1); +lean_dec(x_1); +x_11 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___lambda__1(x_10, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +lean_dec(x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_st_ref_take(x_4, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_11, 0); +x_15 = lean_ctor_get(x_11, 1); +x_16 = lean_array_get_size(x_15); +x_17 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_14, x_31); +lean_dec(x_14); +x_33 = lean_box(0); +x_34 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_34, 0, x_1); +lean_ctor_set(x_34, 1, x_33); +lean_ctor_set(x_34, 2, x_29); +x_35 = lean_array_uset(x_15, x_28, x_34); +x_36 = lean_unsigned_to_nat(4u); +x_37 = lean_nat_mul(x_32, x_36); +x_38 = lean_unsigned_to_nat(3u); +x_39 = lean_nat_div(x_37, x_38); +lean_dec(x_37); +x_40 = lean_array_get_size(x_35); +x_41 = lean_nat_dec_le(x_39, x_40); +lean_dec(x_40); +lean_dec(x_39); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_35); +lean_ctor_set(x_11, 1, x_42); +lean_ctor_set(x_11, 0, x_32); +x_43 = lean_st_ref_set(x_4, x_11, x_12); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +lean_ctor_set(x_43, 0, x_33); +return x_43; +} +else +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_dec(x_43); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_33); +lean_ctor_set(x_47, 1, x_46); +return x_47; +} +} +else +{ +lean_object* x_48; uint8_t x_49; +lean_ctor_set(x_11, 1, x_35); +lean_ctor_set(x_11, 0, x_32); +x_48 = lean_st_ref_set(x_4, x_11, x_12); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; +x_50 = lean_ctor_get(x_48, 0); +lean_dec(x_50); +lean_ctor_set(x_48, 0, x_33); +return x_48; +} +else +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_48, 1); +lean_inc(x_51); +lean_dec(x_48); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_33); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +lean_object* x_53; uint8_t x_54; +lean_dec(x_29); +lean_dec(x_1); +x_53 = lean_st_ref_set(x_4, x_11, x_12); +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_53, 0); +lean_dec(x_55); +x_56 = lean_box(0); +lean_ctor_set(x_53, 0, x_56); +return x_53; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_53, 1); +lean_inc(x_57); +lean_dec(x_53); +x_58 = lean_box(0); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_57); +return x_59; +} +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; uint64_t x_68; uint64_t x_69; size_t x_70; size_t x_71; size_t x_72; size_t x_73; size_t x_74; lean_object* x_75; uint8_t x_76; +x_60 = lean_ctor_get(x_11, 0); +x_61 = lean_ctor_get(x_11, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_11); +x_62 = lean_array_get_size(x_61); +x_63 = l___private_Lean_Expr_0__Lean_hashFVarId____x40_Lean_Expr___hyg_1730_(x_1); +x_64 = 32; +x_65 = lean_uint64_shift_right(x_63, x_64); +x_66 = lean_uint64_xor(x_63, x_65); +x_67 = 16; +x_68 = lean_uint64_shift_right(x_66, x_67); +x_69 = lean_uint64_xor(x_66, x_68); +x_70 = lean_uint64_to_usize(x_69); +x_71 = lean_usize_of_nat(x_62); +lean_dec(x_62); +x_72 = 1; +x_73 = lean_usize_sub(x_71, x_72); +x_74 = lean_usize_land(x_70, x_73); +x_75 = lean_array_uget(x_61, x_74); +x_76 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_MVarId_getNondepPropHyps___spec__1(x_1, x_75); +if (x_76 == 0) +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; +x_77 = lean_unsigned_to_nat(1u); +x_78 = lean_nat_add(x_60, x_77); +lean_dec(x_60); +x_79 = lean_box(0); +x_80 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_80, 0, x_1); +lean_ctor_set(x_80, 1, x_79); +lean_ctor_set(x_80, 2, x_75); +x_81 = lean_array_uset(x_61, x_74, x_80); +x_82 = lean_unsigned_to_nat(4u); +x_83 = lean_nat_mul(x_78, x_82); +x_84 = lean_unsigned_to_nat(3u); +x_85 = lean_nat_div(x_83, x_84); +lean_dec(x_83); +x_86 = lean_array_get_size(x_81); +x_87 = lean_nat_dec_le(x_85, x_86); +lean_dec(x_86); +lean_dec(x_85); +if (x_87 == 0) +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_88 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_MVarId_getNondepPropHyps___spec__7(x_81); +x_89 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_89, 0, x_78); +lean_ctor_set(x_89, 1, x_88); +x_90 = lean_st_ref_set(x_4, x_89, x_12); +x_91 = lean_ctor_get(x_90, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_90)) { + lean_ctor_release(x_90, 0); + lean_ctor_release(x_90, 1); + x_92 = x_90; +} else { + lean_dec_ref(x_90); + x_92 = lean_box(0); +} +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_92; +} +lean_ctor_set(x_93, 0, x_79); +lean_ctor_set(x_93, 1, x_91); +return x_93; +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_94 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_94, 0, x_78); +lean_ctor_set(x_94, 1, x_81); +x_95 = lean_st_ref_set(x_4, x_94, x_12); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_95)) { + lean_ctor_release(x_95, 0); + lean_ctor_release(x_95, 1); + x_97 = x_95; +} else { + lean_dec_ref(x_95); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(0, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_79); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +lean_dec(x_75); +lean_dec(x_1); +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_60); +lean_ctor_set(x_99, 1, x_61); +x_100 = lean_st_ref_set(x_4, x_99, x_12); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_102 = x_100; +} else { + lean_dec_ref(x_100); + x_102 = lean_box(0); +} +x_103 = lean_box(0); +if (lean_is_scalar(x_102)) { + x_104 = lean_alloc_ctor(0, 2, 0); +} else { + x_104 = x_102; +} +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_101); +return x_104; +} +} +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Adding ", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" to the rewritten set", 21, 21); +return x_1; +} +} +static lean_object* _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = lean_usize_dec_eq(x_2, x_3); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_dec(x_4); +x_13 = lean_array_uget(x_1, x_2); +x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4; +x_15 = l_Lean_isTracingEnabledFor___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__1(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_box(0); +x_20 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(x_13, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 1; +x_24 = lean_usize_add(x_2, x_23); +x_2 = x_24; +x_4 = x_21; +x_11 = x_22; +goto _start; +} +else +{ +uint8_t x_26; +x_26 = !lean_is_exclusive(x_15); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; size_t x_40; size_t x_41; +x_27 = lean_ctor_get(x_15, 1); +x_28 = lean_ctor_get(x_15, 0); +lean_dec(x_28); +lean_inc(x_13); +x_29 = l_Lean_Expr_fvar___override(x_13); +x_30 = l_Lean_MessageData_ofExpr(x_29); +x_31 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_30); +lean_ctor_set(x_15, 0, x_31); +x_32 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_15); +lean_ctor_set(x_33, 1, x_32); +x_34 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_14, x_33, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(x_13, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_36); +lean_dec(x_35); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = 1; +x_41 = lean_usize_add(x_2, x_40); +x_2 = x_41; +x_4 = x_38; +x_11 = x_39; +goto _start; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; size_t x_56; size_t x_57; +x_43 = lean_ctor_get(x_15, 1); +lean_inc(x_43); +lean_dec(x_15); +lean_inc(x_13); +x_44 = l_Lean_Expr_fvar___override(x_13); +x_45 = l_Lean_MessageData_ofExpr(x_44); +x_46 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2; +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +x_48 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_addTrace___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_PreProcessM_checkRewritten___spec__2(x_14, x_49, x_5, x_6, x_7, x_8, x_9, x_10, x_43); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(x_13, x_51, x_5, x_6, x_7, x_8, x_9, x_10, x_52); +lean_dec(x_51); +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +x_56 = 1; +x_57 = lean_usize_add(x_2, x_56); +x_2 = x_57; +x_4 = x_54; +x_11 = x_55; +goto _start; +} +} +} +else +{ +lean_object* x_59; +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_4); +lean_ctor_set(x_59, 1, x_11); +return x_59; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_array_get_size(x_1); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_lt(x_10, x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_9); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_8); +return x_13; +} +else +{ +uint8_t x_14; +x_14 = lean_nat_dec_le(x_9, x_9); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_9); +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_8); +return x_16; +} +else +{ +size_t x_17; size_t x_18; lean_object* x_19; lean_object* x_20; +x_17 = 0; +x_18 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_19 = lean_box(0); +x_20 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1(x_1, x_17, x_18, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +return x_20; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeExt; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_bvNormalizeSimprocExt; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_sevalSimpExtension; +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(32u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9() { +_start: +{ +size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = 5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8; +x_3 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7; +x_4 = lean_unsigned_to_nat(0u); +x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_4); +lean_ctor_set(x_5, 3, x_4); +lean_ctor_set_usize(x_5, 4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9; +x_3 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_1); +lean_ctor_set(x_3, 3, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1___boxed), 8, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1; +x_10 = l_Lean_Meta_SimpExtension_getTheorems(x_9, x_6, x_7, x_8); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2; +x_14 = l_Lean_Meta_Simp_SimprocExtension_getSimprocs(x_13, x_6, x_7, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3; +x_18 = l_Lean_Meta_SimpExtension_getTheorems(x_17, x_6, x_7, x_16); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +x_22 = l_Lean_Meta_Simp_getSEvalSimprocs___rarg(x_7, x_21); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +x_26 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_7, x_25); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; uint8_t x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_28 = lean_ctor_get(x_26, 0); +x_29 = lean_ctor_get(x_26, 1); +x_30 = lean_ctor_get(x_2, 1); +lean_inc(x_30); +x_31 = lean_unsigned_to_nat(2u); +x_32 = 0; +x_33 = 1; +x_34 = 0; +x_35 = lean_alloc_ctor(0, 2, 19); +lean_ctor_set(x_35, 0, x_30); +lean_ctor_set(x_35, 1, x_31); +lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 1, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 2, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 3, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 4, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 5, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 6, x_34); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 7, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 8, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 9, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 10, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 11, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 12, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 13, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 14, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 15, x_32); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 16, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 17, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2 + 18, x_33); +x_36 = lean_box(0); +lean_ctor_set_tag(x_26, 1); +lean_ctor_set(x_26, 1, x_36); +lean_ctor_set(x_26, 0, x_20); +lean_ctor_set_tag(x_22, 1); +lean_ctor_set(x_22, 1, x_26); +lean_ctor_set(x_22, 0, x_11); +x_37 = lean_array_mk(x_22); +x_38 = l_Lean_Meta_Simp_mkContext(x_35, x_37, x_28, x_4, x_5, x_6, x_7, x_29); +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_38, 0); +x_41 = lean_ctor_get(x_38, 1); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_42 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_41); +if (lean_obj_tag(x_42) == 0) +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_44 = lean_ctor_get(x_42, 0); +x_45 = lean_ctor_get(x_42, 1); +x_46 = l_Array_isEmpty___rarg(x_44); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_free_object(x_42); +lean_ctor_set_tag(x_38, 1); +lean_ctor_set(x_38, 1, x_36); +lean_ctor_set(x_38, 0, x_24); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_38); +lean_ctor_set(x_18, 0, x_15); +x_47 = lean_array_mk(x_18); +x_48 = lean_box(0); +x_49 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_50 = l_Lean_Meta_simpGoal(x_1, x_40, x_47, x_48, x_33, x_44, x_49, x_4, x_5, x_6, x_7, x_45); +if (lean_obj_tag(x_50) == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_51, 0); +lean_inc(x_52); +lean_dec(x_51); +if (lean_obj_tag(x_52) == 0) +{ +uint8_t x_53; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_53 = !lean_is_exclusive(x_50); +if (x_53 == 0) +{ +lean_object* x_54; +x_54 = lean_ctor_get(x_50, 0); +lean_dec(x_54); +lean_ctor_set(x_50, 0, x_48); +return x_50; +} +else +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_50, 1); +lean_inc(x_55); +lean_dec(x_50); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_48); +lean_ctor_set(x_56, 1, x_55); +return x_56; +} +} +else +{ +uint8_t x_57; +x_57 = !lean_is_exclusive(x_52); +if (x_57 == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_58 = lean_ctor_get(x_52, 0); +x_59 = lean_ctor_get(x_50, 1); +lean_inc(x_59); +lean_dec(x_50); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +lean_inc(x_60); +x_61 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_61, 0, x_60); +x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_63 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_63, 0, x_61); +lean_closure_set(x_63, 1, x_62); +lean_inc(x_60); +x_64 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_60, x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_59); +if (lean_obj_tag(x_64) == 0) +{ +uint8_t x_65; +x_65 = !lean_is_exclusive(x_64); +if (x_65 == 0) +{ +lean_object* x_66; +x_66 = lean_ctor_get(x_64, 0); +lean_dec(x_66); +lean_ctor_set(x_52, 0, x_60); +lean_ctor_set(x_64, 0, x_52); +return x_64; +} +else +{ +lean_object* x_67; lean_object* x_68; +x_67 = lean_ctor_get(x_64, 1); +lean_inc(x_67); +lean_dec(x_64); +lean_ctor_set(x_52, 0, x_60); +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_52); +lean_ctor_set(x_68, 1, x_67); +return x_68; +} +} +else +{ +uint8_t x_69; +lean_dec(x_60); +lean_free_object(x_52); +x_69 = !lean_is_exclusive(x_64); +if (x_69 == 0) +{ +return x_64; +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_64, 0); +x_71 = lean_ctor_get(x_64, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_64); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; +} +} +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_73 = lean_ctor_get(x_52, 0); +lean_inc(x_73); +lean_dec(x_52); +x_74 = lean_ctor_get(x_50, 1); +lean_inc(x_74); +lean_dec(x_50); +x_75 = lean_ctor_get(x_73, 1); +lean_inc(x_75); +lean_dec(x_73); +lean_inc(x_75); +x_76 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_76, 0, x_75); +x_77 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_78 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_78, 0, x_76); +lean_closure_set(x_78, 1, x_77); +lean_inc(x_75); +x_79 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_75, x_78, x_2, x_3, x_4, x_5, x_6, x_7, x_74); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_80 = lean_ctor_get(x_79, 1); +lean_inc(x_80); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_81 = x_79; +} else { + lean_dec_ref(x_79); + x_81 = lean_box(0); +} +x_82 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_82, 0, x_75); +if (lean_is_scalar(x_81)) { + x_83 = lean_alloc_ctor(0, 2, 0); +} else { + x_83 = x_81; +} +lean_ctor_set(x_83, 0, x_82); +lean_ctor_set(x_83, 1, x_80); +return x_83; +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_75); +x_84 = lean_ctor_get(x_79, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_79, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_86 = x_79; +} else { + lean_dec_ref(x_79); + x_86 = lean_box(0); +} +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); +} else { + x_87 = x_86; +} +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; +} +} +} +} +else +{ +uint8_t x_88; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_88 = !lean_is_exclusive(x_50); +if (x_88 == 0) +{ +return x_50; +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_50, 0); +x_90 = lean_ctor_get(x_50, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_50); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +return x_91; +} +} +} +else +{ +lean_object* x_92; +lean_dec(x_44); +lean_free_object(x_38); +lean_dec(x_40); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_1); +lean_ctor_set(x_42, 0, x_92); +return x_42; +} +} +else +{ +lean_object* x_93; lean_object* x_94; uint8_t x_95; +x_93 = lean_ctor_get(x_42, 0); +x_94 = lean_ctor_get(x_42, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_42); +x_95 = l_Array_isEmpty___rarg(x_93); +if (x_95 == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_ctor_set_tag(x_38, 1); +lean_ctor_set(x_38, 1, x_36); +lean_ctor_set(x_38, 0, x_24); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_38); +lean_ctor_set(x_18, 0, x_15); +x_96 = lean_array_mk(x_18); +x_97 = lean_box(0); +x_98 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_99 = l_Lean_Meta_simpGoal(x_1, x_40, x_96, x_97, x_33, x_93, x_98, x_4, x_5, x_6, x_7, x_94); +if (lean_obj_tag(x_99) == 0) +{ +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +lean_dec(x_100); +if (lean_obj_tag(x_101) == 0) +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_102 = lean_ctor_get(x_99, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_103 = x_99; +} else { + lean_dec_ref(x_99); + x_103 = lean_box(0); +} +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(0, 2, 0); +} else { + x_104 = x_103; +} +lean_ctor_set(x_104, 0, x_97); +lean_ctor_set(x_104, 1, x_102); +return x_104; +} +else +{ +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_105 = lean_ctor_get(x_101, 0); +lean_inc(x_105); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + x_106 = x_101; +} else { + lean_dec_ref(x_101); + x_106 = lean_box(0); +} +x_107 = lean_ctor_get(x_99, 1); +lean_inc(x_107); +lean_dec(x_99); +x_108 = lean_ctor_get(x_105, 1); +lean_inc(x_108); +lean_dec(x_105); +lean_inc(x_108); +x_109 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_109, 0, x_108); +x_110 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_111 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_111, 0, x_109); +lean_closure_set(x_111, 1, x_110); +lean_inc(x_108); +x_112 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_108, x_111, x_2, x_3, x_4, x_5, x_6, x_7, x_107); +if (lean_obj_tag(x_112) == 0) +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; +} else { + lean_dec_ref(x_112); + x_114 = lean_box(0); +} +if (lean_is_scalar(x_106)) { + x_115 = lean_alloc_ctor(1, 1, 0); +} else { + x_115 = x_106; +} +lean_ctor_set(x_115, 0, x_108); +if (lean_is_scalar(x_114)) { + x_116 = lean_alloc_ctor(0, 2, 0); +} else { + x_116 = x_114; +} +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_113); +return x_116; +} +else +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_dec(x_108); +lean_dec(x_106); +x_117 = lean_ctor_get(x_112, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_112, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_119 = x_112; +} else { + lean_dec_ref(x_112); + x_119 = lean_box(0); +} +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(1, 2, 0); +} else { + x_120 = x_119; +} +lean_ctor_set(x_120, 0, x_117); +lean_ctor_set(x_120, 1, x_118); +return x_120; +} +} +} +else +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_121 = lean_ctor_get(x_99, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_99, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_123 = x_99; +} else { + lean_dec_ref(x_99); + x_123 = lean_box(0); +} +if (lean_is_scalar(x_123)) { + x_124 = lean_alloc_ctor(1, 2, 0); +} else { + x_124 = x_123; +} +lean_ctor_set(x_124, 0, x_121); +lean_ctor_set(x_124, 1, x_122); +return x_124; +} +} +else +{ +lean_object* x_125; lean_object* x_126; +lean_dec(x_93); +lean_free_object(x_38); +lean_dec(x_40); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_125 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_125, 0, x_1); +x_126 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_94); +return x_126; +} +} +} +else +{ +uint8_t x_127; +lean_free_object(x_38); +lean_dec(x_40); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_127 = !lean_is_exclusive(x_42); +if (x_127 == 0) +{ +return x_42; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_42, 0); +x_129 = lean_ctor_get(x_42, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_42); +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; +} +} +} +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_131 = lean_ctor_get(x_38, 0); +x_132 = lean_ctor_get(x_38, 1); +lean_inc(x_132); +lean_inc(x_131); +lean_dec(x_38); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_133 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_132); +if (lean_obj_tag(x_133) == 0) +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; +x_134 = lean_ctor_get(x_133, 0); +lean_inc(x_134); +x_135 = lean_ctor_get(x_133, 1); +lean_inc(x_135); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_136 = x_133; +} else { + lean_dec_ref(x_133); + x_136 = lean_box(0); +} +x_137 = l_Array_isEmpty___rarg(x_134); +if (x_137 == 0) +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +lean_dec(x_136); +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_24); +lean_ctor_set(x_138, 1, x_36); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_138); +lean_ctor_set(x_18, 0, x_15); +x_139 = lean_array_mk(x_18); +x_140 = lean_box(0); +x_141 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_142 = l_Lean_Meta_simpGoal(x_1, x_131, x_139, x_140, x_33, x_134, x_141, x_4, x_5, x_6, x_7, x_135); +if (lean_obj_tag(x_142) == 0) +{ +lean_object* x_143; lean_object* x_144; +x_143 = lean_ctor_get(x_142, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_143, 0); +lean_inc(x_144); +lean_dec(x_143); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_145 = lean_ctor_get(x_142, 1); +lean_inc(x_145); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + lean_ctor_release(x_142, 1); + x_146 = x_142; +} else { + lean_dec_ref(x_142); + x_146 = lean_box(0); +} +if (lean_is_scalar(x_146)) { + x_147 = lean_alloc_ctor(0, 2, 0); +} else { + x_147 = x_146; +} +lean_ctor_set(x_147, 0, x_140); +lean_ctor_set(x_147, 1, x_145); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + x_149 = x_144; +} else { + lean_dec_ref(x_144); + x_149 = lean_box(0); +} +x_150 = lean_ctor_get(x_142, 1); +lean_inc(x_150); +lean_dec(x_142); +x_151 = lean_ctor_get(x_148, 1); +lean_inc(x_151); +lean_dec(x_148); +lean_inc(x_151); +x_152 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_152, 0, x_151); +x_153 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_154 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_154, 0, x_152); +lean_closure_set(x_154, 1, x_153); +lean_inc(x_151); +x_155 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_151, x_154, x_2, x_3, x_4, x_5, x_6, x_7, x_150); +if (lean_obj_tag(x_155) == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_156 = lean_ctor_get(x_155, 1); +lean_inc(x_156); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_157 = x_155; +} else { + lean_dec_ref(x_155); + x_157 = lean_box(0); +} +if (lean_is_scalar(x_149)) { + x_158 = lean_alloc_ctor(1, 1, 0); +} else { + x_158 = x_149; +} +lean_ctor_set(x_158, 0, x_151); +if (lean_is_scalar(x_157)) { + x_159 = lean_alloc_ctor(0, 2, 0); +} else { + x_159 = x_157; +} +lean_ctor_set(x_159, 0, x_158); +lean_ctor_set(x_159, 1, x_156); +return x_159; +} +else +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +lean_dec(x_151); +lean_dec(x_149); +x_160 = lean_ctor_get(x_155, 0); +lean_inc(x_160); +x_161 = lean_ctor_get(x_155, 1); +lean_inc(x_161); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_162 = x_155; +} else { + lean_dec_ref(x_155); + x_162 = lean_box(0); +} +if (lean_is_scalar(x_162)) { + x_163 = lean_alloc_ctor(1, 2, 0); +} else { + x_163 = x_162; +} +lean_ctor_set(x_163, 0, x_160); +lean_ctor_set(x_163, 1, x_161); +return x_163; +} +} +} +else +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_164 = lean_ctor_get(x_142, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_142, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_142)) { + lean_ctor_release(x_142, 0); + lean_ctor_release(x_142, 1); + x_166 = x_142; +} else { + lean_dec_ref(x_142); + x_166 = lean_box(0); +} +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); +} else { + x_167 = x_166; +} +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; +} +} +else +{ +lean_object* x_168; lean_object* x_169; +lean_dec(x_134); +lean_dec(x_131); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_168 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_168, 0, x_1); +if (lean_is_scalar(x_136)) { + x_169 = lean_alloc_ctor(0, 2, 0); +} else { + x_169 = x_136; +} +lean_ctor_set(x_169, 0, x_168); +lean_ctor_set(x_169, 1, x_135); +return x_169; +} +} +else +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +lean_dec(x_131); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_170 = lean_ctor_get(x_133, 0); +lean_inc(x_170); +x_171 = lean_ctor_get(x_133, 1); +lean_inc(x_171); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_172 = x_133; +} else { + lean_dec_ref(x_133); + x_172 = lean_box(0); +} +if (lean_is_scalar(x_172)) { + x_173 = lean_alloc_ctor(1, 2, 0); +} else { + x_173 = x_172; +} +lean_ctor_set(x_173, 0, x_170); +lean_ctor_set(x_173, 1, x_171); +return x_173; +} +} +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; uint8_t x_178; uint8_t x_179; uint8_t x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +x_174 = lean_ctor_get(x_26, 0); +x_175 = lean_ctor_get(x_26, 1); +lean_inc(x_175); +lean_inc(x_174); +lean_dec(x_26); +x_176 = lean_ctor_get(x_2, 1); +lean_inc(x_176); +x_177 = lean_unsigned_to_nat(2u); +x_178 = 0; +x_179 = 1; +x_180 = 0; +x_181 = lean_alloc_ctor(0, 2, 19); +lean_ctor_set(x_181, 0, x_176); +lean_ctor_set(x_181, 1, x_177); +lean_ctor_set_uint8(x_181, sizeof(void*)*2, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 1, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 2, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 3, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 4, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 5, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 6, x_180); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 7, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 8, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 9, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 10, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 11, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 12, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 13, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 14, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 15, x_178); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 16, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 17, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*2 + 18, x_179); +x_182 = lean_box(0); +x_183 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_183, 0, x_20); +lean_ctor_set(x_183, 1, x_182); +lean_ctor_set_tag(x_22, 1); +lean_ctor_set(x_22, 1, x_183); +lean_ctor_set(x_22, 0, x_11); +x_184 = lean_array_mk(x_22); +x_185 = l_Lean_Meta_Simp_mkContext(x_181, x_184, x_174, x_4, x_5, x_6, x_7, x_175); +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_185, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + x_188 = x_185; +} else { + lean_dec_ref(x_185); + x_188 = lean_box(0); +} +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_189 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_187); +if (lean_obj_tag(x_189) == 0) +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; uint8_t x_193; +x_190 = lean_ctor_get(x_189, 0); +lean_inc(x_190); +x_191 = lean_ctor_get(x_189, 1); +lean_inc(x_191); +if (lean_is_exclusive(x_189)) { + lean_ctor_release(x_189, 0); + lean_ctor_release(x_189, 1); + x_192 = x_189; +} else { + lean_dec_ref(x_189); + x_192 = lean_box(0); +} +x_193 = l_Array_isEmpty___rarg(x_190); +if (x_193 == 0) +{ +lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; +lean_dec(x_192); +if (lean_is_scalar(x_188)) { + x_194 = lean_alloc_ctor(1, 2, 0); +} else { + x_194 = x_188; + lean_ctor_set_tag(x_194, 1); +} +lean_ctor_set(x_194, 0, x_24); +lean_ctor_set(x_194, 1, x_182); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_194); +lean_ctor_set(x_18, 0, x_15); +x_195 = lean_array_mk(x_18); +x_196 = lean_box(0); +x_197 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_198 = l_Lean_Meta_simpGoal(x_1, x_186, x_195, x_196, x_179, x_190, x_197, x_4, x_5, x_6, x_7, x_191); +if (lean_obj_tag(x_198) == 0) +{ +lean_object* x_199; lean_object* x_200; +x_199 = lean_ctor_get(x_198, 0); +lean_inc(x_199); +x_200 = lean_ctor_get(x_199, 0); +lean_inc(x_200); +lean_dec(x_199); +if (lean_obj_tag(x_200) == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_201 = lean_ctor_get(x_198, 1); +lean_inc(x_201); +if (lean_is_exclusive(x_198)) { + lean_ctor_release(x_198, 0); + lean_ctor_release(x_198, 1); + x_202 = x_198; +} else { + lean_dec_ref(x_198); + x_202 = lean_box(0); +} +if (lean_is_scalar(x_202)) { + x_203 = lean_alloc_ctor(0, 2, 0); +} else { + x_203 = x_202; +} +lean_ctor_set(x_203, 0, x_196); +lean_ctor_set(x_203, 1, x_201); +return x_203; +} +else +{ +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_204 = lean_ctor_get(x_200, 0); +lean_inc(x_204); +if (lean_is_exclusive(x_200)) { + lean_ctor_release(x_200, 0); + x_205 = x_200; +} else { + lean_dec_ref(x_200); + x_205 = lean_box(0); +} +x_206 = lean_ctor_get(x_198, 1); +lean_inc(x_206); +lean_dec(x_198); +x_207 = lean_ctor_get(x_204, 1); +lean_inc(x_207); +lean_dec(x_204); +lean_inc(x_207); +x_208 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_208, 0, x_207); +x_209 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_210 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_210, 0, x_208); +lean_closure_set(x_210, 1, x_209); +lean_inc(x_207); +x_211 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_207, x_210, x_2, x_3, x_4, x_5, x_6, x_7, x_206); +if (lean_obj_tag(x_211) == 0) +{ +lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_212 = lean_ctor_get(x_211, 1); +lean_inc(x_212); +if (lean_is_exclusive(x_211)) { + lean_ctor_release(x_211, 0); + lean_ctor_release(x_211, 1); + x_213 = x_211; +} else { + lean_dec_ref(x_211); + x_213 = lean_box(0); +} +if (lean_is_scalar(x_205)) { + x_214 = lean_alloc_ctor(1, 1, 0); +} else { + x_214 = x_205; +} +lean_ctor_set(x_214, 0, x_207); +if (lean_is_scalar(x_213)) { + x_215 = lean_alloc_ctor(0, 2, 0); +} else { + x_215 = x_213; +} +lean_ctor_set(x_215, 0, x_214); +lean_ctor_set(x_215, 1, x_212); +return x_215; +} +else +{ +lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +lean_dec(x_207); +lean_dec(x_205); +x_216 = lean_ctor_get(x_211, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_211, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_211)) { + lean_ctor_release(x_211, 0); + lean_ctor_release(x_211, 1); + x_218 = x_211; +} else { + lean_dec_ref(x_211); + x_218 = lean_box(0); +} +if (lean_is_scalar(x_218)) { + x_219 = lean_alloc_ctor(1, 2, 0); +} else { + x_219 = x_218; +} +lean_ctor_set(x_219, 0, x_216); +lean_ctor_set(x_219, 1, x_217); +return x_219; +} +} +} +else +{ +lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_220 = lean_ctor_get(x_198, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_198, 1); +lean_inc(x_221); +if (lean_is_exclusive(x_198)) { + lean_ctor_release(x_198, 0); + lean_ctor_release(x_198, 1); + x_222 = x_198; +} else { + lean_dec_ref(x_198); + x_222 = lean_box(0); +} +if (lean_is_scalar(x_222)) { + x_223 = lean_alloc_ctor(1, 2, 0); +} else { + x_223 = x_222; +} +lean_ctor_set(x_223, 0, x_220); +lean_ctor_set(x_223, 1, x_221); +return x_223; +} +} +else +{ +lean_object* x_224; lean_object* x_225; +lean_dec(x_190); +lean_dec(x_188); +lean_dec(x_186); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_224 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_224, 0, x_1); +if (lean_is_scalar(x_192)) { + x_225 = lean_alloc_ctor(0, 2, 0); +} else { + x_225 = x_192; +} +lean_ctor_set(x_225, 0, x_224); +lean_ctor_set(x_225, 1, x_191); +return x_225; +} +} +else +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +lean_dec(x_188); +lean_dec(x_186); +lean_dec(x_24); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_226 = lean_ctor_get(x_189, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_189, 1); +lean_inc(x_227); +if (lean_is_exclusive(x_189)) { + lean_ctor_release(x_189, 0); + lean_ctor_release(x_189, 1); + x_228 = x_189; +} else { + lean_dec_ref(x_189); + x_228 = lean_box(0); +} +if (lean_is_scalar(x_228)) { + x_229 = lean_alloc_ctor(1, 2, 0); +} else { + x_229 = x_228; +} +lean_ctor_set(x_229, 0, x_226); +lean_ctor_set(x_229, 1, x_227); +return x_229; +} +} +} +else +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t x_238; uint8_t x_239; uint8_t x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; +x_230 = lean_ctor_get(x_22, 0); +x_231 = lean_ctor_get(x_22, 1); +lean_inc(x_231); +lean_inc(x_230); +lean_dec(x_22); +x_232 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_7, x_231); +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_232, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_232)) { + lean_ctor_release(x_232, 0); + lean_ctor_release(x_232, 1); + x_235 = x_232; +} else { + lean_dec_ref(x_232); + x_235 = lean_box(0); +} +x_236 = lean_ctor_get(x_2, 1); +lean_inc(x_236); +x_237 = lean_unsigned_to_nat(2u); +x_238 = 0; +x_239 = 1; +x_240 = 0; +x_241 = lean_alloc_ctor(0, 2, 19); +lean_ctor_set(x_241, 0, x_236); +lean_ctor_set(x_241, 1, x_237); +lean_ctor_set_uint8(x_241, sizeof(void*)*2, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 1, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 2, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 3, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 4, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 5, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 6, x_240); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 7, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 8, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 9, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 10, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 11, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 12, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 13, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 14, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 15, x_238); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 16, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 17, x_239); +lean_ctor_set_uint8(x_241, sizeof(void*)*2 + 18, x_239); +x_242 = lean_box(0); +if (lean_is_scalar(x_235)) { + x_243 = lean_alloc_ctor(1, 2, 0); +} else { + x_243 = x_235; + lean_ctor_set_tag(x_243, 1); +} +lean_ctor_set(x_243, 0, x_20); +lean_ctor_set(x_243, 1, x_242); +x_244 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_244, 0, x_11); +lean_ctor_set(x_244, 1, x_243); +x_245 = lean_array_mk(x_244); +x_246 = l_Lean_Meta_Simp_mkContext(x_241, x_245, x_233, x_4, x_5, x_6, x_7, x_234); +x_247 = lean_ctor_get(x_246, 0); +lean_inc(x_247); +x_248 = lean_ctor_get(x_246, 1); +lean_inc(x_248); +if (lean_is_exclusive(x_246)) { + lean_ctor_release(x_246, 0); + lean_ctor_release(x_246, 1); + x_249 = x_246; +} else { + lean_dec_ref(x_246); + x_249 = lean_box(0); +} +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_250 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_248); +if (lean_obj_tag(x_250) == 0) +{ +lean_object* x_251; lean_object* x_252; lean_object* x_253; uint8_t x_254; +x_251 = lean_ctor_get(x_250, 0); +lean_inc(x_251); +x_252 = lean_ctor_get(x_250, 1); +lean_inc(x_252); +if (lean_is_exclusive(x_250)) { + lean_ctor_release(x_250, 0); + lean_ctor_release(x_250, 1); + x_253 = x_250; +} else { + lean_dec_ref(x_250); + x_253 = lean_box(0); +} +x_254 = l_Array_isEmpty___rarg(x_251); +if (x_254 == 0) +{ +lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_253); +if (lean_is_scalar(x_249)) { + x_255 = lean_alloc_ctor(1, 2, 0); +} else { + x_255 = x_249; + lean_ctor_set_tag(x_255, 1); +} +lean_ctor_set(x_255, 0, x_230); +lean_ctor_set(x_255, 1, x_242); +lean_ctor_set_tag(x_18, 1); +lean_ctor_set(x_18, 1, x_255); +lean_ctor_set(x_18, 0, x_15); +x_256 = lean_array_mk(x_18); +x_257 = lean_box(0); +x_258 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_259 = l_Lean_Meta_simpGoal(x_1, x_247, x_256, x_257, x_239, x_251, x_258, x_4, x_5, x_6, x_7, x_252); +if (lean_obj_tag(x_259) == 0) +{ +lean_object* x_260; lean_object* x_261; +x_260 = lean_ctor_get(x_259, 0); +lean_inc(x_260); +x_261 = lean_ctor_get(x_260, 0); +lean_inc(x_261); +lean_dec(x_260); +if (lean_obj_tag(x_261) == 0) +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_262 = lean_ctor_get(x_259, 1); +lean_inc(x_262); +if (lean_is_exclusive(x_259)) { + lean_ctor_release(x_259, 0); + lean_ctor_release(x_259, 1); + x_263 = x_259; +} else { + lean_dec_ref(x_259); + x_263 = lean_box(0); +} +if (lean_is_scalar(x_263)) { + x_264 = lean_alloc_ctor(0, 2, 0); +} else { + x_264 = x_263; +} +lean_ctor_set(x_264, 0, x_257); +lean_ctor_set(x_264, 1, x_262); +return x_264; +} +else +{ +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_265 = lean_ctor_get(x_261, 0); +lean_inc(x_265); +if (lean_is_exclusive(x_261)) { + lean_ctor_release(x_261, 0); + x_266 = x_261; +} else { + lean_dec_ref(x_261); + x_266 = lean_box(0); +} +x_267 = lean_ctor_get(x_259, 1); +lean_inc(x_267); +lean_dec(x_259); +x_268 = lean_ctor_get(x_265, 1); +lean_inc(x_268); +lean_dec(x_265); +lean_inc(x_268); +x_269 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_269, 0, x_268); +x_270 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_271 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_271, 0, x_269); +lean_closure_set(x_271, 1, x_270); +lean_inc(x_268); +x_272 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_268, x_271, x_2, x_3, x_4, x_5, x_6, x_7, x_267); +if (lean_obj_tag(x_272) == 0) +{ +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_273 = lean_ctor_get(x_272, 1); +lean_inc(x_273); +if (lean_is_exclusive(x_272)) { + lean_ctor_release(x_272, 0); + lean_ctor_release(x_272, 1); + x_274 = x_272; +} else { + lean_dec_ref(x_272); + x_274 = lean_box(0); +} +if (lean_is_scalar(x_266)) { + x_275 = lean_alloc_ctor(1, 1, 0); +} else { + x_275 = x_266; +} +lean_ctor_set(x_275, 0, x_268); +if (lean_is_scalar(x_274)) { + x_276 = lean_alloc_ctor(0, 2, 0); +} else { + x_276 = x_274; +} +lean_ctor_set(x_276, 0, x_275); +lean_ctor_set(x_276, 1, x_273); +return x_276; +} +else +{ +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +lean_dec(x_268); +lean_dec(x_266); +x_277 = lean_ctor_get(x_272, 0); +lean_inc(x_277); +x_278 = lean_ctor_get(x_272, 1); +lean_inc(x_278); +if (lean_is_exclusive(x_272)) { + lean_ctor_release(x_272, 0); + lean_ctor_release(x_272, 1); + x_279 = x_272; +} else { + lean_dec_ref(x_272); + x_279 = lean_box(0); +} +if (lean_is_scalar(x_279)) { + x_280 = lean_alloc_ctor(1, 2, 0); +} else { + x_280 = x_279; +} +lean_ctor_set(x_280, 0, x_277); +lean_ctor_set(x_280, 1, x_278); +return x_280; +} +} +} +else +{ +lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_281 = lean_ctor_get(x_259, 0); +lean_inc(x_281); +x_282 = lean_ctor_get(x_259, 1); +lean_inc(x_282); +if (lean_is_exclusive(x_259)) { + lean_ctor_release(x_259, 0); + lean_ctor_release(x_259, 1); + x_283 = x_259; +} else { + lean_dec_ref(x_259); + x_283 = lean_box(0); +} +if (lean_is_scalar(x_283)) { + x_284 = lean_alloc_ctor(1, 2, 0); +} else { + x_284 = x_283; +} +lean_ctor_set(x_284, 0, x_281); +lean_ctor_set(x_284, 1, x_282); +return x_284; +} +} +else +{ +lean_object* x_285; lean_object* x_286; +lean_dec(x_251); +lean_dec(x_249); +lean_dec(x_247); +lean_dec(x_230); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_285 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_285, 0, x_1); +if (lean_is_scalar(x_253)) { + x_286 = lean_alloc_ctor(0, 2, 0); +} else { + x_286 = x_253; +} +lean_ctor_set(x_286, 0, x_285); +lean_ctor_set(x_286, 1, x_252); +return x_286; +} +} +else +{ +lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; +lean_dec(x_249); +lean_dec(x_247); +lean_dec(x_230); +lean_free_object(x_18); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_287 = lean_ctor_get(x_250, 0); +lean_inc(x_287); +x_288 = lean_ctor_get(x_250, 1); +lean_inc(x_288); +if (lean_is_exclusive(x_250)) { + lean_ctor_release(x_250, 0); + lean_ctor_release(x_250, 1); + x_289 = x_250; +} else { + lean_dec_ref(x_250); + x_289 = lean_box(0); +} +if (lean_is_scalar(x_289)) { + x_290 = lean_alloc_ctor(1, 2, 0); +} else { + x_290 = x_289; +} +lean_ctor_set(x_290, 0, x_287); +lean_ctor_set(x_290, 1, x_288); +return x_290; +} +} +} +else +{ +lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; uint8_t x_303; uint8_t x_304; uint8_t x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; +x_291 = lean_ctor_get(x_18, 0); +x_292 = lean_ctor_get(x_18, 1); +lean_inc(x_292); +lean_inc(x_291); +lean_dec(x_18); +x_293 = l_Lean_Meta_Simp_getSEvalSimprocs___rarg(x_7, x_292); +x_294 = lean_ctor_get(x_293, 0); +lean_inc(x_294); +x_295 = lean_ctor_get(x_293, 1); +lean_inc(x_295); +if (lean_is_exclusive(x_293)) { + lean_ctor_release(x_293, 0); + lean_ctor_release(x_293, 1); + x_296 = x_293; +} else { + lean_dec_ref(x_293); + x_296 = lean_box(0); +} +x_297 = l_Lean_Meta_getSimpCongrTheorems___rarg(x_7, x_295); +x_298 = lean_ctor_get(x_297, 0); +lean_inc(x_298); +x_299 = lean_ctor_get(x_297, 1); +lean_inc(x_299); +if (lean_is_exclusive(x_297)) { + lean_ctor_release(x_297, 0); + lean_ctor_release(x_297, 1); + x_300 = x_297; +} else { + lean_dec_ref(x_297); + x_300 = lean_box(0); +} +x_301 = lean_ctor_get(x_2, 1); +lean_inc(x_301); +x_302 = lean_unsigned_to_nat(2u); +x_303 = 0; +x_304 = 1; +x_305 = 0; +x_306 = lean_alloc_ctor(0, 2, 19); +lean_ctor_set(x_306, 0, x_301); +lean_ctor_set(x_306, 1, x_302); +lean_ctor_set_uint8(x_306, sizeof(void*)*2, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 1, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 2, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 3, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 4, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 5, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 6, x_305); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 7, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 8, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 9, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 10, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 11, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 12, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 13, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 14, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 15, x_303); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 16, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 17, x_304); +lean_ctor_set_uint8(x_306, sizeof(void*)*2 + 18, x_304); +x_307 = lean_box(0); +if (lean_is_scalar(x_300)) { + x_308 = lean_alloc_ctor(1, 2, 0); +} else { + x_308 = x_300; + lean_ctor_set_tag(x_308, 1); +} +lean_ctor_set(x_308, 0, x_291); +lean_ctor_set(x_308, 1, x_307); +if (lean_is_scalar(x_296)) { + x_309 = lean_alloc_ctor(1, 2, 0); +} else { + x_309 = x_296; + lean_ctor_set_tag(x_309, 1); +} +lean_ctor_set(x_309, 0, x_11); +lean_ctor_set(x_309, 1, x_308); +x_310 = lean_array_mk(x_309); +x_311 = l_Lean_Meta_Simp_mkContext(x_306, x_310, x_298, x_4, x_5, x_6, x_7, x_299); +x_312 = lean_ctor_get(x_311, 0); +lean_inc(x_312); +x_313 = lean_ctor_get(x_311, 1); +lean_inc(x_313); +if (lean_is_exclusive(x_311)) { + lean_ctor_release(x_311, 0); + lean_ctor_release(x_311, 1); + x_314 = x_311; +} else { + lean_dec_ref(x_311); + x_314 = lean_box(0); +} +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_315 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_313); +if (lean_obj_tag(x_315) == 0) +{ +lean_object* x_316; lean_object* x_317; lean_object* x_318; uint8_t x_319; +x_316 = lean_ctor_get(x_315, 0); +lean_inc(x_316); +x_317 = lean_ctor_get(x_315, 1); +lean_inc(x_317); +if (lean_is_exclusive(x_315)) { + lean_ctor_release(x_315, 0); + lean_ctor_release(x_315, 1); + x_318 = x_315; +} else { + lean_dec_ref(x_315); + x_318 = lean_box(0); +} +x_319 = l_Array_isEmpty___rarg(x_316); +if (x_319 == 0) +{ +lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; +lean_dec(x_318); +if (lean_is_scalar(x_314)) { + x_320 = lean_alloc_ctor(1, 2, 0); +} else { + x_320 = x_314; + lean_ctor_set_tag(x_320, 1); +} +lean_ctor_set(x_320, 0, x_294); +lean_ctor_set(x_320, 1, x_307); +x_321 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_321, 0, x_15); +lean_ctor_set(x_321, 1, x_320); +x_322 = lean_array_mk(x_321); +x_323 = lean_box(0); +x_324 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11; +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_325 = l_Lean_Meta_simpGoal(x_1, x_312, x_322, x_323, x_304, x_316, x_324, x_4, x_5, x_6, x_7, x_317); +if (lean_obj_tag(x_325) == 0) +{ +lean_object* x_326; lean_object* x_327; +x_326 = lean_ctor_get(x_325, 0); +lean_inc(x_326); +x_327 = lean_ctor_get(x_326, 0); +lean_inc(x_327); +lean_dec(x_326); +if (lean_obj_tag(x_327) == 0) +{ +lean_object* x_328; lean_object* x_329; lean_object* x_330; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_328 = lean_ctor_get(x_325, 1); +lean_inc(x_328); +if (lean_is_exclusive(x_325)) { + lean_ctor_release(x_325, 0); + lean_ctor_release(x_325, 1); + x_329 = x_325; +} else { + lean_dec_ref(x_325); + x_329 = lean_box(0); +} +if (lean_is_scalar(x_329)) { + x_330 = lean_alloc_ctor(0, 2, 0); +} else { + x_330 = x_329; +} +lean_ctor_set(x_330, 0, x_323); +lean_ctor_set(x_330, 1, x_328); +return x_330; +} +else +{ +lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; +x_331 = lean_ctor_get(x_327, 0); +lean_inc(x_331); +if (lean_is_exclusive(x_327)) { + lean_ctor_release(x_327, 0); + x_332 = x_327; +} else { + lean_dec_ref(x_327); + x_332 = lean_box(0); +} +x_333 = lean_ctor_get(x_325, 1); +lean_inc(x_333); +lean_dec(x_325); +x_334 = lean_ctor_get(x_331, 1); +lean_inc(x_334); +lean_dec(x_331); +lean_inc(x_334); +x_335 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__1___boxed), 8, 1); +lean_closure_set(x_335, 0, x_334); +x_336 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12; +x_337 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__2___rarg), 9, 2); +lean_closure_set(x_337, 0, x_335); +lean_closure_set(x_337, 1, x_336); +lean_inc(x_334); +x_338 = l_Lean_MVarId_withContext___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__3___rarg(x_334, x_337, x_2, x_3, x_4, x_5, x_6, x_7, x_333); +if (lean_obj_tag(x_338) == 0) +{ +lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; +x_339 = lean_ctor_get(x_338, 1); +lean_inc(x_339); +if (lean_is_exclusive(x_338)) { + lean_ctor_release(x_338, 0); + lean_ctor_release(x_338, 1); + x_340 = x_338; +} else { + lean_dec_ref(x_338); + x_340 = lean_box(0); +} +if (lean_is_scalar(x_332)) { + x_341 = lean_alloc_ctor(1, 1, 0); +} else { + x_341 = x_332; +} +lean_ctor_set(x_341, 0, x_334); +if (lean_is_scalar(x_340)) { + x_342 = lean_alloc_ctor(0, 2, 0); +} else { + x_342 = x_340; +} +lean_ctor_set(x_342, 0, x_341); +lean_ctor_set(x_342, 1, x_339); +return x_342; +} +else +{ +lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; +lean_dec(x_334); +lean_dec(x_332); +x_343 = lean_ctor_get(x_338, 0); +lean_inc(x_343); +x_344 = lean_ctor_get(x_338, 1); +lean_inc(x_344); +if (lean_is_exclusive(x_338)) { + lean_ctor_release(x_338, 0); + lean_ctor_release(x_338, 1); + x_345 = x_338; +} else { + lean_dec_ref(x_338); + x_345 = lean_box(0); +} +if (lean_is_scalar(x_345)) { + x_346 = lean_alloc_ctor(1, 2, 0); +} else { + x_346 = x_345; +} +lean_ctor_set(x_346, 0, x_343); +lean_ctor_set(x_346, 1, x_344); +return x_346; +} +} +} +else +{ +lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_347 = lean_ctor_get(x_325, 0); +lean_inc(x_347); +x_348 = lean_ctor_get(x_325, 1); +lean_inc(x_348); +if (lean_is_exclusive(x_325)) { + lean_ctor_release(x_325, 0); + lean_ctor_release(x_325, 1); + x_349 = x_325; +} else { + lean_dec_ref(x_325); + x_349 = lean_box(0); +} +if (lean_is_scalar(x_349)) { + x_350 = lean_alloc_ctor(1, 2, 0); +} else { + x_350 = x_349; +} +lean_ctor_set(x_350, 0, x_347); +lean_ctor_set(x_350, 1, x_348); +return x_350; +} +} +else +{ +lean_object* x_351; lean_object* x_352; +lean_dec(x_316); +lean_dec(x_314); +lean_dec(x_312); +lean_dec(x_294); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_351 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_351, 0, x_1); +if (lean_is_scalar(x_318)) { + x_352 = lean_alloc_ctor(0, 2, 0); +} else { + x_352 = x_318; +} +lean_ctor_set(x_352, 0, x_351); +lean_ctor_set(x_352, 1, x_317); +return x_352; +} +} +else +{ +lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; +lean_dec(x_314); +lean_dec(x_312); +lean_dec(x_294); +lean_dec(x_15); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_353 = lean_ctor_get(x_315, 0); +lean_inc(x_353); +x_354 = lean_ctor_get(x_315, 1); +lean_inc(x_354); +if (lean_is_exclusive(x_315)) { + lean_ctor_release(x_315, 0); + lean_ctor_release(x_315, 1); + x_355 = x_315; +} else { + lean_dec_ref(x_315); + x_355 = lean_box(0); +} +if (lean_is_scalar(x_355)) { + x_356 = lean_alloc_ctor(1, 2, 0); +} else { + x_356 = x_355; +} +lean_ctor_set(x_356, 0, x_353); +lean_ctor_set(x_356, 1, x_354); +return x_356; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("rewriteRules", 12, 12); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1), 8, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +size_t x_12; size_t x_13; lean_object* x_14; +x_12 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_13 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_14 = l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1(x_1, x_12, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_9; +} +} +lean_object* initialize_Lean_Elab_Tactic_Simp(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Rewrite(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Elab_Tactic_Simp(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__2); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__3); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__4); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__5); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__6); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__7); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__8); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__9); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__10); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__11); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__12); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__13); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___spec__1___closed__14); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___lambda__2___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass_getHyps___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__1); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__2); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__3); +l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4 = _init_l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4(); +lean_mark_persistent(l_Array_foldlMUnsafe_fold___at_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___spec__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___elambda__1___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_rewriteRulesPass); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Simproc.c b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Simproc.c new file mode 100644 index 000000000000..4c87535eb473 --- /dev/null +++ b/stage0/stdlib/Lean/Elab/Tactic/BVDecide/Frontend/Normalize/Simproc.c @@ -0,0 +1,11406 @@ +// Lean compiler output +// Module: Lean.Elab.Tactic.BVDecide.Frontend.Normalize.Simproc +// Imports: Std.Tactic.BVDecide.Normalize Std.Tactic.BVDecide.Syntax Lean.Elab.Tactic.Simp Lean.Elab.Tactic.BVDecide.Frontend.Attr +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Simp_Result_getProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1; +lean_object* l_Lean_mkNatLit(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8; +lean_object* l_Lean_mkAppN(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3; +lean_object* l_Lean_Meta_getNatValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13; +lean_object* l_Lean_Meta_mkLt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508_(lean_object*); +lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isApp(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; +lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8; +lean_object* l_Lean_Level_ofNat(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; +uint8_t l_instDecidableNot___rarg(uint8_t); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +lean_object* l_Lean_Name_mkStr7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7; +lean_object* l_BitVec_neg(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; +lean_object* l_Lean_Meta_getBitVecValue_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_BitVec_ofNat(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3; +lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5; +lean_object* l_Lean_Meta_mkDecideProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2; +lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13; +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2; +lean_object* l_BitVec_add(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; +lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_constLevels_x21(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6; +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); +lean_object* lean_nat_pow(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823_(lean_object*); +lean_object* l_Lean_Meta_Simp_registerBuiltinSimproc(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16; +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +lean_object* lean_nat_log2(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952_(lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_mk(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact___boxed(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1; +extern lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085_(lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4; +static lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9; +lean_object* lean_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655_(lean_object*); +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Bool", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("true", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("false", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("cond_neg", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("cond_pos", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_3); +x_14 = lean_simp(x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +x_19 = l_Lean_Expr_cleanupAnnotations(x_18); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; +x_21 = l_Lean_Expr_isConstOf(x_19, x_20); +if (x_21 == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; +x_23 = l_Lean_Expr_isConstOf(x_19, x_22); +lean_dec(x_19); +if (x_23 == 0) +{ +lean_object* x_24; +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_14, 0, x_24); +return x_14; +} +else +{ +lean_object* x_25; +lean_free_object(x_14); +x_25 = l_Lean_Meta_Simp_Result_getProof(x_16, x_9, x_10, x_11, x_12, x_17); +if (lean_obj_tag(x_25) == 0) +{ +uint8_t x_26; +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; +x_27 = lean_ctor_get(x_25, 0); +x_28 = l_Lean_Expr_constLevels_x21(x_1); +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; +x_30 = l_Lean_Expr_const___override(x_29, x_28); +lean_inc(x_5); +x_31 = l_Lean_mkApp4(x_30, x_2, x_3, x_4, x_5); +x_32 = l_Lean_Expr_app___override(x_31, x_27); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_32); +x_34 = 1; +x_35 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_35, 0, x_5); +lean_ctor_set(x_35, 1, x_33); +lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_34); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_25, 0, x_36); +return x_25; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_37 = lean_ctor_get(x_25, 0); +x_38 = lean_ctor_get(x_25, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_25); +x_39 = l_Lean_Expr_constLevels_x21(x_1); +x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; +x_41 = l_Lean_Expr_const___override(x_40, x_39); +lean_inc(x_5); +x_42 = l_Lean_mkApp4(x_41, x_2, x_3, x_4, x_5); +x_43 = l_Lean_Expr_app___override(x_42, x_37); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = 1; +x_46 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_46, 0, x_5); +lean_ctor_set(x_46, 1, x_44); +lean_ctor_set_uint8(x_46, sizeof(void*)*2, x_45); +x_47 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_38); +return x_48; +} +} +else +{ +uint8_t x_49; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_49 = !lean_is_exclusive(x_25); +if (x_49 == 0) +{ +return x_25; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_25, 0); +x_51 = lean_ctor_get(x_25, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_25); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +} +else +{ +lean_object* x_53; +lean_dec(x_19); +lean_free_object(x_14); +x_53 = l_Lean_Meta_Simp_Result_getProof(x_16, x_9, x_10, x_11, x_12, x_17); +if (lean_obj_tag(x_53) == 0) +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; +x_55 = lean_ctor_get(x_53, 0); +x_56 = l_Lean_Expr_constLevels_x21(x_1); +x_57 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; +x_58 = l_Lean_Expr_const___override(x_57, x_56); +lean_inc(x_4); +x_59 = l_Lean_mkApp4(x_58, x_2, x_3, x_4, x_5); +x_60 = l_Lean_Expr_app___override(x_59, x_55); +x_61 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_62 = 1; +x_63 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_63, 0, x_4); +lean_ctor_set(x_63, 1, x_61); +lean_ctor_set_uint8(x_63, sizeof(void*)*2, x_62); +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_53, 0, x_64); +return x_53; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_65 = lean_ctor_get(x_53, 0); +x_66 = lean_ctor_get(x_53, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_53); +x_67 = l_Lean_Expr_constLevels_x21(x_1); +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; +x_69 = l_Lean_Expr_const___override(x_68, x_67); +lean_inc(x_4); +x_70 = l_Lean_mkApp4(x_69, x_2, x_3, x_4, x_5); +x_71 = l_Lean_Expr_app___override(x_70, x_65); +x_72 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_72, 0, x_71); +x_73 = 1; +x_74 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_74, 0, x_4); +lean_ctor_set(x_74, 1, x_72); +lean_ctor_set_uint8(x_74, sizeof(void*)*2, x_73); +x_75 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_75, 0, x_74); +x_76 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_66); +return x_76; +} +} +else +{ +uint8_t x_77; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_77 = !lean_is_exclusive(x_53); +if (x_77 == 0) +{ +return x_53; +} +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_53, 0); +x_79 = lean_ctor_get(x_53, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_53); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +return x_80; +} +} +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +x_81 = lean_ctor_get(x_14, 0); +x_82 = lean_ctor_get(x_14, 1); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_14); +x_83 = lean_ctor_get(x_81, 0); +lean_inc(x_83); +x_84 = l_Lean_Expr_cleanupAnnotations(x_83); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; +x_86 = l_Lean_Expr_isConstOf(x_84, x_85); +if (x_86 == 0) +{ +lean_object* x_87; uint8_t x_88; +x_87 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; +x_88 = l_Lean_Expr_isConstOf(x_84, x_87); +lean_dec(x_84); +if (x_88 == 0) +{ +lean_object* x_89; lean_object* x_90; +lean_dec(x_81); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_89 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_89); +lean_ctor_set(x_90, 1, x_82); +return x_90; +} +else +{ +lean_object* x_91; +x_91 = l_Lean_Meta_Simp_Result_getProof(x_81, x_9, x_10, x_11, x_12, x_82); +if (lean_obj_tag(x_91) == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; uint8_t x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_94 = x_91; +} else { + lean_dec_ref(x_91); + x_94 = lean_box(0); +} +x_95 = l_Lean_Expr_constLevels_x21(x_1); +x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8; +x_97 = l_Lean_Expr_const___override(x_96, x_95); +lean_inc(x_5); +x_98 = l_Lean_mkApp4(x_97, x_2, x_3, x_4, x_5); +x_99 = l_Lean_Expr_app___override(x_98, x_92); +x_100 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_100, 0, x_99); +x_101 = 1; +x_102 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_102, 0, x_5); +lean_ctor_set(x_102, 1, x_100); +lean_ctor_set_uint8(x_102, sizeof(void*)*2, x_101); +x_103 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_103, 0, x_102); +if (lean_is_scalar(x_94)) { + x_104 = lean_alloc_ctor(0, 2, 0); +} else { + x_104 = x_94; +} +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_93); +return x_104; +} +else +{ +lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_105 = lean_ctor_get(x_91, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_91, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_107 = x_91; +} else { + lean_dec_ref(x_91); + x_107 = lean_box(0); +} +if (lean_is_scalar(x_107)) { + x_108 = lean_alloc_ctor(1, 2, 0); +} else { + x_108 = x_107; +} +lean_ctor_set(x_108, 0, x_105); +lean_ctor_set(x_108, 1, x_106); +return x_108; +} +} +} +else +{ +lean_object* x_109; +lean_dec(x_84); +x_109 = l_Lean_Meta_Simp_Result_getProof(x_81, x_9, x_10, x_11, x_12, x_82); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_112 = x_109; +} else { + lean_dec_ref(x_109); + x_112 = lean_box(0); +} +x_113 = l_Lean_Expr_constLevels_x21(x_1); +x_114 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10; +x_115 = l_Lean_Expr_const___override(x_114, x_113); +lean_inc(x_4); +x_116 = l_Lean_mkApp4(x_115, x_2, x_3, x_4, x_5); +x_117 = l_Lean_Expr_app___override(x_116, x_110); +x_118 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_118, 0, x_117); +x_119 = 1; +x_120 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_120, 0, x_4); +lean_ctor_set(x_120, 1, x_118); +lean_ctor_set_uint8(x_120, sizeof(void*)*2, x_119); +x_121 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_121, 0, x_120); +if (lean_is_scalar(x_112)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_112; +} +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_111); +return x_122; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_123 = lean_ctor_get(x_109, 0); +lean_inc(x_123); +x_124 = lean_ctor_get(x_109, 1); +lean_inc(x_124); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_125 = x_109; +} else { + lean_dec_ref(x_109); + x_125 = lean_box(0); +} +if (lean_is_scalar(x_125)) { + x_126 = lean_alloc_ctor(1, 2, 0); +} else { + x_126 = x_125; +} +lean_ctor_set(x_126, 0, x_123); +lean_ctor_set(x_126, 1, x_124); +return x_126; +} +} +} +} +else +{ +uint8_t x_127; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_127 = !lean_is_exclusive(x_14); +if (x_127 == 0) +{ +return x_14; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_14, 0); +x_129 = lean_ctor_get(x_14, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_14); +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +return x_11; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed), 13, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed), 9, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("cond", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = l_Lean_Expr_appArg(x_22, lean_box(0)); +x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_28 = l_Lean_Expr_isApp(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); +x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; +x_34 = l_Lean_Expr_isConstOf(x_32, x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_35 = lean_box(0); +x_36 = lean_apply_9(x_11, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_36; +} +else +{ +lean_object* x_37; +x_37 = lean_apply_13(x_10, x_32, x_31, x_26, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_37; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Elab", 4, 4); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BVDecide", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Frontend", 8, 8); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Normalize", 9, 9); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("reduceCond", 10, 10); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4; +x_2 = lean_unsigned_to_nat(4u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = lean_box(3); +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_builtinBVNormalizeSimprocsRef; +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8; +x_4 = 0; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BEq", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("beq", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Eq", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = l_Lean_Level_ofNat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7; +x_3 = l_Lean_Expr_const___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Std", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_to_beq", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_12 = lean_box(0); +lean_inc(x_1); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_1); +lean_ctor_set(x_13, 1, x_12); +lean_inc(x_2); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_2); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_array_mk(x_14); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3; +x_17 = l_Lean_Meta_mkAppM(x_16, x_15, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; +x_19 = lean_ctor_get(x_17, 0); +x_20 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; +x_23 = l_Lean_mkApp3(x_20, x_21, x_19, x_22); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; +x_25 = l_Lean_mkAppB(x_24, x_2, x_1); +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_27 = 1; +x_28 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_28, 0, x_23); +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set_uint8(x_28, sizeof(void*)*2, x_27); +x_29 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_17, 0, x_29); +return x_17; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_30 = lean_ctor_get(x_17, 0); +x_31 = lean_ctor_get(x_17, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_17); +x_32 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8; +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10; +x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11; +x_35 = l_Lean_mkApp3(x_32, x_33, x_30, x_34); +x_36 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15; +x_37 = l_Lean_mkAppB(x_36, x_2, x_1); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_37); +x_39 = 1; +x_40 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_40, 0, x_35); +lean_ctor_set(x_40, 1, x_38); +lean_ctor_set_uint8(x_40, sizeof(void*)*2, x_39); +x_41 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_41, 0, x_40); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_31); +return x_42; +} +} +else +{ +uint8_t x_43; +lean_dec(x_2); +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_17); +if (x_43 == 0) +{ +return x_17; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_17, 0); +x_45 = lean_ctor_get(x_17, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_17); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_inc(x_2); +x_11 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_2, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_15 = l_Lean_Expr_cleanupAnnotations(x_12); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3; +x_17 = l_Lean_Expr_isConstOf(x_15, x_16); +lean_dec(x_15); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_box(0); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(x_2, x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_2); +lean_dec(x_1); +x_20 = lean_box(0); +x_21 = lean_apply_9(x_14, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_21; +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__2), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; +x_28 = l_Lean_Expr_isConstOf(x_26, x_27); +lean_dec(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_21); +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_30; +} +else +{ +lean_object* x_31; +x_31 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_31; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_12; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eqToBEq", 7, 7); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5; +x_2 = lean_unsigned_to_nat(3u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("BitVec", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("and_ones", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_11); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_12, 0); +x_22 = lean_ctor_get(x_11, 0); +lean_dec(x_22); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_unsigned_to_nat(1u); +x_26 = l_BitVec_ofNat(x_23, x_25); +x_27 = l_BitVec_neg(x_23, x_26); +lean_dec(x_26); +x_28 = lean_nat_dec_eq(x_24, x_27); +lean_dec(x_27); +lean_dec(x_24); +if (x_28 == 0) +{ +lean_object* x_29; +lean_dec(x_23); +lean_free_object(x_12); +lean_dec(x_1); +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_29); +return x_11; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; +x_30 = l_Lean_mkNatLit(x_23); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; +lean_inc(x_1); +x_32 = l_Lean_mkAppB(x_31, x_30, x_1); +lean_ctor_set(x_12, 0, x_32); +x_33 = 1; +x_34 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_34, 0, x_1); +lean_ctor_set(x_34, 1, x_12); +lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_33); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_11, 0, x_35); +return x_11; +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_36 = lean_ctor_get(x_12, 0); +x_37 = lean_ctor_get(x_11, 1); +lean_inc(x_37); +lean_dec(x_11); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_unsigned_to_nat(1u); +x_41 = l_BitVec_ofNat(x_38, x_40); +x_42 = l_BitVec_neg(x_38, x_41); +lean_dec(x_41); +x_43 = lean_nat_dec_eq(x_39, x_42); +lean_dec(x_42); +lean_dec(x_39); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +lean_dec(x_38); +lean_free_object(x_12); +lean_dec(x_1); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_37); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_46 = l_Lean_mkNatLit(x_38); +x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; +lean_inc(x_1); +x_48 = l_Lean_mkAppB(x_47, x_46, x_1); +lean_ctor_set(x_12, 0, x_48); +x_49 = 1; +x_50 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_50, 0, x_1); +lean_ctor_set(x_50, 1, x_12); +lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_49); +x_51 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_37); +return x_52; +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_53 = lean_ctor_get(x_12, 0); +lean_inc(x_53); +lean_dec(x_12); +x_54 = lean_ctor_get(x_11, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_11)) { + lean_ctor_release(x_11, 0); + lean_ctor_release(x_11, 1); + x_55 = x_11; +} else { + lean_dec_ref(x_11); + x_55 = lean_box(0); +} +x_56 = lean_ctor_get(x_53, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_53, 1); +lean_inc(x_57); +lean_dec(x_53); +x_58 = lean_unsigned_to_nat(1u); +x_59 = l_BitVec_ofNat(x_56, x_58); +x_60 = l_BitVec_neg(x_56, x_59); +lean_dec(x_59); +x_61 = lean_nat_dec_eq(x_57, x_60); +lean_dec(x_60); +lean_dec(x_57); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; +lean_dec(x_56); +lean_dec(x_1); +x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_55)) { + x_63 = lean_alloc_ctor(0, 2, 0); +} else { + x_63 = x_55; +} +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_54); +return x_63; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_64 = l_Lean_mkNatLit(x_56); +x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4; +lean_inc(x_1); +x_66 = l_Lean_mkAppB(x_65, x_64, x_1); +x_67 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_67, 0, x_66); +x_68 = 1; +x_69 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_69, 0, x_1); +lean_ctor_set(x_69, 1, x_67); +lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_68); +x_70 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_70, 0, x_69); +if (lean_is_scalar(x_55)) { + x_71 = lean_alloc_ctor(0, 2, 0); +} else { + x_71 = x_55; +} +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_54); +return x_71; +} +} +} +} +else +{ +uint8_t x_72; +lean_dec(x_1); +x_72 = !lean_is_exclusive(x_11); +if (x_72 == 0) +{ +return x_11; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_11, 0); +x_74 = lean_ctor_get(x_11, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_11); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HAnd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hAnd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_43; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_11; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("andOnes", 7, 7); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; +x_2 = lean_unsigned_to_nat(6u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4; +x_2 = lean_unsigned_to_nat(1u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ones_and", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_2); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_11); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_12, 0); +x_22 = lean_ctor_get(x_11, 0); +lean_dec(x_22); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_unsigned_to_nat(1u); +x_26 = l_BitVec_ofNat(x_23, x_25); +x_27 = l_BitVec_neg(x_23, x_26); +lean_dec(x_26); +x_28 = lean_nat_dec_eq(x_24, x_27); +lean_dec(x_27); +lean_dec(x_24); +if (x_28 == 0) +{ +lean_object* x_29; +lean_dec(x_23); +lean_free_object(x_12); +lean_dec(x_2); +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_29); +return x_11; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; +x_30 = l_Lean_mkNatLit(x_23); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; +lean_inc(x_2); +x_32 = l_Lean_mkAppB(x_31, x_30, x_2); +lean_ctor_set(x_12, 0, x_32); +x_33 = 1; +x_34 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_34, 0, x_2); +lean_ctor_set(x_34, 1, x_12); +lean_ctor_set_uint8(x_34, sizeof(void*)*2, x_33); +x_35 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_11, 0, x_35); +return x_11; +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_36 = lean_ctor_get(x_12, 0); +x_37 = lean_ctor_get(x_11, 1); +lean_inc(x_37); +lean_dec(x_11); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_36, 1); +lean_inc(x_39); +lean_dec(x_36); +x_40 = lean_unsigned_to_nat(1u); +x_41 = l_BitVec_ofNat(x_38, x_40); +x_42 = l_BitVec_neg(x_38, x_41); +lean_dec(x_41); +x_43 = lean_nat_dec_eq(x_39, x_42); +lean_dec(x_42); +lean_dec(x_39); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +lean_dec(x_38); +lean_free_object(x_12); +lean_dec(x_2); +x_44 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_37); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_46 = l_Lean_mkNatLit(x_38); +x_47 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; +lean_inc(x_2); +x_48 = l_Lean_mkAppB(x_47, x_46, x_2); +lean_ctor_set(x_12, 0, x_48); +x_49 = 1; +x_50 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_50, 0, x_2); +lean_ctor_set(x_50, 1, x_12); +lean_ctor_set_uint8(x_50, sizeof(void*)*2, x_49); +x_51 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_51, 0, x_50); +x_52 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_37); +return x_52; +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_53 = lean_ctor_get(x_12, 0); +lean_inc(x_53); +lean_dec(x_12); +x_54 = lean_ctor_get(x_11, 1); +lean_inc(x_54); +if (lean_is_exclusive(x_11)) { + lean_ctor_release(x_11, 0); + lean_ctor_release(x_11, 1); + x_55 = x_11; +} else { + lean_dec_ref(x_11); + x_55 = lean_box(0); +} +x_56 = lean_ctor_get(x_53, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_53, 1); +lean_inc(x_57); +lean_dec(x_53); +x_58 = lean_unsigned_to_nat(1u); +x_59 = l_BitVec_ofNat(x_56, x_58); +x_60 = l_BitVec_neg(x_56, x_59); +lean_dec(x_59); +x_61 = lean_nat_dec_eq(x_57, x_60); +lean_dec(x_60); +lean_dec(x_57); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; +lean_dec(x_56); +lean_dec(x_2); +x_62 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_55)) { + x_63 = lean_alloc_ctor(0, 2, 0); +} else { + x_63 = x_55; +} +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_54); +return x_63; +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_64 = l_Lean_mkNatLit(x_56); +x_65 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3; +lean_inc(x_2); +x_66 = l_Lean_mkAppB(x_65, x_64, x_2); +x_67 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_67, 0, x_66); +x_68 = 1; +x_69 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_69, 0, x_2); +lean_ctor_set(x_69, 1, x_67); +lean_ctor_set_uint8(x_69, sizeof(void*)*2, x_68); +x_70 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_70, 0, x_69); +if (lean_is_scalar(x_55)) { + x_71 = lean_alloc_ctor(0, 2, 0); +} else { + x_71 = x_55; +} +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_54); +return x_71; +} +} +} +} +else +{ +uint8_t x_72; +lean_dec(x_2); +x_72 = !lean_is_exclusive(x_11); +if (x_72 == 0) +{ +return x_11; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_11, 0); +x_74 = lean_ctor_get(x_11, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_11); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_43; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_11; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("onesAnd", 7, 7); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("max_ult'", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_2); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_11); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_12, 0); +x_22 = lean_ctor_get(x_11, 0); +lean_dec(x_22); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_unsigned_to_nat(1u); +x_26 = l_BitVec_ofNat(x_23, x_25); +x_27 = l_BitVec_neg(x_23, x_26); +lean_dec(x_26); +x_28 = lean_nat_dec_eq(x_24, x_27); +lean_dec(x_27); +lean_dec(x_24); +if (x_28 == 0) +{ +lean_object* x_29; +lean_dec(x_23); +lean_free_object(x_12); +lean_dec(x_2); +x_29 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_29); +return x_11; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; +x_30 = l_Lean_mkNatLit(x_23); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; +x_32 = l_Lean_mkAppB(x_31, x_30, x_2); +lean_ctor_set(x_12, 0, x_32); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; +x_34 = 1; +x_35 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_12); +lean_ctor_set_uint8(x_35, sizeof(void*)*2, x_34); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_11, 0, x_36); +return x_11; +} +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_37 = lean_ctor_get(x_12, 0); +x_38 = lean_ctor_get(x_11, 1); +lean_inc(x_38); +lean_dec(x_11); +x_39 = lean_ctor_get(x_37, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_37, 1); +lean_inc(x_40); +lean_dec(x_37); +x_41 = lean_unsigned_to_nat(1u); +x_42 = l_BitVec_ofNat(x_39, x_41); +x_43 = l_BitVec_neg(x_39, x_42); +lean_dec(x_42); +x_44 = lean_nat_dec_eq(x_40, x_43); +lean_dec(x_43); +lean_dec(x_40); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +lean_dec(x_39); +lean_free_object(x_12); +lean_dec(x_2); +x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_38); +return x_46; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_47 = l_Lean_mkNatLit(x_39); +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; +x_49 = l_Lean_mkAppB(x_48, x_47, x_2); +lean_ctor_set(x_12, 0, x_49); +x_50 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; +x_51 = 1; +x_52 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_12); +lean_ctor_set_uint8(x_52, sizeof(void*)*2, x_51); +x_53 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_53, 0, x_52); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_38); +return x_54; +} +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_55 = lean_ctor_get(x_12, 0); +lean_inc(x_55); +lean_dec(x_12); +x_56 = lean_ctor_get(x_11, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_11)) { + lean_ctor_release(x_11, 0); + lean_ctor_release(x_11, 1); + x_57 = x_11; +} else { + lean_dec_ref(x_11); + x_57 = lean_box(0); +} +x_58 = lean_ctor_get(x_55, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_55, 1); +lean_inc(x_59); +lean_dec(x_55); +x_60 = lean_unsigned_to_nat(1u); +x_61 = l_BitVec_ofNat(x_58, x_60); +x_62 = l_BitVec_neg(x_58, x_61); +lean_dec(x_61); +x_63 = lean_nat_dec_eq(x_59, x_62); +lean_dec(x_62); +lean_dec(x_59); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +lean_dec(x_58); +lean_dec(x_2); +x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_57)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_57; +} +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_56); +return x_65; +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_66 = l_Lean_mkNatLit(x_58); +x_67 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3; +x_68 = l_Lean_mkAppB(x_67, x_66, x_2); +x_69 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4; +x_71 = 1; +x_72 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_69); +lean_ctor_set_uint8(x_72, sizeof(void*)*2, x_71); +x_73 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_73, 0, x_72); +if (lean_is_scalar(x_57)) { + x_74 = lean_alloc_ctor(0, 2, 0); +} else { + x_74 = x_57; +} +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_56); +return x_74; +} +} +} +} +else +{ +uint8_t x_75; +lean_dec(x_2); +x_75 = !lean_is_exclusive(x_11); +if (x_75 == 0) +{ +return x_11; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_11, 0); +x_77 = lean_ctor_get(x_11, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_11); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ult", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; +x_28 = l_Lean_Expr_isConstOf(x_26, x_27); +lean_dec(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_21); +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_30; +} +else +{ +lean_object* x_31; +x_31 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_31; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_11; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("maxUlt", 6, 6); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3; +x_2 = lean_unsigned_to_nat(3u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("neg_eq_not_add", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Complement", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("complement", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HAdd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hAdd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ofNat", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_11 = l_Lean_Meta_getNatValue_x3f(x_2, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_11, 0); +lean_dec(x_14); +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_11, 0, x_15); +return x_11; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_dec(x_11); +x_17 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_dec(x_11); +x_20 = !lean_is_exclusive(x_12); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_12, 0); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_1); +x_22 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_box(0); +lean_inc(x_21); +x_26 = l_Lean_mkNatLit(x_21); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; +lean_inc(x_1); +lean_inc(x_26); +x_28 = l_Lean_mkAppB(x_27, x_26, x_1); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_1); +lean_ctor_set(x_29, 1, x_25); +x_30 = lean_array_mk(x_29); +x_31 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_32 = l_Lean_Meta_mkAppM(x_31, x_30, x_6, x_7, x_8, x_9, x_24); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = lean_unsigned_to_nat(1u); +x_36 = l_BitVec_ofNat(x_21, x_35); +lean_dec(x_21); +x_37 = l_Lean_mkNatLit(x_36); +x_38 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; +x_39 = l_Lean_mkAppB(x_38, x_26, x_37); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_25); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_33); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_array_mk(x_41); +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_44 = l_Lean_Meta_mkAppM(x_43, x_42, x_6, x_7, x_8, x_9, x_34); +if (lean_obj_tag(x_44) == 0) +{ +uint8_t x_45; +x_45 = !lean_is_exclusive(x_44); +if (x_45 == 0) +{ +lean_object* x_46; uint8_t x_47; lean_object* x_48; lean_object* x_49; +x_46 = lean_ctor_get(x_44, 0); +lean_ctor_set(x_12, 0, x_28); +x_47 = 1; +x_48 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_12); +lean_ctor_set_uint8(x_48, sizeof(void*)*2, x_47); +x_49 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_44, 0, x_49); +return x_44; +} +else +{ +lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_50 = lean_ctor_get(x_44, 0); +x_51 = lean_ctor_get(x_44, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_44); +lean_ctor_set(x_12, 0, x_28); +x_52 = 1; +x_53 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_53, 0, x_50); +lean_ctor_set(x_53, 1, x_12); +lean_ctor_set_uint8(x_53, sizeof(void*)*2, x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_51); +return x_55; +} +} +else +{ +uint8_t x_56; +lean_dec(x_28); +lean_free_object(x_12); +x_56 = !lean_is_exclusive(x_44); +if (x_56 == 0) +{ +return x_44; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_44, 0); +x_58 = lean_ctor_get(x_44, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_44); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; +} +} +} +else +{ +uint8_t x_60; +lean_dec(x_28); +lean_dec(x_26); +lean_free_object(x_12); +lean_dec(x_21); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_60 = !lean_is_exclusive(x_32); +if (x_60 == 0) +{ +return x_32; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_32, 0); +x_62 = lean_ctor_get(x_32, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_32); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; +} +} +} +else +{ +uint8_t x_64; +lean_dec(x_23); +lean_free_object(x_12); +lean_dec(x_21); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_64 = !lean_is_exclusive(x_22); +if (x_64 == 0) +{ +lean_object* x_65; lean_object* x_66; +x_65 = lean_ctor_get(x_22, 0); +lean_dec(x_65); +x_66 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_22, 0, x_66); +return x_22; +} +else +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_22, 1); +lean_inc(x_67); +lean_dec(x_22); +x_68 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_67); +return x_69; +} +} +} +else +{ +uint8_t x_70; +lean_free_object(x_12); +lean_dec(x_21); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_22); +if (x_70 == 0) +{ +return x_22; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_22, 0); +x_72 = lean_ctor_get(x_22, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_22); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} +} +else +{ +lean_object* x_74; lean_object* x_75; +x_74 = lean_ctor_get(x_12, 0); +lean_inc(x_74); +lean_dec(x_12); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_1); +x_75 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_6, x_7, x_8, x_9, x_19); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +if (lean_obj_tag(x_76) == 0) +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +x_78 = lean_box(0); +lean_inc(x_74); +x_79 = l_Lean_mkNatLit(x_74); +x_80 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3; +lean_inc(x_1); +lean_inc(x_79); +x_81 = l_Lean_mkAppB(x_80, x_79, x_1); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_1); +lean_ctor_set(x_82, 1, x_78); +x_83 = lean_array_mk(x_82); +x_84 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_85 = l_Lean_Meta_mkAppM(x_84, x_83, x_6, x_7, x_8, x_9, x_77); +if (lean_obj_tag(x_85) == 0) +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_88 = lean_unsigned_to_nat(1u); +x_89 = l_BitVec_ofNat(x_74, x_88); +lean_dec(x_74); +x_90 = l_Lean_mkNatLit(x_89); +x_91 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12; +x_92 = l_Lean_mkAppB(x_91, x_79, x_90); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_92); +lean_ctor_set(x_93, 1, x_78); +x_94 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_94, 0, x_86); +lean_ctor_set(x_94, 1, x_93); +x_95 = lean_array_mk(x_94); +x_96 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_97 = l_Lean_Meta_mkAppM(x_96, x_95, x_6, x_7, x_8, x_9, x_87); +if (lean_obj_tag(x_97) == 0) +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_98 = lean_ctor_get(x_97, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_97, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_100 = x_97; +} else { + lean_dec_ref(x_97); + x_100 = lean_box(0); +} +x_101 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_101, 0, x_81); +x_102 = 1; +x_103 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_103, 0, x_98); +lean_ctor_set(x_103, 1, x_101); +lean_ctor_set_uint8(x_103, sizeof(void*)*2, x_102); +x_104 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_104, 0, x_103); +if (lean_is_scalar(x_100)) { + x_105 = lean_alloc_ctor(0, 2, 0); +} else { + x_105 = x_100; +} +lean_ctor_set(x_105, 0, x_104); +lean_ctor_set(x_105, 1, x_99); +return x_105; +} +else +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_81); +x_106 = lean_ctor_get(x_97, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_97, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_108 = x_97; +} else { + lean_dec_ref(x_97); + x_108 = lean_box(0); +} +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(1, 2, 0); +} else { + x_109 = x_108; +} +lean_ctor_set(x_109, 0, x_106); +lean_ctor_set(x_109, 1, x_107); +return x_109; +} +} +else +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +lean_dec(x_81); +lean_dec(x_79); +lean_dec(x_74); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +x_110 = lean_ctor_get(x_85, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_85, 1); +lean_inc(x_111); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_112 = x_85; +} else { + lean_dec_ref(x_85); + x_112 = lean_box(0); +} +if (lean_is_scalar(x_112)) { + x_113 = lean_alloc_ctor(1, 2, 0); +} else { + x_113 = x_112; +} +lean_ctor_set(x_113, 0, x_110); +lean_ctor_set(x_113, 1, x_111); +return x_113; +} +} +else +{ +lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_76); +lean_dec(x_74); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_114 = lean_ctor_get(x_75, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_115 = x_75; +} else { + lean_dec_ref(x_75); + x_115 = lean_box(0); +} +x_116 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_115)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_115; +} +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_114); +return x_117; +} +} +else +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +lean_dec(x_74); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_118 = lean_ctor_get(x_75, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_75, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_120 = x_75; +} else { + lean_dec_ref(x_75); + x_120 = lean_box(0); +} +if (lean_is_scalar(x_120)) { + x_121 = lean_alloc_ctor(1, 2, 0); +} else { + x_121 = x_120; +} +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_119); +return x_121; +} +} +} +} +else +{ +uint8_t x_122; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_122 = !lean_is_exclusive(x_11); +if (x_122 == 0) +{ +return x_11; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_11, 0); +x_124 = lean_ctor_get(x_11, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_11); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4; +x_19 = l_Lean_Expr_isConstOf(x_17, x_18); +lean_dec(x_17); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_dec(x_16); +lean_dec(x_2); +x_20 = lean_box(0); +x_21 = lean_apply_9(x_11, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_21; +} +else +{ +lean_object* x_22; +x_22 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_16); +return x_22; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__2), 10, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Neg", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("neg", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; uint8_t x_22; +x_21 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_22 = l_Lean_Expr_isApp(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_21); +lean_dec(x_16); +x_23 = lean_box(0); +x_24 = lean_apply_9(x_11, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_24; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = l_Lean_Expr_appArg(x_21, lean_box(0)); +x_26 = l_Lean_Expr_appFnCleanup(x_21, lean_box(0)); +x_27 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; +x_28 = l_Lean_Expr_isConstOf(x_26, x_27); +lean_dec(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_25); +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_30; +} +else +{ +lean_object* x_31; +x_31 = lean_apply_10(x_10, x_25, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_31; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4; +x_2 = lean_unsigned_to_nat(3u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("add_const_right", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("add_const_left", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_1); +x_12 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_12, 0); +lean_dec(x_15); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_12, 0, x_16); +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_dec(x_12); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; +} +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_13); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_13, 0); +x_22 = lean_ctor_get(x_12, 1); +lean_inc(x_22); +lean_dec(x_12); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_26 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_29 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_28); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_29); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 0); +lean_dec(x_32); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_33); +return x_29; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_dec(x_29); +x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +uint8_t x_37; +x_37 = !lean_is_exclusive(x_30); +if (x_37 == 0) +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_29); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_39 = lean_ctor_get(x_30, 0); +x_40 = lean_ctor_get(x_29, 1); +x_41 = lean_ctor_get(x_29, 0); +lean_dec(x_41); +x_42 = !lean_is_exclusive(x_39); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; uint8_t x_45; +x_43 = lean_ctor_get(x_39, 0); +x_44 = lean_ctor_get(x_39, 1); +x_45 = lean_nat_dec_eq(x_24, x_43); +lean_dec(x_43); +if (x_45 == 0) +{ +lean_object* x_46; +lean_free_object(x_39); +lean_dec(x_44); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_46); +return x_29; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_free_object(x_29); +x_47 = l_BitVec_add(x_24, x_25, x_44); +lean_dec(x_44); +lean_dec(x_25); +x_48 = lean_box(0); +x_49 = l_Lean_mkNatLit(x_24); +x_50 = l_Lean_mkNatLit(x_47); +x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_49); +x_52 = l_Lean_mkAppB(x_51, x_49, x_50); +lean_inc(x_2); +lean_ctor_set_tag(x_39, 1); +lean_ctor_set(x_39, 1, x_48); +lean_ctor_set(x_39, 0, x_2); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_39); +lean_ctor_set(x_21, 0, x_52); +x_53 = lean_array_mk(x_21); +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_55 = l_Lean_Meta_mkAppM(x_54, x_53, x_7, x_8, x_9, x_10, x_40); +if (lean_obj_tag(x_55) == 0) +{ +uint8_t x_56; +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; +x_57 = lean_ctor_get(x_55, 0); +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_59 = l_Lean_mkApp4(x_58, x_49, x_1, x_2, x_3); +lean_ctor_set(x_30, 0, x_59); +x_60 = 1; +x_61 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_61, 0, x_57); +lean_ctor_set(x_61, 1, x_30); +lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_60); +lean_ctor_set(x_13, 0, x_61); +lean_ctor_set(x_55, 0, x_13); +return x_55; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; +x_62 = lean_ctor_get(x_55, 0); +x_63 = lean_ctor_get(x_55, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_55); +x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_65 = l_Lean_mkApp4(x_64, x_49, x_1, x_2, x_3); +lean_ctor_set(x_30, 0, x_65); +x_66 = 1; +x_67 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_67, 0, x_62); +lean_ctor_set(x_67, 1, x_30); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); +lean_ctor_set(x_13, 0, x_67); +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_13); +lean_ctor_set(x_68, 1, x_63); +return x_68; +} +} +else +{ +uint8_t x_69; +lean_dec(x_49); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_69 = !lean_is_exclusive(x_55); +if (x_69 == 0) +{ +return x_55; +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_55, 0); +x_71 = lean_ctor_get(x_55, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_55); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; +} +} +} +} +else +{ +lean_object* x_73; lean_object* x_74; uint8_t x_75; +x_73 = lean_ctor_get(x_39, 0); +x_74 = lean_ctor_get(x_39, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_39); +x_75 = lean_nat_dec_eq(x_24, x_73); +lean_dec(x_73); +if (x_75 == 0) +{ +lean_object* x_76; +lean_dec(x_74); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_76 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_76); +return x_29; +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_free_object(x_29); +x_77 = l_BitVec_add(x_24, x_25, x_74); +lean_dec(x_74); +lean_dec(x_25); +x_78 = lean_box(0); +x_79 = l_Lean_mkNatLit(x_24); +x_80 = l_Lean_mkNatLit(x_77); +x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_79); +x_82 = l_Lean_mkAppB(x_81, x_79, x_80); +lean_inc(x_2); +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_2); +lean_ctor_set(x_83, 1, x_78); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_83); +lean_ctor_set(x_21, 0, x_82); +x_84 = lean_array_mk(x_21); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_86 = l_Lean_Meta_mkAppM(x_85, x_84, x_7, x_8, x_9, x_10, x_40); +if (lean_obj_tag(x_86) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_89 = x_86; +} else { + lean_dec_ref(x_86); + x_89 = lean_box(0); +} +x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_91 = l_Lean_mkApp4(x_90, x_79, x_1, x_2, x_3); +lean_ctor_set(x_30, 0, x_91); +x_92 = 1; +x_93 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_93, 0, x_87); +lean_ctor_set(x_93, 1, x_30); +lean_ctor_set_uint8(x_93, sizeof(void*)*2, x_92); +lean_ctor_set(x_13, 0, x_93); +if (lean_is_scalar(x_89)) { + x_94 = lean_alloc_ctor(0, 2, 0); +} else { + x_94 = x_89; +} +lean_ctor_set(x_94, 0, x_13); +lean_ctor_set(x_94, 1, x_88); +return x_94; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_79); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_95 = lean_ctor_get(x_86, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_86, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_97 = x_86; +} else { + lean_dec_ref(x_86); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_99 = lean_ctor_get(x_30, 0); +x_100 = lean_ctor_get(x_29, 1); +lean_inc(x_100); +lean_dec(x_29); +x_101 = lean_ctor_get(x_99, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_99, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_103 = x_99; +} else { + lean_dec_ref(x_99); + x_103 = lean_box(0); +} +x_104 = lean_nat_dec_eq(x_24, x_101); +lean_dec(x_101); +if (x_104 == 0) +{ +lean_object* x_105; lean_object* x_106; +lean_dec(x_103); +lean_dec(x_102); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_100); +return x_106; +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_107 = l_BitVec_add(x_24, x_25, x_102); +lean_dec(x_102); +lean_dec(x_25); +x_108 = lean_box(0); +x_109 = l_Lean_mkNatLit(x_24); +x_110 = l_Lean_mkNatLit(x_107); +x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_109); +x_112 = l_Lean_mkAppB(x_111, x_109, x_110); +lean_inc(x_2); +if (lean_is_scalar(x_103)) { + x_113 = lean_alloc_ctor(1, 2, 0); +} else { + x_113 = x_103; + lean_ctor_set_tag(x_113, 1); +} +lean_ctor_set(x_113, 0, x_2); +lean_ctor_set(x_113, 1, x_108); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_113); +lean_ctor_set(x_21, 0, x_112); +x_114 = lean_array_mk(x_21); +x_115 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_116 = l_Lean_Meta_mkAppM(x_115, x_114, x_7, x_8, x_9, x_10, x_100); +if (lean_obj_tag(x_116) == 0) +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; +x_117 = lean_ctor_get(x_116, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_116, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_119 = x_116; +} else { + lean_dec_ref(x_116); + x_119 = lean_box(0); +} +x_120 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_121 = l_Lean_mkApp4(x_120, x_109, x_1, x_2, x_3); +lean_ctor_set(x_30, 0, x_121); +x_122 = 1; +x_123 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_123, 0, x_117); +lean_ctor_set(x_123, 1, x_30); +lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_122); +lean_ctor_set(x_13, 0, x_123); +if (lean_is_scalar(x_119)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_119; +} +lean_ctor_set(x_124, 0, x_13); +lean_ctor_set(x_124, 1, x_118); +return x_124; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_109); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_125 = lean_ctor_get(x_116, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_116, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_127 = x_116; +} else { + lean_dec_ref(x_116); + x_127 = lean_box(0); +} +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); +} else { + x_128 = x_127; +} +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; +} +} +} +} +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; +x_129 = lean_ctor_get(x_30, 0); +lean_inc(x_129); +lean_dec(x_30); +x_130 = lean_ctor_get(x_29, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_131 = x_29; +} else { + lean_dec_ref(x_29); + x_131 = lean_box(0); +} +x_132 = lean_ctor_get(x_129, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_129, 1); +lean_inc(x_133); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_134 = x_129; +} else { + lean_dec_ref(x_129); + x_134 = lean_box(0); +} +x_135 = lean_nat_dec_eq(x_24, x_132); +lean_dec(x_132); +if (x_135 == 0) +{ +lean_object* x_136; lean_object* x_137; +lean_dec(x_134); +lean_dec(x_133); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_136 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_131)) { + x_137 = lean_alloc_ctor(0, 2, 0); +} else { + x_137 = x_131; +} +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_130); +return x_137; +} +else +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +lean_dec(x_131); +x_138 = l_BitVec_add(x_24, x_25, x_133); +lean_dec(x_133); +lean_dec(x_25); +x_139 = lean_box(0); +x_140 = l_Lean_mkNatLit(x_24); +x_141 = l_Lean_mkNatLit(x_138); +x_142 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_140); +x_143 = l_Lean_mkAppB(x_142, x_140, x_141); +lean_inc(x_2); +if (lean_is_scalar(x_134)) { + x_144 = lean_alloc_ctor(1, 2, 0); +} else { + x_144 = x_134; + lean_ctor_set_tag(x_144, 1); +} +lean_ctor_set(x_144, 0, x_2); +lean_ctor_set(x_144, 1, x_139); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_144); +lean_ctor_set(x_21, 0, x_143); +x_145 = lean_array_mk(x_21); +x_146 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_147 = l_Lean_Meta_mkAppM(x_146, x_145, x_7, x_8, x_9, x_10, x_130); +if (lean_obj_tag(x_147) == 0) +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_147)) { + lean_ctor_release(x_147, 0); + lean_ctor_release(x_147, 1); + x_150 = x_147; +} else { + lean_dec_ref(x_147); + x_150 = lean_box(0); +} +x_151 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_152 = l_Lean_mkApp4(x_151, x_140, x_1, x_2, x_3); +x_153 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_153, 0, x_152); +x_154 = 1; +x_155 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_155, 0, x_148); +lean_ctor_set(x_155, 1, x_153); +lean_ctor_set_uint8(x_155, sizeof(void*)*2, x_154); +lean_ctor_set(x_13, 0, x_155); +if (lean_is_scalar(x_150)) { + x_156 = lean_alloc_ctor(0, 2, 0); +} else { + x_156 = x_150; +} +lean_ctor_set(x_156, 0, x_13); +lean_ctor_set(x_156, 1, x_149); +return x_156; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_140); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_157 = lean_ctor_get(x_147, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_147, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_147)) { + lean_ctor_release(x_147, 0); + lean_ctor_release(x_147, 1); + x_159 = x_147; +} else { + lean_dec_ref(x_147); + x_159 = lean_box(0); +} +if (lean_is_scalar(x_159)) { + x_160 = lean_alloc_ctor(1, 2, 0); +} else { + x_160 = x_159; +} +lean_ctor_set(x_160, 0, x_157); +lean_ctor_set(x_160, 1, x_158); +return x_160; +} +} +} +} +} +else +{ +uint8_t x_161; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_161 = !lean_is_exclusive(x_29); +if (x_161 == 0) +{ +return x_29; +} +else +{ +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_29, 0); +x_163 = lean_ctor_get(x_29, 1); +lean_inc(x_163); +lean_inc(x_162); +lean_dec(x_29); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_162); +lean_ctor_set(x_164, 1, x_163); +return x_164; +} +} +} +else +{ +uint8_t x_165; +x_165 = !lean_is_exclusive(x_27); +if (x_165 == 0) +{ +uint8_t x_166; +x_166 = !lean_is_exclusive(x_26); +if (x_166 == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; +x_167 = lean_ctor_get(x_27, 0); +x_168 = lean_ctor_get(x_26, 1); +x_169 = lean_ctor_get(x_26, 0); +lean_dec(x_169); +x_170 = !lean_is_exclusive(x_167); +if (x_170 == 0) +{ +lean_object* x_171; lean_object* x_172; uint8_t x_173; +x_171 = lean_ctor_get(x_167, 0); +x_172 = lean_ctor_get(x_167, 1); +x_173 = lean_nat_dec_eq(x_24, x_171); +lean_dec(x_171); +if (x_173 == 0) +{ +lean_object* x_174; +lean_free_object(x_167); +lean_dec(x_172); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_174 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_26, 0, x_174); +return x_26; +} +else +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +lean_free_object(x_26); +x_175 = l_BitVec_add(x_24, x_25, x_172); +lean_dec(x_172); +lean_dec(x_25); +x_176 = lean_box(0); +x_177 = l_Lean_mkNatLit(x_24); +x_178 = l_Lean_mkNatLit(x_175); +x_179 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_177); +x_180 = l_Lean_mkAppB(x_179, x_177, x_178); +lean_inc(x_3); +lean_ctor_set_tag(x_167, 1); +lean_ctor_set(x_167, 1, x_176); +lean_ctor_set(x_167, 0, x_3); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_167); +lean_ctor_set(x_21, 0, x_180); +x_181 = lean_array_mk(x_21); +x_182 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_183 = l_Lean_Meta_mkAppM(x_182, x_181, x_7, x_8, x_9, x_10, x_168); +if (lean_obj_tag(x_183) == 0) +{ +uint8_t x_184; +x_184 = !lean_is_exclusive(x_183); +if (x_184 == 0) +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; lean_object* x_189; +x_185 = lean_ctor_get(x_183, 0); +x_186 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_187 = l_Lean_mkApp4(x_186, x_177, x_1, x_2, x_3); +lean_ctor_set(x_27, 0, x_187); +x_188 = 1; +x_189 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_189, 0, x_185); +lean_ctor_set(x_189, 1, x_27); +lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_188); +lean_ctor_set(x_13, 0, x_189); +lean_ctor_set(x_183, 0, x_13); +return x_183; +} +else +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; lean_object* x_195; lean_object* x_196; +x_190 = lean_ctor_get(x_183, 0); +x_191 = lean_ctor_get(x_183, 1); +lean_inc(x_191); +lean_inc(x_190); +lean_dec(x_183); +x_192 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_193 = l_Lean_mkApp4(x_192, x_177, x_1, x_2, x_3); +lean_ctor_set(x_27, 0, x_193); +x_194 = 1; +x_195 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_195, 0, x_190); +lean_ctor_set(x_195, 1, x_27); +lean_ctor_set_uint8(x_195, sizeof(void*)*2, x_194); +lean_ctor_set(x_13, 0, x_195); +x_196 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_196, 0, x_13); +lean_ctor_set(x_196, 1, x_191); +return x_196; +} +} +else +{ +uint8_t x_197; +lean_dec(x_177); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_197 = !lean_is_exclusive(x_183); +if (x_197 == 0) +{ +return x_183; +} +else +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_198 = lean_ctor_get(x_183, 0); +x_199 = lean_ctor_get(x_183, 1); +lean_inc(x_199); +lean_inc(x_198); +lean_dec(x_183); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_198); +lean_ctor_set(x_200, 1, x_199); +return x_200; +} +} +} +} +else +{ +lean_object* x_201; lean_object* x_202; uint8_t x_203; +x_201 = lean_ctor_get(x_167, 0); +x_202 = lean_ctor_get(x_167, 1); +lean_inc(x_202); +lean_inc(x_201); +lean_dec(x_167); +x_203 = lean_nat_dec_eq(x_24, x_201); +lean_dec(x_201); +if (x_203 == 0) +{ +lean_object* x_204; +lean_dec(x_202); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_204 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_26, 0, x_204); +return x_26; +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +lean_free_object(x_26); +x_205 = l_BitVec_add(x_24, x_25, x_202); +lean_dec(x_202); +lean_dec(x_25); +x_206 = lean_box(0); +x_207 = l_Lean_mkNatLit(x_24); +x_208 = l_Lean_mkNatLit(x_205); +x_209 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_207); +x_210 = l_Lean_mkAppB(x_209, x_207, x_208); +lean_inc(x_3); +x_211 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_211, 0, x_3); +lean_ctor_set(x_211, 1, x_206); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_211); +lean_ctor_set(x_21, 0, x_210); +x_212 = lean_array_mk(x_21); +x_213 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_214 = l_Lean_Meta_mkAppM(x_213, x_212, x_7, x_8, x_9, x_10, x_168); +if (lean_obj_tag(x_214) == 0) +{ +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; lean_object* x_221; lean_object* x_222; +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_214, 1); +lean_inc(x_216); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_217 = x_214; +} else { + lean_dec_ref(x_214); + x_217 = lean_box(0); +} +x_218 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_219 = l_Lean_mkApp4(x_218, x_207, x_1, x_2, x_3); +lean_ctor_set(x_27, 0, x_219); +x_220 = 1; +x_221 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_221, 0, x_215); +lean_ctor_set(x_221, 1, x_27); +lean_ctor_set_uint8(x_221, sizeof(void*)*2, x_220); +lean_ctor_set(x_13, 0, x_221); +if (lean_is_scalar(x_217)) { + x_222 = lean_alloc_ctor(0, 2, 0); +} else { + x_222 = x_217; +} +lean_ctor_set(x_222, 0, x_13); +lean_ctor_set(x_222, 1, x_216); +return x_222; +} +else +{ +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; +lean_dec(x_207); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_223 = lean_ctor_get(x_214, 0); +lean_inc(x_223); +x_224 = lean_ctor_get(x_214, 1); +lean_inc(x_224); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_225 = x_214; +} else { + lean_dec_ref(x_214); + x_225 = lean_box(0); +} +if (lean_is_scalar(x_225)) { + x_226 = lean_alloc_ctor(1, 2, 0); +} else { + x_226 = x_225; +} +lean_ctor_set(x_226, 0, x_223); +lean_ctor_set(x_226, 1, x_224); +return x_226; +} +} +} +} +else +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; uint8_t x_232; +x_227 = lean_ctor_get(x_27, 0); +x_228 = lean_ctor_get(x_26, 1); +lean_inc(x_228); +lean_dec(x_26); +x_229 = lean_ctor_get(x_227, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_227, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_231 = x_227; +} else { + lean_dec_ref(x_227); + x_231 = lean_box(0); +} +x_232 = lean_nat_dec_eq(x_24, x_229); +lean_dec(x_229); +if (x_232 == 0) +{ +lean_object* x_233; lean_object* x_234; +lean_dec(x_231); +lean_dec(x_230); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_233 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_234 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_234, 0, x_233); +lean_ctor_set(x_234, 1, x_228); +return x_234; +} +else +{ +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; +x_235 = l_BitVec_add(x_24, x_25, x_230); +lean_dec(x_230); +lean_dec(x_25); +x_236 = lean_box(0); +x_237 = l_Lean_mkNatLit(x_24); +x_238 = l_Lean_mkNatLit(x_235); +x_239 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_237); +x_240 = l_Lean_mkAppB(x_239, x_237, x_238); +lean_inc(x_3); +if (lean_is_scalar(x_231)) { + x_241 = lean_alloc_ctor(1, 2, 0); +} else { + x_241 = x_231; + lean_ctor_set_tag(x_241, 1); +} +lean_ctor_set(x_241, 0, x_3); +lean_ctor_set(x_241, 1, x_236); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_241); +lean_ctor_set(x_21, 0, x_240); +x_242 = lean_array_mk(x_21); +x_243 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_244 = l_Lean_Meta_mkAppM(x_243, x_242, x_7, x_8, x_9, x_10, x_228); +if (lean_obj_tag(x_244) == 0) +{ +lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; uint8_t x_250; lean_object* x_251; lean_object* x_252; +x_245 = lean_ctor_get(x_244, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_244, 1); +lean_inc(x_246); +if (lean_is_exclusive(x_244)) { + lean_ctor_release(x_244, 0); + lean_ctor_release(x_244, 1); + x_247 = x_244; +} else { + lean_dec_ref(x_244); + x_247 = lean_box(0); +} +x_248 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_249 = l_Lean_mkApp4(x_248, x_237, x_1, x_2, x_3); +lean_ctor_set(x_27, 0, x_249); +x_250 = 1; +x_251 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_251, 0, x_245); +lean_ctor_set(x_251, 1, x_27); +lean_ctor_set_uint8(x_251, sizeof(void*)*2, x_250); +lean_ctor_set(x_13, 0, x_251); +if (lean_is_scalar(x_247)) { + x_252 = lean_alloc_ctor(0, 2, 0); +} else { + x_252 = x_247; +} +lean_ctor_set(x_252, 0, x_13); +lean_ctor_set(x_252, 1, x_246); +return x_252; +} +else +{ +lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +lean_dec(x_237); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_253 = lean_ctor_get(x_244, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_244, 1); +lean_inc(x_254); +if (lean_is_exclusive(x_244)) { + lean_ctor_release(x_244, 0); + lean_ctor_release(x_244, 1); + x_255 = x_244; +} else { + lean_dec_ref(x_244); + x_255 = lean_box(0); +} +if (lean_is_scalar(x_255)) { + x_256 = lean_alloc_ctor(1, 2, 0); +} else { + x_256 = x_255; +} +lean_ctor_set(x_256, 0, x_253); +lean_ctor_set(x_256, 1, x_254); +return x_256; +} +} +} +} +else +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; uint8_t x_263; +x_257 = lean_ctor_get(x_27, 0); +lean_inc(x_257); +lean_dec(x_27); +x_258 = lean_ctor_get(x_26, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_259 = x_26; +} else { + lean_dec_ref(x_26); + x_259 = lean_box(0); +} +x_260 = lean_ctor_get(x_257, 0); +lean_inc(x_260); +x_261 = lean_ctor_get(x_257, 1); +lean_inc(x_261); +if (lean_is_exclusive(x_257)) { + lean_ctor_release(x_257, 0); + lean_ctor_release(x_257, 1); + x_262 = x_257; +} else { + lean_dec_ref(x_257); + x_262 = lean_box(0); +} +x_263 = lean_nat_dec_eq(x_24, x_260); +lean_dec(x_260); +if (x_263 == 0) +{ +lean_object* x_264; lean_object* x_265; +lean_dec(x_262); +lean_dec(x_261); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_264 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_259)) { + x_265 = lean_alloc_ctor(0, 2, 0); +} else { + x_265 = x_259; +} +lean_ctor_set(x_265, 0, x_264); +lean_ctor_set(x_265, 1, x_258); +return x_265; +} +else +{ +lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; +lean_dec(x_259); +x_266 = l_BitVec_add(x_24, x_25, x_261); +lean_dec(x_261); +lean_dec(x_25); +x_267 = lean_box(0); +x_268 = l_Lean_mkNatLit(x_24); +x_269 = l_Lean_mkNatLit(x_266); +x_270 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_268); +x_271 = l_Lean_mkAppB(x_270, x_268, x_269); +lean_inc(x_3); +if (lean_is_scalar(x_262)) { + x_272 = lean_alloc_ctor(1, 2, 0); +} else { + x_272 = x_262; + lean_ctor_set_tag(x_272, 1); +} +lean_ctor_set(x_272, 0, x_3); +lean_ctor_set(x_272, 1, x_267); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_272); +lean_ctor_set(x_21, 0, x_271); +x_273 = lean_array_mk(x_21); +x_274 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_275 = l_Lean_Meta_mkAppM(x_274, x_273, x_7, x_8, x_9, x_10, x_258); +if (lean_obj_tag(x_275) == 0) +{ +lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; uint8_t x_282; lean_object* x_283; lean_object* x_284; +x_276 = lean_ctor_get(x_275, 0); +lean_inc(x_276); +x_277 = lean_ctor_get(x_275, 1); +lean_inc(x_277); +if (lean_is_exclusive(x_275)) { + lean_ctor_release(x_275, 0); + lean_ctor_release(x_275, 1); + x_278 = x_275; +} else { + lean_dec_ref(x_275); + x_278 = lean_box(0); +} +x_279 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_280 = l_Lean_mkApp4(x_279, x_268, x_1, x_2, x_3); +x_281 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_281, 0, x_280); +x_282 = 1; +x_283 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_283, 0, x_276); +lean_ctor_set(x_283, 1, x_281); +lean_ctor_set_uint8(x_283, sizeof(void*)*2, x_282); +lean_ctor_set(x_13, 0, x_283); +if (lean_is_scalar(x_278)) { + x_284 = lean_alloc_ctor(0, 2, 0); +} else { + x_284 = x_278; +} +lean_ctor_set(x_284, 0, x_13); +lean_ctor_set(x_284, 1, x_277); +return x_284; +} +else +{ +lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +lean_dec(x_268); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_285 = lean_ctor_get(x_275, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_275, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_275)) { + lean_ctor_release(x_275, 0); + lean_ctor_release(x_275, 1); + x_287 = x_275; +} else { + lean_dec_ref(x_275); + x_287 = lean_box(0); +} +if (lean_is_scalar(x_287)) { + x_288 = lean_alloc_ctor(1, 2, 0); +} else { + x_288 = x_287; +} +lean_ctor_set(x_288, 0, x_285); +lean_ctor_set(x_288, 1, x_286); +return x_288; +} +} +} +} +} +else +{ +uint8_t x_289; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_289 = !lean_is_exclusive(x_26); +if (x_289 == 0) +{ +return x_26; +} +else +{ +lean_object* x_290; lean_object* x_291; lean_object* x_292; +x_290 = lean_ctor_get(x_26, 0); +x_291 = lean_ctor_get(x_26, 1); +lean_inc(x_291); +lean_inc(x_290); +lean_dec(x_26); +x_292 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_292, 0, x_290); +lean_ctor_set(x_292, 1, x_291); +return x_292; +} +} +} +else +{ +lean_object* x_293; lean_object* x_294; lean_object* x_295; +x_293 = lean_ctor_get(x_21, 0); +x_294 = lean_ctor_get(x_21, 1); +lean_inc(x_294); +lean_inc(x_293); +lean_dec(x_21); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_295 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +if (lean_obj_tag(x_296) == 0) +{ +lean_object* x_297; lean_object* x_298; +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_298 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_297); +if (lean_obj_tag(x_298) == 0) +{ +lean_object* x_299; +x_299 = lean_ctor_get(x_298, 0); +lean_inc(x_299); +if (lean_obj_tag(x_299) == 0) +{ +lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_300 = lean_ctor_get(x_298, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_301 = x_298; +} else { + lean_dec_ref(x_298); + x_301 = lean_box(0); +} +x_302 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_301)) { + x_303 = lean_alloc_ctor(0, 2, 0); +} else { + x_303 = x_301; +} +lean_ctor_set(x_303, 0, x_302); +lean_ctor_set(x_303, 1, x_300); +return x_303; +} +else +{ +lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; uint8_t x_311; +x_304 = lean_ctor_get(x_299, 0); +lean_inc(x_304); +if (lean_is_exclusive(x_299)) { + lean_ctor_release(x_299, 0); + x_305 = x_299; +} else { + lean_dec_ref(x_299); + x_305 = lean_box(0); +} +x_306 = lean_ctor_get(x_298, 1); +lean_inc(x_306); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_307 = x_298; +} else { + lean_dec_ref(x_298); + x_307 = lean_box(0); +} +x_308 = lean_ctor_get(x_304, 0); +lean_inc(x_308); +x_309 = lean_ctor_get(x_304, 1); +lean_inc(x_309); +if (lean_is_exclusive(x_304)) { + lean_ctor_release(x_304, 0); + lean_ctor_release(x_304, 1); + x_310 = x_304; +} else { + lean_dec_ref(x_304); + x_310 = lean_box(0); +} +x_311 = lean_nat_dec_eq(x_293, x_308); +lean_dec(x_308); +if (x_311 == 0) +{ +lean_object* x_312; lean_object* x_313; +lean_dec(x_310); +lean_dec(x_309); +lean_dec(x_305); +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_312 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_307)) { + x_313 = lean_alloc_ctor(0, 2, 0); +} else { + x_313 = x_307; +} +lean_ctor_set(x_313, 0, x_312); +lean_ctor_set(x_313, 1, x_306); +return x_313; +} +else +{ +lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; +lean_dec(x_307); +x_314 = l_BitVec_add(x_293, x_294, x_309); +lean_dec(x_309); +lean_dec(x_294); +x_315 = lean_box(0); +x_316 = l_Lean_mkNatLit(x_293); +x_317 = l_Lean_mkNatLit(x_314); +x_318 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_316); +x_319 = l_Lean_mkAppB(x_318, x_316, x_317); +lean_inc(x_2); +if (lean_is_scalar(x_310)) { + x_320 = lean_alloc_ctor(1, 2, 0); +} else { + x_320 = x_310; + lean_ctor_set_tag(x_320, 1); +} +lean_ctor_set(x_320, 0, x_2); +lean_ctor_set(x_320, 1, x_315); +x_321 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_321, 0, x_319); +lean_ctor_set(x_321, 1, x_320); +x_322 = lean_array_mk(x_321); +x_323 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_324 = l_Lean_Meta_mkAppM(x_323, x_322, x_7, x_8, x_9, x_10, x_306); +if (lean_obj_tag(x_324) == 0) +{ +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; uint8_t x_331; lean_object* x_332; lean_object* x_333; +x_325 = lean_ctor_get(x_324, 0); +lean_inc(x_325); +x_326 = lean_ctor_get(x_324, 1); +lean_inc(x_326); +if (lean_is_exclusive(x_324)) { + lean_ctor_release(x_324, 0); + lean_ctor_release(x_324, 1); + x_327 = x_324; +} else { + lean_dec_ref(x_324); + x_327 = lean_box(0); +} +x_328 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_329 = l_Lean_mkApp4(x_328, x_316, x_1, x_2, x_3); +if (lean_is_scalar(x_305)) { + x_330 = lean_alloc_ctor(1, 1, 0); +} else { + x_330 = x_305; +} +lean_ctor_set(x_330, 0, x_329); +x_331 = 1; +x_332 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_332, 0, x_325); +lean_ctor_set(x_332, 1, x_330); +lean_ctor_set_uint8(x_332, sizeof(void*)*2, x_331); +lean_ctor_set(x_13, 0, x_332); +if (lean_is_scalar(x_327)) { + x_333 = lean_alloc_ctor(0, 2, 0); +} else { + x_333 = x_327; +} +lean_ctor_set(x_333, 0, x_13); +lean_ctor_set(x_333, 1, x_326); +return x_333; +} +else +{ +lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; +lean_dec(x_316); +lean_dec(x_305); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_334 = lean_ctor_get(x_324, 0); +lean_inc(x_334); +x_335 = lean_ctor_get(x_324, 1); +lean_inc(x_335); +if (lean_is_exclusive(x_324)) { + lean_ctor_release(x_324, 0); + lean_ctor_release(x_324, 1); + x_336 = x_324; +} else { + lean_dec_ref(x_324); + x_336 = lean_box(0); +} +if (lean_is_scalar(x_336)) { + x_337 = lean_alloc_ctor(1, 2, 0); +} else { + x_337 = x_336; +} +lean_ctor_set(x_337, 0, x_334); +lean_ctor_set(x_337, 1, x_335); +return x_337; +} +} +} +} +else +{ +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_338 = lean_ctor_get(x_298, 0); +lean_inc(x_338); +x_339 = lean_ctor_get(x_298, 1); +lean_inc(x_339); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_340 = x_298; +} else { + lean_dec_ref(x_298); + x_340 = lean_box(0); +} +if (lean_is_scalar(x_340)) { + x_341 = lean_alloc_ctor(1, 2, 0); +} else { + x_341 = x_340; +} +lean_ctor_set(x_341, 0, x_338); +lean_ctor_set(x_341, 1, x_339); +return x_341; +} +} +else +{ +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; +x_342 = lean_ctor_get(x_296, 0); +lean_inc(x_342); +if (lean_is_exclusive(x_296)) { + lean_ctor_release(x_296, 0); + x_343 = x_296; +} else { + lean_dec_ref(x_296); + x_343 = lean_box(0); +} +x_344 = lean_ctor_get(x_295, 1); +lean_inc(x_344); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_345 = x_295; +} else { + lean_dec_ref(x_295); + x_345 = lean_box(0); +} +x_346 = lean_ctor_get(x_342, 0); +lean_inc(x_346); +x_347 = lean_ctor_get(x_342, 1); +lean_inc(x_347); +if (lean_is_exclusive(x_342)) { + lean_ctor_release(x_342, 0); + lean_ctor_release(x_342, 1); + x_348 = x_342; +} else { + lean_dec_ref(x_342); + x_348 = lean_box(0); +} +x_349 = lean_nat_dec_eq(x_293, x_346); +lean_dec(x_346); +if (x_349 == 0) +{ +lean_object* x_350; lean_object* x_351; +lean_dec(x_348); +lean_dec(x_347); +lean_dec(x_343); +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_350 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_345)) { + x_351 = lean_alloc_ctor(0, 2, 0); +} else { + x_351 = x_345; +} +lean_ctor_set(x_351, 0, x_350); +lean_ctor_set(x_351, 1, x_344); +return x_351; +} +else +{ +lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; +lean_dec(x_345); +x_352 = l_BitVec_add(x_293, x_294, x_347); +lean_dec(x_347); +lean_dec(x_294); +x_353 = lean_box(0); +x_354 = l_Lean_mkNatLit(x_293); +x_355 = l_Lean_mkNatLit(x_352); +x_356 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_354); +x_357 = l_Lean_mkAppB(x_356, x_354, x_355); +lean_inc(x_3); +if (lean_is_scalar(x_348)) { + x_358 = lean_alloc_ctor(1, 2, 0); +} else { + x_358 = x_348; + lean_ctor_set_tag(x_358, 1); +} +lean_ctor_set(x_358, 0, x_3); +lean_ctor_set(x_358, 1, x_353); +x_359 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_359, 0, x_357); +lean_ctor_set(x_359, 1, x_358); +x_360 = lean_array_mk(x_359); +x_361 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_362 = l_Lean_Meta_mkAppM(x_361, x_360, x_7, x_8, x_9, x_10, x_344); +if (lean_obj_tag(x_362) == 0) +{ +lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; uint8_t x_369; lean_object* x_370; lean_object* x_371; +x_363 = lean_ctor_get(x_362, 0); +lean_inc(x_363); +x_364 = lean_ctor_get(x_362, 1); +lean_inc(x_364); +if (lean_is_exclusive(x_362)) { + lean_ctor_release(x_362, 0); + lean_ctor_release(x_362, 1); + x_365 = x_362; +} else { + lean_dec_ref(x_362); + x_365 = lean_box(0); +} +x_366 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_367 = l_Lean_mkApp4(x_366, x_354, x_1, x_2, x_3); +if (lean_is_scalar(x_343)) { + x_368 = lean_alloc_ctor(1, 1, 0); +} else { + x_368 = x_343; +} +lean_ctor_set(x_368, 0, x_367); +x_369 = 1; +x_370 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_370, 0, x_363); +lean_ctor_set(x_370, 1, x_368); +lean_ctor_set_uint8(x_370, sizeof(void*)*2, x_369); +lean_ctor_set(x_13, 0, x_370); +if (lean_is_scalar(x_365)) { + x_371 = lean_alloc_ctor(0, 2, 0); +} else { + x_371 = x_365; +} +lean_ctor_set(x_371, 0, x_13); +lean_ctor_set(x_371, 1, x_364); +return x_371; +} +else +{ +lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; +lean_dec(x_354); +lean_dec(x_343); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_372 = lean_ctor_get(x_362, 0); +lean_inc(x_372); +x_373 = lean_ctor_get(x_362, 1); +lean_inc(x_373); +if (lean_is_exclusive(x_362)) { + lean_ctor_release(x_362, 0); + lean_ctor_release(x_362, 1); + x_374 = x_362; +} else { + lean_dec_ref(x_362); + x_374 = lean_box(0); +} +if (lean_is_scalar(x_374)) { + x_375 = lean_alloc_ctor(1, 2, 0); +} else { + x_375 = x_374; +} +lean_ctor_set(x_375, 0, x_372); +lean_ctor_set(x_375, 1, x_373); +return x_375; +} +} +} +} +else +{ +lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_376 = lean_ctor_get(x_295, 0); +lean_inc(x_376); +x_377 = lean_ctor_get(x_295, 1); +lean_inc(x_377); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_378 = x_295; +} else { + lean_dec_ref(x_295); + x_378 = lean_box(0); +} +if (lean_is_scalar(x_378)) { + x_379 = lean_alloc_ctor(1, 2, 0); +} else { + x_379 = x_378; +} +lean_ctor_set(x_379, 0, x_376); +lean_ctor_set(x_379, 1, x_377); +return x_379; +} +} +} +else +{ +lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; +x_380 = lean_ctor_get(x_13, 0); +lean_inc(x_380); +lean_dec(x_13); +x_381 = lean_ctor_get(x_12, 1); +lean_inc(x_381); +lean_dec(x_12); +x_382 = lean_ctor_get(x_380, 0); +lean_inc(x_382); +x_383 = lean_ctor_get(x_380, 1); +lean_inc(x_383); +if (lean_is_exclusive(x_380)) { + lean_ctor_release(x_380, 0); + lean_ctor_release(x_380, 1); + x_384 = x_380; +} else { + lean_dec_ref(x_380); + x_384 = lean_box(0); +} +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_385 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_381); +if (lean_obj_tag(x_385) == 0) +{ +lean_object* x_386; +x_386 = lean_ctor_get(x_385, 0); +lean_inc(x_386); +if (lean_obj_tag(x_386) == 0) +{ +lean_object* x_387; lean_object* x_388; +x_387 = lean_ctor_get(x_385, 1); +lean_inc(x_387); +lean_dec(x_385); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_388 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_387); +if (lean_obj_tag(x_388) == 0) +{ +lean_object* x_389; +x_389 = lean_ctor_get(x_388, 0); +lean_inc(x_389); +if (lean_obj_tag(x_389) == 0) +{ +lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_390 = lean_ctor_get(x_388, 1); +lean_inc(x_390); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_391 = x_388; +} else { + lean_dec_ref(x_388); + x_391 = lean_box(0); +} +x_392 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_391)) { + x_393 = lean_alloc_ctor(0, 2, 0); +} else { + x_393 = x_391; +} +lean_ctor_set(x_393, 0, x_392); +lean_ctor_set(x_393, 1, x_390); +return x_393; +} +else +{ +lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; uint8_t x_401; +x_394 = lean_ctor_get(x_389, 0); +lean_inc(x_394); +if (lean_is_exclusive(x_389)) { + lean_ctor_release(x_389, 0); + x_395 = x_389; +} else { + lean_dec_ref(x_389); + x_395 = lean_box(0); +} +x_396 = lean_ctor_get(x_388, 1); +lean_inc(x_396); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_397 = x_388; +} else { + lean_dec_ref(x_388); + x_397 = lean_box(0); +} +x_398 = lean_ctor_get(x_394, 0); +lean_inc(x_398); +x_399 = lean_ctor_get(x_394, 1); +lean_inc(x_399); +if (lean_is_exclusive(x_394)) { + lean_ctor_release(x_394, 0); + lean_ctor_release(x_394, 1); + x_400 = x_394; +} else { + lean_dec_ref(x_394); + x_400 = lean_box(0); +} +x_401 = lean_nat_dec_eq(x_382, x_398); +lean_dec(x_398); +if (x_401 == 0) +{ +lean_object* x_402; lean_object* x_403; +lean_dec(x_400); +lean_dec(x_399); +lean_dec(x_395); +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_402 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_397)) { + x_403 = lean_alloc_ctor(0, 2, 0); +} else { + x_403 = x_397; +} +lean_ctor_set(x_403, 0, x_402); +lean_ctor_set(x_403, 1, x_396); +return x_403; +} +else +{ +lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; +lean_dec(x_397); +x_404 = l_BitVec_add(x_382, x_383, x_399); +lean_dec(x_399); +lean_dec(x_383); +x_405 = lean_box(0); +x_406 = l_Lean_mkNatLit(x_382); +x_407 = l_Lean_mkNatLit(x_404); +x_408 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_406); +x_409 = l_Lean_mkAppB(x_408, x_406, x_407); +lean_inc(x_2); +if (lean_is_scalar(x_400)) { + x_410 = lean_alloc_ctor(1, 2, 0); +} else { + x_410 = x_400; + lean_ctor_set_tag(x_410, 1); +} +lean_ctor_set(x_410, 0, x_2); +lean_ctor_set(x_410, 1, x_405); +if (lean_is_scalar(x_384)) { + x_411 = lean_alloc_ctor(1, 2, 0); +} else { + x_411 = x_384; + lean_ctor_set_tag(x_411, 1); +} +lean_ctor_set(x_411, 0, x_409); +lean_ctor_set(x_411, 1, x_410); +x_412 = lean_array_mk(x_411); +x_413 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_414 = l_Lean_Meta_mkAppM(x_413, x_412, x_7, x_8, x_9, x_10, x_396); +if (lean_obj_tag(x_414) == 0) +{ +lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; +x_415 = lean_ctor_get(x_414, 0); +lean_inc(x_415); +x_416 = lean_ctor_get(x_414, 1); +lean_inc(x_416); +if (lean_is_exclusive(x_414)) { + lean_ctor_release(x_414, 0); + lean_ctor_release(x_414, 1); + x_417 = x_414; +} else { + lean_dec_ref(x_414); + x_417 = lean_box(0); +} +x_418 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4; +x_419 = l_Lean_mkApp4(x_418, x_406, x_1, x_2, x_3); +if (lean_is_scalar(x_395)) { + x_420 = lean_alloc_ctor(1, 1, 0); +} else { + x_420 = x_395; +} +lean_ctor_set(x_420, 0, x_419); +x_421 = 1; +x_422 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_422, 0, x_415); +lean_ctor_set(x_422, 1, x_420); +lean_ctor_set_uint8(x_422, sizeof(void*)*2, x_421); +x_423 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_423, 0, x_422); +if (lean_is_scalar(x_417)) { + x_424 = lean_alloc_ctor(0, 2, 0); +} else { + x_424 = x_417; +} +lean_ctor_set(x_424, 0, x_423); +lean_ctor_set(x_424, 1, x_416); +return x_424; +} +else +{ +lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; +lean_dec(x_406); +lean_dec(x_395); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_425 = lean_ctor_get(x_414, 0); +lean_inc(x_425); +x_426 = lean_ctor_get(x_414, 1); +lean_inc(x_426); +if (lean_is_exclusive(x_414)) { + lean_ctor_release(x_414, 0); + lean_ctor_release(x_414, 1); + x_427 = x_414; +} else { + lean_dec_ref(x_414); + x_427 = lean_box(0); +} +if (lean_is_scalar(x_427)) { + x_428 = lean_alloc_ctor(1, 2, 0); +} else { + x_428 = x_427; +} +lean_ctor_set(x_428, 0, x_425); +lean_ctor_set(x_428, 1, x_426); +return x_428; +} +} +} +} +else +{ +lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_429 = lean_ctor_get(x_388, 0); +lean_inc(x_429); +x_430 = lean_ctor_get(x_388, 1); +lean_inc(x_430); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_431 = x_388; +} else { + lean_dec_ref(x_388); + x_431 = lean_box(0); +} +if (lean_is_scalar(x_431)) { + x_432 = lean_alloc_ctor(1, 2, 0); +} else { + x_432 = x_431; +} +lean_ctor_set(x_432, 0, x_429); +lean_ctor_set(x_432, 1, x_430); +return x_432; +} +} +else +{ +lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; uint8_t x_440; +x_433 = lean_ctor_get(x_386, 0); +lean_inc(x_433); +if (lean_is_exclusive(x_386)) { + lean_ctor_release(x_386, 0); + x_434 = x_386; +} else { + lean_dec_ref(x_386); + x_434 = lean_box(0); +} +x_435 = lean_ctor_get(x_385, 1); +lean_inc(x_435); +if (lean_is_exclusive(x_385)) { + lean_ctor_release(x_385, 0); + lean_ctor_release(x_385, 1); + x_436 = x_385; +} else { + lean_dec_ref(x_385); + x_436 = lean_box(0); +} +x_437 = lean_ctor_get(x_433, 0); +lean_inc(x_437); +x_438 = lean_ctor_get(x_433, 1); +lean_inc(x_438); +if (lean_is_exclusive(x_433)) { + lean_ctor_release(x_433, 0); + lean_ctor_release(x_433, 1); + x_439 = x_433; +} else { + lean_dec_ref(x_433); + x_439 = lean_box(0); +} +x_440 = lean_nat_dec_eq(x_382, x_437); +lean_dec(x_437); +if (x_440 == 0) +{ +lean_object* x_441; lean_object* x_442; +lean_dec(x_439); +lean_dec(x_438); +lean_dec(x_434); +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_441 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_436)) { + x_442 = lean_alloc_ctor(0, 2, 0); +} else { + x_442 = x_436; +} +lean_ctor_set(x_442, 0, x_441); +lean_ctor_set(x_442, 1, x_435); +return x_442; +} +else +{ +lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; +lean_dec(x_436); +x_443 = l_BitVec_add(x_382, x_383, x_438); +lean_dec(x_438); +lean_dec(x_383); +x_444 = lean_box(0); +x_445 = l_Lean_mkNatLit(x_382); +x_446 = l_Lean_mkNatLit(x_443); +x_447 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_445); +x_448 = l_Lean_mkAppB(x_447, x_445, x_446); +lean_inc(x_3); +if (lean_is_scalar(x_439)) { + x_449 = lean_alloc_ctor(1, 2, 0); +} else { + x_449 = x_439; + lean_ctor_set_tag(x_449, 1); +} +lean_ctor_set(x_449, 0, x_3); +lean_ctor_set(x_449, 1, x_444); +if (lean_is_scalar(x_384)) { + x_450 = lean_alloc_ctor(1, 2, 0); +} else { + x_450 = x_384; + lean_ctor_set_tag(x_450, 1); +} +lean_ctor_set(x_450, 0, x_448); +lean_ctor_set(x_450, 1, x_449); +x_451 = lean_array_mk(x_450); +x_452 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_453 = l_Lean_Meta_mkAppM(x_452, x_451, x_7, x_8, x_9, x_10, x_435); +if (lean_obj_tag(x_453) == 0) +{ +lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; uint8_t x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; +x_454 = lean_ctor_get(x_453, 0); +lean_inc(x_454); +x_455 = lean_ctor_get(x_453, 1); +lean_inc(x_455); +if (lean_is_exclusive(x_453)) { + lean_ctor_release(x_453, 0); + lean_ctor_release(x_453, 1); + x_456 = x_453; +} else { + lean_dec_ref(x_453); + x_456 = lean_box(0); +} +x_457 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7; +x_458 = l_Lean_mkApp4(x_457, x_445, x_1, x_2, x_3); +if (lean_is_scalar(x_434)) { + x_459 = lean_alloc_ctor(1, 1, 0); +} else { + x_459 = x_434; +} +lean_ctor_set(x_459, 0, x_458); +x_460 = 1; +x_461 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_461, 0, x_454); +lean_ctor_set(x_461, 1, x_459); +lean_ctor_set_uint8(x_461, sizeof(void*)*2, x_460); +x_462 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_462, 0, x_461); +if (lean_is_scalar(x_456)) { + x_463 = lean_alloc_ctor(0, 2, 0); +} else { + x_463 = x_456; +} +lean_ctor_set(x_463, 0, x_462); +lean_ctor_set(x_463, 1, x_455); +return x_463; +} +else +{ +lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; +lean_dec(x_445); +lean_dec(x_434); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_464 = lean_ctor_get(x_453, 0); +lean_inc(x_464); +x_465 = lean_ctor_get(x_453, 1); +lean_inc(x_465); +if (lean_is_exclusive(x_453)) { + lean_ctor_release(x_453, 0); + lean_ctor_release(x_453, 1); + x_466 = x_453; +} else { + lean_dec_ref(x_453); + x_466 = lean_box(0); +} +if (lean_is_scalar(x_466)) { + x_467 = lean_alloc_ctor(1, 2, 0); +} else { + x_467 = x_466; +} +lean_ctor_set(x_467, 0, x_464); +lean_ctor_set(x_467, 1, x_465); +return x_467; +} +} +} +} +else +{ +lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_468 = lean_ctor_get(x_385, 0); +lean_inc(x_468); +x_469 = lean_ctor_get(x_385, 1); +lean_inc(x_469); +if (lean_is_exclusive(x_385)) { + lean_ctor_release(x_385, 0); + lean_ctor_release(x_385, 1); + x_470 = x_385; +} else { + lean_dec_ref(x_385); + x_470 = lean_box(0); +} +if (lean_is_scalar(x_470)) { + x_471 = lean_alloc_ctor(1, 2, 0); +} else { + x_471 = x_470; +} +lean_ctor_set(x_471, 0, x_468); +lean_ctor_set(x_471, 1, x_469); +return x_471; +} +} +} +} +else +{ +uint8_t x_472; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_472 = !lean_is_exclusive(x_12); +if (x_472 == 0) +{ +return x_12; +} +else +{ +lean_object* x_473; lean_object* x_474; lean_object* x_475; +x_473 = lean_ctor_get(x_12, 0); +x_474 = lean_ctor_get(x_12, 1); +lean_inc(x_474); +lean_inc(x_473); +lean_dec(x_12); +x_475 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_475, 0, x_473); +lean_ctor_set(x_475, 1, x_474); +return x_475; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_2); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_1); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_1); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_1); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_1); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_1); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_1); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(x_1, x_21, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_43; +} +} +} +} +} +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__2), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_43; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bv_add_const", 12, 12); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_2 = lean_unsigned_to_nat(6u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("add_const_right'", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("add_const_left'", 15, 15); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_1); +x_12 = l_Lean_Meta_getBitVecValue_x3f(x_1, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_12, 0); +lean_dec(x_15); +x_16 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_12, 0, x_16); +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_dec(x_12); +x_18 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; +} +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_13); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_13, 0); +x_22 = lean_ctor_get(x_12, 1); +lean_inc(x_22); +lean_dec(x_12); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 0); +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_26 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_29 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_28); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +if (lean_obj_tag(x_30) == 0) +{ +uint8_t x_31; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_29); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 0); +lean_dec(x_32); +x_33 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_33); +return x_29; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 1); +lean_inc(x_34); +lean_dec(x_29); +x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_34); +return x_36; +} +} +else +{ +uint8_t x_37; +x_37 = !lean_is_exclusive(x_30); +if (x_37 == 0) +{ +uint8_t x_38; +x_38 = !lean_is_exclusive(x_29); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_39 = lean_ctor_get(x_30, 0); +x_40 = lean_ctor_get(x_29, 1); +x_41 = lean_ctor_get(x_29, 0); +lean_dec(x_41); +x_42 = !lean_is_exclusive(x_39); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; uint8_t x_45; +x_43 = lean_ctor_get(x_39, 0); +x_44 = lean_ctor_get(x_39, 1); +x_45 = lean_nat_dec_eq(x_24, x_43); +lean_dec(x_43); +if (x_45 == 0) +{ +lean_object* x_46; +lean_free_object(x_39); +lean_dec(x_44); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_46); +return x_29; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_free_object(x_29); +x_47 = l_BitVec_add(x_24, x_25, x_44); +lean_dec(x_44); +lean_dec(x_25); +x_48 = lean_box(0); +x_49 = l_Lean_mkNatLit(x_24); +x_50 = l_Lean_mkNatLit(x_47); +x_51 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_49); +x_52 = l_Lean_mkAppB(x_51, x_49, x_50); +lean_inc(x_2); +lean_ctor_set_tag(x_39, 1); +lean_ctor_set(x_39, 1, x_48); +lean_ctor_set(x_39, 0, x_2); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_39); +lean_ctor_set(x_21, 0, x_52); +x_53 = lean_array_mk(x_21); +x_54 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_55 = l_Lean_Meta_mkAppM(x_54, x_53, x_7, x_8, x_9, x_10, x_40); +if (lean_obj_tag(x_55) == 0) +{ +uint8_t x_56; +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; +x_57 = lean_ctor_get(x_55, 0); +x_58 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_59 = l_Lean_mkApp4(x_58, x_49, x_2, x_3, x_1); +lean_ctor_set(x_30, 0, x_59); +x_60 = 1; +x_61 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_61, 0, x_57); +lean_ctor_set(x_61, 1, x_30); +lean_ctor_set_uint8(x_61, sizeof(void*)*2, x_60); +lean_ctor_set(x_13, 0, x_61); +lean_ctor_set(x_55, 0, x_13); +return x_55; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; +x_62 = lean_ctor_get(x_55, 0); +x_63 = lean_ctor_get(x_55, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_55); +x_64 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_65 = l_Lean_mkApp4(x_64, x_49, x_2, x_3, x_1); +lean_ctor_set(x_30, 0, x_65); +x_66 = 1; +x_67 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_67, 0, x_62); +lean_ctor_set(x_67, 1, x_30); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); +lean_ctor_set(x_13, 0, x_67); +x_68 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_68, 0, x_13); +lean_ctor_set(x_68, 1, x_63); +return x_68; +} +} +else +{ +uint8_t x_69; +lean_dec(x_49); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_69 = !lean_is_exclusive(x_55); +if (x_69 == 0) +{ +return x_55; +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_55, 0); +x_71 = lean_ctor_get(x_55, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_55); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; +} +} +} +} +else +{ +lean_object* x_73; lean_object* x_74; uint8_t x_75; +x_73 = lean_ctor_get(x_39, 0); +x_74 = lean_ctor_get(x_39, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_39); +x_75 = lean_nat_dec_eq(x_24, x_73); +lean_dec(x_73); +if (x_75 == 0) +{ +lean_object* x_76; +lean_dec(x_74); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_76 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_29, 0, x_76); +return x_29; +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_free_object(x_29); +x_77 = l_BitVec_add(x_24, x_25, x_74); +lean_dec(x_74); +lean_dec(x_25); +x_78 = lean_box(0); +x_79 = l_Lean_mkNatLit(x_24); +x_80 = l_Lean_mkNatLit(x_77); +x_81 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_79); +x_82 = l_Lean_mkAppB(x_81, x_79, x_80); +lean_inc(x_2); +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_2); +lean_ctor_set(x_83, 1, x_78); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_83); +lean_ctor_set(x_21, 0, x_82); +x_84 = lean_array_mk(x_21); +x_85 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_86 = l_Lean_Meta_mkAppM(x_85, x_84, x_7, x_8, x_9, x_10, x_40); +if (lean_obj_tag(x_86) == 0) +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_89 = x_86; +} else { + lean_dec_ref(x_86); + x_89 = lean_box(0); +} +x_90 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_91 = l_Lean_mkApp4(x_90, x_79, x_2, x_3, x_1); +lean_ctor_set(x_30, 0, x_91); +x_92 = 1; +x_93 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_93, 0, x_87); +lean_ctor_set(x_93, 1, x_30); +lean_ctor_set_uint8(x_93, sizeof(void*)*2, x_92); +lean_ctor_set(x_13, 0, x_93); +if (lean_is_scalar(x_89)) { + x_94 = lean_alloc_ctor(0, 2, 0); +} else { + x_94 = x_89; +} +lean_ctor_set(x_94, 0, x_13); +lean_ctor_set(x_94, 1, x_88); +return x_94; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_79); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_95 = lean_ctor_get(x_86, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_86, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_97 = x_86; +} else { + lean_dec_ref(x_86); + x_97 = lean_box(0); +} +if (lean_is_scalar(x_97)) { + x_98 = lean_alloc_ctor(1, 2, 0); +} else { + x_98 = x_97; +} +lean_ctor_set(x_98, 0, x_95); +lean_ctor_set(x_98, 1, x_96); +return x_98; +} +} +} +} +else +{ +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; uint8_t x_104; +x_99 = lean_ctor_get(x_30, 0); +x_100 = lean_ctor_get(x_29, 1); +lean_inc(x_100); +lean_dec(x_29); +x_101 = lean_ctor_get(x_99, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_99, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_103 = x_99; +} else { + lean_dec_ref(x_99); + x_103 = lean_box(0); +} +x_104 = lean_nat_dec_eq(x_24, x_101); +lean_dec(x_101); +if (x_104 == 0) +{ +lean_object* x_105; lean_object* x_106; +lean_dec(x_103); +lean_dec(x_102); +lean_free_object(x_30); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_105 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_100); +return x_106; +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_107 = l_BitVec_add(x_24, x_25, x_102); +lean_dec(x_102); +lean_dec(x_25); +x_108 = lean_box(0); +x_109 = l_Lean_mkNatLit(x_24); +x_110 = l_Lean_mkNatLit(x_107); +x_111 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_109); +x_112 = l_Lean_mkAppB(x_111, x_109, x_110); +lean_inc(x_2); +if (lean_is_scalar(x_103)) { + x_113 = lean_alloc_ctor(1, 2, 0); +} else { + x_113 = x_103; + lean_ctor_set_tag(x_113, 1); +} +lean_ctor_set(x_113, 0, x_2); +lean_ctor_set(x_113, 1, x_108); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_113); +lean_ctor_set(x_21, 0, x_112); +x_114 = lean_array_mk(x_21); +x_115 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_116 = l_Lean_Meta_mkAppM(x_115, x_114, x_7, x_8, x_9, x_10, x_100); +if (lean_obj_tag(x_116) == 0) +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; +x_117 = lean_ctor_get(x_116, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_116, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_119 = x_116; +} else { + lean_dec_ref(x_116); + x_119 = lean_box(0); +} +x_120 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_121 = l_Lean_mkApp4(x_120, x_109, x_2, x_3, x_1); +lean_ctor_set(x_30, 0, x_121); +x_122 = 1; +x_123 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_123, 0, x_117); +lean_ctor_set(x_123, 1, x_30); +lean_ctor_set_uint8(x_123, sizeof(void*)*2, x_122); +lean_ctor_set(x_13, 0, x_123); +if (lean_is_scalar(x_119)) { + x_124 = lean_alloc_ctor(0, 2, 0); +} else { + x_124 = x_119; +} +lean_ctor_set(x_124, 0, x_13); +lean_ctor_set(x_124, 1, x_118); +return x_124; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_109); +lean_free_object(x_30); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_125 = lean_ctor_get(x_116, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_116, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_127 = x_116; +} else { + lean_dec_ref(x_116); + x_127 = lean_box(0); +} +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); +} else { + x_128 = x_127; +} +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; +} +} +} +} +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; +x_129 = lean_ctor_get(x_30, 0); +lean_inc(x_129); +lean_dec(x_30); +x_130 = lean_ctor_get(x_29, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_131 = x_29; +} else { + lean_dec_ref(x_29); + x_131 = lean_box(0); +} +x_132 = lean_ctor_get(x_129, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_129, 1); +lean_inc(x_133); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_134 = x_129; +} else { + lean_dec_ref(x_129); + x_134 = lean_box(0); +} +x_135 = lean_nat_dec_eq(x_24, x_132); +lean_dec(x_132); +if (x_135 == 0) +{ +lean_object* x_136; lean_object* x_137; +lean_dec(x_134); +lean_dec(x_133); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_136 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_131)) { + x_137 = lean_alloc_ctor(0, 2, 0); +} else { + x_137 = x_131; +} +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_130); +return x_137; +} +else +{ +lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; +lean_dec(x_131); +x_138 = l_BitVec_add(x_24, x_25, x_133); +lean_dec(x_133); +lean_dec(x_25); +x_139 = lean_box(0); +x_140 = l_Lean_mkNatLit(x_24); +x_141 = l_Lean_mkNatLit(x_138); +x_142 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_140); +x_143 = l_Lean_mkAppB(x_142, x_140, x_141); +lean_inc(x_2); +if (lean_is_scalar(x_134)) { + x_144 = lean_alloc_ctor(1, 2, 0); +} else { + x_144 = x_134; + lean_ctor_set_tag(x_144, 1); +} +lean_ctor_set(x_144, 0, x_2); +lean_ctor_set(x_144, 1, x_139); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_144); +lean_ctor_set(x_21, 0, x_143); +x_145 = lean_array_mk(x_21); +x_146 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_147 = l_Lean_Meta_mkAppM(x_146, x_145, x_7, x_8, x_9, x_10, x_130); +if (lean_obj_tag(x_147) == 0) +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_147)) { + lean_ctor_release(x_147, 0); + lean_ctor_release(x_147, 1); + x_150 = x_147; +} else { + lean_dec_ref(x_147); + x_150 = lean_box(0); +} +x_151 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_152 = l_Lean_mkApp4(x_151, x_140, x_2, x_3, x_1); +x_153 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_153, 0, x_152); +x_154 = 1; +x_155 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_155, 0, x_148); +lean_ctor_set(x_155, 1, x_153); +lean_ctor_set_uint8(x_155, sizeof(void*)*2, x_154); +lean_ctor_set(x_13, 0, x_155); +if (lean_is_scalar(x_150)) { + x_156 = lean_alloc_ctor(0, 2, 0); +} else { + x_156 = x_150; +} +lean_ctor_set(x_156, 0, x_13); +lean_ctor_set(x_156, 1, x_149); +return x_156; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_140); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_157 = lean_ctor_get(x_147, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_147, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_147)) { + lean_ctor_release(x_147, 0); + lean_ctor_release(x_147, 1); + x_159 = x_147; +} else { + lean_dec_ref(x_147); + x_159 = lean_box(0); +} +if (lean_is_scalar(x_159)) { + x_160 = lean_alloc_ctor(1, 2, 0); +} else { + x_160 = x_159; +} +lean_ctor_set(x_160, 0, x_157); +lean_ctor_set(x_160, 1, x_158); +return x_160; +} +} +} +} +} +else +{ +uint8_t x_161; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_161 = !lean_is_exclusive(x_29); +if (x_161 == 0) +{ +return x_29; +} +else +{ +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_29, 0); +x_163 = lean_ctor_get(x_29, 1); +lean_inc(x_163); +lean_inc(x_162); +lean_dec(x_29); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_162); +lean_ctor_set(x_164, 1, x_163); +return x_164; +} +} +} +else +{ +uint8_t x_165; +x_165 = !lean_is_exclusive(x_27); +if (x_165 == 0) +{ +uint8_t x_166; +x_166 = !lean_is_exclusive(x_26); +if (x_166 == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; uint8_t x_170; +x_167 = lean_ctor_get(x_27, 0); +x_168 = lean_ctor_get(x_26, 1); +x_169 = lean_ctor_get(x_26, 0); +lean_dec(x_169); +x_170 = !lean_is_exclusive(x_167); +if (x_170 == 0) +{ +lean_object* x_171; lean_object* x_172; uint8_t x_173; +x_171 = lean_ctor_get(x_167, 0); +x_172 = lean_ctor_get(x_167, 1); +x_173 = lean_nat_dec_eq(x_24, x_171); +lean_dec(x_171); +if (x_173 == 0) +{ +lean_object* x_174; +lean_free_object(x_167); +lean_dec(x_172); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_174 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_26, 0, x_174); +return x_26; +} +else +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +lean_free_object(x_26); +x_175 = l_BitVec_add(x_24, x_25, x_172); +lean_dec(x_172); +lean_dec(x_25); +x_176 = lean_box(0); +x_177 = l_Lean_mkNatLit(x_24); +x_178 = l_Lean_mkNatLit(x_175); +x_179 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_177); +x_180 = l_Lean_mkAppB(x_179, x_177, x_178); +lean_inc(x_3); +lean_ctor_set_tag(x_167, 1); +lean_ctor_set(x_167, 1, x_176); +lean_ctor_set(x_167, 0, x_3); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_167); +lean_ctor_set(x_21, 0, x_180); +x_181 = lean_array_mk(x_21); +x_182 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_183 = l_Lean_Meta_mkAppM(x_182, x_181, x_7, x_8, x_9, x_10, x_168); +if (lean_obj_tag(x_183) == 0) +{ +uint8_t x_184; +x_184 = !lean_is_exclusive(x_183); +if (x_184 == 0) +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; uint8_t x_188; lean_object* x_189; +x_185 = lean_ctor_get(x_183, 0); +x_186 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_187 = l_Lean_mkApp4(x_186, x_177, x_2, x_3, x_1); +lean_ctor_set(x_27, 0, x_187); +x_188 = 1; +x_189 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_189, 0, x_185); +lean_ctor_set(x_189, 1, x_27); +lean_ctor_set_uint8(x_189, sizeof(void*)*2, x_188); +lean_ctor_set(x_13, 0, x_189); +lean_ctor_set(x_183, 0, x_13); +return x_183; +} +else +{ +lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; lean_object* x_195; lean_object* x_196; +x_190 = lean_ctor_get(x_183, 0); +x_191 = lean_ctor_get(x_183, 1); +lean_inc(x_191); +lean_inc(x_190); +lean_dec(x_183); +x_192 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_193 = l_Lean_mkApp4(x_192, x_177, x_2, x_3, x_1); +lean_ctor_set(x_27, 0, x_193); +x_194 = 1; +x_195 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_195, 0, x_190); +lean_ctor_set(x_195, 1, x_27); +lean_ctor_set_uint8(x_195, sizeof(void*)*2, x_194); +lean_ctor_set(x_13, 0, x_195); +x_196 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_196, 0, x_13); +lean_ctor_set(x_196, 1, x_191); +return x_196; +} +} +else +{ +uint8_t x_197; +lean_dec(x_177); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_197 = !lean_is_exclusive(x_183); +if (x_197 == 0) +{ +return x_183; +} +else +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_198 = lean_ctor_get(x_183, 0); +x_199 = lean_ctor_get(x_183, 1); +lean_inc(x_199); +lean_inc(x_198); +lean_dec(x_183); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_198); +lean_ctor_set(x_200, 1, x_199); +return x_200; +} +} +} +} +else +{ +lean_object* x_201; lean_object* x_202; uint8_t x_203; +x_201 = lean_ctor_get(x_167, 0); +x_202 = lean_ctor_get(x_167, 1); +lean_inc(x_202); +lean_inc(x_201); +lean_dec(x_167); +x_203 = lean_nat_dec_eq(x_24, x_201); +lean_dec(x_201); +if (x_203 == 0) +{ +lean_object* x_204; +lean_dec(x_202); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_204 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_26, 0, x_204); +return x_26; +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +lean_free_object(x_26); +x_205 = l_BitVec_add(x_24, x_25, x_202); +lean_dec(x_202); +lean_dec(x_25); +x_206 = lean_box(0); +x_207 = l_Lean_mkNatLit(x_24); +x_208 = l_Lean_mkNatLit(x_205); +x_209 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_207); +x_210 = l_Lean_mkAppB(x_209, x_207, x_208); +lean_inc(x_3); +x_211 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_211, 0, x_3); +lean_ctor_set(x_211, 1, x_206); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_211); +lean_ctor_set(x_21, 0, x_210); +x_212 = lean_array_mk(x_21); +x_213 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_214 = l_Lean_Meta_mkAppM(x_213, x_212, x_7, x_8, x_9, x_10, x_168); +if (lean_obj_tag(x_214) == 0) +{ +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; uint8_t x_220; lean_object* x_221; lean_object* x_222; +x_215 = lean_ctor_get(x_214, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_214, 1); +lean_inc(x_216); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_217 = x_214; +} else { + lean_dec_ref(x_214); + x_217 = lean_box(0); +} +x_218 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_219 = l_Lean_mkApp4(x_218, x_207, x_2, x_3, x_1); +lean_ctor_set(x_27, 0, x_219); +x_220 = 1; +x_221 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_221, 0, x_215); +lean_ctor_set(x_221, 1, x_27); +lean_ctor_set_uint8(x_221, sizeof(void*)*2, x_220); +lean_ctor_set(x_13, 0, x_221); +if (lean_is_scalar(x_217)) { + x_222 = lean_alloc_ctor(0, 2, 0); +} else { + x_222 = x_217; +} +lean_ctor_set(x_222, 0, x_13); +lean_ctor_set(x_222, 1, x_216); +return x_222; +} +else +{ +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; +lean_dec(x_207); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_223 = lean_ctor_get(x_214, 0); +lean_inc(x_223); +x_224 = lean_ctor_get(x_214, 1); +lean_inc(x_224); +if (lean_is_exclusive(x_214)) { + lean_ctor_release(x_214, 0); + lean_ctor_release(x_214, 1); + x_225 = x_214; +} else { + lean_dec_ref(x_214); + x_225 = lean_box(0); +} +if (lean_is_scalar(x_225)) { + x_226 = lean_alloc_ctor(1, 2, 0); +} else { + x_226 = x_225; +} +lean_ctor_set(x_226, 0, x_223); +lean_ctor_set(x_226, 1, x_224); +return x_226; +} +} +} +} +else +{ +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; uint8_t x_232; +x_227 = lean_ctor_get(x_27, 0); +x_228 = lean_ctor_get(x_26, 1); +lean_inc(x_228); +lean_dec(x_26); +x_229 = lean_ctor_get(x_227, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_227, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_231 = x_227; +} else { + lean_dec_ref(x_227); + x_231 = lean_box(0); +} +x_232 = lean_nat_dec_eq(x_24, x_229); +lean_dec(x_229); +if (x_232 == 0) +{ +lean_object* x_233; lean_object* x_234; +lean_dec(x_231); +lean_dec(x_230); +lean_free_object(x_27); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_233 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_234 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_234, 0, x_233); +lean_ctor_set(x_234, 1, x_228); +return x_234; +} +else +{ +lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; +x_235 = l_BitVec_add(x_24, x_25, x_230); +lean_dec(x_230); +lean_dec(x_25); +x_236 = lean_box(0); +x_237 = l_Lean_mkNatLit(x_24); +x_238 = l_Lean_mkNatLit(x_235); +x_239 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_237); +x_240 = l_Lean_mkAppB(x_239, x_237, x_238); +lean_inc(x_3); +if (lean_is_scalar(x_231)) { + x_241 = lean_alloc_ctor(1, 2, 0); +} else { + x_241 = x_231; + lean_ctor_set_tag(x_241, 1); +} +lean_ctor_set(x_241, 0, x_3); +lean_ctor_set(x_241, 1, x_236); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_241); +lean_ctor_set(x_21, 0, x_240); +x_242 = lean_array_mk(x_21); +x_243 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_244 = l_Lean_Meta_mkAppM(x_243, x_242, x_7, x_8, x_9, x_10, x_228); +if (lean_obj_tag(x_244) == 0) +{ +lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; uint8_t x_250; lean_object* x_251; lean_object* x_252; +x_245 = lean_ctor_get(x_244, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_244, 1); +lean_inc(x_246); +if (lean_is_exclusive(x_244)) { + lean_ctor_release(x_244, 0); + lean_ctor_release(x_244, 1); + x_247 = x_244; +} else { + lean_dec_ref(x_244); + x_247 = lean_box(0); +} +x_248 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_249 = l_Lean_mkApp4(x_248, x_237, x_2, x_3, x_1); +lean_ctor_set(x_27, 0, x_249); +x_250 = 1; +x_251 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_251, 0, x_245); +lean_ctor_set(x_251, 1, x_27); +lean_ctor_set_uint8(x_251, sizeof(void*)*2, x_250); +lean_ctor_set(x_13, 0, x_251); +if (lean_is_scalar(x_247)) { + x_252 = lean_alloc_ctor(0, 2, 0); +} else { + x_252 = x_247; +} +lean_ctor_set(x_252, 0, x_13); +lean_ctor_set(x_252, 1, x_246); +return x_252; +} +else +{ +lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; +lean_dec(x_237); +lean_free_object(x_27); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_253 = lean_ctor_get(x_244, 0); +lean_inc(x_253); +x_254 = lean_ctor_get(x_244, 1); +lean_inc(x_254); +if (lean_is_exclusive(x_244)) { + lean_ctor_release(x_244, 0); + lean_ctor_release(x_244, 1); + x_255 = x_244; +} else { + lean_dec_ref(x_244); + x_255 = lean_box(0); +} +if (lean_is_scalar(x_255)) { + x_256 = lean_alloc_ctor(1, 2, 0); +} else { + x_256 = x_255; +} +lean_ctor_set(x_256, 0, x_253); +lean_ctor_set(x_256, 1, x_254); +return x_256; +} +} +} +} +else +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; uint8_t x_263; +x_257 = lean_ctor_get(x_27, 0); +lean_inc(x_257); +lean_dec(x_27); +x_258 = lean_ctor_get(x_26, 1); +lean_inc(x_258); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_259 = x_26; +} else { + lean_dec_ref(x_26); + x_259 = lean_box(0); +} +x_260 = lean_ctor_get(x_257, 0); +lean_inc(x_260); +x_261 = lean_ctor_get(x_257, 1); +lean_inc(x_261); +if (lean_is_exclusive(x_257)) { + lean_ctor_release(x_257, 0); + lean_ctor_release(x_257, 1); + x_262 = x_257; +} else { + lean_dec_ref(x_257); + x_262 = lean_box(0); +} +x_263 = lean_nat_dec_eq(x_24, x_260); +lean_dec(x_260); +if (x_263 == 0) +{ +lean_object* x_264; lean_object* x_265; +lean_dec(x_262); +lean_dec(x_261); +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_264 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_259)) { + x_265 = lean_alloc_ctor(0, 2, 0); +} else { + x_265 = x_259; +} +lean_ctor_set(x_265, 0, x_264); +lean_ctor_set(x_265, 1, x_258); +return x_265; +} +else +{ +lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; +lean_dec(x_259); +x_266 = l_BitVec_add(x_24, x_25, x_261); +lean_dec(x_261); +lean_dec(x_25); +x_267 = lean_box(0); +x_268 = l_Lean_mkNatLit(x_24); +x_269 = l_Lean_mkNatLit(x_266); +x_270 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_268); +x_271 = l_Lean_mkAppB(x_270, x_268, x_269); +lean_inc(x_3); +if (lean_is_scalar(x_262)) { + x_272 = lean_alloc_ctor(1, 2, 0); +} else { + x_272 = x_262; + lean_ctor_set_tag(x_272, 1); +} +lean_ctor_set(x_272, 0, x_3); +lean_ctor_set(x_272, 1, x_267); +lean_ctor_set_tag(x_21, 1); +lean_ctor_set(x_21, 1, x_272); +lean_ctor_set(x_21, 0, x_271); +x_273 = lean_array_mk(x_21); +x_274 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_275 = l_Lean_Meta_mkAppM(x_274, x_273, x_7, x_8, x_9, x_10, x_258); +if (lean_obj_tag(x_275) == 0) +{ +lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; uint8_t x_282; lean_object* x_283; lean_object* x_284; +x_276 = lean_ctor_get(x_275, 0); +lean_inc(x_276); +x_277 = lean_ctor_get(x_275, 1); +lean_inc(x_277); +if (lean_is_exclusive(x_275)) { + lean_ctor_release(x_275, 0); + lean_ctor_release(x_275, 1); + x_278 = x_275; +} else { + lean_dec_ref(x_275); + x_278 = lean_box(0); +} +x_279 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_280 = l_Lean_mkApp4(x_279, x_268, x_2, x_3, x_1); +x_281 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_281, 0, x_280); +x_282 = 1; +x_283 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_283, 0, x_276); +lean_ctor_set(x_283, 1, x_281); +lean_ctor_set_uint8(x_283, sizeof(void*)*2, x_282); +lean_ctor_set(x_13, 0, x_283); +if (lean_is_scalar(x_278)) { + x_284 = lean_alloc_ctor(0, 2, 0); +} else { + x_284 = x_278; +} +lean_ctor_set(x_284, 0, x_13); +lean_ctor_set(x_284, 1, x_277); +return x_284; +} +else +{ +lean_object* x_285; lean_object* x_286; lean_object* x_287; lean_object* x_288; +lean_dec(x_268); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_285 = lean_ctor_get(x_275, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_275, 1); +lean_inc(x_286); +if (lean_is_exclusive(x_275)) { + lean_ctor_release(x_275, 0); + lean_ctor_release(x_275, 1); + x_287 = x_275; +} else { + lean_dec_ref(x_275); + x_287 = lean_box(0); +} +if (lean_is_scalar(x_287)) { + x_288 = lean_alloc_ctor(1, 2, 0); +} else { + x_288 = x_287; +} +lean_ctor_set(x_288, 0, x_285); +lean_ctor_set(x_288, 1, x_286); +return x_288; +} +} +} +} +} +else +{ +uint8_t x_289; +lean_free_object(x_21); +lean_dec(x_25); +lean_dec(x_24); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_289 = !lean_is_exclusive(x_26); +if (x_289 == 0) +{ +return x_26; +} +else +{ +lean_object* x_290; lean_object* x_291; lean_object* x_292; +x_290 = lean_ctor_get(x_26, 0); +x_291 = lean_ctor_get(x_26, 1); +lean_inc(x_291); +lean_inc(x_290); +lean_dec(x_26); +x_292 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_292, 0, x_290); +lean_ctor_set(x_292, 1, x_291); +return x_292; +} +} +} +else +{ +lean_object* x_293; lean_object* x_294; lean_object* x_295; +x_293 = lean_ctor_get(x_21, 0); +x_294 = lean_ctor_get(x_21, 1); +lean_inc(x_294); +lean_inc(x_293); +lean_dec(x_21); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_295 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +if (lean_obj_tag(x_296) == 0) +{ +lean_object* x_297; lean_object* x_298; +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_298 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_297); +if (lean_obj_tag(x_298) == 0) +{ +lean_object* x_299; +x_299 = lean_ctor_get(x_298, 0); +lean_inc(x_299); +if (lean_obj_tag(x_299) == 0) +{ +lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_object* x_303; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_300 = lean_ctor_get(x_298, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_301 = x_298; +} else { + lean_dec_ref(x_298); + x_301 = lean_box(0); +} +x_302 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_301)) { + x_303 = lean_alloc_ctor(0, 2, 0); +} else { + x_303 = x_301; +} +lean_ctor_set(x_303, 0, x_302); +lean_ctor_set(x_303, 1, x_300); +return x_303; +} +else +{ +lean_object* x_304; lean_object* x_305; lean_object* x_306; lean_object* x_307; lean_object* x_308; lean_object* x_309; lean_object* x_310; uint8_t x_311; +x_304 = lean_ctor_get(x_299, 0); +lean_inc(x_304); +if (lean_is_exclusive(x_299)) { + lean_ctor_release(x_299, 0); + x_305 = x_299; +} else { + lean_dec_ref(x_299); + x_305 = lean_box(0); +} +x_306 = lean_ctor_get(x_298, 1); +lean_inc(x_306); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_307 = x_298; +} else { + lean_dec_ref(x_298); + x_307 = lean_box(0); +} +x_308 = lean_ctor_get(x_304, 0); +lean_inc(x_308); +x_309 = lean_ctor_get(x_304, 1); +lean_inc(x_309); +if (lean_is_exclusive(x_304)) { + lean_ctor_release(x_304, 0); + lean_ctor_release(x_304, 1); + x_310 = x_304; +} else { + lean_dec_ref(x_304); + x_310 = lean_box(0); +} +x_311 = lean_nat_dec_eq(x_293, x_308); +lean_dec(x_308); +if (x_311 == 0) +{ +lean_object* x_312; lean_object* x_313; +lean_dec(x_310); +lean_dec(x_309); +lean_dec(x_305); +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_312 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_307)) { + x_313 = lean_alloc_ctor(0, 2, 0); +} else { + x_313 = x_307; +} +lean_ctor_set(x_313, 0, x_312); +lean_ctor_set(x_313, 1, x_306); +return x_313; +} +else +{ +lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; +lean_dec(x_307); +x_314 = l_BitVec_add(x_293, x_294, x_309); +lean_dec(x_309); +lean_dec(x_294); +x_315 = lean_box(0); +x_316 = l_Lean_mkNatLit(x_293); +x_317 = l_Lean_mkNatLit(x_314); +x_318 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_316); +x_319 = l_Lean_mkAppB(x_318, x_316, x_317); +lean_inc(x_2); +if (lean_is_scalar(x_310)) { + x_320 = lean_alloc_ctor(1, 2, 0); +} else { + x_320 = x_310; + lean_ctor_set_tag(x_320, 1); +} +lean_ctor_set(x_320, 0, x_2); +lean_ctor_set(x_320, 1, x_315); +x_321 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_321, 0, x_319); +lean_ctor_set(x_321, 1, x_320); +x_322 = lean_array_mk(x_321); +x_323 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_324 = l_Lean_Meta_mkAppM(x_323, x_322, x_7, x_8, x_9, x_10, x_306); +if (lean_obj_tag(x_324) == 0) +{ +lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; uint8_t x_331; lean_object* x_332; lean_object* x_333; +x_325 = lean_ctor_get(x_324, 0); +lean_inc(x_325); +x_326 = lean_ctor_get(x_324, 1); +lean_inc(x_326); +if (lean_is_exclusive(x_324)) { + lean_ctor_release(x_324, 0); + lean_ctor_release(x_324, 1); + x_327 = x_324; +} else { + lean_dec_ref(x_324); + x_327 = lean_box(0); +} +x_328 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_329 = l_Lean_mkApp4(x_328, x_316, x_2, x_3, x_1); +if (lean_is_scalar(x_305)) { + x_330 = lean_alloc_ctor(1, 1, 0); +} else { + x_330 = x_305; +} +lean_ctor_set(x_330, 0, x_329); +x_331 = 1; +x_332 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_332, 0, x_325); +lean_ctor_set(x_332, 1, x_330); +lean_ctor_set_uint8(x_332, sizeof(void*)*2, x_331); +lean_ctor_set(x_13, 0, x_332); +if (lean_is_scalar(x_327)) { + x_333 = lean_alloc_ctor(0, 2, 0); +} else { + x_333 = x_327; +} +lean_ctor_set(x_333, 0, x_13); +lean_ctor_set(x_333, 1, x_326); +return x_333; +} +else +{ +lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; +lean_dec(x_316); +lean_dec(x_305); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_334 = lean_ctor_get(x_324, 0); +lean_inc(x_334); +x_335 = lean_ctor_get(x_324, 1); +lean_inc(x_335); +if (lean_is_exclusive(x_324)) { + lean_ctor_release(x_324, 0); + lean_ctor_release(x_324, 1); + x_336 = x_324; +} else { + lean_dec_ref(x_324); + x_336 = lean_box(0); +} +if (lean_is_scalar(x_336)) { + x_337 = lean_alloc_ctor(1, 2, 0); +} else { + x_337 = x_336; +} +lean_ctor_set(x_337, 0, x_334); +lean_ctor_set(x_337, 1, x_335); +return x_337; +} +} +} +} +else +{ +lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_338 = lean_ctor_get(x_298, 0); +lean_inc(x_338); +x_339 = lean_ctor_get(x_298, 1); +lean_inc(x_339); +if (lean_is_exclusive(x_298)) { + lean_ctor_release(x_298, 0); + lean_ctor_release(x_298, 1); + x_340 = x_298; +} else { + lean_dec_ref(x_298); + x_340 = lean_box(0); +} +if (lean_is_scalar(x_340)) { + x_341 = lean_alloc_ctor(1, 2, 0); +} else { + x_341 = x_340; +} +lean_ctor_set(x_341, 0, x_338); +lean_ctor_set(x_341, 1, x_339); +return x_341; +} +} +else +{ +lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; lean_object* x_348; uint8_t x_349; +x_342 = lean_ctor_get(x_296, 0); +lean_inc(x_342); +if (lean_is_exclusive(x_296)) { + lean_ctor_release(x_296, 0); + x_343 = x_296; +} else { + lean_dec_ref(x_296); + x_343 = lean_box(0); +} +x_344 = lean_ctor_get(x_295, 1); +lean_inc(x_344); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_345 = x_295; +} else { + lean_dec_ref(x_295); + x_345 = lean_box(0); +} +x_346 = lean_ctor_get(x_342, 0); +lean_inc(x_346); +x_347 = lean_ctor_get(x_342, 1); +lean_inc(x_347); +if (lean_is_exclusive(x_342)) { + lean_ctor_release(x_342, 0); + lean_ctor_release(x_342, 1); + x_348 = x_342; +} else { + lean_dec_ref(x_342); + x_348 = lean_box(0); +} +x_349 = lean_nat_dec_eq(x_293, x_346); +lean_dec(x_346); +if (x_349 == 0) +{ +lean_object* x_350; lean_object* x_351; +lean_dec(x_348); +lean_dec(x_347); +lean_dec(x_343); +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_350 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_345)) { + x_351 = lean_alloc_ctor(0, 2, 0); +} else { + x_351 = x_345; +} +lean_ctor_set(x_351, 0, x_350); +lean_ctor_set(x_351, 1, x_344); +return x_351; +} +else +{ +lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; +lean_dec(x_345); +x_352 = l_BitVec_add(x_293, x_294, x_347); +lean_dec(x_347); +lean_dec(x_294); +x_353 = lean_box(0); +x_354 = l_Lean_mkNatLit(x_293); +x_355 = l_Lean_mkNatLit(x_352); +x_356 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_354); +x_357 = l_Lean_mkAppB(x_356, x_354, x_355); +lean_inc(x_3); +if (lean_is_scalar(x_348)) { + x_358 = lean_alloc_ctor(1, 2, 0); +} else { + x_358 = x_348; + lean_ctor_set_tag(x_358, 1); +} +lean_ctor_set(x_358, 0, x_3); +lean_ctor_set(x_358, 1, x_353); +x_359 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_359, 0, x_357); +lean_ctor_set(x_359, 1, x_358); +x_360 = lean_array_mk(x_359); +x_361 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_362 = l_Lean_Meta_mkAppM(x_361, x_360, x_7, x_8, x_9, x_10, x_344); +if (lean_obj_tag(x_362) == 0) +{ +lean_object* x_363; lean_object* x_364; lean_object* x_365; lean_object* x_366; lean_object* x_367; lean_object* x_368; uint8_t x_369; lean_object* x_370; lean_object* x_371; +x_363 = lean_ctor_get(x_362, 0); +lean_inc(x_363); +x_364 = lean_ctor_get(x_362, 1); +lean_inc(x_364); +if (lean_is_exclusive(x_362)) { + lean_ctor_release(x_362, 0); + lean_ctor_release(x_362, 1); + x_365 = x_362; +} else { + lean_dec_ref(x_362); + x_365 = lean_box(0); +} +x_366 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_367 = l_Lean_mkApp4(x_366, x_354, x_2, x_3, x_1); +if (lean_is_scalar(x_343)) { + x_368 = lean_alloc_ctor(1, 1, 0); +} else { + x_368 = x_343; +} +lean_ctor_set(x_368, 0, x_367); +x_369 = 1; +x_370 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_370, 0, x_363); +lean_ctor_set(x_370, 1, x_368); +lean_ctor_set_uint8(x_370, sizeof(void*)*2, x_369); +lean_ctor_set(x_13, 0, x_370); +if (lean_is_scalar(x_365)) { + x_371 = lean_alloc_ctor(0, 2, 0); +} else { + x_371 = x_365; +} +lean_ctor_set(x_371, 0, x_13); +lean_ctor_set(x_371, 1, x_364); +return x_371; +} +else +{ +lean_object* x_372; lean_object* x_373; lean_object* x_374; lean_object* x_375; +lean_dec(x_354); +lean_dec(x_343); +lean_free_object(x_13); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_372 = lean_ctor_get(x_362, 0); +lean_inc(x_372); +x_373 = lean_ctor_get(x_362, 1); +lean_inc(x_373); +if (lean_is_exclusive(x_362)) { + lean_ctor_release(x_362, 0); + lean_ctor_release(x_362, 1); + x_374 = x_362; +} else { + lean_dec_ref(x_362); + x_374 = lean_box(0); +} +if (lean_is_scalar(x_374)) { + x_375 = lean_alloc_ctor(1, 2, 0); +} else { + x_375 = x_374; +} +lean_ctor_set(x_375, 0, x_372); +lean_ctor_set(x_375, 1, x_373); +return x_375; +} +} +} +} +else +{ +lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; +lean_dec(x_294); +lean_dec(x_293); +lean_free_object(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_376 = lean_ctor_get(x_295, 0); +lean_inc(x_376); +x_377 = lean_ctor_get(x_295, 1); +lean_inc(x_377); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_378 = x_295; +} else { + lean_dec_ref(x_295); + x_378 = lean_box(0); +} +if (lean_is_scalar(x_378)) { + x_379 = lean_alloc_ctor(1, 2, 0); +} else { + x_379 = x_378; +} +lean_ctor_set(x_379, 0, x_376); +lean_ctor_set(x_379, 1, x_377); +return x_379; +} +} +} +else +{ +lean_object* x_380; lean_object* x_381; lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; +x_380 = lean_ctor_get(x_13, 0); +lean_inc(x_380); +lean_dec(x_13); +x_381 = lean_ctor_get(x_12, 1); +lean_inc(x_381); +lean_dec(x_12); +x_382 = lean_ctor_get(x_380, 0); +lean_inc(x_382); +x_383 = lean_ctor_get(x_380, 1); +lean_inc(x_383); +if (lean_is_exclusive(x_380)) { + lean_ctor_release(x_380, 0); + lean_ctor_release(x_380, 1); + x_384 = x_380; +} else { + lean_dec_ref(x_380); + x_384 = lean_box(0); +} +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +x_385 = l_Lean_Meta_getBitVecValue_x3f(x_2, x_7, x_8, x_9, x_10, x_381); +if (lean_obj_tag(x_385) == 0) +{ +lean_object* x_386; +x_386 = lean_ctor_get(x_385, 0); +lean_inc(x_386); +if (lean_obj_tag(x_386) == 0) +{ +lean_object* x_387; lean_object* x_388; +x_387 = lean_ctor_get(x_385, 1); +lean_inc(x_387); +lean_dec(x_385); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_3); +x_388 = l_Lean_Meta_getBitVecValue_x3f(x_3, x_7, x_8, x_9, x_10, x_387); +if (lean_obj_tag(x_388) == 0) +{ +lean_object* x_389; +x_389 = lean_ctor_get(x_388, 0); +lean_inc(x_389); +if (lean_obj_tag(x_389) == 0) +{ +lean_object* x_390; lean_object* x_391; lean_object* x_392; lean_object* x_393; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_390 = lean_ctor_get(x_388, 1); +lean_inc(x_390); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_391 = x_388; +} else { + lean_dec_ref(x_388); + x_391 = lean_box(0); +} +x_392 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_391)) { + x_393 = lean_alloc_ctor(0, 2, 0); +} else { + x_393 = x_391; +} +lean_ctor_set(x_393, 0, x_392); +lean_ctor_set(x_393, 1, x_390); +return x_393; +} +else +{ +lean_object* x_394; lean_object* x_395; lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; uint8_t x_401; +x_394 = lean_ctor_get(x_389, 0); +lean_inc(x_394); +if (lean_is_exclusive(x_389)) { + lean_ctor_release(x_389, 0); + x_395 = x_389; +} else { + lean_dec_ref(x_389); + x_395 = lean_box(0); +} +x_396 = lean_ctor_get(x_388, 1); +lean_inc(x_396); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_397 = x_388; +} else { + lean_dec_ref(x_388); + x_397 = lean_box(0); +} +x_398 = lean_ctor_get(x_394, 0); +lean_inc(x_398); +x_399 = lean_ctor_get(x_394, 1); +lean_inc(x_399); +if (lean_is_exclusive(x_394)) { + lean_ctor_release(x_394, 0); + lean_ctor_release(x_394, 1); + x_400 = x_394; +} else { + lean_dec_ref(x_394); + x_400 = lean_box(0); +} +x_401 = lean_nat_dec_eq(x_382, x_398); +lean_dec(x_398); +if (x_401 == 0) +{ +lean_object* x_402; lean_object* x_403; +lean_dec(x_400); +lean_dec(x_399); +lean_dec(x_395); +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_402 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_397)) { + x_403 = lean_alloc_ctor(0, 2, 0); +} else { + x_403 = x_397; +} +lean_ctor_set(x_403, 0, x_402); +lean_ctor_set(x_403, 1, x_396); +return x_403; +} +else +{ +lean_object* x_404; lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; lean_object* x_410; lean_object* x_411; lean_object* x_412; lean_object* x_413; lean_object* x_414; +lean_dec(x_397); +x_404 = l_BitVec_add(x_382, x_383, x_399); +lean_dec(x_399); +lean_dec(x_383); +x_405 = lean_box(0); +x_406 = l_Lean_mkNatLit(x_382); +x_407 = l_Lean_mkNatLit(x_404); +x_408 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_406); +x_409 = l_Lean_mkAppB(x_408, x_406, x_407); +lean_inc(x_2); +if (lean_is_scalar(x_400)) { + x_410 = lean_alloc_ctor(1, 2, 0); +} else { + x_410 = x_400; + lean_ctor_set_tag(x_410, 1); +} +lean_ctor_set(x_410, 0, x_2); +lean_ctor_set(x_410, 1, x_405); +if (lean_is_scalar(x_384)) { + x_411 = lean_alloc_ctor(1, 2, 0); +} else { + x_411 = x_384; + lean_ctor_set_tag(x_411, 1); +} +lean_ctor_set(x_411, 0, x_409); +lean_ctor_set(x_411, 1, x_410); +x_412 = lean_array_mk(x_411); +x_413 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_414 = l_Lean_Meta_mkAppM(x_413, x_412, x_7, x_8, x_9, x_10, x_396); +if (lean_obj_tag(x_414) == 0) +{ +lean_object* x_415; lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; uint8_t x_421; lean_object* x_422; lean_object* x_423; lean_object* x_424; +x_415 = lean_ctor_get(x_414, 0); +lean_inc(x_415); +x_416 = lean_ctor_get(x_414, 1); +lean_inc(x_416); +if (lean_is_exclusive(x_414)) { + lean_ctor_release(x_414, 0); + lean_ctor_release(x_414, 1); + x_417 = x_414; +} else { + lean_dec_ref(x_414); + x_417 = lean_box(0); +} +x_418 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3; +x_419 = l_Lean_mkApp4(x_418, x_406, x_2, x_3, x_1); +if (lean_is_scalar(x_395)) { + x_420 = lean_alloc_ctor(1, 1, 0); +} else { + x_420 = x_395; +} +lean_ctor_set(x_420, 0, x_419); +x_421 = 1; +x_422 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_422, 0, x_415); +lean_ctor_set(x_422, 1, x_420); +lean_ctor_set_uint8(x_422, sizeof(void*)*2, x_421); +x_423 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_423, 0, x_422); +if (lean_is_scalar(x_417)) { + x_424 = lean_alloc_ctor(0, 2, 0); +} else { + x_424 = x_417; +} +lean_ctor_set(x_424, 0, x_423); +lean_ctor_set(x_424, 1, x_416); +return x_424; +} +else +{ +lean_object* x_425; lean_object* x_426; lean_object* x_427; lean_object* x_428; +lean_dec(x_406); +lean_dec(x_395); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_425 = lean_ctor_get(x_414, 0); +lean_inc(x_425); +x_426 = lean_ctor_get(x_414, 1); +lean_inc(x_426); +if (lean_is_exclusive(x_414)) { + lean_ctor_release(x_414, 0); + lean_ctor_release(x_414, 1); + x_427 = x_414; +} else { + lean_dec_ref(x_414); + x_427 = lean_box(0); +} +if (lean_is_scalar(x_427)) { + x_428 = lean_alloc_ctor(1, 2, 0); +} else { + x_428 = x_427; +} +lean_ctor_set(x_428, 0, x_425); +lean_ctor_set(x_428, 1, x_426); +return x_428; +} +} +} +} +else +{ +lean_object* x_429; lean_object* x_430; lean_object* x_431; lean_object* x_432; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_429 = lean_ctor_get(x_388, 0); +lean_inc(x_429); +x_430 = lean_ctor_get(x_388, 1); +lean_inc(x_430); +if (lean_is_exclusive(x_388)) { + lean_ctor_release(x_388, 0); + lean_ctor_release(x_388, 1); + x_431 = x_388; +} else { + lean_dec_ref(x_388); + x_431 = lean_box(0); +} +if (lean_is_scalar(x_431)) { + x_432 = lean_alloc_ctor(1, 2, 0); +} else { + x_432 = x_431; +} +lean_ctor_set(x_432, 0, x_429); +lean_ctor_set(x_432, 1, x_430); +return x_432; +} +} +else +{ +lean_object* x_433; lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; lean_object* x_438; lean_object* x_439; uint8_t x_440; +x_433 = lean_ctor_get(x_386, 0); +lean_inc(x_433); +if (lean_is_exclusive(x_386)) { + lean_ctor_release(x_386, 0); + x_434 = x_386; +} else { + lean_dec_ref(x_386); + x_434 = lean_box(0); +} +x_435 = lean_ctor_get(x_385, 1); +lean_inc(x_435); +if (lean_is_exclusive(x_385)) { + lean_ctor_release(x_385, 0); + lean_ctor_release(x_385, 1); + x_436 = x_385; +} else { + lean_dec_ref(x_385); + x_436 = lean_box(0); +} +x_437 = lean_ctor_get(x_433, 0); +lean_inc(x_437); +x_438 = lean_ctor_get(x_433, 1); +lean_inc(x_438); +if (lean_is_exclusive(x_433)) { + lean_ctor_release(x_433, 0); + lean_ctor_release(x_433, 1); + x_439 = x_433; +} else { + lean_dec_ref(x_433); + x_439 = lean_box(0); +} +x_440 = lean_nat_dec_eq(x_382, x_437); +lean_dec(x_437); +if (x_440 == 0) +{ +lean_object* x_441; lean_object* x_442; +lean_dec(x_439); +lean_dec(x_438); +lean_dec(x_434); +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_441 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +if (lean_is_scalar(x_436)) { + x_442 = lean_alloc_ctor(0, 2, 0); +} else { + x_442 = x_436; +} +lean_ctor_set(x_442, 0, x_441); +lean_ctor_set(x_442, 1, x_435); +return x_442; +} +else +{ +lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; lean_object* x_447; lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; lean_object* x_452; lean_object* x_453; +lean_dec(x_436); +x_443 = l_BitVec_add(x_382, x_383, x_438); +lean_dec(x_438); +lean_dec(x_383); +x_444 = lean_box(0); +x_445 = l_Lean_mkNatLit(x_382); +x_446 = l_Lean_mkNatLit(x_443); +x_447 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1; +lean_inc(x_445); +x_448 = l_Lean_mkAppB(x_447, x_445, x_446); +lean_inc(x_3); +if (lean_is_scalar(x_439)) { + x_449 = lean_alloc_ctor(1, 2, 0); +} else { + x_449 = x_439; + lean_ctor_set_tag(x_449, 1); +} +lean_ctor_set(x_449, 0, x_3); +lean_ctor_set(x_449, 1, x_444); +if (lean_is_scalar(x_384)) { + x_450 = lean_alloc_ctor(1, 2, 0); +} else { + x_450 = x_384; + lean_ctor_set_tag(x_450, 1); +} +lean_ctor_set(x_450, 0, x_448); +lean_ctor_set(x_450, 1, x_449); +x_451 = lean_array_mk(x_450); +x_452 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_453 = l_Lean_Meta_mkAppM(x_452, x_451, x_7, x_8, x_9, x_10, x_435); +if (lean_obj_tag(x_453) == 0) +{ +lean_object* x_454; lean_object* x_455; lean_object* x_456; lean_object* x_457; lean_object* x_458; lean_object* x_459; uint8_t x_460; lean_object* x_461; lean_object* x_462; lean_object* x_463; +x_454 = lean_ctor_get(x_453, 0); +lean_inc(x_454); +x_455 = lean_ctor_get(x_453, 1); +lean_inc(x_455); +if (lean_is_exclusive(x_453)) { + lean_ctor_release(x_453, 0); + lean_ctor_release(x_453, 1); + x_456 = x_453; +} else { + lean_dec_ref(x_453); + x_456 = lean_box(0); +} +x_457 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6; +x_458 = l_Lean_mkApp4(x_457, x_445, x_2, x_3, x_1); +if (lean_is_scalar(x_434)) { + x_459 = lean_alloc_ctor(1, 1, 0); +} else { + x_459 = x_434; +} +lean_ctor_set(x_459, 0, x_458); +x_460 = 1; +x_461 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_461, 0, x_454); +lean_ctor_set(x_461, 1, x_459); +lean_ctor_set_uint8(x_461, sizeof(void*)*2, x_460); +x_462 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_462, 0, x_461); +if (lean_is_scalar(x_456)) { + x_463 = lean_alloc_ctor(0, 2, 0); +} else { + x_463 = x_456; +} +lean_ctor_set(x_463, 0, x_462); +lean_ctor_set(x_463, 1, x_455); +return x_463; +} +else +{ +lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; +lean_dec(x_445); +lean_dec(x_434); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_464 = lean_ctor_get(x_453, 0); +lean_inc(x_464); +x_465 = lean_ctor_get(x_453, 1); +lean_inc(x_465); +if (lean_is_exclusive(x_453)) { + lean_ctor_release(x_453, 0); + lean_ctor_release(x_453, 1); + x_466 = x_453; +} else { + lean_dec_ref(x_453); + x_466 = lean_box(0); +} +if (lean_is_scalar(x_466)) { + x_467 = lean_alloc_ctor(1, 2, 0); +} else { + x_467 = x_466; +} +lean_ctor_set(x_467, 0, x_464); +lean_ctor_set(x_467, 1, x_465); +return x_467; +} +} +} +} +else +{ +lean_object* x_468; lean_object* x_469; lean_object* x_470; lean_object* x_471; +lean_dec(x_384); +lean_dec(x_383); +lean_dec(x_382); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_468 = lean_ctor_get(x_385, 0); +lean_inc(x_468); +x_469 = lean_ctor_get(x_385, 1); +lean_inc(x_469); +if (lean_is_exclusive(x_385)) { + lean_ctor_release(x_385, 0); + lean_ctor_release(x_385, 1); + x_470 = x_385; +} else { + lean_dec_ref(x_385); + x_470 = lean_box(0); +} +if (lean_is_scalar(x_470)) { + x_471 = lean_alloc_ctor(1, 2, 0); +} else { + x_471 = x_470; +} +lean_ctor_set(x_471, 0, x_468); +lean_ctor_set(x_471, 1, x_469); +return x_471; +} +} +} +} +else +{ +uint8_t x_472; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_472 = !lean_is_exclusive(x_12); +if (x_472 == 0) +{ +return x_12; +} +else +{ +lean_object* x_473; lean_object* x_474; lean_object* x_475; +x_473 = lean_ctor_get(x_12, 0); +x_474 = lean_ctor_get(x_12, 1); +lean_inc(x_474); +lean_inc(x_473); +lean_dec(x_12); +x_475 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_475, 0, x_473); +lean_ctor_set(x_475, 1, x_474); +return x_475; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_2); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_2); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_2); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_2); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_2); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +lean_dec(x_2); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(x_2, x_21, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_43; +} +} +} +} +} +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__2), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; uint8_t x_27; +x_26 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_27 = l_Lean_Expr_isApp(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_28 = lean_box(0); +x_29 = lean_apply_9(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_29; +} +else +{ +lean_object* x_30; uint8_t x_31; +x_30 = l_Lean_Expr_appFnCleanup(x_26, lean_box(0)); +x_31 = l_Lean_Expr_isApp(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_30); +lean_dec(x_21); +lean_dec(x_16); +x_32 = lean_box(0); +x_33 = lean_apply_9(x_11, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_33; +} +else +{ +lean_object* x_34; uint8_t x_35; +x_34 = l_Lean_Expr_appFnCleanup(x_30, lean_box(0)); +x_35 = l_Lean_Expr_isApp(x_34); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +lean_dec(x_34); +lean_dec(x_21); +lean_dec(x_16); +x_36 = lean_box(0); +x_37 = lean_apply_9(x_11, x_36, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_37; +} +else +{ +lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_38 = l_Lean_Expr_appFnCleanup(x_34, lean_box(0)); +x_39 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_21); +lean_dec(x_16); +x_41 = lean_box(0); +x_42 = lean_apply_9(x_11, x_41, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = lean_apply_10(x_10, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_43; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_12; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bv_add_const'", 13, 13); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; uint8_t x_4; +x_2 = lean_unsigned_to_nat(0u); +x_3 = lean_nat_dec_eq(x_1, x_2); +x_4 = l_instDecidableNot___rarg(x_3); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_box(0); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_nat_log2(x_1); +x_7 = lean_unsigned_to_nat(2u); +x_8 = lean_nat_pow(x_7, x_6); +x_9 = lean_nat_dec_eq(x_8, x_1); +lean_dec(x_8); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_6); +x_10 = lean_box(0); +return x_10; +} +else +{ +lean_object* x_11; +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_6); +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HPow", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hPow", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_2); +lean_ctor_set(x_9, 1, x_8); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_array_mk(x_10); +x_12 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3; +x_13 = l_Lean_Meta_mkAppM(x_12, x_11, x_3, x_4, x_5, x_6, x_7); +return x_13; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HShiftRight", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hShiftRight", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(2u); +x_2 = l_Lean_mkNatLit(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("udiv_ofNat_eq_of_lt", 19, 19); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_5 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1; +x_6 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5; +x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); +return x_7; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_14 = l_Lean_mkNatLit(x_1); +x_15 = lean_box(0); +lean_inc(x_14); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +lean_inc(x_2); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_2); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_array_mk(x_17); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_20 = l_Lean_Meta_mkAppM(x_19, x_18, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_14); +x_24 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow(x_23, x_14, x_9, x_10, x_11, x_12, x_22); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_mkNatLit(x_3); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_27); +x_28 = l_Lean_Meta_mkEq(x_25, x_27, x_9, x_10, x_11, x_12, x_26); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_31 = l_Lean_Meta_mkDecideProof(x_29, x_9, x_10, x_11, x_12, x_30); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_mkNatLit(x_4); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_34); +lean_inc(x_14); +x_35 = l_Lean_Meta_mkLt(x_14, x_34, x_9, x_10, x_11, x_12, x_33); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = l_Lean_Meta_mkDecideProof(x_36, x_9, x_10, x_11, x_12, x_37); +if (lean_obj_tag(x_38) == 0) +{ +uint8_t x_39; +x_39 = !lean_is_exclusive(x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; +x_40 = lean_ctor_get(x_38, 0); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_15); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_32); +lean_ctor_set(x_42, 1, x_41); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_14); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_27); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_2); +lean_ctor_set(x_45, 1, x_44); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_34); +lean_ctor_set(x_46, 1, x_45); +x_47 = lean_array_mk(x_46); +x_48 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; +x_49 = l_Lean_mkAppN(x_48, x_47); +lean_dec(x_47); +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_51 = 1; +x_52 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_52, 0, x_21); +lean_ctor_set(x_52, 1, x_50); +lean_ctor_set_uint8(x_52, sizeof(void*)*2, x_51); +x_53 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_38, 0, x_53); +return x_38; +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_54 = lean_ctor_get(x_38, 0); +x_55 = lean_ctor_get(x_38, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_38); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_15); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_32); +lean_ctor_set(x_57, 1, x_56); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_14); +lean_ctor_set(x_58, 1, x_57); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_27); +lean_ctor_set(x_59, 1, x_58); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_2); +lean_ctor_set(x_60, 1, x_59); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_34); +lean_ctor_set(x_61, 1, x_60); +x_62 = lean_array_mk(x_61); +x_63 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7; +x_64 = l_Lean_mkAppN(x_63, x_62); +lean_dec(x_62); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = 1; +x_67 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_67, 0, x_21); +lean_ctor_set(x_67, 1, x_65); +lean_ctor_set_uint8(x_67, sizeof(void*)*2, x_66); +x_68 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_68, 0, x_67); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_55); +return x_69; +} +} +else +{ +uint8_t x_70; +lean_dec(x_34); +lean_dec(x_32); +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_14); +lean_dec(x_2); +x_70 = !lean_is_exclusive(x_38); +if (x_70 == 0) +{ +return x_38; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_38, 0); +x_72 = lean_ctor_get(x_38, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_38); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; +} +} +} +else +{ +uint8_t x_74; +lean_dec(x_34); +lean_dec(x_32); +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +x_74 = !lean_is_exclusive(x_35); +if (x_74 == 0) +{ +return x_35; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_35, 0); +x_76 = lean_ctor_get(x_35, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_35); +x_77 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +return x_77; +} +} +} +else +{ +uint8_t x_78; +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_2); +x_78 = !lean_is_exclusive(x_31); +if (x_78 == 0) +{ +return x_31; +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_31, 0); +x_80 = lean_ctor_get(x_31, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_31); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; +} +} +} +else +{ +uint8_t x_82; +lean_dec(x_27); +lean_dec(x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_2); +x_82 = !lean_is_exclusive(x_28); +if (x_82 == 0) +{ +return x_28; +} +else +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_28, 0); +x_84 = lean_ctor_get(x_28, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_28); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +return x_85; +} +} +} +else +{ +uint8_t x_86; +lean_dec(x_21); +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_86 = !lean_is_exclusive(x_24); +if (x_86 == 0) +{ +return x_24; +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_24, 0); +x_88 = lean_ctor_get(x_24, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_24); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +return x_89; +} +} +} +else +{ +uint8_t x_90; +lean_dec(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_90 = !lean_is_exclusive(x_20); +if (x_90 == 0) +{ +return x_20; +} +else +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_20, 0); +x_92 = lean_ctor_get(x_20, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_20); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_15 = l_Lean_Meta_getBitVecValue_x3f(x_6, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_17 = !lean_is_exclusive(x_15); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_15, 0); +lean_dec(x_18); +x_19 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_15, 0, x_19); +return x_15; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_dec(x_15); +x_21 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +} +else +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_16, 0); +lean_inc(x_23); +lean_dec(x_16); +x_24 = !lean_is_exclusive(x_15); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_15, 1); +x_26 = lean_ctor_get(x_15, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_23, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_dec(x_23); +x_29 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_28); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_30 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_15, 0, x_30); +return x_15; +} +else +{ +lean_object* x_31; uint8_t x_32; +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_nat_dec_le(x_27, x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +lean_free_object(x_15); +x_33 = lean_box(0); +x_34 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_31, x_5, x_28, x_27, x_33, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +return x_34; +} +else +{ +lean_object* x_35; +lean_dec(x_31); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_35 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +lean_ctor_set(x_15, 0, x_35); +return x_15; +} +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_15, 1); +lean_inc(x_36); +lean_dec(x_15); +x_37 = lean_ctor_get(x_23, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_23, 1); +lean_inc(x_38); +lean_dec(x_23); +x_39 = l___private_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc_0__Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Nat_log2Exact(x_38); +if (lean_obj_tag(x_39) == 0) +{ +lean_object* x_40; lean_object* x_41; +lean_dec(x_38); +lean_dec(x_37); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_40 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_36); +return x_41; +} +else +{ +lean_object* x_42; uint8_t x_43; +x_42 = lean_ctor_get(x_39, 0); +lean_inc(x_42); +lean_dec(x_39); +x_43 = lean_nat_dec_le(x_37, x_42); +if (x_43 == 0) +{ +lean_object* x_44; lean_object* x_45; +x_44 = lean_box(0); +x_45 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_42, x_5, x_38, x_37, x_44, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_36); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; +lean_dec(x_42); +lean_dec(x_38); +lean_dec(x_37); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_46 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6; +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_36); +return x_47; +} +} +} +} +} +else +{ +uint8_t x_48; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_5); +x_48 = !lean_is_exclusive(x_15); +if (x_48 == 0) +{ +return x_15; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_15, 0); +x_50 = lean_ctor_get(x_15, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_15); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed), 14, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HDiv", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hDiv", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2; +x_2 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1; +x_11 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2; +x_12 = l_Lean_Expr_cleanupAnnotations(x_1); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +x_14 = lean_box(0); +x_15 = lean_apply_9(x_11, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_16 = l_Lean_Expr_appArg(x_12, lean_box(0)); +x_17 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_17); +lean_dec(x_16); +x_19 = lean_box(0); +x_20 = lean_apply_9(x_11, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_16); +x_24 = lean_box(0); +x_25 = lean_apply_9(x_11, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = l_Lean_Expr_appArg(x_22, lean_box(0)); +x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_28 = l_Lean_Expr_isApp(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_29 = lean_box(0); +x_30 = lean_apply_9(x_11, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); +x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); +x_33 = l_Lean_Expr_isApp(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_34 = lean_box(0); +x_35 = lean_apply_9(x_11, x_34, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_36 = l_Lean_Expr_appArg(x_32, lean_box(0)); +x_37 = l_Lean_Expr_appFnCleanup(x_32, lean_box(0)); +x_38 = l_Lean_Expr_isApp(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +lean_dec(x_37); +lean_dec(x_36); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_39 = lean_box(0); +x_40 = lean_apply_9(x_11, x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_40; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_41 = l_Lean_Expr_appArg(x_37, lean_box(0)); +x_42 = l_Lean_Expr_appFnCleanup(x_37, lean_box(0)); +x_43 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; +x_44 = l_Lean_Expr_isConstOf(x_42, x_43); +lean_dec(x_42); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +lean_dec(x_41); +lean_dec(x_36); +lean_dec(x_31); +lean_dec(x_26); +lean_dec(x_21); +lean_dec(x_16); +x_45 = lean_box(0); +x_46 = lean_apply_9(x_11, x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_46; +} +else +{ +lean_object* x_47; +x_47 = lean_apply_14(x_10, x_41, x_36, x_31, x_26, x_21, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_47; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("bv_udiv_of_two_pow", 18, 18); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5; +x_6 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6; +x_7 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1; +x_8 = l_Lean_Name_mkStr7(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +return x_8; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4; +x_2 = lean_unsigned_to_nat(6u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11; +x_2 = lean_unsigned_to_nat(2u); +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(3); +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13; +x_3 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14; +x_2 = lean_array_mk(x_1); +return x_2; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow), 9, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15; +x_4 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16; +x_5 = l_Lean_Meta_Simp_registerBuiltinSimproc(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510_(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; lean_object* x_6; +x_2 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2; +x_3 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2; +x_4 = 1; +x_5 = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1; +x_6 = l_Lean_Meta_Simp_addSimprocBuiltinAttrCore(x_2, x_3, x_4, x_5, x_1); +return x_6; +} +} +lean_object* initialize_Std_Tactic_BVDecide_Normalize(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Tactic_BVDecide_Syntax(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_Simp(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Tactic_BVDecide_Normalize(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Tactic_BVDecide_Syntax(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_Simp(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Elab_Tactic_BVDecide_Frontend_Attr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___lambda__1___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond___closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__8); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__9); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__10); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__11); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__12); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__13); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__14); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__15); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349____closed__16); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_349_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351____closed__2); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_reduceCond_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_351_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__13); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__14); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___lambda__1___closed__15); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq___closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655____closed__8); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_655_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_eqToBEq_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_657_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes___closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__8); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__9); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__10); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__11); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021____closed__12); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1021_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_andOnes_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1023_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd___closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387____closed__3); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1387_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_onesAnd_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1389_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt___closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660____closed__6); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1660_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_maxUlt_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_1662_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__8); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__9); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__10); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__11); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___lambda__1___closed__12); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add___closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083____closed__6); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2083_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_neg__eq__not__add_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2085_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const___closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__8); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__9); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__10); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__11); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__12); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952____closed__13); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2952_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_2954_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27___closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__8); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__9); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__10); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__11); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__12); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__13); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__14); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821____closed__15); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3821_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__add__const_x27_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_3823_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_mkPow___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__4); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__5); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__6); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___lambda__1___closed__7); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__1); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__2); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__3); +l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4 = _init_l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4(); +lean_mark_persistent(l_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow___closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__1); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__2); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__3); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__4); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__5); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__6); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__7); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__8); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__9); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__10); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__11); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__12); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__13); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__14); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__15); +l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508____closed__16); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4508_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1 = _init_l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_bv__udiv__of__two__pow_declare__1____x40_Lean_Elab_Tactic_BVDecide_Frontend_Normalize_Simproc___hyg_4510_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Elab/Tactic/Grind.c b/stage0/stdlib/Lean/Elab/Tactic/Grind.c index f011d032d6b8..bae559343107 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Grind.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Grind.c @@ -15,6 +15,7 @@ extern "C" { #endif lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_KeyedDeclsAttribute_addBuiltin___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_goalsToMessageData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Elab_Tactic_Grind_0__Lean_Elab_Tactic_elabFallback___elambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Grind_0__Lean_Elab_Tactic_elabFallback___closed__4; @@ -104,7 +105,6 @@ static lean_object* l_Lean_Elab_Tactic_elabGrindConfig___lambda__1___closed__3; lean_object* l_Lean_getConstInfo___at_Lean_Elab_Term_mkConst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_eval_const(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Elab_Tactic_Grind_0__Lean_Elab_Tactic_elabFallback___closed__5; -lean_object* l_Lean_Elab_goalsToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabGrindPattern___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at_Lean_Elab_Tactic_elabGrindPattern___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -720,20 +720,21 @@ return x_18; static lean_object* _init_l_Lean_Elab_Tactic_elabGrindConfig___lambda__3___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; uint8_t x_3; lean_object* x_4; -x_1 = lean_unsigned_to_nat(5u); -x_2 = lean_unsigned_to_nat(1000u); -x_3 = 1; -x_4 = lean_alloc_ctor(0, 4, 4); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_1); -lean_ctor_set(x_4, 2, x_1); -lean_ctor_set(x_4, 3, x_2); -lean_ctor_set_uint8(x_4, sizeof(void*)*4, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*4 + 1, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*4 + 2, x_3); -lean_ctor_set_uint8(x_4, sizeof(void*)*4 + 3, x_3); -return x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; +x_1 = lean_unsigned_to_nat(8u); +x_2 = lean_unsigned_to_nat(5u); +x_3 = lean_unsigned_to_nat(1000u); +x_4 = 1; +x_5 = lean_alloc_ctor(0, 4, 4); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_2); +lean_ctor_set(x_5, 3, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*4, x_4); +lean_ctor_set_uint8(x_5, sizeof(void*)*4 + 1, x_4); +lean_ctor_set_uint8(x_5, sizeof(void*)*4 + 2, x_4); +lean_ctor_set_uint8(x_5, sizeof(void*)*4 + 3, x_4); +return x_5; } } LEAN_EXPORT lean_object* l_Lean_Elab_Tactic_elabGrindConfig___lambda__3(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -2630,105 +2631,185 @@ x_13 = lean_ctor_get(x_10, 1); x_14 = l_List_isEmpty___rarg(x_12); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +lean_object* x_15; lean_free_object(x_10); -x_15 = l_Lean_Elab_goalsToMessageData(x_12); -x_16 = l_Lean_Elab_Tactic_grind___closed__2; -x_17 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = l_Lean_Elab_Tactic_elabGrindConfig___lambda__1___closed__6; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_15 = l_Lean_Meta_Grind_goalsToMessageData(x_12, x_5, x_6, x_7, x_8, x_13); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Elab_Tactic_grind___closed__2; x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_19, x_5, x_6, x_7, x_8, x_13); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_16); +x_20 = l_Lean_Elab_Tactic_elabGrindConfig___lambda__1___closed__6; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_21, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_22; +} +else +{ +uint8_t x_23; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -return x_20; +x_23 = !lean_is_exclusive(x_15); +if (x_23 == 0) +{ +return x_15; } else { -lean_object* x_21; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_15, 0); +x_25 = lean_ctor_get(x_15, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_15); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +else +{ +lean_object* x_27; lean_dec(x_12); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_21 = lean_box(0); -lean_ctor_set(x_10, 0, x_21); +x_27 = lean_box(0); +lean_ctor_set(x_10, 0, x_27); return x_10; } } else { -lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_10, 0); -x_23 = lean_ctor_get(x_10, 1); -lean_inc(x_23); -lean_inc(x_22); +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_ctor_get(x_10, 0); +x_29 = lean_ctor_get(x_10, 1); +lean_inc(x_29); +lean_inc(x_28); lean_dec(x_10); -x_24 = l_List_isEmpty___rarg(x_22); -if (x_24 == 0) +x_30 = l_List_isEmpty___rarg(x_28); +if (x_30 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_25 = l_Lean_Elab_goalsToMessageData(x_22); -x_26 = l_Lean_Elab_Tactic_grind___closed__2; -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_25); -x_28 = l_Lean_Elab_Tactic_elabGrindConfig___lambda__1___closed__6; -x_29 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -x_30 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_29, x_5, x_6, x_7, x_8, x_23); +lean_object* x_31; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_31 = l_Lean_Meta_Grind_goalsToMessageData(x_28, x_5, x_6, x_7, x_8, x_29); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_Elab_Tactic_grind___closed__2; +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_32); +x_36 = l_Lean_Elab_Tactic_elabGrindConfig___lambda__1___closed__6; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +x_38 = l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(x_37, x_5, x_6, x_7, x_8, x_33); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -return x_30; +return x_38; } else { -lean_object* x_31; lean_object* x_32; -lean_dec(x_22); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_31 = lean_box(0); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_23); -return x_32; +x_39 = lean_ctor_get(x_31, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_31, 1); +lean_inc(x_40); +if (lean_is_exclusive(x_31)) { + lean_ctor_release(x_31, 0); + lean_ctor_release(x_31, 1); + x_41 = x_31; +} else { + lean_dec_ref(x_31); + x_41 = lean_box(0); +} +if (lean_is_scalar(x_41)) { + x_42 = lean_alloc_ctor(1, 2, 0); +} else { + x_42 = x_41; +} +lean_ctor_set(x_42, 0, x_39); +lean_ctor_set(x_42, 1, x_40); +return x_42; +} +} +else +{ +lean_object* x_43; lean_object* x_44; +lean_dec(x_28); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_43 = lean_box(0); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_29); +return x_44; } } } else { -uint8_t x_33; +uint8_t x_45; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_33 = !lean_is_exclusive(x_10); -if (x_33 == 0) +x_45 = !lean_is_exclusive(x_10); +if (x_45 == 0) { return x_10; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_10, 0); -x_35 = lean_ctor_get(x_10, 1); -lean_inc(x_35); -lean_inc(x_34); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_10, 0); +x_47 = lean_ctor_get(x_10, 1); +lean_inc(x_47); +lean_inc(x_46); lean_dec(x_10); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } } diff --git a/stage0/stdlib/Lean/Elab/Tactic/Simproc.c b/stage0/stdlib/Lean/Elab/Tactic/Simproc.c index 394414eba494..38cb528b259b 100644 --- a/stage0/stdlib/Lean/Elab/Tactic/Simproc.c +++ b/stage0/stdlib/Lean/Elab/Tactic/Simproc.c @@ -2559,8 +2559,6 @@ x_39 = l_Lean_Elab_Command_elabSimprocPatternBuiltin___lambda__1___closed__20; x_40 = l_Lean_mkAppN(x_39, x_32); lean_dec(x_32); x_41 = l_Lean_declareBuiltin(x_37, x_40, x_7, x_8, x_38); -lean_dec(x_8); -lean_dec(x_7); return x_41; } else @@ -2575,8 +2573,6 @@ x_44 = l_Lean_Elab_Command_elabSimprocPatternBuiltin___lambda__1___closed__23; x_45 = l_Lean_mkAppN(x_44, x_32); lean_dec(x_32); x_46 = l_Lean_declareBuiltin(x_42, x_45, x_7, x_8, x_43); -lean_dec(x_8); -lean_dec(x_7); return x_46; } } diff --git a/stage0/stdlib/Lean/Elab/Term.c b/stage0/stdlib/Lean/Elab/Term.c index 88384ad81972..fed62ca2f949 100644 --- a/stage0/stdlib/Lean/Elab/Term.c +++ b/stage0/stdlib/Lean/Elab/Term.c @@ -80850,6 +80850,7 @@ lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_dec(x_1); x_11 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20682____lambda__2___closed__2; x_12 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_11, x_4, x_5, x_8); +lean_dec(x_5); lean_dec(x_4); x_13 = !lean_is_exclusive(x_12); if (x_13 == 0) @@ -80875,13 +80876,13 @@ else lean_object* x_17; lean_object* x_18; x_17 = lean_box(0); x_18 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20682____lambda__1(x_1, x_17, x_4, x_5, x_8); -lean_dec(x_4); return x_18; } } else { uint8_t x_19; +lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); x_19 = !lean_is_exclusive(x_7); @@ -81056,8 +81057,6 @@ LEAN_EXPORT lean_object* l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20682___ { lean_object* x_6; x_6 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20682____lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); return x_6; } @@ -81069,7 +81068,6 @@ uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); x_8 = l_Lean_Elab_initFn____x40_Lean_Elab_Term___hyg_20682____lambda__2(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); return x_8; } } diff --git a/stage0/stdlib/Lean/Elab/Util.c b/stage0/stdlib/Lean/Elab/Util.c index 578ac6183f15..1991ec7f5251 100644 --- a/stage0/stdlib/Lean/Elab/Util.c +++ b/stage0/stdlib/Lean/Elab/Util.c @@ -2341,6 +2341,8 @@ LEAN_EXPORT lean_object* l_Lean_Elab_mkElabAttribute___rarg___lambda__3(uint8_t if (x_1 == 0) { lean_object* x_6; lean_object* x_7; +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); x_6 = lean_box(0); x_7 = lean_alloc_ctor(0, 2, 0); @@ -2429,8 +2431,6 @@ uint8_t x_6; lean_object* x_7; x_6 = lean_unbox(x_1); lean_dec(x_1); x_7 = l_Lean_Elab_mkElabAttribute___rarg___lambda__3(x_6, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); return x_7; } } diff --git a/stage0/stdlib/Lean/KeyedDeclsAttribute.c b/stage0/stdlib/Lean/KeyedDeclsAttribute.c index 3cdc21842dd9..b22d88e657c4 100644 --- a/stage0/stdlib/Lean/KeyedDeclsAttribute.c +++ b/stage0/stdlib/Lean/KeyedDeclsAttribute.c @@ -5783,6 +5783,8 @@ x_43 = lean_array_mk(x_42); x_44 = l_Lean_KeyedDeclsAttribute_init___rarg___lambda__9___closed__10; x_45 = l_Lean_mkAppN(x_44, x_43); lean_dec(x_43); +lean_inc(x_9); +lean_inc(x_8); lean_inc(x_3); x_46 = l_Lean_declareBuiltin(x_3, x_45, x_8, x_9, x_18); if (lean_obj_tag(x_46) == 0) diff --git a/stage0/stdlib/Lean/Linter/MissingDocs.c b/stage0/stdlib/Lean/Linter/MissingDocs.c index b5c70fba95ba..0cba05c5e536 100644 --- a/stage0/stdlib/Lean/Linter/MissingDocs.c +++ b/stage0/stdlib/Lean/Linter/MissingDocs.c @@ -2982,8 +2982,6 @@ else lean_object* x_44; lean_object* x_45; x_44 = lean_box(0); x_45 = l_Lean_Linter_MissingDocs_initFn____x40_Lean_Linter_MissingDocs___hyg_802____lambda__1(x_8, x_15, x_1, x_44, x_4, x_5, x_16); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_8); return x_45; } @@ -2994,8 +2992,6 @@ lean_object* x_46; lean_object* x_47; lean_dec(x_29); x_46 = lean_box(0); x_47 = l_Lean_Linter_MissingDocs_initFn____x40_Lean_Linter_MissingDocs___hyg_802____lambda__1(x_8, x_15, x_1, x_46, x_4, x_5, x_16); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_8); return x_47; } @@ -4091,8 +4087,6 @@ LEAN_EXPORT lean_object* l_Lean_Linter_MissingDocs_initFn____x40_Lean_Linter_Mis { lean_object* x_8; x_8 = l_Lean_Linter_MissingDocs_initFn____x40_Lean_Linter_MissingDocs___hyg_802____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); return x_8; diff --git a/stage0/stdlib/Lean/Linter/UnusedVariables.c b/stage0/stdlib/Lean/Linter/UnusedVariables.c index 8862d98debe7..a4731d61bdcc 100644 --- a/stage0/stdlib/Lean/Linter/UnusedVariables.c +++ b/stage0/stdlib/Lean/Linter/UnusedVariables.c @@ -2324,6 +2324,8 @@ x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_17, x_4, x_5, x_9); +lean_dec(x_5); +lean_dec(x_4); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) { @@ -2355,6 +2357,8 @@ return x_24; else { uint8_t x_25; +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); x_25 = !lean_is_exclusive(x_7); @@ -2423,6 +2427,7 @@ x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); x_17 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_16, x_5, x_6, x_9); +lean_dec(x_6); lean_dec(x_5); x_18 = !lean_is_exclusive(x_17); if (x_18 == 0) @@ -2448,13 +2453,13 @@ else lean_object* x_22; lean_object* x_23; x_22 = lean_box(0); x_23 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(x_2, x_1, x_22, x_5, x_6, x_9); -lean_dec(x_5); return x_23; } } else { uint8_t x_24; +lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); @@ -3227,8 +3232,6 @@ LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables { lean_object* x_6; x_6 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); return x_6; } @@ -3238,8 +3241,6 @@ LEAN_EXPORT lean_object* l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables { lean_object* x_7; x_7 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); return x_7; } @@ -3251,7 +3252,6 @@ uint8_t x_8; lean_object* x_9; x_8 = lean_unbox(x_4); lean_dec(x_4); x_9 = l_Lean_Linter_initFn____x40_Lean_Linter_UnusedVariables___hyg_640____lambda__3(x_1, x_2, x_3, x_8, x_5, x_6, x_7); -lean_dec(x_6); return x_9; } } diff --git a/stage0/stdlib/Lean/Meta/AppBuilder.c b/stage0/stdlib/Lean/Meta/AppBuilder.c index dbc16ff6c192..4798f8711371 100644 --- a/stage0/stdlib/Lean/Meta/AppBuilder.c +++ b/stage0/stdlib/Lean/Meta/AppBuilder.c @@ -25,6 +25,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkLetBodyCongr(lean_object*, lean_object*, static lean_object* l_Lean_Meta_mkCongrArg___closed__1; static lean_object* l_Lean_Meta_mkForallCongr___closed__2; lean_object* l_Lean_getProjFnForField_x3f(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_mkOfEqTrueCore___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_mkEqOfHEq___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkDefault___closed__2; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___closed__2; @@ -46,7 +47,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkPure(lean_object*, lean_object*, lean_obj static lean_object* l_Lean_Meta_mkEqNDRec___closed__5; static lean_object* l_Lean_Meta_mkPropExt___closed__2; static lean_object* l_Lean_Meta_mkNumeral___closed__4; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3; lean_object* l_Lean_Meta_mkFreshLevelMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSome___closed__1; @@ -55,7 +55,9 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue(lean_object*, lean_object*, lean_o static lean_object* l_Lean_Meta_mkImpDepCongrCtx___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_mkNoConfusion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqSymm___closed__5; +static lean_object* l_Lean_Meta_mkOfEqTrueCore___closed__2; static lean_object* l_Lean_Meta_mkEqTrans___closed__2; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs___closed__1; static lean_object* l_Lean_Meta_mkEqSymm___closed__3; lean_object* lean_whnf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -66,7 +68,7 @@ lean_object* l_Lean_Core_instantiateTypeLevelParams(lean_object*, lean_object*, static lean_object* l_Lean_Meta_congrArg_x3f___lambda__4___closed__5; lean_object* l_Lean_ConstantInfo_levelParams(lean_object*); lean_object* l_Lean_indentD(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13; +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrueCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkEqSymm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkBinaryOp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -78,7 +80,6 @@ static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilder static lean_object* l_Lean_Meta_mkMul___closed__3; static lean_object* l_Lean_Meta_mkAdd___closed__4; lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9; LEAN_EXPORT lean_object* l_Lean_Meta_mkCongrFun___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_congrArg_x3f___lambda__4___closed__7; @@ -88,14 +89,14 @@ uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLetFun___closed__1; static lean_object* l_Lean_Meta_mkOfEqTrue___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException(lean_object*); +uint8_t l_Lean_Expr_isApp(lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7; static lean_object* l_Lean_Meta_mkEqRec___closed__2; static lean_object* l_Lean_Meta_mkEqNDRec___closed__4; lean_object* l_Lean_Expr_sort___override(lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10; lean_object* l_Lean_Meta_trySynthInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); +static lean_object* l_Lean_Meta_mkEqTrueCore___closed__1; static lean_object* l_Lean_Meta_mkDecideProof___closed__1; static lean_object* l_Lean_Meta_mkEqNDRec___closed__1; lean_object* lean_array_push(lean_object*, lean_object*); @@ -110,7 +111,6 @@ extern uint8_t l_instInhabitedBool; static lean_object* l_Lean_Meta_mkNumeral___closed__3; static lean_object* l_Lean_Meta_mkIffOfEq___closed__1; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__1___closed__8; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12; static lean_object* l_Lean_Meta_mkEqMPR___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkCongr___closed__2; @@ -118,6 +118,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_infer(lea LEAN_EXPORT lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__3___closed__6; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4; static lean_object* l_Lean_Meta_mkNoConfusion___closed__5; static lean_object* l_Lean_Meta_mkForallCongr___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_mkHEqOfEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -128,16 +129,17 @@ static lean_object* l_Lean_Meta_mkImpCongr___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppOptM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_environment_find(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppOptMAux___closed__4; +static lean_object* l_Lean_Meta_mkOfEqTrueCore___closed__4; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_hasAssignableMVar___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkSome(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkListLit___closed__4; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__1___closed__4; static lean_object* l_Lean_Meta_mkProjection___lambda__2___closed__10; -static lean_object* l_Lean_Meta_mkOfEqTrue___closed__2; uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkEqMPR(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_congrArg_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppOptMAux___closed__9; static lean_object* l_Lean_Meta_mkEqMP___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_mkProjection___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -164,7 +166,6 @@ static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilder static lean_object* l_Lean_Meta_mkImpCongr___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_mkAdd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkCongrArg___closed__2; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5; lean_object* l_Lean_getStructureFields(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkNoConfusion___closed__7; uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -181,9 +182,11 @@ static lean_object* l_Lean_Meta_mkId___closed__2; lean_object* l_Lean_MVarId_assign___at_Lean_Meta_getLevel___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkNoConfusion___closed__6; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppM_x27___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkCongrArg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLe___closed__2; lean_object* lean_expr_instantiate_rev_range(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkEqMP(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -199,7 +202,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_congrArg_x3f___lambda__3(lean_object*, lean static lean_object* l_Lean_Meta_mkFunExt___closed__1; static lean_object* l_Lean_Meta_mkEqFalse_x27___closed__1; static lean_object* l_Lean_Meta_mkProjection___lambda__2___closed__1; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11; static lean_object* l_Lean_Meta_mkDecide___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppM_x27___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkHEqTrans___closed__1; @@ -222,7 +224,6 @@ LEAN_EXPORT lean_object* l_List_anyM___at___private_Lean_Meta_AppBuilder_0__Lean LEAN_EXPORT lean_object* l_Lean_Meta_mkEqNDRec(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkHEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_SavedState_restore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1; static lean_object* l_Lean_Meta_mkLetBodyCongr___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppM___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); @@ -239,6 +240,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkLetCongr(lean_object*, lean_object*, lean static lean_object* l_Lean_Meta_mkMul___closed__1; static lean_object* l_Lean_Meta_mkHEqSymm___closed__3; lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLetBodyCongr___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_mkPropExt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkNumeral___closed__2; @@ -249,6 +251,7 @@ static lean_object* l_Lean_Meta_mkHEqOfEq___closed__2; extern lean_object* l_Lean_checkEmoji; lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrans(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_mkAppM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAppM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -262,6 +265,7 @@ static lean_object* l_Lean_Meta_mkNoConfusion___closed__8; lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkIffOfEq___closed__3; +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); static lean_object* l_Lean_isLevelMVarAssignable___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__4___closed__3; uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); @@ -287,9 +291,10 @@ static lean_object* l_Lean_Meta_mkProjection___lambda__2___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_mkForallCongr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__9; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_mkOfEqTrueCore___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897_(lean_object*); static lean_object* l_Lean_Meta_congrArg_x3f___lambda__4___closed__6; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException___rarg___closed__1; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_mkEqOfHEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLt___closed__2; static lean_object* l_Lean_Meta_mkHEqSymm___closed__1; @@ -311,25 +316,29 @@ lean_object* l_Lean_Expr_appFn_x21(lean_object*); extern lean_object* l_Lean_Meta_instMonadMetaM; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkSub___closed__4; -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417_(lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8; static lean_object* l_Lean_Meta_mkAdd___closed__2; static lean_object* l_Lean_Meta_mkNoConfusion___closed__1; static lean_object* l_Lean_Meta_mkPure___closed__1; static lean_object* l_Lean_isLevelMVarAssignable___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__4___closed__4; lean_object* l_Lean_MessageData_arrayExpr_toMessageData(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppM_x27___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_mkFalseElim(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkProjection___closed__1; lean_object* l_Lean_Meta_withNewMCtxDepth___at_Lean_Meta_matchesInstance___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkDefault(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqNDRec___closed__2; lean_object* l_Array_append___rarg(lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAppOptM___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqFalse___closed__2; static lean_object* l_Lean_Meta_mkListLit___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5; LEAN_EXPORT uint8_t l_Lean_Meta_mkProjection___lambda__1(lean_object*); static lean_object* l_Lean_Meta_mkDecideProof___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_congrArg_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -341,6 +350,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrans_x3f(lean_object*, lean_object*, l static lean_object* l_Lean_Meta_mkLe___closed__1; static lean_object* l_Lean_Meta_mkNone___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_mkCongr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkImpCongr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkLetFun(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -365,9 +375,9 @@ static lean_object* l_Lean_Meta_mkDefault___closed__3; lean_object* l_Lean_MVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__5; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppOptM___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqRec___closed__1; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13; static lean_object* l_Lean_Meta_mkEqSymm___closed__4; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_mkProjection___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -382,6 +392,7 @@ static lean_object* l_List_mapTR_loop___at_Lean_Meta_mkAppOptM___spec__2___close static lean_object* l_Lean_Meta_mkProjection___lambda__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkListLit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLetValCongr___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_mkEqRefl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -392,11 +403,10 @@ static lean_object* l_Lean_Meta_mkEqOfHEq___closed__1; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_hasTypeMsg___closed__2; static lean_object* l_Lean_Meta_mkLetCongr___closed__1; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__3; -static lean_object* l_Lean_Meta_mkEqTrue___closed__1; static lean_object* l_Lean_Meta_mkIffOfEq___closed__2; LEAN_EXPORT lean_object* l_List_mapM_loop___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkFun___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException___rarg___closed__3; +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkForallFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_hasTypeMsg___closed__1; static lean_object* l_Lean_Meta_mkProjection___closed__3; @@ -414,15 +424,16 @@ lean_object* l_Lean_Expr_getAppFn(lean_object*); uint8_t l_Lean_isStructure(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkDecide___closed__1; static lean_object* l_Lean_Meta_mkEqSymm___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrueCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkFunExt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqNDRec___closed__3; -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppOptM_x27___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__1___closed__2; static lean_object* l_Lean_Meta_mkListLit___closed__5; static lean_object* l_Lean_Meta_mkArrayLit___closed__2; static lean_object* l_Lean_isLevelMVarAssignable___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__4___closed__2; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___closed__3; +lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_throwAppTypeMismatch___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkNumeral(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkDefault___closed__1; @@ -443,14 +454,15 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkEqFalse(lean_object*, lean_object*, lean_ static lean_object* l_Lean_Meta_mkProjection___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_mkEqOfHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); -static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppOptMAux___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_congrArg_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_array_size(lean_object*); +static lean_object* l_Lean_Meta_mkOfEqTrueCore___closed__1; lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkProjection___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqMP___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppOptM_x27___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__1___closed__9; @@ -466,15 +478,16 @@ lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_hasAssignableLevelMVar___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException___spec__1(lean_object*); static lean_object* l_Lean_Meta_mkProjection___lambda__2___closed__5; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_hasTypeMsg___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_mkEqTrue___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__7(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkListLit___closed__1; uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqMPR___closed__1; uint8_t lean_usize_dec_lt(size_t, size_t); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9; LEAN_EXPORT lean_object* l_Lean_hasAssignableLevelMVar___at___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkNoConfusion___closed__4; lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -491,7 +504,9 @@ uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_Expr_beta(lean_object*, lean_object*); lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7; static lean_object* l_Lean_Meta_mkEqOfHEq___closed__3; +static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMFinal___closed__1; static lean_object* l_Lean_Meta_mkEqOfHEq___lambda__1___closed__1; static lean_object* l_Lean_Meta_mkId___closed__1; @@ -499,6 +514,7 @@ static lean_object* l_Lean_Meta_mkLetFun___closed__2; uint8_t l_Lean_Expr_isForall(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkAppM_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_mkAppOptM___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkListLitAux___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkOfNonempty(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -513,6 +529,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_mkHEqSymm(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___at_Lean_Meta_mkAppM___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkLT___closed__1; static lean_object* l_Lean_Meta_mkSub___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_mkEqOfHEq___closed__2; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_throwAppBuilderException___rarg___closed__2; static lean_object* l___private_Lean_Meta_AppBuilder_0__Lean_Meta_mkAppMArgs_loop___closed__4; @@ -15825,7 +15842,7 @@ x_13 = l_Lean_Meta_mkAppM(x_12, x_11, x_3, x_4, x_5, x_6, x_7); return x_13; } } -static lean_object* _init_l_Lean_Meta_mkOfEqTrue___closed__1() { +static lean_object* _init_l_Lean_Meta_mkOfEqTrueCore___closed__1() { _start: { lean_object* x_1; @@ -15833,31 +15850,27 @@ x_1 = lean_mk_string_unchecked("of_eq_true", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Meta_mkOfEqTrue___closed__2() { +static lean_object* _init_l_Lean_Meta_mkOfEqTrueCore___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_mkOfEqTrue___closed__1; +x_2 = l_Lean_Meta_mkOfEqTrueCore___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +static lean_object* _init_l_Lean_Meta_mkOfEqTrueCore___closed__3() { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -x_9 = lean_array_mk(x_8); -x_10 = l_Lean_Meta_mkOfEqTrue___closed__2; -x_11 = l_Lean_Meta_mkAppM(x_10, x_9, x_2, x_3, x_4, x_5, x_6); -return x_11; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_mkOfEqTrueCore___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; } } -static lean_object* _init_l_Lean_Meta_mkEqTrue___closed__1() { +static lean_object* _init_l_Lean_Meta_mkOfEqTrueCore___closed__4() { _start: { lean_object* x_1; @@ -15865,29 +15878,454 @@ x_1 = lean_mk_string_unchecked("eq_true", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_mkEqTrue___closed__2() { +static lean_object* _init_l_Lean_Meta_mkOfEqTrueCore___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_mkEqTrue___closed__1; +x_2 = l_Lean_Meta_mkOfEqTrueCore___closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrueCore(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; -x_7 = lean_box(0); -x_8 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_8, 0, x_1); -lean_ctor_set(x_8, 1, x_7); -x_9 = lean_array_mk(x_8); -x_10 = l_Lean_Meta_mkEqTrue___closed__2; -x_11 = l_Lean_Meta_mkAppM(x_10, x_9, x_2, x_3, x_4, x_5, x_6); +lean_object* x_3; uint8_t x_4; +lean_inc(x_2); +x_3 = l_Lean_Expr_cleanupAnnotations(x_2); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +lean_dec(x_3); +x_5 = l_Lean_Meta_mkOfEqTrueCore___closed__3; +x_6 = l_Lean_mkAppB(x_5, x_1, x_2); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_7 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_8 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_9 = l_Lean_Expr_isApp(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_8); +lean_dec(x_7); +x_10 = l_Lean_Meta_mkOfEqTrueCore___closed__3; +x_11 = l_Lean_mkAppB(x_10, x_1, x_2); return x_11; } +else +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_12 = l_Lean_Expr_appFnCleanup(x_8, lean_box(0)); +x_13 = l_Lean_Meta_mkOfEqTrueCore___closed__5; +x_14 = l_Lean_Expr_isConstOf(x_12, x_13); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_7); +x_15 = l_Lean_Meta_mkOfEqTrueCore___closed__3; +x_16 = l_Lean_mkAppB(x_15, x_1, x_2); +return x_16; +} +else +{ +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_1); +lean_ctor_set(x_7, 1, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_8); +x_10 = lean_array_mk(x_9); +x_11 = l_Lean_Meta_mkOfEqTrueCore___closed__2; +x_12 = l_Lean_Meta_mkAppM(x_11, x_10, x_3, x_4, x_5, x_6, x_7); +return x_12; +} +} +static lean_object* _init_l_Lean_Meta_mkOfEqTrue___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_mkOfEqTrue___lambda__1___boxed), 6, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_inc(x_1); +x_7 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_2, x_3, x_4, x_5, x_6); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_7, 1); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Lean_Meta_mkOfEqTrue___closed__1; +x_11 = l_Lean_Expr_cleanupAnnotations(x_8); +x_12 = l_Lean_Expr_isApp(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_11); +x_13 = lean_box(0); +x_14 = l_Lean_Meta_mkOfEqTrue___lambda__2(x_1, x_13, x_2, x_3, x_4, x_5, x_9); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = l_Lean_Expr_appArg(x_11, lean_box(0)); +x_16 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); +x_17 = l_Lean_Expr_isApp(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_16); +lean_dec(x_15); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_mkOfEqTrue___lambda__2(x_1, x_18, x_2, x_3, x_4, x_5, x_9); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); +x_21 = l_Lean_Meta_mkOfEqTrueCore___closed__5; +x_22 = l_Lean_Expr_isConstOf(x_20, x_21); +lean_dec(x_20); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_15); +x_23 = lean_box(0); +x_24 = l_Lean_Meta_mkOfEqTrue___lambda__2(x_1, x_23, x_2, x_3, x_4, x_5, x_9); +return x_24; +} +else +{ +lean_object* x_25; +lean_dec(x_1); +x_25 = lean_apply_6(x_10, x_15, x_2, x_3, x_4, x_5, x_9); +return x_25; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Meta_mkOfEqTrue___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkOfEqTrue___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Meta_mkOfEqTrue___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_2); +return x_8; +} +} +static lean_object* _init_l_Lean_Meta_mkEqTrueCore___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_mkOfEqTrueCore___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrueCore(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint8_t x_4; +lean_inc(x_2); +x_3 = l_Lean_Expr_cleanupAnnotations(x_2); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +lean_dec(x_3); +x_5 = l_Lean_Meta_mkEqTrueCore___closed__1; +x_6 = l_Lean_mkAppB(x_5, x_1, x_2); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_7 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_8 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_9 = l_Lean_Expr_isApp(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_8); +lean_dec(x_7); +x_10 = l_Lean_Meta_mkEqTrueCore___closed__1; +x_11 = l_Lean_mkAppB(x_10, x_1, x_2); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_12 = l_Lean_Expr_appFnCleanup(x_8, lean_box(0)); +x_13 = l_Lean_Meta_mkOfEqTrueCore___closed__2; +x_14 = l_Lean_Expr_isConstOf(x_12, x_13); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_7); +x_15 = l_Lean_Meta_mkEqTrueCore___closed__1; +x_16 = l_Lean_mkAppB(x_15, x_1, x_2); +return x_16; +} +else +{ +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_1); +x_8 = lean_infer_type(x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_8, 0); +x_11 = l_Lean_Meta_mkEqTrueCore___closed__1; +x_12 = l_Lean_mkAppB(x_11, x_10, x_1); +lean_ctor_set(x_8, 0, x_12); +return x_8; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_8, 0); +x_14 = lean_ctor_get(x_8, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_8); +x_15 = l_Lean_Meta_mkEqTrueCore___closed__1; +x_16 = l_Lean_mkAppB(x_15, x_13, x_1); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_14); +return x_17; +} +} +else +{ +uint8_t x_18; +lean_dec(x_1); +x_18 = !lean_is_exclusive(x_8); +if (x_18 == 0) +{ +return x_8; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_8, 0); +x_20 = lean_ctor_get(x_8, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_8); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +lean_inc(x_1); +x_7 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_1, x_2, x_3, x_4, x_5, x_6); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +x_11 = l_Lean_Expr_cleanupAnnotations(x_9); +x_12 = l_Lean_Expr_isApp(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_11); +lean_free_object(x_7); +x_13 = lean_box(0); +x_14 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_13, x_2, x_3, x_4, x_5, x_10); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = l_Lean_Expr_appArg(x_11, lean_box(0)); +x_16 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); +x_17 = l_Lean_Expr_isApp(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_16); +lean_dec(x_15); +lean_free_object(x_7); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_18, x_2, x_3, x_4, x_5, x_10); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = l_Lean_Expr_appFnCleanup(x_16, lean_box(0)); +x_21 = l_Lean_Meta_mkOfEqTrueCore___closed__2; +x_22 = l_Lean_Expr_isConstOf(x_20, x_21); +lean_dec(x_20); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_15); +lean_free_object(x_7); +x_23 = lean_box(0); +x_24 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_23, x_2, x_3, x_4, x_5, x_10); +return x_24; +} +else +{ +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +lean_ctor_set(x_7, 0, x_15); +return x_7; +} +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_ctor_get(x_7, 0); +x_26 = lean_ctor_get(x_7, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_7); +x_27 = l_Lean_Expr_cleanupAnnotations(x_25); +x_28 = l_Lean_Expr_isApp(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_27); +x_29 = lean_box(0); +x_30 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_29, x_2, x_3, x_4, x_5, x_26); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); +x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); +x_33 = l_Lean_Expr_isApp(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_32); +lean_dec(x_31); +x_34 = lean_box(0); +x_35 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_34, x_2, x_3, x_4, x_5, x_26); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_36 = l_Lean_Expr_appFnCleanup(x_32, lean_box(0)); +x_37 = l_Lean_Meta_mkOfEqTrueCore___closed__2; +x_38 = l_Lean_Expr_isConstOf(x_36, x_37); +lean_dec(x_36); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +lean_dec(x_31); +x_39 = lean_box(0); +x_40 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_39, x_2, x_3, x_4, x_5, x_26); +return x_40; +} +else +{ +lean_object* x_41; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_31); +lean_ctor_set(x_41, 1, x_26); +return x_41; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_mkEqTrue___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Meta_mkEqTrue___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_2); +return x_8; +} } static lean_object* _init_l_Lean_Meta_mkEqFalse___closed__1() { _start: @@ -17013,7 +17451,7 @@ return x_16; } } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1() { _start: { lean_object* x_1; @@ -17021,27 +17459,27 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2; x_2 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4() { _start: { lean_object* x_1; @@ -17049,17 +17487,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6() { _start: { lean_object* x_1; @@ -17067,37 +17505,37 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8; x_2 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___lambda__3___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10() { _start: { lean_object* x_1; @@ -17105,17 +17543,17 @@ x_1 = lean_mk_string_unchecked("AppBuilder", 10, 10); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12() { _start: { lean_object* x_1; @@ -17123,33 +17561,33 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11; -x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12; +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11; +x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14() { +static lean_object* _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13; -x_2 = lean_unsigned_to_nat(7417u); +x_1 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13; +x_2 = lean_unsigned_to_nat(7897u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l___private_Lean_Meta_AppBuilder_0__Lean_Meta_withAppBuilderTrace___rarg___closed__1; x_3 = 0; -x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14; +x_4 = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); if (lean_obj_tag(x_5) == 0) { @@ -17628,14 +18066,20 @@ l_Lean_Meta_mkLetBodyCongr___closed__1 = _init_l_Lean_Meta_mkLetBodyCongr___clos lean_mark_persistent(l_Lean_Meta_mkLetBodyCongr___closed__1); l_Lean_Meta_mkLetBodyCongr___closed__2 = _init_l_Lean_Meta_mkLetBodyCongr___closed__2(); lean_mark_persistent(l_Lean_Meta_mkLetBodyCongr___closed__2); +l_Lean_Meta_mkOfEqTrueCore___closed__1 = _init_l_Lean_Meta_mkOfEqTrueCore___closed__1(); +lean_mark_persistent(l_Lean_Meta_mkOfEqTrueCore___closed__1); +l_Lean_Meta_mkOfEqTrueCore___closed__2 = _init_l_Lean_Meta_mkOfEqTrueCore___closed__2(); +lean_mark_persistent(l_Lean_Meta_mkOfEqTrueCore___closed__2); +l_Lean_Meta_mkOfEqTrueCore___closed__3 = _init_l_Lean_Meta_mkOfEqTrueCore___closed__3(); +lean_mark_persistent(l_Lean_Meta_mkOfEqTrueCore___closed__3); +l_Lean_Meta_mkOfEqTrueCore___closed__4 = _init_l_Lean_Meta_mkOfEqTrueCore___closed__4(); +lean_mark_persistent(l_Lean_Meta_mkOfEqTrueCore___closed__4); +l_Lean_Meta_mkOfEqTrueCore___closed__5 = _init_l_Lean_Meta_mkOfEqTrueCore___closed__5(); +lean_mark_persistent(l_Lean_Meta_mkOfEqTrueCore___closed__5); l_Lean_Meta_mkOfEqTrue___closed__1 = _init_l_Lean_Meta_mkOfEqTrue___closed__1(); lean_mark_persistent(l_Lean_Meta_mkOfEqTrue___closed__1); -l_Lean_Meta_mkOfEqTrue___closed__2 = _init_l_Lean_Meta_mkOfEqTrue___closed__2(); -lean_mark_persistent(l_Lean_Meta_mkOfEqTrue___closed__2); -l_Lean_Meta_mkEqTrue___closed__1 = _init_l_Lean_Meta_mkEqTrue___closed__1(); -lean_mark_persistent(l_Lean_Meta_mkEqTrue___closed__1); -l_Lean_Meta_mkEqTrue___closed__2 = _init_l_Lean_Meta_mkEqTrue___closed__2(); -lean_mark_persistent(l_Lean_Meta_mkEqTrue___closed__2); +l_Lean_Meta_mkEqTrueCore___closed__1 = _init_l_Lean_Meta_mkEqTrueCore___closed__1(); +lean_mark_persistent(l_Lean_Meta_mkEqTrueCore___closed__1); l_Lean_Meta_mkEqFalse___closed__1 = _init_l_Lean_Meta_mkEqFalse___closed__1(); lean_mark_persistent(l_Lean_Meta_mkEqFalse___closed__1); l_Lean_Meta_mkEqFalse___closed__2 = _init_l_Lean_Meta_mkEqFalse___closed__2(); @@ -17706,35 +18150,35 @@ l_Lean_Meta_mkIffOfEq___closed__2 = _init_l_Lean_Meta_mkIffOfEq___closed__2(); lean_mark_persistent(l_Lean_Meta_mkIffOfEq___closed__2); l_Lean_Meta_mkIffOfEq___closed__3 = _init_l_Lean_Meta_mkIffOfEq___closed__3(); lean_mark_persistent(l_Lean_Meta_mkIffOfEq___closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__1); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__2); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__3); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__4); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__5); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__6); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__7); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__8); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__9); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__10); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__11); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__12); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__13); -l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14(); -lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417____closed__14); -if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7417_(lean_io_mk_world()); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__1); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__2); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__3); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__4); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__5); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__6); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__7); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__8); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__9); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__10); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__11); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__12); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__13); +l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14 = _init_l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14(); +lean_mark_persistent(l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897____closed__14); +if (builtin) {res = l_Lean_Meta_initFn____x40_Lean_Meta_AppBuilder___hyg_7897_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Basic.c b/stage0/stdlib/Lean/Meta/Basic.c index 10672b3302c2..adf8cec8d6b9 100644 --- a/stage0/stdlib/Lean/Meta/Basic.c +++ b/stage0/stdlib/Lean/Meta/Basic.c @@ -38,7 +38,6 @@ static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_L LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_FVarId_hasForwardDeps___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalInstances___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getZetaDeltaFVarIds___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux_process___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withExistingLocalDeclsImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withErasedFVars___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -106,7 +105,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_orelseMergeErrors(lean_object*, lean_object LEAN_EXPORT lean_object* l_Lean_MVarId_getDecl___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitMain___at_Lean_FVarId_hasForwardDeps___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_FVarId_hasForwardDeps___spec__34___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_mkForallFVars___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_throwMaxRecDepthAt___at_Lean_Meta_withIncRecDepth___spec__1___rarg___closed__4; @@ -290,7 +288,6 @@ LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_sortFVarIds___spec__1 LEAN_EXPORT lean_object* l_Lean_FVarId_isLetVar___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instBEqDefEqCacheKey; static lean_object* l_Lean_Meta_instMonadEnvMetaM___closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_FVarId_throwUnknown___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_instInhabitedProjReductionKind; LEAN_EXPORT lean_object* l_Lean_Meta_lambdaTelescope___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -333,6 +330,7 @@ static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_L LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux(lean_object*); static size_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_recordSynthPendingFailure___spec__2___closed__2; static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprProjReductionKind____x40_Lean_Meta_Basic___hyg_210____closed__21; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncSynthPending(lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewMCtxDepthImp___rarg___closed__3; LEAN_EXPORT lean_object* l_Lean_getExprMVarAssignment_x3f___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassQuick_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -347,6 +345,7 @@ LEAN_EXPORT lean_object* l_Array_isEqvAux___at___private_Lean_Meta_Basic_0__Lean LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_beqSynthInstanceCacheKey____x40_Lean_Meta_Basic___hyg_1516____boxed(lean_object*, lean_object*); uint8_t l_Lean_Name_quickLt(lean_object*, lean_object*); lean_object* lean_io_get_num_heartbeats(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7; LEAN_EXPORT lean_object* l_Lean_LocalContext_foldlM___at_Lean_FVarId_hasForwardDeps___spec__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkFreshExprMVarAtCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); @@ -388,10 +387,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_FVarId_hasForwardDe LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_FVarId_hasForwardDeps___spec__9(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_normalizeLevel___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprProjReductionKind____x40_Lean_Meta_Basic___hyg_210____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwUnknownConstant___at___private_Lean_Meta_Basic_0__Lean_Meta_getConstTemp_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withIncSynthPending___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_3478____closed__6; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_approxDefEqImp(lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__3; static lean_object* l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_3478____closed__7; @@ -402,7 +403,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_getConstTemp_x lean_object* l_Lean_LocalContext_addDecl(lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__5___closed__3; LEAN_EXPORT lean_object* l_Lean_getReducibilityStatus___at___private_Lean_Meta_Basic_0__Lean_Meta_getDefInfoTemp___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_modifyInferTypeCache(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Kernel_Diagnostics_recordUnfold___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclD(lean_object*); @@ -464,9 +464,11 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_r LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingImp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getNumPostponed___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprProjReductionKind____x40_Lean_Meta_Basic___hyg_210____closed__26; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_checkpointDefEq___at_Lean_Meta_isExprDefEq___spec__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_processPostponed___lambda__1___closed__1; size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isReadOnlyOrSyntheticOpaque___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_get_reducibility_status(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_Lean_Meta_Basic___hyg_579____closed__47; @@ -517,7 +519,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_shouldReduceReducibleOnly(lean_object*, lea LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_recordSynthPendingFailure___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_1294____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_sortFVarIds___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6; lean_object* lean_is_expr_def_eq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_fullApproxDefEq___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); @@ -683,7 +684,7 @@ static lean_object* l_Lean_Meta_instAddMessageContextMetaM___closed__1; static lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withDefault___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_isInductivePredicate___closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_mapMetaM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_liftMkBindingM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_FVarId_hasForwardDeps___spec__49___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -691,6 +692,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___rarg___lambda__1(lean LEAN_EXPORT lean_object* l_Lean_Meta_inferType___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3; static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_Lean_Meta_Basic___hyg_579____closed__17; LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_withLocalInstancesImp___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withTrackingZetaDelta___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -711,7 +713,6 @@ LEAN_EXPORT lean_object* l_Lean_MVarId_setType___boxed(lean_object*, lean_object LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visitApp___at_Lean_FVarId_hasForwardDeps___spec__12___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_Lean_Meta_Basic___hyg_579____closed__34; lean_object* l_Lean_LocalInstances_erase(lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_whnfD(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_instInhabitedCache___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withExistingLocalDeclsImp(lean_object*); @@ -772,7 +773,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_approxDefEq___rarg___lambda__1(lean_object* uint8_t l___private_Init_MetaTypes_0__Lean_Meta_beqTransparencyMode____x40_Init_MetaTypes___hyg_73_(uint8_t, uint8_t); uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_withoutProofIrrelevance___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withoutProofIrrelevance___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getParamNames___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -870,6 +870,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_getConfig(lean_object*, lean_object*, lean_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux___rarg(uint8_t, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Level_collectMVars(lean_object*, lean_object*); lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Trace_0__Lean_addTraceNode___spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Meta_withInstImplicitAsImplict___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withRestoreOrSaveFull___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_Lean_Meta_Basic___hyg_579____closed__16; @@ -1068,7 +1069,6 @@ static lean_object* l_Lean_Meta_instMonadMetaM___closed__1; LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Basic_0__Lean_Meta_forallTelescopeReducingAuxAux_process___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_map1MetaM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_orelseMergeErrorsImp(lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withNewBinderInfos___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1135,7 +1135,6 @@ LEAN_EXPORT lean_object* l_Lean_mkFreshLMVarId___at_Lean_Meta_mkFreshLevelMVar__ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_recordSynthPendingFailure___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprProjReductionKind____x40_Lean_Meta_Basic___hyg_210____closed__3; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_getParamNames___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_withLCtx_x27___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); uint8_t l_Lean_LocalDecl_binderInfo(lean_object*); @@ -1269,6 +1268,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_withMCtx___rarg___lambda__1(lean_object*, l LEAN_EXPORT lean_object* l_Lean_Meta_withInTypeClassResolution(lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Meta_withInstImplicitAsImplict___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_withTraceNode___at_Lean_Meta_processPostponed___spec__1___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_forIn___at___private_Lean_Meta_Basic_0__Lean_Meta_processPostponedStep___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Meta_processPostponed___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_getPostponed(lean_object*); @@ -1287,6 +1287,7 @@ static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprProjReductionKi LEAN_EXPORT lean_object* l_Lean_Meta_useEtaStruct___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_reprConfig____x40_Lean_Meta_Basic___hyg_579____closed__36; static lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withNewMCtxDepthImp___rarg___closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_withLocalDeclsD___spec__1___rarg(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_liftMkBindingM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_processPostponed_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -1368,7 +1369,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_setPostponed(lean_object*, lean_object*, le LEAN_EXPORT uint64_t l___private_Lean_Meta_Basic_0__Lean_Meta_Config_toKey(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_forallBoundedTelescopeImp(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_instMonadLCtxMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_ParamInfo_isExplicit(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_MetavarContext_0__Lean_DependsOn_dep_visit___at_Lean_FVarId_hasForwardDeps___spec__10___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_ppExprWithInfos(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -47053,117 +47053,137 @@ lean_dec(x_3); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_8; -x_8 = l_Lean_Meta_whnfD(x_2, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_8) == 0) -{ lean_object* x_9; -x_9 = lean_ctor_get(x_8, 0); -lean_inc(x_9); -if (lean_obj_tag(x_9) == 3) +x_9 = l_Lean_Meta_whnfD(x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_9) == 0) { -uint8_t x_10; -x_10 = !lean_is_exclusive(x_8); -if (x_10 == 0) +lean_object* x_10; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +if (lean_obj_tag(x_10) == 3) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_11 = lean_ctor_get(x_8, 0); -lean_dec(x_11); +uint8_t x_11; +x_11 = !lean_is_exclusive(x_9); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; x_12 = lean_ctor_get(x_9, 0); -lean_inc(x_12); -lean_dec(x_9); -x_13 = l_Lean_levelZero; -x_14 = lean_level_eq(x_12, x_13); lean_dec(x_12); -x_15 = lean_box(x_14); -lean_ctor_set(x_8, 0, x_15); -return x_8; +x_13 = lean_ctor_get(x_10, 0); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l_Lean_levelZero; +x_15 = lean_level_eq(x_13, x_14); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_1); +x_16 = lean_box(0); +lean_ctor_set(x_9, 0, x_16); +return x_9; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_8, 1); -lean_inc(x_16); -lean_dec(x_8); -x_17 = lean_ctor_get(x_9, 0); -lean_inc(x_17); -lean_dec(x_9); -x_18 = l_Lean_levelZero; -x_19 = lean_level_eq(x_17, x_18); -lean_dec(x_17); -x_20 = lean_box(x_19); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_16); -return x_21; +lean_object* x_17; +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_9, 0, x_17); +return x_9; } } else { -uint8_t x_22; +lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); lean_dec(x_9); -x_22 = !lean_is_exclusive(x_8); -if (x_22 == 0) +x_19 = lean_ctor_get(x_10, 0); +lean_inc(x_19); +lean_dec(x_10); +x_20 = l_Lean_levelZero; +x_21 = lean_level_eq(x_19, x_20); +lean_dec(x_19); +if (x_21 == 0) { -lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_8, 0); -lean_dec(x_23); -x_24 = 0; -x_25 = lean_box(x_24); -lean_ctor_set(x_8, 0, x_25); -return x_8; +lean_object* x_22; lean_object* x_23; +lean_dec(x_1); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_18); +return x_23; } else { -lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_26 = lean_ctor_get(x_8, 1); -lean_inc(x_26); -lean_dec(x_8); -x_27 = 0; -x_28 = lean_box(x_27); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_26); -return x_29; +lean_object* x_24; lean_object* x_25; +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_1); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_18); +return x_25; } } } else { -uint8_t x_30; -x_30 = !lean_is_exclusive(x_8); -if (x_30 == 0) +uint8_t x_26; +lean_dec(x_10); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_9); +if (x_26 == 0) { -return x_8; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_9, 0); +lean_dec(x_27); +x_28 = lean_box(0); +lean_ctor_set(x_9, 0, x_28); +return x_9; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_8, 0); -x_32 = lean_ctor_get(x_8, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_8); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_9, 1); +lean_inc(x_29); +lean_dec(x_9); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; } } } +else +{ +uint8_t x_32; +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_9); +if (x_32 == 0) +{ +return x_9; } -static lean_object* _init_l_Lean_Meta_isInductivePredicate___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_isInductivePredicate___lambda__1___boxed), 7, 0); -return x_1; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_9, 0); +x_34 = lean_ctor_get(x_9, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_9); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } -LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; uint8_t x_8; @@ -47180,130 +47200,218 @@ lean_dec(x_9); x_12 = lean_environment_find(x_11, x_1); if (lean_obj_tag(x_12) == 0) { -uint8_t x_13; lean_object* x_14; +lean_object* x_13; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_13 = 0; -x_14 = lean_box(x_13); -lean_ctor_set(x_7, 0, x_14); +x_13 = lean_box(0); +lean_ctor_set(x_7, 0, x_13); return x_7; } else { -lean_object* x_15; -x_15 = lean_ctor_get(x_12, 0); -lean_inc(x_15); +lean_object* x_14; +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); lean_dec(x_12); -if (lean_obj_tag(x_15) == 5) +if (lean_obj_tag(x_14) == 5) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_free_object(x_7); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +lean_dec(x_14); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_15); -x_17 = lean_ctor_get(x_16, 0); +x_17 = lean_ctor_get(x_16, 2); lean_inc(x_17); lean_dec(x_16); -x_18 = lean_ctor_get(x_17, 2); -lean_inc(x_18); -lean_dec(x_17); -x_19 = l_Lean_Meta_isInductivePredicate___closed__1; -x_20 = 0; -x_21 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_18, x_19, x_20, x_2, x_3, x_4, x_5, x_10); -return x_21; +x_18 = lean_alloc_closure((void*)(l_Lean_Meta_isInductivePredicate_x3f___lambda__1___boxed), 8, 1); +lean_closure_set(x_18, 0, x_15); +x_19 = 0; +x_20 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_17, x_18, x_19, x_2, x_3, x_4, x_5, x_10); +return x_20; } else { -uint8_t x_22; lean_object* x_23; -lean_dec(x_15); +lean_object* x_21; +lean_dec(x_14); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_22 = 0; -x_23 = lean_box(x_22); -lean_ctor_set(x_7, 0, x_23); +x_21 = lean_box(0); +lean_ctor_set(x_7, 0, x_21); return x_7; } } } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_7, 0); -x_25 = lean_ctor_get(x_7, 1); -lean_inc(x_25); -lean_inc(x_24); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_7, 0); +x_23 = lean_ctor_get(x_7, 1); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_7); -x_26 = lean_ctor_get(x_24, 0); -lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_environment_find(x_26, x_1); -if (lean_obj_tag(x_27) == 0) +x_24 = lean_ctor_get(x_22, 0); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_environment_find(x_24, x_1); +if (lean_obj_tag(x_25) == 0) { -uint8_t x_28; lean_object* x_29; lean_object* x_30; +lean_object* x_26; lean_object* x_27; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_28 = 0; -x_29 = lean_box(x_28); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_25); -return x_30; +x_26 = lean_box(0); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_23); +return x_27; } else { -lean_object* x_31; -x_31 = lean_ctor_get(x_27, 0); -lean_inc(x_31); -lean_dec(x_27); -if (lean_obj_tag(x_31) == 5) +lean_object* x_28; +x_28 = lean_ctor_get(x_25, 0); +lean_inc(x_28); +lean_dec(x_25); +if (lean_obj_tag(x_28) == 5) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -lean_dec(x_31); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -lean_dec(x_32); -x_34 = lean_ctor_get(x_33, 2); -lean_inc(x_34); -lean_dec(x_33); -x_35 = l_Lean_Meta_isInductivePredicate___closed__1; -x_36 = 0; -x_37 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_34, x_35, x_36, x_2, x_3, x_4, x_5, x_25); -return x_37; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +lean_dec(x_28); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_30, 2); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_alloc_closure((void*)(l_Lean_Meta_isInductivePredicate_x3f___lambda__1___boxed), 8, 1); +lean_closure_set(x_32, 0, x_29); +x_33 = 0; +x_34 = l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(x_31, x_32, x_33, x_2, x_3, x_4, x_5, x_23); +return x_34; } else { -uint8_t x_38; lean_object* x_39; lean_object* x_40; -lean_dec(x_31); +lean_object* x_35; lean_object* x_36; +lean_dec(x_28); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_38 = 0; -x_39 = lean_box(x_38); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_25); -return x_40; +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_23); +return x_36; +} +} } } } +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l_Lean_Meta_isInductivePredicate_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_2); +return x_9; } } -LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Lean_Meta_isInductivePredicate(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { +lean_object* x_7; +x_7 = l_Lean_Meta_isInductivePredicate_x3f(x_1, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_7) == 0) +{ lean_object* x_8; -x_8 = l_Lean_Meta_isInductivePredicate___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_1); -return x_8; +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +if (lean_obj_tag(x_8) == 0) +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_7); +if (x_9 == 0) +{ +lean_object* x_10; uint8_t x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_7, 0); +lean_dec(x_10); +x_11 = 0; +x_12 = lean_box(x_11); +lean_ctor_set(x_7, 0, x_12); +return x_7; +} +else +{ +lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_7, 1); +lean_inc(x_13); +lean_dec(x_7); +x_14 = 0; +x_15 = lean_box(x_14); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_13); +return x_16; +} +} +else +{ +uint8_t x_17; +lean_dec(x_8); +x_17 = !lean_is_exclusive(x_7); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_7, 0); +lean_dec(x_18); +x_19 = 1; +x_20 = lean_box(x_19); +lean_ctor_set(x_7, 0, x_20); +return x_7; +} +else +{ +lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_7, 1); +lean_inc(x_21); +lean_dec(x_7); +x_22 = 1; +x_23 = lean_box(x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_21); +return x_24; +} +} +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_7); +if (x_25 == 0) +{ +return x_7; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_7, 0); +x_27 = lean_ctor_get(x_7, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_7); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} +} } } LEAN_EXPORT lean_object* l_Lean_Meta_isListLevelDefEqAux(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { @@ -58051,7 +58159,7 @@ lean_dec(x_2); return x_7; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -58061,73 +58169,73 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1; +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1; x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_3478____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2; +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2; x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_2486____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3; x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_2486____closed__7; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4; x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_3478____closed__10; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5; +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5; x_2 = l_Lean_Meta_initFn____x40_Lean_Meta_Basic___hyg_3478____closed__12; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6; -x_2 = lean_unsigned_to_nat(19460u); +x_1 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6; +x_2 = lean_unsigned_to_nat(19467u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_processPostponed_loop___closed__3; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7; +x_4 = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -58669,8 +58777,6 @@ l_Lean_Meta_instAlternativeMetaM___closed__3 = _init_l_Lean_Meta_instAlternative lean_mark_persistent(l_Lean_Meta_instAlternativeMetaM___closed__3); l_Lean_Meta_instAlternativeMetaM = _init_l_Lean_Meta_instAlternativeMetaM(); lean_mark_persistent(l_Lean_Meta_instAlternativeMetaM); -l_Lean_Meta_isInductivePredicate___closed__1 = _init_l_Lean_Meta_isInductivePredicate___closed__1(); -lean_mark_persistent(l_Lean_Meta_isInductivePredicate___closed__1); l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__1 = _init_l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__1); l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__2 = _init_l___private_Lean_Meta_Basic_0__Lean_Meta_mkLevelErrorMessageCore___lambda__3___closed__2(); @@ -58732,21 +58838,21 @@ l_Lean_Meta_processPostponed___lambda__1___closed__3 = _init_l_Lean_Meta_process lean_mark_persistent(l_Lean_Meta_processPostponed___lambda__1___closed__3); l_Lean_Meta_processPostponed___lambda__1___closed__4 = _init_l_Lean_Meta_processPostponed___lambda__1___closed__4(); lean_mark_persistent(l_Lean_Meta_processPostponed___lambda__1___closed__4); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__1); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__2); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__3); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__4); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__5); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__6); -l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460____closed__7); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19460_(lean_io_mk_world()); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__1); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__2); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__3); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__4); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__5); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__6); +l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7 = _init_l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467____closed__7); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Basic___hyg_19467_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind.c b/stage0/stdlib/Lean/Meta/Tactic/Grind.c index 1d3922f2ccad..5429de45f6d9 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind -// Imports: Lean.Meta.Tactic.Grind.Attr Lean.Meta.Tactic.Grind.RevertAll Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Util Lean.Meta.Tactic.Grind.Cases Lean.Meta.Tactic.Grind.Injection Lean.Meta.Tactic.Grind.Core Lean.Meta.Tactic.Grind.Canon Lean.Meta.Tactic.Grind.MarkNestedProofs Lean.Meta.Tactic.Grind.Inv Lean.Meta.Tactic.Grind.Proof Lean.Meta.Tactic.Grind.Propagate Lean.Meta.Tactic.Grind.PP Lean.Meta.Tactic.Grind.Simp Lean.Meta.Tactic.Grind.Ctor Lean.Meta.Tactic.Grind.Parser Lean.Meta.Tactic.Grind.EMatchTheorem Lean.Meta.Tactic.Grind.EMatch Lean.Meta.Tactic.Grind.Main Lean.Meta.Tactic.Grind.CasesMatch +// Imports: Lean.Meta.Tactic.Grind.Attr Lean.Meta.Tactic.Grind.RevertAll Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Util Lean.Meta.Tactic.Grind.Cases Lean.Meta.Tactic.Grind.Injection Lean.Meta.Tactic.Grind.Core Lean.Meta.Tactic.Grind.Canon Lean.Meta.Tactic.Grind.MarkNestedProofs Lean.Meta.Tactic.Grind.Inv Lean.Meta.Tactic.Grind.Proof Lean.Meta.Tactic.Grind.Propagate Lean.Meta.Tactic.Grind.PP Lean.Meta.Tactic.Grind.Simp Lean.Meta.Tactic.Grind.Ctor Lean.Meta.Tactic.Grind.Parser Lean.Meta.Tactic.Grind.EMatchTheorem Lean.Meta.Tactic.Grind.EMatch Lean.Meta.Tactic.Grind.Main Lean.Meta.Tactic.Grind.CasesMatch Lean.Meta.Tactic.Grind.Arith #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -15,120 +15,157 @@ extern "C" { #endif static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_78____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__8; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__9; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_300____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_226_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__14; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__10; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_226____closed__3; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671_(lean_object*); -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_448____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_337____closed__3; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_448____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__13; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_411____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_152____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_189____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__11; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_448_(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_411____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_263____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__2; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_41____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_337____closed__1; lean_object* l_Lean_registerTraceClass(lean_object*, uint8_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_152_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_300_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_374____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_226____closed__1; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_374_(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3; lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__6; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_300____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__1; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_78_(lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__5; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_189____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_263____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_41____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__12; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_78____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_189_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_189____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_226____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__16; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_448____closed__3; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_152____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_374____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_374____closed__3; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_41_(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_337____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__15; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_263____closed__1; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_411_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_300____closed__2; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_337_(lean_object*); +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_411____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__18; -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856_(lean_object*); +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4_(lean_object*); -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__3; +static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__7; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__4; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115____closed__2; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485_(lean_object*); LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_263_(lean_object*); static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_152____closed__2; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_78____closed__1; -static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3; static lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_41____closed__2; +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522_(lean_object*); static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1() { _start: { @@ -819,161 +856,154 @@ x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("debug", 5, 5); +x_1 = lean_mk_string_unchecked("offset", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(523u); +x_2 = lean_unsigned_to_nat(522u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("proofs", 6, 6); +x_1 = lean_mk_string_unchecked("dist", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(560u); +x_2 = lean_unsigned_to_nat(559u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("congr", 5, 5); -return x_1; -} -} -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(597u); +x_2 = lean_unsigned_to_nat(596u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("proof", 5, 5); +x_1 = lean_mk_string_unchecked("term", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_115____closed__1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(634u); +x_2 = lean_unsigned_to_nat(633u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2; -x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2; +x_3 = 1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -982,7 +1012,7 @@ static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("proj", 4, 4); +x_1 = lean_mk_string_unchecked("propagate", 9, 9); return x_1; } } @@ -991,7 +1021,7 @@ static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; @@ -1022,7 +1052,7 @@ static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("parent", 6, 6); +x_1 = lean_mk_string_unchecked("eq", 2, 2); return x_1; } } @@ -1031,7 +1061,7 @@ static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708_ { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; @@ -1062,19 +1092,20 @@ static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("final", 5, 5); +x_1 = lean_mk_string_unchecked("to", 2, 2); return x_1; } } static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__1; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } } static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__3() { @@ -1092,13 +1123,333 @@ LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745_( { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__2; -x_3 = 0; +x_3 = 1; x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____closed__3; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("from", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_708____closed__1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(783u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2; +x_3 = 1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("debug", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(822u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("proofs", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(859u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("congr", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(896u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("proof", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(933u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("proj", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(970u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("parent", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(1007u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("final", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(1044u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1() { _start: { lean_object* x_1; @@ -1106,71 +1457,71 @@ x_1 = lean_mk_string_unchecked("forallPropagator", 16, 16); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(782u); +x_2 = lean_unsigned_to_nat(1081u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_411____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(819u); +x_2 = lean_unsigned_to_nat(1118u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1() { _start: { lean_object* x_1; @@ -1178,34 +1529,99 @@ x_1 = lean_mk_string_unchecked("canon", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1; -x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3() { +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(1155u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; +x_2 = lean_unsigned_to_nat(1192u); +x_3 = l_Lean_Name_num___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1; +x_3 = 0; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2; +x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1; +x_3 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__17; -x_2 = lean_unsigned_to_nat(856u); +x_2 = lean_unsigned_to_nat(1229u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2; +x_2 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1; x_3 = 0; -x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3; +x_4 = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2; x_5 = l_Lean_registerTraceClass(x_2, x_3, x_4, x_1); return x_5; } @@ -1230,6 +1646,7 @@ lean_object* initialize_Lean_Meta_Tactic_Grind_EMatchTheorem(uint8_t builtin, le lean_object* initialize_Lean_Meta_Tactic_Grind_EMatch(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Main(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_CasesMatch(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind(uint8_t builtin, lean_object* w) { lean_object * res; @@ -1295,6 +1712,9 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_CasesMatch(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1(); lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__1); l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_4____closed__2(); @@ -1451,40 +1871,38 @@ lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485____cl if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_485_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_523_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_522_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_560_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_559_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_597_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596____closed__2); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_596_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_634_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_633_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_671____closed__1(); @@ -1514,29 +1932,115 @@ lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745____cl if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_745_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_782_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_783_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_822_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_859_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_896_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_933_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_970_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1007_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1044_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1081_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118____closed__2); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1118_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__2); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155____closed__3); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1155_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819____closed__2); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_819_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192____closed__2); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1192_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__1); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__2); -l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3(); -lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856____closed__3); -if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_856_(lean_io_mk_world()); +}l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__1); +l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2 = _init_l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2(); +lean_mark_persistent(l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229____closed__2); +if (builtin) {res = l_Lean_initFn____x40_Lean_Meta_Tactic_Grind___hyg_1229_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith.c new file mode 100644 index 000000000000..3b5252429ccc --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith.c @@ -0,0 +1,41 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith +// Imports: Lean.Meta.Tactic.Grind.Arith.Util Lean.Meta.Tactic.Grind.Arith.Types Lean.Meta.Tactic.Grind.Arith.Offset Lean.Meta.Tactic.Grind.Arith.Main +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Util(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Types(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Offset(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Main(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Tactic_Grind_Arith_Util(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Types(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Main(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Internalize.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Internalize.c new file mode 100644 index 000000000000..e21f41304643 --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Internalize.c @@ -0,0 +1,39 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Internalize +// Imports: Lean.Meta.Tactic.Grind.Arith.Offset +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* l_Lean_Meta_Grind_Arith_Offset_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_internalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Meta_Grind_Arith_Offset_internalize(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; +} +} +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Offset(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Internalize(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Tactic_Grind_Arith_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Inv.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Inv.c new file mode 100644 index 000000000000..2309a6709ba9 --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Inv.c @@ -0,0 +1,39 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Inv +// Imports: Lean.Meta.Tactic.Grind.Arith.Offset +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* l_Lean_Meta_Grind_Arith_Offset_checkInvariants(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_checkInvariants(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_checkInvariants(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_Arith_Offset_checkInvariants(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +return x_10; +} +} +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Offset(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Inv(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Tactic_Grind_Arith_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Main.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Main.c new file mode 100644 index 000000000000..270b8ebb038e --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Main.c @@ -0,0 +1,913 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Main +// Imports: Lean.Meta.Tactic.Grind.PropagatorAttr Lean.Meta.Tactic.Grind.Arith.Offset +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_shift_right(size_t, size_t); +static lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_uint64_to_usize(uint64_t); +lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1; +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4; +lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_assertTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); +lean_object* lean_usize_to_nat(size_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_assertFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Meta_mkOfEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396_(lean_object*); +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2(lean_object*, size_t, lean_object*); +lean_object* l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(lean_object*, uint8_t, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_sub(size_t, size_t); +lean_object* l_Lean_Meta_Grind_isEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object*); +size_t lean_usize_shift_left(size_t, size_t); +lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg(lean_object*); +lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_get_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get_size(lean_object*); +static lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3; +lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_land(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_lt(x_4, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; uint8_t x_10; +x_9 = lean_array_fget(x_1, x_4); +x_10 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_5, x_9); +lean_dec(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_add(x_4, x_11); +lean_dec(x_4); +x_3 = lean_box(0); +x_4 = x_12; +goto _start; +} +else +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_array_fget(x_2, x_4); +lean_dec(x_4); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; +} +} +} +} +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__1() { +_start: +{ +size_t x_1; size_t x_2; size_t x_3; +x_1 = 1; +x_2 = 5; +x_3 = lean_usize_shift_left(x_1, x_2); +return x_3; +} +} +static size_t _init_l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2() { +_start: +{ +size_t x_1; size_t x_2; size_t x_3; +x_1 = 1; +x_2 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__1; +x_3 = lean_usize_sub(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2(lean_object* x_1, size_t x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; size_t x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 0); +x_6 = 5; +x_7 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2; +x_8 = lean_usize_land(x_2, x_7); +x_9 = lean_usize_to_nat(x_8); +x_10 = lean_box(2); +x_11 = lean_array_get(x_10, x_5, x_9); +lean_dec(x_9); +lean_dec(x_5); +switch (lean_obj_tag(x_11)) { +case 0: +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_12); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_13); +lean_free_object(x_1); +x_15 = lean_box(0); +return x_15; +} +else +{ +lean_ctor_set_tag(x_1, 1); +lean_ctor_set(x_1, 0, x_13); +return x_1; +} +} +case 1: +{ +lean_object* x_16; size_t x_17; +lean_free_object(x_1); +x_16 = lean_ctor_get(x_11, 0); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_usize_shift_right(x_2, x_6); +x_1 = x_16; +x_2 = x_17; +goto _start; +} +default: +{ +lean_object* x_19; +lean_free_object(x_1); +x_19 = lean_box(0); +return x_19; +} +} +} +else +{ +lean_object* x_20; size_t x_21; size_t x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +lean_dec(x_1); +x_21 = 5; +x_22 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2; +x_23 = lean_usize_land(x_2, x_22); +x_24 = lean_usize_to_nat(x_23); +x_25 = lean_box(2); +x_26 = lean_array_get(x_25, x_20, x_24); +lean_dec(x_24); +lean_dec(x_20); +switch (lean_obj_tag(x_26)) { +case 0: +{ +lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_27); +lean_dec(x_27); +if (x_29 == 0) +{ +lean_object* x_30; +lean_dec(x_28); +x_30 = lean_box(0); +return x_30; +} +else +{ +lean_object* x_31; +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_28); +return x_31; +} +} +case 1: +{ +lean_object* x_32; size_t x_33; +x_32 = lean_ctor_get(x_26, 0); +lean_inc(x_32); +lean_dec(x_26); +x_33 = lean_usize_shift_right(x_2, x_21); +x_1 = x_32; +x_2 = x_33; +goto _start; +} +default: +{ +lean_object* x_35; +x_35 = lean_box(0); +return x_35; +} +} +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_1, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_1, 1); +lean_inc(x_37); +lean_dec(x_1); +x_38 = lean_unsigned_to_nat(0u); +x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3(x_36, x_37, lean_box(0), x_38, x_3); +lean_dec(x_37); +lean_dec(x_36); +return x_39; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint64_t x_3; size_t x_4; lean_object* x_5; +x_3 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_2); +x_4 = lean_uint64_to_usize(x_3); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2(x_1, x_4, x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_13, 9); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_ctor_get(x_14, 2); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1(x_15, x_1); +lean_ctor_set(x_11, 0, x_16); +return x_11; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_11, 0); +x_18 = lean_ctor_get(x_11, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_11); +x_19 = lean_ctor_get(x_17, 9); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_ctor_get(x_19, 2); +lean_inc(x_20); +lean_dec(x_19); +x_21 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1(x_20, x_1); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_18); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__3(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2(x_1, x_4, x_3); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_assertTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_12 = l_Lean_Meta_mkOfEqTrue(x_2, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_ctor_get(x_1, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_1, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_1, 2); +lean_inc(x_17); +lean_dec(x_1); +x_18 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_15, x_16, x_17, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_18; +} +else +{ +uint8_t x_19; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) +{ +return x_12; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_12, 0); +x_21 = lean_ctor_get(x_12, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_12); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_assertFalse(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_ctor_get(x_13, 0); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse(x_15, x_1, x_2); +x_17 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg(x_1); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +x_20 = lean_ctor_get(x_17, 2); +lean_inc(x_20); +lean_dec(x_17); +x_21 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_18, x_19, x_20, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_21; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_1); +x_12 = l_Lean_Meta_Grind_isEqFalse(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_unbox(x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +uint8_t x_15; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_15 = !lean_is_exclusive(x_12); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_12, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_12, 0, x_17); +return x_12; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_dec(x_12); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_12, 1); +lean_inc(x_21); +lean_dec(x_12); +x_22 = l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_24 = !lean_is_exclusive(x_22); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 0); +lean_dec(x_25); +x_26 = lean_box(0); +lean_ctor_set(x_22, 0, x_26); +return x_22; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_22, 1); +lean_inc(x_27); +lean_dec(x_22); +x_28 = lean_box(0); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_22, 1); +lean_inc(x_30); +lean_dec(x_22); +x_31 = lean_ctor_get(x_23, 0); +lean_inc(x_31); +lean_dec(x_23); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_32 = l_Lean_Meta_Grind_mkEqFalseProof(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_30); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = l_Lean_Meta_Grind_Arith_Offset_assertFalse(x_31, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +return x_35; +} +else +{ +uint8_t x_36; +lean_dec(x_31); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_36 = !lean_is_exclusive(x_32); +if (x_36 == 0) +{ +return x_32; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_32, 0); +x_38 = lean_ctor_get(x_32, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_32); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +} +} +else +{ +uint8_t x_40; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_40 = !lean_is_exclusive(x_12); +if (x_40 == 0) +{ +return x_12; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_12, 0); +x_42 = lean_ctor_get(x_12, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_12); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +lean_inc(x_1); +x_11 = l_Lean_Meta_Grind_isEqTrue(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; uint8_t x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_unbox(x_12); +lean_dec(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = lean_box(0); +x_16 = l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(x_1, x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_11, 1); +lean_inc(x_17); +lean_dec(x_11); +x_18 = l_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_box(0); +x_22 = l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(x_1, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_18, 1); +lean_inc(x_23); +lean_dec(x_18); +x_24 = lean_ctor_get(x_19, 0); +lean_inc(x_24); +lean_dec(x_19); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_25 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_28 = l_Lean_Meta_Grind_Arith_Offset_assertTrue(x_24, x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(x_1, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); +lean_dec(x_29); +return x_31; +} +else +{ +uint8_t x_32; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_32 = !lean_is_exclusive(x_28); +if (x_32 == 0) +{ +return x_28; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_28, 0); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_28); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +} +else +{ +uint8_t x_36; +lean_dec(x_24); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_25); +if (x_36 == 0) +{ +return x_25; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_25, 0); +x_38 = lean_ctor_get(x_25, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_25); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +} +} +else +{ +uint8_t x_40; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_40 = !lean_is_exclusive(x_11); +if (x_40 == 0) +{ +return x_11; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_11, 0); +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_11); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_propagateLE___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Meta_Grind_Arith_propagateLE___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; +} +} +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("LE", 2, 2); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le", 2, 2); +return x_1; +} +} +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1; +x_2 = l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_propagateLE), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396_(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_2 = l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3; +x_3 = 0; +x_4 = l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4; +x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); +return x_5; +} +} +lean_object* initialize_Lean_Meta_Tactic_Grind_PropagatorAttr(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Offset(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Main(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Tactic_Grind_PropagatorAttr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__1 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__1(); +l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2 = _init_l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_isCnstr_x3f___spec__2___closed__2(); +l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__1); +l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2 = _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__2); +l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3 = _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__3); +l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4 = _init_l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396____closed__4); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_Arith_propagateLE_declare__1____x40_Lean_Meta_Tactic_Grind_Arith_Main___hyg_396_(lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +}return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Model.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Model.c new file mode 100644 index 000000000000..775e38a44c0e --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Model.c @@ -0,0 +1,1702 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Model +// Imports: Lean.Meta.Basic Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Util +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3(lean_object*, lean_object*, lean_object*); +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* lean_mk_array(lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3; +lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4; +uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_1294____spec__1(lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2; +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1; +lean_object* lean_nat_to_int(lean_object*); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2; +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_outOfBounds___rarg(lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_isNatOffset_x3f(lean_object*); +extern lean_object* l_Lean_instInhabitedExpr; +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_int_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkModel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1; +lean_object* l_Int_toNat(lean_object*); +lean_object* lean_panic_fn(lean_object*, lean_object*); +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); +size_t lean_usize_add(size_t, size_t); +static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5; +lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_int_add(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f(lean_object*); +lean_object* lean_array_get_size(lean_object*); +static lean_object* l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1; +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1; +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_ctor_get(x_3, 1); +x_6 = lean_ctor_get(x_3, 2); +x_7 = lean_box(0); +x_8 = lean_array_get_size(x_1); +x_9 = lean_nat_dec_lt(x_4, x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_outOfBounds___rarg(x_7); +if (lean_obj_tag(x_10) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +x_14 = lean_int_sub(x_13, x_5); +lean_dec(x_13); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_10, 0, x_14); +x_2 = x_10; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_16; uint8_t x_17; +lean_free_object(x_10); +x_16 = lean_ctor_get(x_2, 0); +lean_inc(x_16); +x_17 = lean_int_dec_lt(x_16, x_14); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_dec(x_14); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_2); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_2, 0); +lean_dec(x_20); +lean_ctor_set(x_2, 0, x_14); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_14); +x_2 = x_22; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_10, 0); +lean_inc(x_24); +lean_dec(x_10); +x_25 = lean_int_sub(x_24, x_5); +lean_dec(x_24); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_26; +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_2 = x_26; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +x_29 = lean_int_dec_lt(x_28, x_25); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_dec(x_25); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_31; lean_object* x_32; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_31 = x_2; +} else { + lean_dec_ref(x_2); + x_31 = lean_box(0); +} +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 1, 0); +} else { + x_32 = x_31; +} +lean_ctor_set(x_32, 0, x_25); +x_2 = x_32; +x_3 = x_6; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_34; +x_34 = lean_array_fget(x_1, x_4); +if (lean_obj_tag(x_34) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 0); +x_38 = lean_int_sub(x_37, x_5); +lean_dec(x_37); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_34, 0, x_38); +x_2 = x_34; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_40; uint8_t x_41; +lean_free_object(x_34); +x_40 = lean_ctor_get(x_2, 0); +lean_inc(x_40); +x_41 = lean_int_dec_lt(x_40, x_38); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_dec(x_38); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_2); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_ctor_get(x_2, 0); +lean_dec(x_44); +lean_ctor_set(x_2, 0, x_38); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_46; +lean_dec(x_2); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_38); +x_2 = x_46; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_34, 0); +lean_inc(x_48); +lean_dec(x_34); +x_49 = lean_int_sub(x_48, x_5); +lean_dec(x_48); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_50; +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_2 = x_50; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_52; uint8_t x_53; +x_52 = lean_ctor_get(x_2, 0); +lean_inc(x_52); +x_53 = lean_int_dec_lt(x_52, x_49); +lean_dec(x_52); +if (x_53 == 0) +{ +lean_dec(x_49); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_55; lean_object* x_56; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_55 = x_2; +} else { + lean_dec_ref(x_2); + x_55 = lean_box(0); +} +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 1, 0); +} else { + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_49); +x_2 = x_56; +x_3 = x_6; +goto _start; +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_ctor_get(x_3, 1); +x_6 = lean_ctor_get(x_3, 2); +x_7 = lean_box(0); +x_8 = lean_array_get_size(x_1); +x_9 = lean_nat_dec_lt(x_4, x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_outOfBounds___rarg(x_7); +if (lean_obj_tag(x_10) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +x_14 = lean_int_add(x_13, x_5); +lean_dec(x_13); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_10, 0, x_14); +x_2 = x_10; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_16; uint8_t x_17; +lean_free_object(x_10); +x_16 = lean_ctor_get(x_2, 0); +lean_inc(x_16); +x_17 = lean_int_dec_lt(x_14, x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_dec(x_14); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_2); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_2, 0); +lean_dec(x_20); +lean_ctor_set(x_2, 0, x_14); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_14); +x_2 = x_22; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_10, 0); +lean_inc(x_24); +lean_dec(x_10); +x_25 = lean_int_add(x_24, x_5); +lean_dec(x_24); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_26; +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_2 = x_26; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +x_29 = lean_int_dec_lt(x_25, x_28); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_dec(x_25); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_31; lean_object* x_32; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_31 = x_2; +} else { + lean_dec_ref(x_2); + x_31 = lean_box(0); +} +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 1, 0); +} else { + x_32 = x_31; +} +lean_ctor_set(x_32, 0, x_25); +x_2 = x_32; +x_3 = x_6; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_34; +x_34 = lean_array_fget(x_1, x_4); +if (lean_obj_tag(x_34) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 0); +x_38 = lean_int_add(x_37, x_5); +lean_dec(x_37); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_34, 0, x_38); +x_2 = x_34; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_40; uint8_t x_41; +lean_free_object(x_34); +x_40 = lean_ctor_get(x_2, 0); +lean_inc(x_40); +x_41 = lean_int_dec_lt(x_38, x_40); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_dec(x_38); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_2); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_ctor_get(x_2, 0); +lean_dec(x_44); +lean_ctor_set(x_2, 0, x_38); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_46; +lean_dec(x_2); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_38); +x_2 = x_46; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_34, 0); +lean_inc(x_48); +lean_dec(x_34); +x_49 = lean_int_add(x_48, x_5); +lean_dec(x_48); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_50; +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_2 = x_50; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_52; uint8_t x_53; +x_52 = lean_ctor_get(x_2, 0); +lean_inc(x_52); +x_53 = lean_int_dec_lt(x_49, x_52); +lean_dec(x_52); +if (x_53 == 0) +{ +lean_dec(x_49); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_55; lean_object* x_56; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_55 = x_2; +} else { + lean_dec_ref(x_2); + x_55 = lean_box(0); +} +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 1, 0); +} else { + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_49); +x_2 = x_56; +x_3 = x_6; +goto _start; +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_4 = lean_ctor_get(x_3, 0); +x_5 = lean_ctor_get(x_3, 1); +x_6 = lean_ctor_get(x_3, 2); +x_7 = lean_box(0); +x_8 = lean_array_get_size(x_1); +x_9 = lean_nat_dec_lt(x_4, x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_outOfBounds___rarg(x_7); +if (lean_obj_tag(x_10) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_10); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_10, 0); +x_14 = lean_int_add(x_13, x_5); +lean_dec(x_13); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_10, 0, x_14); +x_2 = x_10; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_16; uint8_t x_17; +lean_free_object(x_10); +x_16 = lean_ctor_get(x_2, 0); +lean_inc(x_16); +x_17 = lean_int_dec_lt(x_14, x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_dec(x_14); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_2); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = lean_ctor_get(x_2, 0); +lean_dec(x_20); +lean_ctor_set(x_2, 0, x_14); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_22; +lean_dec(x_2); +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_14); +x_2 = x_22; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_10, 0); +lean_inc(x_24); +lean_dec(x_10); +x_25 = lean_int_add(x_24, x_5); +lean_dec(x_24); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_26; +x_26 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_26, 0, x_25); +x_2 = x_26; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_2, 0); +lean_inc(x_28); +x_29 = lean_int_dec_lt(x_25, x_28); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_dec(x_25); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_31; lean_object* x_32; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_31 = x_2; +} else { + lean_dec_ref(x_2); + x_31 = lean_box(0); +} +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 1, 0); +} else { + x_32 = x_31; +} +lean_ctor_set(x_32, 0, x_25); +x_2 = x_32; +x_3 = x_6; +goto _start; +} +} +} +} +} +else +{ +lean_object* x_34; +x_34 = lean_array_fget(x_1, x_4); +if (lean_obj_tag(x_34) == 0) +{ +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_36; +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 0); +x_38 = lean_int_add(x_37, x_5); +lean_dec(x_37); +if (lean_obj_tag(x_2) == 0) +{ +lean_ctor_set(x_34, 0, x_38); +x_2 = x_34; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_40; uint8_t x_41; +lean_free_object(x_34); +x_40 = lean_ctor_get(x_2, 0); +lean_inc(x_40); +x_41 = lean_int_dec_lt(x_38, x_40); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_dec(x_38); +x_3 = x_6; +goto _start; +} +else +{ +uint8_t x_43; +x_43 = !lean_is_exclusive(x_2); +if (x_43 == 0) +{ +lean_object* x_44; +x_44 = lean_ctor_get(x_2, 0); +lean_dec(x_44); +lean_ctor_set(x_2, 0, x_38); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_46; +lean_dec(x_2); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_38); +x_2 = x_46; +x_3 = x_6; +goto _start; +} +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; +x_48 = lean_ctor_get(x_34, 0); +lean_inc(x_48); +lean_dec(x_34); +x_49 = lean_int_add(x_48, x_5); +lean_dec(x_48); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_50; +x_50 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_50, 0, x_49); +x_2 = x_50; +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_52; uint8_t x_53; +x_52 = lean_ctor_get(x_2, 0); +lean_inc(x_52); +x_53 = lean_int_dec_lt(x_49, x_52); +lean_dec(x_52); +if (x_53 == 0) +{ +lean_dec(x_49); +x_3 = x_6; +goto _start; +} +else +{ +lean_object* x_55; lean_object* x_56; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + x_55 = x_2; +} else { + lean_dec_ref(x_2); + x_55 = lean_box(0); +} +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(1, 1, 0); +} else { + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_49); +x_2 = x_56; +x_3 = x_6; +goto _start; +} +} +} +} +} +} +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_4, 1); +x_15 = lean_nat_dec_lt(x_6, x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_6); +lean_dec(x_2); +lean_dec(x_1); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_13); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_17 = lean_box(0); +x_18 = lean_ctor_get(x_1, 4); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 2); +lean_inc(x_19); +x_20 = lean_nat_dec_lt(x_6, x_19); +lean_dec(x_19); +x_21 = lean_ctor_get(x_1, 5); +lean_inc(x_21); +x_22 = lean_ctor_get(x_21, 2); +lean_inc(x_22); +x_23 = lean_nat_dec_lt(x_6, x_22); +lean_dec(x_22); +if (x_20 == 0) +{ +lean_object* x_63; +lean_dec(x_18); +x_63 = l_outOfBounds___rarg(x_17); +x_24 = x_63; +goto block_62; +} +else +{ +lean_object* x_64; +x_64 = l_Lean_PersistentArray_get_x21___rarg(x_17, x_18, x_6); +x_24 = x_64; +goto block_62; +} +block_62: +{ +lean_object* x_25; +lean_inc(x_2); +x_25 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1(x_5, x_2, x_24); +lean_dec(x_24); +if (x_23 == 0) +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_21); +x_26 = l_outOfBounds___rarg(x_17); +x_27 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2(x_5, x_25, x_26); +lean_dec(x_26); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2; +x_29 = lean_array_set(x_5, x_6, x_28); +x_30 = lean_ctor_get(x_4, 2); +x_31 = lean_nat_add(x_6, x_30); +lean_dec(x_6); +x_5 = x_29; +x_6 = x_31; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +else +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_27); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_array_set(x_5, x_6, x_27); +x_35 = lean_ctor_get(x_4, 2); +x_36 = lean_nat_add(x_6, x_35); +lean_dec(x_6); +x_5 = x_34; +x_6 = x_36; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_38 = lean_ctor_get(x_27, 0); +lean_inc(x_38); +lean_dec(x_27); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_38); +x_40 = lean_array_set(x_5, x_6, x_39); +x_41 = lean_ctor_get(x_4, 2); +x_42 = lean_nat_add(x_6, x_41); +lean_dec(x_6); +x_5 = x_40; +x_6 = x_42; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +} +} +else +{ +lean_object* x_44; lean_object* x_45; +x_44 = l_Lean_PersistentArray_get_x21___rarg(x_17, x_21, x_6); +x_45 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3(x_5, x_25, x_44); +lean_dec(x_44); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_46 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2; +x_47 = lean_array_set(x_5, x_6, x_46); +x_48 = lean_ctor_get(x_4, 2); +x_49 = lean_nat_add(x_6, x_48); +lean_dec(x_6); +x_5 = x_47; +x_6 = x_49; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +else +{ +uint8_t x_51; +x_51 = !lean_is_exclusive(x_45); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_array_set(x_5, x_6, x_45); +x_53 = lean_ctor_get(x_4, 2); +x_54 = lean_nat_add(x_6, x_53); +lean_dec(x_6); +x_5 = x_52; +x_6 = x_54; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_56 = lean_ctor_get(x_45, 0); +lean_inc(x_56); +lean_dec(x_45); +x_57 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_57, 0, x_56); +x_58 = lean_array_set(x_5, x_6, x_57); +x_59 = lean_ctor_get(x_4, 2); +x_60 = lean_nat_add(x_6, x_59); +lean_dec(x_6); +x_5 = x_58; +x_6 = x_60; +x_7 = lean_box(0); +x_8 = lean_box(0); +goto _start; +} +} +} +} +} +} +} +static lean_object* _init_l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_instInhabitedMetaM___boxed), 5, 1); +lean_closure_set(x_1, 0, lean_box(0)); +return x_1; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1; +x_8 = lean_panic_fn(x_7, x_1); +x_9 = lean_apply_5(x_8, x_2, x_3, x_4, x_5, x_6); +return x_9; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.Grind.Arith.Model", 34, 34); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.mkModel", 36, 36); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); +return x_1; +} +} +static lean_object* _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2; +x_2 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3; +x_3 = lean_unsigned_to_nat(35u); +x_4 = lean_unsigned_to_nat(30u); +x_5 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_ctor_get(x_7, 1); +x_18 = lean_nat_dec_lt(x_9, x_17); +if (x_18 == 0) +{ +lean_object* x_19; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_1); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_8); +lean_ctor_set(x_19, 1, x_16); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_27; lean_object* x_58; uint8_t x_59; +x_58 = lean_box(0); +x_59 = lean_nat_dec_lt(x_9, x_5); +if (x_59 == 0) +{ +lean_object* x_60; +x_60 = l_outOfBounds___rarg(x_58); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; +x_61 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_62 = l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5(x_61, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_62) == 0) +{ +lean_object* x_63; lean_object* x_64; +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +lean_dec(x_62); +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_8); +x_20 = x_64; +x_21 = x_63; +goto block_26; +} +else +{ +uint8_t x_65; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_65 = !lean_is_exclusive(x_62); +if (x_65 == 0) +{ +return x_62; +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_62, 0); +x_67 = lean_ctor_get(x_62, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_62); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; +} +} +} +else +{ +lean_object* x_69; +x_69 = lean_ctor_get(x_60, 0); +lean_inc(x_69); +lean_dec(x_60); +x_27 = x_69; +goto block_57; +} +} +else +{ +lean_object* x_70; +x_70 = lean_array_fget(x_4, x_9); +if (lean_obj_tag(x_70) == 0) +{ +lean_object* x_71; lean_object* x_72; +x_71 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_72 = l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5(x_71, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +lean_dec(x_72); +x_74 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_74, 0, x_8); +x_20 = x_74; +x_21 = x_73; +goto block_26; +} +else +{ +uint8_t x_75; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_75 = !lean_is_exclusive(x_72); +if (x_75 == 0) +{ +return x_72; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_72, 0); +x_77 = lean_ctor_get(x_72, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_72); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; +} +} +} +else +{ +lean_object* x_79; +x_79 = lean_ctor_get(x_70, 0); +lean_inc(x_79); +lean_dec(x_70); +x_27 = x_79; +goto block_57; +} +} +block_26: +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_ctor_get(x_7, 2); +x_24 = lean_nat_add(x_9, x_23); +lean_dec(x_9); +x_8 = x_22; +x_9 = x_24; +x_10 = lean_box(0); +x_11 = lean_box(0); +x_16 = x_21; +goto _start; +} +block_57: +{ +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_int_sub(x_27, x_6); +lean_dec(x_27); +x_29 = l_Int_toNat(x_28); +lean_dec(x_28); +x_30 = lean_nat_dec_lt(x_9, x_2); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = l_Lean_instInhabitedExpr; +x_32 = l_outOfBounds___rarg(x_31); +lean_inc(x_32); +x_33 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; uint8_t x_36; +lean_inc(x_32); +x_34 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_32); +x_35 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1; +x_36 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_1294____spec__1(x_34, x_35); +lean_dec(x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_32); +lean_ctor_set(x_37, 1, x_29); +x_38 = lean_array_push(x_8, x_37); +x_39 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_39, 0, x_38); +x_20 = x_39; +x_21 = x_16; +goto block_26; +} +else +{ +lean_object* x_40; +lean_dec(x_32); +lean_dec(x_29); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_8); +x_20 = x_40; +x_21 = x_16; +goto block_26; +} +} +else +{ +uint8_t x_41; +lean_dec(x_32); +lean_dec(x_29); +x_41 = !lean_is_exclusive(x_33); +if (x_41 == 0) +{ +lean_object* x_42; +x_42 = lean_ctor_get(x_33, 0); +lean_dec(x_42); +lean_ctor_set(x_33, 0, x_8); +x_20 = x_33; +x_21 = x_16; +goto block_26; +} +else +{ +lean_object* x_43; +lean_dec(x_33); +x_43 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_43, 0, x_8); +x_20 = x_43; +x_21 = x_16; +goto block_26; +} +} +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = l_Lean_instInhabitedExpr; +lean_inc(x_1); +x_45 = l_Lean_PersistentArray_get_x21___rarg(x_44, x_1, x_9); +lean_inc(x_45); +x_46 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_45); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; uint8_t x_49; +lean_inc(x_45); +x_47 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_45); +x_48 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1; +x_49 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Meta_Basic_0__Lean_Meta_beqInfoCacheKey____x40_Lean_Meta_Basic___hyg_1294____spec__1(x_47, x_48); +lean_dec(x_47); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_45); +lean_ctor_set(x_50, 1, x_29); +x_51 = lean_array_push(x_8, x_50); +x_52 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_52, 0, x_51); +x_20 = x_52; +x_21 = x_16; +goto block_26; +} +else +{ +lean_object* x_53; +lean_dec(x_45); +lean_dec(x_29); +x_53 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_53, 0, x_8); +x_20 = x_53; +x_21 = x_16; +goto block_26; +} +} +else +{ +uint8_t x_54; +lean_dec(x_45); +lean_dec(x_29); +x_54 = !lean_is_exclusive(x_46); +if (x_54 == 0) +{ +lean_object* x_55; +x_55 = lean_ctor_get(x_46, 0); +lean_dec(x_55); +lean_ctor_set(x_46, 0, x_8); +x_20 = x_46; +x_21 = x_16; +goto block_26; +} +else +{ +lean_object* x_56; +lean_dec(x_46); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_8); +x_20 = x_56; +x_21 = x_16; +goto block_26; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_eq(x_2, x_3); +if (x_5 == 0) +{ +lean_object* x_6; size_t x_7; size_t x_8; +x_6 = lean_array_uget(x_1, x_2); +x_7 = 1; +x_8 = lean_usize_add(x_2, x_7); +if (lean_obj_tag(x_6) == 0) +{ +x_2 = x_8; +goto _start; +} +else +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_ctor_get(x_6, 0); +lean_inc(x_10); +lean_dec(x_6); +x_11 = lean_int_dec_lt(x_10, x_4); +if (x_11 == 0) +{ +lean_dec(x_10); +x_2 = x_8; +goto _start; +} +else +{ +lean_dec(x_4); +x_2 = x_8; +x_4 = x_10; +goto _start; +} +} +} +else +{ +return x_4; +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkModel(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_7 = lean_ctor_get(x_1, 9); +lean_inc(x_7); +lean_dec(x_1); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_8, 2); +lean_inc(x_9); +x_10 = lean_box(0); +lean_inc(x_9); +x_11 = lean_mk_array(x_9, x_10); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_unsigned_to_nat(1u); +lean_inc(x_9); +x_14 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_9); +lean_ctor_set(x_14, 2, x_13); +x_15 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4(x_7, x_10, x_14, x_14, x_11, x_12, lean_box(0), lean_box(0), x_2, x_3, x_4, x_5, x_6); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_array_get_size(x_16); +x_19 = lean_nat_dec_lt(x_12, x_18); +if (x_19 == 0) +{ +lean_object* x_32; +x_32 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1; +x_20 = x_32; +goto block_31; +} +else +{ +uint8_t x_33; +x_33 = lean_nat_dec_le(x_18, x_18); +if (x_33 == 0) +{ +lean_object* x_34; +x_34 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1; +x_20 = x_34; +goto block_31; +} +else +{ +size_t x_35; size_t x_36; lean_object* x_37; lean_object* x_38; +x_35 = 0; +x_36 = lean_usize_of_nat(x_18); +x_37 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1; +x_38 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7(x_16, x_35, x_36, x_37); +x_20 = x_38; +goto block_31; +} +} +block_31: +{ +lean_object* x_21; lean_object* x_22; +x_21 = l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1; +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6(x_8, x_9, x_14, x_16, x_18, x_20, x_14, x_21, x_12, lean_box(0), lean_box(0), x_2, x_3, x_4, x_5, x_17); +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_14); +lean_dec(x_9); +if (lean_obj_tag(x_22) == 0) +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +return x_22; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_22); +if (x_27 == 0) +{ +return x_22; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_22, 0); +x_29 = lean_ctor_get(x_22, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_22); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__1(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__2(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_AssocList_foldlM___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__3(x_1, x_2, x_3); +lean_dec(x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; +x_17 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_17; +} +} +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__7(x_1, x_5, x_6, x_4); +lean_dec(x_1); +return x_7; +} +} +lean_object* initialize_Lean_Meta_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Util(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Model(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Meta_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Types(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Util(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__1); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__4___closed__2); +l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1 = _init_l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1(); +lean_mark_persistent(l_panic___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__5___closed__1); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__1); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__2); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__3); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__4); +l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5 = _init_l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5(); +lean_mark_persistent(l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_mkModel___spec__6___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkModel___closed__1); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Offset.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Offset.c new file mode 100644 index 000000000000..f436b631a00c --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Offset.c @@ -0,0 +1,19994 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Offset +// Imports: Init.Grind.Offset Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Arith.ProofUtil +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* lean_process_new_offset_eq_lit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2; +lean_object* l_Lean_mkNatLit(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +size_t lean_usize_shift_right(size_t, size_t); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getZeroNode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1; +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_usize_dec_le(size_t, size_t); +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5; +uint64_t lean_uint64_of_nat(lean_object*); +lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); +LEAN_EXPORT lean_object* lean_process_new_offset_eq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_uint64_to_usize(uint64_t); +uint64_t lean_uint64_lor(uint64_t, uint64_t); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7; +size_t lean_usize_mul(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4; +lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static uint64_t l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2; +lean_object* l_Lean_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_checkInvariants(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_int_dec_le(lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_instInhabitedPUnit; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1; +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5; +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___spec__1(lean_object*); +size_t lean_usize_of_nat(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4; +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge_update___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_take(lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_shift_right(uint64_t, uint64_t); +lean_object* lean_nat_to_int(lean_object*); +uint8_t l_Lean_Expr_isEq(lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_get_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l___private_Lean_Expr_0__Lean_natAddFn; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3; +lean_object* l_Lean_Meta_Grind_closeGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5; +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_Meta_check(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5; +lean_object* l_outOfBounds___rarg(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +lean_object* lean_st_ref_get(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_isNatOffset_x3f(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1; +extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +lean_object* l_Lean_Meta_Grind_pushEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_markAsOffsetTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2; +static double l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2; +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l___private_Lean_Expr_0__Lean_natLEPred; +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +extern lean_object* l_Lean_Meta_instMonadMetaM; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2; +lean_object* lean_usize_to_nat(size_t); +LEAN_EXPORT lean_object* l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3; +lean_object* l_Lean_MessageData_ofExpr(lean_object*); +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3; +lean_object* lean_grind_mk_eq_proof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6; +lean_object* lean_nat_abs(lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4; +LEAN_EXPORT lean_object* l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent___boxed(lean_object*); +lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4; +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent(lean_object*); +lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1___boxed(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3; +lean_object* l_Lean_indentExpr(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Int_toNat(lean_object*); +lean_object* lean_panic_fn(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_isEqv(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(lean_object*, lean_object*); +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2; +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t lean_uint64_shift_left(uint64_t, uint64_t); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__5(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__2(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2; +lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_modify_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1; +lean_object* l_List_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_sub(size_t, size_t); +lean_object* lean_array_mk(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_isEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_pushEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Meta_Grind_Arith_isNatAdd(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6(lean_object*, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object*); +size_t lean_usize_add(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_modify_x27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_int_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_traceDists(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2; +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8; +lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +size_t lean_usize_shift_left(size_t, size_t); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_int_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__8(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_get_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(lean_object*, lean_object*); +lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_int_neg(lean_object*); +lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t lean_nat_dec_le(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5; +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1; +uint64_t l_Lean_Meta_TransparencyMode_toUInt64(uint8_t); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_nat_add(lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4; +LEAN_EXPORT lean_object* l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +extern lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge_update(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3; +lean_object* l_ReaderT_instMonad___rarg(lean_object*); +size_t lean_usize_land(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_traceDists___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_get_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_12, 9); +lean_inc(x_13); +lean_dec(x_12); +lean_ctor_set(x_10, 0, x_13); +return x_10; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_10); +x_16 = lean_ctor_get(x_14, 9); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_get_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_modify_x27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_st_ref_take(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_12, 9); +x_16 = lean_apply_1(x_1, x_15); +lean_ctor_set(x_12, 9, x_16); +x_17 = lean_st_ref_set(x_2, x_12, x_13); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +x_20 = lean_box(0); +lean_ctor_set(x_17, 0, x_20); +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; +} +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_24 = lean_ctor_get(x_12, 0); +x_25 = lean_ctor_get(x_12, 1); +x_26 = lean_ctor_get(x_12, 2); +x_27 = lean_ctor_get(x_12, 3); +x_28 = lean_ctor_get(x_12, 4); +x_29 = lean_ctor_get(x_12, 5); +x_30 = lean_ctor_get(x_12, 6); +x_31 = lean_ctor_get_uint8(x_12, sizeof(void*)*23); +x_32 = lean_ctor_get(x_12, 7); +x_33 = lean_ctor_get(x_12, 8); +x_34 = lean_ctor_get(x_12, 9); +x_35 = lean_ctor_get(x_12, 10); +x_36 = lean_ctor_get(x_12, 11); +x_37 = lean_ctor_get(x_12, 12); +x_38 = lean_ctor_get(x_12, 13); +x_39 = lean_ctor_get(x_12, 14); +x_40 = lean_ctor_get(x_12, 15); +x_41 = lean_ctor_get(x_12, 16); +x_42 = lean_ctor_get(x_12, 17); +x_43 = lean_ctor_get(x_12, 18); +x_44 = lean_ctor_get(x_12, 19); +x_45 = lean_ctor_get(x_12, 20); +x_46 = lean_ctor_get(x_12, 21); +x_47 = lean_ctor_get(x_12, 22); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_12); +x_48 = lean_apply_1(x_1, x_34); +x_49 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_49, 0, x_24); +lean_ctor_set(x_49, 1, x_25); +lean_ctor_set(x_49, 2, x_26); +lean_ctor_set(x_49, 3, x_27); +lean_ctor_set(x_49, 4, x_28); +lean_ctor_set(x_49, 5, x_29); +lean_ctor_set(x_49, 6, x_30); +lean_ctor_set(x_49, 7, x_32); +lean_ctor_set(x_49, 8, x_33); +lean_ctor_set(x_49, 9, x_48); +lean_ctor_set(x_49, 10, x_35); +lean_ctor_set(x_49, 11, x_36); +lean_ctor_set(x_49, 12, x_37); +lean_ctor_set(x_49, 13, x_38); +lean_ctor_set(x_49, 14, x_39); +lean_ctor_set(x_49, 15, x_40); +lean_ctor_set(x_49, 16, x_41); +lean_ctor_set(x_49, 17, x_42); +lean_ctor_set(x_49, 18, x_43); +lean_ctor_set(x_49, 19, x_44); +lean_ctor_set(x_49, 20, x_45); +lean_ctor_set(x_49, 21, x_46); +lean_ctor_set(x_49, 22, x_47); +lean_ctor_set_uint8(x_49, sizeof(void*)*23, x_31); +x_50 = lean_st_ref_set(x_2, x_49, x_13); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_52 = x_50; +} else { + lean_dec_ref(x_50); + x_52 = lean_box(0); +} +x_53 = lean_box(0); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); +} else { + x_54 = x_52; +} +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_modify_x27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_Arith_Offset_modify_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_array_get_size(x_2); +x_8 = lean_nat_dec_lt(x_5, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +lean_dec(x_5); +return x_6; +} +else +{ +lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_9 = lean_array_fget(x_2, x_5); +x_10 = lean_array_fget(x_3, x_5); +x_11 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_9); +x_12 = lean_uint64_to_usize(x_11); +x_13 = 1; +x_14 = lean_usize_sub(x_1, x_13); +x_15 = 5; +x_16 = lean_usize_mul(x_15, x_14); +x_17 = lean_usize_shift_right(x_12, x_16); +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_add(x_5, x_18); +lean_dec(x_5); +x_20 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_6, x_17, x_1, x_9, x_10); +x_4 = lean_box(0); +x_5 = x_19; +x_6 = x_20; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_5); +x_8 = lean_nat_dec_lt(x_2, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +uint8_t x_9; +lean_dec(x_2); +x_9 = !lean_is_exclusive(x_1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 1); +lean_dec(x_10); +x_11 = lean_ctor_get(x_1, 0); +lean_dec(x_11); +x_12 = lean_array_push(x_5, x_3); +x_13 = lean_array_push(x_6, x_4); +lean_ctor_set(x_1, 1, x_13); +lean_ctor_set(x_1, 0, x_12); +return x_1; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_14 = lean_array_push(x_5, x_3); +x_15 = lean_array_push(x_6, x_4); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +else +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_fget(x_5, x_2); +x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_6); +lean_dec(x_5); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_add(x_2, x_19); +lean_dec(x_2); +x_2 = x_20; +goto _start; +} +else +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = lean_ctor_get(x_1, 0); +lean_dec(x_24); +x_25 = lean_array_fset(x_5, x_2, x_3); +x_26 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +lean_ctor_set(x_1, 1, x_26); +lean_ctor_set(x_1, 0, x_25); +return x_1; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_array_fset(x_5, x_2, x_3); +x_28 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +} +static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__1() { +_start: +{ +size_t x_1; size_t x_2; size_t x_3; +x_1 = 1; +x_2 = 5; +x_3 = lean_usize_shift_left(x_1, x_2); +return x_3; +} +} +static size_t _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2() { +_start: +{ +size_t x_1; size_t x_2; size_t x_3; +x_1 = 1; +x_2 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__1; +x_3 = lean_usize_sub(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntries(lean_box(0), lean_box(0)); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_1); +if (x_6 == 0) +{ +lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_7 = lean_ctor_get(x_1, 0); +x_8 = 1; +x_9 = 5; +x_10 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_11 = lean_usize_land(x_2, x_10); +x_12 = lean_usize_to_nat(x_11); +x_13 = lean_array_get_size(x_7); +x_14 = lean_nat_dec_lt(x_12, x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_dec(x_12); +lean_dec(x_5); +lean_dec(x_4); +return x_1; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_array_fget(x_7, x_12); +x_16 = lean_box(0); +x_17 = lean_array_fset(x_7, x_12, x_16); +switch (lean_obj_tag(x_15)) { +case 0: +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_free_object(x_15); +x_22 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_array_fset(x_17, x_12, x_23); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_24); +return x_1; +} +else +{ +lean_object* x_25; +lean_dec(x_20); +lean_dec(x_19); +lean_ctor_set(x_15, 1, x_5); +lean_ctor_set(x_15, 0, x_4); +x_25 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_25); +return x_1; +} +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_15, 0); +x_27 = lean_ctor_get(x_15, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_15); +x_28 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_26, x_27, x_4, x_5); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_array_fset(x_17, x_12, x_30); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_31); +return x_1; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_27); +lean_dec(x_26); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_4); +lean_ctor_set(x_32, 1, x_5); +x_33 = lean_array_fset(x_17, x_12, x_32); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_33); +return x_1; +} +} +} +case 1: +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_15); +if (x_34 == 0) +{ +lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_15, 0); +x_36 = lean_usize_shift_right(x_2, x_9); +x_37 = lean_usize_add(x_3, x_8); +x_38 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_35, x_36, x_37, x_4, x_5); +lean_ctor_set(x_15, 0, x_38); +x_39 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_39); +return x_1; +} +else +{ +lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_15, 0); +lean_inc(x_40); +lean_dec(x_15); +x_41 = lean_usize_shift_right(x_2, x_9); +x_42 = lean_usize_add(x_3, x_8); +x_43 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_40, x_41, x_42, x_4, x_5); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = lean_array_fset(x_17, x_12, x_44); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_45); +return x_1; +} +} +default: +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_4); +lean_ctor_set(x_46, 1, x_5); +x_47 = lean_array_fset(x_17, x_12, x_46); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_47); +return x_1; +} +} +} +} +else +{ +lean_object* x_48; size_t x_49; size_t x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_48 = lean_ctor_get(x_1, 0); +lean_inc(x_48); +lean_dec(x_1); +x_49 = 1; +x_50 = 5; +x_51 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_52 = lean_usize_land(x_2, x_51); +x_53 = lean_usize_to_nat(x_52); +x_54 = lean_array_get_size(x_48); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_5); +lean_dec(x_4); +x_56 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_56, 0, x_48); +return x_56; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_array_fget(x_48, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_48, x_53, x_58); +switch (lean_obj_tag(x_57)) { +case 0: +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = lean_ctor_get(x_57, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_57, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_62 = x_57; +} else { + lean_dec_ref(x_57); + x_62 = lean_box(0); +} +x_63 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_60); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_62); +x_64 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_60, x_61, x_4, x_5); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_array_fset(x_59, x_53, x_65); +lean_dec(x_53); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +return x_67; +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_dec(x_61); +lean_dec(x_60); +if (lean_is_scalar(x_62)) { + x_68 = lean_alloc_ctor(0, 2, 0); +} else { + x_68 = x_62; +} +lean_ctor_set(x_68, 0, x_4); +lean_ctor_set(x_68, 1, x_5); +x_69 = lean_array_fset(x_59, x_53, x_68); +lean_dec(x_53); +x_70 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_70, 0, x_69); +return x_70; +} +} +case 1: +{ +lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_71 = lean_ctor_get(x_57, 0); +lean_inc(x_71); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + x_72 = x_57; +} else { + lean_dec_ref(x_57); + x_72 = lean_box(0); +} +x_73 = lean_usize_shift_right(x_2, x_50); +x_74 = lean_usize_add(x_3, x_49); +x_75 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_71, x_73, x_74, x_4, x_5); +if (lean_is_scalar(x_72)) { + x_76 = lean_alloc_ctor(1, 1, 0); +} else { + x_76 = x_72; +} +lean_ctor_set(x_76, 0, x_75); +x_77 = lean_array_fset(x_59, x_53, x_76); +lean_dec(x_53); +x_78 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_78, 0, x_77); +return x_78; +} +default: +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_4); +lean_ctor_set(x_79, 1, x_5); +x_80 = lean_array_fset(x_59, x_53, x_79); +lean_dec(x_53); +x_81 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_81, 0, x_80); +return x_81; +} +} +} +} +} +else +{ +uint8_t x_82; +x_82 = !lean_is_exclusive(x_1); +if (x_82 == 0) +{ +lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; +x_83 = lean_unsigned_to_nat(0u); +x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__4(x_1, x_83, x_4, x_5); +x_85 = 7; +x_86 = lean_usize_dec_le(x_85, x_3); +if (x_86 == 0) +{ +lean_object* x_87; lean_object* x_88; uint8_t x_89; +x_87 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_84); +x_88 = lean_unsigned_to_nat(4u); +x_89 = lean_nat_dec_lt(x_87, x_88); +lean_dec(x_87); +if (x_89 == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_90 = lean_ctor_get(x_84, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_84, 1); +lean_inc(x_91); +lean_dec(x_84); +x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3(x_3, x_90, x_91, lean_box(0), x_83, x_92); +lean_dec(x_91); +lean_dec(x_90); +return x_93; +} +else +{ +return x_84; +} +} +else +{ +return x_84; +} +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; uint8_t x_100; +x_94 = lean_ctor_get(x_1, 0); +x_95 = lean_ctor_get(x_1, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_1); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_unsigned_to_nat(0u); +x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__4(x_96, x_97, x_4, x_5); +x_99 = 7; +x_100 = lean_usize_dec_le(x_99, x_3); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; uint8_t x_103; +x_101 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_98); +x_102 = lean_unsigned_to_nat(4u); +x_103 = lean_nat_dec_lt(x_101, x_102); +lean_dec(x_101); +if (x_103 == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_98, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +lean_dec(x_98); +x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3(x_3, x_104, x_105, lean_box(0), x_97, x_106); +lean_dec(x_105); +lean_dec(x_104); +return x_107; +} +else +{ +return x_98; +} +} +else +{ +return x_98; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint64_t x_4; size_t x_5; size_t x_6; lean_object* x_7; +x_4 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_2); +x_5 = lean_uint64_to_usize(x_4); +x_6 = 1; +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_1, x_5, x_6, x_2, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_lt(x_4, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; uint8_t x_10; +x_9 = lean_array_fget(x_1, x_4); +x_10 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_5, x_9); +lean_dec(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_unsigned_to_nat(1u); +x_12 = lean_nat_add(x_4, x_11); +lean_dec(x_4); +x_3 = lean_box(0); +x_4 = x_12; +goto _start; +} +else +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_array_fget(x_2, x_4); +lean_dec(x_4); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6(lean_object* x_1, size_t x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; size_t x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 0); +x_6 = 5; +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_8 = lean_usize_land(x_2, x_7); +x_9 = lean_usize_to_nat(x_8); +x_10 = lean_box(2); +x_11 = lean_array_get(x_10, x_5, x_9); +lean_dec(x_9); +lean_dec(x_5); +switch (lean_obj_tag(x_11)) { +case 0: +{ +lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_12); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; +lean_dec(x_13); +lean_free_object(x_1); +x_15 = lean_box(0); +return x_15; +} +else +{ +lean_ctor_set_tag(x_1, 1); +lean_ctor_set(x_1, 0, x_13); +return x_1; +} +} +case 1: +{ +lean_object* x_16; size_t x_17; +lean_free_object(x_1); +x_16 = lean_ctor_get(x_11, 0); +lean_inc(x_16); +lean_dec(x_11); +x_17 = lean_usize_shift_right(x_2, x_6); +x_1 = x_16; +x_2 = x_17; +goto _start; +} +default: +{ +lean_object* x_19; +lean_free_object(x_1); +x_19 = lean_box(0); +return x_19; +} +} +} +else +{ +lean_object* x_20; size_t x_21; size_t x_22; size_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_20 = lean_ctor_get(x_1, 0); +lean_inc(x_20); +lean_dec(x_1); +x_21 = 5; +x_22 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_23 = lean_usize_land(x_2, x_22); +x_24 = lean_usize_to_nat(x_23); +x_25 = lean_box(2); +x_26 = lean_array_get(x_25, x_20, x_24); +lean_dec(x_24); +lean_dec(x_20); +switch (lean_obj_tag(x_26)) { +case 0: +{ +lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_27); +lean_dec(x_27); +if (x_29 == 0) +{ +lean_object* x_30; +lean_dec(x_28); +x_30 = lean_box(0); +return x_30; +} +else +{ +lean_object* x_31; +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_28); +return x_31; +} +} +case 1: +{ +lean_object* x_32; size_t x_33; +x_32 = lean_ctor_get(x_26, 0); +lean_inc(x_32); +lean_dec(x_26); +x_33 = lean_usize_shift_right(x_2, x_21); +x_1 = x_32; +x_2 = x_33; +goto _start; +} +default: +{ +lean_object* x_35; +x_35 = lean_box(0); +return x_35; +} +} +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_1, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_1, 1); +lean_inc(x_37); +lean_dec(x_1); +x_38 = lean_unsigned_to_nat(0u); +x_39 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7(x_36, x_37, lean_box(0), x_38, x_3); +lean_dec(x_37); +lean_dec(x_36); +return x_39; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint64_t x_3; size_t x_4; lean_object* x_5; +x_3 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_2); +x_4 = lean_uint64_to_usize(x_3); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6(x_1, x_4, x_2); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_st_ref_take(x_4, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 9); +lean_inc(x_15); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_14, 9); +lean_dec(x_18); +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_20 = lean_ctor_get(x_15, 0); +x_21 = lean_ctor_get(x_15, 1); +x_22 = lean_ctor_get(x_15, 4); +x_23 = lean_ctor_get(x_15, 5); +x_24 = lean_ctor_get(x_15, 6); +lean_inc(x_1); +x_25 = l_Lean_PersistentArray_push___rarg(x_20, x_1); +lean_inc(x_2); +lean_inc(x_1); +x_26 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__1(x_21, x_1, x_2); +x_27 = lean_box(0); +x_28 = l_Lean_PersistentArray_push___rarg(x_22, x_27); +x_29 = l_Lean_PersistentArray_push___rarg(x_23, x_27); +x_30 = l_Lean_PersistentArray_push___rarg(x_24, x_27); +lean_ctor_set(x_15, 6, x_30); +lean_ctor_set(x_15, 5, x_29); +lean_ctor_set(x_15, 4, x_28); +lean_ctor_set(x_15, 1, x_26); +lean_ctor_set(x_15, 0, x_25); +x_31 = lean_st_ref_set(x_4, x_14, x_16); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = l_Lean_Meta_Grind_markAsOffsetTerm(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +if (lean_obj_tag(x_33) == 0) +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; +x_35 = lean_ctor_get(x_33, 0); +lean_dec(x_35); +lean_ctor_set(x_33, 0, x_2); +return x_33; +} +else +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_33, 1); +lean_inc(x_36); +lean_dec(x_33); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_2); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +else +{ +uint8_t x_38; +lean_dec(x_2); +x_38 = !lean_is_exclusive(x_33); +if (x_38 == 0) +{ +return x_33; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_33, 0); +x_40 = lean_ctor_get(x_33, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_33); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_42 = lean_ctor_get(x_15, 0); +x_43 = lean_ctor_get(x_15, 1); +x_44 = lean_ctor_get(x_15, 2); +x_45 = lean_ctor_get(x_15, 3); +x_46 = lean_ctor_get(x_15, 4); +x_47 = lean_ctor_get(x_15, 5); +x_48 = lean_ctor_get(x_15, 6); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_15); +lean_inc(x_1); +x_49 = l_Lean_PersistentArray_push___rarg(x_42, x_1); +lean_inc(x_2); +lean_inc(x_1); +x_50 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__1(x_43, x_1, x_2); +x_51 = lean_box(0); +x_52 = l_Lean_PersistentArray_push___rarg(x_46, x_51); +x_53 = l_Lean_PersistentArray_push___rarg(x_47, x_51); +x_54 = l_Lean_PersistentArray_push___rarg(x_48, x_51); +x_55 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_55, 0, x_49); +lean_ctor_set(x_55, 1, x_50); +lean_ctor_set(x_55, 2, x_44); +lean_ctor_set(x_55, 3, x_45); +lean_ctor_set(x_55, 4, x_52); +lean_ctor_set(x_55, 5, x_53); +lean_ctor_set(x_55, 6, x_54); +lean_ctor_set(x_14, 9, x_55); +x_56 = lean_st_ref_set(x_4, x_14, x_16); +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +lean_dec(x_56); +x_58 = l_Lean_Meta_Grind_markAsOffsetTerm(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_57); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_60 = x_58; +} else { + lean_dec_ref(x_58); + x_60 = lean_box(0); +} +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(0, 2, 0); +} else { + x_61 = x_60; +} +lean_ctor_set(x_61, 0, x_2); +lean_ctor_set(x_61, 1, x_59); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_2); +x_62 = lean_ctor_get(x_58, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_58, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_64 = x_58; +} else { + lean_dec_ref(x_58); + x_64 = lean_box(0); +} +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(1, 2, 0); +} else { + x_65 = x_64; +} +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_63); +return x_65; +} +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_66 = lean_ctor_get(x_14, 0); +x_67 = lean_ctor_get(x_14, 1); +x_68 = lean_ctor_get(x_14, 2); +x_69 = lean_ctor_get(x_14, 3); +x_70 = lean_ctor_get(x_14, 4); +x_71 = lean_ctor_get(x_14, 5); +x_72 = lean_ctor_get(x_14, 6); +x_73 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); +x_74 = lean_ctor_get(x_14, 7); +x_75 = lean_ctor_get(x_14, 8); +x_76 = lean_ctor_get(x_14, 10); +x_77 = lean_ctor_get(x_14, 11); +x_78 = lean_ctor_get(x_14, 12); +x_79 = lean_ctor_get(x_14, 13); +x_80 = lean_ctor_get(x_14, 14); +x_81 = lean_ctor_get(x_14, 15); +x_82 = lean_ctor_get(x_14, 16); +x_83 = lean_ctor_get(x_14, 17); +x_84 = lean_ctor_get(x_14, 18); +x_85 = lean_ctor_get(x_14, 19); +x_86 = lean_ctor_get(x_14, 20); +x_87 = lean_ctor_get(x_14, 21); +x_88 = lean_ctor_get(x_14, 22); +lean_inc(x_88); +lean_inc(x_87); +lean_inc(x_86); +lean_inc(x_85); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_inc(x_80); +lean_inc(x_79); +lean_inc(x_78); +lean_inc(x_77); +lean_inc(x_76); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_14); +x_89 = lean_ctor_get(x_15, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_15, 1); +lean_inc(x_90); +x_91 = lean_ctor_get(x_15, 2); +lean_inc(x_91); +x_92 = lean_ctor_get(x_15, 3); +lean_inc(x_92); +x_93 = lean_ctor_get(x_15, 4); +lean_inc(x_93); +x_94 = lean_ctor_get(x_15, 5); +lean_inc(x_94); +x_95 = lean_ctor_get(x_15, 6); +lean_inc(x_95); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + lean_ctor_release(x_15, 2); + lean_ctor_release(x_15, 3); + lean_ctor_release(x_15, 4); + lean_ctor_release(x_15, 5); + lean_ctor_release(x_15, 6); + x_96 = x_15; +} else { + lean_dec_ref(x_15); + x_96 = lean_box(0); +} +lean_inc(x_1); +x_97 = l_Lean_PersistentArray_push___rarg(x_89, x_1); +lean_inc(x_2); +lean_inc(x_1); +x_98 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__1(x_90, x_1, x_2); +x_99 = lean_box(0); +x_100 = l_Lean_PersistentArray_push___rarg(x_93, x_99); +x_101 = l_Lean_PersistentArray_push___rarg(x_94, x_99); +x_102 = l_Lean_PersistentArray_push___rarg(x_95, x_99); +if (lean_is_scalar(x_96)) { + x_103 = lean_alloc_ctor(0, 7, 0); +} else { + x_103 = x_96; +} +lean_ctor_set(x_103, 0, x_97); +lean_ctor_set(x_103, 1, x_98); +lean_ctor_set(x_103, 2, x_91); +lean_ctor_set(x_103, 3, x_92); +lean_ctor_set(x_103, 4, x_100); +lean_ctor_set(x_103, 5, x_101); +lean_ctor_set(x_103, 6, x_102); +x_104 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_104, 0, x_66); +lean_ctor_set(x_104, 1, x_67); +lean_ctor_set(x_104, 2, x_68); +lean_ctor_set(x_104, 3, x_69); +lean_ctor_set(x_104, 4, x_70); +lean_ctor_set(x_104, 5, x_71); +lean_ctor_set(x_104, 6, x_72); +lean_ctor_set(x_104, 7, x_74); +lean_ctor_set(x_104, 8, x_75); +lean_ctor_set(x_104, 9, x_103); +lean_ctor_set(x_104, 10, x_76); +lean_ctor_set(x_104, 11, x_77); +lean_ctor_set(x_104, 12, x_78); +lean_ctor_set(x_104, 13, x_79); +lean_ctor_set(x_104, 14, x_80); +lean_ctor_set(x_104, 15, x_81); +lean_ctor_set(x_104, 16, x_82); +lean_ctor_set(x_104, 17, x_83); +lean_ctor_set(x_104, 18, x_84); +lean_ctor_set(x_104, 19, x_85); +lean_ctor_set(x_104, 20, x_86); +lean_ctor_set(x_104, 21, x_87); +lean_ctor_set(x_104, 22, x_88); +lean_ctor_set_uint8(x_104, sizeof(void*)*23, x_73); +x_105 = lean_st_ref_set(x_4, x_104, x_16); +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +lean_dec(x_105); +x_107 = l_Lean_Meta_Grind_markAsOffsetTerm(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_106); +if (lean_obj_tag(x_107) == 0) +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_108 = lean_ctor_get(x_107, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_109 = x_107; +} else { + lean_dec_ref(x_107); + x_109 = lean_box(0); +} +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(0, 2, 0); +} else { + x_110 = x_109; +} +lean_ctor_set(x_110, 0, x_2); +lean_ctor_set(x_110, 1, x_108); +return x_110; +} +else +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_dec(x_2); +x_111 = lean_ctor_get(x_107, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_107, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_113 = x_107; +} else { + lean_dec_ref(x_107); + x_113 = lean_box(0); +} +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 2, 0); +} else { + x_114 = x_113; +} +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_112); +return x_114; +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("grind", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("offset", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("internalize", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("term", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ↦ #", 6, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5; +x_19 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_free_object(x_12); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_box(0); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_17, x_23, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_22); +return x_24; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_26 = lean_ctor_get(x_19, 1); +x_27 = lean_ctor_get(x_19, 0); +lean_dec(x_27); +lean_inc(x_1); +x_28 = l_Lean_MessageData_ofExpr(x_1); +x_29 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_28); +lean_ctor_set(x_19, 0, x_29); +x_30 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9; +lean_ctor_set_tag(x_12, 7); +lean_ctor_set(x_12, 1, x_30); +lean_ctor_set(x_12, 0, x_19); +lean_inc(x_17); +x_31 = l___private_Init_Data_Repr_0__Nat_reprFast(x_17); +x_32 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_32, 0, x_31); +x_33 = l_Lean_MessageData_ofFormat(x_32); +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_12); +lean_ctor_set(x_34, 1, x_33); +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_29); +x_36 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_35, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_26); +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_17, x_37, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_38); +lean_dec(x_37); +return x_39; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_40 = lean_ctor_get(x_19, 1); +lean_inc(x_40); +lean_dec(x_19); +lean_inc(x_1); +x_41 = l_Lean_MessageData_ofExpr(x_1); +x_42 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +x_44 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9; +lean_ctor_set_tag(x_12, 7); +lean_ctor_set(x_12, 1, x_44); +lean_ctor_set(x_12, 0, x_43); +lean_inc(x_17); +x_45 = l___private_Init_Data_Repr_0__Nat_reprFast(x_17); +x_46 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l_Lean_MessageData_ofFormat(x_46); +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_12); +lean_ctor_set(x_48, 1, x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_42); +x_50 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_40); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_17, x_51, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_52); +lean_dec(x_51); +return x_53; +} +} +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_54 = lean_ctor_get(x_12, 0); +x_55 = lean_ctor_get(x_12, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_12); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +lean_dec(x_54); +x_57 = lean_ctor_get(x_56, 2); +lean_inc(x_57); +lean_dec(x_56); +x_58 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5; +x_59 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_58, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_55); +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_unbox(x_60); +lean_dec(x_60); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_59, 1); +lean_inc(x_62); +lean_dec(x_59); +x_63 = lean_box(0); +x_64 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_57, x_63, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_62); +return x_64; +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_65 = lean_ctor_get(x_59, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_66 = x_59; +} else { + lean_dec_ref(x_59); + x_66 = lean_box(0); +} +lean_inc(x_1); +x_67 = l_Lean_MessageData_ofExpr(x_1); +x_68 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +if (lean_is_scalar(x_66)) { + x_69 = lean_alloc_ctor(7, 2, 0); +} else { + x_69 = x_66; + lean_ctor_set_tag(x_69, 7); +} +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_67); +x_70 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9; +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +lean_inc(x_57); +x_72 = l___private_Init_Data_Repr_0__Nat_reprFast(x_57); +x_73 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_73, 0, x_72); +x_74 = l_Lean_MessageData_ofFormat(x_73); +x_75 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_75, 0, x_71); +lean_ctor_set(x_75, 1, x_74); +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_68); +x_77 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_58, x_76, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_65); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_57, x_78, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_79); +lean_dec(x_78); +return x_80; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(x_15, x_1); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_free_object(x_11); +x_17 = lean_box(0); +x_18 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_18; +} +else +{ +lean_object* x_19; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = lean_ctor_get(x_16, 0); +lean_inc(x_19); +lean_dec(x_16); +lean_ctor_set(x_11, 0, x_19); +return x_11; +} +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_11, 0); +x_21 = lean_ctor_get(x_11, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_11); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(x_22, x_1); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_box(0); +x_25 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2(x_1, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_26 = lean_ctor_get(x_23, 0); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_21); +return x_27; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__3(x_7, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2(x_1, x_6, x_7, x_4, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__7(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__6(x_1, x_4, x_3); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_ctor_get(x_14, 2); +lean_inc(x_15); +x_16 = lean_nat_dec_lt(x_1, x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +lean_dec(x_14); +x_17 = l_Lean_instInhabitedExpr; +x_18 = l_outOfBounds___rarg(x_17); +lean_ctor_set(x_11, 0, x_18); +return x_11; +} +else +{ +lean_object* x_19; lean_object* x_20; +x_19 = l_Lean_instInhabitedExpr; +x_20 = l_Lean_PersistentArray_get_x21___rarg(x_19, x_14, x_1); +lean_ctor_set(x_11, 0, x_20); +return x_11; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_21 = lean_ctor_get(x_11, 0); +x_22 = lean_ctor_get(x_11, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_11); +x_23 = lean_ctor_get(x_21, 0); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_ctor_get(x_23, 2); +lean_inc(x_24); +x_25 = lean_nat_dec_lt(x_1, x_24); +lean_dec(x_24); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_23); +x_26 = l_Lean_instInhabitedExpr; +x_27 = l_outOfBounds___rarg(x_26); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_22); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = l_Lean_instInhabitedExpr; +x_30 = l_Lean_PersistentArray_get_x21___rarg(x_29, x_23, x_1); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_22); +return x_31; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_2, 1); +x_6 = lean_ctor_get(x_2, 2); +x_7 = lean_nat_dec_eq(x_4, x_1); +if (x_7 == 0) +{ +x_2 = x_6; +goto _start; +} +else +{ +lean_object* x_9; +lean_inc(x_5); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +return x_9; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_box(0); +x_16 = lean_ctor_get(x_14, 5); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +x_18 = lean_nat_dec_lt(x_1, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_16); +x_19 = l_outOfBounds___rarg(x_15); +x_20 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(x_2, x_19); +lean_dec(x_19); +lean_ctor_set(x_12, 0, x_20); +return x_12; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = l_Lean_PersistentArray_get_x21___rarg(x_15, x_16, x_1); +x_22 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(x_2, x_21); +lean_dec(x_21); +lean_ctor_set(x_12, 0, x_22); +return x_12; +} +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_23 = lean_ctor_get(x_12, 0); +x_24 = lean_ctor_get(x_12, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_12); +x_25 = lean_box(0); +x_26 = lean_ctor_get(x_23, 5); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_ctor_get(x_26, 2); +lean_inc(x_27); +x_28 = lean_nat_dec_lt(x_1, x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_26); +x_29 = l_outOfBounds___rarg(x_25); +x_30 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(x_2, x_29); +lean_dec(x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_24); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = l_Lean_PersistentArray_get_x21___rarg(x_25, x_26, x_1); +x_33 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(x_2, x_32); +lean_dec(x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_24); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_2, 1); +x_6 = lean_ctor_get(x_2, 2); +x_7 = lean_nat_dec_eq(x_4, x_1); +if (x_7 == 0) +{ +x_2 = x_6; +goto _start; +} +else +{ +lean_object* x_9; +lean_inc(x_5); +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_5); +return x_9; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; uint8_t x_13; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_box(0); +x_16 = lean_ctor_get(x_14, 6); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +x_18 = lean_nat_dec_lt(x_1, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_16); +x_19 = l_outOfBounds___rarg(x_15); +x_20 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(x_2, x_19); +lean_dec(x_19); +lean_ctor_set(x_12, 0, x_20); +return x_12; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = l_Lean_PersistentArray_get_x21___rarg(x_15, x_16, x_1); +x_22 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(x_2, x_21); +lean_dec(x_21); +lean_ctor_set(x_12, 0, x_22); +return x_12; +} +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_23 = lean_ctor_get(x_12, 0); +x_24 = lean_ctor_get(x_12, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_12); +x_25 = lean_box(0); +x_26 = lean_ctor_get(x_23, 6); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_ctor_get(x_26, 2); +lean_inc(x_27); +x_28 = lean_nat_dec_lt(x_1, x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_26); +x_29 = l_outOfBounds___rarg(x_25); +x_30 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(x_2, x_29); +lean_dec(x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_24); +return x_31; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = l_Lean_PersistentArray_get_x21___rarg(x_25, x_26, x_1); +x_33 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(x_2, x_32); +lean_dec(x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_24); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_AssocList_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___spec__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_8, 5); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_11); +lean_ctor_set(x_15, 1, x_14); +lean_ctor_set_tag(x_12, 1); +lean_ctor_set(x_12, 0, x_15); +return x_12; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_12, 0); +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_12); +lean_inc(x_11); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_11); +lean_ctor_set(x_18, 1, x_16); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("internal `grind` error, term has not been internalized by offset module", 71, 71); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(x_15, x_1); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_free_object(x_11); +x_17 = l_Lean_indentExpr(x_1); +x_18 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +x_20 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +x_22 = l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_22; +} +else +{ +lean_object* x_23; +lean_dec(x_1); +x_23 = lean_ctor_get(x_16, 0); +lean_inc(x_23); +lean_dec(x_16); +lean_ctor_set(x_11, 0, x_23); +return x_11; +} +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_11, 0); +x_25 = lean_ctor_get(x_11, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_11); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__5(x_26, x_1); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_28 = l_Lean_indentExpr(x_1); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +x_31 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_1); +x_34 = lean_ctor_get(x_27, 0); +lean_inc(x_34); +lean_dec(x_27); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_25); +return x_35; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo; +x_3 = lean_panic_fn(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Init.Data.Option.BasicAux", 25, 25); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Option.get!", 11, 11); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("value is none", 13, 13); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2; +x_3 = lean_unsigned_to_nat(16u); +x_4 = lean_unsigned_to_nat(14u); +x_5 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_3, 0); +lean_inc(x_13); +x_14 = lean_nat_dec_eq(x_1, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(x_1, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_13); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4; +x_22 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___spec__1(x_21); +x_23 = lean_ctor_get(x_19, 0); +lean_inc(x_23); +lean_dec(x_19); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkTrans(x_23, x_22, x_3, x_2); +x_3 = x_24; +x_12 = x_20; +goto _start; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_26 = lean_ctor_get(x_16, 0); +lean_inc(x_26); +lean_dec(x_16); +x_27 = lean_ctor_get(x_18, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_18, 1); +lean_inc(x_28); +lean_dec(x_18); +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l_Lean_Meta_Grind_Arith_Offset_mkTrans(x_29, x_26, x_3, x_2); +x_3 = x_30; +x_12 = x_28; +goto _start; +} +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_13); +x_32 = lean_ctor_get(x_3, 2); +lean_inc(x_32); +lean_dec(x_3); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_12); +return x_33; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4; +x_16 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___spec__1(x_15); +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go(x_1, x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_dec(x_12); +x_19 = lean_ctor_get(x_13, 0); +lean_inc(x_19); +lean_dec(x_13); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go(x_1, x_2, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +return x_20; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_12; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_instMonadMetaM; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4; +x_2 = l_instInhabitedPUnit; +x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5; +x_12 = lean_panic_fn(x_11, x_1); +x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("assertion violation: ", 21, 21); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("kuv + kvu < 0\n ", 16, 16); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.Grind.Arith.Offset", 35, 35); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Meta.Tactic.Grind.Arith.Offset.0.Lean.Meta.Grind.Arith.Offset.setUnsat", 84, 84); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6; +x_3 = lean_unsigned_to_nat(88u); +x_4 = lean_unsigned_to_nat(2u); +x_5 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_int_add(x_3, x_5); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_17 = lean_int_dec_lt(x_15, x_16); +lean_dec(x_15); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_4); +x_18 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7; +x_19 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_2, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof(x_24, x_27, x_3, x_4, x_5, x_21); +x_30 = l_Lean_Meta_Grind_closeGoal(x_29, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_28); +return x_30; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT uint8_t l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_2, 2); +x_6 = lean_nat_dec_eq(x_4, x_1); +if (x_6 == 0) +{ +x_2 = x_5; +goto _start; +} +else +{ +uint8_t x_8; +x_8 = 1; +return x_8; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(0); +return x_4; +} +else +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_3, 1); +x_8 = lean_ctor_get(x_3, 2); +x_9 = lean_nat_dec_eq(x_6, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__3(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_10); +return x_3; +} +else +{ +lean_dec(x_7); +lean_dec(x_6); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 0, x_1); +return x_3; +} +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = lean_ctor_get(x_3, 2); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_14 = lean_nat_dec_eq(x_11, x_1); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__3(x_1, x_2, x_13); +x_16 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_12); +lean_ctor_set(x_16, 2, x_15); +return x_16; +} +else +{ +lean_object* x_17; +lean_dec(x_12); +lean_dec(x_11); +x_17 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_2); +lean_ctor_set(x_17, 2, x_13); +return x_17; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2(x_2, x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_1); +return x_5; +} +else +{ +lean_object* x_6; +x_6 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__3(x_2, x_3, x_1); +return x_6; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_4); +if (x_7 == 0) +{ +lean_object* x_8; size_t x_9; size_t x_10; size_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_8 = lean_ctor_get(x_4, 0); +x_9 = lean_usize_shift_right(x_5, x_6); +x_10 = 1; +x_11 = lean_usize_shift_left(x_10, x_6); +x_12 = lean_usize_sub(x_11, x_10); +x_13 = lean_usize_land(x_5, x_12); +x_14 = 5; +x_15 = lean_usize_sub(x_6, x_14); +x_16 = lean_usize_to_nat(x_9); +x_17 = lean_array_get_size(x_8); +x_18 = lean_nat_dec_lt(x_16, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_dec(x_16); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_array_fget(x_8, x_16); +x_20 = lean_box(0); +x_21 = lean_array_fset(x_8, x_16, x_20); +x_22 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(x_1, x_2, x_3, x_19, x_13, x_15); +x_23 = lean_array_fset(x_21, x_16, x_22); +lean_dec(x_16); +lean_ctor_set(x_4, 0, x_23); +return x_4; +} +} +else +{ +lean_object* x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_24 = lean_ctor_get(x_4, 0); +lean_inc(x_24); +lean_dec(x_4); +x_25 = lean_usize_shift_right(x_5, x_6); +x_26 = 1; +x_27 = lean_usize_shift_left(x_26, x_6); +x_28 = lean_usize_sub(x_27, x_26); +x_29 = lean_usize_land(x_5, x_28); +x_30 = 5; +x_31 = lean_usize_sub(x_6, x_30); +x_32 = lean_usize_to_nat(x_25); +x_33 = lean_array_get_size(x_24); +x_34 = lean_nat_dec_lt(x_32, x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; +lean_dec(x_32); +lean_dec(x_2); +lean_dec(x_1); +x_35 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_35, 0, x_24); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_36 = lean_array_fget(x_24, x_32); +x_37 = lean_box(0); +x_38 = lean_array_fset(x_24, x_32, x_37); +x_39 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(x_1, x_2, x_3, x_36, x_29, x_31); +x_40 = lean_array_fset(x_38, x_32, x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_41, 0, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +x_42 = !lean_is_exclusive(x_4); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = lean_ctor_get(x_4, 0); +x_44 = lean_usize_to_nat(x_5); +x_45 = lean_array_get_size(x_43); +x_46 = lean_nat_dec_lt(x_44, x_45); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_dec(x_44); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_array_fget(x_43, x_44); +x_48 = lean_box(0); +x_49 = lean_array_fset(x_43, x_44, x_48); +x_50 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_47, x_1, x_2); +x_51 = lean_array_fset(x_49, x_44, x_50); +lean_dec(x_44); +lean_ctor_set(x_4, 0, x_51); +return x_4; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_52 = lean_ctor_get(x_4, 0); +lean_inc(x_52); +lean_dec(x_4); +x_53 = lean_usize_to_nat(x_5); +x_54 = lean_array_get_size(x_52); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_2); +lean_dec(x_1); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_52); +return x_56; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_57 = lean_array_fget(x_52, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_52, x_53, x_58); +x_60 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_57, x_1, x_2); +x_61 = lean_array_fset(x_59, x_53, x_60); +lean_dec(x_53); +x_62 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_62, 0, x_61); +return x_62; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; size_t x_9; lean_object* x_10; uint8_t x_11; +x_7 = lean_ctor_get(x_4, 0); +x_8 = lean_ctor_get(x_4, 1); +x_9 = lean_ctor_get_usize(x_4, 4); +x_10 = lean_ctor_get(x_4, 3); +x_11 = lean_nat_dec_le(x_10, x_5); +if (x_11 == 0) +{ +size_t x_12; lean_object* x_13; +x_12 = lean_usize_of_nat(x_5); +x_13 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(x_1, x_2, x_3, x_7, x_12, x_9); +lean_ctor_set(x_4, 0, x_13); +return x_4; +} +else +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_nat_sub(x_5, x_10); +x_15 = lean_array_get_size(x_8); +x_16 = lean_nat_dec_lt(x_14, x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_dec(x_14); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_array_fget(x_8, x_14); +x_18 = lean_box(0); +x_19 = lean_array_fset(x_8, x_14, x_18); +x_20 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_17, x_1, x_2); +x_21 = lean_array_fset(x_19, x_14, x_20); +lean_dec(x_14); +lean_ctor_set(x_4, 1, x_21); +return x_4; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; lean_object* x_26; uint8_t x_27; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +x_24 = lean_ctor_get(x_4, 2); +x_25 = lean_ctor_get_usize(x_4, 4); +x_26 = lean_ctor_get(x_4, 3); +lean_inc(x_26); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_4); +x_27 = lean_nat_dec_le(x_26, x_5); +if (x_27 == 0) +{ +size_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_usize_of_nat(x_5); +x_29 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(x_1, x_2, x_3, x_22, x_28, x_25); +x_30 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_24); +lean_ctor_set(x_30, 3, x_26); +lean_ctor_set_usize(x_30, 4, x_25); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_nat_sub(x_5, x_26); +x_32 = lean_array_get_size(x_23); +x_33 = lean_nat_dec_lt(x_31, x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_31); +lean_dec(x_2); +lean_dec(x_1); +x_34 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_34, 0, x_22); +lean_ctor_set(x_34, 1, x_23); +lean_ctor_set(x_34, 2, x_24); +lean_ctor_set(x_34, 3, x_26); +lean_ctor_set_usize(x_34, 4, x_25); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_array_fget(x_23, x_31); +x_36 = lean_box(0); +x_37 = lean_array_fset(x_23, x_31, x_36); +x_38 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_35, x_1, x_2); +x_39 = lean_array_fset(x_37, x_31, x_38); +lean_dec(x_31); +x_40 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_40, 0, x_22); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_24); +lean_ctor_set(x_40, 3, x_26); +lean_ctor_set_usize(x_40, 4, x_25); +return x_40; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_4); +if (x_7 == 0) +{ +lean_object* x_8; size_t x_9; size_t x_10; size_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_8 = lean_ctor_get(x_4, 0); +x_9 = lean_usize_shift_right(x_5, x_6); +x_10 = 1; +x_11 = lean_usize_shift_left(x_10, x_6); +x_12 = lean_usize_sub(x_11, x_10); +x_13 = lean_usize_land(x_5, x_12); +x_14 = 5; +x_15 = lean_usize_sub(x_6, x_14); +x_16 = lean_usize_to_nat(x_9); +x_17 = lean_array_get_size(x_8); +x_18 = lean_nat_dec_lt(x_16, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_dec(x_16); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_array_fget(x_8, x_16); +x_20 = lean_box(0); +x_21 = lean_array_fset(x_8, x_16, x_20); +x_22 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(x_1, x_2, x_3, x_19, x_13, x_15); +x_23 = lean_array_fset(x_21, x_16, x_22); +lean_dec(x_16); +lean_ctor_set(x_4, 0, x_23); +return x_4; +} +} +else +{ +lean_object* x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_24 = lean_ctor_get(x_4, 0); +lean_inc(x_24); +lean_dec(x_4); +x_25 = lean_usize_shift_right(x_5, x_6); +x_26 = 1; +x_27 = lean_usize_shift_left(x_26, x_6); +x_28 = lean_usize_sub(x_27, x_26); +x_29 = lean_usize_land(x_5, x_28); +x_30 = 5; +x_31 = lean_usize_sub(x_6, x_30); +x_32 = lean_usize_to_nat(x_25); +x_33 = lean_array_get_size(x_24); +x_34 = lean_nat_dec_lt(x_32, x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; +lean_dec(x_32); +lean_dec(x_2); +lean_dec(x_1); +x_35 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_35, 0, x_24); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_36 = lean_array_fget(x_24, x_32); +x_37 = lean_box(0); +x_38 = lean_array_fset(x_24, x_32, x_37); +x_39 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(x_1, x_2, x_3, x_36, x_29, x_31); +x_40 = lean_array_fset(x_38, x_32, x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_41, 0, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +x_42 = !lean_is_exclusive(x_4); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = lean_ctor_get(x_4, 0); +x_44 = lean_usize_to_nat(x_5); +x_45 = lean_array_get_size(x_43); +x_46 = lean_nat_dec_lt(x_44, x_45); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_dec(x_44); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_array_fget(x_43, x_44); +x_48 = lean_box(0); +x_49 = lean_array_fset(x_43, x_44, x_48); +x_50 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_47, x_1, x_2); +x_51 = lean_array_fset(x_49, x_44, x_50); +lean_dec(x_44); +lean_ctor_set(x_4, 0, x_51); +return x_4; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_52 = lean_ctor_get(x_4, 0); +lean_inc(x_52); +lean_dec(x_4); +x_53 = lean_usize_to_nat(x_5); +x_54 = lean_array_get_size(x_52); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_2); +lean_dec(x_1); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_52); +return x_56; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_57 = lean_array_fget(x_52, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_52, x_53, x_58); +x_60 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_57, x_1, x_2); +x_61 = lean_array_fset(x_59, x_53, x_60); +lean_dec(x_53); +x_62 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_62, 0, x_61); +return x_62; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; size_t x_9; lean_object* x_10; uint8_t x_11; +x_7 = lean_ctor_get(x_4, 0); +x_8 = lean_ctor_get(x_4, 1); +x_9 = lean_ctor_get_usize(x_4, 4); +x_10 = lean_ctor_get(x_4, 3); +x_11 = lean_nat_dec_le(x_10, x_5); +if (x_11 == 0) +{ +size_t x_12; lean_object* x_13; +x_12 = lean_usize_of_nat(x_5); +x_13 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(x_1, x_2, x_3, x_7, x_12, x_9); +lean_ctor_set(x_4, 0, x_13); +return x_4; +} +else +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_nat_sub(x_5, x_10); +x_15 = lean_array_get_size(x_8); +x_16 = lean_nat_dec_lt(x_14, x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_dec(x_14); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_array_fget(x_8, x_14); +x_18 = lean_box(0); +x_19 = lean_array_fset(x_8, x_14, x_18); +x_20 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_17, x_1, x_2); +x_21 = lean_array_fset(x_19, x_14, x_20); +lean_dec(x_14); +lean_ctor_set(x_4, 1, x_21); +return x_4; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; lean_object* x_26; uint8_t x_27; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +x_24 = lean_ctor_get(x_4, 2); +x_25 = lean_ctor_get_usize(x_4, 4); +x_26 = lean_ctor_get(x_4, 3); +lean_inc(x_26); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_4); +x_27 = lean_nat_dec_le(x_26, x_5); +if (x_27 == 0) +{ +size_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_usize_of_nat(x_5); +x_29 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(x_1, x_2, x_3, x_22, x_28, x_25); +x_30 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_24); +lean_ctor_set(x_30, 3, x_26); +lean_ctor_set_usize(x_30, 4, x_25); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_nat_sub(x_5, x_26); +x_32 = lean_array_get_size(x_23); +x_33 = lean_nat_dec_lt(x_31, x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_31); +lean_dec(x_2); +lean_dec(x_1); +x_34 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_34, 0, x_22); +lean_ctor_set(x_34, 1, x_23); +lean_ctor_set(x_34, 2, x_24); +lean_ctor_set(x_34, 3, x_26); +lean_ctor_set_usize(x_34, 4, x_25); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_array_fget(x_23, x_31); +x_36 = lean_box(0); +x_37 = lean_array_fset(x_23, x_31, x_36); +x_38 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__1(x_35, x_1, x_2); +x_39 = lean_array_fset(x_37, x_31, x_38); +lean_dec(x_31); +x_40 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_40, 0, x_22); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_24); +lean_ctor_set(x_40, 3, x_26); +lean_ctor_set_usize(x_40, 4, x_25); +return x_40; +} +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("#", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ≤ ", 5, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" + ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +x_10 = l___private_Init_Data_Repr_0__Nat_reprFast(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Lean_MessageData_ofFormat(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +lean_inc(x_1); +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_1); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_ctor_get(x_2, 1); +lean_inc(x_20); +lean_dec(x_2); +x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); +x_22 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_1); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_30 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lean_MessageData_ofFormat(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_28); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_16); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_6); +x_34 = lean_ctor_get(x_2, 0); +lean_inc(x_34); +x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_34); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l_Lean_MessageData_ofFormat(x_36); +x_38 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +lean_inc(x_1); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_ctor_get(x_2, 1); +lean_inc(x_45); +lean_dec(x_2); +x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_45); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l_Lean_MessageData_ofFormat(x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_1); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_41); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_53 = lean_nat_abs(x_3); +lean_dec(x_3); +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_53, x_54); +lean_dec(x_53); +x_56 = lean_ctor_get(x_2, 0); +lean_inc(x_56); +x_57 = l___private_Init_Data_Repr_0__Nat_reprFast(x_56); +x_58 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_59 = l_Lean_MessageData_ofFormat(x_58); +x_60 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +lean_inc(x_1); +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_1); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_62); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_nat_add(x_55, x_54); +lean_dec(x_55); +x_68 = l___private_Init_Data_Repr_0__Nat_reprFast(x_67); +x_69 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_MessageData_ofFormat(x_69); +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_ctor_get(x_2, 1); +lean_inc(x_74); +lean_dec(x_2); +x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_77 = l_Lean_MessageData_ofFormat(x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_60); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_1); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = lean_st_ref_take(x_5, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 9); +lean_inc(x_16); +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = lean_ctor_get(x_15, 9); +lean_dec(x_19); +x_20 = !lean_is_exclusive(x_16); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_21 = lean_ctor_get(x_16, 4); +x_22 = lean_ctor_get(x_16, 5); +x_23 = lean_box(0); +lean_inc(x_2); +lean_inc(x_1); +x_24 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(x_1, x_2, x_23, x_21, x_3); +x_25 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(x_3, x_2, x_23, x_22, x_1); +lean_dec(x_1); +lean_ctor_set(x_16, 5, x_25); +lean_ctor_set(x_16, 4, x_24); +x_26 = lean_st_ref_set(x_5, x_15, x_17); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +x_29 = lean_box(0); +lean_ctor_set(x_26, 0, x_29); +return x_26; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_26, 1); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +return x_32; +} +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_33 = lean_ctor_get(x_16, 0); +x_34 = lean_ctor_get(x_16, 1); +x_35 = lean_ctor_get(x_16, 2); +x_36 = lean_ctor_get(x_16, 3); +x_37 = lean_ctor_get(x_16, 4); +x_38 = lean_ctor_get(x_16, 5); +x_39 = lean_ctor_get(x_16, 6); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_16); +x_40 = lean_box(0); +lean_inc(x_2); +lean_inc(x_1); +x_41 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(x_1, x_2, x_40, x_37, x_3); +x_42 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(x_3, x_2, x_40, x_38, x_1); +lean_dec(x_1); +x_43 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_43, 0, x_33); +lean_ctor_set(x_43, 1, x_34); +lean_ctor_set(x_43, 2, x_35); +lean_ctor_set(x_43, 3, x_36); +lean_ctor_set(x_43, 4, x_41); +lean_ctor_set(x_43, 5, x_42); +lean_ctor_set(x_43, 6, x_39); +lean_ctor_set(x_15, 9, x_43); +x_44 = lean_st_ref_set(x_5, x_15, x_17); +x_45 = lean_ctor_get(x_44, 1); +lean_inc(x_45); +if (lean_is_exclusive(x_44)) { + lean_ctor_release(x_44, 0); + lean_ctor_release(x_44, 1); + x_46 = x_44; +} else { + lean_dec_ref(x_44); + x_46 = lean_box(0); +} +x_47 = lean_box(0); +if (lean_is_scalar(x_46)) { + x_48 = lean_alloc_ctor(0, 2, 0); +} else { + x_48 = x_46; +} +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_45); +return x_48; +} +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_49 = lean_ctor_get(x_15, 0); +x_50 = lean_ctor_get(x_15, 1); +x_51 = lean_ctor_get(x_15, 2); +x_52 = lean_ctor_get(x_15, 3); +x_53 = lean_ctor_get(x_15, 4); +x_54 = lean_ctor_get(x_15, 5); +x_55 = lean_ctor_get(x_15, 6); +x_56 = lean_ctor_get_uint8(x_15, sizeof(void*)*23); +x_57 = lean_ctor_get(x_15, 7); +x_58 = lean_ctor_get(x_15, 8); +x_59 = lean_ctor_get(x_15, 10); +x_60 = lean_ctor_get(x_15, 11); +x_61 = lean_ctor_get(x_15, 12); +x_62 = lean_ctor_get(x_15, 13); +x_63 = lean_ctor_get(x_15, 14); +x_64 = lean_ctor_get(x_15, 15); +x_65 = lean_ctor_get(x_15, 16); +x_66 = lean_ctor_get(x_15, 17); +x_67 = lean_ctor_get(x_15, 18); +x_68 = lean_ctor_get(x_15, 19); +x_69 = lean_ctor_get(x_15, 20); +x_70 = lean_ctor_get(x_15, 21); +x_71 = lean_ctor_get(x_15, 22); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_15); +x_72 = lean_ctor_get(x_16, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_16, 1); +lean_inc(x_73); +x_74 = lean_ctor_get(x_16, 2); +lean_inc(x_74); +x_75 = lean_ctor_get(x_16, 3); +lean_inc(x_75); +x_76 = lean_ctor_get(x_16, 4); +lean_inc(x_76); +x_77 = lean_ctor_get(x_16, 5); +lean_inc(x_77); +x_78 = lean_ctor_get(x_16, 6); +lean_inc(x_78); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + lean_ctor_release(x_16, 1); + lean_ctor_release(x_16, 2); + lean_ctor_release(x_16, 3); + lean_ctor_release(x_16, 4); + lean_ctor_release(x_16, 5); + lean_ctor_release(x_16, 6); + x_79 = x_16; +} else { + lean_dec_ref(x_16); + x_79 = lean_box(0); +} +x_80 = lean_box(0); +lean_inc(x_2); +lean_inc(x_1); +x_81 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(x_1, x_2, x_80, x_76, x_3); +x_82 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(x_3, x_2, x_80, x_77, x_1); +lean_dec(x_1); +if (lean_is_scalar(x_79)) { + x_83 = lean_alloc_ctor(0, 7, 0); +} else { + x_83 = x_79; +} +lean_ctor_set(x_83, 0, x_72); +lean_ctor_set(x_83, 1, x_73); +lean_ctor_set(x_83, 2, x_74); +lean_ctor_set(x_83, 3, x_75); +lean_ctor_set(x_83, 4, x_81); +lean_ctor_set(x_83, 5, x_82); +lean_ctor_set(x_83, 6, x_78); +x_84 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_84, 0, x_49); +lean_ctor_set(x_84, 1, x_50); +lean_ctor_set(x_84, 2, x_51); +lean_ctor_set(x_84, 3, x_52); +lean_ctor_set(x_84, 4, x_53); +lean_ctor_set(x_84, 5, x_54); +lean_ctor_set(x_84, 6, x_55); +lean_ctor_set(x_84, 7, x_57); +lean_ctor_set(x_84, 8, x_58); +lean_ctor_set(x_84, 9, x_83); +lean_ctor_set(x_84, 10, x_59); +lean_ctor_set(x_84, 11, x_60); +lean_ctor_set(x_84, 12, x_61); +lean_ctor_set(x_84, 13, x_62); +lean_ctor_set(x_84, 14, x_63); +lean_ctor_set(x_84, 15, x_64); +lean_ctor_set(x_84, 16, x_65); +lean_ctor_set(x_84, 17, x_66); +lean_ctor_set(x_84, 18, x_67); +lean_ctor_set(x_84, 19, x_68); +lean_ctor_set(x_84, 20, x_69); +lean_ctor_set(x_84, 21, x_70); +lean_ctor_set(x_84, 22, x_71); +lean_ctor_set_uint8(x_84, sizeof(void*)*23, x_56); +x_85 = lean_st_ref_set(x_5, x_84, x_17); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_87 = x_85; +} else { + lean_dec_ref(x_85); + x_87 = lean_box(0); +} +x_88 = lean_box(0); +if (lean_is_scalar(x_87)) { + x_89 = lean_alloc_ctor(0, 2, 0); +} else { + x_89 = x_87; +} +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_86); +return x_89; +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("dist", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2; +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_box(0); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(x_1, x_3, x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_14); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_21 = lean_ctor_get(x_14, 1); +x_22 = lean_ctor_get(x_14, 0); +lean_dec(x_22); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_23 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_23, 0, x_1); +lean_ctor_set(x_23, 1, x_2); +lean_ctor_set(x_23, 2, x_3); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_25 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8(x_24, x_23); +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_25); +lean_ctor_set(x_14, 0, x_24); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_14); +lean_ctor_set(x_26, 1, x_24); +x_27 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(x_1, x_3, x_2, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_29); +lean_dec(x_28); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_dec(x_14); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_32 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_32, 0, x_1); +lean_ctor_set(x_32, 1, x_2); +lean_ctor_set(x_32, 2, x_3); +x_33 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_34 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8(x_33, x_32); +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_33); +x_37 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_31); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(x_1, x_3, x_2, x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_39); +lean_dec(x_38); +return x_40; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__2(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_8 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_9 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__5(x_1, x_2, x_3, x_4, x_7, x_8); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__4(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_8 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_9 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__7(x_1, x_2, x_3, x_4, x_7, x_8); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__6(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} +LEAN_EXPORT uint8_t l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = 0; +return x_3; +} +else +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_2, 2); +x_6 = lean_nat_dec_eq(x_4, x_1); +if (x_6 == 0) +{ +x_2 = x_5; +goto _start; +} +else +{ +uint8_t x_8; +x_8 = 1; +return x_8; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(0); +return x_4; +} +else +{ +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_3, 1); +x_8 = lean_ctor_get(x_3, 2); +x_9 = lean_nat_dec_eq(x_6, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +x_10 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__3(x_1, x_2, x_8); +lean_ctor_set(x_3, 2, x_10); +return x_3; +} +else +{ +lean_dec(x_7); +lean_dec(x_6); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 0, x_1); +return x_3; +} +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = lean_ctor_get(x_3, 2); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_14 = lean_nat_dec_eq(x_11, x_1); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__3(x_1, x_2, x_13); +x_16 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_12); +lean_ctor_set(x_16, 2, x_15); +return x_16; +} +else +{ +lean_object* x_17; +lean_dec(x_12); +lean_dec(x_11); +x_17 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_17, 0, x_1); +lean_ctor_set(x_17, 1, x_2); +lean_ctor_set(x_17, 2, x_13); +return x_17; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2(x_2, x_1); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +lean_ctor_set(x_5, 2, x_1); +return x_5; +} +else +{ +lean_object* x_6; +x_6 = l_Lean_AssocList_replace___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__3(x_2, x_3, x_1); +return x_6; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_4); +if (x_7 == 0) +{ +lean_object* x_8; size_t x_9; size_t x_10; size_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_8 = lean_ctor_get(x_4, 0); +x_9 = lean_usize_shift_right(x_5, x_6); +x_10 = 1; +x_11 = lean_usize_shift_left(x_10, x_6); +x_12 = lean_usize_sub(x_11, x_10); +x_13 = lean_usize_land(x_5, x_12); +x_14 = 5; +x_15 = lean_usize_sub(x_6, x_14); +x_16 = lean_usize_to_nat(x_9); +x_17 = lean_array_get_size(x_8); +x_18 = lean_nat_dec_lt(x_16, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_dec(x_16); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_array_fget(x_8, x_16); +x_20 = lean_box(0); +x_21 = lean_array_fset(x_8, x_16, x_20); +x_22 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(x_1, x_2, x_3, x_19, x_13, x_15); +x_23 = lean_array_fset(x_21, x_16, x_22); +lean_dec(x_16); +lean_ctor_set(x_4, 0, x_23); +return x_4; +} +} +else +{ +lean_object* x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_24 = lean_ctor_get(x_4, 0); +lean_inc(x_24); +lean_dec(x_4); +x_25 = lean_usize_shift_right(x_5, x_6); +x_26 = 1; +x_27 = lean_usize_shift_left(x_26, x_6); +x_28 = lean_usize_sub(x_27, x_26); +x_29 = lean_usize_land(x_5, x_28); +x_30 = 5; +x_31 = lean_usize_sub(x_6, x_30); +x_32 = lean_usize_to_nat(x_25); +x_33 = lean_array_get_size(x_24); +x_34 = lean_nat_dec_lt(x_32, x_33); +lean_dec(x_33); +if (x_34 == 0) +{ +lean_object* x_35; +lean_dec(x_32); +lean_dec(x_2); +lean_dec(x_1); +x_35 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_35, 0, x_24); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_36 = lean_array_fget(x_24, x_32); +x_37 = lean_box(0); +x_38 = lean_array_fset(x_24, x_32, x_37); +x_39 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(x_1, x_2, x_3, x_36, x_29, x_31); +x_40 = lean_array_fset(x_38, x_32, x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_41, 0, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +x_42 = !lean_is_exclusive(x_4); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = lean_ctor_get(x_4, 0); +x_44 = lean_usize_to_nat(x_5); +x_45 = lean_array_get_size(x_43); +x_46 = lean_nat_dec_lt(x_44, x_45); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_dec(x_44); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_47 = lean_array_fget(x_43, x_44); +x_48 = lean_box(0); +x_49 = lean_array_fset(x_43, x_44, x_48); +x_50 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(x_47, x_1, x_2); +x_51 = lean_array_fset(x_49, x_44, x_50); +lean_dec(x_44); +lean_ctor_set(x_4, 0, x_51); +return x_4; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_52 = lean_ctor_get(x_4, 0); +lean_inc(x_52); +lean_dec(x_4); +x_53 = lean_usize_to_nat(x_5); +x_54 = lean_array_get_size(x_52); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_2); +lean_dec(x_1); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_52); +return x_56; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_57 = lean_array_fget(x_52, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_52, x_53, x_58); +x_60 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(x_57, x_1, x_2); +x_61 = lean_array_fset(x_59, x_53, x_60); +lean_dec(x_53); +x_62 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_62, 0, x_61); +return x_62; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; size_t x_9; lean_object* x_10; uint8_t x_11; +x_7 = lean_ctor_get(x_4, 0); +x_8 = lean_ctor_get(x_4, 1); +x_9 = lean_ctor_get_usize(x_4, 4); +x_10 = lean_ctor_get(x_4, 3); +x_11 = lean_nat_dec_le(x_10, x_5); +if (x_11 == 0) +{ +size_t x_12; lean_object* x_13; +x_12 = lean_usize_of_nat(x_5); +x_13 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(x_1, x_2, x_3, x_7, x_12, x_9); +lean_ctor_set(x_4, 0, x_13); +return x_4; +} +else +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_nat_sub(x_5, x_10); +x_15 = lean_array_get_size(x_8); +x_16 = lean_nat_dec_lt(x_14, x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_dec(x_14); +lean_dec(x_2); +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_array_fget(x_8, x_14); +x_18 = lean_box(0); +x_19 = lean_array_fset(x_8, x_14, x_18); +x_20 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(x_17, x_1, x_2); +x_21 = lean_array_fset(x_19, x_14, x_20); +lean_dec(x_14); +lean_ctor_set(x_4, 1, x_21); +return x_4; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; lean_object* x_26; uint8_t x_27; +x_22 = lean_ctor_get(x_4, 0); +x_23 = lean_ctor_get(x_4, 1); +x_24 = lean_ctor_get(x_4, 2); +x_25 = lean_ctor_get_usize(x_4, 4); +x_26 = lean_ctor_get(x_4, 3); +lean_inc(x_26); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_4); +x_27 = lean_nat_dec_le(x_26, x_5); +if (x_27 == 0) +{ +size_t x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_usize_of_nat(x_5); +x_29 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(x_1, x_2, x_3, x_22, x_28, x_25); +x_30 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_23); +lean_ctor_set(x_30, 2, x_24); +lean_ctor_set(x_30, 3, x_26); +lean_ctor_set_usize(x_30, 4, x_25); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_nat_sub(x_5, x_26); +x_32 = lean_array_get_size(x_23); +x_33 = lean_nat_dec_lt(x_31, x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; +lean_dec(x_31); +lean_dec(x_2); +lean_dec(x_1); +x_34 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_34, 0, x_22); +lean_ctor_set(x_34, 1, x_23); +lean_ctor_set(x_34, 2, x_24); +lean_ctor_set(x_34, 3, x_26); +lean_ctor_set_usize(x_34, 4, x_25); +return x_34; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_array_fget(x_23, x_31); +x_36 = lean_box(0); +x_37 = lean_array_fset(x_23, x_31, x_36); +x_38 = l_Lean_AssocList_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__1(x_35, x_1, x_2); +x_39 = lean_array_fset(x_37, x_31, x_38); +lean_dec(x_31); +x_40 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_40, 0, x_22); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_24); +lean_ctor_set(x_40, 3, x_26); +lean_ctor_set_usize(x_40, 4, x_25); +return x_40; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_st_ref_take(x_4, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 9); +lean_inc(x_15); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; uint8_t x_19; +x_18 = lean_ctor_get(x_14, 9); +lean_dec(x_18); +x_19 = !lean_is_exclusive(x_15); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_20 = lean_ctor_get(x_15, 6); +x_21 = lean_box(0); +x_22 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(x_2, x_3, x_21, x_20, x_1); +lean_ctor_set(x_15, 6, x_22); +x_23 = lean_st_ref_set(x_4, x_14, x_16); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_23, 0); +lean_dec(x_25); +x_26 = lean_box(0); +lean_ctor_set(x_23, 0, x_26); +return x_23; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_23, 1); +lean_inc(x_27); +lean_dec(x_23); +x_28 = lean_box(0); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_30 = lean_ctor_get(x_15, 0); +x_31 = lean_ctor_get(x_15, 1); +x_32 = lean_ctor_get(x_15, 2); +x_33 = lean_ctor_get(x_15, 3); +x_34 = lean_ctor_get(x_15, 4); +x_35 = lean_ctor_get(x_15, 5); +x_36 = lean_ctor_get(x_15, 6); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_15); +x_37 = lean_box(0); +x_38 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(x_2, x_3, x_37, x_36, x_1); +x_39 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_39, 0, x_30); +lean_ctor_set(x_39, 1, x_31); +lean_ctor_set(x_39, 2, x_32); +lean_ctor_set(x_39, 3, x_33); +lean_ctor_set(x_39, 4, x_34); +lean_ctor_set(x_39, 5, x_35); +lean_ctor_set(x_39, 6, x_38); +lean_ctor_set(x_14, 9, x_39); +x_40 = lean_st_ref_set(x_4, x_14, x_16); +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_42 = x_40; +} else { + lean_dec_ref(x_40); + x_42 = lean_box(0); +} +x_43 = lean_box(0); +if (lean_is_scalar(x_42)) { + x_44 = lean_alloc_ctor(0, 2, 0); +} else { + x_44 = x_42; +} +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_41); +return x_44; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_45 = lean_ctor_get(x_14, 0); +x_46 = lean_ctor_get(x_14, 1); +x_47 = lean_ctor_get(x_14, 2); +x_48 = lean_ctor_get(x_14, 3); +x_49 = lean_ctor_get(x_14, 4); +x_50 = lean_ctor_get(x_14, 5); +x_51 = lean_ctor_get(x_14, 6); +x_52 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); +x_53 = lean_ctor_get(x_14, 7); +x_54 = lean_ctor_get(x_14, 8); +x_55 = lean_ctor_get(x_14, 10); +x_56 = lean_ctor_get(x_14, 11); +x_57 = lean_ctor_get(x_14, 12); +x_58 = lean_ctor_get(x_14, 13); +x_59 = lean_ctor_get(x_14, 14); +x_60 = lean_ctor_get(x_14, 15); +x_61 = lean_ctor_get(x_14, 16); +x_62 = lean_ctor_get(x_14, 17); +x_63 = lean_ctor_get(x_14, 18); +x_64 = lean_ctor_get(x_14, 19); +x_65 = lean_ctor_get(x_14, 20); +x_66 = lean_ctor_get(x_14, 21); +x_67 = lean_ctor_get(x_14, 22); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_14); +x_68 = lean_ctor_get(x_15, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_15, 1); +lean_inc(x_69); +x_70 = lean_ctor_get(x_15, 2); +lean_inc(x_70); +x_71 = lean_ctor_get(x_15, 3); +lean_inc(x_71); +x_72 = lean_ctor_get(x_15, 4); +lean_inc(x_72); +x_73 = lean_ctor_get(x_15, 5); +lean_inc(x_73); +x_74 = lean_ctor_get(x_15, 6); +lean_inc(x_74); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + lean_ctor_release(x_15, 2); + lean_ctor_release(x_15, 3); + lean_ctor_release(x_15, 4); + lean_ctor_release(x_15, 5); + lean_ctor_release(x_15, 6); + x_75 = x_15; +} else { + lean_dec_ref(x_15); + x_75 = lean_box(0); +} +x_76 = lean_box(0); +x_77 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(x_2, x_3, x_76, x_74, x_1); +if (lean_is_scalar(x_75)) { + x_78 = lean_alloc_ctor(0, 7, 0); +} else { + x_78 = x_75; +} +lean_ctor_set(x_78, 0, x_68); +lean_ctor_set(x_78, 1, x_69); +lean_ctor_set(x_78, 2, x_70); +lean_ctor_set(x_78, 3, x_71); +lean_ctor_set(x_78, 4, x_72); +lean_ctor_set(x_78, 5, x_73); +lean_ctor_set(x_78, 6, x_77); +x_79 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_79, 0, x_45); +lean_ctor_set(x_79, 1, x_46); +lean_ctor_set(x_79, 2, x_47); +lean_ctor_set(x_79, 3, x_48); +lean_ctor_set(x_79, 4, x_49); +lean_ctor_set(x_79, 5, x_50); +lean_ctor_set(x_79, 6, x_51); +lean_ctor_set(x_79, 7, x_53); +lean_ctor_set(x_79, 8, x_54); +lean_ctor_set(x_79, 9, x_78); +lean_ctor_set(x_79, 10, x_55); +lean_ctor_set(x_79, 11, x_56); +lean_ctor_set(x_79, 12, x_57); +lean_ctor_set(x_79, 13, x_58); +lean_ctor_set(x_79, 14, x_59); +lean_ctor_set(x_79, 15, x_60); +lean_ctor_set(x_79, 16, x_61); +lean_ctor_set(x_79, 17, x_62); +lean_ctor_set(x_79, 18, x_63); +lean_ctor_set(x_79, 19, x_64); +lean_ctor_set(x_79, 20, x_65); +lean_ctor_set(x_79, 21, x_66); +lean_ctor_set(x_79, 22, x_67); +lean_ctor_set_uint8(x_79, sizeof(void*)*23, x_52); +x_80 = lean_st_ref_set(x_4, x_79, x_16); +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_82 = x_80; +} else { + lean_dec_ref(x_80); + x_82 = lean_box(0); +} +x_83 = lean_box(0); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); +} else { + x_84 = x_82; +} +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__2(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; size_t x_8; lean_object* x_9; +x_7 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_8 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_9 = l_Lean_PersistentArray_modifyAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__5(x_1, x_2, x_3, x_4, x_7, x_8); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentArray_modify___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___spec__4(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_2, 2); +lean_inc(x_16); +lean_dec(x_2); +lean_inc(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_17 = lean_apply_11(x_1, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_2 = x_16; +x_11 = x_18; +goto _start; +} +else +{ +uint8_t x_20; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_2, 2); +lean_inc(x_16); +lean_dec(x_2); +lean_inc(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_17 = lean_apply_11(x_1, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_2 = x_16; +x_11 = x_18; +goto _start; +} +else +{ +uint8_t x_20; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_box(0); +x_16 = lean_ctor_get(x_13, 4); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +x_18 = lean_nat_dec_lt(x_1, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_16); +x_19 = l_outOfBounds___rarg(x_15); +x_20 = l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__1(x_2, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = l_Lean_PersistentArray_get_x21___rarg(x_15, x_16, x_1); +x_22 = l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___spec__2(x_2, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachSourceOf(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_2, 2); +lean_inc(x_16); +lean_dec(x_2); +lean_inc(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_17 = lean_apply_11(x_1, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_2 = x_16; +x_11 = x_18; +goto _start; +} +else +{ +uint8_t x_20; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_12 = lean_box(0); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_2, 2); +lean_inc(x_16); +lean_dec(x_2); +lean_inc(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_17 = lean_apply_11(x_1, x_14, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_2 = x_16; +x_11 = x_18; +goto _start; +} +else +{ +uint8_t x_20; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_17); +if (x_20 == 0) +{ +return x_17; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_12 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_box(0); +x_16 = lean_ctor_get(x_13, 5); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_ctor_get(x_16, 2); +lean_inc(x_17); +x_18 = lean_nat_dec_lt(x_1, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_16); +x_19 = l_outOfBounds___rarg(x_15); +x_20 = l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__1(x_2, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; +x_21 = l_Lean_PersistentArray_get_x21___rarg(x_15, x_16, x_1); +x_22 = l_Lean_AssocList_forM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___spec__2(x_2, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_22; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_forEachTargetOf(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +return x_12; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = 1; +x_18 = lean_box(x_17); +lean_ctor_set(x_13, 0, x_18); +return x_13; +} +else +{ +lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_dec(x_13); +x_20 = 1; +x_21 = lean_box(x_20); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_19); +return x_22; +} +} +else +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_13); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_13, 0); +lean_dec(x_24); +x_25 = lean_ctor_get(x_14, 0); +lean_inc(x_25); +lean_dec(x_14); +x_26 = lean_int_dec_lt(x_3, x_25); +lean_dec(x_25); +x_27 = lean_box(x_26); +lean_ctor_set(x_13, 0, x_27); +return x_13; +} +else +{ +lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; +x_28 = lean_ctor_get(x_13, 1); +lean_inc(x_28); +lean_dec(x_13); +x_29 = lean_ctor_get(x_14, 0); +lean_inc(x_29); +lean_dec(x_14); +x_30 = lean_int_dec_lt(x_3, x_29); +lean_dec(x_29); +x_31 = lean_box(x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_28); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +x_10 = l___private_Init_Data_Repr_0__Nat_reprFast(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Lean_MessageData_ofFormat(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +lean_inc(x_1); +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_1); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_ctor_get(x_2, 1); +lean_inc(x_20); +lean_dec(x_2); +x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); +x_22 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_1); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_30 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lean_MessageData_ofFormat(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_28); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_16); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_6); +x_34 = lean_ctor_get(x_2, 0); +lean_inc(x_34); +x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_34); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l_Lean_MessageData_ofFormat(x_36); +x_38 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +lean_inc(x_1); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_ctor_get(x_2, 1); +lean_inc(x_45); +lean_dec(x_2); +x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_45); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l_Lean_MessageData_ofFormat(x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_1); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_41); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_53 = lean_nat_abs(x_3); +lean_dec(x_3); +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_53, x_54); +lean_dec(x_53); +x_56 = lean_ctor_get(x_2, 0); +lean_inc(x_56); +x_57 = l___private_Init_Data_Repr_0__Nat_reprFast(x_56); +x_58 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_59 = l_Lean_MessageData_ofFormat(x_58); +x_60 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +lean_inc(x_1); +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_1); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_62); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_nat_add(x_55, x_54); +lean_dec(x_55); +x_68 = l___private_Init_Data_Repr_0__Nat_reprFast(x_67); +x_69 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_MessageData_ofFormat(x_69); +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_ctor_get(x_2, 1); +lean_inc(x_74); +lean_dec(x_2); +x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_77 = l_Lean_MessageData_ofFormat(x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_60); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_1); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; lean_object* x_13; +x_11 = 0; +x_12 = lean_box(x_11); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_1, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_18); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof(x_20, x_23, x_3, x_17, x_4); +x_26 = l_Lean_Meta_Grind_pushEqTrue(x_5, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_24); +x_27 = !lean_is_exclusive(x_26); +if (x_27 == 0) +{ +lean_object* x_28; uint8_t x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_26, 0); +lean_dec(x_28); +x_29 = 1; +x_30 = lean_box(x_29); +lean_ctor_set(x_26, 0, x_30); +return x_26; +} +else +{ +lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_dec(x_26); +x_32 = 1; +x_33 = lean_box(x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_31); +return x_34; +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("propagate", 9, 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ==> ", 5, 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" = True", 7, 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1; +x_16 = lean_ctor_get(x_4, 2); +x_17 = lean_int_dec_le(x_3, x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_18 = lean_box(0); +x_19 = lean_apply_10(x_15, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3; +x_21 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_unbox(x_22); +lean_dec(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_box(0); +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(x_1, x_2, x_3, x_16, x_5, x_25, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_24); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_26; +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_28 = lean_ctor_get(x_21, 1); +x_29 = lean_ctor_get(x_21, 0); +lean_dec(x_29); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_30 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_30, 0, x_1); +lean_ctor_set(x_30, 1, x_2); +lean_ctor_set(x_30, 2, x_3); +x_31 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_32 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___spec__1(x_31, x_30); +lean_ctor_set_tag(x_21, 7); +lean_ctor_set(x_21, 1, x_32); +lean_ctor_set(x_21, 0, x_31); +x_33 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5; +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_21); +lean_ctor_set(x_34, 1, x_33); +lean_inc(x_5); +x_35 = l_Lean_MessageData_ofExpr(x_5); +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +x_37 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_20, x_38, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_28); +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_42 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(x_1, x_2, x_3, x_16, x_5, x_40, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_41); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_40); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_42; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_43 = lean_ctor_get(x_21, 1); +lean_inc(x_43); +lean_dec(x_21); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_44 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_44, 0, x_1); +lean_ctor_set(x_44, 1, x_2); +lean_ctor_set(x_44, 2, x_3); +x_45 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_46 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___spec__1(x_45, x_44); +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_48 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +lean_inc(x_5); +x_50 = l_Lean_MessageData_ofExpr(x_5); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +x_52 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_54 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_20, x_53, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_43); +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +x_57 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(x_1, x_2, x_3, x_16, x_5, x_55, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_56); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_55); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_57; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_4); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +x_10 = l___private_Init_Data_Repr_0__Nat_reprFast(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Lean_MessageData_ofFormat(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +lean_inc(x_1); +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_1); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_ctor_get(x_2, 1); +lean_inc(x_20); +lean_dec(x_2); +x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); +x_22 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_1); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_30 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lean_MessageData_ofFormat(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_28); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_16); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_6); +x_34 = lean_ctor_get(x_2, 0); +lean_inc(x_34); +x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_34); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l_Lean_MessageData_ofFormat(x_36); +x_38 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +lean_inc(x_1); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_ctor_get(x_2, 1); +lean_inc(x_45); +lean_dec(x_2); +x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_45); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l_Lean_MessageData_ofFormat(x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_1); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_41); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_53 = lean_nat_abs(x_3); +lean_dec(x_3); +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_53, x_54); +lean_dec(x_53); +x_56 = lean_ctor_get(x_2, 0); +lean_inc(x_56); +x_57 = l___private_Init_Data_Repr_0__Nat_reprFast(x_56); +x_58 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_59 = l_Lean_MessageData_ofFormat(x_58); +x_60 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +lean_inc(x_1); +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_1); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_62); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_nat_add(x_55, x_54); +lean_dec(x_55); +x_68 = l___private_Init_Data_Repr_0__Nat_reprFast(x_67); +x_69 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_MessageData_ofFormat(x_69); +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_ctor_get(x_2, 1); +lean_inc(x_74); +lean_dec(x_2); +x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_77 = l_Lean_MessageData_ofFormat(x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_60); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_1); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_1, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_22); +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof(x_21, x_24, x_3, x_18, x_4); +x_27 = l_Lean_Meta_Grind_pushEqFalse(x_5, x_26, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_25); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_apply_10(x_6, x_28, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_29); +return x_30; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" = False", 8, 8); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1; +x_16 = lean_ctor_get(x_4, 2); +x_17 = lean_int_add(x_3, x_16); +x_18 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_19 = lean_int_dec_lt(x_17, x_18); +lean_dec(x_17); +if (x_19 == 0) +{ +uint8_t x_20; lean_object* x_21; lean_object* x_22; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = 0; +x_21 = lean_box(x_20); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_14); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3; +x_24 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_box(0); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(x_1, x_2, x_3, x_16, x_5, x_15, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_27); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_29; +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_24); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_31 = lean_ctor_get(x_24, 1); +x_32 = lean_ctor_get(x_24, 0); +lean_dec(x_32); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_33 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_33, 0, x_1); +lean_ctor_set(x_33, 1, x_2); +lean_ctor_set(x_33, 2, x_3); +x_34 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_35 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___spec__1(x_34, x_33); +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_35); +lean_ctor_set(x_24, 0, x_34); +x_36 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_24); +lean_ctor_set(x_37, 1, x_36); +lean_inc(x_5); +x_38 = l_Lean_MessageData_ofExpr(x_5); +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +x_40 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_23, x_41, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(x_1, x_2, x_3, x_16, x_5, x_15, x_43, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_44); +lean_dec(x_43); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_45; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_46 = lean_ctor_get(x_24, 1); +lean_inc(x_46); +lean_dec(x_24); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_47 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_47, 0, x_1); +lean_ctor_set(x_47, 1, x_2); +lean_ctor_set(x_47, 2, x_3); +x_48 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_49 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___spec__1(x_48, x_47); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +x_51 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5; +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +lean_inc(x_5); +x_53 = l_Lean_MessageData_ofExpr(x_5); +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +x_55 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2; +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +x_57 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_23, x_56, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_46); +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_57, 1); +lean_inc(x_59); +lean_dec(x_57); +x_60 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(x_1, x_2, x_3, x_16, x_5, x_15, x_58, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_59); +lean_dec(x_58); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_60; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_17; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_4); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_lt(x_4, x_6); +lean_dec(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_4); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_9 = lean_array_fget(x_1, x_4); +x_10 = lean_ctor_get(x_5, 0); +x_11 = lean_ctor_get(x_5, 1); +x_12 = lean_ctor_get(x_9, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_9, 1); +lean_inc(x_13); +lean_dec(x_9); +x_14 = lean_nat_dec_eq(x_10, x_12); +lean_dec(x_12); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_13); +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_add(x_4, x_15); +lean_dec(x_4); +x_3 = lean_box(0); +x_4 = x_16; +goto _start; +} +else +{ +uint8_t x_18; +x_18 = lean_nat_dec_eq(x_11, x_13); +lean_dec(x_13); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_add(x_4, x_19); +lean_dec(x_4); +x_3 = lean_box(0); +x_4 = x_20; +goto _start; +} +else +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_array_fget(x_2, x_4); +lean_dec(x_4); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2(lean_object* x_1, size_t x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; size_t x_6; size_t x_7; size_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_5 = lean_ctor_get(x_1, 0); +x_6 = 5; +x_7 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_8 = lean_usize_land(x_2, x_7); +x_9 = lean_usize_to_nat(x_8); +x_10 = lean_box(2); +x_11 = lean_array_get(x_10, x_5, x_9); +lean_dec(x_9); +lean_dec(x_5); +switch (lean_obj_tag(x_11)) { +case 0: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_ctor_get(x_3, 0); +x_15 = lean_ctor_get(x_3, 1); +x_16 = lean_ctor_get(x_12, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_dec(x_12); +x_18 = lean_nat_dec_eq(x_14, x_16); +lean_dec(x_16); +if (x_18 == 0) +{ +lean_object* x_19; +lean_dec(x_17); +lean_dec(x_13); +lean_free_object(x_1); +x_19 = lean_box(0); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = lean_nat_dec_eq(x_15, x_17); +lean_dec(x_17); +if (x_20 == 0) +{ +lean_object* x_21; +lean_dec(x_13); +lean_free_object(x_1); +x_21 = lean_box(0); +return x_21; +} +else +{ +lean_ctor_set_tag(x_1, 1); +lean_ctor_set(x_1, 0, x_13); +return x_1; +} +} +} +case 1: +{ +lean_object* x_22; size_t x_23; +lean_free_object(x_1); +x_22 = lean_ctor_get(x_11, 0); +lean_inc(x_22); +lean_dec(x_11); +x_23 = lean_usize_shift_right(x_2, x_6); +x_1 = x_22; +x_2 = x_23; +goto _start; +} +default: +{ +lean_object* x_25; +lean_free_object(x_1); +x_25 = lean_box(0); +return x_25; +} +} +} +else +{ +lean_object* x_26; size_t x_27; size_t x_28; size_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); +lean_dec(x_1); +x_27 = 5; +x_28 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_29 = lean_usize_land(x_2, x_28); +x_30 = lean_usize_to_nat(x_29); +x_31 = lean_box(2); +x_32 = lean_array_get(x_31, x_26, x_30); +lean_dec(x_30); +lean_dec(x_26); +switch (lean_obj_tag(x_32)) { +case 0: +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = lean_ctor_get(x_3, 0); +x_36 = lean_ctor_get(x_3, 1); +x_37 = lean_ctor_get(x_33, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_33, 1); +lean_inc(x_38); +lean_dec(x_33); +x_39 = lean_nat_dec_eq(x_35, x_37); +lean_dec(x_37); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_38); +lean_dec(x_34); +x_40 = lean_box(0); +return x_40; +} +else +{ +uint8_t x_41; +x_41 = lean_nat_dec_eq(x_36, x_38); +lean_dec(x_38); +if (x_41 == 0) +{ +lean_object* x_42; +lean_dec(x_34); +x_42 = lean_box(0); +return x_42; +} +else +{ +lean_object* x_43; +x_43 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_43, 0, x_34); +return x_43; +} +} +} +case 1: +{ +lean_object* x_44; size_t x_45; +x_44 = lean_ctor_get(x_32, 0); +lean_inc(x_44); +lean_dec(x_32); +x_45 = lean_usize_shift_right(x_2, x_27); +x_1 = x_44; +x_2 = x_45; +goto _start; +} +default: +{ +lean_object* x_47; +x_47 = lean_box(0); +return x_47; +} +} +} +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_1, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_1, 1); +lean_inc(x_49); +lean_dec(x_1); +x_50 = lean_unsigned_to_nat(0u); +x_51 = l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3(x_48, x_49, lean_box(0), x_50, x_3); +lean_dec(x_49); +lean_dec(x_48); +return x_51; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint64_t x_5; uint64_t x_6; uint64_t x_7; size_t x_8; lean_object* x_9; +x_3 = lean_ctor_get(x_2, 0); +x_4 = lean_ctor_get(x_2, 1); +x_5 = lean_uint64_of_nat(x_3); +x_6 = lean_uint64_of_nat(x_4); +x_7 = lean_uint64_mix_hash(x_5, x_6); +x_8 = lean_uint64_to_usize(x_7); +x_9 = l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2(x_1, x_8, x_2); +return x_9; +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_13; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_3); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_14 = lean_ctor_get(x_2, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + lean_ctor_release(x_2, 1); + x_16 = x_2; +} else { + lean_dec_ref(x_2); + x_16 = lean_box(0); +} +x_23 = lean_ctor_get(x_14, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_inc(x_24); +x_25 = l_Lean_Meta_Grind_isEqTrue(x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_unbox(x_26); +lean_dec(x_26); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +lean_inc(x_24); +x_29 = l_Lean_Meta_Grind_isEqFalse(x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_unbox(x_30); +lean_dec(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +lean_inc(x_1); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_33 = lean_apply_11(x_1, x_23, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; uint8_t x_35; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_unbox(x_34); +lean_dec(x_34); +if (x_35 == 0) +{ +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_33, 1); +lean_inc(x_36); +lean_dec(x_33); +x_37 = 1; +x_17 = x_37; +x_18 = x_36; +goto block_22; +} +else +{ +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_33, 1); +lean_inc(x_38); +lean_dec(x_33); +x_39 = 0; +x_17 = x_39; +x_18 = x_38; +goto block_22; +} +} +else +{ +uint8_t x_40; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_40 = !lean_is_exclusive(x_33); +if (x_40 == 0) +{ +return x_33; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_33, 0); +x_42 = lean_ctor_get(x_33, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_33); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} +} +} +else +{ +lean_object* x_44; uint8_t x_45; +lean_dec(x_24); +lean_dec(x_23); +x_44 = lean_ctor_get(x_29, 1); +lean_inc(x_44); +lean_dec(x_29); +x_45 = 0; +x_17 = x_45; +x_18 = x_44; +goto block_22; +} +} +else +{ +uint8_t x_46; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_46 = !lean_is_exclusive(x_29); +if (x_46 == 0) +{ +return x_29; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_29, 0); +x_48 = lean_ctor_get(x_29, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_29); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; +} +} +} +else +{ +lean_object* x_50; uint8_t x_51; +lean_dec(x_24); +lean_dec(x_23); +x_50 = lean_ctor_get(x_25, 1); +lean_inc(x_50); +lean_dec(x_25); +x_51 = 0; +x_17 = x_51; +x_18 = x_50; +goto block_22; +} +} +else +{ +uint8_t x_52; +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_52 = !lean_is_exclusive(x_25); +if (x_52 == 0) +{ +return x_25; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_25, 0); +x_54 = lean_ctor_get(x_25, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_25); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; +} +} +block_22: +{ +if (x_17 == 0) +{ +lean_dec(x_16); +lean_dec(x_14); +x_2 = x_15; +x_12 = x_18; +goto _start; +} +else +{ +lean_object* x_20; +if (lean_is_scalar(x_16)) { + x_20 = lean_alloc_ctor(1, 2, 0); +} else { + x_20 = x_16; +} +lean_ctor_set(x_20, 0, x_14); +lean_ctor_set(x_20, 1, x_3); +x_2 = x_15; +x_3 = x_20; +x_12 = x_18; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_array_get_size(x_2); +x_8 = lean_nat_dec_lt(x_5, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +lean_dec(x_5); +return x_6; +} +else +{ +lean_object* x_9; lean_object* x_10; size_t x_11; size_t x_12; size_t x_13; size_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; size_t x_22; size_t x_23; lean_object* x_24; +x_9 = lean_array_fget(x_2, x_5); +x_10 = lean_array_fget(x_3, x_5); +x_11 = 1; +x_12 = lean_usize_sub(x_1, x_11); +x_13 = 5; +x_14 = lean_usize_mul(x_13, x_12); +x_15 = lean_unsigned_to_nat(1u); +x_16 = lean_nat_add(x_5, x_15); +lean_dec(x_5); +x_17 = lean_ctor_get(x_9, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_9, 1); +lean_inc(x_18); +x_19 = lean_uint64_of_nat(x_17); +lean_dec(x_17); +x_20 = lean_uint64_of_nat(x_18); +lean_dec(x_18); +x_21 = lean_uint64_mix_hash(x_19, x_20); +x_22 = lean_uint64_to_usize(x_21); +x_23 = lean_usize_shift_right(x_22, x_14); +x_24 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_6, x_23, x_1, x_9, x_10); +x_4 = lean_box(0); +x_5 = x_16; +x_6 = x_24; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_5); +x_8 = lean_nat_dec_lt(x_2, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +uint8_t x_9; +lean_dec(x_2); +x_9 = !lean_is_exclusive(x_1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 1); +lean_dec(x_10); +x_11 = lean_ctor_get(x_1, 0); +lean_dec(x_11); +x_12 = lean_array_push(x_5, x_3); +x_13 = lean_array_push(x_6, x_4); +lean_ctor_set(x_1, 1, x_13); +lean_ctor_set(x_1, 0, x_12); +return x_1; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_14 = lean_array_push(x_5, x_3); +x_15 = lean_array_push(x_6, x_4); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_17 = lean_array_fget(x_5, x_2); +x_18 = lean_ctor_get(x_3, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_3, 1); +lean_inc(x_19); +x_20 = lean_ctor_get(x_17, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_nat_dec_eq(x_18, x_20); +lean_dec(x_20); +lean_dec(x_18); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_21); +lean_dec(x_19); +lean_dec(x_6); +lean_dec(x_5); +x_23 = lean_unsigned_to_nat(1u); +x_24 = lean_nat_add(x_2, x_23); +lean_dec(x_2); +x_2 = x_24; +goto _start; +} +else +{ +uint8_t x_26; +x_26 = lean_nat_dec_eq(x_19, x_21); +lean_dec(x_21); +lean_dec(x_19); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +lean_dec(x_6); +lean_dec(x_5); +x_27 = lean_unsigned_to_nat(1u); +x_28 = lean_nat_add(x_2, x_27); +lean_dec(x_2); +x_2 = x_28; +goto _start; +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_1); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_31 = lean_ctor_get(x_1, 1); +lean_dec(x_31); +x_32 = lean_ctor_get(x_1, 0); +lean_dec(x_32); +x_33 = lean_array_fset(x_5, x_2, x_3); +x_34 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +lean_ctor_set(x_1, 1, x_34); +lean_ctor_set(x_1, 0, x_33); +return x_1; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_1); +x_35 = lean_array_fset(x_5, x_2, x_3); +x_36 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_1); +if (x_6 == 0) +{ +lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_7 = lean_ctor_get(x_1, 0); +x_8 = 1; +x_9 = 5; +x_10 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_11 = lean_usize_land(x_2, x_10); +x_12 = lean_usize_to_nat(x_11); +x_13 = lean_array_get_size(x_7); +x_14 = lean_nat_dec_lt(x_12, x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_dec(x_12); +lean_dec(x_5); +lean_dec(x_4); +return x_1; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_array_fget(x_7, x_12); +x_16 = lean_box(0); +x_17 = lean_array_fset(x_7, x_12, x_16); +switch (lean_obj_tag(x_15)) { +case 0: +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +x_21 = lean_ctor_get(x_4, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_4, 1); +lean_inc(x_22); +x_23 = lean_ctor_get(x_19, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_19, 1); +lean_inc(x_24); +x_25 = lean_nat_dec_eq(x_21, x_23); +lean_dec(x_23); +lean_dec(x_21); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_dec(x_24); +lean_dec(x_22); +lean_free_object(x_15); +x_26 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_26); +x_28 = lean_array_fset(x_17, x_12, x_27); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_28); +return x_1; +} +else +{ +uint8_t x_29; +x_29 = lean_nat_dec_eq(x_22, x_24); +lean_dec(x_24); +lean_dec(x_22); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_free_object(x_15); +x_30 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); +x_31 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_31, 0, x_30); +x_32 = lean_array_fset(x_17, x_12, x_31); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_32); +return x_1; +} +else +{ +lean_object* x_33; +lean_dec(x_20); +lean_dec(x_19); +lean_ctor_set(x_15, 1, x_5); +lean_ctor_set(x_15, 0, x_4); +x_33 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_33); +return x_1; +} +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_34 = lean_ctor_get(x_15, 0); +x_35 = lean_ctor_get(x_15, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_15); +x_36 = lean_ctor_get(x_4, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_4, 1); +lean_inc(x_37); +x_38 = lean_ctor_get(x_34, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_34, 1); +lean_inc(x_39); +x_40 = lean_nat_dec_eq(x_36, x_38); +lean_dec(x_38); +lean_dec(x_36); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_dec(x_39); +lean_dec(x_37); +x_41 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_34, x_35, x_4, x_5); +x_42 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_42, 0, x_41); +x_43 = lean_array_fset(x_17, x_12, x_42); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_43); +return x_1; +} +else +{ +uint8_t x_44; +x_44 = lean_nat_dec_eq(x_37, x_39); +lean_dec(x_39); +lean_dec(x_37); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_34, x_35, x_4, x_5); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = lean_array_fset(x_17, x_12, x_46); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_47); +return x_1; +} +else +{ +lean_object* x_48; lean_object* x_49; +lean_dec(x_35); +lean_dec(x_34); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_4); +lean_ctor_set(x_48, 1, x_5); +x_49 = lean_array_fset(x_17, x_12, x_48); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_49); +return x_1; +} +} +} +} +case 1: +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_15); +if (x_50 == 0) +{ +lean_object* x_51; size_t x_52; size_t x_53; lean_object* x_54; lean_object* x_55; +x_51 = lean_ctor_get(x_15, 0); +x_52 = lean_usize_shift_right(x_2, x_9); +x_53 = lean_usize_add(x_3, x_8); +x_54 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_51, x_52, x_53, x_4, x_5); +lean_ctor_set(x_15, 0, x_54); +x_55 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_55); +return x_1; +} +else +{ +lean_object* x_56; size_t x_57; size_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_56 = lean_ctor_get(x_15, 0); +lean_inc(x_56); +lean_dec(x_15); +x_57 = lean_usize_shift_right(x_2, x_9); +x_58 = lean_usize_add(x_3, x_8); +x_59 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_56, x_57, x_58, x_4, x_5); +x_60 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_60, 0, x_59); +x_61 = lean_array_fset(x_17, x_12, x_60); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_61); +return x_1; +} +} +default: +{ +lean_object* x_62; lean_object* x_63; +x_62 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_62, 0, x_4); +lean_ctor_set(x_62, 1, x_5); +x_63 = lean_array_fset(x_17, x_12, x_62); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_63); +return x_1; +} +} +} +} +else +{ +lean_object* x_64; size_t x_65; size_t x_66; size_t x_67; size_t x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; +x_64 = lean_ctor_get(x_1, 0); +lean_inc(x_64); +lean_dec(x_1); +x_65 = 1; +x_66 = 5; +x_67 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_68 = lean_usize_land(x_2, x_67); +x_69 = lean_usize_to_nat(x_68); +x_70 = lean_array_get_size(x_64); +x_71 = lean_nat_dec_lt(x_69, x_70); +lean_dec(x_70); +if (x_71 == 0) +{ +lean_object* x_72; +lean_dec(x_69); +lean_dec(x_5); +lean_dec(x_4); +x_72 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_72, 0, x_64); +return x_72; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_array_fget(x_64, x_69); +x_74 = lean_box(0); +x_75 = lean_array_fset(x_64, x_69, x_74); +switch (lean_obj_tag(x_73)) { +case 0: +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; +x_76 = lean_ctor_get(x_73, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_73, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_78 = x_73; +} else { + lean_dec_ref(x_73); + x_78 = lean_box(0); +} +x_79 = lean_ctor_get(x_4, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_4, 1); +lean_inc(x_80); +x_81 = lean_ctor_get(x_76, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_76, 1); +lean_inc(x_82); +x_83 = lean_nat_dec_eq(x_79, x_81); +lean_dec(x_81); +lean_dec(x_79); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_82); +lean_dec(x_80); +lean_dec(x_78); +x_84 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_76, x_77, x_4, x_5); +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_84); +x_86 = lean_array_fset(x_75, x_69, x_85); +lean_dec(x_69); +x_87 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_87, 0, x_86); +return x_87; +} +else +{ +uint8_t x_88; +x_88 = lean_nat_dec_eq(x_80, x_82); +lean_dec(x_82); +lean_dec(x_80); +if (x_88 == 0) +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_dec(x_78); +x_89 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_76, x_77, x_4, x_5); +x_90 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_90, 0, x_89); +x_91 = lean_array_fset(x_75, x_69, x_90); +lean_dec(x_69); +x_92 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_92, 0, x_91); +return x_92; +} +else +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(x_77); +lean_dec(x_76); +if (lean_is_scalar(x_78)) { + x_93 = lean_alloc_ctor(0, 2, 0); +} else { + x_93 = x_78; +} +lean_ctor_set(x_93, 0, x_4); +lean_ctor_set(x_93, 1, x_5); +x_94 = lean_array_fset(x_75, x_69, x_93); +lean_dec(x_69); +x_95 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_95, 0, x_94); +return x_95; +} +} +} +case 1: +{ +lean_object* x_96; lean_object* x_97; size_t x_98; size_t x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_96 = lean_ctor_get(x_73, 0); +lean_inc(x_96); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + x_97 = x_73; +} else { + lean_dec_ref(x_73); + x_97 = lean_box(0); +} +x_98 = lean_usize_shift_right(x_2, x_66); +x_99 = lean_usize_add(x_3, x_65); +x_100 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_96, x_98, x_99, x_4, x_5); +if (lean_is_scalar(x_97)) { + x_101 = lean_alloc_ctor(1, 1, 0); +} else { + x_101 = x_97; +} +lean_ctor_set(x_101, 0, x_100); +x_102 = lean_array_fset(x_75, x_69, x_101); +lean_dec(x_69); +x_103 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_103, 0, x_102); +return x_103; +} +default: +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_4); +lean_ctor_set(x_104, 1, x_5); +x_105 = lean_array_fset(x_75, x_69, x_104); +lean_dec(x_69); +x_106 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_106, 0, x_105); +return x_106; +} +} +} +} +} +else +{ +uint8_t x_107; +x_107 = !lean_is_exclusive(x_1); +if (x_107 == 0) +{ +lean_object* x_108; lean_object* x_109; size_t x_110; uint8_t x_111; +x_108 = lean_unsigned_to_nat(0u); +x_109 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__8(x_1, x_108, x_4, x_5); +x_110 = 7; +x_111 = lean_usize_dec_le(x_110, x_3); +if (x_111 == 0) +{ +lean_object* x_112; lean_object* x_113; uint8_t x_114; +x_112 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_109); +x_113 = lean_unsigned_to_nat(4u); +x_114 = lean_nat_dec_lt(x_112, x_113); +lean_dec(x_112); +if (x_114 == 0) +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_115 = lean_ctor_get(x_109, 0); +lean_inc(x_115); +x_116 = lean_ctor_get(x_109, 1); +lean_inc(x_116); +lean_dec(x_109); +x_117 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_118 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7(x_3, x_115, x_116, lean_box(0), x_108, x_117); +lean_dec(x_116); +lean_dec(x_115); +return x_118; +} +else +{ +return x_109; +} +} +else +{ +return x_109; +} +} +else +{ +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; size_t x_124; uint8_t x_125; +x_119 = lean_ctor_get(x_1, 0); +x_120 = lean_ctor_get(x_1, 1); +lean_inc(x_120); +lean_inc(x_119); +lean_dec(x_1); +x_121 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_121, 0, x_119); +lean_ctor_set(x_121, 1, x_120); +x_122 = lean_unsigned_to_nat(0u); +x_123 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__8(x_121, x_122, x_4, x_5); +x_124 = 7; +x_125 = lean_usize_dec_le(x_124, x_3); +if (x_125 == 0) +{ +lean_object* x_126; lean_object* x_127; uint8_t x_128; +x_126 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_123); +x_127 = lean_unsigned_to_nat(4u); +x_128 = lean_nat_dec_lt(x_126, x_127); +lean_dec(x_126); +if (x_128 == 0) +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_129 = lean_ctor_get(x_123, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_123, 1); +lean_inc(x_130); +lean_dec(x_123); +x_131 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_132 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7(x_3, x_129, x_130, lean_box(0), x_122, x_131); +lean_dec(x_130); +lean_dec(x_129); +return x_132; +} +else +{ +return x_123; +} +} +else +{ +return x_123; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; lean_object* x_6; uint64_t x_7; uint64_t x_8; uint64_t x_9; size_t x_10; lean_object* x_11; +x_4 = 1; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +x_7 = lean_uint64_of_nat(x_5); +lean_dec(x_5); +x_8 = lean_uint64_of_nat(x_6); +lean_dec(x_6); +x_9 = lean_uint64_mix_hash(x_7, x_8); +x_10 = lean_uint64_to_usize(x_9); +x_11 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_1, x_10, x_4, x_2, x_3); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; uint8_t x_14; +x_13 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +x_17 = lean_ctor_get(x_15, 3); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_1); +lean_ctor_set(x_18, 1, x_2); +x_19 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_17, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; +lean_dec(x_18); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_20 = lean_box(0); +lean_ctor_set(x_13, 0, x_20); +return x_13; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_free_object(x_13); +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_box(0); +lean_inc(x_4); +x_23 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__4(x_3, x_21, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_List_reverse___rarg(x_24); +x_27 = lean_st_ref_take(x_4, x_25); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_28, 9); +lean_inc(x_29); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = !lean_is_exclusive(x_28); +if (x_31 == 0) +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_28, 9); +lean_dec(x_32); +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_34 = lean_ctor_get(x_29, 3); +x_35 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_34, x_18, x_26); +lean_ctor_set(x_29, 3, x_35); +x_36 = lean_st_ref_set(x_4, x_28, x_30); +lean_dec(x_4); +x_37 = !lean_is_exclusive(x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_36, 0); +lean_dec(x_38); +x_39 = lean_box(0); +lean_ctor_set(x_36, 0, x_39); +return x_36; +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +lean_dec(x_36); +x_41 = lean_box(0); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +return x_42; +} +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_43 = lean_ctor_get(x_29, 0); +x_44 = lean_ctor_get(x_29, 1); +x_45 = lean_ctor_get(x_29, 2); +x_46 = lean_ctor_get(x_29, 3); +x_47 = lean_ctor_get(x_29, 4); +x_48 = lean_ctor_get(x_29, 5); +x_49 = lean_ctor_get(x_29, 6); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_29); +x_50 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_46, x_18, x_26); +x_51 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_51, 0, x_43); +lean_ctor_set(x_51, 1, x_44); +lean_ctor_set(x_51, 2, x_45); +lean_ctor_set(x_51, 3, x_50); +lean_ctor_set(x_51, 4, x_47); +lean_ctor_set(x_51, 5, x_48); +lean_ctor_set(x_51, 6, x_49); +lean_ctor_set(x_28, 9, x_51); +x_52 = lean_st_ref_set(x_4, x_28, x_30); +lean_dec(x_4); +x_53 = lean_ctor_get(x_52, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + x_54 = x_52; +} else { + lean_dec_ref(x_52); + x_54 = lean_box(0); +} +x_55 = lean_box(0); +if (lean_is_scalar(x_54)) { + x_56 = lean_alloc_ctor(0, 2, 0); +} else { + x_56 = x_54; +} +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_53); +return x_56; +} +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_57 = lean_ctor_get(x_28, 0); +x_58 = lean_ctor_get(x_28, 1); +x_59 = lean_ctor_get(x_28, 2); +x_60 = lean_ctor_get(x_28, 3); +x_61 = lean_ctor_get(x_28, 4); +x_62 = lean_ctor_get(x_28, 5); +x_63 = lean_ctor_get(x_28, 6); +x_64 = lean_ctor_get_uint8(x_28, sizeof(void*)*23); +x_65 = lean_ctor_get(x_28, 7); +x_66 = lean_ctor_get(x_28, 8); +x_67 = lean_ctor_get(x_28, 10); +x_68 = lean_ctor_get(x_28, 11); +x_69 = lean_ctor_get(x_28, 12); +x_70 = lean_ctor_get(x_28, 13); +x_71 = lean_ctor_get(x_28, 14); +x_72 = lean_ctor_get(x_28, 15); +x_73 = lean_ctor_get(x_28, 16); +x_74 = lean_ctor_get(x_28, 17); +x_75 = lean_ctor_get(x_28, 18); +x_76 = lean_ctor_get(x_28, 19); +x_77 = lean_ctor_get(x_28, 20); +x_78 = lean_ctor_get(x_28, 21); +x_79 = lean_ctor_get(x_28, 22); +lean_inc(x_79); +lean_inc(x_78); +lean_inc(x_77); +lean_inc(x_76); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_28); +x_80 = lean_ctor_get(x_29, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_29, 1); +lean_inc(x_81); +x_82 = lean_ctor_get(x_29, 2); +lean_inc(x_82); +x_83 = lean_ctor_get(x_29, 3); +lean_inc(x_83); +x_84 = lean_ctor_get(x_29, 4); +lean_inc(x_84); +x_85 = lean_ctor_get(x_29, 5); +lean_inc(x_85); +x_86 = lean_ctor_get(x_29, 6); +lean_inc(x_86); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + lean_ctor_release(x_29, 2); + lean_ctor_release(x_29, 3); + lean_ctor_release(x_29, 4); + lean_ctor_release(x_29, 5); + lean_ctor_release(x_29, 6); + x_87 = x_29; +} else { + lean_dec_ref(x_29); + x_87 = lean_box(0); +} +x_88 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_83, x_18, x_26); +if (lean_is_scalar(x_87)) { + x_89 = lean_alloc_ctor(0, 7, 0); +} else { + x_89 = x_87; +} +lean_ctor_set(x_89, 0, x_80); +lean_ctor_set(x_89, 1, x_81); +lean_ctor_set(x_89, 2, x_82); +lean_ctor_set(x_89, 3, x_88); +lean_ctor_set(x_89, 4, x_84); +lean_ctor_set(x_89, 5, x_85); +lean_ctor_set(x_89, 6, x_86); +x_90 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_90, 0, x_57); +lean_ctor_set(x_90, 1, x_58); +lean_ctor_set(x_90, 2, x_59); +lean_ctor_set(x_90, 3, x_60); +lean_ctor_set(x_90, 4, x_61); +lean_ctor_set(x_90, 5, x_62); +lean_ctor_set(x_90, 6, x_63); +lean_ctor_set(x_90, 7, x_65); +lean_ctor_set(x_90, 8, x_66); +lean_ctor_set(x_90, 9, x_89); +lean_ctor_set(x_90, 10, x_67); +lean_ctor_set(x_90, 11, x_68); +lean_ctor_set(x_90, 12, x_69); +lean_ctor_set(x_90, 13, x_70); +lean_ctor_set(x_90, 14, x_71); +lean_ctor_set(x_90, 15, x_72); +lean_ctor_set(x_90, 16, x_73); +lean_ctor_set(x_90, 17, x_74); +lean_ctor_set(x_90, 18, x_75); +lean_ctor_set(x_90, 19, x_76); +lean_ctor_set(x_90, 20, x_77); +lean_ctor_set(x_90, 21, x_78); +lean_ctor_set(x_90, 22, x_79); +lean_ctor_set_uint8(x_90, sizeof(void*)*23, x_64); +x_91 = lean_st_ref_set(x_4, x_90, x_30); +lean_dec(x_4); +x_92 = lean_ctor_get(x_91, 1); +lean_inc(x_92); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_93 = x_91; +} else { + lean_dec_ref(x_91); + x_93 = lean_box(0); +} +x_94 = lean_box(0); +if (lean_is_scalar(x_93)) { + x_95 = lean_alloc_ctor(0, 2, 0); +} else { + x_95 = x_93; +} +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_95, 1, x_92); +return x_95; +} +} +else +{ +uint8_t x_96; +lean_dec(x_18); +lean_dec(x_4); +x_96 = !lean_is_exclusive(x_23); +if (x_96 == 0) +{ +return x_23; +} +else +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_23, 0); +x_98 = lean_ctor_get(x_23, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_23); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +return x_99; +} +} +} +} +else +{ +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_100 = lean_ctor_get(x_13, 0); +x_101 = lean_ctor_get(x_13, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_13); +x_102 = lean_ctor_get(x_100, 3); +lean_inc(x_102); +lean_dec(x_100); +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_1); +lean_ctor_set(x_103, 1, x_2); +x_104 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_102, x_103); +if (lean_obj_tag(x_104) == 0) +{ +lean_object* x_105; lean_object* x_106; +lean_dec(x_103); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_105 = lean_box(0); +x_106 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_101); +return x_106; +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_104, 0); +lean_inc(x_107); +lean_dec(x_104); +x_108 = lean_box(0); +lean_inc(x_4); +x_109 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__4(x_3, x_107, x_108, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_101); +if (lean_obj_tag(x_109) == 0) +{ +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; uint8_t x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +lean_dec(x_109); +x_112 = l_List_reverse___rarg(x_110); +x_113 = lean_st_ref_take(x_4, x_111); +x_114 = lean_ctor_get(x_113, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_114, 9); +lean_inc(x_115); +x_116 = lean_ctor_get(x_113, 1); +lean_inc(x_116); +lean_dec(x_113); +x_117 = lean_ctor_get(x_114, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_114, 1); +lean_inc(x_118); +x_119 = lean_ctor_get(x_114, 2); +lean_inc(x_119); +x_120 = lean_ctor_get(x_114, 3); +lean_inc(x_120); +x_121 = lean_ctor_get(x_114, 4); +lean_inc(x_121); +x_122 = lean_ctor_get(x_114, 5); +lean_inc(x_122); +x_123 = lean_ctor_get(x_114, 6); +lean_inc(x_123); +x_124 = lean_ctor_get_uint8(x_114, sizeof(void*)*23); +x_125 = lean_ctor_get(x_114, 7); +lean_inc(x_125); +x_126 = lean_ctor_get(x_114, 8); +lean_inc(x_126); +x_127 = lean_ctor_get(x_114, 10); +lean_inc(x_127); +x_128 = lean_ctor_get(x_114, 11); +lean_inc(x_128); +x_129 = lean_ctor_get(x_114, 12); +lean_inc(x_129); +x_130 = lean_ctor_get(x_114, 13); +lean_inc(x_130); +x_131 = lean_ctor_get(x_114, 14); +lean_inc(x_131); +x_132 = lean_ctor_get(x_114, 15); +lean_inc(x_132); +x_133 = lean_ctor_get(x_114, 16); +lean_inc(x_133); +x_134 = lean_ctor_get(x_114, 17); +lean_inc(x_134); +x_135 = lean_ctor_get(x_114, 18); +lean_inc(x_135); +x_136 = lean_ctor_get(x_114, 19); +lean_inc(x_136); +x_137 = lean_ctor_get(x_114, 20); +lean_inc(x_137); +x_138 = lean_ctor_get(x_114, 21); +lean_inc(x_138); +x_139 = lean_ctor_get(x_114, 22); +lean_inc(x_139); +if (lean_is_exclusive(x_114)) { + lean_ctor_release(x_114, 0); + lean_ctor_release(x_114, 1); + lean_ctor_release(x_114, 2); + lean_ctor_release(x_114, 3); + lean_ctor_release(x_114, 4); + lean_ctor_release(x_114, 5); + lean_ctor_release(x_114, 6); + lean_ctor_release(x_114, 7); + lean_ctor_release(x_114, 8); + lean_ctor_release(x_114, 9); + lean_ctor_release(x_114, 10); + lean_ctor_release(x_114, 11); + lean_ctor_release(x_114, 12); + lean_ctor_release(x_114, 13); + lean_ctor_release(x_114, 14); + lean_ctor_release(x_114, 15); + lean_ctor_release(x_114, 16); + lean_ctor_release(x_114, 17); + lean_ctor_release(x_114, 18); + lean_ctor_release(x_114, 19); + lean_ctor_release(x_114, 20); + lean_ctor_release(x_114, 21); + lean_ctor_release(x_114, 22); + x_140 = x_114; +} else { + lean_dec_ref(x_114); + x_140 = lean_box(0); +} +x_141 = lean_ctor_get(x_115, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_115, 1); +lean_inc(x_142); +x_143 = lean_ctor_get(x_115, 2); +lean_inc(x_143); +x_144 = lean_ctor_get(x_115, 3); +lean_inc(x_144); +x_145 = lean_ctor_get(x_115, 4); +lean_inc(x_145); +x_146 = lean_ctor_get(x_115, 5); +lean_inc(x_146); +x_147 = lean_ctor_get(x_115, 6); +lean_inc(x_147); +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + lean_ctor_release(x_115, 2); + lean_ctor_release(x_115, 3); + lean_ctor_release(x_115, 4); + lean_ctor_release(x_115, 5); + lean_ctor_release(x_115, 6); + x_148 = x_115; +} else { + lean_dec_ref(x_115); + x_148 = lean_box(0); +} +x_149 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_144, x_103, x_112); +if (lean_is_scalar(x_148)) { + x_150 = lean_alloc_ctor(0, 7, 0); +} else { + x_150 = x_148; +} +lean_ctor_set(x_150, 0, x_141); +lean_ctor_set(x_150, 1, x_142); +lean_ctor_set(x_150, 2, x_143); +lean_ctor_set(x_150, 3, x_149); +lean_ctor_set(x_150, 4, x_145); +lean_ctor_set(x_150, 5, x_146); +lean_ctor_set(x_150, 6, x_147); +if (lean_is_scalar(x_140)) { + x_151 = lean_alloc_ctor(0, 23, 1); +} else { + x_151 = x_140; +} +lean_ctor_set(x_151, 0, x_117); +lean_ctor_set(x_151, 1, x_118); +lean_ctor_set(x_151, 2, x_119); +lean_ctor_set(x_151, 3, x_120); +lean_ctor_set(x_151, 4, x_121); +lean_ctor_set(x_151, 5, x_122); +lean_ctor_set(x_151, 6, x_123); +lean_ctor_set(x_151, 7, x_125); +lean_ctor_set(x_151, 8, x_126); +lean_ctor_set(x_151, 9, x_150); +lean_ctor_set(x_151, 10, x_127); +lean_ctor_set(x_151, 11, x_128); +lean_ctor_set(x_151, 12, x_129); +lean_ctor_set(x_151, 13, x_130); +lean_ctor_set(x_151, 14, x_131); +lean_ctor_set(x_151, 15, x_132); +lean_ctor_set(x_151, 16, x_133); +lean_ctor_set(x_151, 17, x_134); +lean_ctor_set(x_151, 18, x_135); +lean_ctor_set(x_151, 19, x_136); +lean_ctor_set(x_151, 20, x_137); +lean_ctor_set(x_151, 21, x_138); +lean_ctor_set(x_151, 22, x_139); +lean_ctor_set_uint8(x_151, sizeof(void*)*23, x_124); +x_152 = lean_st_ref_set(x_4, x_151, x_116); +lean_dec(x_4); +x_153 = lean_ctor_get(x_152, 1); +lean_inc(x_153); +if (lean_is_exclusive(x_152)) { + lean_ctor_release(x_152, 0); + lean_ctor_release(x_152, 1); + x_154 = x_152; +} else { + lean_dec_ref(x_152); + x_154 = lean_box(0); +} +x_155 = lean_box(0); +if (lean_is_scalar(x_154)) { + x_156 = lean_alloc_ctor(0, 2, 0); +} else { + x_156 = x_154; +} +lean_ctor_set(x_156, 0, x_155); +lean_ctor_set(x_156, 1, x_153); +return x_156; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_103); +lean_dec(x_4); +x_157 = lean_ctor_get(x_109, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_109, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_109)) { + lean_ctor_release(x_109, 0); + lean_ctor_release(x_109, 1); + x_159 = x_109; +} else { + lean_dec_ref(x_109); + x_159 = lean_box(0); +} +if (lean_is_scalar(x_159)) { + x_160 = lean_alloc_ctor(1, 2, 0); +} else { + x_160 = x_159; +} +lean_ctor_set(x_160, 0, x_157); +lean_ctor_set(x_160, 1, x_158); +return x_160; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__3(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; lean_object* x_5; +x_4 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_5 = l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__2(x_1, x_4, x_3); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__7(x_7, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__6(x_1, x_6, x_7, x_4, x_5); +return x_8; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Grind", 5, 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Nat", 3, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq_of_le_of_le", 14, 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6; +lean_inc(x_2); +lean_inc(x_1); +x_16 = l_Lean_mkApp4(x_15, x_1, x_2, x_3, x_4); +x_17 = 0; +x_18 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_18; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eq", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("from", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1; +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", ", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; uint8_t x_16; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_1, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_2, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_19, 1); +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3; +x_24 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_free_object(x_19); +lean_free_object(x_15); +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); +x_28 = lean_box(0); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_17, x_21, x_28, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_27); +return x_29; +} +else +{ +uint8_t x_30; +x_30 = !lean_is_exclusive(x_24); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_31 = lean_ctor_get(x_24, 1); +x_32 = lean_ctor_get(x_24, 0); +lean_dec(x_32); +lean_inc(x_3); +x_33 = l_Lean_MessageData_ofExpr(x_3); +x_34 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_24, 7); +lean_ctor_set(x_24, 1, x_33); +lean_ctor_set(x_24, 0, x_34); +x_35 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_35); +lean_ctor_set(x_19, 0, x_24); +lean_inc(x_4); +x_36 = l_Lean_MessageData_ofExpr(x_4); +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_36); +lean_ctor_set(x_15, 0, x_19); +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_15); +lean_ctor_set(x_37, 1, x_34); +x_38 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_23, x_37, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_17, x_21, x_39, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_40); +lean_dec(x_39); +return x_41; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_42 = lean_ctor_get(x_24, 1); +lean_inc(x_42); +lean_dec(x_24); +lean_inc(x_3); +x_43 = l_Lean_MessageData_ofExpr(x_3); +x_44 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +x_46 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_46); +lean_ctor_set(x_19, 0, x_45); +lean_inc(x_4); +x_47 = l_Lean_MessageData_ofExpr(x_4); +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_47); +lean_ctor_set(x_15, 0, x_19); +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_15); +lean_ctor_set(x_48, 1, x_44); +x_49 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_23, x_48, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_42); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_17, x_21, x_50, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_51); +lean_dec(x_50); +return x_52; +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_53 = lean_ctor_get(x_19, 0); +x_54 = lean_ctor_get(x_19, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_19); +x_55 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3; +x_56 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_55, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_54); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_unbox(x_57); +lean_dec(x_57); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_free_object(x_15); +x_59 = lean_ctor_get(x_56, 1); +lean_inc(x_59); +lean_dec(x_56); +x_60 = lean_box(0); +x_61 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_17, x_53, x_60, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_59); +return x_61; +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_62 = lean_ctor_get(x_56, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_63 = x_56; +} else { + lean_dec_ref(x_56); + x_63 = lean_box(0); +} +lean_inc(x_3); +x_64 = l_Lean_MessageData_ofExpr(x_3); +x_65 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +if (lean_is_scalar(x_63)) { + x_66 = lean_alloc_ctor(7, 2, 0); +} else { + x_66 = x_63; + lean_ctor_set_tag(x_66, 7); +} +lean_ctor_set(x_66, 0, x_65); +lean_ctor_set(x_66, 1, x_64); +x_67 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +x_68 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +lean_inc(x_4); +x_69 = l_Lean_MessageData_ofExpr(x_4); +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_69); +lean_ctor_set(x_15, 0, x_68); +x_70 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_70, 0, x_15); +lean_ctor_set(x_70, 1, x_65); +x_71 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_55, x_70, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_62); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_17, x_53, x_72, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_73); +lean_dec(x_72); +return x_74; +} +} +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_75 = lean_ctor_get(x_15, 0); +x_76 = lean_ctor_get(x_15, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_15); +x_77 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_2, x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_76); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +if (lean_is_exclusive(x_77)) { + lean_ctor_release(x_77, 0); + lean_ctor_release(x_77, 1); + x_80 = x_77; +} else { + lean_dec_ref(x_77); + x_80 = lean_box(0); +} +x_81 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3; +x_82 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_81, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_79); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +x_84 = lean_unbox(x_83); +lean_dec(x_83); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_80); +x_85 = lean_ctor_get(x_82, 1); +lean_inc(x_85); +lean_dec(x_82); +x_86 = lean_box(0); +x_87 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_75, x_78, x_86, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_85); +return x_87; +} +else +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_88 = lean_ctor_get(x_82, 1); +lean_inc(x_88); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + x_89 = x_82; +} else { + lean_dec_ref(x_82); + x_89 = lean_box(0); +} +lean_inc(x_3); +x_90 = l_Lean_MessageData_ofExpr(x_3); +x_91 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +if (lean_is_scalar(x_89)) { + x_92 = lean_alloc_ctor(7, 2, 0); +} else { + x_92 = x_89; + lean_ctor_set_tag(x_92, 7); +} +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_90); +x_93 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +if (lean_is_scalar(x_80)) { + x_94 = lean_alloc_ctor(7, 2, 0); +} else { + x_94 = x_80; + lean_ctor_set_tag(x_94, 7); +} +lean_ctor_set(x_94, 0, x_92); +lean_ctor_set(x_94, 1, x_93); +lean_inc(x_4); +x_95 = l_Lean_MessageData_ofExpr(x_4); +x_96 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_91); +x_98 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_81, x_97, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_88); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_98, 1); +lean_inc(x_100); +lean_dec(x_98); +x_101 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_3, x_4, x_75, x_78, x_99, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_100); +lean_dec(x_99); +return x_101; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getExpr(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_17); +lean_inc(x_14); +x_19 = l_Lean_Meta_Grind_isEqv(x_14, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; uint8_t x_21; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_box(0); +x_24 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2(x_1, x_2, x_14, x_17, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +return x_24; +} +else +{ +uint8_t x_25; +lean_dec(x_17); +lean_dec(x_14); +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_19, 0); +lean_dec(x_26); +x_27 = lean_box(0); +lean_ctor_set(x_19, 0, x_27); +return x_19; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_19, 1); +lean_inc(x_28); +lean_dec(x_19); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_28); +return x_30; +} +} +} +else +{ +uint8_t x_31; +lean_dec(x_17); +lean_dec(x_14); +x_31 = !lean_is_exclusive(x_19); +if (x_31 == 0) +{ +return x_19; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_19, 0); +x_33 = lean_ctor_get(x_19, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_19); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_13); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = lean_box(0); +lean_ctor_set(x_13, 0, x_17); +return x_13; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 1); +lean_inc(x_18); +lean_dec(x_13); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; +} +} +else +{ +uint8_t x_21; +x_21 = !lean_is_exclusive(x_13); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_13, 1); +x_23 = lean_ctor_get(x_13, 0); +lean_dec(x_23); +x_24 = lean_ctor_get(x_14, 0); +lean_inc(x_24); +lean_dec(x_14); +x_25 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_26 = lean_int_dec_eq(x_24, x_25); +lean_dec(x_24); +if (x_26 == 0) +{ +lean_object* x_27; +x_27 = lean_box(0); +lean_ctor_set(x_13, 0, x_27); +return x_13; +} +else +{ +lean_object* x_28; lean_object* x_29; +lean_free_object(x_13); +x_28 = lean_box(0); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3(x_2, x_1, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_30 = lean_ctor_get(x_13, 1); +lean_inc(x_30); +lean_dec(x_13); +x_31 = lean_ctor_get(x_14, 0); +lean_inc(x_31); +lean_dec(x_14); +x_32 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_33 = lean_int_dec_eq(x_31, x_32); +lean_dec(x_31); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_box(0); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_30); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_box(0); +x_37 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3(x_2, x_1, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; uint8_t x_14; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_14 = lean_int_dec_eq(x_3, x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_12); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4(x_2, x_1, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_18; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_13; +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_15; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_5); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + lean_ctor_release(x_4, 1); + x_18 = x_4; +} else { + lean_dec_ref(x_4); + x_18 = lean_box(0); +} +x_25 = lean_ctor_get(x_16, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_16, 1); +lean_inc(x_26); +lean_inc(x_26); +x_27 = l_Lean_Meta_Grind_isEqTrue(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_unbox(x_28); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +lean_inc(x_26); +x_31 = l_Lean_Meta_Grind_isEqFalse(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_30); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_35 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse(x_1, x_2, x_3, x_25, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_34); +lean_dec(x_25); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_unbox(x_36); +lean_dec(x_36); +if (x_37 == 0) +{ +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_35, 1); +lean_inc(x_38); +lean_dec(x_35); +x_39 = 0; +x_19 = x_39; +x_20 = x_38; +goto block_24; +} +else +{ +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_35, 1); +lean_inc(x_40); +lean_dec(x_35); +x_41 = 1; +x_19 = x_41; +x_20 = x_40; +goto block_24; +} +} +else +{ +uint8_t x_42; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_35); +if (x_42 == 0) +{ +return x_35; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_35, 0); +x_44 = lean_ctor_get(x_35, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_35); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +lean_object* x_46; uint8_t x_47; +lean_dec(x_26); +lean_dec(x_25); +x_46 = lean_ctor_get(x_31, 1); +lean_inc(x_46); +lean_dec(x_31); +x_47 = 0; +x_19 = x_47; +x_20 = x_46; +goto block_24; +} +} +else +{ +uint8_t x_48; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_48 = !lean_is_exclusive(x_31); +if (x_48 == 0) +{ +return x_31; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_31, 0); +x_50 = lean_ctor_get(x_31, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_31); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +lean_object* x_52; uint8_t x_53; +lean_dec(x_26); +lean_dec(x_25); +x_52 = lean_ctor_get(x_27, 1); +lean_inc(x_52); +lean_dec(x_27); +x_53 = 0; +x_19 = x_53; +x_20 = x_52; +goto block_24; +} +} +else +{ +uint8_t x_54; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_54 = !lean_is_exclusive(x_27); +if (x_54 == 0) +{ +return x_27; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_27, 0); +x_56 = lean_ctor_get(x_27, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_27); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +block_24: +{ +if (x_19 == 0) +{ +lean_dec(x_18); +lean_dec(x_16); +x_4 = x_17; +x_14 = x_20; +goto _start; +} +else +{ +lean_object* x_22; +if (lean_is_scalar(x_18)) { + x_22 = lean_alloc_ctor(1, 2, 0); +} else { + x_22 = x_18; +} +lean_ctor_set(x_22, 0, x_16); +lean_ctor_set(x_22, 1, x_5); +x_4 = x_17; +x_5 = x_22; +x_14 = x_20; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_15; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_5); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +if (lean_is_exclusive(x_4)) { + lean_ctor_release(x_4, 0); + lean_ctor_release(x_4, 1); + x_18 = x_4; +} else { + lean_dec_ref(x_4); + x_18 = lean_box(0); +} +x_25 = lean_ctor_get(x_16, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_16, 1); +lean_inc(x_26); +lean_inc(x_26); +x_27 = l_Lean_Meta_Grind_isEqTrue(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_unbox(x_28); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +lean_inc(x_26); +x_31 = l_Lean_Meta_Grind_isEqFalse(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_30); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_35 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(x_1, x_2, x_3, x_25, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_34); +lean_dec(x_25); +if (lean_obj_tag(x_35) == 0) +{ +lean_object* x_36; uint8_t x_37; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_unbox(x_36); +lean_dec(x_36); +if (x_37 == 0) +{ +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_35, 1); +lean_inc(x_38); +lean_dec(x_35); +x_39 = 0; +x_19 = x_39; +x_20 = x_38; +goto block_24; +} +else +{ +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_35, 1); +lean_inc(x_40); +lean_dec(x_35); +x_41 = 1; +x_19 = x_41; +x_20 = x_40; +goto block_24; +} +} +else +{ +uint8_t x_42; +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_35); +if (x_42 == 0) +{ +return x_35; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_35, 0); +x_44 = lean_ctor_get(x_35, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_35); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +lean_object* x_46; uint8_t x_47; +lean_dec(x_26); +lean_dec(x_25); +x_46 = lean_ctor_get(x_31, 1); +lean_inc(x_46); +lean_dec(x_31); +x_47 = 0; +x_19 = x_47; +x_20 = x_46; +goto block_24; +} +} +else +{ +uint8_t x_48; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_48 = !lean_is_exclusive(x_31); +if (x_48 == 0) +{ +return x_31; +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_31, 0); +x_50 = lean_ctor_get(x_31, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_31); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} +} +} +else +{ +lean_object* x_52; uint8_t x_53; +lean_dec(x_26); +lean_dec(x_25); +x_52 = lean_ctor_get(x_27, 1); +lean_inc(x_52); +lean_dec(x_27); +x_53 = 0; +x_19 = x_53; +x_20 = x_52; +goto block_24; +} +} +else +{ +uint8_t x_54; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_54 = !lean_is_exclusive(x_27); +if (x_54 == 0) +{ +return x_27; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_27, 0); +x_56 = lean_ctor_get(x_27, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_27); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +block_24: +{ +if (x_19 == 0) +{ +lean_dec(x_18); +lean_dec(x_16); +x_4 = x_17; +x_14 = x_20; +goto _start; +} +else +{ +lean_object* x_22; +if (lean_is_scalar(x_18)) { + x_22 = lean_alloc_ctor(1, 2, 0); +} else { + x_22 = x_18; +} +lean_ctor_set(x_22, 0, x_16); +lean_ctor_set(x_22, 1, x_5); +x_4 = x_17; +x_5 = x_22; +x_14 = x_20; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_151; uint8_t x_152; +x_151 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_152 = !lean_is_exclusive(x_151); +if (x_152 == 0) +{ +lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_153 = lean_ctor_get(x_151, 0); +x_154 = lean_ctor_get(x_151, 1); +x_155 = lean_ctor_get(x_153, 3); +lean_inc(x_155); +lean_dec(x_153); +lean_inc(x_2); +lean_inc(x_1); +lean_ctor_set(x_151, 1, x_2); +lean_ctor_set(x_151, 0, x_1); +x_156 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_155, x_151); +if (lean_obj_tag(x_156) == 0) +{ +lean_dec(x_151); +x_13 = x_154; +goto block_150; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_157 = lean_ctor_get(x_156, 0); +lean_inc(x_157); +lean_dec(x_156); +x_158 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_159 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__2(x_1, x_2, x_3, x_157, x_158, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_154); +if (lean_obj_tag(x_159) == 0) +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; +x_160 = lean_ctor_get(x_159, 0); +lean_inc(x_160); +x_161 = lean_ctor_get(x_159, 1); +lean_inc(x_161); +lean_dec(x_159); +x_162 = l_List_reverse___rarg(x_160); +x_163 = lean_st_ref_take(x_4, x_161); +x_164 = lean_ctor_get(x_163, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_164, 9); +lean_inc(x_165); +x_166 = lean_ctor_get(x_163, 1); +lean_inc(x_166); +lean_dec(x_163); +x_167 = !lean_is_exclusive(x_164); +if (x_167 == 0) +{ +lean_object* x_168; uint8_t x_169; +x_168 = lean_ctor_get(x_164, 9); +lean_dec(x_168); +x_169 = !lean_is_exclusive(x_165); +if (x_169 == 0) +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_170 = lean_ctor_get(x_165, 3); +x_171 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_170, x_151, x_162); +lean_ctor_set(x_165, 3, x_171); +x_172 = lean_st_ref_set(x_4, x_164, x_166); +x_173 = lean_ctor_get(x_172, 1); +lean_inc(x_173); +lean_dec(x_172); +x_13 = x_173; +goto block_150; +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; +x_174 = lean_ctor_get(x_165, 0); +x_175 = lean_ctor_get(x_165, 1); +x_176 = lean_ctor_get(x_165, 2); +x_177 = lean_ctor_get(x_165, 3); +x_178 = lean_ctor_get(x_165, 4); +x_179 = lean_ctor_get(x_165, 5); +x_180 = lean_ctor_get(x_165, 6); +lean_inc(x_180); +lean_inc(x_179); +lean_inc(x_178); +lean_inc(x_177); +lean_inc(x_176); +lean_inc(x_175); +lean_inc(x_174); +lean_dec(x_165); +x_181 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_177, x_151, x_162); +x_182 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_182, 0, x_174); +lean_ctor_set(x_182, 1, x_175); +lean_ctor_set(x_182, 2, x_176); +lean_ctor_set(x_182, 3, x_181); +lean_ctor_set(x_182, 4, x_178); +lean_ctor_set(x_182, 5, x_179); +lean_ctor_set(x_182, 6, x_180); +lean_ctor_set(x_164, 9, x_182); +x_183 = lean_st_ref_set(x_4, x_164, x_166); +x_184 = lean_ctor_get(x_183, 1); +lean_inc(x_184); +lean_dec(x_183); +x_13 = x_184; +goto block_150; +} +} +else +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; uint8_t x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; +x_185 = lean_ctor_get(x_164, 0); +x_186 = lean_ctor_get(x_164, 1); +x_187 = lean_ctor_get(x_164, 2); +x_188 = lean_ctor_get(x_164, 3); +x_189 = lean_ctor_get(x_164, 4); +x_190 = lean_ctor_get(x_164, 5); +x_191 = lean_ctor_get(x_164, 6); +x_192 = lean_ctor_get_uint8(x_164, sizeof(void*)*23); +x_193 = lean_ctor_get(x_164, 7); +x_194 = lean_ctor_get(x_164, 8); +x_195 = lean_ctor_get(x_164, 10); +x_196 = lean_ctor_get(x_164, 11); +x_197 = lean_ctor_get(x_164, 12); +x_198 = lean_ctor_get(x_164, 13); +x_199 = lean_ctor_get(x_164, 14); +x_200 = lean_ctor_get(x_164, 15); +x_201 = lean_ctor_get(x_164, 16); +x_202 = lean_ctor_get(x_164, 17); +x_203 = lean_ctor_get(x_164, 18); +x_204 = lean_ctor_get(x_164, 19); +x_205 = lean_ctor_get(x_164, 20); +x_206 = lean_ctor_get(x_164, 21); +x_207 = lean_ctor_get(x_164, 22); +lean_inc(x_207); +lean_inc(x_206); +lean_inc(x_205); +lean_inc(x_204); +lean_inc(x_203); +lean_inc(x_202); +lean_inc(x_201); +lean_inc(x_200); +lean_inc(x_199); +lean_inc(x_198); +lean_inc(x_197); +lean_inc(x_196); +lean_inc(x_195); +lean_inc(x_194); +lean_inc(x_193); +lean_inc(x_191); +lean_inc(x_190); +lean_inc(x_189); +lean_inc(x_188); +lean_inc(x_187); +lean_inc(x_186); +lean_inc(x_185); +lean_dec(x_164); +x_208 = lean_ctor_get(x_165, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_165, 1); +lean_inc(x_209); +x_210 = lean_ctor_get(x_165, 2); +lean_inc(x_210); +x_211 = lean_ctor_get(x_165, 3); +lean_inc(x_211); +x_212 = lean_ctor_get(x_165, 4); +lean_inc(x_212); +x_213 = lean_ctor_get(x_165, 5); +lean_inc(x_213); +x_214 = lean_ctor_get(x_165, 6); +lean_inc(x_214); +if (lean_is_exclusive(x_165)) { + lean_ctor_release(x_165, 0); + lean_ctor_release(x_165, 1); + lean_ctor_release(x_165, 2); + lean_ctor_release(x_165, 3); + lean_ctor_release(x_165, 4); + lean_ctor_release(x_165, 5); + lean_ctor_release(x_165, 6); + x_215 = x_165; +} else { + lean_dec_ref(x_165); + x_215 = lean_box(0); +} +x_216 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_211, x_151, x_162); +if (lean_is_scalar(x_215)) { + x_217 = lean_alloc_ctor(0, 7, 0); +} else { + x_217 = x_215; +} +lean_ctor_set(x_217, 0, x_208); +lean_ctor_set(x_217, 1, x_209); +lean_ctor_set(x_217, 2, x_210); +lean_ctor_set(x_217, 3, x_216); +lean_ctor_set(x_217, 4, x_212); +lean_ctor_set(x_217, 5, x_213); +lean_ctor_set(x_217, 6, x_214); +x_218 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_218, 0, x_185); +lean_ctor_set(x_218, 1, x_186); +lean_ctor_set(x_218, 2, x_187); +lean_ctor_set(x_218, 3, x_188); +lean_ctor_set(x_218, 4, x_189); +lean_ctor_set(x_218, 5, x_190); +lean_ctor_set(x_218, 6, x_191); +lean_ctor_set(x_218, 7, x_193); +lean_ctor_set(x_218, 8, x_194); +lean_ctor_set(x_218, 9, x_217); +lean_ctor_set(x_218, 10, x_195); +lean_ctor_set(x_218, 11, x_196); +lean_ctor_set(x_218, 12, x_197); +lean_ctor_set(x_218, 13, x_198); +lean_ctor_set(x_218, 14, x_199); +lean_ctor_set(x_218, 15, x_200); +lean_ctor_set(x_218, 16, x_201); +lean_ctor_set(x_218, 17, x_202); +lean_ctor_set(x_218, 18, x_203); +lean_ctor_set(x_218, 19, x_204); +lean_ctor_set(x_218, 20, x_205); +lean_ctor_set(x_218, 21, x_206); +lean_ctor_set(x_218, 22, x_207); +lean_ctor_set_uint8(x_218, sizeof(void*)*23, x_192); +x_219 = lean_st_ref_set(x_4, x_218, x_166); +x_220 = lean_ctor_get(x_219, 1); +lean_inc(x_220); +lean_dec(x_219); +x_13 = x_220; +goto block_150; +} +} +else +{ +uint8_t x_221; +lean_dec(x_151); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_221 = !lean_is_exclusive(x_159); +if (x_221 == 0) +{ +return x_159; +} +else +{ +lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_222 = lean_ctor_get(x_159, 0); +x_223 = lean_ctor_get(x_159, 1); +lean_inc(x_223); +lean_inc(x_222); +lean_dec(x_159); +x_224 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_224, 0, x_222); +lean_ctor_set(x_224, 1, x_223); +return x_224; +} +} +} +} +else +{ +lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +x_225 = lean_ctor_get(x_151, 0); +x_226 = lean_ctor_get(x_151, 1); +lean_inc(x_226); +lean_inc(x_225); +lean_dec(x_151); +x_227 = lean_ctor_get(x_225, 3); +lean_inc(x_227); +lean_dec(x_225); +lean_inc(x_2); +lean_inc(x_1); +x_228 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_228, 0, x_1); +lean_ctor_set(x_228, 1, x_2); +x_229 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_227, x_228); +if (lean_obj_tag(x_229) == 0) +{ +lean_dec(x_228); +x_13 = x_226; +goto block_150; +} +else +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; +x_230 = lean_ctor_get(x_229, 0); +lean_inc(x_230); +lean_dec(x_229); +x_231 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_232 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__2(x_1, x_2, x_3, x_230, x_231, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_226); +if (lean_obj_tag(x_232) == 0) +{ +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_233 = lean_ctor_get(x_232, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_232, 1); +lean_inc(x_234); +lean_dec(x_232); +x_235 = l_List_reverse___rarg(x_233); +x_236 = lean_st_ref_take(x_4, x_234); +x_237 = lean_ctor_get(x_236, 0); +lean_inc(x_237); +x_238 = lean_ctor_get(x_237, 9); +lean_inc(x_238); +x_239 = lean_ctor_get(x_236, 1); +lean_inc(x_239); +lean_dec(x_236); +x_240 = lean_ctor_get(x_237, 0); +lean_inc(x_240); +x_241 = lean_ctor_get(x_237, 1); +lean_inc(x_241); +x_242 = lean_ctor_get(x_237, 2); +lean_inc(x_242); +x_243 = lean_ctor_get(x_237, 3); +lean_inc(x_243); +x_244 = lean_ctor_get(x_237, 4); +lean_inc(x_244); +x_245 = lean_ctor_get(x_237, 5); +lean_inc(x_245); +x_246 = lean_ctor_get(x_237, 6); +lean_inc(x_246); +x_247 = lean_ctor_get_uint8(x_237, sizeof(void*)*23); +x_248 = lean_ctor_get(x_237, 7); +lean_inc(x_248); +x_249 = lean_ctor_get(x_237, 8); +lean_inc(x_249); +x_250 = lean_ctor_get(x_237, 10); +lean_inc(x_250); +x_251 = lean_ctor_get(x_237, 11); +lean_inc(x_251); +x_252 = lean_ctor_get(x_237, 12); +lean_inc(x_252); +x_253 = lean_ctor_get(x_237, 13); +lean_inc(x_253); +x_254 = lean_ctor_get(x_237, 14); +lean_inc(x_254); +x_255 = lean_ctor_get(x_237, 15); +lean_inc(x_255); +x_256 = lean_ctor_get(x_237, 16); +lean_inc(x_256); +x_257 = lean_ctor_get(x_237, 17); +lean_inc(x_257); +x_258 = lean_ctor_get(x_237, 18); +lean_inc(x_258); +x_259 = lean_ctor_get(x_237, 19); +lean_inc(x_259); +x_260 = lean_ctor_get(x_237, 20); +lean_inc(x_260); +x_261 = lean_ctor_get(x_237, 21); +lean_inc(x_261); +x_262 = lean_ctor_get(x_237, 22); +lean_inc(x_262); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + lean_ctor_release(x_237, 2); + lean_ctor_release(x_237, 3); + lean_ctor_release(x_237, 4); + lean_ctor_release(x_237, 5); + lean_ctor_release(x_237, 6); + lean_ctor_release(x_237, 7); + lean_ctor_release(x_237, 8); + lean_ctor_release(x_237, 9); + lean_ctor_release(x_237, 10); + lean_ctor_release(x_237, 11); + lean_ctor_release(x_237, 12); + lean_ctor_release(x_237, 13); + lean_ctor_release(x_237, 14); + lean_ctor_release(x_237, 15); + lean_ctor_release(x_237, 16); + lean_ctor_release(x_237, 17); + lean_ctor_release(x_237, 18); + lean_ctor_release(x_237, 19); + lean_ctor_release(x_237, 20); + lean_ctor_release(x_237, 21); + lean_ctor_release(x_237, 22); + x_263 = x_237; +} else { + lean_dec_ref(x_237); + x_263 = lean_box(0); +} +x_264 = lean_ctor_get(x_238, 0); +lean_inc(x_264); +x_265 = lean_ctor_get(x_238, 1); +lean_inc(x_265); +x_266 = lean_ctor_get(x_238, 2); +lean_inc(x_266); +x_267 = lean_ctor_get(x_238, 3); +lean_inc(x_267); +x_268 = lean_ctor_get(x_238, 4); +lean_inc(x_268); +x_269 = lean_ctor_get(x_238, 5); +lean_inc(x_269); +x_270 = lean_ctor_get(x_238, 6); +lean_inc(x_270); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + lean_ctor_release(x_238, 2); + lean_ctor_release(x_238, 3); + lean_ctor_release(x_238, 4); + lean_ctor_release(x_238, 5); + lean_ctor_release(x_238, 6); + x_271 = x_238; +} else { + lean_dec_ref(x_238); + x_271 = lean_box(0); +} +x_272 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_267, x_228, x_235); +if (lean_is_scalar(x_271)) { + x_273 = lean_alloc_ctor(0, 7, 0); +} else { + x_273 = x_271; +} +lean_ctor_set(x_273, 0, x_264); +lean_ctor_set(x_273, 1, x_265); +lean_ctor_set(x_273, 2, x_266); +lean_ctor_set(x_273, 3, x_272); +lean_ctor_set(x_273, 4, x_268); +lean_ctor_set(x_273, 5, x_269); +lean_ctor_set(x_273, 6, x_270); +if (lean_is_scalar(x_263)) { + x_274 = lean_alloc_ctor(0, 23, 1); +} else { + x_274 = x_263; +} +lean_ctor_set(x_274, 0, x_240); +lean_ctor_set(x_274, 1, x_241); +lean_ctor_set(x_274, 2, x_242); +lean_ctor_set(x_274, 3, x_243); +lean_ctor_set(x_274, 4, x_244); +lean_ctor_set(x_274, 5, x_245); +lean_ctor_set(x_274, 6, x_246); +lean_ctor_set(x_274, 7, x_248); +lean_ctor_set(x_274, 8, x_249); +lean_ctor_set(x_274, 9, x_273); +lean_ctor_set(x_274, 10, x_250); +lean_ctor_set(x_274, 11, x_251); +lean_ctor_set(x_274, 12, x_252); +lean_ctor_set(x_274, 13, x_253); +lean_ctor_set(x_274, 14, x_254); +lean_ctor_set(x_274, 15, x_255); +lean_ctor_set(x_274, 16, x_256); +lean_ctor_set(x_274, 17, x_257); +lean_ctor_set(x_274, 18, x_258); +lean_ctor_set(x_274, 19, x_259); +lean_ctor_set(x_274, 20, x_260); +lean_ctor_set(x_274, 21, x_261); +lean_ctor_set(x_274, 22, x_262); +lean_ctor_set_uint8(x_274, sizeof(void*)*23, x_247); +x_275 = lean_st_ref_set(x_4, x_274, x_239); +x_276 = lean_ctor_get(x_275, 1); +lean_inc(x_276); +lean_dec(x_275); +x_13 = x_276; +goto block_150; +} +else +{ +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +lean_dec(x_228); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_277 = lean_ctor_get(x_232, 0); +lean_inc(x_277); +x_278 = lean_ctor_get(x_232, 1); +lean_inc(x_278); +if (lean_is_exclusive(x_232)) { + lean_ctor_release(x_232, 0); + lean_ctor_release(x_232, 1); + x_279 = x_232; +} else { + lean_dec_ref(x_232); + x_279 = lean_box(0); +} +if (lean_is_scalar(x_279)) { + x_280 = lean_alloc_ctor(1, 2, 0); +} else { + x_280 = x_279; +} +lean_ctor_set(x_280, 0, x_277); +lean_ctor_set(x_280, 1, x_278); +return x_280; +} +} +} +block_150: +{ +lean_object* x_14; uint8_t x_15; +x_14 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_13); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +x_18 = lean_ctor_get(x_16, 3); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_1); +lean_inc(x_2); +lean_ctor_set(x_14, 1, x_1); +lean_ctor_set(x_14, 0, x_2); +x_19 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_18, x_14); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; +lean_dec(x_14); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_19, 0); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_23 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__1(x_1, x_2, x_3, x_21, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_List_reverse___rarg(x_24); +x_27 = lean_st_ref_take(x_4, x_25); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_28, 9); +lean_inc(x_29); +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = !lean_is_exclusive(x_28); +if (x_31 == 0) +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_28, 9); +lean_dec(x_32); +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_34 = lean_ctor_get(x_29, 3); +x_35 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_34, x_14, x_26); +lean_ctor_set(x_29, 3, x_35); +x_36 = lean_st_ref_set(x_4, x_28, x_30); +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +lean_dec(x_36); +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_37); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_38; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_39 = lean_ctor_get(x_29, 0); +x_40 = lean_ctor_get(x_29, 1); +x_41 = lean_ctor_get(x_29, 2); +x_42 = lean_ctor_get(x_29, 3); +x_43 = lean_ctor_get(x_29, 4); +x_44 = lean_ctor_get(x_29, 5); +x_45 = lean_ctor_get(x_29, 6); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_29); +x_46 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_42, x_14, x_26); +x_47 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_46); +lean_ctor_set(x_47, 4, x_43); +lean_ctor_set(x_47, 5, x_44); +lean_ctor_set(x_47, 6, x_45); +lean_ctor_set(x_28, 9, x_47); +x_48 = lean_st_ref_set(x_4, x_28, x_30); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_49); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_50; +} +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_51 = lean_ctor_get(x_28, 0); +x_52 = lean_ctor_get(x_28, 1); +x_53 = lean_ctor_get(x_28, 2); +x_54 = lean_ctor_get(x_28, 3); +x_55 = lean_ctor_get(x_28, 4); +x_56 = lean_ctor_get(x_28, 5); +x_57 = lean_ctor_get(x_28, 6); +x_58 = lean_ctor_get_uint8(x_28, sizeof(void*)*23); +x_59 = lean_ctor_get(x_28, 7); +x_60 = lean_ctor_get(x_28, 8); +x_61 = lean_ctor_get(x_28, 10); +x_62 = lean_ctor_get(x_28, 11); +x_63 = lean_ctor_get(x_28, 12); +x_64 = lean_ctor_get(x_28, 13); +x_65 = lean_ctor_get(x_28, 14); +x_66 = lean_ctor_get(x_28, 15); +x_67 = lean_ctor_get(x_28, 16); +x_68 = lean_ctor_get(x_28, 17); +x_69 = lean_ctor_get(x_28, 18); +x_70 = lean_ctor_get(x_28, 19); +x_71 = lean_ctor_get(x_28, 20); +x_72 = lean_ctor_get(x_28, 21); +x_73 = lean_ctor_get(x_28, 22); +lean_inc(x_73); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_28); +x_74 = lean_ctor_get(x_29, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_29, 1); +lean_inc(x_75); +x_76 = lean_ctor_get(x_29, 2); +lean_inc(x_76); +x_77 = lean_ctor_get(x_29, 3); +lean_inc(x_77); +x_78 = lean_ctor_get(x_29, 4); +lean_inc(x_78); +x_79 = lean_ctor_get(x_29, 5); +lean_inc(x_79); +x_80 = lean_ctor_get(x_29, 6); +lean_inc(x_80); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + lean_ctor_release(x_29, 2); + lean_ctor_release(x_29, 3); + lean_ctor_release(x_29, 4); + lean_ctor_release(x_29, 5); + lean_ctor_release(x_29, 6); + x_81 = x_29; +} else { + lean_dec_ref(x_29); + x_81 = lean_box(0); +} +x_82 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_77, x_14, x_26); +if (lean_is_scalar(x_81)) { + x_83 = lean_alloc_ctor(0, 7, 0); +} else { + x_83 = x_81; +} +lean_ctor_set(x_83, 0, x_74); +lean_ctor_set(x_83, 1, x_75); +lean_ctor_set(x_83, 2, x_76); +lean_ctor_set(x_83, 3, x_82); +lean_ctor_set(x_83, 4, x_78); +lean_ctor_set(x_83, 5, x_79); +lean_ctor_set(x_83, 6, x_80); +x_84 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_84, 0, x_51); +lean_ctor_set(x_84, 1, x_52); +lean_ctor_set(x_84, 2, x_53); +lean_ctor_set(x_84, 3, x_54); +lean_ctor_set(x_84, 4, x_55); +lean_ctor_set(x_84, 5, x_56); +lean_ctor_set(x_84, 6, x_57); +lean_ctor_set(x_84, 7, x_59); +lean_ctor_set(x_84, 8, x_60); +lean_ctor_set(x_84, 9, x_83); +lean_ctor_set(x_84, 10, x_61); +lean_ctor_set(x_84, 11, x_62); +lean_ctor_set(x_84, 12, x_63); +lean_ctor_set(x_84, 13, x_64); +lean_ctor_set(x_84, 14, x_65); +lean_ctor_set(x_84, 15, x_66); +lean_ctor_set(x_84, 16, x_67); +lean_ctor_set(x_84, 17, x_68); +lean_ctor_set(x_84, 18, x_69); +lean_ctor_set(x_84, 19, x_70); +lean_ctor_set(x_84, 20, x_71); +lean_ctor_set(x_84, 21, x_72); +lean_ctor_set(x_84, 22, x_73); +lean_ctor_set_uint8(x_84, sizeof(void*)*23, x_58); +x_85 = lean_st_ref_set(x_4, x_84, x_30); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +lean_dec(x_85); +x_87 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_86); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_87; +} +} +else +{ +uint8_t x_88; +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_88 = !lean_is_exclusive(x_23); +if (x_88 == 0) +{ +return x_23; +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_23, 0); +x_90 = lean_ctor_get(x_23, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_23); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +return x_91; +} +} +} +} +else +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_92 = lean_ctor_get(x_14, 0); +x_93 = lean_ctor_get(x_14, 1); +lean_inc(x_93); +lean_inc(x_92); +lean_dec(x_14); +x_94 = lean_ctor_get(x_92, 3); +lean_inc(x_94); +lean_dec(x_92); +lean_inc(x_1); +lean_inc(x_2); +x_95 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_95, 0, x_2); +lean_ctor_set(x_95, 1, x_1); +x_96 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_94, x_95); +if (lean_obj_tag(x_96) == 0) +{ +lean_object* x_97; +lean_dec(x_95); +x_97 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_93); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_97; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_96, 0); +lean_inc(x_98); +lean_dec(x_96); +x_99 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_100 = l_List_filterAuxM___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll___spec__1(x_1, x_2, x_3, x_98, x_99, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_93); +if (lean_obj_tag(x_100) == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; uint8_t x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_101 = lean_ctor_get(x_100, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_100, 1); +lean_inc(x_102); +lean_dec(x_100); +x_103 = l_List_reverse___rarg(x_101); +x_104 = lean_st_ref_take(x_4, x_102); +x_105 = lean_ctor_get(x_104, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_105, 9); +lean_inc(x_106); +x_107 = lean_ctor_get(x_104, 1); +lean_inc(x_107); +lean_dec(x_104); +x_108 = lean_ctor_get(x_105, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_105, 1); +lean_inc(x_109); +x_110 = lean_ctor_get(x_105, 2); +lean_inc(x_110); +x_111 = lean_ctor_get(x_105, 3); +lean_inc(x_111); +x_112 = lean_ctor_get(x_105, 4); +lean_inc(x_112); +x_113 = lean_ctor_get(x_105, 5); +lean_inc(x_113); +x_114 = lean_ctor_get(x_105, 6); +lean_inc(x_114); +x_115 = lean_ctor_get_uint8(x_105, sizeof(void*)*23); +x_116 = lean_ctor_get(x_105, 7); +lean_inc(x_116); +x_117 = lean_ctor_get(x_105, 8); +lean_inc(x_117); +x_118 = lean_ctor_get(x_105, 10); +lean_inc(x_118); +x_119 = lean_ctor_get(x_105, 11); +lean_inc(x_119); +x_120 = lean_ctor_get(x_105, 12); +lean_inc(x_120); +x_121 = lean_ctor_get(x_105, 13); +lean_inc(x_121); +x_122 = lean_ctor_get(x_105, 14); +lean_inc(x_122); +x_123 = lean_ctor_get(x_105, 15); +lean_inc(x_123); +x_124 = lean_ctor_get(x_105, 16); +lean_inc(x_124); +x_125 = lean_ctor_get(x_105, 17); +lean_inc(x_125); +x_126 = lean_ctor_get(x_105, 18); +lean_inc(x_126); +x_127 = lean_ctor_get(x_105, 19); +lean_inc(x_127); +x_128 = lean_ctor_get(x_105, 20); +lean_inc(x_128); +x_129 = lean_ctor_get(x_105, 21); +lean_inc(x_129); +x_130 = lean_ctor_get(x_105, 22); +lean_inc(x_130); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + lean_ctor_release(x_105, 2); + lean_ctor_release(x_105, 3); + lean_ctor_release(x_105, 4); + lean_ctor_release(x_105, 5); + lean_ctor_release(x_105, 6); + lean_ctor_release(x_105, 7); + lean_ctor_release(x_105, 8); + lean_ctor_release(x_105, 9); + lean_ctor_release(x_105, 10); + lean_ctor_release(x_105, 11); + lean_ctor_release(x_105, 12); + lean_ctor_release(x_105, 13); + lean_ctor_release(x_105, 14); + lean_ctor_release(x_105, 15); + lean_ctor_release(x_105, 16); + lean_ctor_release(x_105, 17); + lean_ctor_release(x_105, 18); + lean_ctor_release(x_105, 19); + lean_ctor_release(x_105, 20); + lean_ctor_release(x_105, 21); + lean_ctor_release(x_105, 22); + x_131 = x_105; +} else { + lean_dec_ref(x_105); + x_131 = lean_box(0); +} +x_132 = lean_ctor_get(x_106, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_106, 1); +lean_inc(x_133); +x_134 = lean_ctor_get(x_106, 2); +lean_inc(x_134); +x_135 = lean_ctor_get(x_106, 3); +lean_inc(x_135); +x_136 = lean_ctor_get(x_106, 4); +lean_inc(x_136); +x_137 = lean_ctor_get(x_106, 5); +lean_inc(x_137); +x_138 = lean_ctor_get(x_106, 6); +lean_inc(x_138); +if (lean_is_exclusive(x_106)) { + lean_ctor_release(x_106, 0); + lean_ctor_release(x_106, 1); + lean_ctor_release(x_106, 2); + lean_ctor_release(x_106, 3); + lean_ctor_release(x_106, 4); + lean_ctor_release(x_106, 5); + lean_ctor_release(x_106, 6); + x_139 = x_106; +} else { + lean_dec_ref(x_106); + x_139 = lean_box(0); +} +x_140 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_135, x_95, x_103); +if (lean_is_scalar(x_139)) { + x_141 = lean_alloc_ctor(0, 7, 0); +} else { + x_141 = x_139; +} +lean_ctor_set(x_141, 0, x_132); +lean_ctor_set(x_141, 1, x_133); +lean_ctor_set(x_141, 2, x_134); +lean_ctor_set(x_141, 3, x_140); +lean_ctor_set(x_141, 4, x_136); +lean_ctor_set(x_141, 5, x_137); +lean_ctor_set(x_141, 6, x_138); +if (lean_is_scalar(x_131)) { + x_142 = lean_alloc_ctor(0, 23, 1); +} else { + x_142 = x_131; +} +lean_ctor_set(x_142, 0, x_108); +lean_ctor_set(x_142, 1, x_109); +lean_ctor_set(x_142, 2, x_110); +lean_ctor_set(x_142, 3, x_111); +lean_ctor_set(x_142, 4, x_112); +lean_ctor_set(x_142, 5, x_113); +lean_ctor_set(x_142, 6, x_114); +lean_ctor_set(x_142, 7, x_116); +lean_ctor_set(x_142, 8, x_117); +lean_ctor_set(x_142, 9, x_141); +lean_ctor_set(x_142, 10, x_118); +lean_ctor_set(x_142, 11, x_119); +lean_ctor_set(x_142, 12, x_120); +lean_ctor_set(x_142, 13, x_121); +lean_ctor_set(x_142, 14, x_122); +lean_ctor_set(x_142, 15, x_123); +lean_ctor_set(x_142, 16, x_124); +lean_ctor_set(x_142, 17, x_125); +lean_ctor_set(x_142, 18, x_126); +lean_ctor_set(x_142, 19, x_127); +lean_ctor_set(x_142, 20, x_128); +lean_ctor_set(x_142, 21, x_129); +lean_ctor_set(x_142, 22, x_130); +lean_ctor_set_uint8(x_142, sizeof(void*)*23, x_115); +x_143 = lean_st_ref_set(x_4, x_142, x_107); +x_144 = lean_ctor_get(x_143, 1); +lean_inc(x_144); +lean_dec(x_143); +x_145 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_144); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_145; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +lean_dec(x_95); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_146 = lean_ctor_get(x_100, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_100, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_148 = x_100; +} else { + lean_dec_ref(x_100); + x_148 = lean_box(0); +} +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(1, 2, 0); +} else { + x_149 = x_148; +} +lean_ctor_set(x_149, 0, x_146); +lean_ctor_set(x_149, 1, x_147); +return x_149; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +uint8_t x_17; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_14, 0); +lean_dec(x_18); +x_19 = lean_box(0); +lean_ctor_set(x_14, 0, x_19); +return x_14; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_dec(x_14); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_dec(x_14); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_24 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getProof_x3f(x_4, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4; +x_30 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___spec__1(x_29); +lean_inc(x_2); +x_31 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(x_1, x_2, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); +x_33 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_32); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_34 = lean_ctor_get(x_26, 1); +lean_inc(x_34); +lean_dec(x_26); +x_35 = lean_ctor_get(x_27, 0); +lean_inc(x_35); +lean_dec(x_27); +lean_inc(x_2); +x_36 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(x_1, x_2, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_34); +x_37 = lean_ctor_get(x_36, 1); +lean_inc(x_37); +lean_dec(x_36); +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +return x_38; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_3, x_17); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_2, x_16, x_19, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_4 = x_18; +x_13 = x_21; +goto _start; +} +else +{ +uint8_t x_23; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +return x_20; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_3, x_17); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_2); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_2, x_16, x_19, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_4 = x_18; +x_13 = x_21; +goto _start; +} +else +{ +uint8_t x_23; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +return x_20; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_17, x_3); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_19); +lean_inc(x_2); +lean_inc(x_16); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_16, x_2, x_19, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_box(0); +x_26 = lean_ctor_get(x_23, 5); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_ctor_get(x_26, 2); +lean_inc(x_27); +x_28 = lean_nat_dec_lt(x_2, x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_26); +x_29 = l_outOfBounds___rarg(x_25); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_30 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1(x_2, x_16, x_19, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +lean_dec(x_19); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_4 = x_18; +x_13 = x_31; +goto _start; +} +else +{ +uint8_t x_33; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_33 = !lean_is_exclusive(x_30); +if (x_33 == 0) +{ +return x_30; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_30, 0); +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_30); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +else +{ +lean_object* x_37; lean_object* x_38; +x_37 = l_Lean_PersistentArray_get_x21___rarg(x_25, x_26, x_2); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_38 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2(x_2, x_16, x_19, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +lean_dec(x_19); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +x_4 = x_18; +x_13 = x_39; +goto _start; +} +else +{ +uint8_t x_41; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_41 = !lean_is_exclusive(x_38); +if (x_41 == 0) +{ +return x_38; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_38, 0); +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_38); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_45 = !lean_is_exclusive(x_20); +if (x_45 == 0) +{ +return x_20; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_20, 0); +x_47 = lean_ctor_get(x_20, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_20); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_17, x_3); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_19); +lean_inc(x_2); +lean_inc(x_16); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_16, x_2, x_19, x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_box(0); +x_26 = lean_ctor_get(x_23, 5); +lean_inc(x_26); +lean_dec(x_23); +x_27 = lean_ctor_get(x_26, 2); +lean_inc(x_27); +x_28 = lean_nat_dec_lt(x_2, x_27); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_26); +x_29 = l_outOfBounds___rarg(x_25); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_30 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1(x_2, x_16, x_19, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +lean_dec(x_19); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_4 = x_18; +x_13 = x_31; +goto _start; +} +else +{ +uint8_t x_33; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_33 = !lean_is_exclusive(x_30); +if (x_33 == 0) +{ +return x_30; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_30, 0); +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_30); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +else +{ +lean_object* x_37; lean_object* x_38; +x_37 = l_Lean_PersistentArray_get_x21___rarg(x_25, x_26, x_2); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_38 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2(x_2, x_16, x_19, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +lean_dec(x_19); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); +x_4 = x_18; +x_13 = x_39; +goto _start; +} +else +{ +uint8_t x_41; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_41 = !lean_is_exclusive(x_38); +if (x_41 == 0) +{ +return x_38; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_38, 0); +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_38); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_45 = !lean_is_exclusive(x_20); +if (x_45 == 0) +{ +return x_20; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_20, 0); +x_47 = lean_ctor_get(x_20, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_20); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_3, x_17); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_1, x_16, x_19, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_4 = x_18; +x_13 = x_21; +goto _start; +} +else +{ +uint8_t x_23; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +return x_20; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_14 = lean_box(0); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_4, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_4, 1); +lean_inc(x_17); +x_18 = lean_ctor_get(x_4, 2); +lean_inc(x_18); +lean_dec(x_4); +x_19 = lean_int_add(x_3, x_17); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_20 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateIfShorter(x_1, x_16, x_19, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_4 = x_18; +x_13 = x_21; +goto _start; +} +else +{ +uint8_t x_23; +lean_dec(x_18); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +return x_20; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge_update(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_26 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_box(0); +x_30 = lean_ctor_get(x_27, 5); +lean_inc(x_30); +lean_dec(x_27); +x_31 = lean_ctor_get(x_30, 2); +lean_inc(x_31); +x_32 = lean_nat_dec_lt(x_2, x_31); +lean_dec(x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; +lean_dec(x_30); +x_33 = l_outOfBounds___rarg(x_29); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_34 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5(x_1, x_2, x_3, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; +x_35 = lean_ctor_get(x_34, 1); +lean_inc(x_35); +lean_dec(x_34); +x_13 = x_35; +goto block_25; +} +else +{ +uint8_t x_36; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_36 = !lean_is_exclusive(x_34); +if (x_36 == 0) +{ +return x_34; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_34, 0); +x_38 = lean_ctor_get(x_34, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_34); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +else +{ +lean_object* x_40; lean_object* x_41; +x_40 = l_Lean_PersistentArray_get_x21___rarg(x_29, x_30, x_2); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_41 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6(x_1, x_2, x_3, x_40, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); +x_13 = x_42; +goto block_25; +} +else +{ +uint8_t x_43; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_43 = !lean_is_exclusive(x_41); +if (x_43 == 0) +{ +return x_41; +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_41, 0); +x_45 = lean_ctor_get(x_41, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_41); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} +} +} +block_25: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_14 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_box(0); +x_18 = lean_ctor_get(x_15, 4); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_ctor_get(x_18, 2); +lean_inc(x_19); +x_20 = lean_nat_dec_lt(x_1, x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_18); +x_21 = l_outOfBounds___rarg(x_17); +x_22 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3(x_1, x_2, x_3, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +lean_dec(x_1); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; +x_23 = l_Lean_PersistentArray_get_x21___rarg(x_17, x_18, x_1); +x_24 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4(x_1, x_2, x_3, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +lean_dec(x_1); +return x_24; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_2); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forM___at_Lean_Meta_Grind_Arith_Offset_addEdge_update___spec__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_3); +lean_dec(x_2); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge_update___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Meta_Grind_Arith_Offset_addEdge_update(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isShorter(x_1, x_2, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +uint8_t x_18; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_15, 0); +lean_dec(x_19); +x_20 = lean_box(0); +lean_ctor_set(x_15, 0, x_20); +return x_15; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); +lean_dec(x_15); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; +} +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_15, 1); +lean_inc(x_24); +lean_dec(x_15); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_25 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist(x_1, x_2, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_24); +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +lean_inc(x_3); +lean_inc(x_1); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_1); +lean_ctor_set(x_27, 1, x_3); +lean_ctor_set(x_27, 2, x_4); +lean_inc(x_2); +x_28 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setProof(x_1, x_2, x_27, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_26); +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_30 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateAll(x_1, x_2, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 1); +lean_inc(x_31); +lean_dec(x_30); +x_32 = l_Lean_Meta_Grind_Arith_Offset_addEdge_update(x_1, x_2, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_31); +lean_dec(x_3); +return x_32; +} +else +{ +uint8_t x_33; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_33 = !lean_is_exclusive(x_30); +if (x_33 == 0) +{ +return x_30; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_30, 0); +x_35 = lean_ctor_get(x_30, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_30); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_1, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1(x_2, x_1, x_3, x_4, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_dec(x_15); +x_21 = lean_ctor_get(x_16, 0); +lean_inc(x_21); +lean_dec(x_16); +x_22 = lean_int_add(x_21, x_3); +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_24 = lean_int_dec_lt(x_22, x_23); +lean_dec(x_22); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_21); +x_25 = lean_box(0); +x_26 = l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1(x_2, x_1, x_3, x_4, x_25, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); +return x_26; +} +else +{ +lean_object* x_27; +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat(x_2, x_1, x_3, x_4, x_21, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); +lean_dec(x_21); +lean_dec(x_3); +lean_dec(x_1); +lean_dec(x_2); +if (lean_obj_tag(x_27) == 0) +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_27, 0); +lean_dec(x_29); +x_30 = lean_box(0); +lean_ctor_set(x_27, 0, x_30); +return x_27; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_27, 1); +lean_inc(x_31); +lean_dec(x_27); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; +} +} +else +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_27); +if (x_34 == 0) +{ +return x_27; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_27, 0); +x_36 = lean_ctor_get(x_27, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_27); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2(x_2, x_1, x_3, x_4, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); +return x_19; +} +else +{ +uint8_t x_20; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_20 = !lean_is_exclusive(x_14); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_14, 0); +lean_dec(x_21); +x_22 = lean_box(0); +lean_ctor_set(x_14, 0, x_22); +return x_14; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_dec(x_14); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Meta_Grind_Arith_Offset_addEdge___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_array_get_size(x_2); +x_8 = lean_nat_dec_lt(x_5, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +lean_dec(x_5); +return x_6; +} +else +{ +lean_object* x_9; lean_object* x_10; uint64_t x_11; size_t x_12; size_t x_13; size_t x_14; size_t x_15; size_t x_16; size_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_9 = lean_array_fget(x_2, x_5); +x_10 = lean_array_fget(x_3, x_5); +x_11 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_9); +x_12 = lean_uint64_to_usize(x_11); +x_13 = 1; +x_14 = lean_usize_sub(x_1, x_13); +x_15 = 5; +x_16 = lean_usize_mul(x_15, x_14); +x_17 = lean_usize_shift_right(x_12, x_16); +x_18 = lean_unsigned_to_nat(1u); +x_19 = lean_nat_add(x_5, x_18); +lean_dec(x_5); +x_20 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_6, x_17, x_1, x_9, x_10); +x_4 = lean_box(0); +x_5 = x_19; +x_6 = x_20; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_5 = lean_ctor_get(x_1, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +x_7 = lean_array_get_size(x_5); +x_8 = lean_nat_dec_lt(x_2, x_7); +lean_dec(x_7); +if (x_8 == 0) +{ +uint8_t x_9; +lean_dec(x_2); +x_9 = !lean_is_exclusive(x_1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_1, 1); +lean_dec(x_10); +x_11 = lean_ctor_get(x_1, 0); +lean_dec(x_11); +x_12 = lean_array_push(x_5, x_3); +x_13 = lean_array_push(x_6, x_4); +lean_ctor_set(x_1, 1, x_13); +lean_ctor_set(x_1, 0, x_12); +return x_1; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_dec(x_1); +x_14 = lean_array_push(x_5, x_3); +x_15 = lean_array_push(x_6, x_4); +x_16 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +else +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_array_fget(x_5, x_2); +x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_3, x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_6); +lean_dec(x_5); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_add(x_2, x_19); +lean_dec(x_2); +x_2 = x_20; +goto _start; +} +else +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_1); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_23 = lean_ctor_get(x_1, 1); +lean_dec(x_23); +x_24 = lean_ctor_get(x_1, 0); +lean_dec(x_24); +x_25 = lean_array_fset(x_5, x_2, x_3); +x_26 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +lean_ctor_set(x_1, 1, x_26); +lean_ctor_set(x_1, 0, x_25); +return x_1; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_1); +x_27 = lean_array_fset(x_5, x_2, x_3); +x_28 = lean_array_fset(x_6, x_2, x_4); +lean_dec(x_2); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_1); +if (x_6 == 0) +{ +lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; size_t x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_7 = lean_ctor_get(x_1, 0); +x_8 = 1; +x_9 = 5; +x_10 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_11 = lean_usize_land(x_2, x_10); +x_12 = lean_usize_to_nat(x_11); +x_13 = lean_array_get_size(x_7); +x_14 = lean_nat_dec_lt(x_12, x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_dec(x_12); +lean_dec(x_5); +lean_dec(x_4); +return x_1; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_array_fget(x_7, x_12); +x_16 = lean_box(0); +x_17 = lean_array_fset(x_7, x_12, x_16); +switch (lean_obj_tag(x_15)) { +case 0: +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_15, 0); +x_20 = lean_ctor_get(x_15, 1); +x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_free_object(x_15); +x_22 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_19, x_20, x_4, x_5); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_22); +x_24 = lean_array_fset(x_17, x_12, x_23); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_24); +return x_1; +} +else +{ +lean_object* x_25; +lean_dec(x_20); +lean_dec(x_19); +lean_ctor_set(x_15, 1, x_5); +lean_ctor_set(x_15, 0, x_4); +x_25 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_25); +return x_1; +} +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_15, 0); +x_27 = lean_ctor_get(x_15, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_15); +x_28 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_26, x_27, x_4, x_5); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = lean_array_fset(x_17, x_12, x_30); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_31); +return x_1; +} +else +{ +lean_object* x_32; lean_object* x_33; +lean_dec(x_27); +lean_dec(x_26); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_4); +lean_ctor_set(x_32, 1, x_5); +x_33 = lean_array_fset(x_17, x_12, x_32); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_33); +return x_1; +} +} +} +case 1: +{ +uint8_t x_34; +x_34 = !lean_is_exclusive(x_15); +if (x_34 == 0) +{ +lean_object* x_35; size_t x_36; size_t x_37; lean_object* x_38; lean_object* x_39; +x_35 = lean_ctor_get(x_15, 0); +x_36 = lean_usize_shift_right(x_2, x_9); +x_37 = lean_usize_add(x_3, x_8); +x_38 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_35, x_36, x_37, x_4, x_5); +lean_ctor_set(x_15, 0, x_38); +x_39 = lean_array_fset(x_17, x_12, x_15); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_39); +return x_1; +} +else +{ +lean_object* x_40; size_t x_41; size_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_15, 0); +lean_inc(x_40); +lean_dec(x_15); +x_41 = lean_usize_shift_right(x_2, x_9); +x_42 = lean_usize_add(x_3, x_8); +x_43 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_40, x_41, x_42, x_4, x_5); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +x_45 = lean_array_fset(x_17, x_12, x_44); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_45); +return x_1; +} +} +default: +{ +lean_object* x_46; lean_object* x_47; +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_4); +lean_ctor_set(x_46, 1, x_5); +x_47 = lean_array_fset(x_17, x_12, x_46); +lean_dec(x_12); +lean_ctor_set(x_1, 0, x_47); +return x_1; +} +} +} +} +else +{ +lean_object* x_48; size_t x_49; size_t x_50; size_t x_51; size_t x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; +x_48 = lean_ctor_get(x_1, 0); +lean_inc(x_48); +lean_dec(x_1); +x_49 = 1; +x_50 = 5; +x_51 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2; +x_52 = lean_usize_land(x_2, x_51); +x_53 = lean_usize_to_nat(x_52); +x_54 = lean_array_get_size(x_48); +x_55 = lean_nat_dec_lt(x_53, x_54); +lean_dec(x_54); +if (x_55 == 0) +{ +lean_object* x_56; +lean_dec(x_53); +lean_dec(x_5); +lean_dec(x_4); +x_56 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_56, 0, x_48); +return x_56; +} +else +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_array_fget(x_48, x_53); +x_58 = lean_box(0); +x_59 = lean_array_fset(x_48, x_53, x_58); +switch (lean_obj_tag(x_57)) { +case 0: +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = lean_ctor_get(x_57, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_57, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_62 = x_57; +} else { + lean_dec_ref(x_57); + x_62 = lean_box(0); +} +x_63 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_4, x_60); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_dec(x_62); +x_64 = l_Lean_PersistentHashMap_mkCollisionNode___rarg(x_60, x_61, x_4, x_5); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = lean_array_fset(x_59, x_53, x_65); +lean_dec(x_53); +x_67 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_67, 0, x_66); +return x_67; +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_dec(x_61); +lean_dec(x_60); +if (lean_is_scalar(x_62)) { + x_68 = lean_alloc_ctor(0, 2, 0); +} else { + x_68 = x_62; +} +lean_ctor_set(x_68, 0, x_4); +lean_ctor_set(x_68, 1, x_5); +x_69 = lean_array_fset(x_59, x_53, x_68); +lean_dec(x_53); +x_70 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_70, 0, x_69); +return x_70; +} +} +case 1: +{ +lean_object* x_71; lean_object* x_72; size_t x_73; size_t x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_71 = lean_ctor_get(x_57, 0); +lean_inc(x_71); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + x_72 = x_57; +} else { + lean_dec_ref(x_57); + x_72 = lean_box(0); +} +x_73 = lean_usize_shift_right(x_2, x_50); +x_74 = lean_usize_add(x_3, x_49); +x_75 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_71, x_73, x_74, x_4, x_5); +if (lean_is_scalar(x_72)) { + x_76 = lean_alloc_ctor(1, 1, 0); +} else { + x_76 = x_72; +} +lean_ctor_set(x_76, 0, x_75); +x_77 = lean_array_fset(x_59, x_53, x_76); +lean_dec(x_53); +x_78 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_78, 0, x_77); +return x_78; +} +default: +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_4); +lean_ctor_set(x_79, 1, x_5); +x_80 = lean_array_fset(x_59, x_53, x_79); +lean_dec(x_53); +x_81 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_81, 0, x_80); +return x_81; +} +} +} +} +} +else +{ +uint8_t x_82; +x_82 = !lean_is_exclusive(x_1); +if (x_82 == 0) +{ +lean_object* x_83; lean_object* x_84; size_t x_85; uint8_t x_86; +x_83 = lean_unsigned_to_nat(0u); +x_84 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__4(x_1, x_83, x_4, x_5); +x_85 = 7; +x_86 = lean_usize_dec_le(x_85, x_3); +if (x_86 == 0) +{ +lean_object* x_87; lean_object* x_88; uint8_t x_89; +x_87 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_84); +x_88 = lean_unsigned_to_nat(4u); +x_89 = lean_nat_dec_lt(x_87, x_88); +lean_dec(x_87); +if (x_89 == 0) +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_90 = lean_ctor_get(x_84, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_84, 1); +lean_inc(x_91); +lean_dec(x_84); +x_92 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_93 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3(x_3, x_90, x_91, lean_box(0), x_83, x_92); +lean_dec(x_91); +lean_dec(x_90); +return x_93; +} +else +{ +return x_84; +} +} +else +{ +return x_84; +} +} +else +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; size_t x_99; uint8_t x_100; +x_94 = lean_ctor_get(x_1, 0); +x_95 = lean_ctor_get(x_1, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_1); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +x_97 = lean_unsigned_to_nat(0u); +x_98 = l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__4(x_96, x_97, x_4, x_5); +x_99 = 7; +x_100 = lean_usize_dec_le(x_99, x_3); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; uint8_t x_103; +x_101 = l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(x_98); +x_102 = lean_unsigned_to_nat(4u); +x_103 = lean_nat_dec_lt(x_101, x_102); +lean_dec(x_101); +if (x_103 == 0) +{ +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_104 = lean_ctor_get(x_98, 0); +lean_inc(x_104); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +lean_dec(x_98); +x_106 = l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3; +x_107 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3(x_3, x_104, x_105, lean_box(0), x_97, x_106); +lean_dec(x_105); +lean_dec(x_104); +return x_107; +} +else +{ +return x_98; +} +} +else +{ +return x_98; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint64_t x_4; size_t x_5; size_t x_6; lean_object* x_7; +x_4 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_2); +x_5 = lean_uint64_to_usize(x_4); +x_6 = 1; +x_7 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_1, x_5, x_6, x_2, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__5(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +x_10 = l___private_Init_Data_Repr_0__Nat_reprFast(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Lean_MessageData_ofFormat(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +lean_inc(x_1); +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_1); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_ctor_get(x_2, 1); +lean_inc(x_20); +lean_dec(x_2); +x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); +x_22 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_1); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_30 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lean_MessageData_ofFormat(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_28); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_16); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_6); +x_34 = lean_ctor_get(x_2, 0); +lean_inc(x_34); +x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_34); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l_Lean_MessageData_ofFormat(x_36); +x_38 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +lean_inc(x_1); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_ctor_get(x_2, 1); +lean_inc(x_45); +lean_dec(x_2); +x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_45); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l_Lean_MessageData_ofFormat(x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_1); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_41); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_53 = lean_nat_abs(x_3); +lean_dec(x_3); +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_53, x_54); +lean_dec(x_53); +x_56 = lean_ctor_get(x_2, 0); +lean_inc(x_56); +x_57 = l___private_Init_Data_Repr_0__Nat_reprFast(x_56); +x_58 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_59 = l_Lean_MessageData_ofFormat(x_58); +x_60 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +lean_inc(x_1); +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_1); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_62); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_nat_add(x_55, x_54); +lean_dec(x_55); +x_68 = l___private_Init_Data_Repr_0__Nat_reprFast(x_67); +x_69 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_MessageData_ofFormat(x_69); +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_ctor_get(x_2, 1); +lean_inc(x_74); +lean_dec(x_2); +x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_77 = l_Lean_MessageData_ofFormat(x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_60); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_1); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_st_ref_take(x_6, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 9); +lean_inc(x_17); +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_15, 1); +x_20 = lean_ctor_get(x_15, 0); +lean_dec(x_20); +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_16, 9); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_17, 2); +x_25 = lean_ctor_get(x_17, 3); +lean_inc(x_2); +lean_inc(x_1); +x_26 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(x_24, x_1, x_2); +lean_ctor_set(x_15, 1, x_4); +lean_ctor_set(x_15, 0, x_3); +lean_inc(x_25); +x_27 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_25, x_15); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_2); +lean_ctor_set(x_28, 1, x_1); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_25, x_15, x_30); +lean_ctor_set(x_17, 3, x_31); +lean_ctor_set(x_17, 2, x_26); +x_32 = lean_st_ref_set(x_6, x_16, x_19); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_dec(x_34); +x_35 = lean_box(0); +lean_ctor_set(x_32, 0, x_35); +return x_32; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +return x_38; +} +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_39 = lean_ctor_get(x_27, 0); +lean_inc(x_39); +lean_dec(x_27); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_2); +lean_ctor_set(x_40, 1, x_1); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_39); +x_42 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_25, x_15, x_41); +lean_ctor_set(x_17, 3, x_42); +lean_ctor_set(x_17, 2, x_26); +x_43 = lean_st_ref_set(x_6, x_16, x_19); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +x_46 = lean_box(0); +lean_ctor_set(x_43, 0, x_46); +return x_43; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_43, 1); +lean_inc(x_47); +lean_dec(x_43); +x_48 = lean_box(0); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_47); +return x_49; +} +} +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_50 = lean_ctor_get(x_17, 0); +x_51 = lean_ctor_get(x_17, 1); +x_52 = lean_ctor_get(x_17, 2); +x_53 = lean_ctor_get(x_17, 3); +x_54 = lean_ctor_get(x_17, 4); +x_55 = lean_ctor_get(x_17, 5); +x_56 = lean_ctor_get(x_17, 6); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_17); +lean_inc(x_2); +lean_inc(x_1); +x_57 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(x_52, x_1, x_2); +lean_ctor_set(x_15, 1, x_4); +lean_ctor_set(x_15, 0, x_3); +lean_inc(x_53); +x_58 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_53, x_15); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_2); +lean_ctor_set(x_59, 1, x_1); +x_60 = lean_box(0); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +x_62 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_53, x_15, x_61); +x_63 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_63, 0, x_50); +lean_ctor_set(x_63, 1, x_51); +lean_ctor_set(x_63, 2, x_57); +lean_ctor_set(x_63, 3, x_62); +lean_ctor_set(x_63, 4, x_54); +lean_ctor_set(x_63, 5, x_55); +lean_ctor_set(x_63, 6, x_56); +lean_ctor_set(x_16, 9, x_63); +x_64 = lean_st_ref_set(x_6, x_16, x_19); +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; +} else { + lean_dec_ref(x_64); + x_66 = lean_box(0); +} +x_67 = lean_box(0); +if (lean_is_scalar(x_66)) { + x_68 = lean_alloc_ctor(0, 2, 0); +} else { + x_68 = x_66; +} +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_65); +return x_68; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_69 = lean_ctor_get(x_58, 0); +lean_inc(x_69); +lean_dec(x_58); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_2); +lean_ctor_set(x_70, 1, x_1); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_69); +x_72 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_53, x_15, x_71); +x_73 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_73, 0, x_50); +lean_ctor_set(x_73, 1, x_51); +lean_ctor_set(x_73, 2, x_57); +lean_ctor_set(x_73, 3, x_72); +lean_ctor_set(x_73, 4, x_54); +lean_ctor_set(x_73, 5, x_55); +lean_ctor_set(x_73, 6, x_56); +lean_ctor_set(x_16, 9, x_73); +x_74 = lean_st_ref_set(x_6, x_16, x_19); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_76 = x_74; +} else { + lean_dec_ref(x_74); + x_76 = lean_box(0); +} +x_77 = lean_box(0); +if (lean_is_scalar(x_76)) { + x_78 = lean_alloc_ctor(0, 2, 0); +} else { + x_78 = x_76; +} +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_75); +return x_78; +} +} +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_79 = lean_ctor_get(x_16, 0); +x_80 = lean_ctor_get(x_16, 1); +x_81 = lean_ctor_get(x_16, 2); +x_82 = lean_ctor_get(x_16, 3); +x_83 = lean_ctor_get(x_16, 4); +x_84 = lean_ctor_get(x_16, 5); +x_85 = lean_ctor_get(x_16, 6); +x_86 = lean_ctor_get_uint8(x_16, sizeof(void*)*23); +x_87 = lean_ctor_get(x_16, 7); +x_88 = lean_ctor_get(x_16, 8); +x_89 = lean_ctor_get(x_16, 10); +x_90 = lean_ctor_get(x_16, 11); +x_91 = lean_ctor_get(x_16, 12); +x_92 = lean_ctor_get(x_16, 13); +x_93 = lean_ctor_get(x_16, 14); +x_94 = lean_ctor_get(x_16, 15); +x_95 = lean_ctor_get(x_16, 16); +x_96 = lean_ctor_get(x_16, 17); +x_97 = lean_ctor_get(x_16, 18); +x_98 = lean_ctor_get(x_16, 19); +x_99 = lean_ctor_get(x_16, 20); +x_100 = lean_ctor_get(x_16, 21); +x_101 = lean_ctor_get(x_16, 22); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +lean_inc(x_98); +lean_inc(x_97); +lean_inc(x_96); +lean_inc(x_95); +lean_inc(x_94); +lean_inc(x_93); +lean_inc(x_92); +lean_inc(x_91); +lean_inc(x_90); +lean_inc(x_89); +lean_inc(x_88); +lean_inc(x_87); +lean_inc(x_85); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_16); +x_102 = lean_ctor_get(x_17, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_17, 1); +lean_inc(x_103); +x_104 = lean_ctor_get(x_17, 2); +lean_inc(x_104); +x_105 = lean_ctor_get(x_17, 3); +lean_inc(x_105); +x_106 = lean_ctor_get(x_17, 4); +lean_inc(x_106); +x_107 = lean_ctor_get(x_17, 5); +lean_inc(x_107); +x_108 = lean_ctor_get(x_17, 6); +lean_inc(x_108); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + lean_ctor_release(x_17, 2); + lean_ctor_release(x_17, 3); + lean_ctor_release(x_17, 4); + lean_ctor_release(x_17, 5); + lean_ctor_release(x_17, 6); + x_109 = x_17; +} else { + lean_dec_ref(x_17); + x_109 = lean_box(0); +} +lean_inc(x_2); +lean_inc(x_1); +x_110 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(x_104, x_1, x_2); +lean_ctor_set(x_15, 1, x_4); +lean_ctor_set(x_15, 0, x_3); +lean_inc(x_105); +x_111 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_105, x_15); +if (lean_obj_tag(x_111) == 0) +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_112 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_112, 0, x_2); +lean_ctor_set(x_112, 1, x_1); +x_113 = lean_box(0); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +x_115 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_105, x_15, x_114); +if (lean_is_scalar(x_109)) { + x_116 = lean_alloc_ctor(0, 7, 0); +} else { + x_116 = x_109; +} +lean_ctor_set(x_116, 0, x_102); +lean_ctor_set(x_116, 1, x_103); +lean_ctor_set(x_116, 2, x_110); +lean_ctor_set(x_116, 3, x_115); +lean_ctor_set(x_116, 4, x_106); +lean_ctor_set(x_116, 5, x_107); +lean_ctor_set(x_116, 6, x_108); +x_117 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_117, 0, x_79); +lean_ctor_set(x_117, 1, x_80); +lean_ctor_set(x_117, 2, x_81); +lean_ctor_set(x_117, 3, x_82); +lean_ctor_set(x_117, 4, x_83); +lean_ctor_set(x_117, 5, x_84); +lean_ctor_set(x_117, 6, x_85); +lean_ctor_set(x_117, 7, x_87); +lean_ctor_set(x_117, 8, x_88); +lean_ctor_set(x_117, 9, x_116); +lean_ctor_set(x_117, 10, x_89); +lean_ctor_set(x_117, 11, x_90); +lean_ctor_set(x_117, 12, x_91); +lean_ctor_set(x_117, 13, x_92); +lean_ctor_set(x_117, 14, x_93); +lean_ctor_set(x_117, 15, x_94); +lean_ctor_set(x_117, 16, x_95); +lean_ctor_set(x_117, 17, x_96); +lean_ctor_set(x_117, 18, x_97); +lean_ctor_set(x_117, 19, x_98); +lean_ctor_set(x_117, 20, x_99); +lean_ctor_set(x_117, 21, x_100); +lean_ctor_set(x_117, 22, x_101); +lean_ctor_set_uint8(x_117, sizeof(void*)*23, x_86); +x_118 = lean_st_ref_set(x_6, x_117, x_19); +x_119 = lean_ctor_get(x_118, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + lean_ctor_release(x_118, 1); + x_120 = x_118; +} else { + lean_dec_ref(x_118); + x_120 = lean_box(0); +} +x_121 = lean_box(0); +if (lean_is_scalar(x_120)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_120; +} +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_119); +return x_122; +} +else +{ +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_123 = lean_ctor_get(x_111, 0); +lean_inc(x_123); +lean_dec(x_111); +x_124 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_124, 0, x_2); +lean_ctor_set(x_124, 1, x_1); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_124); +lean_ctor_set(x_125, 1, x_123); +x_126 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_105, x_15, x_125); +if (lean_is_scalar(x_109)) { + x_127 = lean_alloc_ctor(0, 7, 0); +} else { + x_127 = x_109; +} +lean_ctor_set(x_127, 0, x_102); +lean_ctor_set(x_127, 1, x_103); +lean_ctor_set(x_127, 2, x_110); +lean_ctor_set(x_127, 3, x_126); +lean_ctor_set(x_127, 4, x_106); +lean_ctor_set(x_127, 5, x_107); +lean_ctor_set(x_127, 6, x_108); +x_128 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_128, 0, x_79); +lean_ctor_set(x_128, 1, x_80); +lean_ctor_set(x_128, 2, x_81); +lean_ctor_set(x_128, 3, x_82); +lean_ctor_set(x_128, 4, x_83); +lean_ctor_set(x_128, 5, x_84); +lean_ctor_set(x_128, 6, x_85); +lean_ctor_set(x_128, 7, x_87); +lean_ctor_set(x_128, 8, x_88); +lean_ctor_set(x_128, 9, x_127); +lean_ctor_set(x_128, 10, x_89); +lean_ctor_set(x_128, 11, x_90); +lean_ctor_set(x_128, 12, x_91); +lean_ctor_set(x_128, 13, x_92); +lean_ctor_set(x_128, 14, x_93); +lean_ctor_set(x_128, 15, x_94); +lean_ctor_set(x_128, 16, x_95); +lean_ctor_set(x_128, 17, x_96); +lean_ctor_set(x_128, 18, x_97); +lean_ctor_set(x_128, 19, x_98); +lean_ctor_set(x_128, 20, x_99); +lean_ctor_set(x_128, 21, x_100); +lean_ctor_set(x_128, 22, x_101); +lean_ctor_set_uint8(x_128, sizeof(void*)*23, x_86); +x_129 = lean_st_ref_set(x_6, x_128, x_19); +x_130 = lean_ctor_get(x_129, 1); +lean_inc(x_130); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_131 = x_129; +} else { + lean_dec_ref(x_129); + x_131 = lean_box(0); +} +x_132 = lean_box(0); +if (lean_is_scalar(x_131)) { + x_133 = lean_alloc_ctor(0, 2, 0); +} else { + x_133 = x_131; +} +lean_ctor_set(x_133, 0, x_132); +lean_ctor_set(x_133, 1, x_130); +return x_133; +} +} +} +else +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; +x_134 = lean_ctor_get(x_15, 1); +lean_inc(x_134); +lean_dec(x_15); +x_135 = lean_ctor_get(x_16, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_16, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_16, 2); +lean_inc(x_137); +x_138 = lean_ctor_get(x_16, 3); +lean_inc(x_138); +x_139 = lean_ctor_get(x_16, 4); +lean_inc(x_139); +x_140 = lean_ctor_get(x_16, 5); +lean_inc(x_140); +x_141 = lean_ctor_get(x_16, 6); +lean_inc(x_141); +x_142 = lean_ctor_get_uint8(x_16, sizeof(void*)*23); +x_143 = lean_ctor_get(x_16, 7); +lean_inc(x_143); +x_144 = lean_ctor_get(x_16, 8); +lean_inc(x_144); +x_145 = lean_ctor_get(x_16, 10); +lean_inc(x_145); +x_146 = lean_ctor_get(x_16, 11); +lean_inc(x_146); +x_147 = lean_ctor_get(x_16, 12); +lean_inc(x_147); +x_148 = lean_ctor_get(x_16, 13); +lean_inc(x_148); +x_149 = lean_ctor_get(x_16, 14); +lean_inc(x_149); +x_150 = lean_ctor_get(x_16, 15); +lean_inc(x_150); +x_151 = lean_ctor_get(x_16, 16); +lean_inc(x_151); +x_152 = lean_ctor_get(x_16, 17); +lean_inc(x_152); +x_153 = lean_ctor_get(x_16, 18); +lean_inc(x_153); +x_154 = lean_ctor_get(x_16, 19); +lean_inc(x_154); +x_155 = lean_ctor_get(x_16, 20); +lean_inc(x_155); +x_156 = lean_ctor_get(x_16, 21); +lean_inc(x_156); +x_157 = lean_ctor_get(x_16, 22); +lean_inc(x_157); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + lean_ctor_release(x_16, 1); + lean_ctor_release(x_16, 2); + lean_ctor_release(x_16, 3); + lean_ctor_release(x_16, 4); + lean_ctor_release(x_16, 5); + lean_ctor_release(x_16, 6); + lean_ctor_release(x_16, 7); + lean_ctor_release(x_16, 8); + lean_ctor_release(x_16, 9); + lean_ctor_release(x_16, 10); + lean_ctor_release(x_16, 11); + lean_ctor_release(x_16, 12); + lean_ctor_release(x_16, 13); + lean_ctor_release(x_16, 14); + lean_ctor_release(x_16, 15); + lean_ctor_release(x_16, 16); + lean_ctor_release(x_16, 17); + lean_ctor_release(x_16, 18); + lean_ctor_release(x_16, 19); + lean_ctor_release(x_16, 20); + lean_ctor_release(x_16, 21); + lean_ctor_release(x_16, 22); + x_158 = x_16; +} else { + lean_dec_ref(x_16); + x_158 = lean_box(0); +} +x_159 = lean_ctor_get(x_17, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_17, 1); +lean_inc(x_160); +x_161 = lean_ctor_get(x_17, 2); +lean_inc(x_161); +x_162 = lean_ctor_get(x_17, 3); +lean_inc(x_162); +x_163 = lean_ctor_get(x_17, 4); +lean_inc(x_163); +x_164 = lean_ctor_get(x_17, 5); +lean_inc(x_164); +x_165 = lean_ctor_get(x_17, 6); +lean_inc(x_165); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + lean_ctor_release(x_17, 2); + lean_ctor_release(x_17, 3); + lean_ctor_release(x_17, 4); + lean_ctor_release(x_17, 5); + lean_ctor_release(x_17, 6); + x_166 = x_17; +} else { + lean_dec_ref(x_17); + x_166 = lean_box(0); +} +lean_inc(x_2); +lean_inc(x_1); +x_167 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__1(x_161, x_1, x_2); +x_168 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_168, 0, x_3); +lean_ctor_set(x_168, 1, x_4); +lean_inc(x_162); +x_169 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__1(x_162, x_168); +if (lean_obj_tag(x_169) == 0) +{ +lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; +x_170 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_170, 0, x_2); +lean_ctor_set(x_170, 1, x_1); +x_171 = lean_box(0); +x_172 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_172, 0, x_170); +lean_ctor_set(x_172, 1, x_171); +x_173 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_162, x_168, x_172); +if (lean_is_scalar(x_166)) { + x_174 = lean_alloc_ctor(0, 7, 0); +} else { + x_174 = x_166; +} +lean_ctor_set(x_174, 0, x_159); +lean_ctor_set(x_174, 1, x_160); +lean_ctor_set(x_174, 2, x_167); +lean_ctor_set(x_174, 3, x_173); +lean_ctor_set(x_174, 4, x_163); +lean_ctor_set(x_174, 5, x_164); +lean_ctor_set(x_174, 6, x_165); +if (lean_is_scalar(x_158)) { + x_175 = lean_alloc_ctor(0, 23, 1); +} else { + x_175 = x_158; +} +lean_ctor_set(x_175, 0, x_135); +lean_ctor_set(x_175, 1, x_136); +lean_ctor_set(x_175, 2, x_137); +lean_ctor_set(x_175, 3, x_138); +lean_ctor_set(x_175, 4, x_139); +lean_ctor_set(x_175, 5, x_140); +lean_ctor_set(x_175, 6, x_141); +lean_ctor_set(x_175, 7, x_143); +lean_ctor_set(x_175, 8, x_144); +lean_ctor_set(x_175, 9, x_174); +lean_ctor_set(x_175, 10, x_145); +lean_ctor_set(x_175, 11, x_146); +lean_ctor_set(x_175, 12, x_147); +lean_ctor_set(x_175, 13, x_148); +lean_ctor_set(x_175, 14, x_149); +lean_ctor_set(x_175, 15, x_150); +lean_ctor_set(x_175, 16, x_151); +lean_ctor_set(x_175, 17, x_152); +lean_ctor_set(x_175, 18, x_153); +lean_ctor_set(x_175, 19, x_154); +lean_ctor_set(x_175, 20, x_155); +lean_ctor_set(x_175, 21, x_156); +lean_ctor_set(x_175, 22, x_157); +lean_ctor_set_uint8(x_175, sizeof(void*)*23, x_142); +x_176 = lean_st_ref_set(x_6, x_175, x_134); +x_177 = lean_ctor_get(x_176, 1); +lean_inc(x_177); +if (lean_is_exclusive(x_176)) { + lean_ctor_release(x_176, 0); + lean_ctor_release(x_176, 1); + x_178 = x_176; +} else { + lean_dec_ref(x_176); + x_178 = lean_box(0); +} +x_179 = lean_box(0); +if (lean_is_scalar(x_178)) { + x_180 = lean_alloc_ctor(0, 2, 0); +} else { + x_180 = x_178; +} +lean_ctor_set(x_180, 0, x_179); +lean_ctor_set(x_180, 1, x_177); +return x_180; +} +else +{ +lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_181 = lean_ctor_get(x_169, 0); +lean_inc(x_181); +lean_dec(x_169); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_2); +lean_ctor_set(x_182, 1, x_1); +x_183 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_183, 0, x_182); +lean_ctor_set(x_183, 1, x_181); +x_184 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_updateCnstrsOf___spec__5(x_162, x_168, x_183); +if (lean_is_scalar(x_166)) { + x_185 = lean_alloc_ctor(0, 7, 0); +} else { + x_185 = x_166; +} +lean_ctor_set(x_185, 0, x_159); +lean_ctor_set(x_185, 1, x_160); +lean_ctor_set(x_185, 2, x_167); +lean_ctor_set(x_185, 3, x_184); +lean_ctor_set(x_185, 4, x_163); +lean_ctor_set(x_185, 5, x_164); +lean_ctor_set(x_185, 6, x_165); +if (lean_is_scalar(x_158)) { + x_186 = lean_alloc_ctor(0, 23, 1); +} else { + x_186 = x_158; +} +lean_ctor_set(x_186, 0, x_135); +lean_ctor_set(x_186, 1, x_136); +lean_ctor_set(x_186, 2, x_137); +lean_ctor_set(x_186, 3, x_138); +lean_ctor_set(x_186, 4, x_139); +lean_ctor_set(x_186, 5, x_140); +lean_ctor_set(x_186, 6, x_141); +lean_ctor_set(x_186, 7, x_143); +lean_ctor_set(x_186, 8, x_144); +lean_ctor_set(x_186, 9, x_185); +lean_ctor_set(x_186, 10, x_145); +lean_ctor_set(x_186, 11, x_146); +lean_ctor_set(x_186, 12, x_147); +lean_ctor_set(x_186, 13, x_148); +lean_ctor_set(x_186, 14, x_149); +lean_ctor_set(x_186, 15, x_150); +lean_ctor_set(x_186, 16, x_151); +lean_ctor_set(x_186, 17, x_152); +lean_ctor_set(x_186, 18, x_153); +lean_ctor_set(x_186, 19, x_154); +lean_ctor_set(x_186, 20, x_155); +lean_ctor_set(x_186, 21, x_156); +lean_ctor_set(x_186, 22, x_157); +lean_ctor_set_uint8(x_186, sizeof(void*)*23, x_142); +x_187 = lean_st_ref_set(x_6, x_186, x_134); +x_188 = lean_ctor_get(x_187, 1); +lean_inc(x_188); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_189 = x_187; +} else { + lean_dec_ref(x_187); + x_189 = lean_box(0); +} +x_190 = lean_box(0); +if (lean_is_scalar(x_189)) { + x_191 = lean_alloc_ctor(0, 2, 0); +} else { + x_191 = x_189; +} +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_188); +return x_191; +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ↦ ", 5, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1; +x_16 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_unbox(x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_box(0); +x_21 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(x_1, x_2, x_3, x_4, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_19); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_23 = lean_ctor_get(x_16, 1); +x_24 = lean_ctor_get(x_16, 0); +lean_dec(x_24); +lean_inc(x_1); +x_25 = l_Lean_MessageData_ofExpr(x_1); +x_26 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_16, 7); +lean_ctor_set(x_16, 1, x_25); +lean_ctor_set(x_16, 0, x_26); +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_16); +lean_ctor_set(x_28, 1, x_27); +lean_inc(x_2); +x_29 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__5(x_26, x_2); +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_26); +x_32 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_15, x_31, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_23); +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(x_1, x_2, x_3, x_4, x_33, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_34); +lean_dec(x_33); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_36 = lean_ctor_get(x_16, 1); +lean_inc(x_36); +lean_dec(x_16); +lean_inc(x_1); +x_37 = l_Lean_MessageData_ofExpr(x_1); +x_38 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +x_40 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +lean_inc(x_2); +x_42 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__5(x_38, x_2); +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_38); +x_45 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_15, x_44, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_36); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(x_1, x_2, x_3, x_4, x_46, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_47); +lean_dec(x_46); +return x_48; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; lean_object* x_16; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_1, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = lean_box(0); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2(x_3, x_4, x_2, x_1, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_15, 1); +lean_inc(x_20); +lean_dec(x_15); +x_21 = lean_ctor_get(x_16, 0); +lean_inc(x_21); +lean_dec(x_16); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_22 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse(x_1, x_2, x_21, x_4, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_unbox(x_23); +lean_dec(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_box(0); +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2(x_3, x_4, x_2, x_1, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +return x_27; +} +else +{ +uint8_t x_28; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_22); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_22, 0); +lean_dec(x_29); +x_30 = lean_box(0); +lean_ctor_set(x_22, 0, x_30); +return x_22; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_22, 1); +lean_inc(x_31); +lean_dec(x_22); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; +} +} +} +else +{ +uint8_t x_34; +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_22); +if (x_34 == 0) +{ +return x_22; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_22, 0); +x_36 = lean_ctor_get(x_22, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_22); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_2, 0); +x_14 = lean_ctor_get(x_2, 1); +x_15 = lean_ctor_get(x_2, 2); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_19 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +lean_inc(x_20); +lean_inc(x_17); +lean_ctor_set(x_2, 1, x_20); +lean_ctor_set(x_2, 0, x_17); +x_22 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_17, x_20, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_box(0); +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(x_20, x_17, x_1, x_2, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_24); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_22, 1); +lean_inc(x_27); +lean_dec(x_22); +x_28 = lean_ctor_get(x_23, 0); +lean_inc(x_28); +lean_dec(x_23); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +lean_inc(x_20); +lean_inc(x_17); +x_29 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(x_17, x_20, x_28, x_2, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_27); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; uint8_t x_31; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_unbox(x_30); +lean_dec(x_30); +if (x_31 == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +x_33 = lean_box(0); +x_34 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(x_20, x_17, x_1, x_2, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_32); +return x_34; +} +else +{ +uint8_t x_35; +lean_dec(x_2); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_29); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; +x_36 = lean_ctor_get(x_29, 0); +lean_dec(x_36); +x_37 = lean_box(0); +lean_ctor_set(x_29, 0, x_37); +return x_29; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_29, 1); +lean_inc(x_38); +lean_dec(x_29); +x_39 = lean_box(0); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_2); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_29); +if (x_41 == 0) +{ +return x_29; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_29, 0); +x_43 = lean_ctor_get(x_29, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_29); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +else +{ +uint8_t x_45; +lean_dec(x_17); +lean_free_object(x_2); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_45 = !lean_is_exclusive(x_19); +if (x_45 == 0) +{ +return x_19; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_19, 0); +x_47 = lean_ctor_get(x_19, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_19); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +else +{ +uint8_t x_49; +lean_free_object(x_2); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_49 = !lean_is_exclusive(x_16); +if (x_49 == 0) +{ +return x_16; +} +else +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_16, 0); +x_51 = lean_ctor_get(x_16, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_16); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_53 = lean_ctor_get(x_2, 0); +x_54 = lean_ctor_get(x_2, 1); +x_55 = lean_ctor_get(x_2, 2); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_2); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_56 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_53, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_56) == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_59 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_54, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_58); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +lean_inc(x_60); +lean_inc(x_57); +x_62 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_62, 0, x_57); +lean_ctor_set(x_62, 1, x_60); +lean_ctor_set(x_62, 2, x_55); +x_63 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getDist_x3f(x_57, x_60, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_61); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +if (lean_obj_tag(x_64) == 0) +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_63, 1); +lean_inc(x_65); +lean_dec(x_63); +x_66 = lean_box(0); +x_67 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(x_60, x_57, x_1, x_62, x_66, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_65); +return x_67; +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_63, 1); +lean_inc(x_68); +lean_dec(x_63); +x_69 = lean_ctor_get(x_64, 0); +lean_inc(x_69); +lean_dec(x_64); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +lean_inc(x_60); +lean_inc(x_57); +x_70 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue(x_57, x_60, x_69, x_62, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_68); +if (lean_obj_tag(x_70) == 0) +{ +lean_object* x_71; uint8_t x_72; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_unbox(x_71); +lean_dec(x_71); +if (x_72 == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_70, 1); +lean_inc(x_73); +lean_dec(x_70); +x_74 = lean_box(0); +x_75 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(x_60, x_57, x_1, x_62, x_74, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_73); +return x_75; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_62); +lean_dec(x_60); +lean_dec(x_57); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_76 = lean_ctor_get(x_70, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_77 = x_70; +} else { + lean_dec_ref(x_70); + x_77 = lean_box(0); +} +x_78 = lean_box(0); +if (lean_is_scalar(x_77)) { + x_79 = lean_alloc_ctor(0, 2, 0); +} else { + x_79 = x_77; +} +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_76); +return x_79; +} +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_62); +lean_dec(x_60); +lean_dec(x_57); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_80 = lean_ctor_get(x_70, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_70, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_70)) { + lean_ctor_release(x_70, 0); + lean_ctor_release(x_70, 1); + x_82 = x_70; +} else { + lean_dec_ref(x_70); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; +} +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; +} +} +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_57); +lean_dec(x_55); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_84 = lean_ctor_get(x_59, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_59, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_86 = x_59; +} else { + lean_dec_ref(x_59); + x_86 = lean_box(0); +} +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); +} else { + x_87 = x_86; +} +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; +} +} +else +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +lean_dec(x_55); +lean_dec(x_54); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_88 = lean_ctor_get(x_56, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_56, 1); +lean_inc(x_89); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_90 = x_56; +} else { + lean_dec_ref(x_56); + x_90 = lean_box(0); +} +if (lean_is_scalar(x_90)) { + x_91 = lean_alloc_ctor(1, 2, 0); +} else { + x_91 = x_90; +} +lean_ctor_set(x_91, 0, x_88); +lean_ctor_set(x_91, 1, x_89); +return x_91; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +size_t x_7; lean_object* x_8; +x_7 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_8 = l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__3(x_7, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_3); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +size_t x_6; size_t x_7; lean_object* x_8; +x_6 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_7 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_8 = l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___spec__2(x_1, x_6, x_7, x_4, x_5); +return x_8; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getZeroNode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_11, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +return x_13; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_refl", 7, 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_offset", 9, 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_13 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3; +x_20 = l_Lean_Expr_app___override(x_19, x_1); +lean_inc(x_3); +x_21 = lean_nat_to_int(x_3); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_20); +lean_inc(x_21); +lean_inc(x_17); +lean_inc(x_14); +x_22 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_14, x_17, x_21, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = lean_int_neg(x_21); +lean_dec(x_21); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_24); +lean_inc(x_14); +x_25 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_17, x_14, x_24, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getZeroNode(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l_Lean_mkNatLit(x_3); +x_31 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6; +x_32 = l_Lean_mkAppB(x_31, x_2, x_30); +x_33 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_28, x_14, x_24, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_29); +return x_33; +} +else +{ +uint8_t x_34; +lean_dec(x_24); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_34 = !lean_is_exclusive(x_27); +if (x_34 == 0) +{ +return x_27; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_27, 0); +x_36 = lean_ctor_get(x_27, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_27); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +uint8_t x_38; +lean_dec(x_24); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_38 = !lean_is_exclusive(x_25); +if (x_38 == 0) +{ +return x_25; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_25, 0); +x_40 = lean_ctor_get(x_25, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_25); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_42 = !lean_is_exclusive(x_22); +if (x_42 == 0) +{ +return x_22; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_22, 0); +x_44 = lean_ctor_get(x_22, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_22); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +uint8_t x_46; +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_46 = !lean_is_exclusive(x_16); +if (x_46 == 0) +{ +return x_16; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_16, 0); +x_48 = lean_ctor_get(x_16, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_16); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; +} +} +} +else +{ +uint8_t x_50; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_13); +if (x_50 == 0) +{ +return x_13; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_13, 0); +x_52 = lean_ctor_get(x_13, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_13); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_11; lean_object* x_12; lean_object* x_13; +x_11 = 0; +x_12 = lean_box(x_11); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_10); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +lean_dec(x_1); +x_15 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_10); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_inc(x_14); +x_18 = l_Lean_Meta_Grind_Arith_isNatAdd(x_14); +if (x_18 == 0) +{ +lean_object* x_19; +x_19 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(x_14, x_17); +if (lean_obj_tag(x_19) == 0) +{ +uint8_t x_20; lean_object* x_21; +x_20 = 1; +x_21 = lean_box(x_20); +lean_ctor_set(x_15, 0, x_21); +return x_15; +} +else +{ +uint8_t x_22; lean_object* x_23; +lean_dec(x_19); +x_22 = 0; +x_23 = lean_box(x_22); +lean_ctor_set(x_15, 0, x_23); +return x_15; +} +} +else +{ +uint8_t x_24; lean_object* x_25; +lean_dec(x_17); +lean_dec(x_14); +x_24 = 0; +x_25 = lean_box(x_24); +lean_ctor_set(x_15, 0, x_25); +return x_15; +} +} +else +{ +lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_26 = lean_ctor_get(x_15, 0); +x_27 = lean_ctor_get(x_15, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_15); +lean_inc(x_14); +x_28 = l_Lean_Meta_Grind_Arith_isNatAdd(x_14); +if (x_28 == 0) +{ +lean_object* x_29; +x_29 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(x_14, x_26); +if (lean_obj_tag(x_29) == 0) +{ +uint8_t x_30; lean_object* x_31; lean_object* x_32; +x_30 = 1; +x_31 = lean_box(x_30); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_27); +return x_32; +} +else +{ +uint8_t x_33; lean_object* x_34; lean_object* x_35; +lean_dec(x_29); +x_33 = 0; +x_34 = lean_box(x_33); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_27); +return x_35; +} +} +else +{ +uint8_t x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_26); +lean_dec(x_14); +x_36 = 0; +x_37 = lean_box(x_36); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_27); +return x_38; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +uint8_t x_2; +x_2 = 0; +return x_2; +} +else +{ +lean_object* x_3; uint8_t x_4; +x_3 = lean_ctor_get(x_1, 0); +x_4 = l_Lean_Expr_isEq(x_3); +return x_4; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_internalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_6, x_7, x_8, x_9, x_10, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +lean_inc(x_13); +lean_inc(x_1); +x_15 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(x_1, x_13); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; uint8_t x_18; +lean_inc(x_2); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isRelevantParent(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_unbox(x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +uint8_t x_19; +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_16); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_16, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_16, 0, x_21); +return x_16; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 1); +lean_inc(x_22); +lean_dec(x_16); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; +} +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_16); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_16, 1); +x_27 = lean_ctor_get(x_16, 0); +lean_dec(x_27); +lean_inc(x_1); +x_28 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_1); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; +lean_inc(x_1); +x_29 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_1); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_30 = lean_box(0); +lean_ctor_set(x_16, 0, x_30); +return x_16; +} +else +{ +lean_object* x_31; uint8_t x_32; +x_31 = lean_ctor_get(x_29, 0); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent(x_2); +lean_dec(x_2); +if (x_32 == 0) +{ +lean_object* x_33; +lean_free_object(x_16); +x_33 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(x_1, x_13, x_31, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_26); +return x_33; +} +else +{ +lean_object* x_34; +lean_dec(x_31); +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_34 = lean_box(0); +lean_ctor_set(x_16, 0, x_34); +return x_16; +} +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_free_object(x_16); +lean_dec(x_13); +lean_dec(x_2); +x_35 = lean_ctor_get(x_28, 0); +lean_inc(x_35); +lean_dec(x_28); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(x_1, x_36, x_37, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_26); +return x_38; +} +} +else +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_16, 1); +lean_inc(x_39); +lean_dec(x_16); +lean_inc(x_1); +x_40 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_1); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; +lean_inc(x_1); +x_41 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_1); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_42 = lean_box(0); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_39); +return x_43; +} +else +{ +lean_object* x_44; uint8_t x_45; +x_44 = lean_ctor_get(x_41, 0); +lean_inc(x_44); +lean_dec(x_41); +x_45 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_isEqParent(x_2); +lean_dec(x_2); +if (x_45 == 0) +{ +lean_object* x_46; +x_46 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(x_1, x_13, x_44, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_39); +return x_46; +} +else +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_44); +lean_dec(x_13); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_47 = lean_box(0); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_39); +return x_48; +} +} +} +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_13); +lean_dec(x_2); +x_49 = lean_ctor_get(x_40, 0); +lean_inc(x_49); +lean_dec(x_40); +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +x_52 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm(x_1, x_50, x_51, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_39); +return x_52; +} +} +} +} +else +{ +lean_object* x_53; lean_object* x_54; +lean_dec(x_13); +lean_dec(x_2); +x_53 = lean_ctor_get(x_15, 0); +lean_inc(x_53); +lean_dec(x_15); +x_54 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr(x_1, x_53, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_54; +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_of_eq_1", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +x_4 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_of_eq_2", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3; +x_4 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +lean_inc(x_1); +x_13 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_inc(x_2); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_19 = lean_grind_mk_eq_proof(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3; +lean_inc(x_20); +lean_inc(x_2); +lean_inc(x_1); +x_23 = l_Lean_mkApp3(x_22, x_1, x_2, x_20); +x_24 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_17); +lean_inc(x_14); +x_25 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_14, x_17, x_24, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6; +x_28 = l_Lean_mkApp3(x_27, x_1, x_2, x_20); +x_29 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_17, x_14, x_24, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); +return x_29; +} +else +{ +uint8_t x_30; +lean_dec(x_20); +lean_dec(x_17); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_30 = !lean_is_exclusive(x_25); +if (x_30 == 0) +{ +return x_25; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_25, 0); +x_32 = lean_ctor_get(x_25, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_25); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; +} +} +} +else +{ +uint8_t x_34; +lean_dec(x_17); +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_19); +if (x_34 == 0) +{ +return x_19; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_19, 0); +x_36 = lean_ctor_get(x_19, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_19); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +uint8_t x_38; +lean_dec(x_14); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_38 = !lean_is_exclusive(x_16); +if (x_38 == 0) +{ +return x_16; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_16, 0); +x_40 = lean_ctor_get(x_16, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_16); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_13); +if (x_42 == 0) +{ +return x_13; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_13, 0); +x_44 = lean_ctor_get(x_13, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_13); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("to", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* lean_process_new_offset_eq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2; +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(x_1, x_2, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_14); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_21 = lean_ctor_get(x_14, 1); +x_22 = lean_ctor_get(x_14, 0); +lean_dec(x_22); +lean_inc(x_1); +x_23 = l_Lean_MessageData_ofExpr(x_1); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_23); +lean_ctor_set(x_14, 0, x_24); +x_25 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_14); +lean_ctor_set(x_26, 1, x_25); +lean_inc(x_2); +x_27 = l_Lean_MessageData_ofExpr(x_2); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_24); +x_30 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_29, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(x_1, x_2, x_31, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_32); +lean_dec(x_31); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_34 = lean_ctor_get(x_14, 1); +lean_inc(x_34); +lean_dec(x_14); +lean_inc(x_1); +x_35 = l_Lean_MessageData_ofExpr(x_1); +x_36 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +lean_inc(x_2); +x_40 = l_Lean_MessageData_ofExpr(x_2); +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_36); +x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_42, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(x_1, x_2, x_44, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_45); +lean_dec(x_44); +return x_46; +} +} +} +else +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_47 = lean_box(0); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_11); +return x_48; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_13; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.processNewOffsetEqLitImpl", 54, 54); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1; +x_3 = lean_unsigned_to_nat(299u); +x_4 = lean_unsigned_to_nat(32u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +lean_inc(x_1); +x_13 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_1); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; +lean_dec(x_2); +lean_dec(x_1); +x_14 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3; +x_15 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_15; +} +else +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); +lean_inc(x_16); +lean_dec(x_13); +lean_inc(x_2); +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_7, x_8, x_9, x_10, x_11, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_23 = l_Lean_Meta_Grind_Arith_Offset_mkNode(x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +lean_inc(x_2); +x_26 = lean_grind_mk_eq_proof(x_2, x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_nat_to_int(x_16); +x_30 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3; +lean_inc(x_27); +lean_inc(x_1); +lean_inc(x_2); +x_31 = l_Lean_mkApp3(x_30, x_2, x_1, x_27); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_29); +lean_inc(x_24); +lean_inc(x_18); +x_32 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_18, x_24, x_29, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_int_neg(x_29); +lean_dec(x_29); +x_35 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6; +x_36 = l_Lean_mkApp3(x_35, x_2, x_1, x_27); +x_37 = l_Lean_Meta_Grind_Arith_Offset_addEdge(x_24, x_18, x_34, x_36, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +return x_37; +} +else +{ +uint8_t x_38; +lean_dec(x_29); +lean_dec(x_27); +lean_dec(x_24); +lean_dec(x_18); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_38 = !lean_is_exclusive(x_32); +if (x_38 == 0) +{ +return x_32; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_32, 0); +x_40 = lean_ctor_get(x_32, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_32); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +uint8_t x_42; +lean_dec(x_24); +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_26); +if (x_42 == 0) +{ +return x_26; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_26, 0); +x_44 = lean_ctor_get(x_26, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_26); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} +} +} +else +{ +uint8_t x_46; +lean_dec(x_18); +lean_dec(x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_46 = !lean_is_exclusive(x_23); +if (x_46 == 0) +{ +return x_23; +} +else +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_23, 0); +x_48 = lean_ctor_get(x_23, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_23); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; +} +} +} +else +{ +uint8_t x_50; +lean_dec(x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_17); +if (x_50 == 0) +{ +return x_17; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_17, 0); +x_52 = lean_ctor_get(x_17, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_17); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; +} +} +} +} +} +LEAN_EXPORT lean_object* lean_process_new_offset_eq_lit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +uint8_t x_12; +x_12 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2; +x_14 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_14, 1); +lean_inc(x_17); +lean_dec(x_14); +x_18 = lean_box(0); +x_19 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(x_2, x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +return x_19; +} +else +{ +uint8_t x_20; +x_20 = !lean_is_exclusive(x_14); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_21 = lean_ctor_get(x_14, 1); +x_22 = lean_ctor_get(x_14, 0); +lean_dec(x_22); +lean_inc(x_1); +x_23 = l_Lean_MessageData_ofExpr(x_1); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_23); +lean_ctor_set(x_14, 0, x_24); +x_25 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_14); +lean_ctor_set(x_26, 1, x_25); +lean_inc(x_2); +x_27 = l_Lean_MessageData_ofExpr(x_2); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_24); +x_30 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_29, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(x_2, x_1, x_31, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_32); +lean_dec(x_31); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_34 = lean_ctor_get(x_14, 1); +lean_inc(x_34); +lean_dec(x_14); +lean_inc(x_1); +x_35 = l_Lean_MessageData_ofExpr(x_1); +x_36 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_37 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +lean_inc(x_2); +x_40 = l_Lean_MessageData_ofExpr(x_2); +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_36); +x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_42, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(x_2, x_1, x_44, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_45); +lean_dec(x_44); +return x_46; +} +} +} +else +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_47 = lean_box(0); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set(x_48, 1, x_11); +return x_48; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_3); +return x_13; +} +} +static double _init_l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_9, 5); +x_13 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_7, x_8, x_9, x_10, x_11); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_st_ref_take(x_10, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_17, 3); +lean_inc(x_18); +x_19 = !lean_is_exclusive(x_16); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_16, 1); +x_21 = lean_ctor_get(x_16, 0); +lean_dec(x_21); +x_22 = !lean_is_exclusive(x_17); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_17, 3); +lean_dec(x_23); +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; double x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_25 = lean_ctor_get(x_18, 0); +x_26 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1; +x_27 = 0; +x_28 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +x_29 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_29, 0, x_1); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set_float(x_29, sizeof(void*)*2, x_26); +lean_ctor_set_float(x_29, sizeof(void*)*2 + 8, x_26); +lean_ctor_set_uint8(x_29, sizeof(void*)*2 + 16, x_27); +x_30 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2; +x_31 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_14); +lean_ctor_set(x_31, 2, x_30); +lean_inc(x_12); +lean_ctor_set(x_16, 1, x_31); +lean_ctor_set(x_16, 0, x_12); +x_32 = l_Lean_PersistentArray_push___rarg(x_25, x_16); +lean_ctor_set(x_18, 0, x_32); +x_33 = lean_st_ref_set(x_10, x_17, x_20); +x_34 = !lean_is_exclusive(x_33); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_33, 0); +lean_dec(x_35); +x_36 = lean_box(0); +lean_ctor_set(x_33, 0, x_36); +return x_33; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_33, 1); +lean_inc(x_37); +lean_dec(x_33); +x_38 = lean_box(0); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +return x_39; +} +} +else +{ +uint64_t x_40; lean_object* x_41; double x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_40 = lean_ctor_get_uint64(x_18, sizeof(void*)*1); +x_41 = lean_ctor_get(x_18, 0); +lean_inc(x_41); +lean_dec(x_18); +x_42 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1; +x_43 = 0; +x_44 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +x_45 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_45, 0, x_1); +lean_ctor_set(x_45, 1, x_44); +lean_ctor_set_float(x_45, sizeof(void*)*2, x_42); +lean_ctor_set_float(x_45, sizeof(void*)*2 + 8, x_42); +lean_ctor_set_uint8(x_45, sizeof(void*)*2 + 16, x_43); +x_46 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2; +x_47 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_14); +lean_ctor_set(x_47, 2, x_46); +lean_inc(x_12); +lean_ctor_set(x_16, 1, x_47); +lean_ctor_set(x_16, 0, x_12); +x_48 = l_Lean_PersistentArray_push___rarg(x_41, x_16); +x_49 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set_uint64(x_49, sizeof(void*)*1, x_40); +lean_ctor_set(x_17, 3, x_49); +x_50 = lean_st_ref_set(x_10, x_17, x_20); +x_51 = lean_ctor_get(x_50, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_52 = x_50; +} else { + lean_dec_ref(x_50); + x_52 = lean_box(0); +} +x_53 = lean_box(0); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); +} else { + x_54 = x_52; +} +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint64_t x_62; lean_object* x_63; lean_object* x_64; double x_65; uint8_t x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_55 = lean_ctor_get(x_17, 0); +x_56 = lean_ctor_get(x_17, 1); +x_57 = lean_ctor_get(x_17, 2); +x_58 = lean_ctor_get(x_17, 4); +x_59 = lean_ctor_get(x_17, 5); +x_60 = lean_ctor_get(x_17, 6); +x_61 = lean_ctor_get(x_17, 7); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_17); +x_62 = lean_ctor_get_uint64(x_18, sizeof(void*)*1); +x_63 = lean_ctor_get(x_18, 0); +lean_inc(x_63); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + x_64 = x_18; +} else { + lean_dec_ref(x_18); + x_64 = lean_box(0); +} +x_65 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1; +x_66 = 0; +x_67 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +x_68 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_68, 0, x_1); +lean_ctor_set(x_68, 1, x_67); +lean_ctor_set_float(x_68, sizeof(void*)*2, x_65); +lean_ctor_set_float(x_68, sizeof(void*)*2 + 8, x_65); +lean_ctor_set_uint8(x_68, sizeof(void*)*2 + 16, x_66); +x_69 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2; +x_70 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_14); +lean_ctor_set(x_70, 2, x_69); +lean_inc(x_12); +lean_ctor_set(x_16, 1, x_70); +lean_ctor_set(x_16, 0, x_12); +x_71 = l_Lean_PersistentArray_push___rarg(x_63, x_16); +if (lean_is_scalar(x_64)) { + x_72 = lean_alloc_ctor(0, 1, 8); +} else { + x_72 = x_64; +} +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set_uint64(x_72, sizeof(void*)*1, x_62); +x_73 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_73, 0, x_55); +lean_ctor_set(x_73, 1, x_56); +lean_ctor_set(x_73, 2, x_57); +lean_ctor_set(x_73, 3, x_72); +lean_ctor_set(x_73, 4, x_58); +lean_ctor_set(x_73, 5, x_59); +lean_ctor_set(x_73, 6, x_60); +lean_ctor_set(x_73, 7, x_61); +x_74 = lean_st_ref_set(x_10, x_73, x_20); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_76 = x_74; +} else { + lean_dec_ref(x_74); + x_76 = lean_box(0); +} +x_77 = lean_box(0); +if (lean_is_scalar(x_76)) { + x_78 = lean_alloc_ctor(0, 2, 0); +} else { + x_78 = x_76; +} +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_75); +return x_78; +} +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint64_t x_88; lean_object* x_89; lean_object* x_90; double x_91; uint8_t x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_79 = lean_ctor_get(x_16, 1); +lean_inc(x_79); +lean_dec(x_16); +x_80 = lean_ctor_get(x_17, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_17, 1); +lean_inc(x_81); +x_82 = lean_ctor_get(x_17, 2); +lean_inc(x_82); +x_83 = lean_ctor_get(x_17, 4); +lean_inc(x_83); +x_84 = lean_ctor_get(x_17, 5); +lean_inc(x_84); +x_85 = lean_ctor_get(x_17, 6); +lean_inc(x_85); +x_86 = lean_ctor_get(x_17, 7); +lean_inc(x_86); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + lean_ctor_release(x_17, 1); + lean_ctor_release(x_17, 2); + lean_ctor_release(x_17, 3); + lean_ctor_release(x_17, 4); + lean_ctor_release(x_17, 5); + lean_ctor_release(x_17, 6); + lean_ctor_release(x_17, 7); + x_87 = x_17; +} else { + lean_dec_ref(x_17); + x_87 = lean_box(0); +} +x_88 = lean_ctor_get_uint64(x_18, sizeof(void*)*1); +x_89 = lean_ctor_get(x_18, 0); +lean_inc(x_89); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + x_90 = x_18; +} else { + lean_dec_ref(x_18); + x_90 = lean_box(0); +} +x_91 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1; +x_92 = 0; +x_93 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6; +x_94 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_94, 0, x_1); +lean_ctor_set(x_94, 1, x_93); +lean_ctor_set_float(x_94, sizeof(void*)*2, x_91); +lean_ctor_set_float(x_94, sizeof(void*)*2 + 8, x_91); +lean_ctor_set_uint8(x_94, sizeof(void*)*2 + 16, x_92); +x_95 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2; +x_96 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_14); +lean_ctor_set(x_96, 2, x_95); +lean_inc(x_12); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_12); +lean_ctor_set(x_97, 1, x_96); +x_98 = l_Lean_PersistentArray_push___rarg(x_89, x_97); +if (lean_is_scalar(x_90)) { + x_99 = lean_alloc_ctor(0, 1, 8); +} else { + x_99 = x_90; +} +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set_uint64(x_99, sizeof(void*)*1, x_88); +if (lean_is_scalar(x_87)) { + x_100 = lean_alloc_ctor(0, 8, 0); +} else { + x_100 = x_87; +} +lean_ctor_set(x_100, 0, x_80); +lean_ctor_set(x_100, 1, x_81); +lean_ctor_set(x_100, 2, x_82); +lean_ctor_set(x_100, 3, x_99); +lean_ctor_set(x_100, 4, x_83); +lean_ctor_set(x_100, 5, x_84); +lean_ctor_set(x_100, 6, x_85); +lean_ctor_set(x_100, 7, x_86); +x_101 = lean_st_ref_set(x_10, x_100, x_79); +x_102 = lean_ctor_get(x_101, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_101)) { + lean_ctor_release(x_101, 0); + lean_ctor_release(x_101, 1); + x_103 = x_101; +} else { + lean_dec_ref(x_101); + x_103 = lean_box(0); +} +x_104 = lean_box(0); +if (lean_is_scalar(x_103)) { + x_105 = lean_alloc_ctor(0, 2, 0); +} else { + x_105 = x_103; +} +lean_ctor_set(x_105, 0, x_104); +lean_ctor_set(x_105, 1, x_102); +return x_105; +} +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" -(", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(")-> #", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("-", 1, 1); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_13; +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_2); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_dec(x_2); +x_14 = lean_ctor_get(x_3, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_3, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_3, 2); +lean_inc(x_16); +lean_dec(x_3); +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_15); +lean_dec(x_14); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_2 = x_22; +x_3 = x_16; +x_12 = x_21; +goto _start; +} +else +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_25 = lean_ctor_get(x_18, 1); +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +lean_inc(x_1); +x_27 = l___private_Init_Data_Repr_0__Nat_reprFast(x_1); +x_28 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_28, 0, x_27); +x_29 = l_Lean_MessageData_ofFormat(x_28); +x_30 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_29); +lean_ctor_set(x_18, 0, x_30); +x_31 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_18); +lean_ctor_set(x_32, 1, x_31); +x_33 = l___private_Init_Data_Repr_0__Nat_reprFast(x_14); +x_34 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_34, 0, x_33); +x_35 = l_Lean_MessageData_ofFormat(x_34); +x_36 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_37 = lean_int_dec_lt(x_15, x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_38 = lean_nat_abs(x_15); +lean_dec(x_15); +x_39 = l___private_Init_Data_Repr_0__Nat_reprFast(x_38); +x_40 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_40, 0, x_39); +x_41 = l_Lean_MessageData_ofFormat(x_40); +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_32); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_35); +x_46 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(x_17, x_47, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_box(0); +x_2 = x_50; +x_3 = x_16; +x_12 = x_49; +goto _start; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_52 = lean_nat_abs(x_15); +lean_dec(x_15); +x_53 = lean_unsigned_to_nat(1u); +x_54 = lean_nat_sub(x_52, x_53); +lean_dec(x_52); +x_55 = lean_nat_add(x_54, x_53); +lean_dec(x_54); +x_56 = l___private_Init_Data_Repr_0__Nat_reprFast(x_55); +x_57 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5; +x_58 = lean_string_append(x_57, x_56); +lean_dec(x_56); +x_59 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_59, 0, x_58); +x_60 = l_Lean_MessageData_ofFormat(x_59); +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_32); +lean_ctor_set(x_61, 1, x_60); +x_62 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4; +x_63 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_35); +x_65 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(x_17, x_66, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +x_68 = lean_ctor_get(x_67, 1); +lean_inc(x_68); +lean_dec(x_67); +x_69 = lean_box(0); +x_2 = x_69; +x_3 = x_16; +x_12 = x_68; +goto _start; +} +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; uint8_t x_83; +x_71 = lean_ctor_get(x_18, 1); +lean_inc(x_71); +lean_dec(x_18); +lean_inc(x_1); +x_72 = l___private_Init_Data_Repr_0__Nat_reprFast(x_1); +x_73 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_73, 0, x_72); +x_74 = l_Lean_MessageData_ofFormat(x_73); +x_75 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_77 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +x_79 = l___private_Init_Data_Repr_0__Nat_reprFast(x_14); +x_80 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_80, 0, x_79); +x_81 = l_Lean_MessageData_ofFormat(x_80); +x_82 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_83 = lean_int_dec_lt(x_15, x_82); +if (x_83 == 0) +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_84 = lean_nat_abs(x_15); +lean_dec(x_15); +x_85 = l___private_Init_Data_Repr_0__Nat_reprFast(x_84); +x_86 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_86, 0, x_85); +x_87 = l_Lean_MessageData_ofFormat(x_86); +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_78); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4; +x_90 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_90, 0, x_88); +lean_ctor_set(x_90, 1, x_89); +x_91 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_81); +x_92 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_93 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_94 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(x_17, x_93, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_71); +x_95 = lean_ctor_get(x_94, 1); +lean_inc(x_95); +lean_dec(x_94); +x_96 = lean_box(0); +x_2 = x_96; +x_3 = x_16; +x_12 = x_95; +goto _start; +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_98 = lean_nat_abs(x_15); +lean_dec(x_15); +x_99 = lean_unsigned_to_nat(1u); +x_100 = lean_nat_sub(x_98, x_99); +lean_dec(x_98); +x_101 = lean_nat_add(x_100, x_99); +lean_dec(x_100); +x_102 = l___private_Init_Data_Repr_0__Nat_reprFast(x_101); +x_103 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5; +x_104 = lean_string_append(x_103, x_102); +lean_dec(x_102); +x_105 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_105, 0, x_104); +x_106 = l_Lean_MessageData_ofFormat(x_105); +x_107 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_107, 0, x_78); +lean_ctor_set(x_107, 1, x_106); +x_108 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4; +x_109 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_109, 0, x_107); +lean_ctor_set(x_109, 1, x_108); +x_110 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_81); +x_111 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_112 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +x_113 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(x_17, x_112, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_71); +x_114 = lean_ctor_get(x_113, 1); +lean_inc(x_114); +lean_dec(x_113); +x_115 = lean_box(0); +x_2 = x_115; +x_3 = x_16; +x_12 = x_114; +goto _start; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_nat_dec_lt(x_4, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_4); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_15); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_3, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_3, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_3, 2); +lean_inc(x_21); +x_22 = lean_nat_dec_lt(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_4); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_15); +return x_23; +} +else +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_3); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_25 = lean_ctor_get(x_3, 2); +lean_dec(x_25); +x_26 = lean_ctor_get(x_3, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_3, 0); +lean_dec(x_27); +x_28 = lean_array_fget(x_19, x_20); +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_add(x_20, x_29); +lean_dec(x_20); +lean_ctor_set(x_3, 1, x_30); +x_31 = lean_box(0); +lean_inc(x_4); +x_32 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2(x_4, x_31, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_ctor_get(x_2, 2); +x_35 = lean_nat_add(x_4, x_34); +lean_dec(x_4); +x_4 = x_35; +x_5 = lean_box(0); +x_6 = lean_box(0); +x_15 = x_33; +goto _start; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_dec(x_3); +x_37 = lean_array_fget(x_19, x_20); +x_38 = lean_unsigned_to_nat(1u); +x_39 = lean_nat_add(x_20, x_38); +lean_dec(x_20); +x_40 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_40, 0, x_19); +lean_ctor_set(x_40, 1, x_39); +lean_ctor_set(x_40, 2, x_21); +x_41 = lean_box(0); +lean_inc(x_4); +x_42 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2(x_4, x_41, x_37, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +x_44 = lean_ctor_get(x_2, 2); +x_45 = lean_nat_add(x_4, x_44); +lean_dec(x_4); +x_3 = x_40; +x_4 = x_45; +x_5 = lean_box(0); +x_6 = lean_box(0); +x_15 = x_43; +goto _start; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_traceDists(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_10 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_11, 5); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_PersistentArray_toArray___rarg(x_13); +x_15 = lean_array_get_size(x_14); +x_16 = lean_unsigned_to_nat(0u); +x_17 = l_Array_toSubarray___rarg(x_14, x_16, x_15); +x_18 = lean_ctor_get(x_13, 2); +lean_inc(x_18); +lean_dec(x_13); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_18); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3(x_20, x_20, x_17, x_16, lean_box(0), lean_box(0), x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +lean_dec(x_20); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +x_24 = lean_box(0); +lean_ctor_set(x_21, 0, x_24); +return x_21; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_dec(x_21); +x_26 = lean_box(0); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; +} +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; +x_16 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_traceDists___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_Arith_Offset_traceDists(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; lean_object* x_71; +x_64 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_64, 1); +lean_inc(x_66); +lean_dec(x_64); +x_67 = lean_ctor_get(x_65, 0); +lean_inc(x_67); +lean_dec(x_65); +x_68 = lean_ctor_get(x_1, 0); +x_69 = lean_ctor_get(x_67, 2); +lean_inc(x_69); +x_70 = lean_nat_dec_lt(x_68, x_69); +lean_dec(x_69); +x_71 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_66); +if (x_70 == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_dec(x_67); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = l_Lean_instInhabitedExpr; +x_75 = l_outOfBounds___rarg(x_74); +x_11 = x_75; +x_12 = x_72; +x_13 = x_73; +goto block_63; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_71, 1); +lean_inc(x_77); +lean_dec(x_71); +x_78 = l_Lean_instInhabitedExpr; +x_79 = l_Lean_PersistentArray_get_x21___rarg(x_78, x_67, x_68); +x_11 = x_79; +x_12 = x_76; +x_13 = x_77; +goto block_63; +} +block_63: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_14 = lean_ctor_get(x_12, 0); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_ctor_get(x_1, 1); +x_16 = lean_ctor_get(x_14, 2); +lean_inc(x_16); +x_17 = lean_nat_dec_lt(x_15, x_16); +lean_dec(x_16); +x_18 = lean_ctor_get(x_1, 2); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_20 = lean_int_dec_eq(x_18, x_19); +if (x_17 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_dec(x_14); +x_21 = l_Lean_instInhabitedExpr; +x_22 = l_outOfBounds___rarg(x_21); +if (x_20 == 0) +{ +uint8_t x_23; +x_23 = lean_int_dec_lt(x_18, x_19); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = l_Int_toNat(x_18); +x_25 = l_Lean_mkNatLit(x_24); +x_26 = l___private_Lean_Expr_0__Lean_natAddFn; +x_27 = l_Lean_mkAppB(x_26, x_22, x_25); +x_28 = l___private_Lean_Expr_0__Lean_natLEPred; +x_29 = l_Lean_mkAppB(x_28, x_11, x_27); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_13); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_31 = lean_int_neg(x_18); +x_32 = l_Int_toNat(x_31); +lean_dec(x_31); +x_33 = l_Lean_mkNatLit(x_32); +x_34 = l___private_Lean_Expr_0__Lean_natAddFn; +x_35 = l_Lean_mkAppB(x_34, x_11, x_33); +x_36 = l___private_Lean_Expr_0__Lean_natLEPred; +x_37 = l_Lean_mkAppB(x_36, x_35, x_22); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_13); +return x_38; +} +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = l___private_Lean_Expr_0__Lean_natLEPred; +x_40 = l_Lean_mkAppB(x_39, x_11, x_22); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_13); +return x_41; +} +} +else +{ +lean_object* x_42; lean_object* x_43; +x_42 = l_Lean_instInhabitedExpr; +x_43 = l_Lean_PersistentArray_get_x21___rarg(x_42, x_14, x_15); +if (x_20 == 0) +{ +uint8_t x_44; +x_44 = lean_int_dec_lt(x_18, x_19); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_45 = l_Int_toNat(x_18); +x_46 = l_Lean_mkNatLit(x_45); +x_47 = l___private_Lean_Expr_0__Lean_natAddFn; +x_48 = l_Lean_mkAppB(x_47, x_43, x_46); +x_49 = l___private_Lean_Expr_0__Lean_natLEPred; +x_50 = l_Lean_mkAppB(x_49, x_11, x_48); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_13); +return x_51; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_52 = lean_int_neg(x_18); +x_53 = l_Int_toNat(x_52); +lean_dec(x_52); +x_54 = l_Lean_mkNatLit(x_53); +x_55 = l___private_Lean_Expr_0__Lean_natAddFn; +x_56 = l_Lean_mkAppB(x_55, x_11, x_54); +x_57 = l___private_Lean_Expr_0__Lean_natLEPred; +x_58 = l_Lean_mkAppB(x_57, x_56, x_43); +x_59 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_13); +return x_59; +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = l___private_Lean_Expr_0__Lean_natLEPred; +x_61 = l_Lean_mkAppB(x_60, x_11, x_43); +x_62 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_13); +return x_62; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5; +x_12 = lean_panic_fn(x_11, x_1); +x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +x_10 = l___private_Init_Data_Repr_0__Nat_reprFast(x_9); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Lean_MessageData_ofFormat(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +lean_inc(x_1); +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_1); +x_16 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = lean_ctor_get(x_2, 1); +lean_inc(x_20); +lean_dec(x_2); +x_21 = l___private_Init_Data_Repr_0__Nat_reprFast(x_20); +x_22 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_22, 0, x_21); +x_23 = l_Lean_MessageData_ofFormat(x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_13); +lean_ctor_set(x_24, 1, x_23); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_1); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_19); +lean_ctor_set(x_26, 1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +x_29 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_30 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_30, 0, x_29); +x_31 = l_Lean_MessageData_ofFormat(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_28); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_16); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_dec(x_6); +x_34 = lean_ctor_get(x_2, 0); +lean_inc(x_34); +x_35 = l___private_Init_Data_Repr_0__Nat_reprFast(x_34); +x_36 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_36, 0, x_35); +x_37 = l_Lean_MessageData_ofFormat(x_36); +x_38 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +lean_inc(x_1); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_40); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_ctor_get(x_2, 1); +lean_inc(x_45); +lean_dec(x_2); +x_46 = l___private_Init_Data_Repr_0__Nat_reprFast(x_45); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l_Lean_MessageData_ofFormat(x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_38); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_1); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_44); +lean_ctor_set(x_51, 1, x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_41); +return x_52; +} +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_53 = lean_nat_abs(x_3); +lean_dec(x_3); +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_53, x_54); +lean_dec(x_53); +x_56 = lean_ctor_get(x_2, 0); +lean_inc(x_56); +x_57 = l___private_Init_Data_Repr_0__Nat_reprFast(x_56); +x_58 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_58, 0, x_57); +x_59 = l_Lean_MessageData_ofFormat(x_58); +x_60 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2; +x_61 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_59); +lean_inc(x_1); +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_61); +lean_ctor_set(x_62, 1, x_1); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_64 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_64, 0, x_63); +lean_ctor_set(x_64, 1, x_62); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_nat_add(x_55, x_54); +lean_dec(x_55); +x_68 = l___private_Init_Data_Repr_0__Nat_reprFast(x_67); +x_69 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_69, 0, x_68); +x_70 = l_Lean_MessageData_ofFormat(x_69); +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_66); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4; +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_ctor_get(x_2, 1); +lean_inc(x_74); +lean_dec(x_2); +x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_77 = l_Lean_MessageData_ofFormat(x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_60); +lean_ctor_set(x_78, 1, x_77); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_1); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_73); +lean_ctor_set(x_80, 1, x_79); +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_63); +return x_81; +} +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.checkInvariants", 44, 44); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5; +x_2 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1; +x_3 = lean_unsigned_to_nat(333u); +x_4 = lean_unsigned_to_nat(8u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2; +x_12 = l_panic___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__1(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_12, 0); +lean_dec(x_14); +x_15 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +lean_ctor_set(x_12, 0, x_15); +return x_12; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_12, 1); +lean_inc(x_16); +lean_dec(x_12); +x_17 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) +{ +return x_12; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_12, 0); +x_21 = lean_ctor_get(x_12, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_12); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +static uint64_t _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1() { +_start: +{ +uint8_t x_1; uint64_t x_2; +x_1 = 1; +x_2 = l_Lean_Meta_TransparencyMode_toUInt64(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("failed: ", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" =\?= ", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_1); +x_14 = l_Lean_Meta_check(x_1, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_1); +x_16 = lean_infer_type(x_1, x_9, x_10, x_11, x_12, x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +x_20 = lean_ctor_get(x_9, 0); +lean_inc(x_20); +x_21 = !lean_is_exclusive(x_19); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; uint64_t x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_22 = lean_ctor_get(x_19, 0); +x_23 = lean_ctor_get(x_19, 1); +x_24 = lean_ctor_get_uint64(x_9, sizeof(void*)*7); +x_25 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 8); +x_26 = lean_ctor_get(x_9, 1); +lean_inc(x_26); +x_27 = lean_ctor_get(x_9, 2); +lean_inc(x_27); +x_28 = lean_ctor_get(x_9, 3); +lean_inc(x_28); +x_29 = lean_ctor_get(x_9, 4); +lean_inc(x_29); +x_30 = lean_ctor_get(x_9, 5); +lean_inc(x_30); +x_31 = lean_ctor_get(x_9, 6); +lean_inc(x_31); +x_32 = !lean_is_exclusive(x_20); +if (x_32 == 0) +{ +uint8_t x_33; uint8_t x_34; uint8_t x_35; uint64_t x_36; uint64_t x_37; uint64_t x_38; uint64_t x_39; uint64_t x_40; lean_object* x_41; lean_object* x_42; +x_33 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 9); +x_34 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 10); +x_35 = 1; +lean_ctor_set_uint8(x_20, 9, x_35); +x_36 = 2; +x_37 = lean_uint64_shift_right(x_24, x_36); +x_38 = lean_uint64_shift_left(x_37, x_36); +x_39 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1; +x_40 = lean_uint64_lor(x_38, x_39); +x_41 = lean_alloc_ctor(0, 7, 11); +lean_ctor_set(x_41, 0, x_20); +lean_ctor_set(x_41, 1, x_26); +lean_ctor_set(x_41, 2, x_27); +lean_ctor_set(x_41, 3, x_28); +lean_ctor_set(x_41, 4, x_29); +lean_ctor_set(x_41, 5, x_30); +lean_ctor_set(x_41, 6, x_31); +lean_ctor_set_uint64(x_41, sizeof(void*)*7, x_40); +lean_ctor_set_uint8(x_41, sizeof(void*)*7 + 8, x_25); +lean_ctor_set_uint8(x_41, sizeof(void*)*7 + 9, x_33); +lean_ctor_set_uint8(x_41, sizeof(void*)*7 + 10, x_34); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_42 = l_Lean_Meta_isExprDefEq(x_17, x_22, x_41, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; uint8_t x_44; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_unbox(x_43); +lean_dec(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_42, 1); +lean_inc(x_45); +lean_dec(x_42); +lean_inc(x_3); +x_46 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_45); +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_ctor_get(x_46, 1); +x_50 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2; +x_51 = lean_unbox(x_48); +lean_dec(x_48); +if (x_51 == 0) +{ +lean_object* x_52; lean_object* x_53; +lean_free_object(x_46); +lean_free_object(x_19); +lean_dec(x_3); +lean_dec(x_1); +x_52 = lean_box(0); +x_53 = lean_apply_10(x_50, x_52, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_49); +return x_53; +} +else +{ +lean_object* x_54; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_54 = lean_infer_type(x_1, x_9, x_10, x_11, x_12, x_49); +if (lean_obj_tag(x_54) == 0) +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +x_57 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_56); +x_58 = !lean_is_exclusive(x_57); +if (x_58 == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_59 = lean_ctor_get(x_57, 0); +x_60 = lean_ctor_get(x_57, 1); +x_61 = l_Lean_MessageData_ofExpr(x_55); +x_62 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +lean_ctor_set_tag(x_57, 7); +lean_ctor_set(x_57, 1, x_61); +lean_ctor_set(x_57, 0, x_62); +x_63 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +lean_ctor_set_tag(x_46, 7); +lean_ctor_set(x_46, 1, x_63); +lean_ctor_set(x_46, 0, x_57); +x_64 = l_Lean_MessageData_ofExpr(x_59); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_64); +lean_ctor_set(x_19, 0, x_46); +x_65 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_19); +lean_ctor_set(x_66, 1, x_65); +x_67 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_3, x_66, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_60); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_apply_10(x_50, x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_69); +return x_70; +} +else +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_71 = lean_ctor_get(x_57, 0); +x_72 = lean_ctor_get(x_57, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_57); +x_73 = l_Lean_MessageData_ofExpr(x_55); +x_74 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +x_75 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_73); +x_76 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +lean_ctor_set_tag(x_46, 7); +lean_ctor_set(x_46, 1, x_76); +lean_ctor_set(x_46, 0, x_75); +x_77 = l_Lean_MessageData_ofExpr(x_71); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_77); +lean_ctor_set(x_19, 0, x_46); +x_78 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_19); +lean_ctor_set(x_79, 1, x_78); +x_80 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_3, x_79, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_72); +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +x_83 = lean_apply_10(x_50, x_81, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_82); +return x_83; +} +} +else +{ +uint8_t x_84; +lean_free_object(x_46); +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_84 = !lean_is_exclusive(x_54); +if (x_84 == 0) +{ +return x_54; +} +else +{ +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_54, 0); +x_86 = lean_ctor_get(x_54, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_54); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; +} +} +} +} +else +{ +lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_88 = lean_ctor_get(x_46, 0); +x_89 = lean_ctor_get(x_46, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_46); +x_90 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2; +x_91 = lean_unbox(x_88); +lean_dec(x_88); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; +lean_free_object(x_19); +lean_dec(x_3); +lean_dec(x_1); +x_92 = lean_box(0); +x_93 = lean_apply_10(x_90, x_92, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_89); +return x_93; +} +else +{ +lean_object* x_94; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_94 = lean_infer_type(x_1, x_9, x_10, x_11, x_12, x_89); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_96); +x_98 = lean_ctor_get(x_97, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_97, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + x_100 = x_97; +} else { + lean_dec_ref(x_97); + x_100 = lean_box(0); +} +x_101 = l_Lean_MessageData_ofExpr(x_95); +x_102 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +if (lean_is_scalar(x_100)) { + x_103 = lean_alloc_ctor(7, 2, 0); +} else { + x_103 = x_100; + lean_ctor_set_tag(x_103, 7); +} +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_101); +x_104 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +x_105 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +x_106 = l_Lean_MessageData_ofExpr(x_98); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_106); +lean_ctor_set(x_19, 0, x_105); +x_107 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_108 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_108, 0, x_19); +lean_ctor_set(x_108, 1, x_107); +x_109 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_3, x_108, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_99); +x_110 = lean_ctor_get(x_109, 0); +lean_inc(x_110); +x_111 = lean_ctor_get(x_109, 1); +lean_inc(x_111); +lean_dec(x_109); +x_112 = lean_apply_10(x_90, x_110, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_111); +return x_112; +} +else +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_113 = lean_ctor_get(x_94, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_94, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_115 = x_94; +} else { + lean_dec_ref(x_94); + x_115 = lean_box(0); +} +if (lean_is_scalar(x_115)) { + x_116 = lean_alloc_ctor(1, 2, 0); +} else { + x_116 = x_115; +} +lean_ctor_set(x_116, 0, x_113); +lean_ctor_set(x_116, 1, x_114); +return x_116; +} +} +} +} +else +{ +uint8_t x_117; +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_117 = !lean_is_exclusive(x_42); +if (x_117 == 0) +{ +lean_object* x_118; lean_object* x_119; +x_118 = lean_ctor_get(x_42, 0); +lean_dec(x_118); +x_119 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +lean_ctor_set(x_42, 0, x_119); +return x_42; +} +else +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_ctor_get(x_42, 1); +lean_inc(x_120); +lean_dec(x_42); +x_121 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +x_122 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_122, 0, x_121); +lean_ctor_set(x_122, 1, x_120); +return x_122; +} +} +} +else +{ +uint8_t x_123; +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_123 = !lean_is_exclusive(x_42); +if (x_123 == 0) +{ +return x_42; +} +else +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_124 = lean_ctor_get(x_42, 0); +x_125 = lean_ctor_get(x_42, 1); +lean_inc(x_125); +lean_inc(x_124); +lean_dec(x_42); +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; +} +} +} +else +{ +uint8_t x_127; uint8_t x_128; uint8_t x_129; uint8_t x_130; uint8_t x_131; uint8_t x_132; uint8_t x_133; uint8_t x_134; uint8_t x_135; uint8_t x_136; uint8_t x_137; uint8_t x_138; uint8_t x_139; uint8_t x_140; uint8_t x_141; uint8_t x_142; uint8_t x_143; uint8_t x_144; uint8_t x_145; lean_object* x_146; uint64_t x_147; uint64_t x_148; uint64_t x_149; uint64_t x_150; uint64_t x_151; lean_object* x_152; lean_object* x_153; +x_127 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 9); +x_128 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 10); +x_129 = lean_ctor_get_uint8(x_20, 0); +x_130 = lean_ctor_get_uint8(x_20, 1); +x_131 = lean_ctor_get_uint8(x_20, 2); +x_132 = lean_ctor_get_uint8(x_20, 3); +x_133 = lean_ctor_get_uint8(x_20, 4); +x_134 = lean_ctor_get_uint8(x_20, 5); +x_135 = lean_ctor_get_uint8(x_20, 6); +x_136 = lean_ctor_get_uint8(x_20, 7); +x_137 = lean_ctor_get_uint8(x_20, 8); +x_138 = lean_ctor_get_uint8(x_20, 10); +x_139 = lean_ctor_get_uint8(x_20, 11); +x_140 = lean_ctor_get_uint8(x_20, 12); +x_141 = lean_ctor_get_uint8(x_20, 13); +x_142 = lean_ctor_get_uint8(x_20, 14); +x_143 = lean_ctor_get_uint8(x_20, 15); +x_144 = lean_ctor_get_uint8(x_20, 16); +lean_dec(x_20); +x_145 = 1; +x_146 = lean_alloc_ctor(0, 0, 17); +lean_ctor_set_uint8(x_146, 0, x_129); +lean_ctor_set_uint8(x_146, 1, x_130); +lean_ctor_set_uint8(x_146, 2, x_131); +lean_ctor_set_uint8(x_146, 3, x_132); +lean_ctor_set_uint8(x_146, 4, x_133); +lean_ctor_set_uint8(x_146, 5, x_134); +lean_ctor_set_uint8(x_146, 6, x_135); +lean_ctor_set_uint8(x_146, 7, x_136); +lean_ctor_set_uint8(x_146, 8, x_137); +lean_ctor_set_uint8(x_146, 9, x_145); +lean_ctor_set_uint8(x_146, 10, x_138); +lean_ctor_set_uint8(x_146, 11, x_139); +lean_ctor_set_uint8(x_146, 12, x_140); +lean_ctor_set_uint8(x_146, 13, x_141); +lean_ctor_set_uint8(x_146, 14, x_142); +lean_ctor_set_uint8(x_146, 15, x_143); +lean_ctor_set_uint8(x_146, 16, x_144); +x_147 = 2; +x_148 = lean_uint64_shift_right(x_24, x_147); +x_149 = lean_uint64_shift_left(x_148, x_147); +x_150 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1; +x_151 = lean_uint64_lor(x_149, x_150); +x_152 = lean_alloc_ctor(0, 7, 11); +lean_ctor_set(x_152, 0, x_146); +lean_ctor_set(x_152, 1, x_26); +lean_ctor_set(x_152, 2, x_27); +lean_ctor_set(x_152, 3, x_28); +lean_ctor_set(x_152, 4, x_29); +lean_ctor_set(x_152, 5, x_30); +lean_ctor_set(x_152, 6, x_31); +lean_ctor_set_uint64(x_152, sizeof(void*)*7, x_151); +lean_ctor_set_uint8(x_152, sizeof(void*)*7 + 8, x_25); +lean_ctor_set_uint8(x_152, sizeof(void*)*7 + 9, x_127); +lean_ctor_set_uint8(x_152, sizeof(void*)*7 + 10, x_128); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_153 = l_Lean_Meta_isExprDefEq(x_17, x_22, x_152, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_153) == 0) +{ +lean_object* x_154; uint8_t x_155; +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +x_155 = lean_unbox(x_154); +lean_dec(x_154); +if (x_155 == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_156 = lean_ctor_get(x_153, 1); +lean_inc(x_156); +lean_dec(x_153); +lean_inc(x_3); +x_157 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_156); +x_158 = lean_ctor_get(x_157, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_157, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_160 = x_157; +} else { + lean_dec_ref(x_157); + x_160 = lean_box(0); +} +x_161 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2; +x_162 = lean_unbox(x_158); +lean_dec(x_158); +if (x_162 == 0) +{ +lean_object* x_163; lean_object* x_164; +lean_dec(x_160); +lean_free_object(x_19); +lean_dec(x_3); +lean_dec(x_1); +x_163 = lean_box(0); +x_164 = lean_apply_10(x_161, x_163, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_159); +return x_164; +} +else +{ +lean_object* x_165; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_165 = lean_infer_type(x_1, x_9, x_10, x_11, x_12, x_159); +if (lean_obj_tag(x_165) == 0) +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +x_166 = lean_ctor_get(x_165, 0); +lean_inc(x_166); +x_167 = lean_ctor_get(x_165, 1); +lean_inc(x_167); +lean_dec(x_165); +x_168 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_167); +x_169 = lean_ctor_get(x_168, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_171 = x_168; +} else { + lean_dec_ref(x_168); + x_171 = lean_box(0); +} +x_172 = l_Lean_MessageData_ofExpr(x_166); +x_173 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +if (lean_is_scalar(x_171)) { + x_174 = lean_alloc_ctor(7, 2, 0); +} else { + x_174 = x_171; + lean_ctor_set_tag(x_174, 7); +} +lean_ctor_set(x_174, 0, x_173); +lean_ctor_set(x_174, 1, x_172); +x_175 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +if (lean_is_scalar(x_160)) { + x_176 = lean_alloc_ctor(7, 2, 0); +} else { + x_176 = x_160; + lean_ctor_set_tag(x_176, 7); +} +lean_ctor_set(x_176, 0, x_174); +lean_ctor_set(x_176, 1, x_175); +x_177 = l_Lean_MessageData_ofExpr(x_169); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_177); +lean_ctor_set(x_19, 0, x_176); +x_178 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_179 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_179, 0, x_19); +lean_ctor_set(x_179, 1, x_178); +x_180 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_3, x_179, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_170); +x_181 = lean_ctor_get(x_180, 0); +lean_inc(x_181); +x_182 = lean_ctor_get(x_180, 1); +lean_inc(x_182); +lean_dec(x_180); +x_183 = lean_apply_10(x_161, x_181, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_182); +return x_183; +} +else +{ +lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +lean_dec(x_160); +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_184 = lean_ctor_get(x_165, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_165, 1); +lean_inc(x_185); +if (lean_is_exclusive(x_165)) { + lean_ctor_release(x_165, 0); + lean_ctor_release(x_165, 1); + x_186 = x_165; +} else { + lean_dec_ref(x_165); + x_186 = lean_box(0); +} +if (lean_is_scalar(x_186)) { + x_187 = lean_alloc_ctor(1, 2, 0); +} else { + x_187 = x_186; +} +lean_ctor_set(x_187, 0, x_184); +lean_ctor_set(x_187, 1, x_185); +return x_187; +} +} +} +else +{ +lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_188 = lean_ctor_get(x_153, 1); +lean_inc(x_188); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + lean_ctor_release(x_153, 1); + x_189 = x_153; +} else { + lean_dec_ref(x_153); + x_189 = lean_box(0); +} +x_190 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +if (lean_is_scalar(x_189)) { + x_191 = lean_alloc_ctor(0, 2, 0); +} else { + x_191 = x_189; +} +lean_ctor_set(x_191, 0, x_190); +lean_ctor_set(x_191, 1, x_188); +return x_191; +} +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +lean_free_object(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_192 = lean_ctor_get(x_153, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_153, 1); +lean_inc(x_193); +if (lean_is_exclusive(x_153)) { + lean_ctor_release(x_153, 0); + lean_ctor_release(x_153, 1); + x_194 = x_153; +} else { + lean_dec_ref(x_153); + x_194 = lean_box(0); +} +if (lean_is_scalar(x_194)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_194; +} +lean_ctor_set(x_195, 0, x_192); +lean_ctor_set(x_195, 1, x_193); +return x_195; +} +} +} +else +{ +lean_object* x_196; lean_object* x_197; uint64_t x_198; uint8_t x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; uint8_t x_207; uint8_t x_208; uint8_t x_209; uint8_t x_210; uint8_t x_211; uint8_t x_212; uint8_t x_213; uint8_t x_214; uint8_t x_215; uint8_t x_216; uint8_t x_217; uint8_t x_218; uint8_t x_219; uint8_t x_220; uint8_t x_221; uint8_t x_222; uint8_t x_223; lean_object* x_224; uint8_t x_225; lean_object* x_226; uint64_t x_227; uint64_t x_228; uint64_t x_229; uint64_t x_230; uint64_t x_231; lean_object* x_232; lean_object* x_233; +x_196 = lean_ctor_get(x_19, 0); +x_197 = lean_ctor_get(x_19, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_19); +x_198 = lean_ctor_get_uint64(x_9, sizeof(void*)*7); +x_199 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 8); +x_200 = lean_ctor_get(x_9, 1); +lean_inc(x_200); +x_201 = lean_ctor_get(x_9, 2); +lean_inc(x_201); +x_202 = lean_ctor_get(x_9, 3); +lean_inc(x_202); +x_203 = lean_ctor_get(x_9, 4); +lean_inc(x_203); +x_204 = lean_ctor_get(x_9, 5); +lean_inc(x_204); +x_205 = lean_ctor_get(x_9, 6); +lean_inc(x_205); +x_206 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 9); +x_207 = lean_ctor_get_uint8(x_9, sizeof(void*)*7 + 10); +x_208 = lean_ctor_get_uint8(x_20, 0); +x_209 = lean_ctor_get_uint8(x_20, 1); +x_210 = lean_ctor_get_uint8(x_20, 2); +x_211 = lean_ctor_get_uint8(x_20, 3); +x_212 = lean_ctor_get_uint8(x_20, 4); +x_213 = lean_ctor_get_uint8(x_20, 5); +x_214 = lean_ctor_get_uint8(x_20, 6); +x_215 = lean_ctor_get_uint8(x_20, 7); +x_216 = lean_ctor_get_uint8(x_20, 8); +x_217 = lean_ctor_get_uint8(x_20, 10); +x_218 = lean_ctor_get_uint8(x_20, 11); +x_219 = lean_ctor_get_uint8(x_20, 12); +x_220 = lean_ctor_get_uint8(x_20, 13); +x_221 = lean_ctor_get_uint8(x_20, 14); +x_222 = lean_ctor_get_uint8(x_20, 15); +x_223 = lean_ctor_get_uint8(x_20, 16); +if (lean_is_exclusive(x_20)) { + x_224 = x_20; +} else { + lean_dec_ref(x_20); + x_224 = lean_box(0); +} +x_225 = 1; +if (lean_is_scalar(x_224)) { + x_226 = lean_alloc_ctor(0, 0, 17); +} else { + x_226 = x_224; +} +lean_ctor_set_uint8(x_226, 0, x_208); +lean_ctor_set_uint8(x_226, 1, x_209); +lean_ctor_set_uint8(x_226, 2, x_210); +lean_ctor_set_uint8(x_226, 3, x_211); +lean_ctor_set_uint8(x_226, 4, x_212); +lean_ctor_set_uint8(x_226, 5, x_213); +lean_ctor_set_uint8(x_226, 6, x_214); +lean_ctor_set_uint8(x_226, 7, x_215); +lean_ctor_set_uint8(x_226, 8, x_216); +lean_ctor_set_uint8(x_226, 9, x_225); +lean_ctor_set_uint8(x_226, 10, x_217); +lean_ctor_set_uint8(x_226, 11, x_218); +lean_ctor_set_uint8(x_226, 12, x_219); +lean_ctor_set_uint8(x_226, 13, x_220); +lean_ctor_set_uint8(x_226, 14, x_221); +lean_ctor_set_uint8(x_226, 15, x_222); +lean_ctor_set_uint8(x_226, 16, x_223); +x_227 = 2; +x_228 = lean_uint64_shift_right(x_198, x_227); +x_229 = lean_uint64_shift_left(x_228, x_227); +x_230 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1; +x_231 = lean_uint64_lor(x_229, x_230); +x_232 = lean_alloc_ctor(0, 7, 11); +lean_ctor_set(x_232, 0, x_226); +lean_ctor_set(x_232, 1, x_200); +lean_ctor_set(x_232, 2, x_201); +lean_ctor_set(x_232, 3, x_202); +lean_ctor_set(x_232, 4, x_203); +lean_ctor_set(x_232, 5, x_204); +lean_ctor_set(x_232, 6, x_205); +lean_ctor_set_uint64(x_232, sizeof(void*)*7, x_231); +lean_ctor_set_uint8(x_232, sizeof(void*)*7 + 8, x_199); +lean_ctor_set_uint8(x_232, sizeof(void*)*7 + 9, x_206); +lean_ctor_set_uint8(x_232, sizeof(void*)*7 + 10, x_207); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_233 = l_Lean_Meta_isExprDefEq(x_17, x_196, x_232, x_10, x_11, x_12, x_197); +if (lean_obj_tag(x_233) == 0) +{ +lean_object* x_234; uint8_t x_235; +x_234 = lean_ctor_get(x_233, 0); +lean_inc(x_234); +x_235 = lean_unbox(x_234); +lean_dec(x_234); +if (x_235 == 0) +{ +lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; uint8_t x_242; +x_236 = lean_ctor_get(x_233, 1); +lean_inc(x_236); +lean_dec(x_233); +lean_inc(x_3); +x_237 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_236); +x_238 = lean_ctor_get(x_237, 0); +lean_inc(x_238); +x_239 = lean_ctor_get(x_237, 1); +lean_inc(x_239); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + x_240 = x_237; +} else { + lean_dec_ref(x_237); + x_240 = lean_box(0); +} +x_241 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2; +x_242 = lean_unbox(x_238); +lean_dec(x_238); +if (x_242 == 0) +{ +lean_object* x_243; lean_object* x_244; +lean_dec(x_240); +lean_dec(x_3); +lean_dec(x_1); +x_243 = lean_box(0); +x_244 = lean_apply_10(x_241, x_243, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_239); +return x_244; +} +else +{ +lean_object* x_245; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_245 = lean_infer_type(x_1, x_9, x_10, x_11, x_12, x_239); +if (lean_obj_tag(x_245) == 0) +{ +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_246 = lean_ctor_get(x_245, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_245, 1); +lean_inc(x_247); +lean_dec(x_245); +x_248 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_toExpr(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_247); +x_249 = lean_ctor_get(x_248, 0); +lean_inc(x_249); +x_250 = lean_ctor_get(x_248, 1); +lean_inc(x_250); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_251 = x_248; +} else { + lean_dec_ref(x_248); + x_251 = lean_box(0); +} +x_252 = l_Lean_MessageData_ofExpr(x_246); +x_253 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4; +if (lean_is_scalar(x_251)) { + x_254 = lean_alloc_ctor(7, 2, 0); +} else { + x_254 = x_251; + lean_ctor_set_tag(x_254, 7); +} +lean_ctor_set(x_254, 0, x_253); +lean_ctor_set(x_254, 1, x_252); +x_255 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6; +if (lean_is_scalar(x_240)) { + x_256 = lean_alloc_ctor(7, 2, 0); +} else { + x_256 = x_240; + lean_ctor_set_tag(x_256, 7); +} +lean_ctor_set(x_256, 0, x_254); +lean_ctor_set(x_256, 1, x_255); +x_257 = l_Lean_MessageData_ofExpr(x_249); +x_258 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_258, 0, x_256); +lean_ctor_set(x_258, 1, x_257); +x_259 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_260 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_260, 0, x_258); +lean_ctor_set(x_260, 1, x_259); +x_261 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_3, x_260, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_250); +x_262 = lean_ctor_get(x_261, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_261, 1); +lean_inc(x_263); +lean_dec(x_261); +x_264 = lean_apply_10(x_241, x_262, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_263); +return x_264; +} +else +{ +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_240); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_265 = lean_ctor_get(x_245, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_245, 1); +lean_inc(x_266); +if (lean_is_exclusive(x_245)) { + lean_ctor_release(x_245, 0); + lean_ctor_release(x_245, 1); + x_267 = x_245; +} else { + lean_dec_ref(x_245); + x_267 = lean_box(0); +} +if (lean_is_scalar(x_267)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_267; +} +lean_ctor_set(x_268, 0, x_265); +lean_ctor_set(x_268, 1, x_266); +return x_268; +} +} +} +else +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_269 = lean_ctor_get(x_233, 1); +lean_inc(x_269); +if (lean_is_exclusive(x_233)) { + lean_ctor_release(x_233, 0); + lean_ctor_release(x_233, 1); + x_270 = x_233; +} else { + lean_dec_ref(x_233); + x_270 = lean_box(0); +} +x_271 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3; +if (lean_is_scalar(x_270)) { + x_272 = lean_alloc_ctor(0, 2, 0); +} else { + x_272 = x_270; +} +lean_ctor_set(x_272, 0, x_271); +lean_ctor_set(x_272, 1, x_269); +return x_272; +} +} +else +{ +lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_273 = lean_ctor_get(x_233, 0); +lean_inc(x_273); +x_274 = lean_ctor_get(x_233, 1); +lean_inc(x_274); +if (lean_is_exclusive(x_233)) { + lean_ctor_release(x_233, 0); + lean_ctor_release(x_233, 1); + x_275 = x_233; +} else { + lean_dec_ref(x_233); + x_275 = lean_box(0); +} +if (lean_is_scalar(x_275)) { + x_276 = lean_alloc_ctor(1, 2, 0); +} else { + x_276 = x_275; +} +lean_ctor_set(x_276, 0, x_273); +lean_ctor_set(x_276, 1, x_274); +return x_276; +} +} +} +else +{ +uint8_t x_277; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_277 = !lean_is_exclusive(x_16); +if (x_277 == 0) +{ +return x_16; +} +else +{ +lean_object* x_278; lean_object* x_279; lean_object* x_280; +x_278 = lean_ctor_get(x_16, 0); +x_279 = lean_ctor_get(x_16, 1); +lean_inc(x_279); +lean_inc(x_278); +lean_dec(x_16); +x_280 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_280, 0, x_278); +lean_ctor_set(x_280, 1, x_279); +return x_280; +} +} +} +else +{ +uint8_t x_281; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_281 = !lean_is_exclusive(x_14); +if (x_281 == 0) +{ +return x_14; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; +x_282 = lean_ctor_get(x_14, 0); +x_283 = lean_ctor_get(x_14, 1); +lean_inc(x_283); +lean_inc(x_282); +lean_dec(x_14); +x_284 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_284, 0, x_282); +lean_ctor_set(x_284, 1, x_283); +return x_284; +} +} +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("debug", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("proof", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_4 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" : ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; uint8_t x_15; +x_14 = l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +x_18 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3; +x_19 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_free_object(x_14); +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_box(0); +x_24 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_16, x_3, x_18, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +return x_24; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_19, 1); +x_27 = lean_ctor_get(x_19, 0); +lean_dec(x_27); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_16); +x_28 = lean_infer_type(x_16, x_9, x_10, x_11, x_12, x_26); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +lean_inc(x_16); +x_31 = l_Lean_MessageData_ofExpr(x_16); +x_32 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_31); +lean_ctor_set(x_19, 0, x_32); +x_33 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5; +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_33); +lean_ctor_set(x_14, 0, x_19); +x_34 = l_Lean_MessageData_ofExpr(x_29); +x_35 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_35, 0, x_14); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_32); +x_37 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_30); +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_16, x_3, x_18, x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); +lean_dec(x_38); +return x_40; +} +else +{ +uint8_t x_41; +lean_free_object(x_19); +lean_free_object(x_14); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_41 = !lean_is_exclusive(x_28); +if (x_41 == 0) +{ +return x_28; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_28, 0); +x_43 = lean_ctor_get(x_28, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_28); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +else +{ +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_19, 1); +lean_inc(x_45); +lean_dec(x_19); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_16); +x_46 = lean_infer_type(x_16, x_9, x_10, x_11, x_12, x_45); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +lean_inc(x_16); +x_49 = l_Lean_MessageData_ofExpr(x_16); +x_50 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_49); +x_52 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5; +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_52); +lean_ctor_set(x_14, 0, x_51); +x_53 = l_Lean_MessageData_ofExpr(x_47); +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_14); +lean_ctor_set(x_54, 1, x_53); +x_55 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_50); +x_56 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_48); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +x_59 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_16, x_3, x_18, x_57, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_58); +lean_dec(x_57); +return x_59; +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +lean_free_object(x_14); +lean_dec(x_16); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_60 = lean_ctor_get(x_46, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_46, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_62 = x_46; +} else { + lean_dec_ref(x_46); + x_62 = lean_box(0); +} +if (lean_is_scalar(x_62)) { + x_63 = lean_alloc_ctor(1, 2, 0); +} else { + x_63 = x_62; +} +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_61); +return x_63; +} +} +} +} +else +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; +x_64 = lean_ctor_get(x_14, 0); +x_65 = lean_ctor_get(x_14, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_14); +x_66 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3; +x_67 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_66, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_65); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_unbox(x_68); +lean_dec(x_68); +if (x_69 == 0) +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_67, 1); +lean_inc(x_70); +lean_dec(x_67); +x_71 = lean_box(0); +x_72 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_64, x_3, x_66, x_71, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_70); +return x_72; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_67, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + x_74 = x_67; +} else { + lean_dec_ref(x_67); + x_74 = lean_box(0); +} +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_64); +x_75 = lean_infer_type(x_64, x_9, x_10, x_11, x_12, x_73); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +lean_inc(x_64); +x_78 = l_Lean_MessageData_ofExpr(x_64); +x_79 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +if (lean_is_scalar(x_74)) { + x_80 = lean_alloc_ctor(7, 2, 0); +} else { + x_80 = x_74; + lean_ctor_set_tag(x_80, 7); +} +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_78); +x_81 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5; +x_82 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +x_83 = l_Lean_MessageData_ofExpr(x_76); +x_84 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_79); +x_86 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_66, x_85, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_77); +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_64, x_3, x_66, x_87, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_88); +lean_dec(x_87); +return x_89; +} +else +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_74); +lean_dec(x_64); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_90 = lean_ctor_get(x_75, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_75, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_92 = x_75; +} else { + lean_dec_ref(x_75); + x_92 = lean_box(0); +} +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); +} else { + x_93 = x_92; +} +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; +} +} +} +} +} +static lean_object* _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1; +x_2 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_13; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_2); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} +else +{ +uint8_t x_14; +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_3); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_15 = lean_ctor_get(x_3, 0); +x_16 = lean_ctor_get(x_3, 1); +x_17 = lean_ctor_get(x_3, 2); +lean_inc(x_15); +lean_inc(x_1); +lean_ctor_set_tag(x_3, 0); +lean_ctor_set(x_3, 2, x_16); +lean_ctor_set(x_3, 1, x_15); +lean_ctor_set(x_3, 0, x_1); +x_18 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1; +x_19 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_unbox(x_20); +lean_dec(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_19, 1); +lean_inc(x_22); +lean_dec(x_19); +x_23 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_24 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_15, x_3, x_23, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +lean_dec(x_3); +lean_dec(x_15); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +if (lean_obj_tag(x_25) == 0) +{ +uint8_t x_26; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_24); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_24, 0); +lean_dec(x_27); +x_28 = lean_ctor_get(x_25, 0); +lean_inc(x_28); +lean_dec(x_25); +lean_ctor_set(x_24, 0, x_28); +return x_24; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 1); +lean_inc(x_29); +lean_dec(x_24); +x_30 = lean_ctor_get(x_25, 0); +lean_inc(x_30); +lean_dec(x_25); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; +} +} +else +{ +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_24, 1); +lean_inc(x_32); +lean_dec(x_24); +x_33 = lean_ctor_get(x_25, 0); +lean_inc(x_33); +lean_dec(x_25); +x_2 = x_33; +x_3 = x_17; +x_12 = x_32; +goto _start; +} +} +else +{ +uint8_t x_35; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_24); +if (x_35 == 0) +{ +return x_24; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_24, 0); +x_37 = lean_ctor_get(x_24, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_24); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} +} +} +else +{ +uint8_t x_39; +x_39 = !lean_is_exclusive(x_19); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_40 = lean_ctor_get(x_19, 1); +x_41 = lean_ctor_get(x_19, 0); +lean_dec(x_41); +x_42 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_inc(x_3); +x_43 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__2(x_42, x_3); +lean_ctor_set_tag(x_19, 7); +lean_ctor_set(x_19, 1, x_43); +lean_ctor_set(x_19, 0, x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_19); +lean_ctor_set(x_44, 1, x_42); +x_45 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_44, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_40); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_48 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_15, x_3, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +lean_dec(x_46); +lean_dec(x_3); +lean_dec(x_15); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +if (lean_obj_tag(x_49) == 0) +{ +uint8_t x_50; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_48); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_ctor_get(x_49, 0); +lean_inc(x_52); +lean_dec(x_49); +lean_ctor_set(x_48, 0, x_52); +return x_48; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_48, 1); +lean_inc(x_53); +lean_dec(x_48); +x_54 = lean_ctor_get(x_49, 0); +lean_inc(x_54); +lean_dec(x_49); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_53); +return x_55; +} +} +else +{ +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +lean_dec(x_48); +x_57 = lean_ctor_get(x_49, 0); +lean_inc(x_57); +lean_dec(x_49); +x_2 = x_57; +x_3 = x_17; +x_12 = x_56; +goto _start; +} +} +else +{ +uint8_t x_59; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_59 = !lean_is_exclusive(x_48); +if (x_59 == 0) +{ +return x_48; +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_48, 0); +x_61 = lean_ctor_get(x_48, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_48); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; +} +} +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_63 = lean_ctor_get(x_19, 1); +lean_inc(x_63); +lean_dec(x_19); +x_64 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_inc(x_3); +x_65 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__2(x_64, x_3); +x_66 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +x_67 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_64); +x_68 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_18, x_67, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_63); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_71 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_15, x_3, x_69, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +lean_dec(x_69); +lean_dec(x_3); +lean_dec(x_15); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_74 = x_71; +} else { + lean_dec_ref(x_71); + x_74 = lean_box(0); +} +x_75 = lean_ctor_get(x_72, 0); +lean_inc(x_75); +lean_dec(x_72); +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 2, 0); +} else { + x_76 = x_74; +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_73); +return x_76; +} +else +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_71, 1); +lean_inc(x_77); +lean_dec(x_71); +x_78 = lean_ctor_get(x_72, 0); +lean_inc(x_78); +lean_dec(x_72); +x_2 = x_78; +x_3 = x_17; +x_12 = x_77; +goto _start; +} +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_17); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_80 = lean_ctor_get(x_71, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_71, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_82 = x_71; +} else { + lean_dec_ref(x_71); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; +} +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; +} +} +} +} +else +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; +x_84 = lean_ctor_get(x_3, 0); +x_85 = lean_ctor_get(x_3, 1); +x_86 = lean_ctor_get(x_3, 2); +lean_inc(x_86); +lean_inc(x_85); +lean_inc(x_84); +lean_dec(x_3); +lean_inc(x_84); +lean_inc(x_1); +x_87 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_87, 0, x_1); +lean_ctor_set(x_87, 1, x_84); +lean_ctor_set(x_87, 2, x_85); +x_88 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1; +x_89 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_88, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_unbox(x_90); +lean_dec(x_90); +if (x_91 == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_89, 1); +lean_inc(x_92); +lean_dec(x_89); +x_93 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_94 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_84, x_87, x_93, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_92); +lean_dec(x_87); +lean_dec(x_84); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +if (lean_obj_tag(x_95) == 0) +{ +lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_dec(x_86); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_97 = x_94; +} else { + lean_dec_ref(x_94); + x_97 = lean_box(0); +} +x_98 = lean_ctor_get(x_95, 0); +lean_inc(x_98); +lean_dec(x_95); +if (lean_is_scalar(x_97)) { + x_99 = lean_alloc_ctor(0, 2, 0); +} else { + x_99 = x_97; +} +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_96); +return x_99; +} +else +{ +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_94, 1); +lean_inc(x_100); +lean_dec(x_94); +x_101 = lean_ctor_get(x_95, 0); +lean_inc(x_101); +lean_dec(x_95); +x_2 = x_101; +x_3 = x_86; +x_12 = x_100; +goto _start; +} +} +else +{ +lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +lean_dec(x_86); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_103 = lean_ctor_get(x_94, 0); +lean_inc(x_103); +x_104 = lean_ctor_get(x_94, 1); +lean_inc(x_104); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_105 = x_94; +} else { + lean_dec_ref(x_94); + x_105 = lean_box(0); +} +if (lean_is_scalar(x_105)) { + x_106 = lean_alloc_ctor(1, 2, 0); +} else { + x_106 = x_105; +} +lean_ctor_set(x_106, 0, x_103); +lean_ctor_set(x_106, 1, x_104); +return x_106; +} +} +else +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_107 = lean_ctor_get(x_89, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_89)) { + lean_ctor_release(x_89, 0); + lean_ctor_release(x_89, 1); + x_108 = x_89; +} else { + lean_dec_ref(x_89); + x_108 = lean_box(0); +} +x_109 = l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7; +lean_inc(x_87); +x_110 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__2(x_109, x_87); +if (lean_is_scalar(x_108)) { + x_111 = lean_alloc_ctor(7, 2, 0); +} else { + x_111 = x_108; + lean_ctor_set_tag(x_111, 7); +} +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +x_112 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_109); +x_113 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_88, x_112, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_107); +x_114 = lean_ctor_get(x_113, 0); +lean_inc(x_114); +x_115 = lean_ctor_get(x_113, 1); +lean_inc(x_115); +lean_dec(x_113); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_116 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_84, x_87, x_114, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_115); +lean_dec(x_114); +lean_dec(x_87); +lean_dec(x_84); +if (lean_obj_tag(x_116) == 0) +{ +lean_object* x_117; +x_117 = lean_ctor_get(x_116, 0); +lean_inc(x_117); +if (lean_obj_tag(x_117) == 0) +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +lean_dec(x_86); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_118 = lean_ctor_get(x_116, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_119 = x_116; +} else { + lean_dec_ref(x_116); + x_119 = lean_box(0); +} +x_120 = lean_ctor_get(x_117, 0); +lean_inc(x_120); +lean_dec(x_117); +if (lean_is_scalar(x_119)) { + x_121 = lean_alloc_ctor(0, 2, 0); +} else { + x_121 = x_119; +} +lean_ctor_set(x_121, 0, x_120); +lean_ctor_set(x_121, 1, x_118); +return x_121; +} +else +{ +lean_object* x_122; lean_object* x_123; +x_122 = lean_ctor_get(x_116, 1); +lean_inc(x_122); +lean_dec(x_116); +x_123 = lean_ctor_get(x_117, 0); +lean_inc(x_123); +lean_dec(x_117); +x_2 = x_123; +x_3 = x_86; +x_12 = x_122; +goto _start; +} +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +lean_dec(x_86); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_125 = lean_ctor_get(x_116, 0); +lean_inc(x_125); +x_126 = lean_ctor_get(x_116, 1); +lean_inc(x_126); +if (lean_is_exclusive(x_116)) { + lean_ctor_release(x_116, 0); + lean_ctor_release(x_116, 1); + x_127 = x_116; +} else { + lean_dec_ref(x_116); + x_127 = lean_box(0); +} +if (lean_is_scalar(x_127)) { + x_128 = lean_alloc_ctor(1, 2, 0); +} else { + x_128 = x_127; +} +lean_ctor_set(x_128, 0, x_125); +lean_ctor_set(x_128, 1, x_126); +return x_128; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_2, 1); +x_17 = lean_nat_dec_lt(x_4, x_16); +if (x_17 == 0) +{ +lean_object* x_18; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_3); +lean_ctor_set(x_18, 1, x_15); +return x_18; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_3, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_3, 1); +lean_inc(x_20); +x_21 = lean_ctor_get(x_3, 2); +lean_inc(x_21); +x_22 = lean_nat_dec_lt(x_20, x_21); +if (x_22 == 0) +{ +lean_object* x_23; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_15); +return x_23; +} +else +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_3); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_25 = lean_ctor_get(x_3, 2); +lean_dec(x_25); +x_26 = lean_ctor_get(x_3, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_3, 0); +lean_dec(x_27); +x_28 = lean_array_fget(x_19, x_20); +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_add(x_20, x_29); +lean_dec(x_20); +lean_ctor_set(x_3, 1, x_30); +x_31 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_32 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3(x_4, x_31, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_32) == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = lean_ctor_get(x_2, 2); +x_35 = lean_nat_add(x_4, x_34); +lean_dec(x_4); +x_4 = x_35; +x_5 = lean_box(0); +x_6 = lean_box(0); +x_15 = x_33; +goto _start; +} +else +{ +uint8_t x_37; +lean_dec(x_3); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_37 = !lean_is_exclusive(x_32); +if (x_37 == 0) +{ +return x_32; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_32, 0); +x_39 = lean_ctor_get(x_32, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_32); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +lean_dec(x_3); +x_41 = lean_array_fget(x_19, x_20); +x_42 = lean_unsigned_to_nat(1u); +x_43 = lean_nat_add(x_20, x_42); +lean_dec(x_20); +x_44 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_44, 0, x_19); +lean_ctor_set(x_44, 1, x_43); +lean_ctor_set(x_44, 2, x_21); +x_45 = lean_box(0); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_4); +x_46 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3(x_4, x_45, x_41, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_46) == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = lean_ctor_get(x_2, 2); +x_49 = lean_nat_add(x_4, x_48); +lean_dec(x_4); +x_3 = x_44; +x_4 = x_49; +x_5 = lean_box(0); +x_6 = lean_box(0); +x_15 = x_47; +goto _start; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_dec(x_44); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_4); +x_51 = lean_ctor_get(x_46, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_46, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_53 = x_46; +} else { + lean_dec_ref(x_46); + x_53 = lean_box(0); +} +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(1, 2, 0); +} else { + x_54 = x_53; +} +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_52); +return x_54; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_checkInvariants(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_10 = l_Lean_Meta_Grind_Arith_Offset_get_x27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_ctor_get(x_11, 5); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_PersistentArray_toArray___rarg(x_13); +x_15 = lean_array_get_size(x_14); +x_16 = lean_unsigned_to_nat(0u); +x_17 = l_Array_toSubarray___rarg(x_14, x_16, x_15); +x_18 = lean_ctor_get(x_13, 2); +lean_inc(x_18); +lean_dec(x_13); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_20, 0, x_16); +lean_ctor_set(x_20, 1, x_18); +lean_ctor_set(x_20, 2, x_19); +x_21 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4(x_20, x_20, x_17, x_16, lean_box(0), lean_box(0), x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +lean_dec(x_20); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +x_24 = lean_box(0); +lean_ctor_set(x_21, 0, x_24); +return x_21; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_dec(x_21); +x_26 = lean_box(0); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; +} +} +else +{ +uint8_t x_28; +x_28 = !lean_is_exclusive(x_21); +if (x_28 == 0) +{ +return x_21; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_21, 0); +x_30 = lean_ctor_get(x_21, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_21); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +lean_dec(x_2); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +_start: +{ +lean_object* x_16; +x_16 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_2); +lean_dec(x_1); +return x_16; +} +} +lean_object* initialize_Init_Grind_Offset(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_ProofUtil(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Offset(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Grind_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Types(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_ProofUtil(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__1(); +l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__2(); +l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3(); +lean_mark_persistent(l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_Arith_Offset_mkNode___spec__2___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkNode___lambda__2___closed__9); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_getNodeId___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_mkProofForPath_go___closed__4); +l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1(); +lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__1); +l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2(); +lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__2); +l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3(); +lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__3); +l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4(); +lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__4); +l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5(); +lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__6); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___closed__7); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__1); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__2); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__3); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__4); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__5); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___spec__8___closed__6); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setDist___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__6); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateTrue___closed__7); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateFalse___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__1___closed__6); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_propagateEq___lambda__2___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeCnstr___lambda__2___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_internalizeTerm___closed__6); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__1); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__2); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__3); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__4); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__5); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___lambda__1___closed__6); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__1); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqImpl___closed__2); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__1); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__2); +l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_processNewOffsetEqLitImpl___lambda__1___closed__3); +l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__1(); +l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__1___closed__2); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__1); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__2); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__3); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__4); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_traceDists___spec__2___closed__5); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__1); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__2); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__1___closed__3); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__1(); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__2); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__3); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__4); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__5); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__2___closed__6); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__1); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__2); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__3); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__4); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___lambda__3___closed__5); +l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1 = _init_l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1(); +lean_mark_persistent(l_Lean_AssocList_forIn_loop___at_Lean_Meta_Grind_Arith_Offset_checkInvariants___spec__3___closed__1); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/ProofUtil.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/ProofUtil.c new file mode 100644 index 000000000000..074375c83bdd --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/ProofUtil.c @@ -0,0 +1,2733 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.ProofUtil +// Imports: Init.Grind.Offset Init.Grind.Lemmas Lean.Meta.Tactic.Grind.Types +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkNatLit(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32; +lean_object* l_Lean_mkApp7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27; +lean_object* l_Lean_mkApp8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4; +lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8; +uint8_t lean_int_dec_le(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10; +lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3; +lean_object* lean_nat_to_int(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2; +lean_object* l_outOfBounds___rarg(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +extern lean_object* l_Lean_instInhabitedExpr; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4; +lean_object* l_panic___at_Lean_Expr_appFn_x21___spec__1(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___boxed(lean_object*); +lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9; +uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8; +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +lean_object* l_Int_toNat(lean_object*); +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2; +lean_object* l_Lean_PersistentArray_get_x21___rarg(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1; +lean_object* lean_int_add(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14; +uint8_t lean_int_dec_eq(lean_object*, lean_object*); +lean_object* lean_string_append(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17; +lean_object* lean_int_neg(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22; +lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Grind", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("rfl_true", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5; +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("assertion violation: ", 21, 21); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("n >= 0\n ", 9, 9); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.Grind.Arith.ProofUtil", 38, 38); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Meta.Tactic.Grind.Arith.ProofUtil.0.Lean.Meta.Grind.Arith.Offset.toExprN", 86, 86); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6; +x_3 = lean_unsigned_to_nat(23u); +x_4 = lean_unsigned_to_nat(2u); +x_5 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_3 = lean_int_dec_le(x_2, x_1); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; +x_4 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7; +x_5 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = l_Int_toNat(x_1); +x_7 = l_Lean_mkNatLit(x_6); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_1); +lean_dec(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Nat", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_ro", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_lo_1", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_lo_2", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_le", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_ro_2", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_ro_1", 7, 7); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_lo", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_le", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_lo", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_ro", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_trans", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; uint8_t x_14; uint8_t x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +x_6 = lean_ctor_get(x_2, 1); +lean_inc(x_6); +x_7 = lean_ctor_get(x_2, 2); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +x_9 = lean_ctor_get(x_3, 1); +lean_inc(x_9); +x_10 = lean_ctor_get(x_3, 2); +lean_inc(x_10); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + lean_ctor_release(x_3, 1); + lean_ctor_release(x_3, 2); + x_11 = x_3; +} else { + lean_dec_ref(x_3); + x_11 = lean_box(0); +} +x_12 = lean_ctor_get(x_1, 2); +lean_inc(x_12); +x_13 = lean_nat_dec_lt(x_5, x_12); +x_14 = lean_nat_dec_lt(x_8, x_12); +x_15 = lean_nat_dec_lt(x_4, x_12); +lean_dec(x_12); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_17 = lean_int_dec_eq(x_6, x_16); +x_18 = lean_int_add(x_6, x_9); +if (x_13 == 0) +{ +lean_object* x_91; lean_object* x_92; +x_91 = l_Lean_instInhabitedExpr; +x_92 = l_outOfBounds___rarg(x_91); +x_19 = x_92; +goto block_90; +} +else +{ +lean_object* x_93; lean_object* x_94; +x_93 = l_Lean_instInhabitedExpr; +lean_inc(x_1); +x_94 = l_Lean_PersistentArray_get_x21___rarg(x_93, x_1, x_5); +x_19 = x_94; +goto block_90; +} +block_90: +{ +lean_object* x_20; +if (x_14 == 0) +{ +lean_object* x_86; lean_object* x_87; +lean_dec(x_8); +x_86 = l_Lean_instInhabitedExpr; +x_87 = l_outOfBounds___rarg(x_86); +x_20 = x_87; +goto block_85; +} +else +{ +lean_object* x_88; lean_object* x_89; +x_88 = l_Lean_instInhabitedExpr; +lean_inc(x_1); +x_89 = l_Lean_PersistentArray_get_x21___rarg(x_88, x_1, x_8); +lean_dec(x_8); +x_20 = x_89; +goto block_85; +} +block_85: +{ +lean_object* x_21; +if (x_15 == 0) +{ +lean_object* x_81; lean_object* x_82; +lean_dec(x_1); +x_81 = l_Lean_instInhabitedExpr; +x_82 = l_outOfBounds___rarg(x_81); +x_21 = x_82; +goto block_80; +} +else +{ +lean_object* x_83; lean_object* x_84; +x_83 = l_Lean_instInhabitedExpr; +x_84 = l_Lean_PersistentArray_get_x21___rarg(x_83, x_1, x_4); +x_21 = x_84; +goto block_80; +} +block_80: +{ +if (x_17 == 0) +{ +uint8_t x_22; +x_22 = lean_int_dec_lt(x_6, x_16); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_6); +x_24 = lean_int_dec_eq(x_9, x_16); +if (x_24 == 0) +{ +uint8_t x_25; +x_25 = lean_int_dec_lt(x_9, x_16); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_6); +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_9); +lean_dec(x_9); +x_27 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4; +x_28 = l_Lean_mkApp7(x_27, x_19, x_20, x_21, x_23, x_26, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_29 = lean_alloc_ctor(0, 3, 0); +} else { + x_29 = x_11; +} +lean_ctor_set(x_29, 0, x_5); +lean_ctor_set(x_29, 1, x_18); +lean_ctor_set(x_29, 2, x_28); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_int_neg(x_9); +lean_dec(x_9); +x_31 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_30); +x_32 = lean_int_dec_lt(x_6, x_30); +lean_dec(x_30); +lean_dec(x_6); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7; +x_34 = l_Lean_mkApp7(x_33, x_19, x_20, x_21, x_23, x_31, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_35 = lean_alloc_ctor(0, 3, 0); +} else { + x_35 = x_11; +} +lean_ctor_set(x_35, 0, x_5); +lean_ctor_set(x_35, 1, x_18); +lean_ctor_set(x_35, 2, x_34); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10; +x_37 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_38 = l_Lean_mkApp8(x_36, x_19, x_20, x_21, x_23, x_31, x_37, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_39 = lean_alloc_ctor(0, 3, 0); +} else { + x_39 = x_11; +} +lean_ctor_set(x_39, 0, x_5); +lean_ctor_set(x_39, 1, x_18); +lean_ctor_set(x_39, 2, x_38); +return x_39; +} +} +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; +lean_dec(x_9); +lean_dec(x_6); +x_40 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13; +x_41 = l_Lean_mkApp6(x_40, x_19, x_20, x_21, x_23, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_42 = lean_alloc_ctor(0, 3, 0); +} else { + x_42 = x_11; +} +lean_ctor_set(x_42, 0, x_5); +lean_ctor_set(x_42, 1, x_18); +lean_ctor_set(x_42, 2, x_41); +return x_42; +} +} +else +{ +lean_object* x_43; uint8_t x_44; +x_43 = lean_int_neg(x_6); +lean_dec(x_6); +x_44 = lean_int_dec_eq(x_9, x_16); +if (x_44 == 0) +{ +uint8_t x_45; +x_45 = lean_int_dec_lt(x_9, x_16); +if (x_45 == 0) +{ +lean_object* x_46; lean_object* x_47; uint8_t x_48; +x_46 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_43); +x_47 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_9); +x_48 = lean_int_dec_lt(x_9, x_43); +lean_dec(x_43); +lean_dec(x_9); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16; +x_50 = l_Lean_mkApp7(x_49, x_19, x_20, x_21, x_46, x_47, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_51 = lean_alloc_ctor(0, 3, 0); +} else { + x_51 = x_11; +} +lean_ctor_set(x_51, 0, x_5); +lean_ctor_set(x_51, 1, x_18); +lean_ctor_set(x_51, 2, x_50); +return x_51; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_52 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19; +x_53 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_54 = l_Lean_mkApp8(x_52, x_19, x_20, x_21, x_46, x_47, x_53, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_55 = lean_alloc_ctor(0, 3, 0); +} else { + x_55 = x_11; +} +lean_ctor_set(x_55, 0, x_5); +lean_ctor_set(x_55, 1, x_18); +lean_ctor_set(x_55, 2, x_54); +return x_55; +} +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_56 = lean_int_neg(x_9); +lean_dec(x_9); +x_57 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_43); +lean_dec(x_43); +x_58 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_56); +lean_dec(x_56); +x_59 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22; +x_60 = l_Lean_mkApp7(x_59, x_19, x_20, x_21, x_57, x_58, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_61 = lean_alloc_ctor(0, 3, 0); +} else { + x_61 = x_11; +} +lean_ctor_set(x_61, 0, x_5); +lean_ctor_set(x_61, 1, x_18); +lean_ctor_set(x_61, 2, x_60); +return x_61; +} +} +else +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_9); +x_62 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_43); +lean_dec(x_43); +x_63 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25; +x_64 = l_Lean_mkApp6(x_63, x_19, x_20, x_21, x_62, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_65 = lean_alloc_ctor(0, 3, 0); +} else { + x_65 = x_11; +} +lean_ctor_set(x_65, 0, x_5); +lean_ctor_set(x_65, 1, x_18); +lean_ctor_set(x_65, 2, x_64); +return x_65; +} +} +} +else +{ +uint8_t x_66; +lean_dec(x_6); +x_66 = lean_int_dec_eq(x_9, x_16); +if (x_66 == 0) +{ +uint8_t x_67; +x_67 = lean_int_dec_lt(x_16, x_9); +if (x_67 == 0) +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_68 = lean_int_neg(x_9); +lean_dec(x_9); +x_69 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_68); +lean_dec(x_68); +x_70 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28; +x_71 = l_Lean_mkApp6(x_70, x_19, x_20, x_21, x_69, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_72 = lean_alloc_ctor(0, 3, 0); +} else { + x_72 = x_11; +} +lean_ctor_set(x_72, 0, x_5); +lean_ctor_set(x_72, 1, x_18); +lean_ctor_set(x_72, 2, x_71); +return x_72; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_73 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_9); +lean_dec(x_9); +x_74 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31; +x_75 = l_Lean_mkApp6(x_74, x_19, x_20, x_21, x_73, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_76 = lean_alloc_ctor(0, 3, 0); +} else { + x_76 = x_11; +} +lean_ctor_set(x_76, 0, x_5); +lean_ctor_set(x_76, 1, x_18); +lean_ctor_set(x_76, 2, x_75); +return x_76; +} +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_9); +x_77 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34; +x_78 = l_Lean_mkApp5(x_77, x_19, x_20, x_21, x_7, x_10); +if (lean_is_scalar(x_11)) { + x_79 = lean_alloc_ctor(0, 3, 0); +} else { + x_79 = x_11; +} +lean_ctor_set(x_79, 0, x_5); +lean_ctor_set(x_79, 1, x_18); +lean_ctor_set(x_79, 2, x_78); +return x_79; +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkTrans___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkTrans(x_1, x_2, x_3, x_4); +lean_dec(x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1; +x_2 = lean_int_neg(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_ro_eq_false", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_lo_eq_false", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_lo_eq_false_1", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_le_eq_false", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; +x_4 = lean_ctor_get(x_2, 0); +x_5 = lean_ctor_get(x_1, 2); +lean_inc(x_5); +x_6 = lean_nat_dec_lt(x_4, x_5); +x_7 = lean_ctor_get(x_2, 1); +x_8 = lean_nat_dec_lt(x_7, x_5); +lean_dec(x_5); +x_9 = lean_ctor_get(x_2, 2); +x_10 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_11 = lean_int_dec_eq(x_9, x_10); +if (x_6 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = l_Lean_instInhabitedExpr; +x_35 = l_outOfBounds___rarg(x_34); +x_12 = x_35; +goto block_33; +} +else +{ +lean_object* x_36; lean_object* x_37; +x_36 = l_Lean_instInhabitedExpr; +lean_inc(x_1); +x_37 = l_Lean_PersistentArray_get_x21___rarg(x_36, x_1, x_4); +x_12 = x_37; +goto block_33; +} +block_33: +{ +lean_object* x_13; +if (x_8 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_1); +x_29 = l_Lean_instInhabitedExpr; +x_30 = l_outOfBounds___rarg(x_29); +x_13 = x_30; +goto block_28; +} +else +{ +lean_object* x_31; lean_object* x_32; +x_31 = l_Lean_instInhabitedExpr; +x_32 = l_Lean_PersistentArray_get_x21___rarg(x_31, x_1, x_7); +x_13 = x_32; +goto block_28; +} +block_28: +{ +if (x_11 == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2; +x_15 = lean_int_dec_eq(x_9, x_14); +if (x_15 == 0) +{ +uint8_t x_16; +x_16 = lean_int_dec_lt(x_9, x_10); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_9); +x_18 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5; +x_19 = l_Lean_mkApp4(x_18, x_12, x_13, x_17, x_3); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_int_neg(x_9); +x_21 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_20); +lean_dec(x_20); +x_22 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8; +x_23 = l_Lean_mkApp4(x_22, x_12, x_13, x_21, x_3); +return x_23; +} +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11; +x_25 = l_Lean_mkApp3(x_24, x_12, x_13, x_3); +return x_25; +} +} +else +{ +lean_object* x_26; lean_object* x_27; +x_26 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14; +x_27 = l_Lean_mkApp3(x_26, x_12, x_13, x_3); +return x_27; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("kuv > 0 && kvu < 0\n ", 23, 23); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.mkUnsatProof", 41, 41); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3; +x_3 = lean_unsigned_to_nat(110u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unsat_lo_ro", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("kvu < 0\n ", 14, 14); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3; +x_3 = lean_unsigned_to_nat(107u); +x_4 = lean_unsigned_to_nat(6u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unsat_lo_lo", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unsat_le_lo", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("kvu < 0\n ", 12, 12); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3; +x_3 = lean_unsigned_to_nat(99u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_8 = lean_int_dec_eq(x_3, x_7); +if (x_8 == 0) +{ +uint8_t x_9; +x_9 = lean_int_dec_eq(x_5, x_7); +if (x_9 == 0) +{ +uint8_t x_10; +x_10 = lean_int_dec_lt(x_3, x_7); +if (x_10 == 0) +{ +uint8_t x_11; +x_11 = lean_int_dec_lt(x_7, x_3); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_12 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4; +x_13 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_12); +return x_13; +} +else +{ +uint8_t x_14; +x_14 = lean_int_dec_lt(x_5, x_7); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_15 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4; +x_16 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_15); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_int_neg(x_5); +x_18 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_17); +lean_dec(x_17); +x_19 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_3); +x_20 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7; +x_21 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_22 = l_Lean_mkApp7(x_20, x_2, x_1, x_18, x_19, x_21, x_6, x_4); +return x_22; +} +} +} +else +{ +uint8_t x_23; +x_23 = lean_int_dec_lt(x_7, x_5); +if (x_23 == 0) +{ +uint8_t x_24; +x_24 = lean_int_dec_lt(x_5, x_7); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_25 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10; +x_26 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_25); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_27 = lean_int_neg(x_3); +x_28 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_27); +lean_dec(x_27); +x_29 = lean_int_neg(x_5); +x_30 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_29); +lean_dec(x_29); +x_31 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13; +x_32 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_33 = l_Lean_mkApp7(x_31, x_1, x_2, x_28, x_30, x_32, x_4, x_6); +return x_33; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_34 = lean_int_neg(x_3); +x_35 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_34); +lean_dec(x_34); +x_36 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_5); +x_37 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7; +x_38 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_39 = l_Lean_mkApp7(x_37, x_1, x_2, x_35, x_36, x_38, x_4, x_6); +return x_39; +} +} +} +else +{ +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_40 = lean_int_neg(x_3); +x_41 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_40); +lean_dec(x_40); +x_42 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16; +x_43 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_44 = l_Lean_mkApp6(x_42, x_2, x_1, x_41, x_43, x_6, x_4); +return x_44; +} +} +else +{ +uint8_t x_45; +x_45 = lean_int_dec_lt(x_5, x_7); +if (x_45 == 0) +{ +lean_object* x_46; lean_object* x_47; +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_46 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19; +x_47 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_46); +return x_47; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_48 = lean_int_neg(x_5); +x_49 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_48); +lean_dec(x_48); +x_50 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16; +x_51 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_52 = l_Lean_mkApp6(x_50, x_1, x_2, x_49, x_51, x_4, x_6); +return x_52; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_3); +return x_7; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("k > 0\n ", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.mkPropagateEqTrueProof", 51, 51); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3; +x_3 = lean_unsigned_to_nat(136u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("k' > 0\n ", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3; +x_3 = lean_unsigned_to_nat(137u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_eq_true_of_ro", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("k' > 0\n ", 13, 13); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3; +x_3 = lean_unsigned_to_nat(133u); +x_4 = lean_unsigned_to_nat(6u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_eq_true_of_lo", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_eq_true_of_lo", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_eq_true_of_lo", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3; +x_3 = lean_unsigned_to_nat(123u); +x_4 = lean_unsigned_to_nat(6u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_eq_true_of_le", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_eq_true_of_le", 16, 16); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_7 = lean_int_dec_eq(x_3, x_6); +if (x_7 == 0) +{ +uint8_t x_8; +x_8 = lean_int_dec_lt(x_3, x_6); +if (x_8 == 0) +{ +uint8_t x_9; +x_9 = lean_int_dec_lt(x_6, x_3); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_10 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4; +x_11 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_10); +return x_11; +} +else +{ +uint8_t x_12; +x_12 = lean_int_dec_lt(x_6, x_5); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_13 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7; +x_14 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_13); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_3); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_5); +x_17 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10; +x_18 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_19 = l_Lean_mkApp6(x_17, x_1, x_2, x_15, x_16, x_18, x_4); +return x_19; +} +} +} +else +{ +lean_object* x_20; uint8_t x_21; +x_20 = lean_int_neg(x_3); +x_21 = lean_int_dec_eq(x_5, x_6); +if (x_21 == 0) +{ +uint8_t x_22; +x_22 = lean_int_dec_lt(x_5, x_6); +if (x_22 == 0) +{ +uint8_t x_23; +x_23 = lean_int_dec_lt(x_6, x_5); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_20); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_24 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13; +x_25 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_24); +return x_25; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_20); +lean_dec(x_20); +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_5); +x_28 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16; +x_29 = l_Lean_mkApp5(x_28, x_1, x_2, x_26, x_27, x_4); +return x_29; +} +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_30 = lean_int_neg(x_5); +x_31 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_20); +lean_dec(x_20); +x_32 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_30); +lean_dec(x_30); +x_33 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19; +x_34 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_35 = l_Lean_mkApp6(x_33, x_1, x_2, x_31, x_32, x_34, x_4); +return x_35; +} +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_20); +lean_dec(x_20); +x_37 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22; +x_38 = l_Lean_mkApp4(x_37, x_1, x_2, x_36, x_4); +return x_38; +} +} +} +else +{ +uint8_t x_39; +x_39 = lean_int_dec_eq(x_5, x_6); +if (x_39 == 0) +{ +uint8_t x_40; +x_40 = lean_int_dec_lt(x_6, x_5); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_41 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23; +x_42 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_41); +return x_42; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_5); +x_44 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26; +x_45 = l_Lean_mkApp4(x_44, x_1, x_2, x_43, x_4); +return x_45; +} +} +else +{ +lean_object* x_46; lean_object* x_47; +x_46 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29; +x_47 = l_Lean_mkApp3(x_46, x_1, x_2, x_4); +return x_47; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Grind.Arith.Offset.mkPropagateEqFalseProof", 52, 52); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1; +x_3 = lean_unsigned_to_nat(161u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("k' < 0\n ", 11, 11); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3; +x_3 = lean_string_append(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1; +x_3 = lean_unsigned_to_nat(162u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_eq_false_of_ro", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1; +x_3 = lean_unsigned_to_nat(158u); +x_4 = lean_unsigned_to_nat(6u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ro_eq_false_of_lo", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_eq_false_of_lo", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le_eq_false_of_lo", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5; +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1; +x_3 = lean_unsigned_to_nat(147u); +x_4 = lean_unsigned_to_nat(4u); +x_5 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("lo_eq_false_of_le", 17, 17); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2; +x_3 = l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1; +x_4 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; uint8_t x_7; +x_6 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1; +x_7 = lean_int_dec_eq(x_3, x_6); +if (x_7 == 0) +{ +uint8_t x_8; +x_8 = lean_int_dec_lt(x_3, x_6); +if (x_8 == 0) +{ +uint8_t x_9; +x_9 = lean_int_dec_lt(x_6, x_3); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_10 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2; +x_11 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_10); +return x_11; +} +else +{ +uint8_t x_12; +x_12 = lean_int_dec_lt(x_5, x_6); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_13 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5; +x_14 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_13); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_int_neg(x_5); +x_16 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_3); +x_17 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_15); +lean_dec(x_15); +x_18 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8; +x_19 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_20 = l_Lean_mkApp6(x_18, x_1, x_2, x_16, x_17, x_19, x_4); +return x_20; +} +} +} +else +{ +lean_object* x_21; uint8_t x_22; +x_21 = lean_int_neg(x_3); +x_22 = lean_int_dec_eq(x_5, x_6); +if (x_22 == 0) +{ +uint8_t x_23; +x_23 = lean_int_dec_lt(x_5, x_6); +if (x_23 == 0) +{ +uint8_t x_24; +x_24 = lean_int_dec_lt(x_6, x_5); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_21); +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_25 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9; +x_26 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_25); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_27 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_21); +lean_dec(x_21); +x_28 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_5); +x_29 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12; +x_30 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_31 = l_Lean_mkApp6(x_29, x_1, x_2, x_27, x_28, x_30, x_4); +return x_31; +} +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_32 = lean_int_neg(x_5); +x_33 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_21); +lean_dec(x_21); +x_34 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_32); +lean_dec(x_32); +x_35 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15; +x_36 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_37 = l_Lean_mkApp6(x_35, x_1, x_2, x_33, x_34, x_36, x_4); +return x_37; +} +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_38 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_21); +lean_dec(x_21); +x_39 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18; +x_40 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_41 = l_Lean_mkApp5(x_39, x_1, x_2, x_38, x_40, x_4); +return x_41; +} +} +} +else +{ +uint8_t x_42; +x_42 = lean_int_dec_lt(x_5, x_6); +if (x_42 == 0) +{ +lean_object* x_43; lean_object* x_44; +lean_dec(x_4); +lean_dec(x_2); +lean_dec(x_1); +x_43 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19; +x_44 = l_panic___at_Lean_Expr_appFn_x21___spec__1(x_43); +return x_44; +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_45 = lean_int_neg(x_5); +x_46 = l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN(x_45); +lean_dec(x_45); +x_47 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22; +x_48 = l_Lean_Meta_Grind_Arith_Offset_rfl__true; +x_49 = l_Lean_mkApp5(x_47, x_1, x_2, x_46, x_48, x_4); +return x_49; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_5); +lean_dec(x_3); +return x_6; +} +} +lean_object* initialize_Init_Grind_Offset(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Grind_Lemmas(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_ProofUtil(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Grind_Offset(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_Grind_Lemmas(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Types(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__1); +l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__2); +l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__3); +l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__4); +l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true___closed__5); +l_Lean_Meta_Grind_Arith_Offset_rfl__true = _init_l_Lean_Meta_Grind_Arith_Offset_rfl__true(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_rfl__true); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__1); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__2); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__3); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__4); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__5); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__6); +l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Arith_ProofUtil_0__Lean_Meta_Grind_Arith_Offset_toExprN___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__9); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__10); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__11); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__12); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__13); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__14); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__15); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__16); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__17); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__18); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__19); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__20); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__21); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__22); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__23); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__24); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__25); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__26); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__27); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__28); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__29); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__30); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__31); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__32); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__33); +l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34 = _init_l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkTrans___closed__34); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__9); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__10); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__11); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__12); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__13); +l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14 = _init_l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkOfNegEqFalse___closed__14); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__9); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__10); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__11); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__12); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__13); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__14); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__15); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__16); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__17); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__18); +l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19 = _init_l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkUnsatProof___closed__19); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__9); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__10); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__11); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__12); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__13); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__14); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__15); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__16); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__17); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__18); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__19); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__20); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__21); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__22); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__23); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__24); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__25); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__26); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__27); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__28); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqTrueProof___closed__29); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__1); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__2); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__3); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__4); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__5); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__6); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__7); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__8); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__9); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__10); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__11); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__12); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__13); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__14); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__15); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__16); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__17); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__18); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__19); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__20); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__21); +l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22 = _init_l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_mkPropagateEqFalseProof___closed__22); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Types.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Types.c new file mode 100644 index 000000000000..2d224abbbfab --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Types.c @@ -0,0 +1,509 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Types +// Imports: Lean.Data.PersistentArray Lean.Meta.Tactic.Grind.ENodeKey Lean.Meta.Tactic.Grind.Arith.Util +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7; +lean_object* l_Lean_Expr_bvar___override(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6; +size_t lean_usize_of_nat(lean_object*); +lean_object* l_Lean_stringToMessageData(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6; +lean_object* lean_nat_to_int(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4; +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_instInhabitedState; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4; +lean_object* lean_nat_abs(lean_object*); +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2; +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedState; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3; +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1; +static size_t l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo; +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId(lean_object*); +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("#", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ≤ ", 5, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" + ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = lean_ctor_get(x_1, 2); +lean_inc(x_2); +x_3 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1; +x_4 = lean_int_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_nat_abs(x_2); +lean_dec(x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +x_9 = l___private_Init_Data_Repr_0__Nat_reprFast(x_8); +x_10 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_10, 0, x_9); +x_11 = l_Lean_MessageData_ofFormat(x_10); +x_12 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5; +x_13 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +x_14 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7; +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = lean_ctor_get(x_1, 1); +lean_inc(x_19); +lean_dec(x_1); +x_20 = l___private_Init_Data_Repr_0__Nat_reprFast(x_19); +x_21 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l_Lean_MessageData_ofFormat(x_21); +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_12); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_14); +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_18); +lean_ctor_set(x_25, 1, x_24); +x_26 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +x_28 = l___private_Init_Data_Repr_0__Nat_reprFast(x_5); +x_29 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_29, 0, x_28); +x_30 = l_Lean_MessageData_ofFormat(x_29); +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_14); +return x_32; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_5); +x_33 = lean_ctor_get(x_1, 0); +lean_inc(x_33); +x_34 = l___private_Init_Data_Repr_0__Nat_reprFast(x_33); +x_35 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_35, 0, x_34); +x_36 = l_Lean_MessageData_ofFormat(x_35); +x_37 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +x_39 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +x_42 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_ctor_get(x_1, 1); +lean_inc(x_44); +lean_dec(x_1); +x_45 = l___private_Init_Data_Repr_0__Nat_reprFast(x_44); +x_46 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l_Lean_MessageData_ofFormat(x_46); +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_37); +lean_ctor_set(x_48, 1, x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_39); +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_43); +lean_ctor_set(x_50, 1, x_49); +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_39); +return x_51; +} +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_52 = lean_nat_abs(x_2); +lean_dec(x_2); +x_53 = lean_unsigned_to_nat(1u); +x_54 = lean_nat_sub(x_52, x_53); +lean_dec(x_52); +x_55 = lean_ctor_get(x_1, 0); +lean_inc(x_55); +x_56 = l___private_Init_Data_Repr_0__Nat_reprFast(x_55); +x_57 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_57, 0, x_56); +x_58 = l_Lean_MessageData_ofFormat(x_57); +x_59 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5; +x_60 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_58); +x_61 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3; +x_62 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +x_63 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +x_64 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9; +x_65 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +x_66 = lean_nat_add(x_54, x_53); +lean_dec(x_54); +x_67 = l___private_Init_Data_Repr_0__Nat_reprFast(x_66); +x_68 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_68, 0, x_67); +x_69 = l_Lean_MessageData_ofFormat(x_68); +x_70 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_70, 0, x_65); +lean_ctor_set(x_70, 1, x_69); +x_71 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7; +x_72 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +x_73 = lean_ctor_get(x_1, 1); +lean_inc(x_73); +lean_dec(x_1); +x_74 = l___private_Init_Data_Repr_0__Nat_reprFast(x_73); +x_75 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_75, 0, x_74); +x_76 = l_Lean_MessageData_ofFormat(x_75); +x_77 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_77, 0, x_59); +lean_ctor_set(x_77, 1, x_76); +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_61); +x_79 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_79, 0, x_72); +lean_ctor_set(x_79, 1, x_78); +x_80 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_80, 0, x_79); +lean_ctor_set(x_80, 1, x_61); +return x_80; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Expr_bvar___override(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1; +x_3 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1; +x_4 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2; +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static size_t _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__3() { +_start: +{ +lean_object* x_1; size_t x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_usize_of_nat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; size_t x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1; +x_3 = lean_unsigned_to_nat(0u); +x_4 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__3; +x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_3); +lean_ctor_set_usize(x_5, 4, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4; +x_2 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6; +x_3 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 2, x_2); +lean_ctor_set(x_3, 3, x_2); +lean_ctor_set(x_3, 4, x_1); +lean_ctor_set(x_3, 5, x_1); +lean_ctor_set(x_3, 6, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7; +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_instInhabitedState() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7; +return x_1; +} +} +lean_object* initialize_Lean_Data_PersistentArray(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_ENodeKey(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Util(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Types(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Data_PersistentArray(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_ENodeKey(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Util(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__1); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__2); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__3); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__4); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__5); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__6); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__7); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__8); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_Offset_instToMessageDataCnstrNodeId___spec__1___closed__9); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__1); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo___closed__2); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedProofInfo); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__1); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__2); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__3(); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__4); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__5); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__6); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState___closed__7); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedState = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedState(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedState); +l_Lean_Meta_Grind_Arith_instInhabitedState = _init_l_Lean_Meta_Grind_Arith_instInhabitedState(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_instInhabitedState); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Util.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Util.c new file mode 100644 index 000000000000..e02d8fd13db8 --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Arith/Util.c @@ -0,0 +1,1736 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.Arith.Util +// Imports: Lean.Expr Lean.Message +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3; +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isInstAddNat(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatType___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___boxed(lean_object*); +uint8_t l_Lean_Expr_isApp(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__1(lean_object*); +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); +lean_object* l_Lean_stringToMessageData(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1; +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5; +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isNatType(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isInstLENat(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2___boxed(lean_object*); +lean_object* lean_nat_to_int(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +static lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2(lean_object*); +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffset_x3f(lean_object*); +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatAdd_x3f(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatType___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f_go(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg(lean_object*); +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2; +lean_object* lean_int_sub(lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofExpr(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatType___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isInstLENat___boxed(lean_object*); +lean_object* lean_nat_abs(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isInstLENat___closed__2; +uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1; +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1; +uint8_t lean_int_dec_lt(lean_object*, lean_object*); +lean_object* lean_nat_sub(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2; +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1; +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isNatAdd(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatAdd___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4; +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isInstLENat___closed__1; +lean_object* lean_int_neg(lean_object*); +lean_object* lean_nat_add(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6; +lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +static lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2; +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatType___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Nat", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatType___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_isNatType___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isNatType(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Meta_Grind_Arith_isNatType___closed__2; +x_3 = l_Lean_Expr_isConstOf(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatType___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_isNatType(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("instHAdd", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("instAddNat", 10, 10); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isInstAddNat(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = 0; +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = l_Lean_Expr_appArg(x_2, lean_box(0)); +x_6 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_7 = l_Lean_Expr_isApp(x_6); +if (x_7 == 0) +{ +uint8_t x_8; +lean_dec(x_6); +lean_dec(x_5); +x_8 = 0; +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = l_Lean_Expr_appArg(x_6, lean_box(0)); +x_10 = l_Lean_Expr_appFnCleanup(x_6, lean_box(0)); +x_11 = l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2; +x_12 = l_Lean_Expr_isConstOf(x_10, x_11); +lean_dec(x_10); +if (x_12 == 0) +{ +uint8_t x_13; +lean_dec(x_9); +lean_dec(x_5); +x_13 = 0; +return x_13; +} +else +{ +uint8_t x_14; +x_14 = l_Lean_Meta_Grind_Arith_isNatType(x_9); +lean_dec(x_9); +if (x_14 == 0) +{ +uint8_t x_15; +lean_dec(x_5); +x_15 = 0; +return x_15; +} +else +{ +lean_object* x_16; uint8_t x_17; +x_16 = l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4; +x_17 = l_Lean_Expr_isConstOf(x_5, x_16); +lean_dec(x_5); +return x_17; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isInstAddNat___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_isInstAddNat(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstLENat___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("instLENat", 9, 9); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isInstLENat___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_isInstLENat___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isInstLENat(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Meta_Grind_Arith_isInstLENat___closed__2; +x_3 = l_Lean_Expr_isConstOf(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isInstLENat___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_isInstLENat(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("HAdd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("hAdd", 4, 4); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatAdd_x3f(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) +{ +lean_object* x_4; +lean_dec(x_2); +x_4 = lean_box(0); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = l_Lean_Expr_appArg(x_2, lean_box(0)); +x_6 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_7 = l_Lean_Expr_isApp(x_6); +if (x_7 == 0) +{ +lean_object* x_8; +lean_dec(x_6); +lean_dec(x_5); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = l_Lean_Expr_appArg(x_6, lean_box(0)); +x_10 = l_Lean_Expr_appFnCleanup(x_6, lean_box(0)); +x_11 = l_Lean_Expr_isApp(x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_5); +x_12 = lean_box(0); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Expr_appArg(x_10, lean_box(0)); +x_14 = l_Lean_Expr_appFnCleanup(x_10, lean_box(0)); +x_15 = l_Lean_Expr_isApp(x_14); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +x_16 = lean_box(0); +return x_16; +} +else +{ +lean_object* x_17; uint8_t x_18; +x_17 = l_Lean_Expr_appFnCleanup(x_14, lean_box(0)); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) +{ +lean_object* x_19; +lean_dec(x_17); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +x_19 = lean_box(0); +return x_19; +} +else +{ +lean_object* x_20; uint8_t x_21; +x_20 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_21 = l_Lean_Expr_isApp(x_20); +if (x_21 == 0) +{ +lean_object* x_22; +lean_dec(x_20); +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +x_22 = lean_box(0); +return x_22; +} +else +{ +lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_23 = l_Lean_Expr_appFnCleanup(x_20, lean_box(0)); +x_24 = l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3; +x_25 = l_Lean_Expr_isConstOf(x_23, x_24); +lean_dec(x_23); +if (x_25 == 0) +{ +lean_object* x_26; +lean_dec(x_13); +lean_dec(x_9); +lean_dec(x_5); +x_26 = lean_box(0); +return x_26; +} +else +{ +uint8_t x_27; +x_27 = l_Lean_Meta_Grind_Arith_isInstAddNat(x_13); +if (x_27 == 0) +{ +lean_object* x_28; +lean_dec(x_9); +lean_dec(x_5); +x_28 = lean_box(0); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_9); +lean_ctor_set(x_29, 1, x_5); +x_30 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_30, 0, x_29); +return x_30; +} +} +} +} +} +} +} +} +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_Arith_isNatAdd(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) +{ +uint8_t x_4; +lean_dec(x_2); +x_4 = 0; +return x_4; +} +else +{ +lean_object* x_5; uint8_t x_6; +x_5 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_6 = l_Lean_Expr_isApp(x_5); +if (x_6 == 0) +{ +uint8_t x_7; +lean_dec(x_5); +x_7 = 0; +return x_7; +} +else +{ +lean_object* x_8; uint8_t x_9; +x_8 = l_Lean_Expr_appFnCleanup(x_5, lean_box(0)); +x_9 = l_Lean_Expr_isApp(x_8); +if (x_9 == 0) +{ +uint8_t x_10; +lean_dec(x_8); +x_10 = 0; +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l_Lean_Expr_appArg(x_8, lean_box(0)); +x_12 = l_Lean_Expr_appFnCleanup(x_8, lean_box(0)); +x_13 = l_Lean_Expr_isApp(x_12); +if (x_13 == 0) +{ +uint8_t x_14; +lean_dec(x_12); +lean_dec(x_11); +x_14 = 0; +return x_14; +} +else +{ +lean_object* x_15; uint8_t x_16; +x_15 = l_Lean_Expr_appFnCleanup(x_12, lean_box(0)); +x_16 = l_Lean_Expr_isApp(x_15); +if (x_16 == 0) +{ +uint8_t x_17; +lean_dec(x_15); +lean_dec(x_11); +x_17 = 0; +return x_17; +} +else +{ +lean_object* x_18; uint8_t x_19; +x_18 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_19 = l_Lean_Expr_isApp(x_18); +if (x_19 == 0) +{ +uint8_t x_20; +lean_dec(x_18); +lean_dec(x_11); +x_20 = 0; +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = l_Lean_Expr_appFnCleanup(x_18, lean_box(0)); +x_22 = l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3; +x_23 = l_Lean_Expr_isConstOf(x_21, x_22); +lean_dec(x_21); +if (x_23 == 0) +{ +uint8_t x_24; +lean_dec(x_11); +x_24 = 0; +return x_24; +} +else +{ +uint8_t x_25; +x_25 = l_Lean_Meta_Grind_Arith_isInstAddNat(x_11); +return x_25; +} +} +} +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatAdd___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_isNatAdd(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__1(lean_object* x_1) { +_start: +{ +if (lean_obj_tag(x_1) == 9) +{ +lean_object* x_2; +x_2 = lean_ctor_get(x_1, 0); +lean_inc(x_2); +lean_dec(x_1); +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_ctor_set_tag(x_2, 1); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; +} +} +else +{ +lean_object* x_6; +lean_dec(x_2); +x_6 = lean_box(0); +return x_6; +} +} +else +{ +lean_object* x_7; +lean_dec(x_1); +x_7 = lean_box(0); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_box(0); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2; +x_2 = lean_box(0); +x_3 = lean_apply_1(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("instOfNatNat", 12, 12); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1; +x_3 = l_Lean_Expr_cleanupAnnotations(x_1); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) +{ +lean_object* x_5; +lean_dec(x_3); +x_5 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_7 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_8 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5; +x_9 = l_Lean_Expr_isConstOf(x_7, x_8); +lean_dec(x_7); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_6); +x_10 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_10; +} +else +{ +lean_object* x_11; +x_11 = lean_apply_1(x_2, x_6); +return x_11; +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ofNat", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2; +x_2 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1; +x_3 = l_Lean_Expr_cleanupAnnotations(x_1); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) +{ +lean_object* x_5; +lean_dec(x_3); +x_5 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_7 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_8 = l_Lean_Expr_isApp(x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_7); +lean_dec(x_6); +x_9 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_9; +} +else +{ +lean_object* x_10; uint8_t x_11; +x_10 = l_Lean_Expr_appFnCleanup(x_7, lean_box(0)); +x_11 = l_Lean_Expr_isApp(x_10); +if (x_11 == 0) +{ +lean_object* x_12; +lean_dec(x_10); +lean_dec(x_6); +x_12 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Expr_appFnCleanup(x_10, lean_box(0)); +x_14 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4; +x_15 = l_Lean_Expr_isConstOf(x_13, x_14); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_6); +x_16 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3; +return x_16; +} +else +{ +lean_object* x_17; +x_17 = lean_apply_1(x_2, x_6); +return x_17; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__2(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffset_x3f(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Meta_Grind_Arith_isNatAdd_x3f(x_1); +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; +x_3 = lean_box(0); +return x_3; +} +else +{ +lean_object* x_4; uint8_t x_5; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = !lean_is_exclusive(x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_4, 0); +x_7 = lean_ctor_get(x_4, 1); +x_8 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; +lean_free_object(x_4); +lean_dec(x_6); +x_9 = lean_box(0); +return x_9; +} +else +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_8); +if (x_10 == 0) +{ +lean_object* x_11; +x_11 = lean_ctor_get(x_8, 0); +lean_ctor_set(x_4, 1, x_11); +lean_ctor_set(x_8, 0, x_4); +return x_8; +} +else +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_8, 0); +lean_inc(x_12); +lean_dec(x_8); +lean_ctor_set(x_4, 1, x_12); +x_13 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_13, 0, x_4); +return x_13; +} +} +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_4, 0); +x_15 = lean_ctor_get(x_4, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_4); +x_16 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_15); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; +lean_dec(x_14); +x_17 = lean_box(0); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + x_19 = x_16; +} else { + lean_dec_ref(x_16); + x_19 = lean_box(0); +} +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_14); +lean_ctor_set(x_20, 1, x_18); +if (lean_is_scalar(x_19)) { + x_21 = lean_alloc_ctor(1, 1, 0); +} else { + x_21 = x_19; +} +lean_ctor_set(x_21, 0, x_20); +return x_21; +} +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1; +lean_inc(x_1); +x_3 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_1); +lean_ctor_set(x_3, 2, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg), 1, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg(lean_object* x_1) { +_start: +{ +uint8_t x_2; +x_2 = !lean_is_exclusive(x_1); +if (x_2 == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_3 = lean_ctor_get(x_1, 0); +x_4 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_1, 2); +x_6 = lean_int_neg(x_5); +lean_dec(x_5); +x_7 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1; +x_8 = lean_int_sub(x_6, x_7); +lean_dec(x_6); +lean_ctor_set(x_1, 2, x_8); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_4); +return x_1; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_9 = lean_ctor_get(x_1, 0); +x_10 = lean_ctor_get(x_1, 1); +x_11 = lean_ctor_get(x_1, 2); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_dec(x_1); +x_12 = lean_int_neg(x_11); +lean_dec(x_11); +x_13 = l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1; +x_14 = lean_int_sub(x_12, x_13); +lean_dec(x_12); +x_15 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_15, 0, x_10); +lean_ctor_set(x_15, 1, x_9); +lean_ctor_set(x_15, 2, x_14); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg), 1, 0); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ≤ ", 5, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" + ", 3, 3); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_2, 2); +lean_inc(x_3); +x_4 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1; +x_5 = lean_int_dec_lt(x_3, x_4); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_nat_abs(x_3); +lean_dec(x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_nat_dec_eq(x_6, x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_inc(x_1); +x_10 = lean_apply_1(x_1, x_9); +x_11 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_12 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +x_13 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_14 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +x_15 = lean_ctor_get(x_2, 1); +lean_inc(x_15); +lean_dec(x_2); +x_16 = lean_apply_1(x_1, x_15); +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_14); +lean_ctor_set(x_17, 1, x_16); +x_18 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6; +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = l___private_Init_Data_Repr_0__Nat_reprFast(x_6); +x_21 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_21, 0, x_20); +x_22 = l_Lean_MessageData_ofFormat(x_21); +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_19); +lean_ctor_set(x_23, 1, x_22); +x_24 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_11); +return x_24; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_6); +x_25 = lean_ctor_get(x_2, 0); +lean_inc(x_25); +lean_inc(x_1); +x_26 = lean_apply_1(x_1, x_25); +x_27 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +x_31 = lean_ctor_get(x_2, 1); +lean_inc(x_31); +lean_dec(x_2); +x_32 = lean_apply_1(x_1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_30); +lean_ctor_set(x_33, 1, x_32); +x_34 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_27); +return x_34; +} +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_35 = lean_nat_abs(x_3); +lean_dec(x_3); +x_36 = lean_unsigned_to_nat(1u); +x_37 = lean_nat_sub(x_35, x_36); +lean_dec(x_35); +x_38 = lean_ctor_get(x_2, 0); +lean_inc(x_38); +lean_inc(x_1); +x_39 = lean_apply_1(x_1, x_38); +x_40 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_39); +x_42 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6; +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +x_44 = lean_nat_add(x_37, x_36); +lean_dec(x_37); +x_45 = l___private_Init_Data_Repr_0__Nat_reprFast(x_44); +x_46 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_46, 0, x_45); +x_47 = l_Lean_MessageData_ofFormat(x_46); +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_43); +lean_ctor_set(x_48, 1, x_47); +x_49 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +x_51 = lean_ctor_get(x_2, 1); +lean_inc(x_51); +lean_dec(x_2); +x_52 = lean_apply_1(x_1, x_51); +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_50); +lean_ctor_set(x_53, 1, x_52); +x_54 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_40); +return x_54; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = lean_ctor_get(x_1, 2); +lean_inc(x_2); +x_3 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1; +x_4 = lean_int_dec_lt(x_2, x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_nat_abs(x_2); +lean_dec(x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_nat_dec_eq(x_5, x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_8 = lean_ctor_get(x_1, 0); +lean_inc(x_8); +x_9 = l_Lean_MessageData_ofExpr(x_8); +x_10 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_11 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_11, 0, x_10); +lean_ctor_set(x_11, 1, x_9); +x_12 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_13 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +lean_dec(x_1); +x_15 = l_Lean_MessageData_ofExpr(x_14); +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_13); +lean_ctor_set(x_16, 1, x_15); +x_17 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6; +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l___private_Init_Data_Repr_0__Nat_reprFast(x_5); +x_20 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_20, 0, x_19); +x_21 = l_Lean_MessageData_ofFormat(x_20); +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_18); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_10); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_5); +x_24 = lean_ctor_get(x_1, 0); +lean_inc(x_24); +x_25 = l_Lean_MessageData_ofExpr(x_24); +x_26 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +x_28 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +x_30 = lean_ctor_get(x_1, 1); +lean_inc(x_30); +lean_dec(x_1); +x_31 = l_Lean_MessageData_ofExpr(x_30); +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_29); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_26); +return x_33; +} +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_34 = lean_nat_abs(x_2); +lean_dec(x_2); +x_35 = lean_unsigned_to_nat(1u); +x_36 = lean_nat_sub(x_34, x_35); +lean_dec(x_34); +x_37 = lean_ctor_get(x_1, 0); +lean_inc(x_37); +x_38 = l_Lean_MessageData_ofExpr(x_37); +x_39 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +x_41 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = lean_nat_add(x_36, x_35); +lean_dec(x_36); +x_44 = l___private_Init_Data_Repr_0__Nat_reprFast(x_43); +x_45 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_45, 0, x_44); +x_46 = l_Lean_MessageData_ofFormat(x_45); +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_42); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4; +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = lean_ctor_get(x_1, 1); +lean_inc(x_50); +lean_dec(x_1); +x_51 = l_Lean_MessageData_ofExpr(x_50); +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_49); +lean_ctor_set(x_52, 1, x_51); +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_39); +return x_53; +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_Arith_Offset_toMessageData___at_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___spec__1), 1, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f_go(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +lean_inc(x_2); +x_4 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_2); +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_5; +lean_inc(x_3); +x_5 = l_Lean_Meta_Grind_Arith_isNatOffset_x3f(x_3); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; +lean_inc(x_2); +x_6 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_2); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +lean_inc(x_3); +x_7 = l_Lean_Meta_Grind_Arith_isNatNum_x3f(x_3); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_dec(x_1); +x_8 = l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1; +x_9 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_9, 0, x_2); +lean_ctor_set(x_9, 1, x_3); +lean_ctor_set(x_9, 2, x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; +} +else +{ +uint8_t x_11; +lean_dec(x_3); +x_11 = !lean_is_exclusive(x_7); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_7, 0); +x_13 = lean_nat_to_int(x_12); +x_14 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_14, 0, x_2); +lean_ctor_set(x_14, 1, x_1); +lean_ctor_set(x_14, 2, x_13); +lean_ctor_set(x_7, 0, x_14); +return x_7; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_7, 0); +lean_inc(x_15); +lean_dec(x_7); +x_16 = lean_nat_to_int(x_15); +x_17 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_17, 0, x_2); +lean_ctor_set(x_17, 1, x_1); +lean_ctor_set(x_17, 2, x_16); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_17); +return x_18; +} +} +} +else +{ +uint8_t x_19; +lean_dec(x_2); +x_19 = !lean_is_exclusive(x_6); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_6, 0); +x_21 = lean_nat_to_int(x_20); +x_22 = lean_int_neg(x_21); +lean_dec(x_21); +x_23 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_23, 0, x_1); +lean_ctor_set(x_23, 1, x_3); +lean_ctor_set(x_23, 2, x_22); +lean_ctor_set(x_6, 0, x_23); +return x_6; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_6, 0); +lean_inc(x_24); +lean_dec(x_6); +x_25 = lean_nat_to_int(x_24); +x_26 = lean_int_neg(x_25); +lean_dec(x_25); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_1); +lean_ctor_set(x_27, 1, x_3); +lean_ctor_set(x_27, 2, x_26); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_27); +return x_28; +} +} +} +else +{ +uint8_t x_29; +lean_dec(x_3); +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_5); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_5, 0); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = lean_nat_to_int(x_32); +x_34 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_34, 0, x_2); +lean_ctor_set(x_34, 1, x_31); +lean_ctor_set(x_34, 2, x_33); +lean_ctor_set(x_5, 0, x_34); +return x_5; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_35 = lean_ctor_get(x_5, 0); +lean_inc(x_35); +lean_dec(x_5); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_nat_to_int(x_37); +x_39 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_39, 0, x_2); +lean_ctor_set(x_39, 1, x_36); +lean_ctor_set(x_39, 2, x_38); +x_40 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_40, 0, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_2); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_4); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_42 = lean_ctor_get(x_4, 0); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = lean_nat_to_int(x_44); +x_46 = lean_int_neg(x_45); +lean_dec(x_45); +x_47 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_47, 0, x_43); +lean_ctor_set(x_47, 1, x_3); +lean_ctor_set(x_47, 2, x_46); +lean_ctor_set(x_4, 0, x_47); +return x_4; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_48 = lean_ctor_get(x_4, 0); +lean_inc(x_48); +lean_dec(x_4); +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_51 = lean_nat_to_int(x_50); +x_52 = lean_int_neg(x_51); +lean_dec(x_51); +x_53 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_53, 0, x_49); +lean_ctor_set(x_53, 1, x_3); +lean_ctor_set(x_53, 2, x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +return x_54; +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("LE", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1; +x_2 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint8_t x_4; +x_3 = l_Lean_Expr_cleanupAnnotations(x_1); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) +{ +lean_object* x_5; +lean_dec(x_3); +lean_dec(x_2); +x_5 = lean_box(0); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_7 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_8 = l_Lean_Expr_isApp(x_7); +if (x_8 == 0) +{ +lean_object* x_9; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_2); +x_9 = lean_box(0); +return x_9; +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = l_Lean_Expr_appArg(x_7, lean_box(0)); +x_11 = l_Lean_Expr_appFnCleanup(x_7, lean_box(0)); +x_12 = l_Lean_Expr_isApp(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_13 = lean_box(0); +return x_13; +} +else +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = l_Lean_Expr_appArg(x_11, lean_box(0)); +x_15 = l_Lean_Expr_appFnCleanup(x_11, lean_box(0)); +x_16 = l_Lean_Expr_isApp(x_15); +if (x_16 == 0) +{ +lean_object* x_17; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_17 = lean_box(0); +return x_17; +} +else +{ +lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_18 = l_Lean_Expr_appFnCleanup(x_15, lean_box(0)); +x_19 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3; +x_20 = l_Lean_Expr_isConstOf(x_18, x_19); +lean_dec(x_18); +if (x_20 == 0) +{ +lean_object* x_21; +lean_dec(x_14); +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_21 = lean_box(0); +return x_21; +} +else +{ +uint8_t x_22; +x_22 = l_Lean_Meta_Grind_Arith_isInstLENat(x_14); +lean_dec(x_14); +if (x_22 == 0) +{ +lean_object* x_23; +lean_dec(x_10); +lean_dec(x_6); +lean_dec(x_2); +x_23 = lean_box(0); +return x_23; +} +else +{ +lean_object* x_24; +x_24 = l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f_go(x_2, x_10, x_6); +return x_24; +} +} +} +} +} +} +} +} +lean_object* initialize_Lean_Expr(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Message(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Util(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Expr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Lean_Message(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Meta_Grind_Arith_isNatType___closed__1 = _init_l_Lean_Meta_Grind_Arith_isNatType___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatType___closed__1); +l_Lean_Meta_Grind_Arith_isNatType___closed__2 = _init_l_Lean_Meta_Grind_Arith_isNatType___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatType___closed__2); +l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1 = _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstAddNat___closed__1); +l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2 = _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstAddNat___closed__2); +l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3 = _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstAddNat___closed__3); +l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4 = _init_l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstAddNat___closed__4); +l_Lean_Meta_Grind_Arith_isInstLENat___closed__1 = _init_l_Lean_Meta_Grind_Arith_isInstLENat___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstLENat___closed__1); +l_Lean_Meta_Grind_Arith_isInstLENat___closed__2 = _init_l_Lean_Meta_Grind_Arith_isInstLENat___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isInstLENat___closed__2); +l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1 = _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__1); +l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2 = _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__2); +l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3 = _init_l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatAdd_x3f___closed__3); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__1); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__2); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__3); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__4); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___lambda__3___closed__5); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__1); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__2); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__3); +l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4 = _init_l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatNum_x3f___closed__4); +l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_instInhabitedCnstr___rarg___closed__1); +l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_Cnstr_neg___rarg___closed__1); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__1); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__2); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__3); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__4); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__5); +l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6 = _init_l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_Offset_toMessageData___rarg___closed__6); +l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1 = _init_l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr___closed__1); +l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr = _init_l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_instToMessageDataCnstrExpr); +l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1 = _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__1); +l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2 = _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__2); +l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3 = _init_l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Arith_isNatOffsetCnstr_x3f___closed__3); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Canon.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Canon.c index b1a5fae1b06b..4330b8f13ba3 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Canon.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Canon.c @@ -16266,7 +16266,7 @@ static lean_object* _init_l_Lean_Meta_Grind_Canon_canonImpl_visit___lambda__3___ lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_Canon_canonImpl_visit___lambda__3___closed__1; x_2 = l_Lean_Meta_Grind_Canon_canonImpl_visit___lambda__3___closed__2; -x_3 = lean_unsigned_to_nat(190u); +x_3 = lean_unsigned_to_nat(192u); x_4 = lean_unsigned_to_nat(13u); x_5 = l_Lean_Meta_Grind_Canon_canonImpl_visit___lambda__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Combinators.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Combinators.c index a1cc45a523d7..685bc0cc9b0f 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Combinators.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Combinators.c @@ -1191,7 +1191,7 @@ if (lean_obj_tag(x_17) == 0) lean_object* x_18; uint8_t x_19; x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -x_19 = lean_ctor_get_uint8(x_18, sizeof(void*)*20); +x_19 = lean_ctor_get_uint8(x_18, sizeof(void*)*23); if (x_19 == 0) { uint8_t x_20; diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Core.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Core.c index a061c68ec77f..3f08910f71da 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Core.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Core.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind.Core -// Imports: Init.Grind.Util Lean.Meta.LitValues Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Inv Lean.Meta.Tactic.Grind.PP Lean.Meta.Tactic.Grind.Ctor Lean.Meta.Tactic.Grind.Internalize +// Imports: Init.Grind.Util Lean.Meta.LitValues Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Inv Lean.Meta.Tactic.Grind.PP Lean.Meta.Tactic.Grind.Ctor Lean.Meta.Tactic.Grind.Util Lean.Meta.Tactic.Grind.Internalize #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -19,16 +19,17 @@ static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Gr static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__3; static lean_object* l_Lean_Meta_Grind_add___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__5; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -36,6 +37,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_a LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -43,6 +45,8 @@ lean_object* l_Lean_Meta_Grind_propagateCtor(lean_object*, lean_object*, lean_ob uint8_t l_Lean_Expr_isApp(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_Grind_isCongruent(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_checkSystem(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; @@ -61,13 +65,14 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tact LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents___spec__1___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_setENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goFact(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse___closed__4; lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -79,13 +84,14 @@ lean_object* l_Lean_Meta_Grind_propagateUp(lean_object*, lean_object*, lean_obje LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqMP(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getFalseExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -106,9 +112,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Gr LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addNewEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_closeGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -126,9 +132,9 @@ lean_object* l_Lean_Meta_Grind_addCongrTable(lean_object*, lean_object*, lean_ob LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_checkInvariants(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_ppState(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,7 +143,7 @@ static size_t l_Lean_PersistentHashMap_eraseAux___at___private_Lean_Meta_Tactic_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); @@ -145,48 +151,52 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Gr static lean_object* l_Lean_Meta_Grind_add___closed__2; lean_object* l_Lean_Meta_Grind_getParents(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1; +lean_object* lean_process_new_offset_eq_lit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___closed__1; lean_object* l_Lean_Meta_Grind_updateLastTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__10; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents___spec__1___closed__2; lean_object* l_Lean_MessageData_ofExpr(lean_object*); lean_object* l_Lean_Meta_Grind_copyParentsTo(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addHypothesis(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_ppState(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_grind_mk_eq_proof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_process_new_offset_eq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2___boxed(lean_object**); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__6; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__4; lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__6; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_markAsInconsistent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_isNatNum(lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -195,20 +205,21 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Gr static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_eraseAux___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isProp(lean_object*); static lean_object* l_Lean_Meta_Grind_add_go___closed__2; -lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__4; lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___boxed(lean_object**); lean_object* l_Lean_Meta_Grind_ppENodeRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__8; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); lean_object* l_Lean_Meta_Grind_getParentsAndReset(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isTrue(lean_object*); +static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -219,6 +230,7 @@ LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_Tactic_Grin lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_add_go___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -227,22 +239,24 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Gr static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__2; lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__7; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goFact___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__9; lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6___boxed(lean_object**); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__13; static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse___closed__3; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_propagateOffsetEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_add___lambda__3___closed__2; lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__2; -lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__14; @@ -261,25 +275,27 @@ x_18 = lean_ctor_get(x_1, 4); lean_dec(x_18); lean_ctor_set(x_1, 5, x_3); lean_ctor_set(x_1, 4, x_2); -lean_ctor_set_uint8(x_1, sizeof(void*)*10, x_4); +lean_ctor_set_uint8(x_1, sizeof(void*)*11, x_4); x_19 = l_Lean_Meta_Grind_setENode(x_5, x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); return x_19; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; uint8_t x_26; uint8_t x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; uint8_t x_26; uint8_t x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; x_20 = lean_ctor_get(x_1, 0); x_21 = lean_ctor_get(x_1, 1); x_22 = lean_ctor_get(x_1, 2); x_23 = lean_ctor_get(x_1, 3); x_24 = lean_ctor_get(x_1, 6); -x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 1); -x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 2); -x_27 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 3); -x_28 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 4); +x_25 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 1); +x_26 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 2); +x_27 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 3); +x_28 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 4); x_29 = lean_ctor_get(x_1, 7); x_30 = lean_ctor_get(x_1, 8); x_31 = lean_ctor_get(x_1, 9); +x_32 = lean_ctor_get(x_1, 10); +lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); @@ -289,255 +305,262 @@ lean_inc(x_22); lean_inc(x_21); lean_inc(x_20); lean_dec(x_1); -x_32 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_32, 0, x_20); -lean_ctor_set(x_32, 1, x_21); -lean_ctor_set(x_32, 2, x_22); -lean_ctor_set(x_32, 3, x_23); -lean_ctor_set(x_32, 4, x_2); -lean_ctor_set(x_32, 5, x_3); -lean_ctor_set(x_32, 6, x_24); -lean_ctor_set(x_32, 7, x_29); -lean_ctor_set(x_32, 8, x_30); -lean_ctor_set(x_32, 9, x_31); -lean_ctor_set_uint8(x_32, sizeof(void*)*10, x_4); -lean_ctor_set_uint8(x_32, sizeof(void*)*10 + 1, x_25); -lean_ctor_set_uint8(x_32, sizeof(void*)*10 + 2, x_26); -lean_ctor_set_uint8(x_32, sizeof(void*)*10 + 3, x_27); -lean_ctor_set_uint8(x_32, sizeof(void*)*10 + 4, x_28); -x_33 = l_Lean_Meta_Grind_setENode(x_5, x_32, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -return x_33; +x_33 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_33, 0, x_20); +lean_ctor_set(x_33, 1, x_21); +lean_ctor_set(x_33, 2, x_22); +lean_ctor_set(x_33, 3, x_23); +lean_ctor_set(x_33, 4, x_2); +lean_ctor_set(x_33, 5, x_3); +lean_ctor_set(x_33, 6, x_24); +lean_ctor_set(x_33, 7, x_29); +lean_ctor_set(x_33, 8, x_30); +lean_ctor_set(x_33, 9, x_31); +lean_ctor_set(x_33, 10, x_32); +lean_ctor_set_uint8(x_33, sizeof(void*)*11, x_4); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 1, x_25); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 2, x_26); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 3, x_27); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 4, x_28); +x_34 = l_Lean_Meta_Grind_setENode(x_5, x_33, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +return x_34; } } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_14; -lean_inc(x_1); -x_14 = l_Lean_Meta_Grind_getENode(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_st_ref_get(x_5, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -x_16 = lean_ctor_get(x_15, 4); +x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); -if (lean_obj_tag(x_16) == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); lean_dec(x_14); -x_18 = lean_box(0); -x_19 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_15, x_3, x_4, x_2, x_1, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -return x_19; +lean_inc(x_1); +x_17 = l_Lean_Meta_Grind_Goal_getENode(x_15, x_1, x_11, x_12, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_18, 4); +lean_inc(x_19); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = lean_box(0); +x_22 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_18, x_3, x_4, x_2, x_1, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +return x_22; } else { -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_dec(x_14); -x_21 = lean_ctor_get(x_15, 5); -lean_inc(x_21); -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) +lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_dec(x_17); +x_24 = lean_ctor_get(x_18, 5); +lean_inc(x_24); +x_25 = !lean_is_exclusive(x_19); +if (x_25 == 0) { -uint8_t x_23; lean_object* x_24; -x_23 = lean_ctor_get_uint8(x_15, sizeof(void*)*10); -x_24 = lean_ctor_get(x_16, 0); +uint8_t x_26; lean_object* x_27; +x_26 = lean_ctor_get_uint8(x_18, sizeof(void*)*11); +x_27 = lean_ctor_get(x_19, 0); lean_inc(x_1); -lean_ctor_set(x_16, 0, x_1); -if (x_23 == 0) +lean_ctor_set(x_19, 0, x_1); +if (x_26 == 0) { -uint8_t x_25; lean_object* x_26; -x_25 = 1; -x_26 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_24, x_25, x_16, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_26) == 0) +uint8_t x_28; lean_object* x_29; +x_28 = 1; +x_29 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_27, x_28, x_19, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_15, x_3, x_4, x_2, x_1, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); -lean_dec(x_27); -return x_29; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_18, x_3, x_4, x_2, x_1, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_31); +lean_dec(x_30); +return x_32; } else { -uint8_t x_30; -lean_dec(x_15); +uint8_t x_33; +lean_dec(x_18); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) +x_33 = !lean_is_exclusive(x_29); +if (x_33 == 0) { -return x_26; +return x_29; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_29, 0); +x_35 = lean_ctor_get(x_29, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_29); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } else { -uint8_t x_34; lean_object* x_35; -x_34 = 0; -x_35 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_24, x_34, x_16, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_35) == 0) +uint8_t x_37; lean_object* x_38; +x_37 = 0; +x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_27, x_37, x_19, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_15, x_3, x_4, x_2, x_1, x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); -lean_dec(x_36); -return x_38; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_18, x_3, x_4, x_2, x_1, x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_40); +lean_dec(x_39); +return x_41; } else { -uint8_t x_39; -lean_dec(x_15); +uint8_t x_42; +lean_dec(x_18); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_35); -if (x_39 == 0) +x_42 = !lean_is_exclusive(x_38); +if (x_42 == 0) { -return x_35; +return x_38; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_35, 0); -x_41 = lean_ctor_get(x_35, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_35); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_40); -lean_ctor_set(x_42, 1, x_41); -return x_42; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_38, 0); +x_44 = lean_ctor_get(x_38, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_38); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } } else { -uint8_t x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get_uint8(x_15, sizeof(void*)*10); -x_44 = lean_ctor_get(x_16, 0); -lean_inc(x_44); -lean_dec(x_16); +uint8_t x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get_uint8(x_18, sizeof(void*)*11); +x_47 = lean_ctor_get(x_19, 0); +lean_inc(x_47); +lean_dec(x_19); lean_inc(x_1); -x_45 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_45, 0, x_1); -if (x_43 == 0) +x_48 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_48, 0, x_1); +if (x_46 == 0) { -uint8_t x_46; lean_object* x_47; -x_46 = 1; -x_47 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_44, x_46, x_45, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_47) == 0) +uint8_t x_49; lean_object* x_50; +x_49 = 1; +x_50 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_47, x_49, x_48, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -lean_dec(x_47); -x_50 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_15, x_3, x_4, x_2, x_1, x_48, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_49); -lean_dec(x_48); -return x_50; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_18, x_3, x_4, x_2, x_1, x_51, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_52); +lean_dec(x_51); +return x_53; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -lean_dec(x_15); +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_dec(x_18); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_51 = lean_ctor_get(x_47, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_47, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_53 = x_47; +x_54 = lean_ctor_get(x_50, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_50, 1); +lean_inc(x_55); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_56 = x_50; } else { - lean_dec_ref(x_47); - x_53 = lean_box(0); + lean_dec_ref(x_50); + x_56 = lean_box(0); } -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_56)) { + x_57 = lean_alloc_ctor(1, 2, 0); } else { - x_54 = x_53; + x_57 = x_56; } -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_52); -return x_54; +lean_ctor_set(x_57, 0, x_54); +lean_ctor_set(x_57, 1, x_55); +return x_57; } } else { -uint8_t x_55; lean_object* x_56; -x_55 = 0; -x_56 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_44, x_55, x_45, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_56) == 0) +uint8_t x_58; lean_object* x_59; +x_58 = 0; +x_59 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go(x_47, x_58, x_48, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_15, x_3, x_4, x_2, x_1, x_57, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_58); -lean_dec(x_57); -return x_59; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_62 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans_go___lambda__1(x_18, x_3, x_4, x_2, x_1, x_60, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_61); +lean_dec(x_60); +return x_62; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -lean_dec(x_15); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +lean_dec(x_18); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_60 = lean_ctor_get(x_56, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_56, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_56)) { - lean_ctor_release(x_56, 0); - lean_ctor_release(x_56, 1); - x_62 = x_56; +x_63 = lean_ctor_get(x_59, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_59, 1); +lean_inc(x_64); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_65 = x_59; } else { - lean_dec_ref(x_56); - x_62 = lean_box(0); + lean_dec_ref(x_59); + x_65 = lean_box(0); } -if (lean_is_scalar(x_62)) { - x_63 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_65)) { + x_66 = lean_alloc_ctor(1, 2, 0); } else { - x_63 = x_62; + x_66 = x_65; } -lean_ctor_set(x_63, 0, x_60); -lean_ctor_set(x_63, 1, x_61); -return x_63; +lean_ctor_set(x_66, 0, x_63); +lean_ctor_set(x_66, 1, x_64); +return x_66; } } } @@ -545,27 +568,27 @@ return x_63; } else { -uint8_t x_64; +uint8_t x_67; lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_64 = !lean_is_exclusive(x_14); -if (x_64 == 0) +x_67 = !lean_is_exclusive(x_17); +if (x_67 == 0) { -return x_14; +return x_17; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_14, 0); -x_66 = lean_ctor_get(x_14, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_14); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_17, 0); +x_69 = lean_ctor_get(x_17, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_17); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } } @@ -637,7 +660,7 @@ LEAN_EXPORT lean_object* l_Array_indexOfAux___at___private_Lean_Meta_Tactic_Grin _start: { lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_1, 2); lean_inc(x_5); x_6 = lean_array_get_size(x_2); x_7 = lean_nat_dec_lt(x_4, x_6); @@ -707,7 +730,7 @@ if (lean_obj_tag(x_2) == 0) lean_object* x_5; lean_object* x_6; size_t x_7; size_t x_8; size_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; x_5 = lean_ctor_get(x_2, 0); lean_inc(x_5); -x_6 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_1, 2); lean_inc(x_6); x_7 = 5; x_8 = l_Lean_PersistentHashMap_eraseAux___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__2___closed__2; @@ -1012,7 +1035,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at___private_Lean_Meta _start: { lean_object* x_4; uint64_t x_5; size_t x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); lean_inc(x_4); lean_inc(x_3); x_5 = l_Lean_Meta_Grind_congrHash(x_4, x_3); @@ -1034,7 +1057,7 @@ return x_2; LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; x_12 = lean_st_ref_take(x_3, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); @@ -1053,9 +1076,9 @@ x_19 = lean_ctor_get(x_13, 4); lean_inc(x_19); x_20 = lean_ctor_get(x_13, 5); lean_inc(x_20); -x_21 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_22 = lean_ctor_get(x_13, 6); -lean_inc(x_22); +x_21 = lean_ctor_get(x_13, 6); +lean_inc(x_21); +x_22 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_23 = lean_ctor_get(x_13, 7); lean_inc(x_23); x_24 = lean_ctor_get(x_13, 8); @@ -1082,123 +1105,138 @@ x_34 = lean_ctor_get(x_13, 18); lean_inc(x_34); x_35 = lean_ctor_get(x_13, 19); lean_inc(x_35); +x_36 = lean_ctor_get(x_13, 20); +lean_inc(x_36); +x_37 = lean_ctor_get(x_13, 21); +lean_inc(x_37); +x_38 = lean_ctor_get(x_13, 22); +lean_inc(x_38); lean_inc(x_13); -x_36 = l_Lean_PersistentHashMap_erase___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__1(x_13, x_18, x_1); -x_37 = !lean_is_exclusive(x_13); -if (x_37 == 0) +x_39 = l_Lean_PersistentHashMap_erase___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__1(x_13, x_19, x_1); +x_40 = !lean_is_exclusive(x_13); +if (x_40 == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_38 = lean_ctor_get(x_13, 19); -lean_dec(x_38); -x_39 = lean_ctor_get(x_13, 18); -lean_dec(x_39); -x_40 = lean_ctor_get(x_13, 17); -lean_dec(x_40); -x_41 = lean_ctor_get(x_13, 16); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; +x_41 = lean_ctor_get(x_13, 22); lean_dec(x_41); -x_42 = lean_ctor_get(x_13, 15); +x_42 = lean_ctor_get(x_13, 21); lean_dec(x_42); -x_43 = lean_ctor_get(x_13, 14); +x_43 = lean_ctor_get(x_13, 20); lean_dec(x_43); -x_44 = lean_ctor_get(x_13, 13); +x_44 = lean_ctor_get(x_13, 19); lean_dec(x_44); -x_45 = lean_ctor_get(x_13, 12); +x_45 = lean_ctor_get(x_13, 18); lean_dec(x_45); -x_46 = lean_ctor_get(x_13, 11); +x_46 = lean_ctor_get(x_13, 17); lean_dec(x_46); -x_47 = lean_ctor_get(x_13, 10); +x_47 = lean_ctor_get(x_13, 16); lean_dec(x_47); -x_48 = lean_ctor_get(x_13, 9); +x_48 = lean_ctor_get(x_13, 15); lean_dec(x_48); -x_49 = lean_ctor_get(x_13, 8); +x_49 = lean_ctor_get(x_13, 14); lean_dec(x_49); -x_50 = lean_ctor_get(x_13, 7); +x_50 = lean_ctor_get(x_13, 13); lean_dec(x_50); -x_51 = lean_ctor_get(x_13, 6); +x_51 = lean_ctor_get(x_13, 12); lean_dec(x_51); -x_52 = lean_ctor_get(x_13, 5); +x_52 = lean_ctor_get(x_13, 11); lean_dec(x_52); -x_53 = lean_ctor_get(x_13, 4); +x_53 = lean_ctor_get(x_13, 10); lean_dec(x_53); -x_54 = lean_ctor_get(x_13, 3); +x_54 = lean_ctor_get(x_13, 9); lean_dec(x_54); -x_55 = lean_ctor_get(x_13, 2); +x_55 = lean_ctor_get(x_13, 8); lean_dec(x_55); -x_56 = lean_ctor_get(x_13, 1); +x_56 = lean_ctor_get(x_13, 7); lean_dec(x_56); -x_57 = lean_ctor_get(x_13, 0); +x_57 = lean_ctor_get(x_13, 6); lean_dec(x_57); -lean_ctor_set(x_13, 3, x_36); -x_58 = lean_st_ref_set(x_3, x_13, x_14); -x_59 = !lean_is_exclusive(x_58); -if (x_59 == 0) -{ -lean_object* x_60; lean_object* x_61; -x_60 = lean_ctor_get(x_58, 0); +x_58 = lean_ctor_get(x_13, 5); +lean_dec(x_58); +x_59 = lean_ctor_get(x_13, 4); +lean_dec(x_59); +x_60 = lean_ctor_get(x_13, 3); lean_dec(x_60); -x_61 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; -lean_ctor_set(x_58, 0, x_61); -return x_58; +x_61 = lean_ctor_get(x_13, 2); +lean_dec(x_61); +x_62 = lean_ctor_get(x_13, 1); +lean_dec(x_62); +x_63 = lean_ctor_get(x_13, 0); +lean_dec(x_63); +lean_ctor_set(x_13, 4, x_39); +x_64 = lean_st_ref_set(x_3, x_13, x_14); +x_65 = !lean_is_exclusive(x_64); +if (x_65 == 0) +{ +lean_object* x_66; lean_object* x_67; +x_66 = lean_ctor_get(x_64, 0); +lean_dec(x_66); +x_67 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; +lean_ctor_set(x_64, 0, x_67); +return x_64; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_58, 1); -lean_inc(x_62); -lean_dec(x_58); -x_63 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_62); -return x_64; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_64, 1); +lean_inc(x_68); +lean_dec(x_64); +x_69 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_68); +return x_70; } } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_dec(x_13); -x_65 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_65, 0, x_15); -lean_ctor_set(x_65, 1, x_16); -lean_ctor_set(x_65, 2, x_17); -lean_ctor_set(x_65, 3, x_36); -lean_ctor_set(x_65, 4, x_19); -lean_ctor_set(x_65, 5, x_20); -lean_ctor_set(x_65, 6, x_22); -lean_ctor_set(x_65, 7, x_23); -lean_ctor_set(x_65, 8, x_24); -lean_ctor_set(x_65, 9, x_25); -lean_ctor_set(x_65, 10, x_26); -lean_ctor_set(x_65, 11, x_27); -lean_ctor_set(x_65, 12, x_28); -lean_ctor_set(x_65, 13, x_29); -lean_ctor_set(x_65, 14, x_30); -lean_ctor_set(x_65, 15, x_31); -lean_ctor_set(x_65, 16, x_32); -lean_ctor_set(x_65, 17, x_33); -lean_ctor_set(x_65, 18, x_34); -lean_ctor_set(x_65, 19, x_35); -lean_ctor_set_uint8(x_65, sizeof(void*)*20, x_21); -x_66 = lean_st_ref_set(x_3, x_65, x_14); -x_67 = lean_ctor_get(x_66, 1); -lean_inc(x_67); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_68 = x_66; +x_71 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_71, 0, x_15); +lean_ctor_set(x_71, 1, x_16); +lean_ctor_set(x_71, 2, x_17); +lean_ctor_set(x_71, 3, x_18); +lean_ctor_set(x_71, 4, x_39); +lean_ctor_set(x_71, 5, x_20); +lean_ctor_set(x_71, 6, x_21); +lean_ctor_set(x_71, 7, x_23); +lean_ctor_set(x_71, 8, x_24); +lean_ctor_set(x_71, 9, x_25); +lean_ctor_set(x_71, 10, x_26); +lean_ctor_set(x_71, 11, x_27); +lean_ctor_set(x_71, 12, x_28); +lean_ctor_set(x_71, 13, x_29); +lean_ctor_set(x_71, 14, x_30); +lean_ctor_set(x_71, 15, x_31); +lean_ctor_set(x_71, 16, x_32); +lean_ctor_set(x_71, 17, x_33); +lean_ctor_set(x_71, 18, x_34); +lean_ctor_set(x_71, 19, x_35); +lean_ctor_set(x_71, 20, x_36); +lean_ctor_set(x_71, 21, x_37); +lean_ctor_set(x_71, 22, x_38); +lean_ctor_set_uint8(x_71, sizeof(void*)*23, x_22); +x_72 = lean_st_ref_set(x_3, x_71, x_14); +x_73 = lean_ctor_get(x_72, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_72)) { + lean_ctor_release(x_72, 0); + lean_ctor_release(x_72, 1); + x_74 = x_72; } else { - lean_dec_ref(x_66); - x_68 = lean_box(0); + lean_dec_ref(x_72); + x_74 = lean_box(0); } -x_69 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; -if (lean_is_scalar(x_68)) { - x_70 = lean_alloc_ctor(0, 2, 0); +x_75 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___lambda__1___closed__1; +if (lean_is_scalar(x_74)) { + x_76 = lean_alloc_ctor(0, 2, 0); } else { - x_70 = x_68; + x_76 = x_74; } -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_67); -return x_70; +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_73); +return x_76; } } } @@ -3104,275 +3142,287 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_dec(x_19); x_24 = lean_ctor_get(x_18, 1); lean_inc(x_24); lean_dec(x_18); -lean_inc(x_16); -x_25 = l_Lean_Meta_Grind_getENode(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24); -if (lean_obj_tag(x_25) == 0) -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_st_ref_get(x_4, x_24); x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); x_27 = lean_ctor_get(x_25, 1); lean_inc(x_27); lean_dec(x_25); -x_28 = !lean_is_exclusive(x_26); -if (x_28 == 0) +lean_inc(x_16); +x_28 = l_Lean_Meta_Grind_Goal_getENode(x_26, x_16, x_10, x_11, x_27); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_29 = lean_ctor_get(x_26, 0); -x_30 = lean_ctor_get(x_26, 1); -x_31 = lean_ctor_get(x_26, 2); -x_32 = lean_ctor_get(x_26, 3); -x_33 = lean_ctor_get(x_26, 4); -x_34 = lean_ctor_get(x_26, 5); -x_35 = lean_ctor_get(x_26, 6); -x_36 = lean_ctor_get(x_26, 7); -x_37 = lean_ctor_get(x_26, 8); -x_38 = lean_ctor_get(x_26, 9); -x_39 = lean_nat_dec_lt(x_38, x_1); -lean_dec(x_38); -if (x_39 == 0) +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = !lean_is_exclusive(x_29); +if (x_31 == 0) { -lean_object* x_40; -lean_free_object(x_26); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +x_32 = lean_ctor_get(x_29, 0); +x_33 = lean_ctor_get(x_29, 1); +x_34 = lean_ctor_get(x_29, 2); +x_35 = lean_ctor_get(x_29, 3); +x_36 = lean_ctor_get(x_29, 4); +x_37 = lean_ctor_get(x_29, 5); +x_38 = lean_ctor_get(x_29, 6); +x_39 = lean_ctor_get(x_29, 7); +x_40 = lean_ctor_get(x_29, 8); +x_41 = lean_ctor_get(x_29, 9); +x_42 = lean_ctor_get(x_29, 10); +x_43 = lean_nat_dec_lt(x_41, x_1); +lean_dec(x_41); +if (x_43 == 0) +{ +lean_object* x_44; +lean_free_object(x_29); +lean_dec(x_42); +lean_dec(x_40); +lean_dec(x_39); +lean_dec(x_38); lean_dec(x_37); lean_dec(x_36); lean_dec(x_35); lean_dec(x_34); lean_dec(x_33); lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); lean_dec(x_16); -x_40 = lean_box(0); +x_44 = lean_box(0); x_2 = x_17; -x_3 = x_40; -x_12 = x_27; +x_3 = x_44; +x_12 = x_30; goto _start; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_inc(x_1); -lean_ctor_set(x_26, 9, x_1); +lean_ctor_set(x_29, 9, x_1); lean_inc(x_16); -x_42 = l_Lean_Meta_Grind_setENode(x_16, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_43); +x_46 = l_Lean_Meta_Grind_setENode(x_16, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +x_48 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); lean_dec(x_16); -if (lean_obj_tag(x_44) == 0) +if (lean_obj_tag(x_48) == 0) { -lean_object* x_45; lean_object* x_46; -x_45 = lean_ctor_get(x_44, 1); -lean_inc(x_45); -lean_dec(x_44); -x_46 = lean_box(0); +lean_object* x_49; lean_object* x_50; +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = lean_box(0); x_2 = x_17; -x_3 = x_46; -x_12 = x_45; +x_3 = x_50; +x_12 = x_49; goto _start; } else { -uint8_t x_48; +uint8_t x_52; lean_dec(x_17); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_44); -if (x_48 == 0) +x_52 = !lean_is_exclusive(x_48); +if (x_52 == 0) { -return x_44; +return x_48; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_44, 0); -x_50 = lean_ctor_get(x_44, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_44); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_48, 0); +x_54 = lean_ctor_get(x_48, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_48); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; uint8_t x_60; uint8_t x_61; uint8_t x_62; uint8_t x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_52 = lean_ctor_get(x_26, 0); -x_53 = lean_ctor_get(x_26, 1); -x_54 = lean_ctor_get(x_26, 2); -x_55 = lean_ctor_get(x_26, 3); -x_56 = lean_ctor_get(x_26, 4); -x_57 = lean_ctor_get(x_26, 5); -x_58 = lean_ctor_get_uint8(x_26, sizeof(void*)*10); -x_59 = lean_ctor_get(x_26, 6); -x_60 = lean_ctor_get_uint8(x_26, sizeof(void*)*10 + 1); -x_61 = lean_ctor_get_uint8(x_26, sizeof(void*)*10 + 2); -x_62 = lean_ctor_get_uint8(x_26, sizeof(void*)*10 + 3); -x_63 = lean_ctor_get_uint8(x_26, sizeof(void*)*10 + 4); -x_64 = lean_ctor_get(x_26, 7); -x_65 = lean_ctor_get(x_26, 8); -x_66 = lean_ctor_get(x_26, 9); -lean_inc(x_66); -lean_inc(x_65); -lean_inc(x_64); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; uint8_t x_64; uint8_t x_65; uint8_t x_66; uint8_t x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; +x_56 = lean_ctor_get(x_29, 0); +x_57 = lean_ctor_get(x_29, 1); +x_58 = lean_ctor_get(x_29, 2); +x_59 = lean_ctor_get(x_29, 3); +x_60 = lean_ctor_get(x_29, 4); +x_61 = lean_ctor_get(x_29, 5); +x_62 = lean_ctor_get_uint8(x_29, sizeof(void*)*11); +x_63 = lean_ctor_get(x_29, 6); +x_64 = lean_ctor_get_uint8(x_29, sizeof(void*)*11 + 1); +x_65 = lean_ctor_get_uint8(x_29, sizeof(void*)*11 + 2); +x_66 = lean_ctor_get_uint8(x_29, sizeof(void*)*11 + 3); +x_67 = lean_ctor_get_uint8(x_29, sizeof(void*)*11 + 4); +x_68 = lean_ctor_get(x_29, 7); +x_69 = lean_ctor_get(x_29, 8); +x_70 = lean_ctor_get(x_29, 9); +x_71 = lean_ctor_get(x_29, 10); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_63); +lean_inc(x_61); +lean_inc(x_60); lean_inc(x_59); +lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_26); -x_67 = lean_nat_dec_lt(x_66, x_1); -lean_dec(x_66); -if (x_67 == 0) +lean_dec(x_29); +x_72 = lean_nat_dec_lt(x_70, x_1); +lean_dec(x_70); +if (x_72 == 0) { -lean_object* x_68; -lean_dec(x_65); -lean_dec(x_64); +lean_object* x_73; +lean_dec(x_71); +lean_dec(x_69); +lean_dec(x_68); +lean_dec(x_63); +lean_dec(x_61); +lean_dec(x_60); lean_dec(x_59); +lean_dec(x_58); lean_dec(x_57); lean_dec(x_56); -lean_dec(x_55); -lean_dec(x_54); -lean_dec(x_53); -lean_dec(x_52); lean_dec(x_16); -x_68 = lean_box(0); +x_73 = lean_box(0); x_2 = x_17; -x_3 = x_68; -x_12 = x_27; +x_3 = x_73; +x_12 = x_30; goto _start; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_inc(x_1); -x_70 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_70, 0, x_52); -lean_ctor_set(x_70, 1, x_53); -lean_ctor_set(x_70, 2, x_54); -lean_ctor_set(x_70, 3, x_55); -lean_ctor_set(x_70, 4, x_56); -lean_ctor_set(x_70, 5, x_57); -lean_ctor_set(x_70, 6, x_59); -lean_ctor_set(x_70, 7, x_64); -lean_ctor_set(x_70, 8, x_65); -lean_ctor_set(x_70, 9, x_1); -lean_ctor_set_uint8(x_70, sizeof(void*)*10, x_58); -lean_ctor_set_uint8(x_70, sizeof(void*)*10 + 1, x_60); -lean_ctor_set_uint8(x_70, sizeof(void*)*10 + 2, x_61); -lean_ctor_set_uint8(x_70, sizeof(void*)*10 + 3, x_62); -lean_ctor_set_uint8(x_70, sizeof(void*)*10 + 4, x_63); +x_75 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_75, 0, x_56); +lean_ctor_set(x_75, 1, x_57); +lean_ctor_set(x_75, 2, x_58); +lean_ctor_set(x_75, 3, x_59); +lean_ctor_set(x_75, 4, x_60); +lean_ctor_set(x_75, 5, x_61); +lean_ctor_set(x_75, 6, x_63); +lean_ctor_set(x_75, 7, x_68); +lean_ctor_set(x_75, 8, x_69); +lean_ctor_set(x_75, 9, x_1); +lean_ctor_set(x_75, 10, x_71); +lean_ctor_set_uint8(x_75, sizeof(void*)*11, x_62); +lean_ctor_set_uint8(x_75, sizeof(void*)*11 + 1, x_64); +lean_ctor_set_uint8(x_75, sizeof(void*)*11 + 2, x_65); +lean_ctor_set_uint8(x_75, sizeof(void*)*11 + 3, x_66); +lean_ctor_set_uint8(x_75, sizeof(void*)*11 + 4, x_67); lean_inc(x_16); -x_71 = l_Lean_Meta_Grind_setENode(x_16, x_70, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -lean_dec(x_71); -x_73 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_72); +x_76 = l_Lean_Meta_Grind_setENode(x_16, x_75, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); +x_78 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_16, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_77); lean_dec(x_16); -if (lean_obj_tag(x_73) == 0) +if (lean_obj_tag(x_78) == 0) { -lean_object* x_74; lean_object* x_75; -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -lean_dec(x_73); -x_75 = lean_box(0); +lean_object* x_79; lean_object* x_80; +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = lean_box(0); x_2 = x_17; -x_3 = x_75; -x_12 = x_74; +x_3 = x_80; +x_12 = x_79; goto _start; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_dec(x_17); lean_dec(x_1); -x_77 = lean_ctor_get(x_73, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_73, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_79 = x_73; +x_82 = lean_ctor_get(x_78, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_78, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_84 = x_78; } else { - lean_dec_ref(x_73); - x_79 = lean_box(0); + lean_dec_ref(x_78); + x_84 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_79; + x_85 = x_84; } -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_85, 0, x_82); +lean_ctor_set(x_85, 1, x_83); +return x_85; } } } } else { -uint8_t x_81; +uint8_t x_86; lean_dec(x_17); lean_dec(x_16); lean_dec(x_1); -x_81 = !lean_is_exclusive(x_25); -if (x_81 == 0) +x_86 = !lean_is_exclusive(x_28); +if (x_86 == 0) { -return x_25; +return x_28; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_25, 0); -x_83 = lean_ctor_get(x_25, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_25); -x_84 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_84, 0, x_82); -lean_ctor_set(x_84, 1, x_83); -return x_84; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_28, 0); +x_88 = lean_ctor_get(x_28, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_28); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +return x_89; } } } } else { -uint8_t x_85; +uint8_t x_90; lean_dec(x_17); lean_dec(x_16); lean_dec(x_1); -x_85 = !lean_is_exclusive(x_18); -if (x_85 == 0) +x_90 = !lean_is_exclusive(x_18); +if (x_90 == 0) { return x_18; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_18, 0); -x_87 = lean_ctor_get(x_18, 1); -lean_inc(x_87); -lean_inc(x_86); +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_18, 0); +x_92 = lean_ctor_get(x_18, 1); +lean_inc(x_92); +lean_inc(x_91); lean_dec(x_18); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +return x_93; } } } @@ -3388,7 +3438,7 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 6); +x_14 = lean_ctor_get(x_12, 7); lean_inc(x_14); lean_dec(x_12); x_15 = l_Lean_Meta_Grind_getParents(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); @@ -3480,112 +3530,51 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_14; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_propagateOffsetEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_14; -x_14 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_3); -if (x_14 == 0) +lean_object* x_12; +x_12 = lean_ctor_get(x_2, 10); +lean_inc(x_12); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_15; -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_2, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; -} -else +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = lean_ctor_get(x_2, 0); +lean_inc(x_13); +lean_dec(x_2); +lean_inc(x_13); +x_14 = l_Lean_Meta_Grind_isNatNum(x_13); +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) { lean_object* x_16; lean_object* x_17; -lean_dec(x_12); -lean_dec(x_11); +lean_dec(x_13); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); +lean_dec(x_1); x_16 = lean_box(0); x_17 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_13); +lean_ctor_set(x_17, 1, x_11); return x_17; } -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -lean_object* x_13; -lean_inc(x_3); -x_13 = l_Lean_Meta_Grind_getENode(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) +lean_object* x_18; +x_18 = lean_ctor_get(x_1, 10); +lean_inc(x_18); +lean_dec(x_1); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); +lean_object* x_19; lean_object* x_20; lean_dec(x_13); -x_16 = !lean_is_exclusive(x_14); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_14, 2); -lean_dec(x_18); -lean_inc(x_2); -lean_inc(x_17); -lean_ctor_set(x_14, 2, x_2); -lean_inc(x_3); -x_19 = l_Lean_Meta_Grind_setENode(x_3, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = l_Lean_Meta_Grind_isInconsistent(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_unbox(x_22); -lean_dec(x_22); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; -x_24 = lean_ctor_get(x_21, 1); -lean_inc(x_24); -lean_dec(x_21); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_25 = l_Lean_Meta_Grind_propagateDown(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24); -if (lean_obj_tag(x_25) == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(x_1, x_2, x_17, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); -lean_dec(x_26); -return x_28; -} -else -{ -uint8_t x_29; -lean_dec(x_17); -lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3593,126 +3582,73 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); -x_29 = !lean_is_exclusive(x_25); -if (x_29 == 0) +lean_dec(x_3); +x_19 = lean_box(0); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_11); +return x_20; +} +else { -return x_25; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_18, 0); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_process_new_offset_eq_lit(x_21, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_22; +} +} } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_25, 0); -x_31 = lean_ctor_get(x_25, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_25); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; -} -} -} -else +lean_object* x_23; +lean_dec(x_2); +x_23 = lean_ctor_get(x_1, 10); +lean_inc(x_23); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -lean_dec(x_3); -x_33 = lean_ctor_get(x_21, 1); -lean_inc(x_33); -lean_dec(x_21); -x_34 = lean_box(0); -x_35 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(x_1, x_2, x_17, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); -return x_35; -} -} -else +uint8_t x_24; +x_24 = !lean_is_exclusive(x_12); +if (x_24 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_36 = lean_ctor_get(x_14, 0); -x_37 = lean_ctor_get(x_14, 1); -x_38 = lean_ctor_get(x_14, 3); -x_39 = lean_ctor_get(x_14, 4); -x_40 = lean_ctor_get(x_14, 5); -x_41 = lean_ctor_get_uint8(x_14, sizeof(void*)*10); -x_42 = lean_ctor_get(x_14, 6); -x_43 = lean_ctor_get_uint8(x_14, sizeof(void*)*10 + 1); -x_44 = lean_ctor_get_uint8(x_14, sizeof(void*)*10 + 2); -x_45 = lean_ctor_get_uint8(x_14, sizeof(void*)*10 + 3); -x_46 = lean_ctor_get_uint8(x_14, sizeof(void*)*10 + 4); -x_47 = lean_ctor_get(x_14, 7); -x_48 = lean_ctor_get(x_14, 8); -x_49 = lean_ctor_get(x_14, 9); -lean_inc(x_49); -lean_inc(x_48); -lean_inc(x_47); -lean_inc(x_42); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_14); -lean_inc(x_2); -lean_inc(x_37); -x_50 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_50, 0, x_36); -lean_ctor_set(x_50, 1, x_37); -lean_ctor_set(x_50, 2, x_2); -lean_ctor_set(x_50, 3, x_38); -lean_ctor_set(x_50, 4, x_39); -lean_ctor_set(x_50, 5, x_40); -lean_ctor_set(x_50, 6, x_42); -lean_ctor_set(x_50, 7, x_47); -lean_ctor_set(x_50, 8, x_48); -lean_ctor_set(x_50, 9, x_49); -lean_ctor_set_uint8(x_50, sizeof(void*)*10, x_41); -lean_ctor_set_uint8(x_50, sizeof(void*)*10 + 1, x_43); -lean_ctor_set_uint8(x_50, sizeof(void*)*10 + 2, x_44); -lean_ctor_set_uint8(x_50, sizeof(void*)*10 + 3, x_45); -lean_ctor_set_uint8(x_50, sizeof(void*)*10 + 4, x_46); -lean_inc(x_3); -x_51 = l_Lean_Meta_Grind_setENode(x_3, x_50, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -lean_dec(x_51); -x_53 = l_Lean_Meta_Grind_isInconsistent(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_52); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_unbox(x_54); -lean_dec(x_54); -if (x_55 == 0) +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_ctor_get(x_12, 0); +x_26 = lean_ctor_get(x_1, 0); +lean_inc(x_26); +lean_dec(x_1); +lean_inc(x_26); +x_27 = l_Lean_Meta_Grind_isNatNum(x_26); +x_28 = lean_unbox(x_27); +lean_dec(x_27); +if (x_28 == 0) { -lean_object* x_56; lean_object* x_57; -x_56 = lean_ctor_get(x_53, 1); -lean_inc(x_56); -lean_dec(x_53); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_57 = l_Lean_Meta_Grind_propagateDown(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -if (lean_obj_tag(x_57) == 0) +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_29 = lean_st_ref_get(x_3, x_11); +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l_Lean_Meta_Grind_Goal_getENode(x_30, x_26, x_9, x_10, x_31); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(x_1, x_2, x_37, x_58, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_59); -lean_dec(x_58); -return x_60; -} -else +lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = !lean_is_exclusive(x_33); +if (x_35 == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_33, 0); +x_37 = lean_ctor_get(x_33, 10); lean_dec(x_37); -lean_dec(x_11); +lean_inc(x_36); +lean_ctor_set(x_33, 10, x_12); +x_38 = l_Lean_Meta_Grind_setENode(x_36, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3720,46 +3656,73 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); -x_61 = lean_ctor_get(x_57, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_57, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_63 = x_57; -} else { - lean_dec_ref(x_57); - x_63 = lean_box(0); -} -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; -} -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; -} +lean_dec(x_3); +return x_38; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; uint8_t x_47; uint8_t x_48; uint8_t x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_39 = lean_ctor_get(x_33, 0); +x_40 = lean_ctor_get(x_33, 1); +x_41 = lean_ctor_get(x_33, 2); +x_42 = lean_ctor_get(x_33, 3); +x_43 = lean_ctor_get(x_33, 4); +x_44 = lean_ctor_get(x_33, 5); +x_45 = lean_ctor_get_uint8(x_33, sizeof(void*)*11); +x_46 = lean_ctor_get(x_33, 6); +x_47 = lean_ctor_get_uint8(x_33, sizeof(void*)*11 + 1); +x_48 = lean_ctor_get_uint8(x_33, sizeof(void*)*11 + 2); +x_49 = lean_ctor_get_uint8(x_33, sizeof(void*)*11 + 3); +x_50 = lean_ctor_get_uint8(x_33, sizeof(void*)*11 + 4); +x_51 = lean_ctor_get(x_33, 7); +x_52 = lean_ctor_get(x_33, 8); +x_53 = lean_ctor_get(x_33, 9); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_46); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_33); +lean_inc(x_39); +x_54 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_54, 0, x_39); +lean_ctor_set(x_54, 1, x_40); +lean_ctor_set(x_54, 2, x_41); +lean_ctor_set(x_54, 3, x_42); +lean_ctor_set(x_54, 4, x_43); +lean_ctor_set(x_54, 5, x_44); +lean_ctor_set(x_54, 6, x_46); +lean_ctor_set(x_54, 7, x_51); +lean_ctor_set(x_54, 8, x_52); +lean_ctor_set(x_54, 9, x_53); +lean_ctor_set(x_54, 10, x_12); +lean_ctor_set_uint8(x_54, sizeof(void*)*11, x_45); +lean_ctor_set_uint8(x_54, sizeof(void*)*11 + 1, x_47); +lean_ctor_set_uint8(x_54, sizeof(void*)*11 + 2, x_48); +lean_ctor_set_uint8(x_54, sizeof(void*)*11 + 3, x_49); +lean_ctor_set_uint8(x_54, sizeof(void*)*11 + 4, x_50); +x_55 = l_Lean_Meta_Grind_setENode(x_39, x_54, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_34); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); -x_65 = lean_ctor_get(x_53, 1); -lean_inc(x_65); -lean_dec(x_53); -x_66 = lean_box(0); -x_67 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(x_1, x_2, x_37, x_66, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_65); -return x_67; -} +return x_55; } } else { -uint8_t x_68; -lean_dec(x_11); +uint8_t x_56; +lean_free_object(x_12); +lean_dec(x_25); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3768,73 +3731,132 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -x_68 = !lean_is_exclusive(x_13); -if (x_68 == 0) +x_56 = !lean_is_exclusive(x_32); +if (x_56 == 0) { -return x_13; +return x_32; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_13, 0); -x_70 = lean_ctor_get(x_13, 1); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_13); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -return x_71; -} +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_32, 0); +x_58 = lean_ctor_get(x_32, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_32); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); -lean_dec(x_1); -return x_14; +lean_object* x_60; +lean_free_object(x_12); +x_60 = lean_process_new_offset_eq_lit(x_25, x_26, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_60; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); +lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; +x_61 = lean_ctor_get(x_12, 0); +lean_inc(x_61); +lean_dec(x_12); +x_62 = lean_ctor_get(x_1, 0); +lean_inc(x_62); lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +lean_inc(x_62); +x_63 = l_Lean_Meta_Grind_isNatNum(x_62); +x_64 = lean_unbox(x_63); +lean_dec(x_63); +if (x_64 == 0) { -lean_object* x_13; -x_13 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_65 = lean_st_ref_get(x_3, x_11); +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = l_Lean_Meta_Grind_Goal_getENode(x_66, x_62, x_9, x_10, x_67); +if (lean_obj_tag(x_68) == 0) { -lean_object* x_12; -lean_inc(x_1); -x_12 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_2, x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_1); -return x_12; +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_69, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_69, 1); +lean_inc(x_72); +x_73 = lean_ctor_get(x_69, 2); +lean_inc(x_73); +x_74 = lean_ctor_get(x_69, 3); +lean_inc(x_74); +x_75 = lean_ctor_get(x_69, 4); +lean_inc(x_75); +x_76 = lean_ctor_get(x_69, 5); +lean_inc(x_76); +x_77 = lean_ctor_get_uint8(x_69, sizeof(void*)*11); +x_78 = lean_ctor_get(x_69, 6); +lean_inc(x_78); +x_79 = lean_ctor_get_uint8(x_69, sizeof(void*)*11 + 1); +x_80 = lean_ctor_get_uint8(x_69, sizeof(void*)*11 + 2); +x_81 = lean_ctor_get_uint8(x_69, sizeof(void*)*11 + 3); +x_82 = lean_ctor_get_uint8(x_69, sizeof(void*)*11 + 4); +x_83 = lean_ctor_get(x_69, 7); +lean_inc(x_83); +x_84 = lean_ctor_get(x_69, 8); +lean_inc(x_84); +x_85 = lean_ctor_get(x_69, 9); +lean_inc(x_85); +if (lean_is_exclusive(x_69)) { + lean_ctor_release(x_69, 0); + lean_ctor_release(x_69, 1); + lean_ctor_release(x_69, 2); + lean_ctor_release(x_69, 3); + lean_ctor_release(x_69, 4); + lean_ctor_release(x_69, 5); + lean_ctor_release(x_69, 6); + lean_ctor_release(x_69, 7); + lean_ctor_release(x_69, 8); + lean_ctor_release(x_69, 9); + lean_ctor_release(x_69, 10); + x_86 = x_69; +} else { + lean_dec_ref(x_69); + x_86 = lean_box(0); } +x_87 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_87, 0, x_61); +lean_inc(x_71); +if (lean_is_scalar(x_86)) { + x_88 = lean_alloc_ctor(0, 11, 5); +} else { + x_88 = x_86; } -LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -if (lean_obj_tag(x_1) == 0) -{ -lean_object* x_12; lean_object* x_13; +lean_ctor_set(x_88, 0, x_71); +lean_ctor_set(x_88, 1, x_72); +lean_ctor_set(x_88, 2, x_73); +lean_ctor_set(x_88, 3, x_74); +lean_ctor_set(x_88, 4, x_75); +lean_ctor_set(x_88, 5, x_76); +lean_ctor_set(x_88, 6, x_78); +lean_ctor_set(x_88, 7, x_83); +lean_ctor_set(x_88, 8, x_84); +lean_ctor_set(x_88, 9, x_85); +lean_ctor_set(x_88, 10, x_87); +lean_ctor_set_uint8(x_88, sizeof(void*)*11, x_77); +lean_ctor_set_uint8(x_88, sizeof(void*)*11 + 1, x_79); +lean_ctor_set_uint8(x_88, sizeof(void*)*11 + 2, x_80); +lean_ctor_set_uint8(x_88, sizeof(void*)*11 + 3, x_81); +lean_ctor_set_uint8(x_88, sizeof(void*)*11 + 4, x_82); +x_89 = l_Lean_Meta_Grind_setENode(x_71, x_88, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_70); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3843,42 +3865,12 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_2); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +return x_89; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_14 = lean_ctor_get(x_1, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -x_16 = lean_ctor_get(x_1, 3); -lean_inc(x_16); -lean_dec(x_1); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -x_17 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -if (lean_obj_tag(x_18) == 0) -{ -uint8_t x_19; -lean_dec(x_16); -lean_dec(x_15); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_dec(x_61); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3887,33 +3879,130 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_19 = !lean_is_exclusive(x_17); -if (x_19 == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_17, 0); -lean_dec(x_20); -return x_17; -} +x_90 = lean_ctor_get(x_68, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_68, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_92 = x_68; +} else { + lean_dec_ref(x_68); + x_92 = lean_box(0); +} +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); +} else { + x_93 = x_92; +} +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; +} +} else { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_17, 1); -lean_inc(x_21); -lean_dec(x_17); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_18); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_94; +x_94 = lean_process_new_offset_eq_lit(x_61, x_62, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_94; +} } } else { -lean_object* x_23; lean_object* x_24; -lean_dec(x_18); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_dec(x_17); +lean_object* x_95; lean_object* x_96; lean_object* x_97; +lean_dec(x_1); +x_95 = lean_ctor_get(x_12, 0); +lean_inc(x_95); +lean_dec(x_12); +x_96 = lean_ctor_get(x_23, 0); +lean_inc(x_96); +lean_dec(x_23); +x_97 = lean_process_new_offset_eq(x_95, x_96, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_97; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_13); +return x_17; +} +} +static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_13 = lean_ctor_get(x_3, 1); +lean_inc(x_13); +if (lean_is_exclusive(x_3)) { + lean_ctor_release(x_3, 0); + lean_ctor_release(x_3, 1); + x_14 = x_3; +} else { + lean_dec_ref(x_3); + x_14 = lean_box(0); +} +x_15 = lean_st_ref_get(x_4, x_12); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +lean_inc(x_13); +x_18 = l_Lean_Meta_Grind_Goal_getENode(x_16, x_13, x_10, x_11, x_17); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_35; lean_object* x_36; uint8_t x_37; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + x_21 = x_18; +} else { + lean_dec_ref(x_18); + x_21 = lean_box(0); +} +x_35 = l_Lean_Meta_Grind_isInconsistent(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_unbox(x_36); +lean_dec(x_36); +if (x_37 == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_35, 1); +lean_inc(x_38); +lean_dec(x_35); +x_39 = lean_ctor_get(x_19, 0); +lean_inc(x_39); +lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); @@ -3921,24 +4010,24 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_3); -x_24 = l_Lean_Meta_Grind_propagateUp(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); -if (lean_obj_tag(x_24) == 0) +x_40 = l_Lean_Meta_Grind_propagateDown(x_39, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_box(0); -x_1 = x_16; -x_2 = x_26; -x_11 = x_25; -goto _start; +lean_object* x_41; +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); +x_22 = x_41; +goto block_34; } else { -uint8_t x_28; -lean_dec(x_16); +uint8_t x_42; +lean_dec(x_21); +lean_dec(x_19); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3946,33 +4035,70 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_28 = !lean_is_exclusive(x_24); -if (x_28 == 0) +lean_dec(x_2); +x_42 = !lean_is_exclusive(x_40); +if (x_42 == 0) { -return x_24; +return x_40; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 0); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_24); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_40, 0); +x_44 = lean_ctor_get(x_40, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_40); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} } } +else +{ +lean_object* x_46; +x_46 = lean_ctor_get(x_35, 1); +lean_inc(x_46); +lean_dec(x_35); +x_22 = x_46; +goto block_34; } +block_34: +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_19, 1); +lean_inc(x_23); +x_24 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_23, x_1); +lean_dec(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_21); +lean_dec(x_14); +x_25 = lean_box(0); +lean_inc(x_2); +x_26 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1(x_19, x_2, x_13, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +lean_dec(x_13); +lean_dec(x_19); +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_ctor_get(x_27, 0); +lean_inc(x_29); +lean_dec(x_27); +x_3 = x_29; +x_12 = x_28; +goto _start; } else { -uint8_t x_32; -lean_dec(x_16); -lean_dec(x_15); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_dec(x_19); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -3980,1960 +4106,5046 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -x_32 = !lean_is_exclusive(x_17); -if (x_32 == 0) -{ -return x_17; -} -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_17, 0); -x_34 = lean_ctor_get(x_17, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_17); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_dec(x_2); +x_31 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; +if (lean_is_scalar(x_14)) { + x_32 = lean_alloc_ctor(0, 2, 0); +} else { + x_32 = x_14; } +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_13); +if (lean_is_scalar(x_21)) { + x_33 = lean_alloc_ctor(0, 2, 0); +} else { + x_33 = x_21; } +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_22); +return x_33; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = l_Lean_Meta_Grind_isInconsistent(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_unbox(x_13); +uint8_t x_47; +lean_dec(x_14); lean_dec(x_13); -if (x_14 == 0) +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_2); +x_47 = !lean_is_exclusive(x_18); +if (x_47 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -return x_16; +return x_18; } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_12, 0); +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_18, 0); +x_49 = lean_ctor_get(x_18, 1); +lean_inc(x_49); +lean_inc(x_48); lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_12, 0, x_19); -return x_12; -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_12, 1); -lean_inc(x_20); -lean_dec(x_12); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, uint8_t x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_21; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_box(0); lean_inc(x_1); -x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_21) == 0) +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_1); +x_13 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1(x_1, x_11, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = l_Lean_Meta_Grind_getENode(x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_22); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; uint8_t x_33; uint8_t x_34; uint8_t x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_ctor_get(x_24, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_24, 2); -lean_inc(x_27); -x_28 = lean_ctor_get(x_24, 3); -lean_inc(x_28); -x_29 = lean_ctor_get(x_24, 4); -lean_inc(x_29); -x_30 = lean_ctor_get(x_24, 5); -lean_inc(x_30); -x_31 = lean_ctor_get_uint8(x_24, sizeof(void*)*10); -x_32 = lean_ctor_get(x_24, 6); -lean_inc(x_32); -x_33 = lean_ctor_get_uint8(x_24, sizeof(void*)*10 + 1); -x_34 = lean_ctor_get_uint8(x_24, sizeof(void*)*10 + 2); -x_35 = lean_ctor_get_uint8(x_24, sizeof(void*)*10 + 3); -x_36 = lean_ctor_get_uint8(x_24, sizeof(void*)*10 + 4); -x_37 = lean_ctor_get(x_24, 7); -lean_inc(x_37); -x_38 = lean_ctor_get(x_24, 8); -lean_inc(x_38); -x_39 = lean_ctor_get(x_24, 9); -lean_inc(x_39); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - lean_ctor_release(x_24, 1); - lean_ctor_release(x_24, 2); - lean_ctor_release(x_24, 3); - lean_ctor_release(x_24, 4); - lean_ctor_release(x_24, 5); - lean_ctor_release(x_24, 6); - lean_ctor_release(x_24, 7); - lean_ctor_release(x_24, 8); - lean_ctor_release(x_24, 9); - x_40 = x_24; -} else { - lean_dec_ref(x_24); - x_40 = lean_box(0); -} -x_41 = !lean_is_exclusive(x_3); -if (x_41 == 0) +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +lean_dec(x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; lean_object* x_48; uint8_t x_49; uint8_t x_50; uint8_t x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_59; -x_42 = lean_ctor_get(x_3, 0); -x_43 = lean_ctor_get(x_3, 2); -x_44 = lean_ctor_get(x_3, 3); -x_45 = lean_ctor_get(x_3, 4); -x_46 = lean_ctor_get(x_3, 5); -x_47 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); -x_48 = lean_ctor_get(x_3, 6); -x_49 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 1); -x_50 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 2); -x_51 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 3); -x_52 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 4); -x_53 = lean_ctor_get(x_3, 7); -x_54 = lean_ctor_get(x_3, 8); -x_55 = lean_ctor_get(x_3, 9); -lean_ctor_set(x_3, 9, x_39); -lean_ctor_set(x_3, 8, x_38); -lean_ctor_set(x_3, 7, x_37); -lean_ctor_set(x_3, 6, x_32); -lean_ctor_set(x_3, 5, x_30); -lean_ctor_set(x_3, 4, x_29); -lean_ctor_set(x_3, 3, x_28); -lean_ctor_set(x_3, 2, x_27); -lean_ctor_set(x_3, 0, x_26); -lean_ctor_set_uint8(x_3, sizeof(void*)*10, x_31); -lean_ctor_set_uint8(x_3, sizeof(void*)*10 + 1, x_33); -lean_ctor_set_uint8(x_3, sizeof(void*)*10 + 2, x_34); -lean_ctor_set_uint8(x_3, sizeof(void*)*10 + 3, x_35); -lean_ctor_set_uint8(x_3, sizeof(void*)*10 + 4, x_36); -x_56 = l_Lean_Meta_Grind_setENode(x_4, x_3, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_25); -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -x_58 = lean_nat_add(x_48, x_5); -lean_dec(x_48); -if (x_51 == 0) +uint8_t x_16; +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) { -x_59 = x_10; -goto block_84; +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_13, 0); +lean_dec(x_17); +x_18 = lean_box(0); +lean_ctor_set(x_13, 0, x_18); +return x_13; } else { -uint8_t x_85; -x_85 = 1; -x_59 = x_85; -goto block_84; +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_dec(x_13); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; } -block_84: -{ -uint8_t x_60; -if (x_8 == 0) +} +else { -if (x_52 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_13); +if (x_22 == 0) { -x_60 = x_9; -goto block_81; +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_13, 0); +lean_dec(x_23); +x_24 = lean_ctor_get(x_15, 0); +lean_inc(x_24); +lean_dec(x_15); +lean_ctor_set(x_13, 0, x_24); +return x_13; } else { -uint8_t x_82; -x_82 = 1; -x_60 = x_82; -goto block_81; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_13, 1); +lean_inc(x_25); +lean_dec(x_13); +x_26 = lean_ctor_get(x_15, 0); +lean_inc(x_26); +lean_dec(x_15); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; } } -else -{ -uint8_t x_83; -x_83 = 1; -x_60 = x_83; -goto block_81; } -block_81: -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -lean_inc(x_42); -if (lean_is_scalar(x_40)) { - x_61 = lean_alloc_ctor(0, 10, 5); -} else { - x_61 = x_40; -} -lean_ctor_set(x_61, 0, x_42); -lean_ctor_set(x_61, 1, x_6); -lean_ctor_set(x_61, 2, x_43); -lean_ctor_set(x_61, 3, x_44); -lean_ctor_set(x_61, 4, x_45); -lean_ctor_set(x_61, 5, x_46); -lean_ctor_set(x_61, 6, x_58); -lean_ctor_set(x_61, 7, x_53); -lean_ctor_set(x_61, 8, x_54); -lean_ctor_set(x_61, 9, x_55); -lean_ctor_set_uint8(x_61, sizeof(void*)*10, x_47); -lean_ctor_set_uint8(x_61, sizeof(void*)*10 + 1, x_49); -lean_ctor_set_uint8(x_61, sizeof(void*)*10 + 2, x_50); -lean_ctor_set_uint8(x_61, sizeof(void*)*10 + 3, x_59); -lean_ctor_set_uint8(x_61, sizeof(void*)*10 + 4, x_60); -lean_inc(x_7); -x_62 = l_Lean_Meta_Grind_setENode(x_7, x_61, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_57); -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -lean_dec(x_62); -lean_inc(x_1); -x_64 = l_Lean_Meta_Grind_copyParentsTo(x_1, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_63); -x_65 = lean_ctor_get(x_64, 1); -lean_inc(x_65); -lean_dec(x_64); -x_66 = l_Lean_Meta_Grind_isInconsistent(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_65); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_unbox(x_67); -lean_dec(x_67); -if (x_68 == 0) +else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_66, 1); -lean_inc(x_69); -lean_dec(x_66); -x_70 = lean_box(0); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_71 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(x_1, x_70, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_69); -if (lean_obj_tag(x_71) == 0) +uint8_t x_28; +x_28 = !lean_is_exclusive(x_13); +if (x_28 == 0) { -lean_object* x_72; lean_object* x_73; -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -lean_dec(x_71); -x_73 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_42, x_70, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_72); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_42); -return x_73; +return x_13; } else { -uint8_t x_74; -lean_dec(x_42); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_13, 0); +x_30 = lean_ctor_get(x_13, 1); +lean_inc(x_30); +lean_inc(x_29); lean_dec(x_13); -lean_dec(x_12); -x_74 = !lean_is_exclusive(x_71); -if (x_74 == 0) -{ -return x_71; +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_71, 0); -x_76 = lean_ctor_get(x_71, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_71); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; } } } -else +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_1); -x_78 = lean_ctor_get(x_66, 1); -lean_inc(x_78); -lean_dec(x_66); -x_79 = lean_box(0); -x_80 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_42, x_79, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_78); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_14; +x_14 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); lean_dec(x_12); -lean_dec(x_42); -return x_80; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_14; } } +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_1); +return x_13; } } -else -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; lean_object* x_93; uint8_t x_94; uint8_t x_95; uint8_t x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; -x_86 = lean_ctor_get(x_3, 0); -x_87 = lean_ctor_get(x_3, 1); -x_88 = lean_ctor_get(x_3, 2); -x_89 = lean_ctor_get(x_3, 3); -x_90 = lean_ctor_get(x_3, 4); -x_91 = lean_ctor_get(x_3, 5); -x_92 = lean_ctor_get_uint8(x_3, sizeof(void*)*10); -x_93 = lean_ctor_get(x_3, 6); -x_94 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 1); -x_95 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 2); -x_96 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 3); -x_97 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 4); -x_98 = lean_ctor_get(x_3, 7); -x_99 = lean_ctor_get(x_3, 8); -x_100 = lean_ctor_get(x_3, 9); -lean_inc(x_100); -lean_inc(x_99); -lean_inc(x_98); -lean_inc(x_93); -lean_inc(x_91); -lean_inc(x_90); -lean_inc(x_89); -lean_inc(x_88); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_3); -x_101 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_101, 0, x_26); -lean_ctor_set(x_101, 1, x_87); -lean_ctor_set(x_101, 2, x_27); -lean_ctor_set(x_101, 3, x_28); -lean_ctor_set(x_101, 4, x_29); -lean_ctor_set(x_101, 5, x_30); -lean_ctor_set(x_101, 6, x_32); -lean_ctor_set(x_101, 7, x_37); -lean_ctor_set(x_101, 8, x_38); -lean_ctor_set(x_101, 9, x_39); -lean_ctor_set_uint8(x_101, sizeof(void*)*10, x_31); -lean_ctor_set_uint8(x_101, sizeof(void*)*10 + 1, x_33); -lean_ctor_set_uint8(x_101, sizeof(void*)*10 + 2, x_34); -lean_ctor_set_uint8(x_101, sizeof(void*)*10 + 3, x_35); -lean_ctor_set_uint8(x_101, sizeof(void*)*10 + 4, x_36); -x_102 = l_Lean_Meta_Grind_setENode(x_4, x_101, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_25); -x_103 = lean_ctor_get(x_102, 1); -lean_inc(x_103); -lean_dec(x_102); -x_104 = lean_nat_add(x_93, x_5); -lean_dec(x_93); -if (x_96 == 0) +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -x_105 = x_10; -goto block_130; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_1); +lean_ctor_set(x_14, 1, x_2); +x_15 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_15, 0, x_14); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_13); +return x_16; } -else -{ -uint8_t x_131; -x_131 = 1; -x_105 = x_131; -goto block_130; } -block_130: +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; +x_14 = !lean_is_exclusive(x_4); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_4, 1); +x_16 = lean_ctor_get(x_4, 0); +lean_dec(x_16); +x_17 = lean_st_ref_get(x_5, x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_15); +x_20 = l_Lean_Meta_Grind_Goal_getENode(x_18, x_15, x_11, x_12, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) { -uint8_t x_106; -if (x_8 == 0) +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_24 = lean_ctor_get(x_21, 0); +x_25 = lean_ctor_get(x_21, 1); +x_26 = lean_ctor_get(x_21, 2); +lean_dec(x_26); +lean_inc(x_2); +lean_inc(x_25); +lean_inc(x_24); +lean_ctor_set(x_21, 2, x_2); +x_27 = l_Lean_Meta_Grind_setENode(x_24, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +x_28 = !lean_is_exclusive(x_27); +if (x_28 == 0) { -if (x_97 == 0) +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_27, 1); +x_30 = lean_ctor_get(x_27, 0); +lean_dec(x_30); +x_31 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_25, x_1); +if (x_31 == 0) { -x_106 = x_9; -goto block_127; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_free_object(x_27); +lean_free_object(x_4); +x_32 = lean_box(0); +lean_inc(x_3); +x_33 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(x_3, x_25, x_15, x_32, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_29); +lean_dec(x_15); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = lean_ctor_get(x_34, 0); +lean_inc(x_36); +lean_dec(x_34); +x_4 = x_36; +x_13 = x_35; +goto _start; } else { -uint8_t x_128; -x_128 = 1; -x_106 = x_128; -goto block_127; +lean_object* x_38; +lean_dec(x_25); +lean_dec(x_3); +lean_dec(x_2); +x_38 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; +lean_ctor_set(x_4, 0, x_38); +lean_ctor_set(x_27, 0, x_4); +return x_27; } } else { -uint8_t x_129; -x_129 = 1; -x_106 = x_129; -goto block_127; +lean_object* x_39; uint8_t x_40; +x_39 = lean_ctor_get(x_27, 1); +lean_inc(x_39); +lean_dec(x_27); +x_40 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_25, x_1); +if (x_40 == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_free_object(x_4); +x_41 = lean_box(0); +lean_inc(x_3); +x_42 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(x_3, x_25, x_15, x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); +lean_dec(x_15); +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = lean_ctor_get(x_43, 0); +lean_inc(x_45); +lean_dec(x_43); +x_4 = x_45; +x_13 = x_44; +goto _start; } -block_127: +else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; uint8_t x_114; -lean_inc(x_86); -if (lean_is_scalar(x_40)) { - x_107 = lean_alloc_ctor(0, 10, 5); -} else { - x_107 = x_40; -} -lean_ctor_set(x_107, 0, x_86); -lean_ctor_set(x_107, 1, x_6); -lean_ctor_set(x_107, 2, x_88); -lean_ctor_set(x_107, 3, x_89); -lean_ctor_set(x_107, 4, x_90); -lean_ctor_set(x_107, 5, x_91); -lean_ctor_set(x_107, 6, x_104); -lean_ctor_set(x_107, 7, x_98); -lean_ctor_set(x_107, 8, x_99); -lean_ctor_set(x_107, 9, x_100); -lean_ctor_set_uint8(x_107, sizeof(void*)*10, x_92); -lean_ctor_set_uint8(x_107, sizeof(void*)*10 + 1, x_94); -lean_ctor_set_uint8(x_107, sizeof(void*)*10 + 2, x_95); -lean_ctor_set_uint8(x_107, sizeof(void*)*10 + 3, x_105); -lean_ctor_set_uint8(x_107, sizeof(void*)*10 + 4, x_106); -lean_inc(x_7); -x_108 = l_Lean_Meta_Grind_setENode(x_7, x_107, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_103); -x_109 = lean_ctor_get(x_108, 1); -lean_inc(x_109); -lean_dec(x_108); -lean_inc(x_1); -x_110 = l_Lean_Meta_Grind_copyParentsTo(x_1, x_7, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_109); -x_111 = lean_ctor_get(x_110, 1); -lean_inc(x_111); -lean_dec(x_110); -x_112 = l_Lean_Meta_Grind_isInconsistent(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_111); -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -x_114 = lean_unbox(x_113); -lean_dec(x_113); -if (x_114 == 0) +lean_object* x_47; lean_object* x_48; +lean_dec(x_25); +lean_dec(x_3); +lean_dec(x_2); +x_47 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; +lean_ctor_set(x_4, 0, x_47); +x_48 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_48, 0, x_4); +lean_ctor_set(x_48, 1, x_39); +return x_48; +} +} +} +else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_115 = lean_ctor_get(x_112, 1); -lean_inc(x_115); -lean_dec(x_112); -x_116 = lean_box(0); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_117 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(x_1, x_116, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_115); -if (lean_obj_tag(x_117) == 0) +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; uint8_t x_56; uint8_t x_57; uint8_t x_58; uint8_t x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; +x_49 = lean_ctor_get(x_21, 0); +x_50 = lean_ctor_get(x_21, 1); +x_51 = lean_ctor_get(x_21, 3); +x_52 = lean_ctor_get(x_21, 4); +x_53 = lean_ctor_get(x_21, 5); +x_54 = lean_ctor_get_uint8(x_21, sizeof(void*)*11); +x_55 = lean_ctor_get(x_21, 6); +x_56 = lean_ctor_get_uint8(x_21, sizeof(void*)*11 + 1); +x_57 = lean_ctor_get_uint8(x_21, sizeof(void*)*11 + 2); +x_58 = lean_ctor_get_uint8(x_21, sizeof(void*)*11 + 3); +x_59 = lean_ctor_get_uint8(x_21, sizeof(void*)*11 + 4); +x_60 = lean_ctor_get(x_21, 7); +x_61 = lean_ctor_get(x_21, 8); +x_62 = lean_ctor_get(x_21, 9); +x_63 = lean_ctor_get(x_21, 10); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_55); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_21); +lean_inc(x_2); +lean_inc(x_50); +lean_inc(x_49); +x_64 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_64, 0, x_49); +lean_ctor_set(x_64, 1, x_50); +lean_ctor_set(x_64, 2, x_2); +lean_ctor_set(x_64, 3, x_51); +lean_ctor_set(x_64, 4, x_52); +lean_ctor_set(x_64, 5, x_53); +lean_ctor_set(x_64, 6, x_55); +lean_ctor_set(x_64, 7, x_60); +lean_ctor_set(x_64, 8, x_61); +lean_ctor_set(x_64, 9, x_62); +lean_ctor_set(x_64, 10, x_63); +lean_ctor_set_uint8(x_64, sizeof(void*)*11, x_54); +lean_ctor_set_uint8(x_64, sizeof(void*)*11 + 1, x_56); +lean_ctor_set_uint8(x_64, sizeof(void*)*11 + 2, x_57); +lean_ctor_set_uint8(x_64, sizeof(void*)*11 + 3, x_58); +lean_ctor_set_uint8(x_64, sizeof(void*)*11 + 4, x_59); +x_65 = l_Lean_Meta_Grind_setENode(x_49, x_64, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_67 = x_65; +} else { + lean_dec_ref(x_65); + x_67 = lean_box(0); +} +x_68 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_50, x_1); +if (x_68 == 0) { -lean_object* x_118; lean_object* x_119; -x_118 = lean_ctor_get(x_117, 1); -lean_inc(x_118); -lean_dec(x_117); -x_119 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_86, x_116, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_118); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_dec(x_67); +lean_free_object(x_4); +x_69 = lean_box(0); +lean_inc(x_3); +x_70 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(x_3, x_50, x_15, x_69, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_66); lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_86); -return x_119; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_ctor_get(x_71, 0); +lean_inc(x_73); +lean_dec(x_71); +x_4 = x_73; +x_13 = x_72; +goto _start; } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; -lean_dec(x_86); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_120 = lean_ctor_get(x_117, 0); -lean_inc(x_120); -x_121 = lean_ctor_get(x_117, 1); -lean_inc(x_121); -if (lean_is_exclusive(x_117)) { - lean_ctor_release(x_117, 0); - lean_ctor_release(x_117, 1); - x_122 = x_117; +lean_object* x_75; lean_object* x_76; +lean_dec(x_50); +lean_dec(x_3); +lean_dec(x_2); +x_75 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; +lean_ctor_set(x_4, 0, x_75); +if (lean_is_scalar(x_67)) { + x_76 = lean_alloc_ctor(0, 2, 0); } else { - lean_dec_ref(x_117); - x_122 = lean_box(0); + x_76 = x_67; } -if (lean_is_scalar(x_122)) { - x_123 = lean_alloc_ctor(1, 2, 0); -} else { - x_123 = x_122; +lean_ctor_set(x_76, 0, x_4); +lean_ctor_set(x_76, 1, x_66); +return x_76; } -lean_ctor_set(x_123, 0, x_120); -lean_ctor_set(x_123, 1, x_121); -return x_123; } } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; -lean_dec(x_1); -x_124 = lean_ctor_get(x_112, 1); -lean_inc(x_124); -lean_dec(x_112); -x_125 = lean_box(0); -x_126 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_86, x_125, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_124); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); +uint8_t x_77; +lean_free_object(x_4); lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_86); -return x_126; -} +lean_dec(x_3); +lean_dec(x_2); +x_77 = !lean_is_exclusive(x_20); +if (x_77 == 0) +{ +return x_20; } +else +{ +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_20, 0); +x_79 = lean_ctor_get(x_20, 1); +lean_inc(x_79); +lean_inc(x_78); +lean_dec(x_20); +x_80 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_80, 0, x_78); +lean_ctor_set(x_80, 1, x_79); +return x_80; } } } else { -uint8_t x_132; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_81 = lean_ctor_get(x_4, 1); +lean_inc(x_81); lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_132 = !lean_is_exclusive(x_23); -if (x_132 == 0) -{ -return x_23; -} -else +x_82 = lean_st_ref_get(x_5, x_13); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +lean_dec(x_82); +lean_inc(x_81); +x_85 = l_Lean_Meta_Grind_Goal_getENode(x_83, x_81, x_11, x_12, x_84); +if (lean_obj_tag(x_85) == 0) { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_133 = lean_ctor_get(x_23, 0); -x_134 = lean_ctor_get(x_23, 1); -lean_inc(x_134); -lean_inc(x_133); -lean_dec(x_23); -x_135 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_135, 0, x_133); -lean_ctor_set(x_135, 1, x_134); -return x_135; +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; uint8_t x_95; uint8_t x_96; uint8_t x_97; uint8_t x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; +x_86 = lean_ctor_get(x_85, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_88 = lean_ctor_get(x_86, 0); +lean_inc(x_88); +x_89 = lean_ctor_get(x_86, 1); +lean_inc(x_89); +x_90 = lean_ctor_get(x_86, 3); +lean_inc(x_90); +x_91 = lean_ctor_get(x_86, 4); +lean_inc(x_91); +x_92 = lean_ctor_get(x_86, 5); +lean_inc(x_92); +x_93 = lean_ctor_get_uint8(x_86, sizeof(void*)*11); +x_94 = lean_ctor_get(x_86, 6); +lean_inc(x_94); +x_95 = lean_ctor_get_uint8(x_86, sizeof(void*)*11 + 1); +x_96 = lean_ctor_get_uint8(x_86, sizeof(void*)*11 + 2); +x_97 = lean_ctor_get_uint8(x_86, sizeof(void*)*11 + 3); +x_98 = lean_ctor_get_uint8(x_86, sizeof(void*)*11 + 4); +x_99 = lean_ctor_get(x_86, 7); +lean_inc(x_99); +x_100 = lean_ctor_get(x_86, 8); +lean_inc(x_100); +x_101 = lean_ctor_get(x_86, 9); +lean_inc(x_101); +x_102 = lean_ctor_get(x_86, 10); +lean_inc(x_102); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + lean_ctor_release(x_86, 2); + lean_ctor_release(x_86, 3); + lean_ctor_release(x_86, 4); + lean_ctor_release(x_86, 5); + lean_ctor_release(x_86, 6); + lean_ctor_release(x_86, 7); + lean_ctor_release(x_86, 8); + lean_ctor_release(x_86, 9); + lean_ctor_release(x_86, 10); + x_103 = x_86; +} else { + lean_dec_ref(x_86); + x_103 = lean_box(0); } +lean_inc(x_2); +lean_inc(x_89); +lean_inc(x_88); +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(0, 11, 5); +} else { + x_104 = x_103; +} +lean_ctor_set(x_104, 0, x_88); +lean_ctor_set(x_104, 1, x_89); +lean_ctor_set(x_104, 2, x_2); +lean_ctor_set(x_104, 3, x_90); +lean_ctor_set(x_104, 4, x_91); +lean_ctor_set(x_104, 5, x_92); +lean_ctor_set(x_104, 6, x_94); +lean_ctor_set(x_104, 7, x_99); +lean_ctor_set(x_104, 8, x_100); +lean_ctor_set(x_104, 9, x_101); +lean_ctor_set(x_104, 10, x_102); +lean_ctor_set_uint8(x_104, sizeof(void*)*11, x_93); +lean_ctor_set_uint8(x_104, sizeof(void*)*11 + 1, x_95); +lean_ctor_set_uint8(x_104, sizeof(void*)*11 + 2, x_96); +lean_ctor_set_uint8(x_104, sizeof(void*)*11 + 3, x_97); +lean_ctor_set_uint8(x_104, sizeof(void*)*11 + 4, x_98); +x_105 = l_Lean_Meta_Grind_setENode(x_88, x_104, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_87); +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; +} else { + lean_dec_ref(x_105); + x_107 = lean_box(0); } +x_108 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_89, x_1); +if (x_108 == 0) +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; +lean_dec(x_107); +x_109 = lean_box(0); +lean_inc(x_3); +x_110 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(x_3, x_89, x_81, x_109, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_106); +lean_dec(x_81); +x_111 = lean_ctor_get(x_110, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_110, 1); +lean_inc(x_112); +lean_dec(x_110); +x_113 = lean_ctor_get(x_111, 0); +lean_inc(x_113); +lean_dec(x_111); +x_4 = x_113; +x_13 = x_112; +goto _start; } else { -uint8_t x_136; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); +lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_89); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_136 = !lean_is_exclusive(x_21); -if (x_136 == 0) -{ -return x_21; +x_115 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1; +x_116 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_81); +if (lean_is_scalar(x_107)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_107; +} +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_106); +return x_117; +} } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_137 = lean_ctor_get(x_21, 0); -x_138 = lean_ctor_get(x_21, 1); -lean_inc(x_138); -lean_inc(x_137); -lean_dec(x_21); -x_139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -return x_139; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +lean_dec(x_81); +lean_dec(x_3); +lean_dec(x_2); +x_118 = lean_ctor_get(x_85, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_85, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_120 = x_85; +} else { + lean_dec_ref(x_85); + x_120 = lean_box(0); } +if (lean_is_scalar(x_120)) { + x_121 = lean_alloc_ctor(1, 2, 0); +} else { + x_121 = x_120; } +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_119); +return x_121; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" new root ", 10, 10); -return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__3() { -_start: +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +lean_inc(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_1); +x_14 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1(x_1, x_2, x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", ", 2, 2); -return x_1; -} +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +if (lean_obj_tag(x_16) == 0) +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_14, 0); +lean_dec(x_18); +x_19 = lean_box(0); +lean_ctor_set(x_14, 0, x_19); +return x_14; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__3; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_dec(x_14); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { -_start: -{ -lean_object* x_21; -lean_inc(x_1); -x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_21) == 0) +else { -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_21, 1); -lean_inc(x_22); -lean_dec(x_21); -x_23 = !lean_is_exclusive(x_2); +uint8_t x_23; +x_23 = !lean_is_exclusive(x_14); if (x_23 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_24 = lean_ctor_get(x_2, 2); -x_25 = lean_ctor_get(x_2, 5); -lean_dec(x_25); -x_26 = lean_ctor_get(x_2, 4); -lean_dec(x_26); -x_27 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_27, 0, x_3); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_4); -lean_inc(x_24); -lean_ctor_set(x_2, 5, x_28); -lean_ctor_set(x_2, 4, x_27); -lean_ctor_set_uint8(x_2, sizeof(void*)*10, x_5); -lean_inc(x_1); -x_29 = l_Lean_Meta_Grind_setENode(x_1, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_22); -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +lean_dec(x_24); +x_25 = lean_ctor_get(x_16, 0); +lean_inc(x_25); +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_25); +return x_14; +} +else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; -x_31 = lean_ctor_get(x_29, 1); -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = lean_ctor_get(x_6, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_6, 1); -lean_inc(x_34); -x_35 = lean_ctor_get(x_6, 6); -lean_inc(x_35); -x_36 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 3); -x_37 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 4); -lean_dec(x_6); -x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_33, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_31); -if (lean_obj_tag(x_38) == 0) +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 1); +lean_inc(x_26); +lean_dec(x_14); +x_27 = lean_ctor_get(x_16, 0); +lean_inc(x_27); +lean_dec(x_16); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +return x_28; +} +} +} +else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_39 = lean_ctor_get(x_38, 0); -lean_inc(x_39); -x_40 = lean_ctor_get(x_38, 1); -lean_inc(x_40); -lean_dec(x_38); -x_41 = lean_ctor_get(x_7, 2); -lean_inc(x_41); -lean_dec(x_7); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_41); -lean_inc(x_1); -x_42 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_41, x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_40); -if (lean_obj_tag(x_42) == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -lean_inc(x_8); -x_44 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_43); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_unbox(x_45); -lean_dec(x_45); -if (x_46 == 0) +return x_14; +} +else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -lean_free_object(x_29); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_1); -x_47 = lean_ctor_get(x_44, 1); -lean_inc(x_47); -lean_dec(x_44); -x_48 = lean_box(0); -x_49 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_48, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_47); -lean_dec(x_35); -return x_49; +return x_14; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_50; -x_50 = !lean_is_exclusive(x_44); -if (x_50 == 0) +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_44, 1); -x_52 = lean_ctor_get(x_44, 0); -lean_dec(x_52); -x_53 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_51); -if (lean_obj_tag(x_53) == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -lean_dec(x_53); -x_55 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_54); -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) +lean_object* x_12; lean_object* x_13; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_12 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_12, 0, x_2); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_ctor_get(x_55, 1); -x_59 = l_Lean_Meta_Grind_ppENodeRef(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_58); -x_60 = !lean_is_exclusive(x_59); -if (x_60 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_1, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_1, 1); +lean_inc(x_15); +x_16 = lean_ctor_get(x_1, 3); +lean_inc(x_16); +lean_dec(x_1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_17 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; -x_61 = lean_ctor_get(x_59, 0); -x_62 = lean_ctor_get(x_59, 1); -x_63 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_62); -if (lean_obj_tag(x_63) == 0) +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -x_66 = l_Lean_Meta_Grind_ppENodeRef(x_64, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_65); -lean_dec(x_64); -x_67 = !lean_is_exclusive(x_66); -if (x_67 == 0) +uint8_t x_19; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_68 = lean_ctor_get(x_66, 0); -x_69 = lean_ctor_get(x_66, 1); -x_70 = l_Lean_MessageData_ofFormat(x_57); -x_71 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -lean_ctor_set_tag(x_66, 7); -lean_ctor_set(x_66, 1, x_70); -lean_ctor_set(x_66, 0, x_71); -x_72 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -lean_ctor_set_tag(x_59, 7); -lean_ctor_set(x_59, 1, x_72); -lean_ctor_set(x_59, 0, x_66); -x_73 = l_Lean_MessageData_ofFormat(x_61); -lean_ctor_set_tag(x_55, 7); -lean_ctor_set(x_55, 1, x_73); -lean_ctor_set(x_55, 0, x_59); -x_74 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -lean_ctor_set_tag(x_44, 7); -lean_ctor_set(x_44, 1, x_74); -lean_ctor_set(x_44, 0, x_55); -x_75 = l_Lean_MessageData_ofFormat(x_68); -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_75); -lean_ctor_set(x_29, 0, x_44); -x_76 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_76, 0, x_29); -lean_ctor_set(x_76, 1, x_71); -x_77 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_76, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_69); -x_78 = lean_ctor_get(x_77, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_77, 1); -lean_inc(x_79); -lean_dec(x_77); -x_80 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_78, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_79); -lean_dec(x_78); -lean_dec(x_35); -return x_80; +lean_object* x_20; +x_20 = lean_ctor_get(x_17, 0); +lean_dec(x_20); +return x_17; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_81 = lean_ctor_get(x_66, 0); -x_82 = lean_ctor_get(x_66, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_66); -x_83 = l_Lean_MessageData_ofFormat(x_57); -x_84 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_85 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_83); -x_86 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -lean_ctor_set_tag(x_59, 7); -lean_ctor_set(x_59, 1, x_86); -lean_ctor_set(x_59, 0, x_85); -x_87 = l_Lean_MessageData_ofFormat(x_61); -lean_ctor_set_tag(x_55, 7); -lean_ctor_set(x_55, 1, x_87); -lean_ctor_set(x_55, 0, x_59); -x_88 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -lean_ctor_set_tag(x_44, 7); -lean_ctor_set(x_44, 1, x_88); -lean_ctor_set(x_44, 0, x_55); -x_89 = l_Lean_MessageData_ofFormat(x_81); -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_89); -lean_ctor_set(x_29, 0, x_44); -x_90 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_90, 0, x_29); -lean_ctor_set(x_90, 1, x_84); -x_91 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_90, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_82); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_18); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +else +{ +lean_object* x_23; lean_object* x_24; +lean_dec(x_18); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_dec(x_17); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_24 = l_Lean_Meta_Grind_propagateUp(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_23); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = lean_box(0); +x_1 = x_16; +x_2 = x_26; +x_11 = x_25; +goto _start; +} +else +{ +uint8_t x_28; +lean_dec(x_16); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) +{ +return x_24; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +} +} +else +{ +uint8_t x_32; +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_32 = !lean_is_exclusive(x_17); +if (x_32 == 0) +{ +return x_17; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_17, 0); +x_34 = lean_ctor_get(x_17, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_17); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_propagateOffsetEq(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_unbox(x_17); +lean_dec(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_box(0); +x_21 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___spec__1(x_3, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_19); +if (lean_obj_tag(x_21) == 0) +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +lean_ctor_set(x_21, 0, x_20); +return x_21; +} +else +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_20); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +else +{ +uint8_t x_26; +x_26 = !lean_is_exclusive(x_21); +if (x_26 == 0) +{ +return x_21; +} +else +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_21, 0); +x_28 = lean_ctor_get(x_21, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_21); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; +} +} +} +else +{ +uint8_t x_30; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_30 = !lean_is_exclusive(x_16); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_16, 0); +lean_dec(x_31); +x_32 = lean_box(0); +lean_ctor_set(x_16, 0, x_32); +return x_16; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_16, 1); +lean_inc(x_33); +lean_dec(x_16); +x_34 = lean_box(0); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_33); +return x_35; +} +} +} +else +{ +uint8_t x_36; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +x_36 = !lean_is_exclusive(x_14); +if (x_36 == 0) +{ +return x_14; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_14, 0); +x_38 = lean_ctor_get(x_14, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_14); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, uint8_t x_11, uint8_t x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22) { +_start: +{ +lean_object* x_23; +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_1); +x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_reinsertParents(x_1, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_23, 1); +lean_inc(x_24); +lean_dec(x_23); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +x_25 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown(x_2, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_24); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = lean_st_ref_get(x_14, x_26); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l_Lean_Meta_Grind_Goal_getENode(x_28, x_3, x_20, x_21, x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = !lean_is_exclusive(x_31); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; uint8_t x_43; uint8_t x_44; uint8_t x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_34 = lean_ctor_get(x_31, 1); +lean_dec(x_34); +x_35 = lean_ctor_get(x_4, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_4, 1); +lean_inc(x_36); +x_37 = lean_ctor_get(x_4, 2); +lean_inc(x_37); +x_38 = lean_ctor_get(x_4, 3); +lean_inc(x_38); +x_39 = lean_ctor_get(x_4, 4); +lean_inc(x_39); +x_40 = lean_ctor_get(x_4, 5); +lean_inc(x_40); +x_41 = lean_ctor_get_uint8(x_4, sizeof(void*)*11); +x_42 = lean_ctor_get(x_4, 6); +lean_inc(x_42); +x_43 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 1); +x_44 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 2); +x_45 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 3); +x_46 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 4); +x_47 = lean_ctor_get(x_4, 7); +lean_inc(x_47); +x_48 = lean_ctor_get(x_4, 8); +lean_inc(x_48); +x_49 = lean_ctor_get(x_4, 9); +lean_inc(x_49); +x_50 = lean_ctor_get(x_4, 10); +lean_inc(x_50); +lean_ctor_set(x_31, 1, x_36); +x_51 = l_Lean_Meta_Grind_setENode(x_5, x_31, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_32); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +lean_dec(x_51); +x_53 = lean_nat_add(x_42, x_6); +lean_dec(x_42); +if (x_45 == 0) +{ +x_54 = x_12; +goto block_79; +} +else +{ +uint8_t x_80; +x_80 = 1; +x_54 = x_80; +goto block_79; +} +block_79: +{ +uint8_t x_55; +if (x_10 == 0) +{ +if (x_46 == 0) +{ +x_55 = x_11; +goto block_76; +} +else +{ +uint8_t x_77; +x_77 = 1; +x_55 = x_77; +goto block_76; +} +} +else +{ +uint8_t x_78; +x_78 = 1; +x_55 = x_78; +goto block_76; +} +block_76: +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +lean_inc(x_35); +x_56 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_56, 0, x_35); +lean_ctor_set(x_56, 1, x_7); +lean_ctor_set(x_56, 2, x_37); +lean_ctor_set(x_56, 3, x_38); +lean_ctor_set(x_56, 4, x_39); +lean_ctor_set(x_56, 5, x_40); +lean_ctor_set(x_56, 6, x_53); +lean_ctor_set(x_56, 7, x_47); +lean_ctor_set(x_56, 8, x_48); +lean_ctor_set(x_56, 9, x_49); +lean_ctor_set(x_56, 10, x_50); +lean_ctor_set_uint8(x_56, sizeof(void*)*11, x_41); +lean_ctor_set_uint8(x_56, sizeof(void*)*11 + 1, x_43); +lean_ctor_set_uint8(x_56, sizeof(void*)*11 + 2, x_44); +lean_ctor_set_uint8(x_56, sizeof(void*)*11 + 3, x_54); +lean_ctor_set_uint8(x_56, sizeof(void*)*11 + 4, x_55); +lean_inc(x_8); +x_57 = l_Lean_Meta_Grind_setENode(x_8, x_56, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_52); +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +lean_dec(x_57); +lean_inc(x_1); +x_59 = l_Lean_Meta_Grind_copyParentsTo(x_1, x_8, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_58); +x_60 = lean_ctor_get(x_59, 1); +lean_inc(x_60); +lean_dec(x_59); +x_61 = l_Lean_Meta_Grind_isInconsistent(x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_60); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_unbox(x_62); +lean_dec(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_ctor_get(x_61, 1); +lean_inc(x_64); +lean_dec(x_61); +x_65 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_35, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_64); +lean_dec(x_35); +if (lean_obj_tag(x_65) == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_4, x_9, x_1, x_66, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_67); +lean_dec(x_66); +return x_68; +} +else +{ +uint8_t x_69; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_1); +x_69 = !lean_is_exclusive(x_65); +if (x_69 == 0) +{ +return x_65; +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_65, 0); +x_71 = lean_ctor_get(x_65, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_65); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; +} +} +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_dec(x_35); +x_73 = lean_ctor_get(x_61, 1); +lean_inc(x_73); +lean_dec(x_61); +x_74 = lean_box(0); +x_75 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_4, x_9, x_1, x_74, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_73); +return x_75; +} +} +} +} +else +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; lean_object* x_87; uint8_t x_88; uint8_t x_89; uint8_t x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; uint8_t x_104; uint8_t x_105; uint8_t x_106; uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; +x_81 = lean_ctor_get(x_31, 0); +x_82 = lean_ctor_get(x_31, 2); +x_83 = lean_ctor_get(x_31, 3); +x_84 = lean_ctor_get(x_31, 4); +x_85 = lean_ctor_get(x_31, 5); +x_86 = lean_ctor_get_uint8(x_31, sizeof(void*)*11); +x_87 = lean_ctor_get(x_31, 6); +x_88 = lean_ctor_get_uint8(x_31, sizeof(void*)*11 + 1); +x_89 = lean_ctor_get_uint8(x_31, sizeof(void*)*11 + 2); +x_90 = lean_ctor_get_uint8(x_31, sizeof(void*)*11 + 3); +x_91 = lean_ctor_get_uint8(x_31, sizeof(void*)*11 + 4); +x_92 = lean_ctor_get(x_31, 7); +x_93 = lean_ctor_get(x_31, 8); +x_94 = lean_ctor_get(x_31, 9); +x_95 = lean_ctor_get(x_31, 10); +lean_inc(x_95); +lean_inc(x_94); +lean_inc(x_93); +lean_inc(x_92); +lean_inc(x_87); +lean_inc(x_85); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_dec(x_31); +x_96 = lean_ctor_get(x_4, 0); +lean_inc(x_96); +x_97 = lean_ctor_get(x_4, 1); +lean_inc(x_97); +x_98 = lean_ctor_get(x_4, 2); +lean_inc(x_98); +x_99 = lean_ctor_get(x_4, 3); +lean_inc(x_99); +x_100 = lean_ctor_get(x_4, 4); +lean_inc(x_100); +x_101 = lean_ctor_get(x_4, 5); +lean_inc(x_101); +x_102 = lean_ctor_get_uint8(x_4, sizeof(void*)*11); +x_103 = lean_ctor_get(x_4, 6); +lean_inc(x_103); +x_104 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 1); +x_105 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 2); +x_106 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 3); +x_107 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 4); +x_108 = lean_ctor_get(x_4, 7); +lean_inc(x_108); +x_109 = lean_ctor_get(x_4, 8); +lean_inc(x_109); +x_110 = lean_ctor_get(x_4, 9); +lean_inc(x_110); +x_111 = lean_ctor_get(x_4, 10); +lean_inc(x_111); +x_112 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_112, 0, x_81); +lean_ctor_set(x_112, 1, x_97); +lean_ctor_set(x_112, 2, x_82); +lean_ctor_set(x_112, 3, x_83); +lean_ctor_set(x_112, 4, x_84); +lean_ctor_set(x_112, 5, x_85); +lean_ctor_set(x_112, 6, x_87); +lean_ctor_set(x_112, 7, x_92); +lean_ctor_set(x_112, 8, x_93); +lean_ctor_set(x_112, 9, x_94); +lean_ctor_set(x_112, 10, x_95); +lean_ctor_set_uint8(x_112, sizeof(void*)*11, x_86); +lean_ctor_set_uint8(x_112, sizeof(void*)*11 + 1, x_88); +lean_ctor_set_uint8(x_112, sizeof(void*)*11 + 2, x_89); +lean_ctor_set_uint8(x_112, sizeof(void*)*11 + 3, x_90); +lean_ctor_set_uint8(x_112, sizeof(void*)*11 + 4, x_91); +x_113 = l_Lean_Meta_Grind_setENode(x_5, x_112, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_32); +x_114 = lean_ctor_get(x_113, 1); +lean_inc(x_114); +lean_dec(x_113); +x_115 = lean_nat_add(x_103, x_6); +lean_dec(x_103); +if (x_106 == 0) +{ +x_116 = x_12; +goto block_141; +} +else +{ +uint8_t x_142; +x_142 = 1; +x_116 = x_142; +goto block_141; +} +block_141: +{ +uint8_t x_117; +if (x_10 == 0) +{ +if (x_107 == 0) +{ +x_117 = x_11; +goto block_138; +} +else +{ +uint8_t x_139; +x_139 = 1; +x_117 = x_139; +goto block_138; +} +} +else +{ +uint8_t x_140; +x_140 = 1; +x_117 = x_140; +goto block_138; +} +block_138: +{ +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; +lean_inc(x_96); +x_118 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_118, 0, x_96); +lean_ctor_set(x_118, 1, x_7); +lean_ctor_set(x_118, 2, x_98); +lean_ctor_set(x_118, 3, x_99); +lean_ctor_set(x_118, 4, x_100); +lean_ctor_set(x_118, 5, x_101); +lean_ctor_set(x_118, 6, x_115); +lean_ctor_set(x_118, 7, x_108); +lean_ctor_set(x_118, 8, x_109); +lean_ctor_set(x_118, 9, x_110); +lean_ctor_set(x_118, 10, x_111); +lean_ctor_set_uint8(x_118, sizeof(void*)*11, x_102); +lean_ctor_set_uint8(x_118, sizeof(void*)*11 + 1, x_104); +lean_ctor_set_uint8(x_118, sizeof(void*)*11 + 2, x_105); +lean_ctor_set_uint8(x_118, sizeof(void*)*11 + 3, x_116); +lean_ctor_set_uint8(x_118, sizeof(void*)*11 + 4, x_117); +lean_inc(x_8); +x_119 = l_Lean_Meta_Grind_setENode(x_8, x_118, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_114); +x_120 = lean_ctor_get(x_119, 1); +lean_inc(x_120); +lean_dec(x_119); +lean_inc(x_1); +x_121 = l_Lean_Meta_Grind_copyParentsTo(x_1, x_8, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_120); +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +lean_dec(x_121); +x_123 = l_Lean_Meta_Grind_isInconsistent(x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_122); +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +x_125 = lean_unbox(x_124); +lean_dec(x_124); +if (x_125 == 0) +{ +lean_object* x_126; lean_object* x_127; +x_126 = lean_ctor_get(x_123, 1); +lean_inc(x_126); +lean_dec(x_123); +x_127 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_updateMT(x_96, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_126); +lean_dec(x_96); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +x_130 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_4, x_9, x_1, x_128, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_129); +lean_dec(x_128); +return x_130; +} +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); +lean_dec(x_4); +lean_dec(x_1); +x_131 = lean_ctor_get(x_127, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_127, 1); +lean_inc(x_132); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_133 = x_127; +} else { + lean_dec_ref(x_127); + x_133 = lean_box(0); +} +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); +} else { + x_134 = x_133; +} +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; +} +} +else +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; +lean_dec(x_96); +x_135 = lean_ctor_get(x_123, 1); +lean_inc(x_135); +lean_dec(x_123); +x_136 = lean_box(0); +x_137 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_4, x_9, x_1, x_136, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_135); +return x_137; +} +} +} +} +} +else +{ +uint8_t x_143; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_143 = !lean_is_exclusive(x_30); +if (x_143 == 0) +{ +return x_30; +} +else +{ +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_30, 0); +x_145 = lean_ctor_get(x_30, 1); +lean_inc(x_145); +lean_inc(x_144); +lean_dec(x_30); +x_146 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +return x_146; +} +} +} +else +{ +uint8_t x_147; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_147 = !lean_is_exclusive(x_25); +if (x_147 == 0) +{ +return x_25; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_148 = lean_ctor_get(x_25, 0); +x_149 = lean_ctor_get(x_25, 1); +lean_inc(x_149); +lean_inc(x_148); +lean_dec(x_25); +x_150 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 1, x_149); +return x_150; +} +} +} +else +{ +uint8_t x_151; +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_151 = !lean_is_exclusive(x_23); +if (x_151 == 0) +{ +return x_23; +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_23, 0); +x_153 = lean_ctor_get(x_23, 1); +lean_inc(x_153); +lean_inc(x_152); +lean_dec(x_23); +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_152); +lean_ctor_set(x_154, 1, x_153); +return x_154; +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" new root ", 10, 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", ", 2, 2); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +_start: +{ +lean_object* x_21; +lean_inc(x_1); +x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_invertTrans(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_21, 1); +lean_inc(x_22); +lean_dec(x_21); +x_23 = !lean_is_exclusive(x_2); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_24 = lean_ctor_get(x_2, 2); +x_25 = lean_ctor_get(x_2, 5); +lean_dec(x_25); +x_26 = lean_ctor_get(x_2, 4); +lean_dec(x_26); +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_3); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_4); +lean_inc(x_24); +lean_ctor_set(x_2, 5, x_28); +lean_ctor_set(x_2, 4, x_27); +lean_ctor_set_uint8(x_2, sizeof(void*)*11, x_5); +lean_inc(x_1); +x_29 = l_Lean_Meta_Grind_setENode(x_1, x_2, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_22); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; uint8_t x_37; lean_object* x_38; +x_31 = lean_ctor_get(x_29, 1); +x_32 = lean_ctor_get(x_29, 0); +lean_dec(x_32); +x_33 = lean_ctor_get(x_6, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_6, 1); +lean_inc(x_34); +x_35 = lean_ctor_get(x_6, 6); +lean_inc(x_35); +x_36 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 3); +x_37 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 4); +x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_33, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_31); +if (lean_obj_tag(x_38) == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_ctor_get(x_7, 2); +lean_inc(x_41); +lean_dec(x_7); +lean_inc(x_41); +lean_inc(x_1); +x_42 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(x_1, x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_40); +if (lean_obj_tag(x_42) == 0) +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +lean_inc(x_8); +x_44 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_43); +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_unbox(x_45); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_free_object(x_29); +lean_dec(x_8); +x_47 = lean_ctor_get(x_44, 1); +lean_inc(x_47); +lean_dec(x_44); +x_48 = lean_box(0); +x_49 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_1, x_33, x_9, x_24, x_35, x_34, x_41, x_6, x_10, x_37, x_36, x_48, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_47); +lean_dec(x_35); +return x_49; +} +else +{ +uint8_t x_50; +x_50 = !lean_is_exclusive(x_44); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_44, 1); +x_52 = lean_ctor_get(x_44, 0); +lean_dec(x_52); +x_53 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_51); +if (lean_obj_tag(x_53) == 0) +{ +lean_object* x_54; lean_object* x_55; +x_54 = lean_ctor_get(x_53, 1); +lean_inc(x_54); +lean_dec(x_53); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_1); +x_55 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_54); +if (lean_obj_tag(x_55) == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_41); +x_58 = l_Lean_Meta_Grind_ppENodeRef(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_57); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); +x_61 = lean_st_ref_get(x_12, x_60); +x_62 = !lean_is_exclusive(x_61); +if (x_62 == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_61, 0); +x_64 = lean_ctor_get(x_61, 1); +lean_inc(x_1); +x_65 = l_Lean_Meta_Grind_Goal_getRoot(x_63, x_1, x_18, x_19, x_64); +if (lean_obj_tag(x_65) == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_68 = l_Lean_Meta_Grind_ppENodeRef(x_66, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_67); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +lean_ctor_set_tag(x_61, 7); +lean_ctor_set(x_61, 1, x_56); +lean_ctor_set(x_61, 0, x_71); +x_72 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_72); +lean_ctor_set(x_44, 0, x_61); +lean_ctor_set_tag(x_29, 7); +lean_ctor_set(x_29, 1, x_59); +lean_ctor_set(x_29, 0, x_44); +x_73 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; +x_74 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_74, 0, x_29); +lean_ctor_set(x_74, 1, x_73); +x_75 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_69); +x_76 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_71); +x_77 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_76, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_70); +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_1, x_33, x_9, x_24, x_35, x_34, x_41, x_6, x_10, x_37, x_36, x_78, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_79); +lean_dec(x_78); +lean_dec(x_35); +return x_80; +} +else +{ +uint8_t x_81; +lean_free_object(x_61); +lean_dec(x_59); +lean_dec(x_56); +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_81 = !lean_is_exclusive(x_68); +if (x_81 == 0) +{ +return x_68; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_68, 0); +x_83 = lean_ctor_get(x_68, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_68); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; +} +} +} +else +{ +uint8_t x_85; +lean_free_object(x_61); +lean_dec(x_59); +lean_dec(x_56); +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_85 = !lean_is_exclusive(x_65); +if (x_85 == 0) +{ +return x_65; +} +else +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_65, 0); +x_87 = lean_ctor_get(x_65, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_65); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; +} +} +} +else +{ +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_61, 0); +x_90 = lean_ctor_get(x_61, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_61); +lean_inc(x_1); +x_91 = l_Lean_Meta_Grind_Goal_getRoot(x_89, x_1, x_18, x_19, x_90); +if (lean_obj_tag(x_91) == 0) +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); lean_dec(x_91); -x_94 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_92, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_93); -lean_dec(x_92); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_94 = l_Lean_Meta_Grind_ppENodeRef(x_92, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_93); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_98 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_56); +x_99 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; +lean_ctor_set_tag(x_44, 7); +lean_ctor_set(x_44, 1, x_99); +lean_ctor_set(x_44, 0, x_98); +lean_ctor_set_tag(x_29, 7); +lean_ctor_set(x_29, 1, x_59); +lean_ctor_set(x_29, 0, x_44); +x_100 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; +x_101 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_101, 0, x_29); +lean_ctor_set(x_101, 1, x_100); +x_102 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_102, 0, x_101); +lean_ctor_set(x_102, 1, x_95); +x_103 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_103, 0, x_102); +lean_ctor_set(x_103, 1, x_97); +x_104 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_103, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_96); +x_105 = lean_ctor_get(x_104, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_104, 1); +lean_inc(x_106); +lean_dec(x_104); +x_107 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_1, x_33, x_9, x_24, x_35, x_34, x_41, x_6, x_10, x_37, x_36, x_105, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_106); +lean_dec(x_105); +lean_dec(x_35); +return x_107; +} +else +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +lean_dec(x_59); +lean_dec(x_56); +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_108 = lean_ctor_get(x_94, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_94, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_110 = x_94; +} else { + lean_dec_ref(x_94); + x_110 = lean_box(0); +} +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(1, 2, 0); +} else { + x_111 = x_110; +} +lean_ctor_set(x_111, 0, x_108); +lean_ctor_set(x_111, 1, x_109); +return x_111; +} +} +else +{ +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +lean_dec(x_59); +lean_dec(x_56); +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_112 = lean_ctor_get(x_91, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_91, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_91)) { + lean_ctor_release(x_91, 0); + lean_ctor_release(x_91, 1); + x_114 = x_91; +} else { + lean_dec_ref(x_91); + x_114 = lean_box(0); +} +if (lean_is_scalar(x_114)) { + x_115 = lean_alloc_ctor(1, 2, 0); +} else { + x_115 = x_114; +} +lean_ctor_set(x_115, 0, x_112); +lean_ctor_set(x_115, 1, x_113); +return x_115; +} +} +} +else +{ +uint8_t x_116; +lean_dec(x_56); +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_116 = !lean_is_exclusive(x_58); +if (x_116 == 0) +{ +return x_58; +} +else +{ +lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_117 = lean_ctor_get(x_58, 0); +x_118 = lean_ctor_get(x_58, 1); +lean_inc(x_118); +lean_inc(x_117); +lean_dec(x_58); +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_117); +lean_ctor_set(x_119, 1, x_118); +return x_119; +} +} +} +else +{ +uint8_t x_120; +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_120 = !lean_is_exclusive(x_55); +if (x_120 == 0) +{ +return x_55; +} +else +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; +x_121 = lean_ctor_get(x_55, 0); +x_122 = lean_ctor_get(x_55, 1); +lean_inc(x_122); +lean_inc(x_121); +lean_dec(x_55); +x_123 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_123, 0, x_121); +lean_ctor_set(x_123, 1, x_122); +return x_123; +} +} +} +else +{ +uint8_t x_124; +lean_free_object(x_44); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_124 = !lean_is_exclusive(x_53); +if (x_124 == 0) +{ +return x_53; +} +else +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_53, 0); +x_126 = lean_ctor_get(x_53, 1); +lean_inc(x_126); +lean_inc(x_125); +lean_dec(x_53); +x_127 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_127, 0, x_125); +lean_ctor_set(x_127, 1, x_126); +return x_127; +} +} +} +else +{ +lean_object* x_128; lean_object* x_129; +x_128 = lean_ctor_get(x_44, 1); +lean_inc(x_128); +lean_dec(x_44); +x_129 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_128); +if (lean_obj_tag(x_129) == 0) +{ +lean_object* x_130; lean_object* x_131; +x_130 = lean_ctor_get(x_129, 1); +lean_inc(x_130); +lean_dec(x_129); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_1); +x_131 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_130); +if (lean_obj_tag(x_131) == 0) +{ +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_131, 1); +lean_inc(x_133); +lean_dec(x_131); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_41); +x_134 = l_Lean_Meta_Grind_ppENodeRef(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_133); +if (lean_obj_tag(x_134) == 0) +{ +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_135 = lean_ctor_get(x_134, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_134, 1); +lean_inc(x_136); +lean_dec(x_134); +x_137 = lean_st_ref_get(x_12, x_136); +x_138 = lean_ctor_get(x_137, 0); +lean_inc(x_138); +x_139 = lean_ctor_get(x_137, 1); +lean_inc(x_139); +if (lean_is_exclusive(x_137)) { + lean_ctor_release(x_137, 0); + lean_ctor_release(x_137, 1); + x_140 = x_137; +} else { + lean_dec_ref(x_137); + x_140 = lean_box(0); +} +lean_inc(x_1); +x_141 = l_Lean_Meta_Grind_Goal_getRoot(x_138, x_1, x_18, x_19, x_139); +if (lean_obj_tag(x_141) == 0) +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_142 = lean_ctor_get(x_141, 0); +lean_inc(x_142); +x_143 = lean_ctor_get(x_141, 1); +lean_inc(x_143); +lean_dec(x_141); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_144 = l_Lean_Meta_Grind_ppENodeRef(x_142, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_143); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_140)) { + x_148 = lean_alloc_ctor(7, 2, 0); +} else { + x_148 = x_140; + lean_ctor_set_tag(x_148, 7); +} +lean_ctor_set(x_148, 0, x_147); +lean_ctor_set(x_148, 1, x_132); +x_149 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; +x_150 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_150, 0, x_148); +lean_ctor_set(x_150, 1, x_149); +lean_ctor_set_tag(x_29, 7); +lean_ctor_set(x_29, 1, x_135); +lean_ctor_set(x_29, 0, x_150); +x_151 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; +x_152 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_152, 0, x_29); +lean_ctor_set(x_152, 1, x_151); +x_153 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_153, 0, x_152); +lean_ctor_set(x_153, 1, x_145); +x_154 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_154, 0, x_153); +lean_ctor_set(x_154, 1, x_147); +x_155 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_154, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_146); +x_156 = lean_ctor_get(x_155, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +lean_dec(x_155); +x_158 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_1, x_33, x_9, x_24, x_35, x_34, x_41, x_6, x_10, x_37, x_36, x_156, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_157); +lean_dec(x_156); lean_dec(x_35); -return x_94; +return x_158; +} +else +{ +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; +lean_dec(x_140); +lean_dec(x_135); +lean_dec(x_132); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_159 = lean_ctor_get(x_144, 0); +lean_inc(x_159); +x_160 = lean_ctor_get(x_144, 1); +lean_inc(x_160); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_161 = x_144; +} else { + lean_dec_ref(x_144); + x_161 = lean_box(0); +} +if (lean_is_scalar(x_161)) { + x_162 = lean_alloc_ctor(1, 2, 0); +} else { + x_162 = x_161; +} +lean_ctor_set(x_162, 0, x_159); +lean_ctor_set(x_162, 1, x_160); +return x_162; +} +} +else +{ +lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; +lean_dec(x_140); +lean_dec(x_135); +lean_dec(x_132); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_163 = lean_ctor_get(x_141, 0); +lean_inc(x_163); +x_164 = lean_ctor_get(x_141, 1); +lean_inc(x_164); +if (lean_is_exclusive(x_141)) { + lean_ctor_release(x_141, 0); + lean_ctor_release(x_141, 1); + x_165 = x_141; +} else { + lean_dec_ref(x_141); + x_165 = lean_box(0); +} +if (lean_is_scalar(x_165)) { + x_166 = lean_alloc_ctor(1, 2, 0); +} else { + x_166 = x_165; +} +lean_ctor_set(x_166, 0, x_163); +lean_ctor_set(x_166, 1, x_164); +return x_166; +} +} +else +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; +lean_dec(x_132); +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_167 = lean_ctor_get(x_134, 0); +lean_inc(x_167); +x_168 = lean_ctor_get(x_134, 1); +lean_inc(x_168); +if (lean_is_exclusive(x_134)) { + lean_ctor_release(x_134, 0); + lean_ctor_release(x_134, 1); + x_169 = x_134; +} else { + lean_dec_ref(x_134); + x_169 = lean_box(0); +} +if (lean_is_scalar(x_169)) { + x_170 = lean_alloc_ctor(1, 2, 0); +} else { + x_170 = x_169; +} +lean_ctor_set(x_170, 0, x_167); +lean_ctor_set(x_170, 1, x_168); +return x_170; +} +} +else +{ +lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_171 = lean_ctor_get(x_131, 0); +lean_inc(x_171); +x_172 = lean_ctor_get(x_131, 1); +lean_inc(x_172); +if (lean_is_exclusive(x_131)) { + lean_ctor_release(x_131, 0); + lean_ctor_release(x_131, 1); + x_173 = x_131; +} else { + lean_dec_ref(x_131); + x_173 = lean_box(0); +} +if (lean_is_scalar(x_173)) { + x_174 = lean_alloc_ctor(1, 2, 0); +} else { + x_174 = x_173; +} +lean_ctor_set(x_174, 0, x_171); +lean_ctor_set(x_174, 1, x_172); +return x_174; +} +} +else +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_175 = lean_ctor_get(x_129, 0); +lean_inc(x_175); +x_176 = lean_ctor_get(x_129, 1); +lean_inc(x_176); +if (lean_is_exclusive(x_129)) { + lean_ctor_release(x_129, 0); + lean_ctor_release(x_129, 1); + x_177 = x_129; +} else { + lean_dec_ref(x_129); + x_177 = lean_box(0); +} +if (lean_is_scalar(x_177)) { + x_178 = lean_alloc_ctor(1, 2, 0); +} else { + x_178 = x_177; +} +lean_ctor_set(x_178, 0, x_175); +lean_ctor_set(x_178, 1, x_176); +return x_178; +} +} +} +} +else +{ +uint8_t x_179; +lean_dec(x_41); +lean_dec(x_39); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_179 = !lean_is_exclusive(x_42); +if (x_179 == 0) +{ +return x_42; +} +else +{ +lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_42, 0); +x_181 = lean_ctor_get(x_42, 1); +lean_inc(x_181); +lean_inc(x_180); +lean_dec(x_42); +x_182 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_182, 0, x_180); +lean_ctor_set(x_182, 1, x_181); +return x_182; +} +} +} +else +{ +uint8_t x_183; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); +lean_free_object(x_29); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_183 = !lean_is_exclusive(x_38); +if (x_183 == 0) +{ +return x_38; +} +else +{ +lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_184 = lean_ctor_get(x_38, 0); +x_185 = lean_ctor_get(x_38, 1); +lean_inc(x_185); +lean_inc(x_184); +lean_dec(x_38); +x_186 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_186, 0, x_184); +lean_ctor_set(x_186, 1, x_185); +return x_186; +} +} +} +else +{ +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; uint8_t x_191; uint8_t x_192; lean_object* x_193; +x_187 = lean_ctor_get(x_29, 1); +lean_inc(x_187); +lean_dec(x_29); +x_188 = lean_ctor_get(x_6, 0); +lean_inc(x_188); +x_189 = lean_ctor_get(x_6, 1); +lean_inc(x_189); +x_190 = lean_ctor_get(x_6, 6); +lean_inc(x_190); +x_191 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 3); +x_192 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 4); +x_193 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_188, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_187); +if (lean_obj_tag(x_193) == 0) +{ +lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; +x_194 = lean_ctor_get(x_193, 0); +lean_inc(x_194); +x_195 = lean_ctor_get(x_193, 1); +lean_inc(x_195); +lean_dec(x_193); +x_196 = lean_ctor_get(x_7, 2); +lean_inc(x_196); +lean_dec(x_7); +lean_inc(x_196); +lean_inc(x_1); +x_197 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(x_1, x_196, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_195); +if (lean_obj_tag(x_197) == 0) +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; uint8_t x_201; +x_198 = lean_ctor_get(x_197, 1); +lean_inc(x_198); +lean_dec(x_197); +lean_inc(x_8); +x_199 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_198); +x_200 = lean_ctor_get(x_199, 0); +lean_inc(x_200); +x_201 = lean_unbox(x_200); +lean_dec(x_200); +if (x_201 == 0) +{ +lean_object* x_202; lean_object* x_203; lean_object* x_204; +lean_dec(x_8); +x_202 = lean_ctor_get(x_199, 1); +lean_inc(x_202); +lean_dec(x_199); +x_203 = lean_box(0); +x_204 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_194, x_1, x_188, x_9, x_24, x_190, x_189, x_196, x_6, x_10, x_192, x_191, x_203, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_202); +lean_dec(x_190); +return x_204; +} +else +{ +lean_object* x_205; lean_object* x_206; lean_object* x_207; +x_205 = lean_ctor_get(x_199, 1); +lean_inc(x_205); +if (lean_is_exclusive(x_199)) { + lean_ctor_release(x_199, 0); + lean_ctor_release(x_199, 1); + x_206 = x_199; +} else { + lean_dec_ref(x_199); + x_206 = lean_box(0); +} +x_207 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_205); +if (lean_obj_tag(x_207) == 0) +{ +lean_object* x_208; lean_object* x_209; +x_208 = lean_ctor_get(x_207, 1); +lean_inc(x_208); +lean_dec(x_207); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_1); +x_209 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_208); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_196); +x_212 = l_Lean_Meta_Grind_ppENodeRef(x_196, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_211); +if (lean_obj_tag(x_212) == 0) +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; +x_213 = lean_ctor_get(x_212, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_212, 1); +lean_inc(x_214); +lean_dec(x_212); +x_215 = lean_st_ref_get(x_12, x_214); +x_216 = lean_ctor_get(x_215, 0); +lean_inc(x_216); +x_217 = lean_ctor_get(x_215, 1); +lean_inc(x_217); +if (lean_is_exclusive(x_215)) { + lean_ctor_release(x_215, 0); + lean_ctor_release(x_215, 1); + x_218 = x_215; +} else { + lean_dec_ref(x_215); + x_218 = lean_box(0); +} +lean_inc(x_1); +x_219 = l_Lean_Meta_Grind_Goal_getRoot(x_216, x_1, x_18, x_19, x_217); +if (lean_obj_tag(x_219) == 0) +{ +lean_object* x_220; lean_object* x_221; lean_object* x_222; +x_220 = lean_ctor_get(x_219, 0); +lean_inc(x_220); +x_221 = lean_ctor_get(x_219, 1); +lean_inc(x_221); +lean_dec(x_219); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_222 = l_Lean_Meta_Grind_ppENodeRef(x_220, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_221); +if (lean_obj_tag(x_222) == 0) +{ +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; +x_223 = lean_ctor_get(x_222, 0); +lean_inc(x_223); +x_224 = lean_ctor_get(x_222, 1); +lean_inc(x_224); +lean_dec(x_222); +x_225 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_218)) { + x_226 = lean_alloc_ctor(7, 2, 0); +} else { + x_226 = x_218; + lean_ctor_set_tag(x_226, 7); +} +lean_ctor_set(x_226, 0, x_225); +lean_ctor_set(x_226, 1, x_210); +x_227 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; +if (lean_is_scalar(x_206)) { + x_228 = lean_alloc_ctor(7, 2, 0); +} else { + x_228 = x_206; + lean_ctor_set_tag(x_228, 7); +} +lean_ctor_set(x_228, 0, x_226); +lean_ctor_set(x_228, 1, x_227); +x_229 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_229, 0, x_228); +lean_ctor_set(x_229, 1, x_213); +x_230 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; +x_231 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_231, 0, x_229); +lean_ctor_set(x_231, 1, x_230); +x_232 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_232, 0, x_231); +lean_ctor_set(x_232, 1, x_223); +x_233 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_233, 0, x_232); +lean_ctor_set(x_233, 1, x_225); +x_234 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_233, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_224); +x_235 = lean_ctor_get(x_234, 0); +lean_inc(x_235); +x_236 = lean_ctor_get(x_234, 1); +lean_inc(x_236); +lean_dec(x_234); +x_237 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_194, x_1, x_188, x_9, x_24, x_190, x_189, x_196, x_6, x_10, x_192, x_191, x_235, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_236); +lean_dec(x_235); +lean_dec(x_190); +return x_237; +} +else +{ +lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +lean_dec(x_218); +lean_dec(x_213); +lean_dec(x_210); +lean_dec(x_206); +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_238 = lean_ctor_get(x_222, 0); +lean_inc(x_238); +x_239 = lean_ctor_get(x_222, 1); +lean_inc(x_239); +if (lean_is_exclusive(x_222)) { + lean_ctor_release(x_222, 0); + lean_ctor_release(x_222, 1); + x_240 = x_222; +} else { + lean_dec_ref(x_222); + x_240 = lean_box(0); +} +if (lean_is_scalar(x_240)) { + x_241 = lean_alloc_ctor(1, 2, 0); +} else { + x_241 = x_240; +} +lean_ctor_set(x_241, 0, x_238); +lean_ctor_set(x_241, 1, x_239); +return x_241; +} +} +else +{ +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +lean_dec(x_218); +lean_dec(x_213); +lean_dec(x_210); +lean_dec(x_206); +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_242 = lean_ctor_get(x_219, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_219, 1); +lean_inc(x_243); +if (lean_is_exclusive(x_219)) { + lean_ctor_release(x_219, 0); + lean_ctor_release(x_219, 1); + x_244 = x_219; +} else { + lean_dec_ref(x_219); + x_244 = lean_box(0); +} +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(1, 2, 0); +} else { + x_245 = x_244; +} +lean_ctor_set(x_245, 0, x_242); +lean_ctor_set(x_245, 1, x_243); +return x_245; +} +} +else +{ +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_210); +lean_dec(x_206); +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_246 = lean_ctor_get(x_212, 0); +lean_inc(x_246); +x_247 = lean_ctor_get(x_212, 1); +lean_inc(x_247); +if (lean_is_exclusive(x_212)) { + lean_ctor_release(x_212, 0); + lean_ctor_release(x_212, 1); + x_248 = x_212; +} else { + lean_dec_ref(x_212); + x_248 = lean_box(0); +} +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); +} else { + x_249 = x_248; +} +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; +} +} +else +{ +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; +lean_dec(x_206); +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_250 = lean_ctor_get(x_209, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_209, 1); +lean_inc(x_251); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_252 = x_209; +} else { + lean_dec_ref(x_209); + x_252 = lean_box(0); +} +if (lean_is_scalar(x_252)) { + x_253 = lean_alloc_ctor(1, 2, 0); +} else { + x_253 = x_252; +} +lean_ctor_set(x_253, 0, x_250); +lean_ctor_set(x_253, 1, x_251); +return x_253; +} +} +else +{ +lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; +lean_dec(x_206); +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_254 = lean_ctor_get(x_207, 0); +lean_inc(x_254); +x_255 = lean_ctor_get(x_207, 1); +lean_inc(x_255); +if (lean_is_exclusive(x_207)) { + lean_ctor_release(x_207, 0); + lean_ctor_release(x_207, 1); + x_256 = x_207; +} else { + lean_dec_ref(x_207); + x_256 = lean_box(0); +} +if (lean_is_scalar(x_256)) { + x_257 = lean_alloc_ctor(1, 2, 0); +} else { + x_257 = x_256; +} +lean_ctor_set(x_257, 0, x_254); +lean_ctor_set(x_257, 1, x_255); +return x_257; +} +} +} +else +{ +lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; +lean_dec(x_196); +lean_dec(x_194); +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_258 = lean_ctor_get(x_197, 0); +lean_inc(x_258); +x_259 = lean_ctor_get(x_197, 1); +lean_inc(x_259); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_260 = x_197; +} else { + lean_dec_ref(x_197); + x_260 = lean_box(0); +} +if (lean_is_scalar(x_260)) { + x_261 = lean_alloc_ctor(1, 2, 0); +} else { + x_261 = x_260; +} +lean_ctor_set(x_261, 0, x_258); +lean_ctor_set(x_261, 1, x_259); +return x_261; +} +} +else +{ +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; +lean_dec(x_190); +lean_dec(x_189); +lean_dec(x_188); +lean_dec(x_24); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_262 = lean_ctor_get(x_193, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_193, 1); +lean_inc(x_263); +if (lean_is_exclusive(x_193)) { + lean_ctor_release(x_193, 0); + lean_ctor_release(x_193, 1); + x_264 = x_193; +} else { + lean_dec_ref(x_193); + x_264 = lean_box(0); +} +if (lean_is_scalar(x_264)) { + x_265 = lean_alloc_ctor(1, 2, 0); +} else { + x_265 = x_264; +} +lean_ctor_set(x_265, 0, x_262); +lean_ctor_set(x_265, 1, x_263); +return x_265; +} +} +} +else +{ +lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; lean_object* x_270; uint8_t x_271; uint8_t x_272; uint8_t x_273; uint8_t x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_object* x_286; lean_object* x_287; uint8_t x_288; uint8_t x_289; lean_object* x_290; +x_266 = lean_ctor_get(x_2, 0); +x_267 = lean_ctor_get(x_2, 1); +x_268 = lean_ctor_get(x_2, 2); +x_269 = lean_ctor_get(x_2, 3); +x_270 = lean_ctor_get(x_2, 6); +x_271 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 1); +x_272 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 2); +x_273 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 3); +x_274 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 4); +x_275 = lean_ctor_get(x_2, 7); +x_276 = lean_ctor_get(x_2, 8); +x_277 = lean_ctor_get(x_2, 9); +x_278 = lean_ctor_get(x_2, 10); +lean_inc(x_278); +lean_inc(x_277); +lean_inc(x_276); +lean_inc(x_275); +lean_inc(x_270); +lean_inc(x_269); +lean_inc(x_268); +lean_inc(x_267); +lean_inc(x_266); +lean_dec(x_2); +x_279 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_279, 0, x_3); +x_280 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_280, 0, x_4); +lean_inc(x_268); +x_281 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_281, 0, x_266); +lean_ctor_set(x_281, 1, x_267); +lean_ctor_set(x_281, 2, x_268); +lean_ctor_set(x_281, 3, x_269); +lean_ctor_set(x_281, 4, x_279); +lean_ctor_set(x_281, 5, x_280); +lean_ctor_set(x_281, 6, x_270); +lean_ctor_set(x_281, 7, x_275); +lean_ctor_set(x_281, 8, x_276); +lean_ctor_set(x_281, 9, x_277); +lean_ctor_set(x_281, 10, x_278); +lean_ctor_set_uint8(x_281, sizeof(void*)*11, x_5); +lean_ctor_set_uint8(x_281, sizeof(void*)*11 + 1, x_271); +lean_ctor_set_uint8(x_281, sizeof(void*)*11 + 2, x_272); +lean_ctor_set_uint8(x_281, sizeof(void*)*11 + 3, x_273); +lean_ctor_set_uint8(x_281, sizeof(void*)*11 + 4, x_274); +lean_inc(x_1); +x_282 = l_Lean_Meta_Grind_setENode(x_1, x_281, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_22); +x_283 = lean_ctor_get(x_282, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_282)) { + lean_ctor_release(x_282, 0); + lean_ctor_release(x_282, 1); + x_284 = x_282; +} else { + lean_dec_ref(x_282); + x_284 = lean_box(0); +} +x_285 = lean_ctor_get(x_6, 0); +lean_inc(x_285); +x_286 = lean_ctor_get(x_6, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_6, 6); +lean_inc(x_287); +x_288 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 3); +x_289 = lean_ctor_get_uint8(x_6, sizeof(void*)*11 + 4); +x_290 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_285, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_283); +if (lean_obj_tag(x_290) == 0) +{ +lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; +x_291 = lean_ctor_get(x_290, 0); +lean_inc(x_291); +x_292 = lean_ctor_get(x_290, 1); +lean_inc(x_292); +lean_dec(x_290); +x_293 = lean_ctor_get(x_7, 2); +lean_inc(x_293); +lean_dec(x_7); +lean_inc(x_293); +lean_inc(x_1); +x_294 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots(x_1, x_293, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_292); +if (lean_obj_tag(x_294) == 0) +{ +lean_object* x_295; lean_object* x_296; lean_object* x_297; uint8_t x_298; +x_295 = lean_ctor_get(x_294, 1); +lean_inc(x_295); +lean_dec(x_294); +lean_inc(x_8); +x_296 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_295); +x_297 = lean_ctor_get(x_296, 0); +lean_inc(x_297); +x_298 = lean_unbox(x_297); +lean_dec(x_297); +if (x_298 == 0) +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; +lean_dec(x_284); +lean_dec(x_8); +x_299 = lean_ctor_get(x_296, 1); +lean_inc(x_299); +lean_dec(x_296); +x_300 = lean_box(0); +x_301 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_291, x_1, x_285, x_9, x_268, x_287, x_286, x_293, x_6, x_10, x_289, x_288, x_300, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_299); +lean_dec(x_287); +return x_301; +} +else +{ +lean_object* x_302; lean_object* x_303; lean_object* x_304; +x_302 = lean_ctor_get(x_296, 1); +lean_inc(x_302); +if (lean_is_exclusive(x_296)) { + lean_ctor_release(x_296, 0); + lean_ctor_release(x_296, 1); + x_303 = x_296; +} else { + lean_dec_ref(x_296); + x_303 = lean_box(0); +} +x_304 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_302); +if (lean_obj_tag(x_304) == 0) +{ +lean_object* x_305; lean_object* x_306; +x_305 = lean_ctor_get(x_304, 1); +lean_inc(x_305); +lean_dec(x_304); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_1); +x_306 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_305); +if (lean_obj_tag(x_306) == 0) +{ +lean_object* x_307; lean_object* x_308; lean_object* x_309; +x_307 = lean_ctor_get(x_306, 0); +lean_inc(x_307); +x_308 = lean_ctor_get(x_306, 1); +lean_inc(x_308); +lean_dec(x_306); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_293); +x_309 = l_Lean_Meta_Grind_ppENodeRef(x_293, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_308); +if (lean_obj_tag(x_309) == 0) +{ +lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; lean_object* x_314; lean_object* x_315; lean_object* x_316; +x_310 = lean_ctor_get(x_309, 0); +lean_inc(x_310); +x_311 = lean_ctor_get(x_309, 1); +lean_inc(x_311); +lean_dec(x_309); +x_312 = lean_st_ref_get(x_12, x_311); +x_313 = lean_ctor_get(x_312, 0); +lean_inc(x_313); +x_314 = lean_ctor_get(x_312, 1); +lean_inc(x_314); +if (lean_is_exclusive(x_312)) { + lean_ctor_release(x_312, 0); + lean_ctor_release(x_312, 1); + x_315 = x_312; +} else { + lean_dec_ref(x_312); + x_315 = lean_box(0); +} +lean_inc(x_1); +x_316 = l_Lean_Meta_Grind_Goal_getRoot(x_313, x_1, x_18, x_19, x_314); +if (lean_obj_tag(x_316) == 0) +{ +lean_object* x_317; lean_object* x_318; lean_object* x_319; +x_317 = lean_ctor_get(x_316, 0); +lean_inc(x_317); +x_318 = lean_ctor_get(x_316, 1); +lean_inc(x_318); +lean_dec(x_316); +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +x_319 = l_Lean_Meta_Grind_ppENodeRef(x_317, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_318); +if (lean_obj_tag(x_319) == 0) +{ +lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; +x_320 = lean_ctor_get(x_319, 0); +lean_inc(x_320); +x_321 = lean_ctor_get(x_319, 1); +lean_inc(x_321); +lean_dec(x_319); +x_322 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_315)) { + x_323 = lean_alloc_ctor(7, 2, 0); +} else { + x_323 = x_315; + lean_ctor_set_tag(x_323, 7); +} +lean_ctor_set(x_323, 0, x_322); +lean_ctor_set(x_323, 1, x_307); +x_324 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; +if (lean_is_scalar(x_303)) { + x_325 = lean_alloc_ctor(7, 2, 0); +} else { + x_325 = x_303; + lean_ctor_set_tag(x_325, 7); +} +lean_ctor_set(x_325, 0, x_323); +lean_ctor_set(x_325, 1, x_324); +if (lean_is_scalar(x_284)) { + x_326 = lean_alloc_ctor(7, 2, 0); +} else { + x_326 = x_284; + lean_ctor_set_tag(x_326, 7); +} +lean_ctor_set(x_326, 0, x_325); +lean_ctor_set(x_326, 1, x_310); +x_327 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; +x_328 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_328, 0, x_326); +lean_ctor_set(x_328, 1, x_327); +x_329 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_329, 0, x_328); +lean_ctor_set(x_329, 1, x_320); +x_330 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_330, 0, x_329); +lean_ctor_set(x_330, 1, x_322); +x_331 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_330, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_321); +x_332 = lean_ctor_get(x_331, 0); +lean_inc(x_332); +x_333 = lean_ctor_get(x_331, 1); +lean_inc(x_333); +lean_dec(x_331); +x_334 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_291, x_1, x_285, x_9, x_268, x_287, x_286, x_293, x_6, x_10, x_289, x_288, x_332, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_333); +lean_dec(x_332); +lean_dec(x_287); +return x_334; +} +else +{ +lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; +lean_dec(x_315); +lean_dec(x_310); +lean_dec(x_307); +lean_dec(x_303); +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_335 = lean_ctor_get(x_319, 0); +lean_inc(x_335); +x_336 = lean_ctor_get(x_319, 1); +lean_inc(x_336); +if (lean_is_exclusive(x_319)) { + lean_ctor_release(x_319, 0); + lean_ctor_release(x_319, 1); + x_337 = x_319; +} else { + lean_dec_ref(x_319); + x_337 = lean_box(0); +} +if (lean_is_scalar(x_337)) { + x_338 = lean_alloc_ctor(1, 2, 0); +} else { + x_338 = x_337; +} +lean_ctor_set(x_338, 0, x_335); +lean_ctor_set(x_338, 1, x_336); +return x_338; +} +} +else +{ +lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; +lean_dec(x_315); +lean_dec(x_310); +lean_dec(x_307); +lean_dec(x_303); +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_339 = lean_ctor_get(x_316, 0); +lean_inc(x_339); +x_340 = lean_ctor_get(x_316, 1); +lean_inc(x_340); +if (lean_is_exclusive(x_316)) { + lean_ctor_release(x_316, 0); + lean_ctor_release(x_316, 1); + x_341 = x_316; +} else { + lean_dec_ref(x_316); + x_341 = lean_box(0); +} +if (lean_is_scalar(x_341)) { + x_342 = lean_alloc_ctor(1, 2, 0); +} else { + x_342 = x_341; +} +lean_ctor_set(x_342, 0, x_339); +lean_ctor_set(x_342, 1, x_340); +return x_342; +} +} +else +{ +lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; +lean_dec(x_307); +lean_dec(x_303); +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_343 = lean_ctor_get(x_309, 0); +lean_inc(x_343); +x_344 = lean_ctor_get(x_309, 1); +lean_inc(x_344); +if (lean_is_exclusive(x_309)) { + lean_ctor_release(x_309, 0); + lean_ctor_release(x_309, 1); + x_345 = x_309; +} else { + lean_dec_ref(x_309); + x_345 = lean_box(0); +} +if (lean_is_scalar(x_345)) { + x_346 = lean_alloc_ctor(1, 2, 0); +} else { + x_346 = x_345; +} +lean_ctor_set(x_346, 0, x_343); +lean_ctor_set(x_346, 1, x_344); +return x_346; +} +} +else +{ +lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; +lean_dec(x_303); +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_347 = lean_ctor_get(x_306, 0); +lean_inc(x_347); +x_348 = lean_ctor_get(x_306, 1); +lean_inc(x_348); +if (lean_is_exclusive(x_306)) { + lean_ctor_release(x_306, 0); + lean_ctor_release(x_306, 1); + x_349 = x_306; +} else { + lean_dec_ref(x_306); + x_349 = lean_box(0); +} +if (lean_is_scalar(x_349)) { + x_350 = lean_alloc_ctor(1, 2, 0); +} else { + x_350 = x_349; +} +lean_ctor_set(x_350, 0, x_347); +lean_ctor_set(x_350, 1, x_348); +return x_350; +} +} +else +{ +lean_object* x_351; lean_object* x_352; lean_object* x_353; lean_object* x_354; +lean_dec(x_303); +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_351 = lean_ctor_get(x_304, 0); +lean_inc(x_351); +x_352 = lean_ctor_get(x_304, 1); +lean_inc(x_352); +if (lean_is_exclusive(x_304)) { + lean_ctor_release(x_304, 0); + lean_ctor_release(x_304, 1); + x_353 = x_304; +} else { + lean_dec_ref(x_304); + x_353 = lean_box(0); +} +if (lean_is_scalar(x_353)) { + x_354 = lean_alloc_ctor(1, 2, 0); +} else { + x_354 = x_353; +} +lean_ctor_set(x_354, 0, x_351); +lean_ctor_set(x_354, 1, x_352); +return x_354; +} +} +} +else +{ +lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; +lean_dec(x_293); +lean_dec(x_291); +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_355 = lean_ctor_get(x_294, 0); +lean_inc(x_355); +x_356 = lean_ctor_get(x_294, 1); +lean_inc(x_356); +if (lean_is_exclusive(x_294)) { + lean_ctor_release(x_294, 0); + lean_ctor_release(x_294, 1); + x_357 = x_294; +} else { + lean_dec_ref(x_294); + x_357 = lean_box(0); +} +if (lean_is_scalar(x_357)) { + x_358 = lean_alloc_ctor(1, 2, 0); +} else { + x_358 = x_357; +} +lean_ctor_set(x_358, 0, x_355); +lean_ctor_set(x_358, 1, x_356); +return x_358; +} +} +else +{ +lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; +lean_dec(x_287); +lean_dec(x_286); +lean_dec(x_285); +lean_dec(x_284); +lean_dec(x_268); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_1); +x_359 = lean_ctor_get(x_290, 0); +lean_inc(x_359); +x_360 = lean_ctor_get(x_290, 1); +lean_inc(x_360); +if (lean_is_exclusive(x_290)) { + lean_ctor_release(x_290, 0); + lean_ctor_release(x_290, 1); + x_361 = x_290; +} else { + lean_dec_ref(x_290); + x_361 = lean_box(0); +} +if (lean_is_scalar(x_361)) { + x_362 = lean_alloc_ctor(1, 2, 0); +} else { + x_362 = x_361; +} +lean_ctor_set(x_362, 0, x_359); +lean_ctor_set(x_362, 1, x_360); +return x_362; +} +} +} +else +{ +uint8_t x_363; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_363 = !lean_is_exclusive(x_21); +if (x_363 == 0) +{ +return x_21; +} +else +{ +lean_object* x_364; lean_object* x_365; lean_object* x_366; +x_364 = lean_ctor_get(x_21, 0); +x_365 = lean_ctor_get(x_21, 1); +lean_inc(x_365); +lean_inc(x_364); +lean_dec(x_21); +x_366 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_366, 0, x_364); +lean_ctor_set(x_366, 1, x_365); +return x_366; +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; +x_2 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__2; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("adding ", 7, 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" ↦ ", 5, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; +x_20 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_unbox(x_21); +lean_dec(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = lean_box(0); +x_25 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_23); +return x_25; +} +else +{ +uint8_t x_26; +x_26 = !lean_is_exclusive(x_20); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_20, 1); +x_28 = lean_ctor_get(x_20, 0); +lean_dec(x_28); +x_29 = l_Lean_Meta_Grind_updateLastTag(x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_27); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_29, 1); +lean_inc(x_30); +lean_dec(x_29); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_3); +x_31 = l_Lean_Meta_Grind_ppENodeRef(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_30); +if (lean_obj_tag(x_31) == 0) +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_4); +x_34 = l_Lean_Meta_Grind_ppENodeRef(x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_33); +if (lean_obj_tag(x_34) == 0) +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; +lean_ctor_set_tag(x_20, 7); +lean_ctor_set(x_20, 1, x_32); +lean_ctor_set(x_20, 0, x_37); +x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; +x_39 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_39, 0, x_20); +lean_ctor_set(x_39, 1, x_38); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_35); +x_41 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_42, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_36); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_44, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_45); +lean_dec(x_44); +return x_46; +} +else +{ +uint8_t x_47; +lean_dec(x_32); +lean_free_object(x_20); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_47 = !lean_is_exclusive(x_34); +if (x_47 == 0) +{ +return x_34; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_34, 0); +x_49 = lean_ctor_get(x_34, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_34); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; +} +} +} +else +{ +uint8_t x_51; +lean_free_object(x_20); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_51 = !lean_is_exclusive(x_31); +if (x_51 == 0) +{ +return x_31; +} +else +{ +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_31, 0); +x_53 = lean_ctor_get(x_31, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_31); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +} +} +else +{ +uint8_t x_55; +lean_free_object(x_20); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_55 = !lean_is_exclusive(x_29); +if (x_55 == 0) +{ +return x_29; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_29, 0); +x_57 = lean_ctor_get(x_29, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_29); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; +} +} +} +else +{ +lean_object* x_59; lean_object* x_60; +x_59 = lean_ctor_get(x_20, 1); +lean_inc(x_59); +lean_dec(x_20); +x_60 = l_Lean_Meta_Grind_updateLastTag(x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_59); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_60, 1); +lean_inc(x_61); +lean_dec(x_60); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_3); +x_62 = l_Lean_Meta_Grind_ppENodeRef(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_61); +if (lean_obj_tag(x_62) == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_62, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_62, 1); +lean_inc(x_64); +lean_dec(x_62); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_4); +x_65 = l_Lean_Meta_Grind_ppENodeRef(x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_64); +if (lean_obj_tag(x_65) == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; +x_69 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_63); +x_70 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +x_72 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_66); +x_73 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_74 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +x_75 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_74, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_67); +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +lean_dec(x_75); +x_78 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_76, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_77); +lean_dec(x_76); +return x_78; +} +else +{ +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +lean_dec(x_63); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_79 = lean_ctor_get(x_65, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_65, 1); +lean_inc(x_80); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_81 = x_65; +} else { + lean_dec_ref(x_65); + x_81 = lean_box(0); +} +if (lean_is_scalar(x_81)) { + x_82 = lean_alloc_ctor(1, 2, 0); +} else { + x_82 = x_81; +} +lean_ctor_set(x_82, 0, x_79); +lean_ctor_set(x_82, 1, x_80); +return x_82; } } else { -uint8_t x_95; -lean_free_object(x_59); -lean_dec(x_61); -lean_free_object(x_55); -lean_dec(x_57); -lean_free_object(x_44); -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_83 = lean_ctor_get(x_62, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_62, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_85 = x_62; +} else { + lean_dec_ref(x_62); + x_85 = lean_box(0); +} +if (lean_is_scalar(x_85)) { + x_86 = lean_alloc_ctor(1, 2, 0); +} else { + x_86 = x_85; +} +lean_ctor_set(x_86, 0, x_83); +lean_ctor_set(x_86, 1, x_84); +return x_86; +} +} +else +{ +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_87 = lean_ctor_get(x_60, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_60, 1); +lean_inc(x_88); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_89 = x_60; +} else { + lean_dec_ref(x_60); + x_89 = lean_box(0); +} +if (lean_is_scalar(x_89)) { + x_90 = lean_alloc_ctor(1, 2, 0); +} else { + x_90 = x_89; +} +lean_ctor_set(x_90, 0, x_87); +lean_ctor_set(x_90, 1, x_88); +return x_90; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +lean_object* x_21 = _args[20]; +lean_object* x_22 = _args[21]; +_start: +{ +uint8_t x_23; uint8_t x_24; uint8_t x_25; lean_object* x_26; +x_23 = lean_unbox(x_10); +lean_dec(x_10); +x_24 = lean_unbox(x_11); +lean_dec(x_11); +x_25 = lean_unbox(x_12); +lean_dec(x_12); +x_26 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23, x_24, x_25, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22); +lean_dec(x_13); +lean_dec(x_6); +return x_26; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +_start: +{ +uint8_t x_21; uint8_t x_22; lean_object* x_23; +x_21 = lean_unbox(x_5); +lean_dec(x_5); +x_22 = lean_unbox(x_10); +lean_dec(x_10); +x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_1, x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_9, x_22, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +lean_dec(x_11); +return x_23; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +_start: +{ +uint8_t x_19; uint8_t x_20; lean_object* x_21; +x_19 = lean_unbox(x_2); +lean_dec(x_2); +x_20 = lean_unbox(x_9); +lean_dec(x_9); +x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_1, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +return x_21; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; lean_object* x_12; +x_11 = 0; +x_12 = l_Lean_Meta_Grind_checkInvariants(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_12; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("after addEqStep, ", 17, 17); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; +x_12 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1; +x_17 = lean_unbox(x_14); +lean_dec(x_14); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_free_object(x_12); +x_18 = lean_box(0); +x_19 = lean_apply_10(x_16, x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); +return x_19; +} +else +{ +lean_object* x_20; +x_20 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_get(x_2, x_21); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_26 = l_Lean_Meta_Grind_Goal_ppState(x_24, x_6, x_7, x_8, x_9, x_25); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; +lean_ctor_set_tag(x_22, 7); +lean_ctor_set(x_22, 1, x_27); +lean_ctor_set(x_22, 0, x_29); +x_30 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +lean_ctor_set_tag(x_12, 7); +lean_ctor_set(x_12, 1, x_30); +lean_ctor_set(x_12, 0, x_22); +x_31 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_11, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_28); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = lean_apply_10(x_16, x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_33); +return x_34; +} +else +{ +uint8_t x_35; +lean_free_object(x_22); +lean_free_object(x_12); lean_dec(x_9); lean_dec(x_8); -x_95 = !lean_is_exclusive(x_63); -if (x_95 == 0) +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_35 = !lean_is_exclusive(x_26); +if (x_35 == 0) { -return x_63; +return x_26; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_63, 0); -x_97 = lean_ctor_get(x_63, 1); -lean_inc(x_97); -lean_inc(x_96); -lean_dec(x_63); -x_98 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_26, 0); +x_37 = lean_ctor_get(x_26, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_26); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_59, 0); -x_100 = lean_ctor_get(x_59, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_59); -x_101 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_100); -if (lean_obj_tag(x_101) == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_22, 0); +x_40 = lean_ctor_get(x_22, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_22); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_41 = l_Lean_Meta_Grind_Goal_ppState(x_39, x_6, x_7, x_8, x_9, x_40); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_102 = lean_ctor_get(x_101, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_101, 1); -lean_inc(x_103); -lean_dec(x_101); -x_104 = l_Lean_Meta_Grind_ppENodeRef(x_102, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_103); -lean_dec(x_102); -x_105 = lean_ctor_get(x_104, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_104, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_104)) { - lean_ctor_release(x_104, 0); - lean_ctor_release(x_104, 1); - x_107 = x_104; -} else { - lean_dec_ref(x_104); - x_107 = lean_box(0); -} -x_108 = l_Lean_MessageData_ofFormat(x_57); -x_109 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_107)) { - x_110 = lean_alloc_ctor(7, 2, 0); -} else { - x_110 = x_107; - lean_ctor_set_tag(x_110, 7); -} -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_108); -x_111 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -x_112 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -x_113 = l_Lean_MessageData_ofFormat(x_99); -lean_ctor_set_tag(x_55, 7); -lean_ctor_set(x_55, 1, x_113); -lean_ctor_set(x_55, 0, x_112); -x_114 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -lean_ctor_set_tag(x_44, 7); -lean_ctor_set(x_44, 1, x_114); -lean_ctor_set(x_44, 0, x_55); -x_115 = l_Lean_MessageData_ofFormat(x_105); -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_115); -lean_ctor_set(x_29, 0, x_44); -x_116 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_116, 0, x_29); -lean_ctor_set(x_116, 1, x_109); -x_117 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_116, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_106); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_117, 1); -lean_inc(x_119); -lean_dec(x_117); -x_120 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_118, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_119); -lean_dec(x_118); -lean_dec(x_35); -return x_120; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_ctor_get(x_41, 1); +lean_inc(x_43); +lean_dec(x_41); +x_44 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_42); +x_46 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +lean_ctor_set_tag(x_12, 7); +lean_ctor_set(x_12, 1, x_46); +lean_ctor_set(x_12, 0, x_45); +x_47 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_11, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_43); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_apply_10(x_16, x_48, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_49); +return x_50; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -lean_dec(x_99); -lean_free_object(x_55); -lean_dec(x_57); -lean_free_object(x_44); -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_free_object(x_12); lean_dec(x_9); lean_dec(x_8); -x_121 = lean_ctor_get(x_101, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_101, 1); -lean_inc(x_122); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_123 = x_101; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_51 = lean_ctor_get(x_41, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_41, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + lean_ctor_release(x_41, 1); + x_53 = x_41; } else { - lean_dec_ref(x_101); - x_123 = lean_box(0); + lean_dec_ref(x_41); + x_53 = lean_box(0); } -if (lean_is_scalar(x_123)) { - x_124 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(1, 2, 0); } else { - x_124 = x_123; + x_54 = x_53; } -lean_ctor_set(x_124, 0, x_121); -lean_ctor_set(x_124, 1, x_122); -return x_124; +lean_ctor_set(x_54, 0, x_51); +lean_ctor_set(x_54, 1, x_52); +return x_54; } } } else { -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; -x_125 = lean_ctor_get(x_55, 0); -x_126 = lean_ctor_get(x_55, 1); -lean_inc(x_126); -lean_inc(x_125); -lean_dec(x_55); -x_127 = l_Lean_Meta_Grind_ppENodeRef(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_126); -x_128 = lean_ctor_get(x_127, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_127, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_127)) { - lean_ctor_release(x_127, 0); - lean_ctor_release(x_127, 1); - x_130 = x_127; -} else { - lean_dec_ref(x_127); - x_130 = lean_box(0); -} -x_131 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_129); -if (lean_obj_tag(x_131) == 0) +uint8_t x_55; +lean_free_object(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_55 = !lean_is_exclusive(x_20); +if (x_55 == 0) { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_132 = lean_ctor_get(x_131, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_131, 1); -lean_inc(x_133); -lean_dec(x_131); -x_134 = l_Lean_Meta_Grind_ppENodeRef(x_132, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_133); -lean_dec(x_132); -x_135 = lean_ctor_get(x_134, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_134, 1); -lean_inc(x_136); -if (lean_is_exclusive(x_134)) { - lean_ctor_release(x_134, 0); - lean_ctor_release(x_134, 1); - x_137 = x_134; -} else { - lean_dec_ref(x_134); - x_137 = lean_box(0); -} -x_138 = l_Lean_MessageData_ofFormat(x_125); -x_139 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_137)) { - x_140 = lean_alloc_ctor(7, 2, 0); -} else { - x_140 = x_137; - lean_ctor_set_tag(x_140, 7); -} -lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_138); -x_141 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -if (lean_is_scalar(x_130)) { - x_142 = lean_alloc_ctor(7, 2, 0); -} else { - x_142 = x_130; - lean_ctor_set_tag(x_142, 7); -} -lean_ctor_set(x_142, 0, x_140); -lean_ctor_set(x_142, 1, x_141); -x_143 = l_Lean_MessageData_ofFormat(x_128); -x_144 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_144, 0, x_142); -lean_ctor_set(x_144, 1, x_143); -x_145 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -lean_ctor_set_tag(x_44, 7); -lean_ctor_set(x_44, 1, x_145); -lean_ctor_set(x_44, 0, x_144); -x_146 = l_Lean_MessageData_ofFormat(x_135); -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_146); -lean_ctor_set(x_29, 0, x_44); -x_147 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_147, 0, x_29); -lean_ctor_set(x_147, 1, x_139); -x_148 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_147, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_136); -x_149 = lean_ctor_get(x_148, 0); -lean_inc(x_149); -x_150 = lean_ctor_get(x_148, 1); -lean_inc(x_150); -lean_dec(x_148); -x_151 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_149, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_150); -lean_dec(x_149); -lean_dec(x_35); -return x_151; +return x_20; } else { -lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; -lean_dec(x_130); -lean_dec(x_128); -lean_dec(x_125); -lean_free_object(x_44); -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_152 = lean_ctor_get(x_131, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_131, 1); -lean_inc(x_153); -if (lean_is_exclusive(x_131)) { - lean_ctor_release(x_131, 0); - lean_ctor_release(x_131, 1); - x_154 = x_131; -} else { - lean_dec_ref(x_131); - x_154 = lean_box(0); -} -if (lean_is_scalar(x_154)) { - x_155 = lean_alloc_ctor(1, 2, 0); -} else { - x_155 = x_154; +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_20, 0); +x_57 = lean_ctor_get(x_20, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_20); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; } -lean_ctor_set(x_155, 0, x_152); -lean_ctor_set(x_155, 1, x_153); -return x_155; } } } else { -uint8_t x_156; -lean_free_object(x_44); -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_59 = lean_ctor_get(x_12, 0); +x_60 = lean_ctor_get(x_12, 1); +lean_inc(x_60); +lean_inc(x_59); lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_156 = !lean_is_exclusive(x_53); -if (x_156 == 0) +x_61 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1; +x_62 = lean_unbox(x_59); +lean_dec(x_59); +if (x_62 == 0) { -return x_53; +lean_object* x_63; lean_object* x_64; +x_63 = lean_box(0); +x_64 = lean_apply_10(x_61, x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); +return x_64; +} +else +{ +lean_object* x_65; +x_65 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_60); +if (lean_obj_tag(x_65) == 0) +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_66 = lean_ctor_get(x_65, 1); +lean_inc(x_66); +lean_dec(x_65); +x_67 = lean_st_ref_get(x_2, x_66); +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_67)) { + lean_ctor_release(x_67, 0); + lean_ctor_release(x_67, 1); + x_70 = x_67; +} else { + lean_dec_ref(x_67); + x_70 = lean_box(0); +} +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_71 = l_Lean_Meta_Grind_Goal_ppState(x_68, x_6, x_7, x_8, x_9, x_69); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; +if (lean_is_scalar(x_70)) { + x_75 = lean_alloc_ctor(7, 2, 0); +} else { + x_75 = x_70; + lean_ctor_set_tag(x_75, 7); +} +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_72); +x_76 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_77 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +x_78 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_11, x_77, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_73); +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +x_81 = lean_apply_10(x_61, x_79, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_80); +return x_81; } else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_157 = lean_ctor_get(x_53, 0); -x_158 = lean_ctor_get(x_53, 1); -lean_inc(x_158); -lean_inc(x_157); -lean_dec(x_53); -x_159 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_159, 0, x_157); -lean_ctor_set(x_159, 1, x_158); -return x_159; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_dec(x_70); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_82 = lean_ctor_get(x_71, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_71, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_84 = x_71; +} else { + lean_dec_ref(x_71); + x_84 = lean_box(0); +} +if (lean_is_scalar(x_84)) { + x_85 = lean_alloc_ctor(1, 2, 0); +} else { + x_85 = x_84; } +lean_ctor_set(x_85, 0, x_82); +lean_ctor_set(x_85, 1, x_83); +return x_85; } } else { -lean_object* x_160; lean_object* x_161; -x_160 = lean_ctor_get(x_44, 1); -lean_inc(x_160); -lean_dec(x_44); -x_161 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_160); -if (lean_obj_tag(x_161) == 0) -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; -x_162 = lean_ctor_get(x_161, 1); -lean_inc(x_162); -lean_dec(x_161); -x_163 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_162); -x_164 = lean_ctor_get(x_163, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_163, 1); -lean_inc(x_165); -if (lean_is_exclusive(x_163)) { - lean_ctor_release(x_163, 0); - lean_ctor_release(x_163, 1); - x_166 = x_163; -} else { - lean_dec_ref(x_163); - x_166 = lean_box(0); -} -x_167 = l_Lean_Meta_Grind_ppENodeRef(x_41, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_165); -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_167, 1); -lean_inc(x_169); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_170 = x_167; +lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_86 = lean_ctor_get(x_65, 0); +lean_inc(x_86); +x_87 = lean_ctor_get(x_65, 1); +lean_inc(x_87); +if (lean_is_exclusive(x_65)) { + lean_ctor_release(x_65, 0); + lean_ctor_release(x_65, 1); + x_88 = x_65; } else { - lean_dec_ref(x_167); - x_170 = lean_box(0); + lean_dec_ref(x_65); + x_88 = lean_box(0); } -x_171 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_169); -if (lean_obj_tag(x_171) == 0) -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_171, 1); -lean_inc(x_173); -lean_dec(x_171); -x_174 = l_Lean_Meta_Grind_ppENodeRef(x_172, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_173); -lean_dec(x_172); -x_175 = lean_ctor_get(x_174, 0); -lean_inc(x_175); -x_176 = lean_ctor_get(x_174, 1); -lean_inc(x_176); -if (lean_is_exclusive(x_174)) { - lean_ctor_release(x_174, 0); - lean_ctor_release(x_174, 1); - x_177 = x_174; +if (lean_is_scalar(x_88)) { + x_89 = lean_alloc_ctor(1, 2, 0); } else { - lean_dec_ref(x_174); - x_177 = lean_box(0); + x_89 = x_88; } -x_178 = l_Lean_MessageData_ofFormat(x_164); -x_179 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_177)) { - x_180 = lean_alloc_ctor(7, 2, 0); -} else { - x_180 = x_177; - lean_ctor_set_tag(x_180, 7); +lean_ctor_set(x_89, 0, x_86); +lean_ctor_set(x_89, 1, x_87); +return x_89; } -lean_ctor_set(x_180, 0, x_179); -lean_ctor_set(x_180, 1, x_178); -x_181 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -if (lean_is_scalar(x_170)) { - x_182 = lean_alloc_ctor(7, 2, 0); -} else { - x_182 = x_170; - lean_ctor_set_tag(x_182, 7); } -lean_ctor_set(x_182, 0, x_180); -lean_ctor_set(x_182, 1, x_181); -x_183 = l_Lean_MessageData_ofFormat(x_168); -if (lean_is_scalar(x_166)) { - x_184 = lean_alloc_ctor(7, 2, 0); -} else { - x_184 = x_166; - lean_ctor_set_tag(x_184, 7); } -lean_ctor_set(x_184, 0, x_182); -lean_ctor_set(x_184, 1, x_183); -x_185 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -x_186 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_186, 0, x_184); -lean_ctor_set(x_186, 1, x_185); -x_187 = l_Lean_MessageData_ofFormat(x_175); -lean_ctor_set_tag(x_29, 7); -lean_ctor_set(x_29, 1, x_187); -lean_ctor_set(x_29, 0, x_186); -x_188 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_188, 0, x_29); -lean_ctor_set(x_188, 1, x_179); -x_189 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_188, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_176); -x_190 = lean_ctor_get(x_189, 0); -lean_inc(x_190); -x_191 = lean_ctor_get(x_189, 1); -lean_inc(x_191); -lean_dec(x_189); -x_192 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_39, x_33, x_9, x_24, x_35, x_34, x_41, x_10, x_37, x_36, x_190, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_191); -lean_dec(x_190); -lean_dec(x_35); -return x_192; } -else +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___closed__1() { +_start: { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; -lean_dec(x_170); -lean_dec(x_168); -lean_dec(x_166); -lean_dec(x_164); -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___boxed), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_14 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); lean_dec(x_14); -lean_dec(x_13); +x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___closed__1; +x_18 = lean_unbox(x_15); +lean_dec(x_15); +if (x_18 == 0) +{ +if (x_1 == 0) +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_3); +lean_dec(x_2); +x_19 = lean_box(0); +x_20 = lean_apply_10(x_17, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_2, 0); +lean_inc(x_21); +lean_dec(x_2); +x_22 = lean_ctor_get(x_3, 0); +lean_inc(x_22); +lean_dec(x_3); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq(x_21, x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_apply_10(x_17, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +return x_26; +} +else +{ +uint8_t x_27; lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -x_193 = lean_ctor_get(x_171, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_171, 1); -lean_inc(x_194); -if (lean_is_exclusive(x_171)) { - lean_ctor_release(x_171, 0); - lean_ctor_release(x_171, 1); - x_195 = x_171; -} else { - lean_dec_ref(x_171); - x_195 = lean_box(0); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_27 = !lean_is_exclusive(x_23); +if (x_27 == 0) +{ +return x_23; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_23, 0); +x_29 = lean_ctor_get(x_23, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_23); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; } -if (lean_is_scalar(x_195)) { - x_196 = lean_alloc_ctor(1, 2, 0); -} else { - x_196 = x_195; } -lean_ctor_set(x_196, 0, x_193); -lean_ctor_set(x_196, 1, x_194); -return x_196; } } else { -lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_197 = lean_ctor_get(x_161, 0); -lean_inc(x_197); -x_198 = lean_ctor_get(x_161, 1); -lean_inc(x_198); -if (lean_is_exclusive(x_161)) { - lean_ctor_release(x_161, 0); - lean_ctor_release(x_161, 1); - x_199 = x_161; -} else { - lean_dec_ref(x_161); - x_199 = lean_box(0); +lean_object* x_31; lean_object* x_32; +lean_dec(x_3); +lean_dec(x_2); +x_31 = lean_box(0); +x_32 = lean_apply_10(x_17, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_32; } -if (lean_is_scalar(x_199)) { - x_200 = lean_alloc_ctor(1, 2, 0); -} else { - x_200 = x_199; } -lean_ctor_set(x_200, 0, x_197); -lean_ctor_set(x_200, 1, x_198); -return x_200; } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_14 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_unbox(x_15); +lean_dec(x_15); +if (x_16 == 0) +{ +uint8_t x_17; +x_17 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 2); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_14, 1); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_box(0); +x_20 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +return x_20; } +else +{ +uint8_t x_21; +x_21 = lean_ctor_get_uint8(x_3, sizeof(void*)*11 + 2); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_14, 1); +lean_inc(x_22); +lean_dec(x_14); +x_23 = lean_box(0); +x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +return x_24; } +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_14, 1); +lean_inc(x_25); +lean_dec(x_14); +x_26 = lean_ctor_get(x_2, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_28 = l_Lean_Meta_Grind_propagateCtor(x_26, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_30); +lean_dec(x_29); +return x_31; } else { -uint8_t x_201; -lean_dec(x_41); -lean_dec(x_39); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_32; lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_1); -x_201 = !lean_is_exclusive(x_42); -if (x_201 == 0) +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_32 = !lean_is_exclusive(x_28); +if (x_32 == 0) { -return x_42; +return x_28; } else { -lean_object* x_202; lean_object* x_203; lean_object* x_204; -x_202 = lean_ctor_get(x_42, 0); -x_203 = lean_ctor_get(x_42, 1); -lean_inc(x_203); -lean_inc(x_202); -lean_dec(x_42); -x_204 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_204, 0, x_202); -lean_ctor_set(x_204, 1, x_203); -return x_204; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_28, 0); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_28); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} } } } else { -uint8_t x_205; -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_free_object(x_29); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_14, 1); +lean_inc(x_36); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_1); -x_205 = !lean_is_exclusive(x_38); -if (x_205 == 0) -{ +x_37 = lean_box(0); +x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_36); return x_38; } -else -{ -lean_object* x_206; lean_object* x_207; lean_object* x_208; -x_206 = lean_ctor_get(x_38, 0); -x_207 = lean_ctor_get(x_38, 1); -lean_inc(x_207); -lean_inc(x_206); -lean_dec(x_38); -x_208 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_208, 0, x_206); -lean_ctor_set(x_208, 1, x_207); -return x_208; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(uint8_t x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +if (x_4 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_box(0); +x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_1, x_2, x_3, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_16; } else { -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; uint8_t x_213; uint8_t x_214; lean_object* x_215; -x_209 = lean_ctor_get(x_29, 1); -lean_inc(x_209); -lean_dec(x_29); -x_210 = lean_ctor_get(x_6, 0); -lean_inc(x_210); -x_211 = lean_ctor_get(x_6, 1); -lean_inc(x_211); -x_212 = lean_ctor_get(x_6, 6); -lean_inc(x_212); -x_213 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 3); -x_214 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 4); -lean_dec(x_6); -x_215 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_210, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_209); -if (lean_obj_tag(x_215) == 0) -{ -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; -x_216 = lean_ctor_get(x_215, 0); -lean_inc(x_216); -x_217 = lean_ctor_get(x_215, 1); -lean_inc(x_217); -lean_dec(x_215); -x_218 = lean_ctor_get(x_7, 2); -lean_inc(x_218); -lean_dec(x_7); -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); +lean_object* x_17; lean_inc(x_13); lean_inc(x_12); -lean_inc(x_218); -lean_inc(x_1); -x_219 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_218, x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_217); -if (lean_obj_tag(x_219) == 0) -{ -lean_object* x_220; lean_object* x_221; lean_object* x_222; uint8_t x_223; -x_220 = lean_ctor_get(x_219, 1); -lean_inc(x_220); -lean_dec(x_219); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); lean_inc(x_8); -x_221 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_220); -x_222 = lean_ctor_get(x_221, 0); -lean_inc(x_222); -x_223 = lean_unbox(x_222); -lean_dec(x_222); -if (x_223 == 0) -{ -lean_object* x_224; lean_object* x_225; lean_object* x_226; -lean_dec(x_8); -lean_dec(x_1); -x_224 = lean_ctor_get(x_221, 1); -lean_inc(x_224); -lean_dec(x_221); -x_225 = lean_box(0); -x_226 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_216, x_210, x_9, x_24, x_212, x_211, x_218, x_10, x_214, x_213, x_225, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_224); -lean_dec(x_212); -return x_226; -} -else -{ -lean_object* x_227; lean_object* x_228; lean_object* x_229; -x_227 = lean_ctor_get(x_221, 1); -lean_inc(x_227); -if (lean_is_exclusive(x_221)) { - lean_ctor_release(x_221, 0); - lean_ctor_release(x_221, 1); - x_228 = x_221; -} else { - lean_dec_ref(x_221); - x_228 = lean_box(0); -} -x_229 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_227); -if (lean_obj_tag(x_229) == 0) -{ -lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_230 = lean_ctor_get(x_229, 1); -lean_inc(x_230); -lean_dec(x_229); -x_231 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_230); -x_232 = lean_ctor_get(x_231, 0); -lean_inc(x_232); -x_233 = lean_ctor_get(x_231, 1); -lean_inc(x_233); -if (lean_is_exclusive(x_231)) { - lean_ctor_release(x_231, 0); - lean_ctor_release(x_231, 1); - x_234 = x_231; -} else { - lean_dec_ref(x_231); - x_234 = lean_box(0); -} -x_235 = l_Lean_Meta_Grind_ppENodeRef(x_218, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_233); -x_236 = lean_ctor_get(x_235, 0); -lean_inc(x_236); -x_237 = lean_ctor_get(x_235, 1); -lean_inc(x_237); -if (lean_is_exclusive(x_235)) { - lean_ctor_release(x_235, 0); - lean_ctor_release(x_235, 1); - x_238 = x_235; -} else { - lean_dec_ref(x_235); - x_238 = lean_box(0); -} -x_239 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_237); -if (lean_obj_tag(x_239) == 0) -{ -lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; -x_240 = lean_ctor_get(x_239, 0); -lean_inc(x_240); -x_241 = lean_ctor_get(x_239, 1); -lean_inc(x_241); -lean_dec(x_239); -x_242 = l_Lean_Meta_Grind_ppENodeRef(x_240, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_241); -lean_dec(x_240); -x_243 = lean_ctor_get(x_242, 0); -lean_inc(x_243); -x_244 = lean_ctor_get(x_242, 1); -lean_inc(x_244); -if (lean_is_exclusive(x_242)) { - lean_ctor_release(x_242, 0); - lean_ctor_release(x_242, 1); - x_245 = x_242; -} else { - lean_dec_ref(x_242); - x_245 = lean_box(0); -} -x_246 = l_Lean_MessageData_ofFormat(x_232); -x_247 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_245)) { - x_248 = lean_alloc_ctor(7, 2, 0); -} else { - x_248 = x_245; - lean_ctor_set_tag(x_248, 7); -} -lean_ctor_set(x_248, 0, x_247); -lean_ctor_set(x_248, 1, x_246); -x_249 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -if (lean_is_scalar(x_238)) { - x_250 = lean_alloc_ctor(7, 2, 0); -} else { - x_250 = x_238; - lean_ctor_set_tag(x_250, 7); -} -lean_ctor_set(x_250, 0, x_248); -lean_ctor_set(x_250, 1, x_249); -x_251 = l_Lean_MessageData_ofFormat(x_236); -if (lean_is_scalar(x_234)) { - x_252 = lean_alloc_ctor(7, 2, 0); -} else { - x_252 = x_234; - lean_ctor_set_tag(x_252, 7); -} -lean_ctor_set(x_252, 0, x_250); -lean_ctor_set(x_252, 1, x_251); -x_253 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -if (lean_is_scalar(x_228)) { - x_254 = lean_alloc_ctor(7, 2, 0); -} else { - x_254 = x_228; - lean_ctor_set_tag(x_254, 7); -} -lean_ctor_set(x_254, 0, x_252); -lean_ctor_set(x_254, 1, x_253); -x_255 = l_Lean_MessageData_ofFormat(x_243); -x_256 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_256, 0, x_254); -lean_ctor_set(x_256, 1, x_255); -x_257 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_257, 0, x_256); -lean_ctor_set(x_257, 1, x_247); -x_258 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_257, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_244); -x_259 = lean_ctor_get(x_258, 0); -lean_inc(x_259); -x_260 = lean_ctor_get(x_258, 1); -lean_inc(x_260); -lean_dec(x_258); -x_261 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_216, x_210, x_9, x_24, x_212, x_211, x_218, x_10, x_214, x_213, x_259, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_260); -lean_dec(x_259); -lean_dec(x_212); -return x_261; -} -else +lean_inc(x_7); +lean_inc(x_6); +x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; -lean_dec(x_238); -lean_dec(x_236); -lean_dec(x_234); -lean_dec(x_232); -lean_dec(x_228); -lean_dec(x_218); -lean_dec(x_216); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_262 = lean_ctor_get(x_239, 0); -lean_inc(x_262); -x_263 = lean_ctor_get(x_239, 1); -lean_inc(x_263); -if (lean_is_exclusive(x_239)) { - lean_ctor_release(x_239, 0); - lean_ctor_release(x_239, 1); - x_264 = x_239; -} else { - lean_dec_ref(x_239); - x_264 = lean_box(0); -} -if (lean_is_scalar(x_264)) { - x_265 = lean_alloc_ctor(1, 2, 0); -} else { - x_265 = x_264; -} -lean_ctor_set(x_265, 0, x_262); -lean_ctor_set(x_265, 1, x_263); -return x_265; -} -} -else -{ -lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_269; -lean_dec(x_228); -lean_dec(x_218); -lean_dec(x_216); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_24); -lean_dec(x_19); +x_20 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_1, x_2, x_3, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_19); lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_266 = lean_ctor_get(x_229, 0); -lean_inc(x_266); -x_267 = lean_ctor_get(x_229, 1); -lean_inc(x_267); -if (lean_is_exclusive(x_229)) { - lean_ctor_release(x_229, 0); - lean_ctor_release(x_229, 1); - x_268 = x_229; -} else { - lean_dec_ref(x_229); - x_268 = lean_box(0); -} -if (lean_is_scalar(x_268)) { - x_269 = lean_alloc_ctor(1, 2, 0); -} else { - x_269 = x_268; -} -lean_ctor_set(x_269, 0, x_266); -lean_ctor_set(x_269, 1, x_267); -return x_269; -} -} +return x_20; } else { -lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; -lean_dec(x_218); -lean_dec(x_216); -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); +uint8_t x_21; lean_dec(x_13); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_1); -x_270 = lean_ctor_get(x_219, 0); -lean_inc(x_270); -x_271 = lean_ctor_get(x_219, 1); -lean_inc(x_271); -if (lean_is_exclusive(x_219)) { - lean_ctor_release(x_219, 0); - lean_ctor_release(x_219, 1); - x_272 = x_219; -} else { - lean_dec_ref(x_219); - x_272 = lean_box(0); -} -if (lean_is_scalar(x_272)) { - x_273 = lean_alloc_ctor(1, 2, 0); -} else { - x_273 = x_272; -} -lean_ctor_set(x_273, 0, x_270); -lean_ctor_set(x_273, 1, x_271); -return x_273; -} +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_3); +lean_dec(x_2); +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +return x_17; } else { -lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; -lean_dec(x_212); -lean_dec(x_211); -lean_dec(x_210); -lean_dec(x_24); -lean_dec(x_19); -lean_dec(x_18); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_1); -x_274 = lean_ctor_get(x_215, 0); -lean_inc(x_274); -x_275 = lean_ctor_get(x_215, 1); -lean_inc(x_275); -if (lean_is_exclusive(x_215)) { - lean_ctor_release(x_215, 0); - lean_ctor_release(x_215, 1); - x_276 = x_215; -} else { - lean_dec_ref(x_215); - x_276 = lean_box(0); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} } -if (lean_is_scalar(x_276)) { - x_277 = lean_alloc_ctor(1, 2, 0); -} else { - x_277 = x_276; } -lean_ctor_set(x_277, 0, x_274); -lean_ctor_set(x_277, 1, x_275); -return x_277; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { +_start: +{ +lean_object* x_21; uint8_t x_64; +x_64 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 1); +if (x_64 == 0) +{ +uint8_t x_65; +x_65 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 2); +if (x_65 == 0) +{ +lean_object* x_66; +x_66 = lean_box(0); +x_21 = x_66; +goto block_63; } else { -lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; uint8_t x_283; uint8_t x_284; uint8_t x_285; uint8_t x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; lean_object* x_298; uint8_t x_299; uint8_t x_300; lean_object* x_301; -x_278 = lean_ctor_get(x_2, 0); -x_279 = lean_ctor_get(x_2, 1); -x_280 = lean_ctor_get(x_2, 2); -x_281 = lean_ctor_get(x_2, 3); -x_282 = lean_ctor_get(x_2, 6); -x_283 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 1); -x_284 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 2); -x_285 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 3); -x_286 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 4); -x_287 = lean_ctor_get(x_2, 7); -x_288 = lean_ctor_get(x_2, 8); -x_289 = lean_ctor_get(x_2, 9); -lean_inc(x_289); -lean_inc(x_288); -lean_inc(x_287); -lean_inc(x_282); -lean_inc(x_281); -lean_inc(x_280); -lean_inc(x_279); -lean_inc(x_278); -lean_dec(x_2); -x_290 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_290, 0, x_3); -x_291 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_291, 0, x_4); -lean_inc(x_280); -x_292 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_292, 0, x_278); -lean_ctor_set(x_292, 1, x_279); -lean_ctor_set(x_292, 2, x_280); -lean_ctor_set(x_292, 3, x_281); -lean_ctor_set(x_292, 4, x_290); -lean_ctor_set(x_292, 5, x_291); -lean_ctor_set(x_292, 6, x_282); -lean_ctor_set(x_292, 7, x_287); -lean_ctor_set(x_292, 8, x_288); -lean_ctor_set(x_292, 9, x_289); -lean_ctor_set_uint8(x_292, sizeof(void*)*10, x_5); -lean_ctor_set_uint8(x_292, sizeof(void*)*10 + 1, x_283); -lean_ctor_set_uint8(x_292, sizeof(void*)*10 + 2, x_284); -lean_ctor_set_uint8(x_292, sizeof(void*)*10 + 3, x_285); -lean_ctor_set_uint8(x_292, sizeof(void*)*10 + 4, x_286); -lean_inc(x_1); -x_293 = l_Lean_Meta_Grind_setENode(x_1, x_292, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_22); -x_294 = lean_ctor_get(x_293, 1); -lean_inc(x_294); -if (lean_is_exclusive(x_293)) { - lean_ctor_release(x_293, 0); - lean_ctor_release(x_293, 1); - x_295 = x_293; -} else { - lean_dec_ref(x_293); - x_295 = lean_box(0); -} -x_296 = lean_ctor_get(x_6, 0); -lean_inc(x_296); -x_297 = lean_ctor_get(x_6, 1); -lean_inc(x_297); -x_298 = lean_ctor_get(x_6, 6); -lean_inc(x_298); -x_299 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 3); -x_300 = lean_ctor_get_uint8(x_6, sizeof(void*)*10 + 4); -lean_dec(x_6); -x_301 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents(x_296, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_294); -if (lean_obj_tag(x_301) == 0) +uint8_t x_67; +x_67 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 2); +if (x_67 == 0) { -lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; -x_302 = lean_ctor_get(x_301, 0); -lean_inc(x_302); -x_303 = lean_ctor_get(x_301, 1); -lean_inc(x_303); -lean_dec(x_301); -x_304 = lean_ctor_get(x_7, 2); -lean_inc(x_304); -lean_dec(x_7); +uint8_t x_68; lean_object* x_69; +x_68 = 1; lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); @@ -5942,179 +9154,24 @@ lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_304); lean_inc(x_1); -x_305 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_updateRoots_loop(x_1, x_304, x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_303); -if (lean_obj_tag(x_305) == 0) -{ -lean_object* x_306; lean_object* x_307; lean_object* x_308; uint8_t x_309; -x_306 = lean_ctor_get(x_305, 1); -lean_inc(x_306); -lean_dec(x_305); -lean_inc(x_8); -x_307 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_8, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_306); -x_308 = lean_ctor_get(x_307, 0); -lean_inc(x_308); -x_309 = lean_unbox(x_308); -lean_dec(x_308); -if (x_309 == 0) +lean_inc(x_2); +x_69 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_68, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_69) == 0) { -lean_object* x_310; lean_object* x_311; lean_object* x_312; -lean_dec(x_295); -lean_dec(x_8); -lean_dec(x_1); -x_310 = lean_ctor_get(x_307, 1); -lean_inc(x_310); -lean_dec(x_307); -x_311 = lean_box(0); -x_312 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_302, x_296, x_9, x_280, x_298, x_297, x_304, x_10, x_300, x_299, x_311, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_310); -lean_dec(x_298); -return x_312; +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_70, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_71); +lean_dec(x_70); +return x_72; } else { -lean_object* x_313; lean_object* x_314; lean_object* x_315; -x_313 = lean_ctor_get(x_307, 1); -lean_inc(x_313); -if (lean_is_exclusive(x_307)) { - lean_ctor_release(x_307, 0); - lean_ctor_release(x_307, 1); - x_314 = x_307; -} else { - lean_dec_ref(x_307); - x_314 = lean_box(0); -} -x_315 = l_Lean_Meta_Grind_updateLastTag(x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_313); -if (lean_obj_tag(x_315) == 0) -{ -lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; lean_object* x_324; lean_object* x_325; -x_316 = lean_ctor_get(x_315, 1); -lean_inc(x_316); -lean_dec(x_315); -x_317 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_316); -x_318 = lean_ctor_get(x_317, 0); -lean_inc(x_318); -x_319 = lean_ctor_get(x_317, 1); -lean_inc(x_319); -if (lean_is_exclusive(x_317)) { - lean_ctor_release(x_317, 0); - lean_ctor_release(x_317, 1); - x_320 = x_317; -} else { - lean_dec_ref(x_317); - x_320 = lean_box(0); -} -x_321 = l_Lean_Meta_Grind_ppENodeRef(x_304, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_319); -x_322 = lean_ctor_get(x_321, 0); -lean_inc(x_322); -x_323 = lean_ctor_get(x_321, 1); -lean_inc(x_323); -if (lean_is_exclusive(x_321)) { - lean_ctor_release(x_321, 0); - lean_ctor_release(x_321, 1); - x_324 = x_321; -} else { - lean_dec_ref(x_321); - x_324 = lean_box(0); -} -x_325 = l_Lean_Meta_Grind_getRoot(x_1, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_323); -if (lean_obj_tag(x_325) == 0) -{ -lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_333; lean_object* x_334; lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; lean_object* x_344; lean_object* x_345; lean_object* x_346; lean_object* x_347; -x_326 = lean_ctor_get(x_325, 0); -lean_inc(x_326); -x_327 = lean_ctor_get(x_325, 1); -lean_inc(x_327); -lean_dec(x_325); -x_328 = l_Lean_Meta_Grind_ppENodeRef(x_326, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_327); -lean_dec(x_326); -x_329 = lean_ctor_get(x_328, 0); -lean_inc(x_329); -x_330 = lean_ctor_get(x_328, 1); -lean_inc(x_330); -if (lean_is_exclusive(x_328)) { - lean_ctor_release(x_328, 0); - lean_ctor_release(x_328, 1); - x_331 = x_328; -} else { - lean_dec_ref(x_328); - x_331 = lean_box(0); -} -x_332 = l_Lean_MessageData_ofFormat(x_318); -x_333 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_331)) { - x_334 = lean_alloc_ctor(7, 2, 0); -} else { - x_334 = x_331; - lean_ctor_set_tag(x_334, 7); -} -lean_ctor_set(x_334, 0, x_333); -lean_ctor_set(x_334, 1, x_332); -x_335 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2; -if (lean_is_scalar(x_324)) { - x_336 = lean_alloc_ctor(7, 2, 0); -} else { - x_336 = x_324; - lean_ctor_set_tag(x_336, 7); -} -lean_ctor_set(x_336, 0, x_334); -lean_ctor_set(x_336, 1, x_335); -x_337 = l_Lean_MessageData_ofFormat(x_322); -if (lean_is_scalar(x_320)) { - x_338 = lean_alloc_ctor(7, 2, 0); -} else { - x_338 = x_320; - lean_ctor_set_tag(x_338, 7); -} -lean_ctor_set(x_338, 0, x_336); -lean_ctor_set(x_338, 1, x_337); -x_339 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__4; -if (lean_is_scalar(x_314)) { - x_340 = lean_alloc_ctor(7, 2, 0); -} else { - x_340 = x_314; - lean_ctor_set_tag(x_340, 7); -} -lean_ctor_set(x_340, 0, x_338); -lean_ctor_set(x_340, 1, x_339); -x_341 = l_Lean_MessageData_ofFormat(x_329); -if (lean_is_scalar(x_295)) { - x_342 = lean_alloc_ctor(7, 2, 0); -} else { - x_342 = x_295; - lean_ctor_set_tag(x_342, 7); -} -lean_ctor_set(x_342, 0, x_340); -lean_ctor_set(x_342, 1, x_341); -x_343 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_343, 0, x_342); -lean_ctor_set(x_343, 1, x_333); -x_344 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_8, x_343, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_330); -x_345 = lean_ctor_get(x_344, 0); -lean_inc(x_345); -x_346 = lean_ctor_get(x_344, 1); -lean_inc(x_346); -lean_dec(x_344); -x_347 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_302, x_296, x_9, x_280, x_298, x_297, x_304, x_10, x_300, x_299, x_345, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_346); -lean_dec(x_345); -lean_dec(x_298); -return x_347; -} -else -{ -lean_object* x_348; lean_object* x_349; lean_object* x_350; lean_object* x_351; -lean_dec(x_324); -lean_dec(x_322); -lean_dec(x_320); -lean_dec(x_318); -lean_dec(x_314); -lean_dec(x_304); -lean_dec(x_302); -lean_dec(x_298); -lean_dec(x_297); -lean_dec(x_296); -lean_dec(x_295); -lean_dec(x_280); +uint8_t x_73; lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); @@ -6123,164 +9180,71 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -x_348 = lean_ctor_get(x_325, 0); -lean_inc(x_348); -x_349 = lean_ctor_get(x_325, 1); -lean_inc(x_349); -if (lean_is_exclusive(x_325)) { - lean_ctor_release(x_325, 0); - lean_ctor_release(x_325, 1); - x_350 = x_325; -} else { - lean_dec_ref(x_325); - x_350 = lean_box(0); -} -if (lean_is_scalar(x_350)) { - x_351 = lean_alloc_ctor(1, 2, 0); -} else { - x_351 = x_350; -} -lean_ctor_set(x_351, 0, x_348); -lean_ctor_set(x_351, 1, x_349); -return x_351; -} +lean_dec(x_2); +lean_dec(x_1); +x_73 = !lean_is_exclusive(x_69); +if (x_73 == 0) +{ +return x_69; } else { -lean_object* x_352; lean_object* x_353; lean_object* x_354; lean_object* x_355; -lean_dec(x_314); -lean_dec(x_304); -lean_dec(x_302); -lean_dec(x_298); -lean_dec(x_297); -lean_dec(x_296); -lean_dec(x_295); -lean_dec(x_280); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_352 = lean_ctor_get(x_315, 0); -lean_inc(x_352); -x_353 = lean_ctor_get(x_315, 1); -lean_inc(x_353); -if (lean_is_exclusive(x_315)) { - lean_ctor_release(x_315, 0); - lean_ctor_release(x_315, 1); - x_354 = x_315; -} else { - lean_dec_ref(x_315); - x_354 = lean_box(0); -} -if (lean_is_scalar(x_354)) { - x_355 = lean_alloc_ctor(1, 2, 0); -} else { - x_355 = x_354; -} -lean_ctor_set(x_355, 0, x_352); -lean_ctor_set(x_355, 1, x_353); -return x_355; +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_69, 0); +x_75 = lean_ctor_get(x_69, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_69); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; } } } else { -lean_object* x_356; lean_object* x_357; lean_object* x_358; lean_object* x_359; -lean_dec(x_304); -lean_dec(x_302); -lean_dec(x_298); -lean_dec(x_297); -lean_dec(x_296); -lean_dec(x_295); -lean_dec(x_280); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_1); -x_356 = lean_ctor_get(x_305, 0); -lean_inc(x_356); -x_357 = lean_ctor_get(x_305, 1); -lean_inc(x_357); -if (lean_is_exclusive(x_305)) { - lean_ctor_release(x_305, 0); - lean_ctor_release(x_305, 1); - x_358 = x_305; -} else { - lean_dec_ref(x_305); - x_358 = lean_box(0); -} -if (lean_is_scalar(x_358)) { - x_359 = lean_alloc_ctor(1, 2, 0); -} else { - x_359 = x_358; +lean_object* x_77; +x_77 = lean_box(0); +x_21 = x_77; +goto block_63; } -lean_ctor_set(x_359, 0, x_356); -lean_ctor_set(x_359, 1, x_357); -return x_359; } } else { -lean_object* x_360; lean_object* x_361; lean_object* x_362; lean_object* x_363; -lean_dec(x_298); -lean_dec(x_297); -lean_dec(x_296); -lean_dec(x_295); -lean_dec(x_280); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_1); -x_360 = lean_ctor_get(x_301, 0); -lean_inc(x_360); -x_361 = lean_ctor_get(x_301, 1); -lean_inc(x_361); -if (lean_is_exclusive(x_301)) { - lean_ctor_release(x_301, 0); - lean_ctor_release(x_301, 1); - x_362 = x_301; -} else { - lean_dec_ref(x_301); - x_362 = lean_box(0); -} -if (lean_is_scalar(x_362)) { - x_363 = lean_alloc_ctor(1, 2, 0); -} else { - x_363 = x_362; -} -lean_ctor_set(x_363, 0, x_360); -lean_ctor_set(x_363, 1, x_361); -return x_363; -} -} +uint8_t x_78; +x_78 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 1); +if (x_78 == 0) +{ +uint8_t x_79; lean_object* x_80; +x_79 = 1; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +lean_inc(x_2); +x_80 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_79, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_80) == 0) +{ +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_80, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_80, 1); +lean_inc(x_82); +lean_dec(x_80); +x_83 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_81, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_82); +lean_dec(x_81); +return x_83; } else { -uint8_t x_364; +uint8_t x_84; lean_dec(x_19); lean_dec(x_18); lean_dec(x_17); @@ -6289,2748 +9253,2895 @@ lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_364 = !lean_is_exclusive(x_21); -if (x_364 == 0) +x_84 = !lean_is_exclusive(x_80); +if (x_84 == 0) { -return x_21; +return x_80; } else { -lean_object* x_365; lean_object* x_366; lean_object* x_367; -x_365 = lean_ctor_get(x_21, 0); -x_366 = lean_ctor_get(x_21, 1); -lean_inc(x_366); -lean_inc(x_365); -lean_dec(x_21); -x_367 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_367, 0, x_365); -lean_ctor_set(x_367, 1, x_366); -return x_367; -} -} -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; -x_2 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__2; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_80, 0); +x_86 = lean_ctor_get(x_80, 1); +lean_inc(x_86); +lean_inc(x_85); +lean_dec(x_80); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("adding ", 7, 7); -return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__4() { -_start: +uint8_t x_88; +x_88 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 2); +if (x_88 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" ↦ ", 5, 3); -return x_1; -} +lean_object* x_89; +x_89 = lean_box(0); +x_21 = x_89; +goto block_63; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__4; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { -_start: +uint8_t x_90; +x_90 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 2); +if (x_90 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_19 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; -x_20 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_19, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_unbox(x_21); -lean_dec(x_21); -if (x_22 == 0) +uint8_t x_91; lean_object* x_92; +x_91 = 1; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +lean_inc(x_2); +x_92 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_91, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_92) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_dec(x_20); -x_24 = lean_box(0); -x_25 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_24, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_23); -return x_25; +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_93, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_94); +lean_dec(x_93); +return x_95; } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_20, 1); -x_28 = lean_ctor_get(x_20, 0); -lean_dec(x_28); -x_29 = l_Lean_Meta_Grind_updateLastTag(x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_27); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = lean_ctor_get(x_29, 1); -lean_inc(x_30); -lean_dec(x_29); -x_31 = l_Lean_Meta_Grind_ppENodeRef(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_30); -x_32 = !lean_is_exclusive(x_31); -if (x_32 == 0) -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = lean_ctor_get(x_31, 0); -x_34 = lean_ctor_get(x_31, 1); -x_35 = l_Lean_Meta_Grind_ppENodeRef(x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_34); -x_36 = !lean_is_exclusive(x_35); -if (x_36 == 0) +uint8_t x_96; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_2); +lean_dec(x_1); +x_96 = !lean_is_exclusive(x_92); +if (x_96 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_37 = lean_ctor_get(x_35, 0); -x_38 = lean_ctor_get(x_35, 1); -x_39 = l_Lean_MessageData_ofFormat(x_33); -x_40 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; -lean_ctor_set_tag(x_35, 7); -lean_ctor_set(x_35, 1, x_39); -lean_ctor_set(x_35, 0, x_40); -x_41 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; -lean_ctor_set_tag(x_31, 7); -lean_ctor_set(x_31, 1, x_41); -lean_ctor_set(x_31, 0, x_35); -x_42 = l_Lean_MessageData_ofFormat(x_37); -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_42); -lean_ctor_set(x_20, 0, x_31); -x_43 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_44 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_44, 0, x_20); -lean_ctor_set(x_44, 1, x_43); -x_45 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_44, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_38); -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_46, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_47); -lean_dec(x_46); -return x_48; +return x_92; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_49 = lean_ctor_get(x_35, 0); -x_50 = lean_ctor_get(x_35, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_35); -x_51 = l_Lean_MessageData_ofFormat(x_33); -x_52 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; -x_53 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_51); -x_54 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; -lean_ctor_set_tag(x_31, 7); -lean_ctor_set(x_31, 1, x_54); -lean_ctor_set(x_31, 0, x_53); -x_55 = l_Lean_MessageData_ofFormat(x_49); -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_55); -lean_ctor_set(x_20, 0, x_31); -x_56 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_57 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_57, 0, x_20); -lean_ctor_set(x_57, 1, x_56); -x_58 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_57, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_50); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -lean_dec(x_58); -x_61 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_59, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_60); -lean_dec(x_59); -return x_61; +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_92, 0); +x_98 = lean_ctor_get(x_92, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_92); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +return x_99; +} } } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_62 = lean_ctor_get(x_31, 0); -x_63 = lean_ctor_get(x_31, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_31); -x_64 = l_Lean_Meta_Grind_ppENodeRef(x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_63); -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_64, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_64)) { - lean_ctor_release(x_64, 0); - lean_ctor_release(x_64, 1); - x_67 = x_64; -} else { - lean_dec_ref(x_64); - x_67 = lean_box(0); +lean_object* x_100; +x_100 = lean_box(0); +x_21 = x_100; +goto block_63; } -x_68 = l_Lean_MessageData_ofFormat(x_62); -x_69 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; -if (lean_is_scalar(x_67)) { - x_70 = lean_alloc_ctor(7, 2, 0); -} else { - x_70 = x_67; - lean_ctor_set_tag(x_70, 7); } -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_68); -x_71 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; -x_72 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -x_73 = l_Lean_MessageData_ofFormat(x_65); -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_73); -lean_ctor_set(x_20, 0, x_72); -x_74 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_75 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_75, 0, x_20); -lean_ctor_set(x_75, 1, x_74); -x_76 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_75, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_66); -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_76, 1); -lean_inc(x_78); -lean_dec(x_76); -x_79 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_77, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_78); -lean_dec(x_77); -return x_79; } } +block_63: +{ +lean_object* x_22; lean_object* x_23; uint8_t x_24; +lean_dec(x_21); +x_22 = lean_ctor_get(x_2, 6); +lean_inc(x_22); +x_23 = lean_ctor_get(x_1, 6); +lean_inc(x_23); +x_24 = lean_nat_dec_lt(x_22, x_23); +lean_dec(x_23); +lean_dec(x_22); +if (x_24 == 0) +{ +uint8_t x_25; lean_object* x_26; +x_25 = 0; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_2); +lean_inc(x_1); +x_26 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_25, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_27, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_28); +lean_dec(x_27); +return x_29; +} else { -uint8_t x_80; -lean_free_object(x_20); +uint8_t x_30; +lean_dec(x_19); +lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_80 = !lean_is_exclusive(x_29); -if (x_80 == 0) +x_30 = !lean_is_exclusive(x_26); +if (x_30 == 0) { -return x_29; +return x_26; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_29, 0); -x_82 = lean_ctor_get(x_29, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_29); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_26, 0); +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_26); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } else { -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_20, 1); -lean_inc(x_84); -lean_dec(x_20); -x_85 = l_Lean_Meta_Grind_updateLastTag(x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_84); -if (lean_obj_tag(x_85) == 0) +uint8_t x_34; +x_34 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 1); +if (x_34 == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -lean_dec(x_85); -x_87 = l_Lean_Meta_Grind_ppENodeRef(x_3, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_86); -x_88 = lean_ctor_get(x_87, 0); -lean_inc(x_88); -x_89 = lean_ctor_get(x_87, 1); -lean_inc(x_89); -if (lean_is_exclusive(x_87)) { - lean_ctor_release(x_87, 0); - lean_ctor_release(x_87, 1); - x_90 = x_87; -} else { - lean_dec_ref(x_87); - x_90 = lean_box(0); -} -x_91 = l_Lean_Meta_Grind_ppENodeRef(x_4, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_89); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_94 = x_91; -} else { - lean_dec_ref(x_91); - x_94 = lean_box(0); -} -x_95 = l_Lean_MessageData_ofFormat(x_88); -x_96 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__3; -if (lean_is_scalar(x_94)) { - x_97 = lean_alloc_ctor(7, 2, 0); -} else { - x_97 = x_94; - lean_ctor_set_tag(x_97, 7); -} -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_95); -x_98 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__5; -if (lean_is_scalar(x_90)) { - x_99 = lean_alloc_ctor(7, 2, 0); -} else { - x_99 = x_90; - lean_ctor_set_tag(x_99, 7); -} -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -x_100 = l_Lean_MessageData_ofFormat(x_92); -x_101 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_101, 0, x_99); -lean_ctor_set(x_101, 1, x_100); -x_102 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_103 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -x_104 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_19, x_103, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_93); -x_105 = lean_ctor_get(x_104, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_104, 1); -lean_inc(x_106); -lean_dec(x_104); -x_107 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_3, x_5, x_4, x_1, x_9, x_7, x_6, x_19, x_8, x_2, x_105, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_106); -lean_dec(x_105); -return x_107; +uint8_t x_35; +x_35 = lean_ctor_get_uint8(x_2, sizeof(void*)*11 + 2); +if (x_35 == 0) +{ +uint8_t x_36; lean_object* x_37; +x_36 = 1; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +lean_inc(x_2); +x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_36, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_38, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_39); +lean_dec(x_38); +return x_40; } else { -lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +uint8_t x_41; +lean_dec(x_19); +lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_108 = lean_ctor_get(x_85, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_85, 1); -lean_inc(x_109); -if (lean_is_exclusive(x_85)) { - lean_ctor_release(x_85, 0); - lean_ctor_release(x_85, 1); - x_110 = x_85; -} else { - lean_dec_ref(x_85); - x_110 = lean_box(0); -} -if (lean_is_scalar(x_110)) { - x_111 = lean_alloc_ctor(1, 2, 0); -} else { - x_111 = x_110; -} -lean_ctor_set(x_111, 0, x_108); -lean_ctor_set(x_111, 1, x_109); -return x_111; -} -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -_start: +x_41 = !lean_is_exclusive(x_37); +if (x_41 == 0) { -uint8_t x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; -x_21 = lean_unbox(x_8); -lean_dec(x_8); -x_22 = lean_unbox(x_9); -lean_dec(x_9); -x_23 = lean_unbox(x_10); -lean_dec(x_10); -x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_21, x_22, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -lean_dec(x_11); -lean_dec(x_5); -return x_24; -} +return x_37; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -_start: +else { -uint8_t x_21; uint8_t x_22; lean_object* x_23; -x_21 = lean_unbox(x_5); -lean_dec(x_5); -x_22 = lean_unbox(x_10); -lean_dec(x_10); -x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3(x_1, x_2, x_3, x_4, x_21, x_6, x_7, x_8, x_9, x_22, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -lean_dec(x_11); -return x_23; -} +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_37, 0); +x_43 = lean_ctor_get(x_37, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_37); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -_start: -{ -uint8_t x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_unbox(x_2); -lean_dec(x_2); -x_20 = lean_unbox(x_9); -lean_dec(x_9); -x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_1, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_20, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -uint8_t x_11; lean_object* x_12; -x_11 = 0; -x_12 = l_Lean_Meta_Grind_checkInvariants(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_12; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1() { -_start: +uint8_t x_45; lean_object* x_46; +x_45 = 0; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_2); +lean_inc(x_1); +x_46 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_45, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1___boxed), 10, 0); -return x_1; -} +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_49 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_47, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_48); +lean_dec(x_47); +return x_49; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__2() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("after addEqStep, ", 17, 17); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3() { -_start: +uint8_t x_50; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_2); +lean_dec(x_1); +x_50 = !lean_is_exclusive(x_46); +if (x_50 == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +return x_46; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; -x_12 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1; -x_17 = lean_unbox(x_14); -lean_dec(x_14); -if (x_17 == 0) +else { -lean_object* x_18; lean_object* x_19; -lean_free_object(x_12); -x_18 = lean_box(0); -x_19 = lean_apply_10(x_16, x_18, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); -return x_19; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_46, 0); +x_52 = lean_ctor_get(x_46, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_46); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; +} +} +} } else { -lean_object* x_20; -x_20 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); -if (lean_obj_tag(x_20) == 0) -{ -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_20, 1); -lean_inc(x_21); -lean_dec(x_20); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); +uint8_t x_54; lean_object* x_55; +x_54 = 0; +lean_inc(x_19); +lean_inc(x_18); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); lean_inc(x_2); -x_22 = l_Lean_Meta_Grind_ppState(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_21); -if (lean_obj_tag(x_22) == 0) +lean_inc(x_1); +x_55 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_54, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +if (lean_obj_tag(x_55) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = l_Lean_MessageData_ofFormat(x_23); -x_26 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; -lean_ctor_set_tag(x_12, 7); -lean_ctor_set(x_12, 1, x_25); -lean_ctor_set(x_12, 0, x_26); -x_27 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_28 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_28, 0, x_12); -lean_ctor_set(x_28, 1, x_27); -x_29 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_11, x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_24); -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_apply_10(x_16, x_30, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_31); -return x_32; +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_55, 1); +lean_inc(x_57); +lean_dec(x_55); +x_58 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_56, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_57); +lean_dec(x_56); +return x_58; } else { -uint8_t x_33; -lean_free_object(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +uint8_t x_59; +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_2); -x_33 = !lean_is_exclusive(x_22); -if (x_33 == 0) +lean_dec(x_1); +x_59 = !lean_is_exclusive(x_55); +if (x_59 == 0) { -return x_22; +return x_55; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_22, 0); -x_35 = lean_ctor_get(x_22, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_22); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_55, 0); +x_61 = lean_ctor_get(x_55, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_55); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; } } } -else +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -uint8_t x_37; -lean_free_object(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_37 = !lean_is_exclusive(x_20); -if (x_37 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_17 = lean_ctor_get(x_1, 2); +lean_inc(x_17); +x_18 = lean_st_ref_get(x_8, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_17); +x_21 = l_Lean_Meta_Grind_Goal_getENode(x_19, x_17, x_14, x_15, x_20); +if (lean_obj_tag(x_21) == 0) { -return x_20; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_ctor_get(x_2, 2); +lean_inc(x_24); +x_25 = lean_st_ref_get(x_8, x_23); +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +lean_inc(x_24); +x_28 = l_Lean_Meta_Grind_Goal_getENode(x_26, x_24, x_14, x_15, x_27); +if (lean_obj_tag(x_28) == 0) +{ +uint8_t x_29; +x_29 = lean_ctor_get_uint8(x_22, sizeof(void*)*11 + 1); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_24); +lean_dec(x_17); +x_30 = lean_ctor_get(x_28, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_28, 1); +lean_inc(x_31); +lean_dec(x_28); +x_32 = 0; +x_33 = lean_box(0); +x_34 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_22, x_30, x_3, x_4, x_5, x_6, x_1, x_2, x_32, x_32, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_31); +return x_34; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_20, 0); -x_39 = lean_ctor_get(x_20, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_20); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_28, 0); +lean_inc(x_35); +x_36 = lean_ctor_get_uint8(x_35, sizeof(void*)*11 + 1); +if (x_36 == 0) +{ +lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; +lean_dec(x_24); +lean_dec(x_17); +x_37 = lean_ctor_get(x_28, 1); +lean_inc(x_37); +lean_dec(x_28); +x_38 = 0; +x_39 = lean_box(0); +x_40 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_22, x_35, x_3, x_4, x_5, x_6, x_1, x_2, x_38, x_38, x_39, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_37); return x_40; } -} -} -} else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_41 = lean_ctor_get(x_12, 0); -x_42 = lean_ctor_get(x_12, 1); -lean_inc(x_42); +lean_object* x_41; uint8_t x_42; +x_41 = lean_ctor_get(x_28, 1); lean_inc(x_41); -lean_dec(x_12); -x_43 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__1; -x_44 = lean_unbox(x_41); -lean_dec(x_41); -if (x_44 == 0) +lean_dec(x_28); +x_42 = l_Lean_Expr_isTrue(x_17); +if (x_42 == 0) { -lean_object* x_45; lean_object* x_46; -x_45 = lean_box(0); -x_46 = lean_apply_10(x_43, x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -return x_46; +uint8_t x_43; +x_43 = l_Lean_Expr_isTrue(x_24); +if (x_43 == 0) +{ +uint8_t x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; +x_44 = 0; +x_45 = 1; +x_46 = lean_box(0); +x_47 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_22, x_35, x_3, x_4, x_5, x_6, x_1, x_2, x_44, x_45, x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_41); +return x_47; } else { -lean_object* x_47; -x_47 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; lean_object* x_49; -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); +lean_object* x_48; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_49 = l_Lean_Meta_Grind_ppState(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_48); -if (lean_obj_tag(x_49) == 0) +x_48 = l_Lean_Meta_Grind_markAsInconsistent(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_41); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_MessageData_ofFormat(x_50); -x_53 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___closed__3; -x_54 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_54, 0, x_53); -lean_ctor_set(x_54, 1, x_52); -x_55 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_56 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -x_57 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_11, x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_51); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = lean_apply_10(x_43, x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_59); -return x_60; +lean_object* x_49; uint8_t x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = 1; +x_51 = 0; +x_52 = lean_box(0); +x_53 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_22, x_35, x_3, x_4, x_5, x_6, x_1, x_2, x_50, x_51, x_52, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_49); +return x_53; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +uint8_t x_54; +lean_dec(x_35); +lean_dec(x_22); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_61 = lean_ctor_get(x_49, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_49, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_63 = x_49; -} else { - lean_dec_ref(x_49); - x_63 = lean_box(0); +lean_dec(x_1); +x_54 = !lean_is_exclusive(x_48); +if (x_54 == 0) +{ +return x_48; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_48, 0); +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_48); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} } -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(1, 2, 0); -} else { - x_64 = x_63; } -lean_ctor_set(x_64, 0, x_61); -lean_ctor_set(x_64, 1, x_62); -return x_64; } +else +{ +lean_object* x_58; +lean_dec(x_24); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +x_58 = l_Lean_Meta_Grind_markAsInconsistent(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_41); +if (lean_obj_tag(x_58) == 0) +{ +lean_object* x_59; uint8_t x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +lean_dec(x_58); +x_60 = 1; +x_61 = 0; +x_62 = lean_box(0); +x_63 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_22, x_35, x_3, x_4, x_5, x_6, x_1, x_2, x_60, x_61, x_62, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_59); +return x_63; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +uint8_t x_64; +lean_dec(x_35); +lean_dec(x_22); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_65 = lean_ctor_get(x_47, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_47, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_67 = x_47; -} else { - lean_dec_ref(x_47); - x_67 = lean_box(0); -} -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); -} else { - x_68 = x_67; -} -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; +lean_dec(x_1); +x_64 = !lean_is_exclusive(x_58); +if (x_64 == 0) +{ +return x_58; } +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_58, 0); +x_66 = lean_ctor_get(x_58, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_58); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } } } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___boxed), 10, 0); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___closed__1; -x_18 = lean_unbox(x_15); +uint8_t x_68; +lean_dec(x_24); +lean_dec(x_22); +lean_dec(x_17); lean_dec(x_15); -if (x_18 == 0) -{ -if (x_1 == 0) -{ -lean_object* x_19; lean_object* x_20; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_19 = lean_box(0); -x_20 = lean_apply_10(x_17, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_20; +lean_dec(x_1); +x_68 = !lean_is_exclusive(x_28); +if (x_68 == 0) +{ +return x_28; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_2, 0); -lean_inc(x_21); -lean_dec(x_2); -x_22 = lean_ctor_get(x_3, 0); -lean_inc(x_22); -lean_dec(x_3); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq(x_21, x_22, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_apply_10(x_17, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); -return x_26; +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_28, 0); +x_70 = lean_ctor_get(x_28, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_28); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} } else { -uint8_t x_27; +uint8_t x_72; +lean_dec(x_17); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_27 = !lean_is_exclusive(x_23); -if (x_27 == 0) +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_72 = !lean_is_exclusive(x_21); +if (x_72 == 0) { -return x_23; +return x_21; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 0); -x_29 = lean_ctor_get(x_23, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_23); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_21, 0); +x_74 = lean_ctor_get(x_21, 1); +lean_inc(x_74); +lean_inc(x_73); +lean_dec(x_21); +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; } } } } -else +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__1() { +_start: { -lean_object* x_31; lean_object* x_32; -lean_dec(x_3); -lean_dec(x_2); -x_31 = lean_box(0); -x_32 = lean_apply_10(x_17, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_32; -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eqc", 3, 3); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__2() { _start: { -lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_14 = l_Lean_Meta_Grind_isInconsistent(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_unbox(x_15); -lean_dec(x_15); -if (x_16 == 0) +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: { -uint8_t x_17; -x_17 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 2); -if (x_17 == 0) +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__2; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_14, 1); -lean_inc(x_18); -lean_dec(x_14); -x_19 = lean_box(0); -x_20 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); -return x_20; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_22, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_21); +return x_23; } else { -uint8_t x_21; -x_21 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 2); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_14, 1); -lean_inc(x_22); -lean_dec(x_14); -x_23 = lean_box(0); -x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_18, 1); +lean_inc(x_24); +if (lean_is_exclusive(x_18)) { + lean_ctor_release(x_18, 0); + lean_ctor_release(x_18, 1); + x_25 = x_18; +} else { + lean_dec_ref(x_18); + x_25 = lean_box(0); } -else +x_26 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_24); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_14, 1); -lean_inc(x_25); -lean_dec(x_14); -x_26 = lean_ctor_get(x_2, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_3, 0); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_26, 1); lean_inc(x_27); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); +lean_dec(x_26); +if (x_4 == 0) +{ +lean_object* x_39; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); lean_inc(x_6); lean_inc(x_5); -x_28 = l_Lean_Meta_Grind_propagateCtor(x_26, x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); -if (lean_obj_tag(x_28) == 0) +x_39 = l_Lean_Meta_mkEq(x_5, x_6, x_12, x_13, x_14, x_15, x_27); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_30); -lean_dec(x_29); -return x_31; +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_28 = x_40; +x_29 = x_41; +goto block_38; } else { -uint8_t x_32; +uint8_t x_42; +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_32 = !lean_is_exclusive(x_28); -if (x_32 == 0) -{ -return x_28; -} -else +lean_dec(x_1); +x_42 = !lean_is_exclusive(x_39); +if (x_42 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_28, 0); -x_34 = lean_ctor_get(x_28, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_28); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; -} -} -} -} +return x_39; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_14, 1); -lean_inc(x_36); -lean_dec(x_14); -x_37 = lean_box(0); -x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_1, x_2, x_3, x_37, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_36); -return x_38; -} +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 0); +x_44 = lean_ctor_get(x_39, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_39); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(uint8_t x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -if (x_4 == 0) -{ -lean_object* x_15; lean_object* x_16; -x_15 = lean_box(0); -x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_1, x_2, x_3, x_15, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_16; } else { -lean_object* x_17; +lean_object* x_46; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); lean_inc(x_6); -x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithTrueEqFalse(x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_17) == 0) +lean_inc(x_5); +x_46 = l_Lean_Meta_mkHEq(x_5, x_6, x_12, x_13, x_14, x_15, x_27); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_1, x_2, x_3, x_18, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_19); -lean_dec(x_18); -return x_20; +lean_object* x_47; lean_object* x_48; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +lean_dec(x_46); +x_28 = x_47; +x_29 = x_48; +goto block_38; } else { -uint8_t x_21; +uint8_t x_49; +lean_dec(x_25); +lean_dec(x_15); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); -x_21 = !lean_is_exclusive(x_17); -if (x_21 == 0) +lean_dec(x_1); +x_49 = !lean_is_exclusive(x_46); +if (x_49 == 0) { -return x_17; +return x_46; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_17, 0); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_17); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; -} -} +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_46, 0); +x_51 = lean_ctor_get(x_46, 1); +lean_inc(x_51); +lean_inc(x_50); +lean_dec(x_46); +x_52 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +return x_52; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20) { -_start: -{ -lean_object* x_21; uint8_t x_64; -x_64 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 1); -if (x_64 == 0) -{ -uint8_t x_65; -x_65 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 2); -if (x_65 == 0) +block_38: { -lean_object* x_66; -x_66 = lean_box(0); -x_21 = x_66; -goto block_63; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_30 = l_Lean_MessageData_ofExpr(x_28); +x_31 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_25)) { + x_32 = lean_alloc_ctor(7, 2, 0); +} else { + x_32 = x_25; + lean_ctor_set_tag(x_32, 7); +} +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +x_34 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_17, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_29); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_35, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_36); +lean_dec(x_35); +return x_37; } -else -{ -uint8_t x_67; -x_67 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 2); -if (x_67 == 0) -{ -uint8_t x_68; lean_object* x_69; -x_68 = 1; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_1); -lean_inc(x_2); -x_69 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_68, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); -lean_inc(x_71); -lean_dec(x_69); -x_72 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_70, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_71); -lean_dec(x_70); -return x_72; } else { -uint8_t x_73; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); +uint8_t x_53; +lean_dec(x_25); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_73 = !lean_is_exclusive(x_69); -if (x_73 == 0) +x_53 = !lean_is_exclusive(x_26); +if (x_53 == 0) +{ +return x_26; +} +else +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_54 = lean_ctor_get(x_26, 0); +x_55 = lean_ctor_get(x_26, 1); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_26); +x_56 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_56, 0, x_54); +lean_ctor_set(x_56, 1, x_55); +return x_56; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +return x_12; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1() { +_start: { -return x_69; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9___boxed), 10, 0); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__2() { +_start: { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_69, 0); -x_75 = lean_ctor_get(x_69, 1); -lean_inc(x_75); -lean_inc(x_74); -lean_dec(x_69); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" and ", 5, 5); +return x_1; } } +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} } -else +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__4() { +_start: { -lean_object* x_77; -x_77 = lean_box(0); -x_21 = x_77; -goto block_63; +lean_object* x_1; +x_1 = lean_mk_string_unchecked(" are already in the same equivalence class", 42, 42); +return x_1; } } +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__4; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -uint8_t x_78; -x_78 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 1); -if (x_78 == 0) +lean_object* x_14; uint8_t x_15; +x_14 = lean_st_ref_get(x_5, x_13); +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -uint8_t x_79; lean_object* x_80; -x_79 = 1; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); lean_inc(x_1); +x_18 = l_Lean_Meta_Grind_Goal_getENode(x_16, x_1, x_11, x_12, x_17); +if (lean_obj_tag(x_18) == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_st_ref_get(x_5, x_20); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); lean_inc(x_2); -x_80 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_79, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_80) == 0) +x_25 = l_Lean_Meta_Grind_Goal_getENode(x_23, x_2, x_11, x_12, x_24); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -lean_dec(x_80); -x_83 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_81, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_82); -lean_dec(x_81); -return x_83; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = lean_ctor_get(x_19, 2); +lean_inc(x_28); +x_29 = lean_ctor_get(x_26, 2); +lean_inc(x_29); +x_30 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_28, x_29); +lean_dec(x_29); +lean_dec(x_28); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +lean_free_object(x_21); +lean_free_object(x_14); +x_31 = lean_box(0); +x_32 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_19, x_26, x_3, x_4, x_1, x_2, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_27); +return x_32; } else { -uint8_t x_84; +lean_object* x_33; lean_object* x_34; uint8_t x_35; +lean_dec(x_26); lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_2); -lean_dec(x_1); -x_84 = !lean_is_exclusive(x_80); -if (x_84 == 0) +lean_dec(x_3); +x_33 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; +x_34 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_33, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_27); +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) { -return x_80; -} -else +lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_36 = lean_ctor_get(x_34, 0); +x_37 = lean_ctor_get(x_34, 1); +x_38 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; +x_39 = lean_unbox(x_36); +lean_dec(x_36); +if (x_39 == 0) { -lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_85 = lean_ctor_get(x_80, 0); -x_86 = lean_ctor_get(x_80, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_80); -x_87 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_87, 0, x_85); -lean_ctor_set(x_87, 1, x_86); -return x_87; -} -} +lean_object* x_40; lean_object* x_41; +lean_free_object(x_34); +lean_free_object(x_21); +lean_free_object(x_14); +lean_dec(x_2); +lean_dec(x_1); +x_40 = lean_box(0); +x_41 = lean_apply_10(x_38, x_40, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +return x_41; } else { -uint8_t x_88; -x_88 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 2); -if (x_88 == 0) -{ -lean_object* x_89; -x_89 = lean_box(0); -x_21 = x_89; -goto block_63; -} -else +lean_object* x_42; +x_42 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +if (lean_obj_tag(x_42) == 0) { -uint8_t x_90; -x_90 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 2); -if (x_90 == 0) +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_44 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_43); +if (lean_obj_tag(x_44) == 0) { -uint8_t x_91; lean_object* x_92; -x_91 = 1; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); lean_inc(x_12); -lean_inc(x_1); -lean_inc(x_2); -x_92 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_91, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_92) == 0) +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_47 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_46); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_92, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_92, 1); -lean_inc(x_94); -lean_dec(x_92); -x_95 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_93, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_94); -lean_dec(x_93); -return x_95; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +lean_ctor_set_tag(x_34, 7); +lean_ctor_set(x_34, 1, x_45); +lean_ctor_set(x_34, 0, x_50); +x_51 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; +lean_ctor_set_tag(x_21, 7); +lean_ctor_set(x_21, 1, x_51); +lean_ctor_set(x_21, 0, x_34); +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_48); +lean_ctor_set(x_14, 0, x_21); +x_52 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_14); +lean_ctor_set(x_53, 1, x_52); +x_54 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_33, x_53, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_49); +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); +x_57 = lean_apply_10(x_38, x_55, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_56); +return x_57; } else { -uint8_t x_96; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_58; +lean_dec(x_45); +lean_free_object(x_34); +lean_free_object(x_21); +lean_free_object(x_14); lean_dec(x_12); -lean_dec(x_2); -lean_dec(x_1); -x_96 = !lean_is_exclusive(x_92); -if (x_96 == 0) +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_58 = !lean_is_exclusive(x_47); +if (x_58 == 0) { -return x_92; +return x_47; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_92, 0); -x_98 = lean_ctor_get(x_92, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_92); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_47, 0); +x_60 = lean_ctor_get(x_47, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_47); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } else { -lean_object* x_100; -x_100 = lean_box(0); -x_21 = x_100; -goto block_63; -} +uint8_t x_62; +lean_free_object(x_34); +lean_free_object(x_21); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_62 = !lean_is_exclusive(x_44); +if (x_62 == 0) +{ +return x_44; } +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_44, 0); +x_64 = lean_ctor_get(x_44, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_44); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } -block_63: -{ -lean_object* x_22; lean_object* x_23; uint8_t x_24; -lean_dec(x_21); -x_22 = lean_ctor_get(x_2, 6); -lean_inc(x_22); -x_23 = lean_ctor_get(x_1, 6); -lean_inc(x_23); -x_24 = lean_nat_dec_lt(x_22, x_23); -lean_dec(x_23); -lean_dec(x_22); -if (x_24 == 0) -{ -uint8_t x_25; lean_object* x_26; -x_25 = 0; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_2); -lean_inc(x_1); -x_26 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_25, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_27, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_28); -lean_dec(x_27); -return x_29; } else { -uint8_t x_30; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_66; +lean_free_object(x_34); +lean_free_object(x_21); +lean_free_object(x_14); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) +x_66 = !lean_is_exclusive(x_42); +if (x_66 == 0) { -return x_26; +return x_42; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_42, 0); +x_68 = lean_ctor_get(x_42, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_42); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; +} } } } else { -uint8_t x_34; -x_34 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 1); -if (x_34 == 0) +lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; +x_70 = lean_ctor_get(x_34, 0); +x_71 = lean_ctor_get(x_34, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_34); +x_72 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; +x_73 = lean_unbox(x_70); +lean_dec(x_70); +if (x_73 == 0) { -uint8_t x_35; -x_35 = lean_ctor_get_uint8(x_2, sizeof(void*)*10 + 2); -if (x_35 == 0) +lean_object* x_74; lean_object* x_75; +lean_free_object(x_21); +lean_free_object(x_14); +lean_dec(x_2); +lean_dec(x_1); +x_74 = lean_box(0); +x_75 = lean_apply_10(x_72, x_74, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_71); +return x_75; +} +else { -uint8_t x_36; lean_object* x_37; -x_36 = 1; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_76; +x_76 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_71); +if (lean_obj_tag(x_76) == 0) +{ +lean_object* x_77; lean_object* x_78; +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +lean_dec(x_76); lean_inc(x_12); -lean_inc(x_1); -lean_inc(x_2); -x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_6, x_5, x_8, x_7, x_2, x_1, x_36, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_37) == 0) +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_78 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_77); +if (lean_obj_tag(x_78) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -lean_dec(x_37); -x_40 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_38, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_39); -lean_dec(x_38); -return x_40; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_78, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_81 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_80); +if (lean_obj_tag(x_81) == 0) +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +lean_dec(x_81); +x_84 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_85 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_79); +x_86 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; +lean_ctor_set_tag(x_21, 7); +lean_ctor_set(x_21, 1, x_86); +lean_ctor_set(x_21, 0, x_85); +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_82); +lean_ctor_set(x_14, 0, x_21); +x_87 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; +x_88 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_88, 0, x_14); +lean_ctor_set(x_88, 1, x_87); +x_89 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_33, x_88, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_83); +x_90 = lean_ctor_get(x_89, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_89, 1); +lean_inc(x_91); +lean_dec(x_89); +x_92 = lean_apply_10(x_72, x_90, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_91); +return x_92; } else { -uint8_t x_41; -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_dec(x_79); +lean_free_object(x_21); +lean_free_object(x_14); lean_dec(x_12); -lean_dec(x_2); -lean_dec(x_1); -x_41 = !lean_is_exclusive(x_37); -if (x_41 == 0) -{ -return x_37; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_93 = lean_ctor_get(x_81, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_81, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_95 = x_81; +} else { + lean_dec_ref(x_81); + x_95 = lean_box(0); +} +if (lean_is_scalar(x_95)) { + x_96 = lean_alloc_ctor(1, 2, 0); +} else { + x_96 = x_95; +} +lean_ctor_set(x_96, 0, x_93); +lean_ctor_set(x_96, 1, x_94); +return x_96; +} } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_37, 0); -x_43 = lean_ctor_get(x_37, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_37); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +lean_free_object(x_21); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_97 = lean_ctor_get(x_78, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_78, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_78)) { + lean_ctor_release(x_78, 0); + lean_ctor_release(x_78, 1); + x_99 = x_78; +} else { + lean_dec_ref(x_78); + x_99 = lean_box(0); +} +if (lean_is_scalar(x_99)) { + x_100 = lean_alloc_ctor(1, 2, 0); +} else { + x_100 = x_99; } +lean_ctor_set(x_100, 0, x_97); +lean_ctor_set(x_100, 1, x_98); +return x_100; } } else { -uint8_t x_45; lean_object* x_46; -x_45 = 0; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_2); -lean_inc(x_1); -x_46 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_45, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_47, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_48); -lean_dec(x_47); -return x_49; +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +lean_free_object(x_21); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_101 = lean_ctor_get(x_76, 0); +lean_inc(x_101); +x_102 = lean_ctor_get(x_76, 1); +lean_inc(x_102); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_103 = x_76; +} else { + lean_dec_ref(x_76); + x_103 = lean_box(0); +} +if (lean_is_scalar(x_103)) { + x_104 = lean_alloc_ctor(1, 2, 0); +} else { + x_104 = x_103; +} +lean_ctor_set(x_104, 0, x_101); +lean_ctor_set(x_104, 1, x_102); +return x_104; +} +} +} +} } else { -uint8_t x_50; +uint8_t x_105; +lean_free_object(x_21); lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_free_object(x_14); lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_50 = !lean_is_exclusive(x_46); -if (x_50 == 0) +x_105 = !lean_is_exclusive(x_25); +if (x_105 == 0) { -return x_46; +return x_25; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_51 = lean_ctor_get(x_46, 0); -x_52 = lean_ctor_get(x_46, 1); -lean_inc(x_52); -lean_inc(x_51); -lean_dec(x_46); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_51); -lean_ctor_set(x_53, 1, x_52); -return x_53; -} +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_25, 0); +x_107 = lean_ctor_get(x_25, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_25); +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 1, x_107); +return x_108; } } } else { -uint8_t x_54; lean_object* x_55; -x_54 = 0; -lean_inc(x_19); -lean_inc(x_18); -lean_inc(x_17); -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_21, 0); +x_110 = lean_ctor_get(x_21, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_21); lean_inc(x_2); -lean_inc(x_1); -x_55 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go(x_3, x_4, x_5, x_6, x_7, x_8, x_1, x_2, x_54, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_55) == 0) +x_111 = l_Lean_Meta_Grind_Goal_getENode(x_109, x_2, x_11, x_12, x_110); +if (lean_obj_tag(x_111) == 0) { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_55, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_55, 1); -lean_inc(x_57); -lean_dec(x_55); -x_58 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_10, x_1, x_2, x_9, x_56, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_57); -lean_dec(x_56); -return x_58; +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; +x_112 = lean_ctor_get(x_111, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 1); +lean_inc(x_113); +lean_dec(x_111); +x_114 = lean_ctor_get(x_19, 2); +lean_inc(x_114); +x_115 = lean_ctor_get(x_112, 2); +lean_inc(x_115); +x_116 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_114, x_115); +lean_dec(x_115); +lean_dec(x_114); +if (x_116 == 0) +{ +lean_object* x_117; lean_object* x_118; +lean_free_object(x_14); +x_117 = lean_box(0); +x_118 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_19, x_112, x_3, x_4, x_1, x_2, x_117, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_113); +return x_118; } else { -uint8_t x_59; +lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; +lean_dec(x_112); lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +lean_dec(x_3); +x_119 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; +x_120 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_119, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_113); +x_121 = lean_ctor_get(x_120, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_120, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_123 = x_120; +} else { + lean_dec_ref(x_120); + x_123 = lean_box(0); +} +x_124 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; +x_125 = lean_unbox(x_121); +lean_dec(x_121); +if (x_125 == 0) +{ +lean_object* x_126; lean_object* x_127; +lean_dec(x_123); +lean_free_object(x_14); lean_dec(x_2); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_55); -if (x_59 == 0) -{ -return x_55; +x_126 = lean_box(0); +x_127 = lean_apply_10(x_124, x_126, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_122); +return x_127; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_55, 0); -x_61 = lean_ctor_get(x_55, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_55); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +lean_object* x_128; +x_128 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_122); +if (lean_obj_tag(x_128) == 0) +{ +lean_object* x_129; lean_object* x_130; +x_129 = lean_ctor_get(x_128, 1); +lean_inc(x_129); +lean_dec(x_128); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_130 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_129); +if (lean_obj_tag(x_130) == 0) +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_131 = lean_ctor_get(x_130, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_130, 1); +lean_inc(x_132); +lean_dec(x_130); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_133 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_132); +if (lean_obj_tag(x_133) == 0) +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_134 = lean_ctor_get(x_133, 0); +lean_inc(x_134); +x_135 = lean_ctor_get(x_133, 1); +lean_inc(x_135); +lean_dec(x_133); +x_136 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_123)) { + x_137 = lean_alloc_ctor(7, 2, 0); +} else { + x_137 = x_123; + lean_ctor_set_tag(x_137, 7); } +lean_ctor_set(x_137, 0, x_136); +lean_ctor_set(x_137, 1, x_131); +x_138 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; +x_139 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_139, 0, x_137); +lean_ctor_set(x_139, 1, x_138); +lean_ctor_set_tag(x_14, 7); +lean_ctor_set(x_14, 1, x_134); +lean_ctor_set(x_14, 0, x_139); +x_140 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; +x_141 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_141, 0, x_14); +lean_ctor_set(x_141, 1, x_140); +x_142 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_119, x_141, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_135); +x_143 = lean_ctor_get(x_142, 0); +lean_inc(x_143); +x_144 = lean_ctor_get(x_142, 1); +lean_inc(x_144); +lean_dec(x_142); +x_145 = lean_apply_10(x_124, x_143, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_144); +return x_145; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +lean_dec(x_131); +lean_dec(x_123); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_146 = lean_ctor_get(x_133, 0); +lean_inc(x_146); +x_147 = lean_ctor_get(x_133, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_133)) { + lean_ctor_release(x_133, 0); + lean_ctor_release(x_133, 1); + x_148 = x_133; +} else { + lean_dec_ref(x_133); + x_148 = lean_box(0); } +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(1, 2, 0); +} else { + x_149 = x_148; } +lean_ctor_set(x_149, 0, x_146); +lean_ctor_set(x_149, 1, x_147); +return x_149; } } +else +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +lean_dec(x_123); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_150 = lean_ctor_get(x_130, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_130, 1); +lean_inc(x_151); +if (lean_is_exclusive(x_130)) { + lean_ctor_release(x_130, 0); + lean_ctor_release(x_130, 1); + x_152 = x_130; +} else { + lean_dec_ref(x_130); + x_152 = lean_box(0); } +if (lean_is_scalar(x_152)) { + x_153 = lean_alloc_ctor(1, 2, 0); +} else { + x_153 = x_152; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_1, 2); -lean_inc(x_17); -lean_inc(x_17); -x_18 = l_Lean_Meta_Grind_getENode(x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_2, 2); -lean_inc(x_21); -lean_inc(x_21); -x_22 = l_Lean_Meta_Grind_getENode(x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_22) == 0) -{ -uint8_t x_23; -x_23 = lean_ctor_get_uint8(x_19, sizeof(void*)*10 + 1); -if (x_23 == 0) -{ -lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; -lean_dec(x_21); -lean_dec(x_17); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = 0; -x_27 = lean_box(0); -x_28 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_19, x_24, x_3, x_4, x_5, x_6, x_1, x_2, x_26, x_26, x_27, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_25); -return x_28; +lean_ctor_set(x_153, 0, x_150); +lean_ctor_set(x_153, 1, x_151); +return x_153; } -else -{ -lean_object* x_29; uint8_t x_30; -x_29 = lean_ctor_get(x_22, 0); -lean_inc(x_29); -x_30 = lean_ctor_get_uint8(x_29, sizeof(void*)*10 + 1); -if (x_30 == 0) -{ -lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; -lean_dec(x_21); -lean_dec(x_17); -x_31 = lean_ctor_get(x_22, 1); -lean_inc(x_31); -lean_dec(x_22); -x_32 = 0; -x_33 = lean_box(0); -x_34 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_19, x_29, x_3, x_4, x_5, x_6, x_1, x_2, x_32, x_32, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_31); -return x_34; } else { -lean_object* x_35; uint8_t x_36; -x_35 = lean_ctor_get(x_22, 1); -lean_inc(x_35); -lean_dec(x_22); -x_36 = l_Lean_Expr_isTrue(x_17); -if (x_36 == 0) -{ -uint8_t x_37; -x_37 = l_Lean_Expr_isTrue(x_21); -if (x_37 == 0) -{ -uint8_t x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; -x_38 = 0; -x_39 = 1; -x_40 = lean_box(0); -x_41 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_19, x_29, x_3, x_4, x_5, x_6, x_1, x_2, x_38, x_39, x_40, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_35); -return x_41; +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; +lean_dec(x_123); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_154 = lean_ctor_get(x_128, 0); +lean_inc(x_154); +x_155 = lean_ctor_get(x_128, 1); +lean_inc(x_155); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + x_156 = x_128; +} else { + lean_dec_ref(x_128); + x_156 = lean_box(0); +} +if (lean_is_scalar(x_156)) { + x_157 = lean_alloc_ctor(1, 2, 0); +} else { + x_157 = x_156; +} +lean_ctor_set(x_157, 0, x_154); +lean_ctor_set(x_157, 1, x_155); +return x_157; +} +} +} } else { -lean_object* x_42; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -x_42 = l_Lean_Meta_Grind_markAsInconsistent(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_35); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; uint8_t x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; -x_43 = lean_ctor_get(x_42, 1); -lean_inc(x_43); -lean_dec(x_42); -x_44 = 1; -x_45 = 0; -x_46 = lean_box(0); -x_47 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_19, x_29, x_3, x_4, x_5, x_6, x_1, x_2, x_44, x_45, x_46, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); -return x_47; +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; +lean_dec(x_19); +lean_free_object(x_14); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_158 = lean_ctor_get(x_111, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_111, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + x_160 = x_111; +} else { + lean_dec_ref(x_111); + x_160 = lean_box(0); +} +if (lean_is_scalar(x_160)) { + x_161 = lean_alloc_ctor(1, 2, 0); +} else { + x_161 = x_160; +} +lean_ctor_set(x_161, 0, x_158); +lean_ctor_set(x_161, 1, x_159); +return x_161; +} +} } else { -uint8_t x_48; -lean_dec(x_29); -lean_dec(x_19); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +uint8_t x_162; +lean_free_object(x_14); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_42); -if (x_48 == 0) +x_162 = !lean_is_exclusive(x_18); +if (x_162 == 0) { -return x_42; +return x_18; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_42, 0); -x_50 = lean_ctor_get(x_42, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_42); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_163; lean_object* x_164; lean_object* x_165; +x_163 = lean_ctor_get(x_18, 0); +x_164 = lean_ctor_get(x_18, 1); +lean_inc(x_164); +lean_inc(x_163); +lean_dec(x_18); +x_165 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_165, 0, x_163); +lean_ctor_set(x_165, 1, x_164); +return x_165; } } } +else +{ +lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_166 = lean_ctor_get(x_14, 0); +x_167 = lean_ctor_get(x_14, 1); +lean_inc(x_167); +lean_inc(x_166); +lean_dec(x_14); +lean_inc(x_1); +x_168 = l_Lean_Meta_Grind_Goal_getENode(x_166, x_1, x_11, x_12, x_167); +if (lean_obj_tag(x_168) == 0) +{ +lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_169 = lean_ctor_get(x_168, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +x_171 = lean_st_ref_get(x_5, x_170); +x_172 = lean_ctor_get(x_171, 0); +lean_inc(x_172); +x_173 = lean_ctor_get(x_171, 1); +lean_inc(x_173); +if (lean_is_exclusive(x_171)) { + lean_ctor_release(x_171, 0); + lean_ctor_release(x_171, 1); + x_174 = x_171; +} else { + lean_dec_ref(x_171); + x_174 = lean_box(0); +} +lean_inc(x_2); +x_175 = l_Lean_Meta_Grind_Goal_getENode(x_172, x_2, x_11, x_12, x_173); +if (lean_obj_tag(x_175) == 0) +{ +lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; uint8_t x_180; +x_176 = lean_ctor_get(x_175, 0); +lean_inc(x_176); +x_177 = lean_ctor_get(x_175, 1); +lean_inc(x_177); +lean_dec(x_175); +x_178 = lean_ctor_get(x_169, 2); +lean_inc(x_178); +x_179 = lean_ctor_get(x_176, 2); +lean_inc(x_179); +x_180 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_178, x_179); +lean_dec(x_179); +lean_dec(x_178); +if (x_180 == 0) +{ +lean_object* x_181; lean_object* x_182; +lean_dec(x_174); +x_181 = lean_box(0); +x_182 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_169, x_176, x_3, x_4, x_1, x_2, x_181, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_177); +return x_182; +} +else +{ +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; uint8_t x_189; +lean_dec(x_176); +lean_dec(x_169); +lean_dec(x_3); +x_183 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; +x_184 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_183, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_177); +x_185 = lean_ctor_get(x_184, 0); +lean_inc(x_185); +x_186 = lean_ctor_get(x_184, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_184)) { + lean_ctor_release(x_184, 0); + lean_ctor_release(x_184, 1); + x_187 = x_184; +} else { + lean_dec_ref(x_184); + x_187 = lean_box(0); +} +x_188 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; +x_189 = lean_unbox(x_185); +lean_dec(x_185); +if (x_189 == 0) +{ +lean_object* x_190; lean_object* x_191; +lean_dec(x_187); +lean_dec(x_174); +lean_dec(x_2); +lean_dec(x_1); +x_190 = lean_box(0); +x_191 = lean_apply_10(x_188, x_190, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_186); +return x_191; } else { -lean_object* x_52; -lean_dec(x_21); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_192; +x_192 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_186); +if (lean_obj_tag(x_192) == 0) +{ +lean_object* x_193; lean_object* x_194; +x_193 = lean_ctor_get(x_192, 1); +lean_inc(x_193); +lean_dec(x_192); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -x_52 = l_Lean_Meta_Grind_markAsInconsistent(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_35); -if (lean_obj_tag(x_52) == 0) +x_194 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_193); +if (lean_obj_tag(x_194) == 0) +{ +lean_object* x_195; lean_object* x_196; lean_object* x_197; +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_ctor_get(x_194, 1); +lean_inc(x_196); +lean_dec(x_194); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_197 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_196); +if (lean_obj_tag(x_197) == 0) { -lean_object* x_53; uint8_t x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = 1; -x_55 = 0; -x_56 = lean_box(0); -x_57 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_19, x_29, x_3, x_4, x_5, x_6, x_1, x_2, x_54, x_55, x_56, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_53); -return x_57; +lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; +x_198 = lean_ctor_get(x_197, 0); +lean_inc(x_198); +x_199 = lean_ctor_get(x_197, 1); +lean_inc(x_199); +lean_dec(x_197); +x_200 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_187)) { + x_201 = lean_alloc_ctor(7, 2, 0); +} else { + x_201 = x_187; + lean_ctor_set_tag(x_201, 7); +} +lean_ctor_set(x_201, 0, x_200); +lean_ctor_set(x_201, 1, x_195); +x_202 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; +if (lean_is_scalar(x_174)) { + x_203 = lean_alloc_ctor(7, 2, 0); +} else { + x_203 = x_174; + lean_ctor_set_tag(x_203, 7); +} +lean_ctor_set(x_203, 0, x_201); +lean_ctor_set(x_203, 1, x_202); +x_204 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_204, 0, x_203); +lean_ctor_set(x_204, 1, x_198); +x_205 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; +x_206 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_206, 0, x_204); +lean_ctor_set(x_206, 1, x_205); +x_207 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_183, x_206, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_199); +x_208 = lean_ctor_get(x_207, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_207, 1); +lean_inc(x_209); +lean_dec(x_207); +x_210 = lean_apply_10(x_188, x_208, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_209); +return x_210; } else { -uint8_t x_58; -lean_dec(x_29); -lean_dec(x_19); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +lean_dec(x_195); +lean_dec(x_187); +lean_dec(x_174); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_58 = !lean_is_exclusive(x_52); -if (x_58 == 0) +x_211 = lean_ctor_get(x_197, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_197, 1); +lean_inc(x_212); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_213 = x_197; +} else { + lean_dec_ref(x_197); + x_213 = lean_box(0); +} +if (lean_is_scalar(x_213)) { + x_214 = lean_alloc_ctor(1, 2, 0); +} else { + x_214 = x_213; +} +lean_ctor_set(x_214, 0, x_211); +lean_ctor_set(x_214, 1, x_212); +return x_214; +} +} +else { -return x_52; +lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; +lean_dec(x_187); +lean_dec(x_174); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +x_215 = lean_ctor_get(x_194, 0); +lean_inc(x_215); +x_216 = lean_ctor_get(x_194, 1); +lean_inc(x_216); +if (lean_is_exclusive(x_194)) { + lean_ctor_release(x_194, 0); + lean_ctor_release(x_194, 1); + x_217 = x_194; +} else { + lean_dec_ref(x_194); + x_217 = lean_box(0); +} +if (lean_is_scalar(x_217)) { + x_218 = lean_alloc_ctor(1, 2, 0); +} else { + x_218 = x_217; +} +lean_ctor_set(x_218, 0, x_215); +lean_ctor_set(x_218, 1, x_216); +return x_218; +} } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_52, 0); -x_60 = lean_ctor_get(x_52, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_52); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; +lean_dec(x_187); +lean_dec(x_174); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_2); +lean_dec(x_1); +x_219 = lean_ctor_get(x_192, 0); +lean_inc(x_219); +x_220 = lean_ctor_get(x_192, 1); +lean_inc(x_220); +if (lean_is_exclusive(x_192)) { + lean_ctor_release(x_192, 0); + lean_ctor_release(x_192, 1); + x_221 = x_192; +} else { + lean_dec_ref(x_192); + x_221 = lean_box(0); } +if (lean_is_scalar(x_221)) { + x_222 = lean_alloc_ctor(1, 2, 0); +} else { + x_222 = x_221; } +lean_ctor_set(x_222, 0, x_219); +lean_ctor_set(x_222, 1, x_220); +return x_222; } } } } else { -uint8_t x_62; -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; +lean_dec(x_174); +lean_dec(x_169); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_62 = !lean_is_exclusive(x_22); -if (x_62 == 0) -{ -return x_22; +x_223 = lean_ctor_get(x_175, 0); +lean_inc(x_223); +x_224 = lean_ctor_get(x_175, 1); +lean_inc(x_224); +if (lean_is_exclusive(x_175)) { + lean_ctor_release(x_175, 0); + lean_ctor_release(x_175, 1); + x_225 = x_175; +} else { + lean_dec_ref(x_175); + x_225 = lean_box(0); } -else -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_22, 0); -x_64 = lean_ctor_get(x_22, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_22); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; +if (lean_is_scalar(x_225)) { + x_226 = lean_alloc_ctor(1, 2, 0); +} else { + x_226 = x_225; } +lean_ctor_set(x_226, 0, x_223); +lean_ctor_set(x_226, 1, x_224); +return x_226; } } else { -uint8_t x_66; -lean_dec(x_17); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); +lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_66 = !lean_is_exclusive(x_18); -if (x_66 == 0) +x_227 = lean_ctor_get(x_168, 0); +lean_inc(x_227); +x_228 = lean_ctor_get(x_168, 1); +lean_inc(x_228); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_229 = x_168; +} else { + lean_dec_ref(x_168); + x_229 = lean_box(0); +} +if (lean_is_scalar(x_229)) { + x_230 = lean_alloc_ctor(1, 2, 0); +} else { + x_230 = x_229; +} +lean_ctor_set(x_230, 0, x_227); +lean_ctor_set(x_230, 1, x_228); +return x_230; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -return x_18; +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_18, 0); -x_68 = lean_ctor_get(x_18, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_18); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_1); +lean_dec(x_1); +x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_1); +lean_dec(x_1); +x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; uint8_t x_16; lean_object* x_17; +x_15 = lean_unbox(x_1); +lean_dec(x_1); +x_16 = lean_unbox(x_4); +lean_dec(x_4); +x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_15, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +return x_17; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +lean_object* x_18 = _args[17]; +lean_object* x_19 = _args[18]; +lean_object* x_20 = _args[19]; +_start: +{ +uint8_t x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; +x_21 = lean_unbox(x_4); +lean_dec(x_4); +x_22 = lean_unbox(x_9); +lean_dec(x_9); +x_23 = lean_unbox(x_10); +lean_dec(x_10); +x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_1, x_2, x_3, x_21, x_5, x_6, x_7, x_8, x_22, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); +lean_dec(x_11); +return x_24; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__1() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("eqc", 3, 3); -return x_1; +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_4); +lean_dec(x_4); +x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +return x_18; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_4); +lean_dec(x_4); +x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___closed__2; -x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_unbox(x_19); -lean_dec(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_18, 1); -lean_inc(x_21); -lean_dec(x_18); -x_22 = lean_box(0); -x_23 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_22, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_21); -return x_23; -} -else -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_18, 1); -lean_inc(x_24); -if (lean_is_exclusive(x_18)) { - lean_ctor_release(x_18, 0); - lean_ctor_release(x_18, 1); - x_25 = x_18; -} else { - lean_dec_ref(x_18); - x_25 = lean_box(0); -} -x_26 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_24); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 1); -lean_inc(x_27); -lean_dec(x_26); -if (x_4 == 0) -{ -lean_object* x_39; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_6); -lean_inc(x_5); -x_39 = l_Lean_Meta_mkEq(x_5, x_6, x_12, x_13, x_14, x_15, x_27); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); -lean_inc(x_41); -lean_dec(x_39); -x_28 = x_40; -x_29 = x_41; -goto block_38; -} -else -{ -uint8_t x_42; -lean_dec(x_25); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_42 = !lean_is_exclusive(x_39); -if (x_42 == 0) -{ -return x_39; +return x_11; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_39, 0); -x_44 = lean_ctor_get(x_39, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_39); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_46; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_10 = lean_st_ref_take(x_1, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); -lean_inc(x_6); -lean_inc(x_5); -x_46 = l_Lean_Meta_mkHEq(x_5, x_6, x_12, x_13, x_14, x_15, x_27); -if (lean_obj_tag(x_46) == 0) -{ -lean_object* x_47; lean_object* x_48; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_28 = x_47; -x_29 = x_48; -goto block_38; -} -else +lean_dec(x_10); +x_13 = !lean_is_exclusive(x_11); +if (x_13 == 0) { -uint8_t x_49; -lean_dec(x_25); -lean_dec(x_15); +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = lean_ctor_get(x_11, 6); lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_49 = !lean_is_exclusive(x_46); -if (x_49 == 0) +x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1; +lean_ctor_set(x_11, 6, x_15); +x_16 = lean_st_ref_set(x_1, x_11, x_12); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -return x_46; +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +x_19 = lean_box(0); +lean_ctor_set(x_16, 0, x_19); +return x_16; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_46, 0); -x_51 = lean_ctor_get(x_46, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_46); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); +lean_dec(x_16); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; } } +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_23 = lean_ctor_get(x_11, 0); +x_24 = lean_ctor_get(x_11, 1); +x_25 = lean_ctor_get(x_11, 2); +x_26 = lean_ctor_get(x_11, 3); +x_27 = lean_ctor_get(x_11, 4); +x_28 = lean_ctor_get(x_11, 5); +x_29 = lean_ctor_get_uint8(x_11, sizeof(void*)*23); +x_30 = lean_ctor_get(x_11, 7); +x_31 = lean_ctor_get(x_11, 8); +x_32 = lean_ctor_get(x_11, 9); +x_33 = lean_ctor_get(x_11, 10); +x_34 = lean_ctor_get(x_11, 11); +x_35 = lean_ctor_get(x_11, 12); +x_36 = lean_ctor_get(x_11, 13); +x_37 = lean_ctor_get(x_11, 14); +x_38 = lean_ctor_get(x_11, 15); +x_39 = lean_ctor_get(x_11, 16); +x_40 = lean_ctor_get(x_11, 17); +x_41 = lean_ctor_get(x_11, 18); +x_42 = lean_ctor_get(x_11, 19); +x_43 = lean_ctor_get(x_11, 20); +x_44 = lean_ctor_get(x_11, 21); +x_45 = lean_ctor_get(x_11, 22); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_28); +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_11); +x_46 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1; +x_47 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_47, 0, x_23); +lean_ctor_set(x_47, 1, x_24); +lean_ctor_set(x_47, 2, x_25); +lean_ctor_set(x_47, 3, x_26); +lean_ctor_set(x_47, 4, x_27); +lean_ctor_set(x_47, 5, x_28); +lean_ctor_set(x_47, 6, x_46); +lean_ctor_set(x_47, 7, x_30); +lean_ctor_set(x_47, 8, x_31); +lean_ctor_set(x_47, 9, x_32); +lean_ctor_set(x_47, 10, x_33); +lean_ctor_set(x_47, 11, x_34); +lean_ctor_set(x_47, 12, x_35); +lean_ctor_set(x_47, 13, x_36); +lean_ctor_set(x_47, 14, x_37); +lean_ctor_set(x_47, 15, x_38); +lean_ctor_set(x_47, 16, x_39); +lean_ctor_set(x_47, 17, x_40); +lean_ctor_set(x_47, 18, x_41); +lean_ctor_set(x_47, 19, x_42); +lean_ctor_set(x_47, 20, x_43); +lean_ctor_set(x_47, 21, x_44); +lean_ctor_set(x_47, 22, x_45); +lean_ctor_set_uint8(x_47, sizeof(void*)*23, x_29); +x_48 = lean_st_ref_set(x_1, x_47, x_12); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_50 = x_48; +} else { + lean_dec_ref(x_48); + x_50 = lean_box(0); } -block_38: -{ -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_30 = l_Lean_MessageData_ofExpr(x_28); -x_31 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_25)) { - x_32 = lean_alloc_ctor(7, 2, 0); +x_51 = lean_box(0); +if (lean_is_scalar(x_50)) { + x_52 = lean_alloc_ctor(0, 2, 0); } else { - x_32 = x_25; - lean_ctor_set_tag(x_32, 7); + x_52 = x_50; } -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_30); -x_33 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_31); -x_34 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_17, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_29); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_35, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_36); -lean_dec(x_35); -return x_37; +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_49); +return x_52; } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_53; -lean_dec(x_25); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_10; +x_10 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_53 = !lean_is_exclusive(x_26); -if (x_53 == 0) -{ -return x_26; -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_26, 0); -x_55 = lean_ctor_get(x_26, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_26); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; -} -} -} +return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); +lean_object* x_12; x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_10); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); return x_12; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9___boxed), 10, 0); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" and ", 5, 5); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__4() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(" are already in the same equivalence class", 42, 42); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__4; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_14; -lean_inc(x_1); -x_14 = l_Lean_Meta_Grind_getENode(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); -lean_inc(x_16); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_ctor_get(x_12, 6); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Array_back_x3f___rarg(x_14); lean_dec(x_14); -lean_inc(x_2); -x_17 = l_Lean_Meta_Grind_getENode(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -if (lean_obj_tag(x_17) == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_ctor_get(x_15, 2); -lean_inc(x_20); -x_21 = lean_ctor_get(x_18, 2); -lean_inc(x_21); -x_22 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_20, x_21); -lean_dec(x_21); -lean_dec(x_20); -if (x_22 == 0) +if (lean_obj_tag(x_15) == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_box(0); -x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_15, x_18, x_3, x_4, x_1, x_2, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_19); -return x_24; +lean_ctor_set(x_10, 0, x_15); +return x_10; } else { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -lean_dec(x_18); -lean_dec(x_15); -lean_dec(x_3); -x_25 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___closed__1; -x_26 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_19); -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_free_object(x_10); +x_16 = lean_st_ref_take(x_1, x_13); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = !lean_is_exclusive(x_17); +if (x_19 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_28 = lean_ctor_get(x_26, 0); -x_29 = lean_ctor_get(x_26, 1); -x_30 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; -x_31 = lean_unbox(x_28); -lean_dec(x_28); -if (x_31 == 0) +lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_20 = lean_ctor_get(x_17, 6); +x_21 = lean_array_pop(x_20); +lean_ctor_set(x_17, 6, x_21); +x_22 = lean_st_ref_set(x_1, x_17, x_18); +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) { -lean_object* x_32; lean_object* x_33; -lean_free_object(x_26); -lean_dec(x_2); -lean_dec(x_1); -x_32 = lean_box(0); -x_33 = lean_apply_10(x_30, x_32, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_29); -return x_33; +lean_object* x_24; +x_24 = lean_ctor_get(x_22, 0); +lean_dec(x_24); +lean_ctor_set(x_22, 0, x_15); +return x_22; } else { -lean_object* x_34; -x_34 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_29); -if (lean_obj_tag(x_34) == 0) -{ -lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_35 = lean_ctor_get(x_34, 1); -lean_inc(x_35); -lean_dec(x_34); -x_36 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_35); -lean_dec(x_1); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_38 = lean_ctor_get(x_36, 0); -x_39 = lean_ctor_get(x_36, 1); -x_40 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); -lean_dec(x_2); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) -{ -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_42 = lean_ctor_get(x_40, 0); -x_43 = lean_ctor_get(x_40, 1); -x_44 = l_Lean_MessageData_ofFormat(x_38); -x_45 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -lean_ctor_set_tag(x_40, 7); -lean_ctor_set(x_40, 1, x_44); -lean_ctor_set(x_40, 0, x_45); -x_46 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; -lean_ctor_set_tag(x_36, 7); -lean_ctor_set(x_36, 1, x_46); -lean_ctor_set(x_36, 0, x_40); -x_47 = l_Lean_MessageData_ofFormat(x_42); -lean_ctor_set_tag(x_26, 7); -lean_ctor_set(x_26, 1, x_47); -lean_ctor_set(x_26, 0, x_36); -x_48 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; -x_49 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_49, 0, x_26); -lean_ctor_set(x_49, 1, x_48); -x_50 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_25, x_49, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_43); -x_51 = lean_ctor_get(x_50, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_50, 1); -lean_inc(x_52); -lean_dec(x_50); -x_53 = lean_apply_10(x_30, x_51, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_52); -return x_53; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +lean_dec(x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_15); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_54 = lean_ctor_get(x_40, 0); -x_55 = lean_ctor_get(x_40, 1); -lean_inc(x_55); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +x_27 = lean_ctor_get(x_17, 0); +x_28 = lean_ctor_get(x_17, 1); +x_29 = lean_ctor_get(x_17, 2); +x_30 = lean_ctor_get(x_17, 3); +x_31 = lean_ctor_get(x_17, 4); +x_32 = lean_ctor_get(x_17, 5); +x_33 = lean_ctor_get(x_17, 6); +x_34 = lean_ctor_get_uint8(x_17, sizeof(void*)*23); +x_35 = lean_ctor_get(x_17, 7); +x_36 = lean_ctor_get(x_17, 8); +x_37 = lean_ctor_get(x_17, 9); +x_38 = lean_ctor_get(x_17, 10); +x_39 = lean_ctor_get(x_17, 11); +x_40 = lean_ctor_get(x_17, 12); +x_41 = lean_ctor_get(x_17, 13); +x_42 = lean_ctor_get(x_17, 14); +x_43 = lean_ctor_get(x_17, 15); +x_44 = lean_ctor_get(x_17, 16); +x_45 = lean_ctor_get(x_17, 17); +x_46 = lean_ctor_get(x_17, 18); +x_47 = lean_ctor_get(x_17, 19); +x_48 = lean_ctor_get(x_17, 20); +x_49 = lean_ctor_get(x_17, 21); +x_50 = lean_ctor_get(x_17, 22); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_17); +x_51 = lean_array_pop(x_33); +x_52 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_52, 0, x_27); +lean_ctor_set(x_52, 1, x_28); +lean_ctor_set(x_52, 2, x_29); +lean_ctor_set(x_52, 3, x_30); +lean_ctor_set(x_52, 4, x_31); +lean_ctor_set(x_52, 5, x_32); +lean_ctor_set(x_52, 6, x_51); +lean_ctor_set(x_52, 7, x_35); +lean_ctor_set(x_52, 8, x_36); +lean_ctor_set(x_52, 9, x_37); +lean_ctor_set(x_52, 10, x_38); +lean_ctor_set(x_52, 11, x_39); +lean_ctor_set(x_52, 12, x_40); +lean_ctor_set(x_52, 13, x_41); +lean_ctor_set(x_52, 14, x_42); +lean_ctor_set(x_52, 15, x_43); +lean_ctor_set(x_52, 16, x_44); +lean_ctor_set(x_52, 17, x_45); +lean_ctor_set(x_52, 18, x_46); +lean_ctor_set(x_52, 19, x_47); +lean_ctor_set(x_52, 20, x_48); +lean_ctor_set(x_52, 21, x_49); +lean_ctor_set(x_52, 22, x_50); +lean_ctor_set_uint8(x_52, sizeof(void*)*23, x_34); +x_53 = lean_st_ref_set(x_1, x_52, x_18); +x_54 = lean_ctor_get(x_53, 1); lean_inc(x_54); -lean_dec(x_40); -x_56 = l_Lean_MessageData_ofFormat(x_38); -x_57 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_58 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_56); -x_59 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; -lean_ctor_set_tag(x_36, 7); -lean_ctor_set(x_36, 1, x_59); -lean_ctor_set(x_36, 0, x_58); -x_60 = l_Lean_MessageData_ofFormat(x_54); -lean_ctor_set_tag(x_26, 7); -lean_ctor_set(x_26, 1, x_60); -lean_ctor_set(x_26, 0, x_36); -x_61 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; -x_62 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_62, 0, x_26); -lean_ctor_set(x_62, 1, x_61); -x_63 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_25, x_62, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_55); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -x_66 = lean_apply_10(x_30, x_64, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_65); -return x_66; -} -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_67 = lean_ctor_get(x_36, 0); -x_68 = lean_ctor_get(x_36, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_36); -x_69 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_68); -lean_dec(x_2); -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_72 = x_69; +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_55 = x_53; } else { - lean_dec_ref(x_69); - x_72 = lean_box(0); + lean_dec_ref(x_53); + x_55 = lean_box(0); } -x_73 = l_Lean_MessageData_ofFormat(x_67); -x_74 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_72)) { - x_75 = lean_alloc_ctor(7, 2, 0); +if (lean_is_scalar(x_55)) { + x_56 = lean_alloc_ctor(0, 2, 0); } else { - x_75 = x_72; - lean_ctor_set_tag(x_75, 7); + x_56 = x_55; +} +lean_ctor_set(x_56, 0, x_15); +lean_ctor_set(x_56, 1, x_54); +return x_56; } -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_73); -x_76 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; -x_77 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -x_78 = l_Lean_MessageData_ofFormat(x_70); -lean_ctor_set_tag(x_26, 7); -lean_ctor_set(x_26, 1, x_78); -lean_ctor_set(x_26, 0, x_77); -x_79 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; -x_80 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_80, 0, x_26); -lean_ctor_set(x_80, 1, x_79); -x_81 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_25, x_80, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_71); -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_apply_10(x_30, x_82, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_83); -return x_84; } } else { -uint8_t x_85; -lean_free_object(x_26); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_10, 0); +x_58 = lean_ctor_get(x_10, 1); +lean_inc(x_58); +lean_inc(x_57); lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_2); -lean_dec(x_1); -x_85 = !lean_is_exclusive(x_34); -if (x_85 == 0) +x_59 = lean_ctor_get(x_57, 6); +lean_inc(x_59); +lean_dec(x_57); +x_60 = l_Array_back_x3f___rarg(x_59); +lean_dec(x_59); +if (lean_obj_tag(x_60) == 0) { -return x_34; +lean_object* x_61; +x_61 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_34, 0); -x_87 = lean_ctor_get(x_34, 1); -lean_inc(x_87); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_62 = lean_st_ref_take(x_1, x_58); +x_63 = lean_ctor_get(x_62, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_62, 1); +lean_inc(x_64); +lean_dec(x_62); +x_65 = lean_ctor_get(x_63, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_63, 1); +lean_inc(x_66); +x_67 = lean_ctor_get(x_63, 2); +lean_inc(x_67); +x_68 = lean_ctor_get(x_63, 3); +lean_inc(x_68); +x_69 = lean_ctor_get(x_63, 4); +lean_inc(x_69); +x_70 = lean_ctor_get(x_63, 5); +lean_inc(x_70); +x_71 = lean_ctor_get(x_63, 6); +lean_inc(x_71); +x_72 = lean_ctor_get_uint8(x_63, sizeof(void*)*23); +x_73 = lean_ctor_get(x_63, 7); +lean_inc(x_73); +x_74 = lean_ctor_get(x_63, 8); +lean_inc(x_74); +x_75 = lean_ctor_get(x_63, 9); +lean_inc(x_75); +x_76 = lean_ctor_get(x_63, 10); +lean_inc(x_76); +x_77 = lean_ctor_get(x_63, 11); +lean_inc(x_77); +x_78 = lean_ctor_get(x_63, 12); +lean_inc(x_78); +x_79 = lean_ctor_get(x_63, 13); +lean_inc(x_79); +x_80 = lean_ctor_get(x_63, 14); +lean_inc(x_80); +x_81 = lean_ctor_get(x_63, 15); +lean_inc(x_81); +x_82 = lean_ctor_get(x_63, 16); +lean_inc(x_82); +x_83 = lean_ctor_get(x_63, 17); +lean_inc(x_83); +x_84 = lean_ctor_get(x_63, 18); +lean_inc(x_84); +x_85 = lean_ctor_get(x_63, 19); +lean_inc(x_85); +x_86 = lean_ctor_get(x_63, 20); lean_inc(x_86); -lean_dec(x_34); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; +x_87 = lean_ctor_get(x_63, 21); +lean_inc(x_87); +x_88 = lean_ctor_get(x_63, 22); +lean_inc(x_88); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + lean_ctor_release(x_63, 2); + lean_ctor_release(x_63, 3); + lean_ctor_release(x_63, 4); + lean_ctor_release(x_63, 5); + lean_ctor_release(x_63, 6); + lean_ctor_release(x_63, 7); + lean_ctor_release(x_63, 8); + lean_ctor_release(x_63, 9); + lean_ctor_release(x_63, 10); + lean_ctor_release(x_63, 11); + lean_ctor_release(x_63, 12); + lean_ctor_release(x_63, 13); + lean_ctor_release(x_63, 14); + lean_ctor_release(x_63, 15); + lean_ctor_release(x_63, 16); + lean_ctor_release(x_63, 17); + lean_ctor_release(x_63, 18); + lean_ctor_release(x_63, 19); + lean_ctor_release(x_63, 20); + lean_ctor_release(x_63, 21); + lean_ctor_release(x_63, 22); + x_89 = x_63; +} else { + lean_dec_ref(x_63); + x_89 = lean_box(0); } +x_90 = lean_array_pop(x_71); +if (lean_is_scalar(x_89)) { + x_91 = lean_alloc_ctor(0, 23, 1); +} else { + x_91 = x_89; +} +lean_ctor_set(x_91, 0, x_65); +lean_ctor_set(x_91, 1, x_66); +lean_ctor_set(x_91, 2, x_67); +lean_ctor_set(x_91, 3, x_68); +lean_ctor_set(x_91, 4, x_69); +lean_ctor_set(x_91, 5, x_70); +lean_ctor_set(x_91, 6, x_90); +lean_ctor_set(x_91, 7, x_73); +lean_ctor_set(x_91, 8, x_74); +lean_ctor_set(x_91, 9, x_75); +lean_ctor_set(x_91, 10, x_76); +lean_ctor_set(x_91, 11, x_77); +lean_ctor_set(x_91, 12, x_78); +lean_ctor_set(x_91, 13, x_79); +lean_ctor_set(x_91, 14, x_80); +lean_ctor_set(x_91, 15, x_81); +lean_ctor_set(x_91, 16, x_82); +lean_ctor_set(x_91, 17, x_83); +lean_ctor_set(x_91, 18, x_84); +lean_ctor_set(x_91, 19, x_85); +lean_ctor_set(x_91, 20, x_86); +lean_ctor_set(x_91, 21, x_87); +lean_ctor_set(x_91, 22, x_88); +lean_ctor_set_uint8(x_91, sizeof(void*)*23, x_72); +x_92 = lean_st_ref_set(x_1, x_91, x_64); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_94 = x_92; +} else { + lean_dec_ref(x_92); + x_94 = lean_box(0); } +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(0, 2, 0); +} else { + x_95 = x_94; } +lean_ctor_set(x_95, 0, x_60); +lean_ctor_set(x_95, 1, x_93); +return x_95; } -else -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_92; -x_89 = lean_ctor_get(x_26, 0); -x_90 = lean_ctor_get(x_26, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_26); -x_91 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__1; -x_92 = lean_unbox(x_89); -lean_dec(x_89); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; -lean_dec(x_2); -lean_dec(x_1); -x_93 = lean_box(0); -x_94 = lean_apply_10(x_91, x_93, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_90); -return x_94; } -else -{ -lean_object* x_95; -x_95 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_90); -if (lean_obj_tag(x_95) == 0) -{ -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_96 = lean_ctor_get(x_95, 1); -lean_inc(x_96); -lean_dec(x_95); -x_97 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_96); -lean_dec(x_1); -x_98 = lean_ctor_get(x_97, 0); -lean_inc(x_98); -x_99 = lean_ctor_get(x_97, 1); -lean_inc(x_99); -if (lean_is_exclusive(x_97)) { - lean_ctor_release(x_97, 0); - lean_ctor_release(x_97, 1); - x_100 = x_97; -} else { - lean_dec_ref(x_97); - x_100 = lean_box(0); } -x_101 = l_Lean_Meta_Grind_ppENodeRef(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_99); -lean_dec(x_2); -x_102 = lean_ctor_get(x_101, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_101, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_104 = x_101; -} else { - lean_dec_ref(x_101); - x_104 = lean_box(0); -} -x_105 = l_Lean_MessageData_ofFormat(x_98); -x_106 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -if (lean_is_scalar(x_104)) { - x_107 = lean_alloc_ctor(7, 2, 0); -} else { - x_107 = x_104; - lean_ctor_set_tag(x_107, 7); -} -lean_ctor_set(x_107, 0, x_106); -lean_ctor_set(x_107, 1, x_105); -x_108 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__3; -if (lean_is_scalar(x_100)) { - x_109 = lean_alloc_ctor(7, 2, 0); -} else { - x_109 = x_100; - lean_ctor_set_tag(x_109, 7); -} -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_108); -x_110 = l_Lean_MessageData_ofFormat(x_102); -x_111 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -x_112 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___closed__5; -x_113 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -x_114 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_25, x_113, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_103); -x_115 = lean_ctor_get(x_114, 0); -lean_inc(x_115); -x_116 = lean_ctor_get(x_114, 1); -lean_inc(x_116); -lean_dec(x_114); -x_117 = lean_apply_10(x_91, x_115, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_116); -return x_117; } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_118 = lean_ctor_get(x_95, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_95, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - x_120 = x_95; -} else { - lean_dec_ref(x_95); - x_120 = lean_box(0); -} -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); -} else { - x_121 = x_120; -} -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_119); -return x_121; -} -} -} +return x_12; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_122; -lean_dec(x_15); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_10; +x_10 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_122 = !lean_is_exclusive(x_17); -if (x_122 == 0) -{ -return x_17; -} -else -{ -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_17, 0); -x_124 = lean_ctor_get(x_17, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_17); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; -} +return x_10; } } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; +x_12 = l_Lean_Core_checkSystem(x_11, x_8, x_9, x_10); +if (lean_obj_tag(x_12) == 0) { -uint8_t x_126; +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 1); +lean_inc(x_13); lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_126 = !lean_is_exclusive(x_14); -if (x_126 == 0) +x_16 = !lean_is_exclusive(x_14); +if (x_16 == 0) { +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_14, 0); +lean_dec(x_17); +x_18 = lean_box(0); +lean_ctor_set(x_14, 0, x_18); return x_14; } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_127 = lean_ctor_get(x_14, 0); -x_128 = lean_ctor_get(x_14, 1); -lean_inc(x_128); -lean_inc(x_127); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); lean_dec(x_14); -x_129 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_129, 0, x_127); -lean_ctor_set(x_129, 1, x_128); -return x_129; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_1); -lean_dec(x_1); -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__3(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); -return x_15; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; +x_22 = lean_ctor_get(x_15, 0); +lean_inc(x_22); +lean_dec(x_15); +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_dec(x_14); +x_24 = lean_ctor_get(x_22, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_22, 1); +lean_inc(x_25); +x_26 = lean_ctor_get(x_22, 2); +lean_inc(x_26); +x_27 = lean_ctor_get_uint8(x_22, sizeof(void*)*3); +lean_dec(x_22); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_28 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_24, x_25, x_26, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +if (lean_obj_tag(x_28) == 0) { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_1); -lean_dec(x_1); -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__4(x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_4); -return x_15; -} +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_28, 1); +lean_inc(x_29); +lean_dec(x_28); +x_30 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); +return x_30; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: +else { -uint8_t x_15; uint8_t x_16; lean_object* x_17; -x_15 = lean_unbox(x_1); -lean_dec(x_1); -x_16 = lean_unbox(x_4); -lean_dec(x_4); -x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__5(x_15, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +uint8_t x_31; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_17; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -_start: -{ -uint8_t x_21; uint8_t x_22; uint8_t x_23; lean_object* x_24; -x_21 = lean_unbox(x_4); lean_dec(x_4); -x_22 = lean_unbox(x_9); -lean_dec(x_9); -x_23 = lean_unbox(x_10); -lean_dec(x_10); -x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__6(x_1, x_2, x_3, x_21, x_5, x_6, x_7, x_8, x_22, x_23, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -lean_dec(x_11); -return x_24; -} +lean_dec(x_3); +lean_dec(x_2); +x_31 = !lean_is_exclusive(x_28); +if (x_31 == 0) +{ +return x_28; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -uint8_t x_17; lean_object* x_18; -x_17 = lean_unbox(x_4); -lean_dec(x_4); -x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__7(x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -return x_18; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_28, 0); +x_33 = lean_ctor_get(x_28, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_28); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; lean_object* x_18; -x_17 = lean_unbox(x_4); -lean_dec(x_4); -x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__8(x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -return x_18; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_35; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -9039,270 +12150,254 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_11; -} +x_35 = !lean_is_exclusive(x_12); +if (x_35 == 0) +{ +return x_12; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: +else { -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_12, 0); +x_37 = lean_ctor_get(x_12, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_12); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1() { +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___closed__1() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1___boxed), 10, 0); +return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_st_ref_take(x_1, x_9); +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_11, 5); -lean_dec(x_14); -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1; -lean_ctor_set(x_11, 5, x_15); -x_16 = lean_st_ref_set(x_1, x_11, x_12); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_16, 0); -lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_16, 0, x_19); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___closed__1; +x_15 = lean_box(0); +x_16 = lean_apply_10(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); return x_16; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_16, 1); -lean_inc(x_20); -lean_dec(x_16); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; -} -} -else +lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_17 = lean_ctor_get(x_10, 1); +lean_inc(x_17); +lean_dec(x_10); +x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_23 = lean_ctor_get(x_11, 0); -x_24 = lean_ctor_get(x_11, 1); -x_25 = lean_ctor_get(x_11, 2); -x_26 = lean_ctor_get(x_11, 3); -x_27 = lean_ctor_get(x_11, 4); -x_28 = lean_ctor_get_uint8(x_11, sizeof(void*)*20); -x_29 = lean_ctor_get(x_11, 6); -x_30 = lean_ctor_get(x_11, 7); -x_31 = lean_ctor_get(x_11, 8); -x_32 = lean_ctor_get(x_11, 9); -x_33 = lean_ctor_get(x_11, 10); -x_34 = lean_ctor_get(x_11, 11); -x_35 = lean_ctor_get(x_11, 12); -x_36 = lean_ctor_get(x_11, 13); -x_37 = lean_ctor_get(x_11, 14); -x_38 = lean_ctor_get(x_11, 15); -x_39 = lean_ctor_get(x_11, 16); -x_40 = lean_ctor_get(x_11, 17); -x_41 = lean_ctor_get(x_11, 18); -x_42 = lean_ctor_get(x_11, 19); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_27); -lean_inc(x_26); -lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_11); -x_43 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___closed__1; -x_44 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_44, 0, x_23); -lean_ctor_set(x_44, 1, x_24); -lean_ctor_set(x_44, 2, x_25); -lean_ctor_set(x_44, 3, x_26); -lean_ctor_set(x_44, 4, x_27); -lean_ctor_set(x_44, 5, x_43); -lean_ctor_set(x_44, 6, x_29); -lean_ctor_set(x_44, 7, x_30); -lean_ctor_set(x_44, 8, x_31); -lean_ctor_set(x_44, 9, x_32); -lean_ctor_set(x_44, 10, x_33); -lean_ctor_set(x_44, 11, x_34); -lean_ctor_set(x_44, 12, x_35); -lean_ctor_set(x_44, 13, x_36); -lean_ctor_set(x_44, 14, x_37); -lean_ctor_set(x_44, 15, x_38); -lean_ctor_set(x_44, 16, x_39); -lean_ctor_set(x_44, 17, x_40); -lean_ctor_set(x_44, 18, x_41); -lean_ctor_set(x_44, 19, x_42); -lean_ctor_set_uint8(x_44, sizeof(void*)*20, x_28); -x_45 = lean_st_ref_set(x_1, x_44, x_12); -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_47 = x_45; -} else { - lean_dec_ref(x_45); - x_47 = lean_box(0); +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_18, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_18, 0, x_21); +return x_18; } -x_48 = lean_box(0); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_47; +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_18, 1); +lean_inc(x_22); +lean_dec(x_18); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_46); -return x_49; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); +return x_16; +} +else +{ +uint8_t x_17; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_10; +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) +{ +return x_14; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_14, 0); +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_14); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_12; -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_11); -return x_12; +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_ref_get(x_1, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = lean_ctor_get(x_12, 5); -lean_inc(x_14); -lean_dec(x_12); -x_15 = l_Array_back_x3f___rarg(x_14); -lean_dec(x_14); -if (lean_obj_tag(x_15) == 0) +uint8_t x_13; lean_object* x_14; +x_13 = 0; +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addHEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_ctor_set(x_10, 0, x_15); -return x_10; +uint8_t x_13; lean_object* x_14; +x_13 = 1; +x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +return x_14; } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_free_object(x_10); -x_16 = lean_st_ref_take(x_1, x_13); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = !lean_is_exclusive(x_17); -if (x_19 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_st_ref_take(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_ctor_get(x_17, 5); -x_21 = lean_array_pop(x_20); -lean_ctor_set(x_17, 5, x_21); -x_22 = lean_st_ref_set(x_1, x_17, x_18); -x_23 = !lean_is_exclusive(x_22); -if (x_23 == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_12, 22); +x_16 = l_Lean_PersistentArray_push___rarg(x_15, x_1); +lean_ctor_set(x_12, 22, x_16); +x_17 = lean_st_ref_set(x_2, x_12, x_13); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_dec(x_24); -lean_ctor_set(x_22, 0, x_15); -return x_22; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +lean_dec(x_19); +x_20 = lean_box(0); +lean_ctor_set(x_17, 0, x_20); +return x_17; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_15); -lean_ctor_set(x_26, 1, x_25); -return x_26; +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_17, 1); +lean_inc(x_21); +lean_dec(x_17); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_27 = lean_ctor_get(x_17, 0); -x_28 = lean_ctor_get(x_17, 1); -x_29 = lean_ctor_get(x_17, 2); -x_30 = lean_ctor_get(x_17, 3); -x_31 = lean_ctor_get(x_17, 4); -x_32 = lean_ctor_get(x_17, 5); -x_33 = lean_ctor_get_uint8(x_17, sizeof(void*)*20); -x_34 = lean_ctor_get(x_17, 6); -x_35 = lean_ctor_get(x_17, 7); -x_36 = lean_ctor_get(x_17, 8); -x_37 = lean_ctor_get(x_17, 9); -x_38 = lean_ctor_get(x_17, 10); -x_39 = lean_ctor_get(x_17, 11); -x_40 = lean_ctor_get(x_17, 12); -x_41 = lean_ctor_get(x_17, 13); -x_42 = lean_ctor_get(x_17, 14); -x_43 = lean_ctor_get(x_17, 15); -x_44 = lean_ctor_get(x_17, 16); -x_45 = lean_ctor_get(x_17, 17); -x_46 = lean_ctor_get(x_17, 18); -x_47 = lean_ctor_get(x_17, 19); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_24 = lean_ctor_get(x_12, 0); +x_25 = lean_ctor_get(x_12, 1); +x_26 = lean_ctor_get(x_12, 2); +x_27 = lean_ctor_get(x_12, 3); +x_28 = lean_ctor_get(x_12, 4); +x_29 = lean_ctor_get(x_12, 5); +x_30 = lean_ctor_get(x_12, 6); +x_31 = lean_ctor_get_uint8(x_12, sizeof(void*)*23); +x_32 = lean_ctor_get(x_12, 7); +x_33 = lean_ctor_get(x_12, 8); +x_34 = lean_ctor_get(x_12, 9); +x_35 = lean_ctor_get(x_12, 10); +x_36 = lean_ctor_get(x_12, 11); +x_37 = lean_ctor_get(x_12, 12); +x_38 = lean_ctor_get(x_12, 13); +x_39 = lean_ctor_get(x_12, 14); +x_40 = lean_ctor_get(x_12, 15); +x_41 = lean_ctor_get(x_12, 16); +x_42 = lean_ctor_get(x_12, 17); +x_43 = lean_ctor_get(x_12, 18); +x_44 = lean_ctor_get(x_12, 19); +x_45 = lean_ctor_get(x_12, 20); +x_46 = lean_ctor_get(x_12, 21); +x_47 = lean_ctor_get(x_12, 22); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); @@ -9317,37 +12412,43 @@ lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); -lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); -lean_dec(x_17); -x_48 = lean_array_pop(x_32); -x_49 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_49, 0, x_27); -lean_ctor_set(x_49, 1, x_28); -lean_ctor_set(x_49, 2, x_29); -lean_ctor_set(x_49, 3, x_30); -lean_ctor_set(x_49, 4, x_31); -lean_ctor_set(x_49, 5, x_48); -lean_ctor_set(x_49, 6, x_34); -lean_ctor_set(x_49, 7, x_35); -lean_ctor_set(x_49, 8, x_36); -lean_ctor_set(x_49, 9, x_37); -lean_ctor_set(x_49, 10, x_38); -lean_ctor_set(x_49, 11, x_39); -lean_ctor_set(x_49, 12, x_40); -lean_ctor_set(x_49, 13, x_41); -lean_ctor_set(x_49, 14, x_42); -lean_ctor_set(x_49, 15, x_43); -lean_ctor_set(x_49, 16, x_44); -lean_ctor_set(x_49, 17, x_45); -lean_ctor_set(x_49, 18, x_46); -lean_ctor_set(x_49, 19, x_47); -lean_ctor_set_uint8(x_49, sizeof(void*)*20, x_33); -x_50 = lean_st_ref_set(x_1, x_49, x_18); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_12); +x_48 = l_Lean_PersistentArray_push___rarg(x_47, x_1); +x_49 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_49, 0, x_24); +lean_ctor_set(x_49, 1, x_25); +lean_ctor_set(x_49, 2, x_26); +lean_ctor_set(x_49, 3, x_27); +lean_ctor_set(x_49, 4, x_28); +lean_ctor_set(x_49, 5, x_29); +lean_ctor_set(x_49, 6, x_30); +lean_ctor_set(x_49, 7, x_32); +lean_ctor_set(x_49, 8, x_33); +lean_ctor_set(x_49, 9, x_34); +lean_ctor_set(x_49, 10, x_35); +lean_ctor_set(x_49, 11, x_36); +lean_ctor_set(x_49, 12, x_37); +lean_ctor_set(x_49, 13, x_38); +lean_ctor_set(x_49, 14, x_39); +lean_ctor_set(x_49, 15, x_40); +lean_ctor_set(x_49, 16, x_41); +lean_ctor_set(x_49, 17, x_42); +lean_ctor_set(x_49, 18, x_43); +lean_ctor_set(x_49, 19, x_44); +lean_ctor_set(x_49, 20, x_45); +lean_ctor_set(x_49, 21, x_46); +lean_ctor_set(x_49, 22, x_48); +lean_ctor_set_uint8(x_49, sizeof(void*)*23, x_31); +x_50 = lean_st_ref_set(x_2, x_49, x_13); x_51 = lean_ctor_get(x_50, 1); lean_inc(x_51); if (lean_is_exclusive(x_50)) { @@ -9358,170 +12459,23 @@ if (lean_is_exclusive(x_50)) { lean_dec_ref(x_50); x_52 = lean_box(0); } -if (lean_is_scalar(x_52)) { - x_53 = lean_alloc_ctor(0, 2, 0); -} else { - x_53 = x_52; -} -lean_ctor_set(x_53, 0, x_15); -lean_ctor_set(x_53, 1, x_51); -return x_53; -} -} -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_54 = lean_ctor_get(x_10, 0); -x_55 = lean_ctor_get(x_10, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_10); -x_56 = lean_ctor_get(x_54, 5); -lean_inc(x_56); -lean_dec(x_54); -x_57 = l_Array_back_x3f___rarg(x_56); -lean_dec(x_56); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; -x_58 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_55); -return x_58; -} -else -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_59 = lean_st_ref_take(x_1, x_55); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_59, 1); -lean_inc(x_61); -lean_dec(x_59); -x_62 = lean_ctor_get(x_60, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_60, 1); -lean_inc(x_63); -x_64 = lean_ctor_get(x_60, 2); -lean_inc(x_64); -x_65 = lean_ctor_get(x_60, 3); -lean_inc(x_65); -x_66 = lean_ctor_get(x_60, 4); -lean_inc(x_66); -x_67 = lean_ctor_get(x_60, 5); -lean_inc(x_67); -x_68 = lean_ctor_get_uint8(x_60, sizeof(void*)*20); -x_69 = lean_ctor_get(x_60, 6); -lean_inc(x_69); -x_70 = lean_ctor_get(x_60, 7); -lean_inc(x_70); -x_71 = lean_ctor_get(x_60, 8); -lean_inc(x_71); -x_72 = lean_ctor_get(x_60, 9); -lean_inc(x_72); -x_73 = lean_ctor_get(x_60, 10); -lean_inc(x_73); -x_74 = lean_ctor_get(x_60, 11); -lean_inc(x_74); -x_75 = lean_ctor_get(x_60, 12); -lean_inc(x_75); -x_76 = lean_ctor_get(x_60, 13); -lean_inc(x_76); -x_77 = lean_ctor_get(x_60, 14); -lean_inc(x_77); -x_78 = lean_ctor_get(x_60, 15); -lean_inc(x_78); -x_79 = lean_ctor_get(x_60, 16); -lean_inc(x_79); -x_80 = lean_ctor_get(x_60, 17); -lean_inc(x_80); -x_81 = lean_ctor_get(x_60, 18); -lean_inc(x_81); -x_82 = lean_ctor_get(x_60, 19); -lean_inc(x_82); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - lean_ctor_release(x_60, 2); - lean_ctor_release(x_60, 3); - lean_ctor_release(x_60, 4); - lean_ctor_release(x_60, 5); - lean_ctor_release(x_60, 6); - lean_ctor_release(x_60, 7); - lean_ctor_release(x_60, 8); - lean_ctor_release(x_60, 9); - lean_ctor_release(x_60, 10); - lean_ctor_release(x_60, 11); - lean_ctor_release(x_60, 12); - lean_ctor_release(x_60, 13); - lean_ctor_release(x_60, 14); - lean_ctor_release(x_60, 15); - lean_ctor_release(x_60, 16); - lean_ctor_release(x_60, 17); - lean_ctor_release(x_60, 18); - lean_ctor_release(x_60, 19); - x_83 = x_60; -} else { - lean_dec_ref(x_60); - x_83 = lean_box(0); -} -x_84 = lean_array_pop(x_67); -if (lean_is_scalar(x_83)) { - x_85 = lean_alloc_ctor(0, 20, 1); -} else { - x_85 = x_83; -} -lean_ctor_set(x_85, 0, x_62); -lean_ctor_set(x_85, 1, x_63); -lean_ctor_set(x_85, 2, x_64); -lean_ctor_set(x_85, 3, x_65); -lean_ctor_set(x_85, 4, x_66); -lean_ctor_set(x_85, 5, x_84); -lean_ctor_set(x_85, 6, x_69); -lean_ctor_set(x_85, 7, x_70); -lean_ctor_set(x_85, 8, x_71); -lean_ctor_set(x_85, 9, x_72); -lean_ctor_set(x_85, 10, x_73); -lean_ctor_set(x_85, 11, x_74); -lean_ctor_set(x_85, 12, x_75); -lean_ctor_set(x_85, 13, x_76); -lean_ctor_set(x_85, 14, x_77); -lean_ctor_set(x_85, 15, x_78); -lean_ctor_set(x_85, 16, x_79); -lean_ctor_set(x_85, 17, x_80); -lean_ctor_set(x_85, 18, x_81); -lean_ctor_set(x_85, 19, x_82); -lean_ctor_set_uint8(x_85, sizeof(void*)*20, x_68); -x_86 = lean_st_ref_set(x_1, x_85, x_61); -x_87 = lean_ctor_get(x_86, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_88 = x_86; -} else { - lean_dec_ref(x_86); - x_88 = lean_box(0); -} -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(0, 2, 0); -} else { - x_89 = x_88; -} -lean_ctor_set(x_89, 0, x_57); -lean_ctor_set(x_89, 1, x_87); -return x_89; +x_53 = lean_box(0); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); +} else { + x_54 = x_52; } +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -9530,144 +12484,114 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_12; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_10; +return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addNewEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__1; -x_12 = l_Lean_Core_checkSystem(x_11, x_8, x_9, x_10); -if (lean_obj_tag(x_12) == 0) +lean_object* x_14; +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_2); +lean_inc(x_1); +x_14 = l_Lean_Meta_mkEq(x_1, x_2, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_popNextEq_x3f(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); -if (lean_obj_tag(x_15) == 0) -{ -uint8_t x_16; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_16 = !lean_is_exclusive(x_14); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_14, 0); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_inc(x_15); +x_17 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); lean_dec(x_17); -x_18 = lean_box(0); -lean_ctor_set(x_14, 0, x_18); -return x_14; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_14, 1); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_15); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); lean_inc(x_19); -lean_dec(x_14); -x_20 = lean_box(0); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_19); -return x_21; -} -} -else +lean_inc(x_4); +lean_inc(x_1); +x_20 = l_Lean_Meta_Grind_internalize(x_1, x_4, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; -x_22 = lean_ctor_get(x_15, 0); -lean_inc(x_22); -lean_dec(x_15); -x_23 = lean_ctor_get(x_14, 1); -lean_inc(x_23); -lean_dec(x_14); -x_24 = lean_ctor_get(x_22, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -x_26 = lean_ctor_get(x_22, 2); -lean_inc(x_26); -x_27 = lean_ctor_get_uint8(x_22, sizeof(void*)*3); -lean_dec(x_22); +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); lean_inc(x_2); -x_28 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_24, x_25, x_26, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); -if (lean_obj_tag(x_28) == 0) +x_22 = l_Lean_Meta_Grind_internalize(x_2, x_4, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_29; lean_object* x_30; -x_29 = lean_ctor_get(x_28, 1); -lean_inc(x_29); -lean_dec(x_28); -x_30 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_29); -return x_30; +lean_object* x_23; uint8_t x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_22, 1); +lean_inc(x_23); +lean_dec(x_22); +x_24 = 0; +x_25 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +return x_25; } else { -uint8_t x_31; +uint8_t x_26; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_31 = !lean_is_exclusive(x_28); -if (x_31 == 0) +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_22); +if (x_26 == 0) { -return x_28; +return x_22; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_28, 0); -x_33 = lean_ctor_get(x_28, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_28); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; -} +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_22, 0); +x_28 = lean_ctor_get(x_22, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_22); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } else { -uint8_t x_35; +uint8_t x_30; +lean_dec(x_19); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -9676,62 +12600,34 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_35 = !lean_is_exclusive(x_12); -if (x_35 == 0) +lean_dec(x_1); +x_30 = !lean_is_exclusive(x_20); +if (x_30 == 0) { -return x_12; +return x_20; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_12, 0); -x_37 = lean_ctor_get(x_12, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_12); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; -} -} -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1___boxed), 10, 0); -return x_1; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_20, 0); +x_32 = lean_ctor_get(x_20, 1); +lean_inc(x_32); +lean_inc(x_31); +lean_dec(x_20); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); -lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___closed__1; -x_15 = lean_box(0); -x_16 = lean_apply_10(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -return x_16; } else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = lean_ctor_get(x_10, 1); -lean_inc(x_17); +uint8_t x_34; +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -x_18 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_resetNewEqs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_17); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -9740,44 +12636,32 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +x_34 = !lean_is_exclusive(x_14); +if (x_34 == 0) { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_18, 0); -lean_dec(x_20); -x_21 = lean_box(0); -lean_ctor_set(x_18, 0, x_21); -return x_18; +return x_14; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_18, 1); -lean_inc(x_22); -lean_dec(x_18); -x_23 = lean_box(0); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_22); -return x_24; -} -} +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_14, 0); +x_36 = lean_ctor_get(x_14, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_14); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goFact(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_14; +lean_object* x_14; lean_object* x_15; +x_14 = lean_box(0); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -9786,19 +12670,43 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +lean_inc(x_3); +x_15 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore_processTodo(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); -return x_16; +if (x_4 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_15, 1); +lean_inc(x_16); +lean_dec(x_15); +x_17 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_8, x_9, x_10, x_11, x_12, x_16); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_20 = l_Lean_Meta_mkEqTrue(x_1, x_9, x_10, x_11, x_12, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = 0; +x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_3, x_18, x_21, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +return x_24; } else { -uint8_t x_17; +uint8_t x_25; +lean_dec(x_18); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -9807,99 +12715,60 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_17 = !lean_is_exclusive(x_14); -if (x_17 == 0) -{ -return x_14; -} -else +lean_dec(x_3); +x_25 = !lean_is_exclusive(x_20); +if (x_25 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_14, 0); -x_19 = lean_ctor_get(x_14, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_14); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); return x_20; } -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -uint8_t x_14; lean_object* x_15; -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -uint8_t x_13; lean_object* x_14; -x_13 = 0; -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_14; -} +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_20, 0); +x_27 = lean_ctor_get(x_20, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_20); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addHEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; lean_object* x_14; -x_13 = 1; -x_14 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addNewEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { -_start: -{ -lean_object* x_14; -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_1); -x_14 = l_Lean_Meta_Grind_internalize(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_15, 1); +lean_inc(x_29); +lean_dec(x_15); +x_30 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_8, x_9, x_10, x_11, x_12, x_29); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_2); -x_16 = l_Lean_Meta_Grind_internalize(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); -if (lean_obj_tag(x_16) == 0) +x_33 = l_Lean_Meta_mkEqFalse(x_1, x_9, x_10, x_11, x_12, x_32); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = 0; -x_19 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_2, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -return x_19; +lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +lean_dec(x_33); +x_36 = 0; +x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_3, x_31, x_34, x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_35); +return x_37; } else { -uint8_t x_20; +uint8_t x_38; +lean_dec(x_31); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -9909,31 +12778,30 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_20 = !lean_is_exclusive(x_16); -if (x_20 == 0) +x_38 = !lean_is_exclusive(x_33); +if (x_38 == 0) { -return x_16; +return x_33; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_16, 0); -x_22 = lean_ctor_get(x_16, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_16); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_33, 0); +x_40 = lean_ctor_get(x_33, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_33); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} } } } else { -uint8_t x_24; +uint8_t x_42; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -9942,38 +12810,47 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_14); -if (x_24 == 0) +x_42 = !lean_is_exclusive(x_15); +if (x_42 == 0) { -return x_14; +return x_15; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_14, 0); -x_26 = lean_ctor_get(x_14, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_14); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_15, 0); +x_44 = lean_ctor_get(x_15, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_15); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; +} } } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goFact___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; +} } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_goEq(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { if (x_6 == 0) { -lean_object* x_17; -lean_dec(x_3); +lean_object* x_17; lean_object* x_18; +x_17 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_17, 0, x_3); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -9982,15 +12859,16 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); +lean_inc(x_17); lean_inc(x_2); lean_inc(x_4); -x_17 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_17) == 0) +x_18 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -10000,19 +12878,19 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_5); -x_19 = l_Lean_Meta_Grind_internalize(x_5, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_18); -if (lean_obj_tag(x_19) == 0) +x_20 = l_Lean_Meta_Grind_internalize(x_5, x_2, x_17, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); -x_21 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_4, x_5, x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_20); -return x_21; +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_4, x_5, x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_21); +return x_22; } else { -uint8_t x_22; +uint8_t x_23; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -10024,29 +12902,30 @@ lean_dec(x_8); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_22 = !lean_is_exclusive(x_19); -if (x_22 == 0) +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) { -return x_19; +return x_20; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } else { -uint8_t x_26; +uint8_t x_27; +lean_dec(x_17); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -10059,31 +12938,32 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_26 = !lean_is_exclusive(x_17); -if (x_26 == 0) +x_27 = !lean_is_exclusive(x_18); +if (x_27 == 0) { -return x_17; +return x_18; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_17, 0); -x_28 = lean_ctor_get(x_17, 1); +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_18, 0); +x_29 = lean_ctor_get(x_18, 1); +lean_inc(x_29); lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_17); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_dec(x_18); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } } else { -lean_object* x_30; +lean_object* x_31; lean_object* x_32; lean_dec(x_5); lean_dec(x_4); +x_31 = lean_box(0); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -10093,40 +12973,40 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_3); -x_30 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_30) == 0) +x_32 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_31, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_31 = lean_ctor_get(x_30, 1); -lean_inc(x_31); -lean_dec(x_30); -x_32 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_11, x_12, x_13, x_14, x_15, x_31); -x_33 = lean_ctor_get(x_32, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_33 = lean_ctor_get(x_32, 1); lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); lean_dec(x_32); +x_34 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_11, x_12, x_13, x_14, x_15, x_33); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_35 = l_Lean_Meta_mkEqFalse(x_1, x_12, x_13, x_14, x_15, x_34); -if (lean_obj_tag(x_35) == 0) +x_37 = l_Lean_Meta_mkEqFalse(x_1, x_12, x_13, x_14, x_15, x_36); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = 0; -x_39 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_3, x_33, x_36, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_37); -return x_39; +lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = 0; +x_41 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_3, x_35, x_38, x_40, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_39); +return x_41; } else { -uint8_t x_40; -lean_dec(x_33); +uint8_t x_42; +lean_dec(x_35); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -10136,29 +13016,29 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_3); -x_40 = !lean_is_exclusive(x_35); -if (x_40 == 0) +x_42 = !lean_is_exclusive(x_37); +if (x_42 == 0) { -return x_35; +return x_37; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_35, 0); -x_42 = lean_ctor_get(x_35, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_35); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_37, 0); +x_44 = lean_ctor_get(x_37, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_37); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } else { -uint8_t x_44; +uint8_t x_46; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -10169,23 +13049,23 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_3); lean_dec(x_1); -x_44 = !lean_is_exclusive(x_30); -if (x_44 == 0) +x_46 = !lean_is_exclusive(x_32); +if (x_46 == 0) { -return x_30; +return x_32; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_30, 0); -x_46 = lean_ctor_get(x_30, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_30); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_32, 0); +x_48 = lean_ctor_get(x_32, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_32); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } } @@ -10212,189 +13092,35 @@ x_17 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_5, x_6, x_4, x_16, x_7, x_8, return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -uint8_t x_16; lean_object* x_17; -x_16 = 0; -x_17 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_5, x_6, x_4, x_16, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -return x_17; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_15; -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_15 = l_Lean_Meta_Grind_internalize(x_1, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) -{ -if (x_3 == 0) -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_9, x_10, x_11, x_12, x_13, x_16); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_20 = l_Lean_Meta_mkEqTrue(x_4, x_10, x_11, x_12, x_13, x_19); -if (lean_obj_tag(x_20) == 0) +uint8_t x_17; +x_17 = l_Lean_Expr_isProp(x_5); +if (x_17 == 0) { -lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = 0; -x_24 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_18, x_21, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); -return x_24; +uint8_t x_18; lean_object* x_19; +x_18 = 0; +x_19 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_6, x_7, x_4, x_18, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +return x_19; } else { -uint8_t x_25; -lean_dec(x_18); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); +lean_object* x_20; lean_dec(x_7); lean_dec(x_6); -lean_dec(x_1); -x_25 = !lean_is_exclusive(x_20); -if (x_25 == 0) -{ +x_20 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); return x_20; } -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_20, 0); -x_27 = lean_ctor_get(x_20, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_20); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; -} -} -} -else -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_15, 1); -lean_inc(x_29); -lean_dec(x_15); -x_30 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_9, x_10, x_11, x_12, x_13, x_29); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_33 = l_Lean_Meta_mkEqFalse(x_4, x_10, x_11, x_12, x_13, x_32); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = 0; -x_37 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqCore(x_1, x_31, x_34, x_36, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); -return x_37; -} -else -{ -uint8_t x_38; -lean_dec(x_31); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_1); -x_38 = !lean_is_exclusive(x_33); -if (x_38 == 0) -{ -return x_33; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_33, 0); -x_40 = lean_ctor_get(x_33, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_33); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} -} } } -else -{ -uint8_t x_42; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); -lean_dec(x_1); -x_42 = !lean_is_exclusive(x_15); -if (x_42 == 0) +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: { +lean_object* x_15; +x_15 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); return x_15; } -else -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_15, 0); -x_44 = lean_ctor_get(x_15, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_15); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; -} -} -} } static lean_object* _init_l_Lean_Meta_Grind_add_go___closed__1() { _start: @@ -10439,98 +13165,92 @@ x_17 = l_Lean_Expr_cleanupAnnotations(x_15); x_18 = l_Lean_Expr_isApp(x_17); if (x_18 == 0) { -lean_object* x_19; lean_object* x_20; +lean_object* x_19; lean_dec(x_17); -x_19 = lean_box(0); -x_20 = l_Lean_Meta_Grind_add_go___lambda__3(x_3, x_2, x_4, x_1, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_20; +x_19 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_19; } else { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = l_Lean_Expr_appArg(x_17, lean_box(0)); -x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); -x_23 = l_Lean_Expr_isApp(x_22); -if (x_23 == 0) +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = l_Lean_Expr_appArg(x_17, lean_box(0)); +x_21 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_22 = l_Lean_Expr_isApp(x_21); +if (x_22 == 0) { -lean_object* x_24; lean_object* x_25; -lean_dec(x_22); +lean_object* x_23; lean_dec(x_21); -x_24 = lean_box(0); -x_25 = l_Lean_Meta_Grind_add_go___lambda__3(x_3, x_2, x_4, x_1, x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_25; +lean_dec(x_20); +x_23 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_23; } else { -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = l_Lean_Expr_appArg(x_22, lean_box(0)); -x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); -x_28 = l_Lean_Expr_isApp(x_27); -if (x_28 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = l_Lean_Expr_appArg(x_21, lean_box(0)); +x_25 = l_Lean_Expr_appFnCleanup(x_21, lean_box(0)); +x_26 = l_Lean_Expr_isApp(x_25); +if (x_26 == 0) { -lean_object* x_29; lean_object* x_30; -lean_dec(x_27); -lean_dec(x_26); -lean_dec(x_21); -x_29 = lean_box(0); -x_30 = l_Lean_Meta_Grind_add_go___lambda__3(x_3, x_2, x_4, x_1, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_30; +lean_object* x_27; +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_20); +x_27 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_27; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_31 = l_Lean_Expr_appArg(x_27, lean_box(0)); -x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); -x_33 = l_Lean_Meta_Grind_add_go___closed__1; -x_34 = l_Lean_Expr_isConstOf(x_32, x_33); -if (x_34 == 0) +lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_28 = l_Lean_Expr_appArg(x_25, lean_box(0)); +x_29 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); +x_30 = l_Lean_Meta_Grind_add_go___closed__1; +x_31 = l_Lean_Expr_isConstOf(x_29, x_30); +if (x_31 == 0) { -uint8_t x_35; -lean_dec(x_26); -x_35 = l_Lean_Expr_isApp(x_32); -if (x_35 == 0) +uint8_t x_32; +lean_dec(x_24); +x_32 = l_Lean_Expr_isApp(x_29); +if (x_32 == 0) { -lean_object* x_36; lean_object* x_37; -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_21); -x_36 = lean_box(0); -x_37 = l_Lean_Meta_Grind_add_go___lambda__3(x_3, x_2, x_4, x_1, x_36, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_37; +lean_object* x_33; +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_20); +x_33 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_33; } else { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = l_Lean_Expr_appFnCleanup(x_32, lean_box(0)); -x_39 = l_Lean_Meta_Grind_add_go___closed__3; -x_40 = l_Lean_Expr_isConstOf(x_38, x_39); -lean_dec(x_38); -if (x_40 == 0) +lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_34 = l_Lean_Expr_appFnCleanup(x_29, lean_box(0)); +x_35 = l_Lean_Meta_Grind_add_go___closed__3; +x_36 = l_Lean_Expr_isConstOf(x_34, x_35); +lean_dec(x_34); +if (x_36 == 0) { -lean_object* x_41; lean_object* x_42; -lean_dec(x_31); -lean_dec(x_21); -x_41 = lean_box(0); -x_42 = l_Lean_Meta_Grind_add_go___lambda__3(x_3, x_2, x_4, x_1, x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_42; +lean_object* x_37; +lean_dec(x_28); +lean_dec(x_20); +x_37 = l_Lean_Meta_Grind_add_goFact(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_37; } else { -uint8_t x_43; lean_object* x_44; -x_43 = 1; -x_44 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_31, x_21, x_4, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_44; +uint8_t x_38; lean_object* x_39; +x_38 = 1; +x_39 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_28, x_20, x_4, x_38, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_39; } } } else { -uint8_t x_45; lean_object* x_46; -lean_dec(x_32); -lean_dec(x_31); -x_45 = 0; -x_46 = l_Lean_Meta_Grind_add_goEq(x_1, x_2, x_3, x_26, x_21, x_4, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -return x_46; +lean_object* x_40; +lean_dec(x_29); +x_40 = l_Lean_Meta_Grind_add_go___lambda__2(x_1, x_2, x_3, x_4, x_28, x_24, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +lean_dec(x_28); +return x_40; } } } @@ -10547,23 +13267,24 @@ x_17 = l_Lean_Meta_Grind_add_go___lambda__1(x_1, x_2, x_3, x_16, x_5, x_6, x_7, return x_17; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -uint8_t x_16; lean_object* x_17; -x_16 = lean_unbox(x_4); +uint8_t x_17; lean_object* x_18; +x_17 = lean_unbox(x_4); lean_dec(x_4); -x_17 = l_Lean_Meta_Grind_add_go___lambda__2(x_1, x_2, x_3, x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -return x_17; +x_18 = l_Lean_Meta_Grind_add_go___lambda__2(x_1, x_2, x_3, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_5); +return x_18; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add_go___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { uint8_t x_15; lean_object* x_16; -x_15 = lean_unbox(x_3); -lean_dec(x_3); -x_16 = l_Lean_Meta_Grind_add_go___lambda__3(x_1, x_2, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = l_Lean_Meta_Grind_add_go___lambda__3(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_5); return x_16; } @@ -10739,63 +13460,74 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_add(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = l_Lean_Meta_Grind_add___closed__2; -x_14 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_unbox(x_15); -lean_dec(x_15); -if (x_16 == 0) +lean_object* x_13; uint8_t x_14; +lean_inc(x_1); +x_13 = l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_storeFact(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = lean_box(0); -x_19 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -return x_19; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_15 = lean_ctor_get(x_13, 1); +x_16 = lean_ctor_get(x_13, 0); +lean_dec(x_16); +x_17 = l_Lean_Meta_Grind_add___closed__2; +x_18 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_unbox(x_19); +lean_dec(x_19); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_free_object(x_13); +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = lean_box(0); +x_23 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); +return x_23; } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_14); -if (x_20 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_18); +if (x_24 == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_14, 1); -x_22 = lean_ctor_get(x_14, 0); -lean_dec(x_22); -x_23 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); -if (lean_obj_tag(x_23) == 0) +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_18, 1); +x_26 = lean_ctor_get(x_18, 0); +lean_dec(x_26); +x_27 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); lean_inc(x_1); -x_25 = l_Lean_MessageData_ofExpr(x_1); -x_26 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -lean_ctor_set_tag(x_14, 7); -lean_ctor_set(x_14, 1, x_25); -lean_ctor_set(x_14, 0, x_26); -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_14); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -lean_dec(x_29); -return x_31; +x_29 = l_Lean_MessageData_ofExpr(x_1); +x_30 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +lean_ctor_set_tag(x_18, 7); +lean_ctor_set(x_18, 1, x_29); +lean_ctor_set(x_18, 0, x_30); +lean_ctor_set_tag(x_13, 7); +lean_ctor_set(x_13, 1, x_30); +lean_ctor_set(x_13, 0, x_18); +x_31 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_17, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +x_32 = lean_ctor_get(x_31, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_31, 1); +lean_inc(x_33); +lean_dec(x_31); +x_34 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +lean_dec(x_32); +return x_34; } else { -uint8_t x_32; -lean_free_object(x_14); +uint8_t x_35; +lean_free_object(x_18); +lean_free_object(x_13); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10807,61 +13539,62 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_23); -if (x_32 == 0) +x_35 = !lean_is_exclusive(x_27); +if (x_35 == 0) { -return x_23; +return x_27; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_23, 0); -x_34 = lean_ctor_get(x_23, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_23); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_27, 0); +x_37 = lean_ctor_get(x_27, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_27); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; } } } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_14, 1); -lean_inc(x_36); -lean_dec(x_14); -x_37 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_36); -if (lean_obj_tag(x_37) == 0) +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_18, 1); +lean_inc(x_39); +lean_dec(x_18); +x_40 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_39); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_41 = lean_ctor_get(x_40, 1); +lean_inc(x_41); +lean_dec(x_40); lean_inc(x_1); -x_39 = l_Lean_MessageData_ofExpr(x_1); -x_40 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_39); -x_42 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_40); -x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_42, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); -lean_inc(x_45); -lean_dec(x_43); -x_46 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_44, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_45); -lean_dec(x_44); -return x_46; +x_42 = l_Lean_MessageData_ofExpr(x_1); +x_43 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_42); +lean_ctor_set_tag(x_13, 7); +lean_ctor_set(x_13, 1, x_43); +lean_ctor_set(x_13, 0, x_44); +x_45 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_17, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_41); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +lean_dec(x_46); +return x_48; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_free_object(x_13); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10873,26 +13606,131 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_47 = lean_ctor_get(x_37, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_37, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_49 = x_37; +x_49 = lean_ctor_get(x_40, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_40, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_51 = x_40; } else { - lean_dec_ref(x_37); - x_49 = lean_box(0); + lean_dec_ref(x_40); + x_51 = lean_box(0); } -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_51)) { + x_52 = lean_alloc_ctor(1, 2, 0); } else { - x_50 = x_49; + x_52 = x_51; +} +lean_ctor_set(x_52, 0, x_49); +lean_ctor_set(x_52, 1, x_50); +return x_52; +} +} } -lean_ctor_set(x_50, 0, x_47); -lean_ctor_set(x_50, 1, x_48); -return x_50; +} +else +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; +x_53 = lean_ctor_get(x_13, 1); +lean_inc(x_53); +lean_dec(x_13); +x_54 = l_Lean_Meta_Grind_add___closed__2; +x_55 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_54, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_53); +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); +x_57 = lean_unbox(x_56); +lean_dec(x_56); +if (x_57 == 0) +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_55, 1); +lean_inc(x_58); +lean_dec(x_55); +x_59 = lean_box(0); +x_60 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_59, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_58); +return x_60; +} +else +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_55, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_62 = x_55; +} else { + lean_dec_ref(x_55); + x_62 = lean_box(0); +} +x_63 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_61); +if (lean_obj_tag(x_63) == 0) +{ +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_64 = lean_ctor_get(x_63, 1); +lean_inc(x_64); +lean_dec(x_63); +lean_inc(x_1); +x_65 = l_Lean_MessageData_ofExpr(x_1); +x_66 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_removeParents___spec__4___closed__8; +if (lean_is_scalar(x_62)) { + x_67 = lean_alloc_ctor(7, 2, 0); +} else { + x_67 = x_62; + lean_ctor_set_tag(x_67, 7); +} +lean_ctor_set(x_67, 0, x_66); +lean_ctor_set(x_67, 1, x_65); +x_68 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_66); +x_69 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_54, x_68, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_64); +x_70 = lean_ctor_get(x_69, 0); +lean_inc(x_70); +x_71 = lean_ctor_get(x_69, 1); +lean_inc(x_71); +lean_dec(x_69); +x_72 = l_Lean_Meta_Grind_add___lambda__4(x_1, x_2, x_3, x_70, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_71); +lean_dec(x_70); +return x_72; +} +else +{ +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_dec(x_62); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_73 = lean_ctor_get(x_63, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_63, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_75 = x_63; +} else { + lean_dec_ref(x_63); + x_75 = lean_box(0); +} +if (lean_is_scalar(x_75)) { + x_76 = lean_alloc_ctor(1, 2, 0); +} else { + x_76 = x_75; +} +lean_ctor_set(x_76, 0, x_73); +lean_ctor_set(x_76, 1, x_74); +return x_76; } } } @@ -10984,6 +13822,7 @@ lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_objec lean_object* initialize_Lean_Meta_Tactic_Grind_Inv(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_PP(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Ctor(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Util(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Internalize(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Core(uint8_t builtin, lean_object* w) { @@ -11008,6 +13847,9 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Ctor(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Util(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Internalize(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -11075,6 +13917,8 @@ l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__15); l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__16 = _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__16(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_closeGoalWithValuesEq___closed__16); +l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1 = _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1(); +lean_mark_persistent(l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_propagateEqcDown___spec__1___closed__1); l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__1); l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Core_0__Lean_Meta_Grind_addEqStep_go___lambda__3___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c index 33e0caa7696d..d4df32fcbd83 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatch.c @@ -88,6 +88,7 @@ lean_object* lean_environment_find(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatch_ematchTheorems___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematchAndAssert(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___boxed(lean_object**); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_assign_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___lambda__2___closed__3; @@ -117,6 +118,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_assign_x3f___spec__1___closed__5; LEAN_EXPORT lean_object* l_Lean_mkConstWithLevelParams___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedPUnit; +lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematchAndAssert___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); @@ -271,7 +273,6 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatch_ematchTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_forallMetaBoundedTelescope(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_EMatch_ematchTheorems___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Meta_Grind_ENode_isCongrRoot(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematchAndAssert___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getConstInfo___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_addNewInstance___spec__5___closed__3; @@ -326,7 +327,6 @@ uint64_t lean_uint64_shift_left(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematchAndAssert___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_annotateMatchEqnType___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___spec__5___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); @@ -358,7 +358,7 @@ static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_G static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f___closed__7; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___spec__3___closed__11; @@ -404,7 +404,7 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_instantiateTheorem___lambda__2___closed__5; lean_object* l_ReaderT_instMonad___rarg(lean_object*); -lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_ematchAndAssert___closed__2; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -2152,85 +2152,91 @@ return x_13; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_15; -x_15 = l_Lean_Meta_Grind_getNext(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_st_ref_get(x_6, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Meta_Grind_Goal_getNext(x_16, x_2, x_12, x_13, x_17); +if (lean_obj_tag(x_18) == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_15, 0); -x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_17, x_1); -if (x_18 == 0) +lean_object* x_20; uint8_t x_21; +x_20 = lean_ctor_get(x_18, 0); +x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_20, x_1); +if (x_21 == 0) { -lean_object* x_19; -x_19 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_15, 0, x_19); -return x_15; +lean_object* x_22; +x_22 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_18, 0, x_22); +return x_18; } else { -lean_object* x_20; -x_20 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_20, 0, x_17); -lean_ctor_set(x_15, 0, x_20); -return x_15; +lean_object* x_23; +x_23 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_23, 0, x_20); +lean_ctor_set(x_18, 0, x_23); +return x_18; } } else { -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_15, 0); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_15); -x_23 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_21, x_1); -if (x_23 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_18, 0); +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_18); +x_26 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_24, x_1); +if (x_26 == 0) { -lean_object* x_24; lean_object* x_25; -x_24 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_24, 0, x_21); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_22); -return x_25; +lean_object* x_27; lean_object* x_28; +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_24); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_25); +return x_28; } else { -lean_object* x_26; lean_object* x_27; -x_26 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_26, 0, x_21); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_22); -return x_27; +lean_object* x_29; lean_object* x_30; +x_29 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_29, 0, x_24); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_25); +return x_30; } } } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_15); -if (x_28 == 0) +uint8_t x_31; +x_31 = !lean_is_exclusive(x_18); +if (x_31 == 0) { -return x_15; +return x_18; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_15, 0); -x_30 = lean_ctor_get(x_15, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_15); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_18, 0); +x_33 = lean_ctor_get(x_18, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_18); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } @@ -2238,42 +2244,48 @@ return x_31; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { -lean_object* x_19; lean_object* x_20; lean_object* x_26; -lean_inc(x_7); -x_26 = l_Lean_Meta_Grind_getENode(x_7, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -if (lean_obj_tag(x_26) == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_81; +lean_object* x_19; lean_object* x_20; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_26 = lean_st_ref_get(x_10, x_18); x_27 = lean_ctor_get(x_26, 0); lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 8); -lean_inc(x_29); -x_81 = lean_nat_dec_lt(x_29, x_4); -if (x_81 == 0) +lean_inc(x_7); +x_29 = l_Lean_Meta_Grind_Goal_getENode(x_27, x_7, x_16, x_17, x_28); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_82; lean_object* x_83; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_84; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); lean_dec(x_29); -lean_dec(x_27); -x_82 = lean_box(0); -x_83 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_82, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_28); -if (lean_obj_tag(x_83) == 0) +x_32 = lean_ctor_get(x_30, 8); +lean_inc(x_32); +x_84 = lean_nat_dec_lt(x_32, x_4); +if (x_84 == 0) { -lean_object* x_84; lean_object* x_85; -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); -lean_inc(x_85); -lean_dec(x_83); -x_19 = x_84; -x_20 = x_85; +lean_object* x_85; lean_object* x_86; +lean_dec(x_32); +lean_dec(x_30); +x_85 = lean_box(0); +x_86 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_85, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_86) == 0) +{ +lean_object* x_87; lean_object* x_88; +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_19 = x_87; +x_20 = x_88; goto block_25; } else { -uint8_t x_86; +uint8_t x_89; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2283,56 +2295,56 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_86 = !lean_is_exclusive(x_83); -if (x_86 == 0) +x_89 = !lean_is_exclusive(x_86); +if (x_89 == 0) { -return x_83; +return x_86; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_83, 0); -x_88 = lean_ctor_get(x_83, 1); -lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_83); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_86, 0); +x_91 = lean_ctor_get(x_86, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_86); +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; } } } else { -uint8_t x_90; -x_90 = lean_ctor_get_uint8(x_27, sizeof(void*)*10 + 4); -if (x_90 == 0) +uint8_t x_93; +x_93 = lean_ctor_get_uint8(x_30, sizeof(void*)*11 + 4); +if (x_93 == 0) { -uint8_t x_91; -x_91 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_27); -lean_dec(x_27); -if (x_91 == 0) +uint8_t x_94; +x_94 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_30); +lean_dec(x_30); +if (x_94 == 0) { -lean_object* x_92; lean_object* x_93; -lean_dec(x_29); -x_92 = lean_box(0); -x_93 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_92, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_28); -if (lean_obj_tag(x_93) == 0) +lean_object* x_95; lean_object* x_96; +lean_dec(x_32); +x_95 = lean_box(0); +x_96 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_95, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_96) == 0) { -lean_object* x_94; lean_object* x_95; -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -lean_dec(x_93); -x_19 = x_94; -x_20 = x_95; +lean_object* x_97; lean_object* x_98; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +x_19 = x_97; +x_20 = x_98; goto block_25; } else { -uint8_t x_96; +uint8_t x_99; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2342,71 +2354,71 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_96 = !lean_is_exclusive(x_93); -if (x_96 == 0) +x_99 = !lean_is_exclusive(x_96); +if (x_99 == 0) { -return x_93; +return x_96; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_97 = lean_ctor_get(x_93, 0); -x_98 = lean_ctor_get(x_93, 1); -lean_inc(x_98); -lean_inc(x_97); -lean_dec(x_93); -x_99 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_99, 0, x_97); -lean_ctor_set(x_99, 1, x_98); -return x_99; +lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_100 = lean_ctor_get(x_96, 0); +x_101 = lean_ctor_get(x_96, 1); +lean_inc(x_101); +lean_inc(x_100); +lean_dec(x_96); +x_102 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_102, 0, x_100); +lean_ctor_set(x_102, 1, x_101); +return x_102; } } } else { -lean_object* x_100; -x_100 = lean_box(0); -x_30 = x_100; -goto block_80; +lean_object* x_103; +x_103 = lean_box(0); +x_33 = x_103; +goto block_83; } } else { -lean_object* x_101; -lean_dec(x_27); -x_101 = lean_box(0); -x_30 = x_101; -goto block_80; +lean_object* x_104; +lean_dec(x_30); +x_104 = lean_box(0); +x_33 = x_104; +goto block_83; } } -block_80: +block_83: { -lean_object* x_31; uint8_t x_32; -lean_dec(x_30); -x_31 = l_Lean_Expr_getAppFn(x_7); -x_32 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_eqvFunctions(x_5, x_31); -lean_dec(x_31); -if (x_32 == 0) +lean_object* x_34; uint8_t x_35; +lean_dec(x_33); +x_34 = l_Lean_Expr_getAppFn(x_7); +x_35 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_eqvFunctions(x_5, x_34); +lean_dec(x_34); +if (x_35 == 0) { -lean_object* x_33; lean_object* x_34; -lean_dec(x_29); -x_33 = lean_box(0); -x_34 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_28); -if (lean_obj_tag(x_34) == 0) +lean_object* x_36; lean_object* x_37; +lean_dec(x_32); +x_36 = lean_box(0); +x_37 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_36, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_35; lean_object* x_36; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_19 = x_35; -x_20 = x_36; +lean_object* x_38; lean_object* x_39; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_19 = x_38; +x_20 = x_39; goto block_25; } else { -uint8_t x_37; +uint8_t x_40; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2416,54 +2428,54 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_34); -if (x_37 == 0) +x_40 = !lean_is_exclusive(x_37); +if (x_40 == 0) { -return x_34; +return x_37; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_34, 0); -x_39 = lean_ctor_get(x_34, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_34); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_37, 0); +x_42 = lean_ctor_get(x_37, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_37); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_41 = lean_unsigned_to_nat(0u); -x_42 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_41); -x_43 = lean_nat_dec_eq(x_42, x_6); -lean_dec(x_42); -if (x_43 == 0) +lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_44 = lean_unsigned_to_nat(0u); +x_45 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_7, x_44); +x_46 = lean_nat_dec_eq(x_45, x_6); +lean_dec(x_45); +if (x_46 == 0) { -lean_object* x_44; lean_object* x_45; -lean_dec(x_29); -x_44 = lean_box(0); -x_45 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_44, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_28); -if (lean_obj_tag(x_45) == 0) +lean_object* x_47; lean_object* x_48; +lean_dec(x_32); +x_47 = lean_box(0); +x_48 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_47, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_19 = x_46; -x_20 = x_47; +lean_object* x_49; lean_object* x_50; +x_49 = lean_ctor_get(x_48, 0); +lean_inc(x_49); +x_50 = lean_ctor_get(x_48, 1); +lean_inc(x_50); +lean_dec(x_48); +x_19 = x_49; +x_20 = x_50; goto block_25; } else { -uint8_t x_48; +uint8_t x_51; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2473,29 +2485,29 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_48 = !lean_is_exclusive(x_45); -if (x_48 == 0) +x_51 = !lean_is_exclusive(x_48); +if (x_51 == 0) { -return x_45; +return x_48; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_45, 0); -x_50 = lean_ctor_get(x_45, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_45); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_48, 0); +x_53 = lean_ctor_get(x_48, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_48); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; } } } else { -lean_object* x_52; +lean_object* x_55; lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); @@ -2505,36 +2517,36 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_1); -x_52 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_1, x_2, x_7, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_28); -if (lean_obj_tag(x_52) == 0) -{ -lean_object* x_53; -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -if (lean_obj_tag(x_53) == 0) +x_55 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_1, x_2, x_7, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_31); +if (lean_obj_tag(x_55) == 0) { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_29); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = lean_box(0); -x_56 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_55, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_54); +lean_object* x_56; +x_56 = lean_ctor_get(x_55, 0); +lean_inc(x_56); if (lean_obj_tag(x_56) == 0) { -lean_object* x_57; lean_object* x_58; -x_57 = lean_ctor_get(x_56, 0); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_dec(x_32); +x_57 = lean_ctor_get(x_55, 1); lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_19 = x_57; -x_20 = x_58; +lean_dec(x_55); +x_58 = lean_box(0); +x_59 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_58, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_57); +if (lean_obj_tag(x_59) == 0) +{ +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +x_19 = x_60; +x_20 = x_61; goto block_25; } else { -uint8_t x_59; +uint8_t x_62; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2544,59 +2556,59 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_56); -if (x_59 == 0) +x_62 = !lean_is_exclusive(x_59); +if (x_62 == 0) { -return x_56; +return x_59; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_56, 0); -x_61 = lean_ctor_get(x_56, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_56); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_59, 0); +x_64 = lean_ctor_get(x_59, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_59); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_63 = lean_ctor_get(x_52, 1); -lean_inc(x_63); -lean_dec(x_52); -x_64 = lean_ctor_get(x_53, 0); -lean_inc(x_64); -lean_dec(x_53); -x_65 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_64, x_29); -x_66 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_65, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_63); -x_67 = lean_ctor_get(x_66, 0); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_66 = lean_ctor_get(x_55, 1); +lean_inc(x_66); +lean_dec(x_55); +x_67 = lean_ctor_get(x_56, 0); lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_67, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_68); -lean_dec(x_67); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; lean_object* x_71; +lean_dec(x_56); +x_68 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_67, x_32); +x_69 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_68, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_66); x_70 = lean_ctor_get(x_69, 0); lean_inc(x_70); x_71 = lean_ctor_get(x_69, 1); lean_inc(x_71); lean_dec(x_69); -x_19 = x_70; -x_20 = x_71; +x_72 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_3, x_7, x_70, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_71); +lean_dec(x_70); +if (lean_obj_tag(x_72) == 0) +{ +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); +x_19 = x_73; +x_20 = x_74; goto block_25; } else { -uint8_t x_72; +uint8_t x_75; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2606,31 +2618,31 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_1); -x_72 = !lean_is_exclusive(x_69); -if (x_72 == 0) +x_75 = !lean_is_exclusive(x_72); +if (x_75 == 0) { -return x_69; +return x_72; } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_69, 0); -x_74 = lean_ctor_get(x_69, 1); -lean_inc(x_74); -lean_inc(x_73); -lean_dec(x_69); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -return x_75; +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_72, 0); +x_77 = lean_ctor_get(x_72, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_72); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; } } } } else { -uint8_t x_76; -lean_dec(x_29); +uint8_t x_79; +lean_dec(x_32); lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2641,23 +2653,23 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_7); lean_dec(x_1); -x_76 = !lean_is_exclusive(x_52); -if (x_76 == 0) +x_79 = !lean_is_exclusive(x_55); +if (x_79 == 0) { -return x_52; +return x_55; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_52, 0); -x_78 = lean_ctor_get(x_52, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_52); -x_79 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_78); -return x_79; +lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_80 = lean_ctor_get(x_55, 0); +x_81 = lean_ctor_get(x_55, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_55); +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +return x_82; } } } @@ -2666,7 +2678,7 @@ return x_79; } else { -uint8_t x_102; +uint8_t x_105; lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); @@ -2677,23 +2689,23 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_7); lean_dec(x_1); -x_102 = !lean_is_exclusive(x_26); -if (x_102 == 0) +x_105 = !lean_is_exclusive(x_29); +if (x_105 == 0) { -return x_26; +return x_29; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_26, 0); -x_104 = lean_ctor_get(x_26, 1); -lean_inc(x_104); -lean_inc(x_103); -lean_dec(x_26); -x_105 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -return x_105; +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_29, 0); +x_107 = lean_ctor_get(x_29, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_29); +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 1, x_107); +return x_108; } } block_25: @@ -2867,56 +2879,45 @@ return x_15; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processOffset___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { -lean_object* x_18; lean_object* x_34; -lean_inc(x_6); -x_34 = l_Lean_Meta_Grind_getENode(x_6, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_34) == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +lean_object* x_18; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_34 = lean_st_ref_get(x_9, x_17); x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); x_36 = lean_ctor_get(x_34, 1); lean_inc(x_36); lean_dec(x_34); -x_37 = lean_ctor_get(x_35, 8); -lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_nat_dec_lt(x_37, x_5); -if (x_38 == 0) +lean_inc(x_6); +x_37 = l_Lean_Meta_Grind_Goal_getENode(x_35, x_6, x_15, x_16, x_36); +if (lean_obj_tag(x_37) == 0) { -lean_object* x_39; lean_object* x_40; +lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); lean_dec(x_37); -x_39 = lean_box(0); -x_40 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_39, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_36); -x_18 = x_40; +x_40 = lean_ctor_get(x_38, 8); +lean_inc(x_40); +lean_dec(x_38); +x_41 = lean_nat_dec_lt(x_40, x_5); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; +lean_dec(x_40); +x_42 = lean_box(0); +x_43 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_42, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_39); +x_18 = x_43; goto block_33; } else { -lean_object* x_41; -lean_inc(x_16); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_6); -x_41 = l_Lean_Meta_isOffset_x3f(x_6, x_13, x_14, x_15, x_16, x_36); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -if (lean_obj_tag(x_42) == 0) -{ -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_41, 1); -lean_inc(x_43); -lean_dec(x_41); +lean_object* x_44; lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_6); -x_44 = l_Lean_Meta_evalNat(x_6, x_13, x_14, x_15, x_16, x_43); +x_44 = l_Lean_Meta_isOffset_x3f(x_6, x_13, x_14, x_15, x_16, x_39); if (lean_obj_tag(x_44) == 0) { lean_object* x_45; @@ -2924,63 +2925,81 @@ x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); if (lean_obj_tag(x_45) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -lean_dec(x_37); +lean_object* x_46; lean_object* x_47; x_46 = lean_ctor_get(x_44, 1); lean_inc(x_46); lean_dec(x_44); -x_47 = lean_box(0); -x_48 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_46); -x_18 = x_48; +lean_inc(x_16); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_6); +x_47 = l_Lean_Meta_evalNat(x_6, x_13, x_14, x_15, x_16, x_46); +if (lean_obj_tag(x_47) == 0) +{ +lean_object* x_48; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +if (lean_obj_tag(x_48) == 0) +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_40); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = lean_box(0); +x_51 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_50, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_49); +x_18 = x_51; goto block_33; } else { -lean_object* x_49; lean_object* x_50; uint8_t x_51; -x_49 = lean_ctor_get(x_44, 1); -lean_inc(x_49); -lean_dec(x_44); -x_50 = lean_ctor_get(x_45, 0); -lean_inc(x_50); -lean_dec(x_45); -x_51 = lean_nat_dec_le(x_3, x_50); -if (x_51 == 0) +lean_object* x_52; lean_object* x_53; uint8_t x_54; +x_52 = lean_ctor_get(x_47, 1); +lean_inc(x_52); +lean_dec(x_47); +x_53 = lean_ctor_get(x_48, 0); +lean_inc(x_53); +lean_dec(x_48); +x_54 = lean_nat_dec_le(x_3, x_53); +if (x_54 == 0) { -lean_object* x_52; lean_object* x_53; -lean_dec(x_50); -lean_dec(x_37); -x_52 = lean_box(0); -x_53 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_52, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_49); -x_18 = x_53; +lean_object* x_55; lean_object* x_56; +lean_dec(x_53); +lean_dec(x_40); +x_55 = lean_box(0); +x_56 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_55, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_52); +x_18 = x_56; goto block_33; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_nat_sub(x_50, x_3); -lean_dec(x_50); -x_55 = l_Lean_mkNatLit(x_54); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_nat_sub(x_53, x_3); +lean_dec(x_53); +x_58 = l_Lean_mkNatLit(x_57); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); -x_56 = l_Lean_Meta_Grind_canon(x_55, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_49); -if (lean_obj_tag(x_56) == 0) +x_59 = l_Lean_Meta_Grind_canon(x_58, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_52); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = l_Lean_Meta_Grind_shareCommon(x_57, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_58); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_60 = lean_ctor_get(x_59, 0); lean_inc(x_60); x_61 = lean_ctor_get(x_59, 1); lean_inc(x_61); lean_dec(x_59); -x_62 = lean_unsigned_to_nat(1u); -x_63 = lean_nat_add(x_37, x_62); +x_62 = l_Lean_Meta_Grind_shareCommon(x_60, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_61); +x_63 = lean_ctor_get(x_62, 0); +lean_inc(x_63); +x_64 = lean_ctor_get(x_62, 1); +lean_inc(x_64); +lean_dec(x_62); +x_65 = lean_unsigned_to_nat(1u); +x_66 = lean_nat_add(x_40, x_65); +x_67 = lean_box(0); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -2989,14 +3008,14 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_60); -x_64 = l_Lean_Meta_Grind_internalize(x_60, x_63, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_61); -if (lean_obj_tag(x_64) == 0) +lean_inc(x_63); +x_68 = l_Lean_Meta_Grind_internalize(x_63, x_66, x_67, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_64); +if (lean_obj_tag(x_68) == 0) { -lean_object* x_65; lean_object* x_66; -x_65 = lean_ctor_get(x_64, 1); -lean_inc(x_65); -lean_dec(x_64); +lean_object* x_69; lean_object* x_70; +x_69 = lean_ctor_get(x_68, 1); +lean_inc(x_69); +lean_dec(x_68); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3007,93 +3026,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); lean_inc(x_1); -x_66 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_60, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_65); -if (lean_obj_tag(x_66) == 0) +x_70 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_63, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_69); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_67; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -if (lean_obj_tag(x_67) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -lean_dec(x_37); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_box(0); -x_70 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_69, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_68); -x_18 = x_70; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_dec(x_40); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_73, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_72); +x_18 = x_74; goto block_33; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_71 = lean_ctor_get(x_66, 1); -lean_inc(x_71); -lean_dec(x_66); -x_72 = lean_ctor_get(x_67, 0); -lean_inc(x_72); -lean_dec(x_67); -x_73 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_72, x_37); -x_74 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_73, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_71); -x_75 = lean_ctor_get(x_74, 0); +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); lean_inc(x_76); -lean_dec(x_74); -x_77 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_75, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_76); -lean_dec(x_75); -x_18 = x_77; -goto block_33; -} -} -else -{ -uint8_t x_78; -lean_dec(x_37); -lean_dec(x_6); -x_78 = !lean_is_exclusive(x_66); -if (x_78 == 0) -{ -x_18 = x_66; -goto block_33; -} -else -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_66, 0); -x_80 = lean_ctor_get(x_66, 1); -lean_inc(x_80); +lean_dec(x_71); +x_77 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_76, x_40); +x_78 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_77, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_75); +x_79 = lean_ctor_get(x_78, 0); lean_inc(x_79); -lean_dec(x_66); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); +x_80 = lean_ctor_get(x_78, 1); +lean_inc(x_80); +lean_dec(x_78); +x_81 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_79, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_80); +lean_dec(x_79); x_18 = x_81; goto block_33; } } -} else { uint8_t x_82; -lean_dec(x_60); -lean_dec(x_37); +lean_dec(x_40); lean_dec(x_6); -x_82 = !lean_is_exclusive(x_64); +x_82 = !lean_is_exclusive(x_70); if (x_82 == 0) { -x_18 = x_64; +x_18 = x_70; goto block_33; } else { lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_64, 0); -x_84 = lean_ctor_get(x_64, 1); +x_83 = lean_ctor_get(x_70, 0); +x_84 = lean_ctor_get(x_70, 1); lean_inc(x_84); lean_inc(x_83); -lean_dec(x_64); +lean_dec(x_70); x_85 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_85, 0, x_83); lean_ctor_set(x_85, 1, x_84); @@ -3105,22 +3096,23 @@ goto block_33; else { uint8_t x_86; -lean_dec(x_37); +lean_dec(x_63); +lean_dec(x_40); lean_dec(x_6); -x_86 = !lean_is_exclusive(x_56); +x_86 = !lean_is_exclusive(x_68); if (x_86 == 0) { -x_18 = x_56; +x_18 = x_68; goto block_33; } else { lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_56, 0); -x_88 = lean_ctor_get(x_56, 1); +x_87 = lean_ctor_get(x_68, 0); +x_88 = lean_ctor_get(x_68, 1); lean_inc(x_88); lean_inc(x_87); -lean_dec(x_56); +lean_dec(x_68); x_89 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_89, 0, x_87); lean_ctor_set(x_89, 1, x_88); @@ -3129,27 +3121,25 @@ goto block_33; } } } -} -} else { uint8_t x_90; -lean_dec(x_37); +lean_dec(x_40); lean_dec(x_6); -x_90 = !lean_is_exclusive(x_44); +x_90 = !lean_is_exclusive(x_59); if (x_90 == 0) { -x_18 = x_44; +x_18 = x_59; goto block_33; } else { lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_44, 0); -x_92 = lean_ctor_get(x_44, 1); +x_91 = lean_ctor_get(x_59, 0); +x_92 = lean_ctor_get(x_59, 1); lean_inc(x_92); lean_inc(x_91); -lean_dec(x_44); +lean_dec(x_59); x_93 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_93, 0, x_91); lean_ctor_set(x_93, 1, x_92); @@ -3158,71 +3148,101 @@ goto block_33; } } } +} +} else { -lean_object* x_94; lean_object* x_95; uint8_t x_96; -x_94 = lean_ctor_get(x_42, 0); -lean_inc(x_94); -lean_dec(x_42); -x_95 = lean_ctor_get(x_41, 1); -lean_inc(x_95); -lean_dec(x_41); -x_96 = !lean_is_exclusive(x_94); -if (x_96 == 0) +uint8_t x_94; +lean_dec(x_40); +lean_dec(x_6); +x_94 = !lean_is_exclusive(x_47); +if (x_94 == 0) { -lean_object* x_97; lean_object* x_98; uint8_t x_99; -x_97 = lean_ctor_get(x_94, 0); -x_98 = lean_ctor_get(x_94, 1); -x_99 = lean_nat_dec_lt(x_98, x_3); -if (x_99 == 0) +x_18 = x_47; +goto block_33; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_47, 0); +x_96 = lean_ctor_get(x_47, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_47); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +x_18 = x_97; +goto block_33; +} +} +} +else { -uint8_t x_100; -lean_free_object(x_94); -x_100 = lean_nat_dec_eq(x_98, x_3); +lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_98 = lean_ctor_get(x_45, 0); +lean_inc(x_98); +lean_dec(x_45); +x_99 = lean_ctor_get(x_44, 1); +lean_inc(x_99); +lean_dec(x_44); +x_100 = !lean_is_exclusive(x_98); if (x_100 == 0) { -uint8_t x_101; -x_101 = lean_nat_dec_lt(x_3, x_98); -if (x_101 == 0) +lean_object* x_101; lean_object* x_102; uint8_t x_103; +x_101 = lean_ctor_get(x_98, 0); +x_102 = lean_ctor_get(x_98, 1); +x_103 = lean_nat_dec_lt(x_102, x_3); +if (x_103 == 0) { -lean_object* x_102; lean_object* x_103; -lean_dec(x_98); -lean_dec(x_97); -lean_dec(x_37); -x_102 = lean_box(0); -x_103 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_102, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -x_18 = x_103; +uint8_t x_104; +lean_free_object(x_98); +x_104 = lean_nat_dec_eq(x_102, x_3); +if (x_104 == 0) +{ +uint8_t x_105; +x_105 = lean_nat_dec_lt(x_3, x_102); +if (x_105 == 0) +{ +lean_object* x_106; lean_object* x_107; +lean_dec(x_102); +lean_dec(x_101); +lean_dec(x_40); +x_106 = lean_box(0); +x_107 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_106, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +x_18 = x_107; goto block_33; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_104 = lean_nat_sub(x_98, x_3); -lean_dec(x_98); -x_105 = l_Lean_mkNatLit(x_104); -x_106 = l___private_Lean_Expr_0__Lean_natAddFn; -x_107 = l_Lean_mkAppB(x_106, x_97, x_105); +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_108 = lean_nat_sub(x_102, x_3); +lean_dec(x_102); +x_109 = l_Lean_mkNatLit(x_108); +x_110 = l___private_Lean_Expr_0__Lean_natAddFn; +x_111 = l_Lean_mkAppB(x_110, x_101, x_109); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); -x_108 = l_Lean_Meta_Grind_canon(x_107, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -if (lean_obj_tag(x_108) == 0) +x_112 = l_Lean_Meta_Grind_canon(x_111, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +if (lean_obj_tag(x_112) == 0) { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_109 = lean_ctor_get(x_108, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_108, 1); -lean_inc(x_110); -lean_dec(x_108); -x_111 = l_Lean_Meta_Grind_shareCommon(x_109, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_110); -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 1); +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_113 = lean_ctor_get(x_112, 0); lean_inc(x_113); -lean_dec(x_111); -x_114 = lean_unsigned_to_nat(1u); -x_115 = lean_nat_add(x_37, x_114); +x_114 = lean_ctor_get(x_112, 1); +lean_inc(x_114); +lean_dec(x_112); +x_115 = l_Lean_Meta_Grind_shareCommon(x_113, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_114); +x_116 = lean_ctor_get(x_115, 0); +lean_inc(x_116); +x_117 = lean_ctor_get(x_115, 1); +lean_inc(x_117); +lean_dec(x_115); +x_118 = lean_unsigned_to_nat(1u); +x_119 = lean_nat_add(x_40, x_118); +x_120 = lean_box(0); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3231,14 +3251,14 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_112); -x_116 = l_Lean_Meta_Grind_internalize(x_112, x_115, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_113); -if (lean_obj_tag(x_116) == 0) +lean_inc(x_116); +x_121 = l_Lean_Meta_Grind_internalize(x_116, x_119, x_120, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_117); +if (lean_obj_tag(x_121) == 0) { -lean_object* x_117; lean_object* x_118; -x_117 = lean_ctor_get(x_116, 1); -lean_inc(x_117); -lean_dec(x_116); +lean_object* x_122; lean_object* x_123; +x_122 = lean_ctor_get(x_121, 1); +lean_inc(x_122); +lean_dec(x_121); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3249,124 +3269,124 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); lean_inc(x_1); -x_118 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_112, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_117); -if (lean_obj_tag(x_118) == 0) +x_123 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_116, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_122); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_119; -x_119 = lean_ctor_get(x_118, 0); -lean_inc(x_119); -if (lean_obj_tag(x_119) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_dec(x_37); -x_120 = lean_ctor_get(x_118, 1); -lean_inc(x_120); -lean_dec(x_118); -x_121 = lean_box(0); -x_122 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_121, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_120); -x_18 = x_122; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_dec(x_40); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_126, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_125); +x_18 = x_127; goto block_33; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_123 = lean_ctor_get(x_118, 1); -lean_inc(x_123); -lean_dec(x_118); -x_124 = lean_ctor_get(x_119, 0); -lean_inc(x_124); -lean_dec(x_119); -x_125 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_124, x_37); -x_126 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_125, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_123); -x_127 = lean_ctor_get(x_126, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_126, 1); +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_128 = lean_ctor_get(x_123, 1); lean_inc(x_128); -lean_dec(x_126); -x_129 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_127, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_128); -lean_dec(x_127); -x_18 = x_129; +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_129, x_40); +x_131 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_130, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_128); +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_131, 1); +lean_inc(x_133); +lean_dec(x_131); +x_134 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_132, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_133); +lean_dec(x_132); +x_18 = x_134; goto block_33; } } else { -uint8_t x_130; -lean_dec(x_37); +uint8_t x_135; +lean_dec(x_40); lean_dec(x_6); -x_130 = !lean_is_exclusive(x_118); -if (x_130 == 0) +x_135 = !lean_is_exclusive(x_123); +if (x_135 == 0) { -x_18 = x_118; +x_18 = x_123; goto block_33; } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_131 = lean_ctor_get(x_118, 0); -x_132 = lean_ctor_get(x_118, 1); -lean_inc(x_132); -lean_inc(x_131); -lean_dec(x_118); -x_133 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_133, 0, x_131); -lean_ctor_set(x_133, 1, x_132); -x_18 = x_133; +lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_136 = lean_ctor_get(x_123, 0); +x_137 = lean_ctor_get(x_123, 1); +lean_inc(x_137); +lean_inc(x_136); +lean_dec(x_123); +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +x_18 = x_138; goto block_33; } } } else { -uint8_t x_134; -lean_dec(x_112); -lean_dec(x_37); +uint8_t x_139; +lean_dec(x_116); +lean_dec(x_40); lean_dec(x_6); -x_134 = !lean_is_exclusive(x_116); -if (x_134 == 0) +x_139 = !lean_is_exclusive(x_121); +if (x_139 == 0) { -x_18 = x_116; +x_18 = x_121; goto block_33; } else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_135 = lean_ctor_get(x_116, 0); -x_136 = lean_ctor_get(x_116, 1); -lean_inc(x_136); -lean_inc(x_135); -lean_dec(x_116); -x_137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_137, 0, x_135); -lean_ctor_set(x_137, 1, x_136); -x_18 = x_137; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_121, 0); +x_141 = lean_ctor_get(x_121, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_121); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +x_18 = x_142; goto block_33; } } } else { -uint8_t x_138; -lean_dec(x_37); +uint8_t x_143; +lean_dec(x_40); lean_dec(x_6); -x_138 = !lean_is_exclusive(x_108); -if (x_138 == 0) +x_143 = !lean_is_exclusive(x_112); +if (x_143 == 0) { -x_18 = x_108; +x_18 = x_112; goto block_33; } else { -lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_139 = lean_ctor_get(x_108, 0); -x_140 = lean_ctor_get(x_108, 1); -lean_inc(x_140); -lean_inc(x_139); -lean_dec(x_108); -x_141 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -x_18 = x_141; +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_112, 0); +x_145 = lean_ctor_get(x_112, 1); +lean_inc(x_145); +lean_inc(x_144); +lean_dec(x_112); +x_146 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_18 = x_146; goto block_33; } } @@ -3374,8 +3394,8 @@ goto block_33; } else { -lean_object* x_142; -lean_dec(x_98); +lean_object* x_147; +lean_dec(x_102); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3386,69 +3406,69 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); lean_inc(x_1); -x_142 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_97, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -if (lean_obj_tag(x_142) == 0) +x_147 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_101, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_143; -x_143 = lean_ctor_get(x_142, 0); -lean_inc(x_143); -if (lean_obj_tag(x_143) == 0) +lean_object* x_148; +x_148 = lean_ctor_get(x_147, 0); +lean_inc(x_148); +if (lean_obj_tag(x_148) == 0) { -lean_object* x_144; lean_object* x_145; lean_object* x_146; -lean_dec(x_37); -x_144 = lean_ctor_get(x_142, 1); -lean_inc(x_144); -lean_dec(x_142); -x_145 = lean_box(0); -x_146 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_145, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_144); -x_18 = x_146; +lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_40); +x_149 = lean_ctor_get(x_147, 1); +lean_inc(x_149); +lean_dec(x_147); +x_150 = lean_box(0); +x_151 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_150, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_149); +x_18 = x_151; goto block_33; } else { -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; -x_147 = lean_ctor_get(x_142, 1); -lean_inc(x_147); -lean_dec(x_142); -x_148 = lean_ctor_get(x_143, 0); -lean_inc(x_148); -lean_dec(x_143); -x_149 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_148, x_37); -x_150 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_149, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_147); -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_150, 1); +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_152 = lean_ctor_get(x_147, 1); lean_inc(x_152); -lean_dec(x_150); -x_153 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_151, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_152); -lean_dec(x_151); -x_18 = x_153; +lean_dec(x_147); +x_153 = lean_ctor_get(x_148, 0); +lean_inc(x_153); +lean_dec(x_148); +x_154 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_153, x_40); +x_155 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_154, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_152); +x_156 = lean_ctor_get(x_155, 0); +lean_inc(x_156); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +lean_dec(x_155); +x_158 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_156, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_157); +lean_dec(x_156); +x_18 = x_158; goto block_33; } } else { -uint8_t x_154; -lean_dec(x_37); +uint8_t x_159; +lean_dec(x_40); lean_dec(x_6); -x_154 = !lean_is_exclusive(x_142); -if (x_154 == 0) +x_159 = !lean_is_exclusive(x_147); +if (x_159 == 0) { -x_18 = x_142; +x_18 = x_147; goto block_33; } else { -lean_object* x_155; lean_object* x_156; lean_object* x_157; -x_155 = lean_ctor_get(x_142, 0); -x_156 = lean_ctor_get(x_142, 1); -lean_inc(x_156); -lean_inc(x_155); -lean_dec(x_142); -x_157 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_157, 0, x_155); -lean_ctor_set(x_157, 1, x_156); -x_18 = x_157; +lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_160 = lean_ctor_get(x_147, 0); +x_161 = lean_ctor_get(x_147, 1); +lean_inc(x_161); +lean_inc(x_160); +lean_dec(x_147); +x_162 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_162, 0, x_160); +lean_ctor_set(x_162, 1, x_161); +x_18 = x_162; goto block_33; } } @@ -3456,123 +3476,124 @@ goto block_33; } else { -lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; +lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_inc(x_1); -x_158 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_1, x_37); -x_159 = lean_nat_sub(x_3, x_98); -lean_dec(x_98); +x_163 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_1, x_40); +x_164 = lean_nat_sub(x_3, x_102); +lean_dec(x_102); lean_inc(x_2); -x_160 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_160, 0, x_2); -lean_ctor_set(x_160, 1, x_159); -lean_ctor_set(x_160, 2, x_97); -x_161 = !lean_is_exclusive(x_158); -if (x_161 == 0) -{ -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_162 = lean_ctor_get(x_158, 0); -lean_ctor_set_tag(x_94, 1); -lean_ctor_set(x_94, 1, x_162); -lean_ctor_set(x_94, 0, x_160); -lean_ctor_set(x_158, 0, x_94); -x_163 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_158, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -x_164 = lean_ctor_get(x_163, 0); -lean_inc(x_164); -x_165 = lean_ctor_get(x_163, 1); -lean_inc(x_165); -lean_dec(x_163); -x_166 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_164, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_165); -lean_dec(x_164); -x_18 = x_166; +x_165 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_165, 0, x_2); +lean_ctor_set(x_165, 1, x_164); +lean_ctor_set(x_165, 2, x_101); +x_166 = !lean_is_exclusive(x_163); +if (x_166 == 0) +{ +lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +x_167 = lean_ctor_get(x_163, 0); +lean_ctor_set_tag(x_98, 1); +lean_ctor_set(x_98, 1, x_167); +lean_ctor_set(x_98, 0, x_165); +lean_ctor_set(x_163, 0, x_98); +x_168 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_163, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +x_169 = lean_ctor_get(x_168, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +x_171 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_169, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_170); +lean_dec(x_169); +x_18 = x_171; goto block_33; } else { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_167 = lean_ctor_get(x_158, 0); -x_168 = lean_ctor_get(x_158, 1); -x_169 = lean_ctor_get(x_158, 2); -lean_inc(x_169); -lean_inc(x_168); -lean_inc(x_167); -lean_dec(x_158); -lean_ctor_set_tag(x_94, 1); -lean_ctor_set(x_94, 1, x_167); -lean_ctor_set(x_94, 0, x_160); -x_170 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_170, 0, x_94); -lean_ctor_set(x_170, 1, x_168); -lean_ctor_set(x_170, 2, x_169); -x_171 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_170, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_171, 1); +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_172 = lean_ctor_get(x_163, 0); +x_173 = lean_ctor_get(x_163, 1); +x_174 = lean_ctor_get(x_163, 2); +lean_inc(x_174); lean_inc(x_173); -lean_dec(x_171); -x_174 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_172, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_173); -lean_dec(x_172); -x_18 = x_174; +lean_inc(x_172); +lean_dec(x_163); +lean_ctor_set_tag(x_98, 1); +lean_ctor_set(x_98, 1, x_172); +lean_ctor_set(x_98, 0, x_165); +x_175 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_175, 0, x_98); +lean_ctor_set(x_175, 1, x_173); +lean_ctor_set(x_175, 2, x_174); +x_176 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_175, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +x_177 = lean_ctor_get(x_176, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_176, 1); +lean_inc(x_178); +lean_dec(x_176); +x_179 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_177, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_178); +lean_dec(x_177); +x_18 = x_179; goto block_33; } } } else { -lean_object* x_175; lean_object* x_176; uint8_t x_177; -x_175 = lean_ctor_get(x_94, 0); -x_176 = lean_ctor_get(x_94, 1); -lean_inc(x_176); -lean_inc(x_175); -lean_dec(x_94); -x_177 = lean_nat_dec_lt(x_176, x_3); -if (x_177 == 0) +lean_object* x_180; lean_object* x_181; uint8_t x_182; +x_180 = lean_ctor_get(x_98, 0); +x_181 = lean_ctor_get(x_98, 1); +lean_inc(x_181); +lean_inc(x_180); +lean_dec(x_98); +x_182 = lean_nat_dec_lt(x_181, x_3); +if (x_182 == 0) { -uint8_t x_178; -x_178 = lean_nat_dec_eq(x_176, x_3); -if (x_178 == 0) +uint8_t x_183; +x_183 = lean_nat_dec_eq(x_181, x_3); +if (x_183 == 0) { -uint8_t x_179; -x_179 = lean_nat_dec_lt(x_3, x_176); -if (x_179 == 0) +uint8_t x_184; +x_184 = lean_nat_dec_lt(x_3, x_181); +if (x_184 == 0) { -lean_object* x_180; lean_object* x_181; -lean_dec(x_176); -lean_dec(x_175); -lean_dec(x_37); -x_180 = lean_box(0); -x_181 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_180, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -x_18 = x_181; +lean_object* x_185; lean_object* x_186; +lean_dec(x_181); +lean_dec(x_180); +lean_dec(x_40); +x_185 = lean_box(0); +x_186 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_185, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +x_18 = x_186; goto block_33; } else { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; -x_182 = lean_nat_sub(x_176, x_3); -lean_dec(x_176); -x_183 = l_Lean_mkNatLit(x_182); -x_184 = l___private_Lean_Expr_0__Lean_natAddFn; -x_185 = l_Lean_mkAppB(x_184, x_175, x_183); +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; +x_187 = lean_nat_sub(x_181, x_3); +lean_dec(x_181); +x_188 = l_Lean_mkNatLit(x_187); +x_189 = l___private_Lean_Expr_0__Lean_natAddFn; +x_190 = l_Lean_mkAppB(x_189, x_180, x_188); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); -x_186 = l_Lean_Meta_Grind_canon(x_185, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -if (lean_obj_tag(x_186) == 0) +x_191 = l_Lean_Meta_Grind_canon(x_190, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +if (lean_obj_tag(x_191) == 0) { -lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; -x_187 = lean_ctor_get(x_186, 0); -lean_inc(x_187); -x_188 = lean_ctor_get(x_186, 1); -lean_inc(x_188); -lean_dec(x_186); -x_189 = l_Lean_Meta_Grind_shareCommon(x_187, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_188); -x_190 = lean_ctor_get(x_189, 0); -lean_inc(x_190); -x_191 = lean_ctor_get(x_189, 1); -lean_inc(x_191); -lean_dec(x_189); -x_192 = lean_unsigned_to_nat(1u); -x_193 = lean_nat_add(x_37, x_192); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_191, 0); +lean_inc(x_192); +x_193 = lean_ctor_get(x_191, 1); +lean_inc(x_193); +lean_dec(x_191); +x_194 = l_Lean_Meta_Grind_shareCommon(x_192, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_193); +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_ctor_get(x_194, 1); +lean_inc(x_196); +lean_dec(x_194); +x_197 = lean_unsigned_to_nat(1u); +x_198 = lean_nat_add(x_40, x_197); +x_199 = lean_box(0); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3581,14 +3602,14 @@ lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_190); -x_194 = l_Lean_Meta_Grind_internalize(x_190, x_193, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_191); -if (lean_obj_tag(x_194) == 0) -{ -lean_object* x_195; lean_object* x_196; -x_195 = lean_ctor_get(x_194, 1); lean_inc(x_195); -lean_dec(x_194); +x_200 = l_Lean_Meta_Grind_internalize(x_195, x_198, x_199, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_196); +if (lean_obj_tag(x_200) == 0) +{ +lean_object* x_201; lean_object* x_202; +x_201 = lean_ctor_get(x_200, 1); +lean_inc(x_201); +lean_dec(x_200); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3599,136 +3620,136 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); lean_inc(x_1); -x_196 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_190, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_195); -if (lean_obj_tag(x_196) == 0) +x_202 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_195, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_201); +if (lean_obj_tag(x_202) == 0) { -lean_object* x_197; -x_197 = lean_ctor_get(x_196, 0); -lean_inc(x_197); -if (lean_obj_tag(x_197) == 0) +lean_object* x_203; +x_203 = lean_ctor_get(x_202, 0); +lean_inc(x_203); +if (lean_obj_tag(x_203) == 0) { -lean_object* x_198; lean_object* x_199; lean_object* x_200; -lean_dec(x_37); -x_198 = lean_ctor_get(x_196, 1); -lean_inc(x_198); -lean_dec(x_196); -x_199 = lean_box(0); -x_200 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_199, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_198); -x_18 = x_200; +lean_object* x_204; lean_object* x_205; lean_object* x_206; +lean_dec(x_40); +x_204 = lean_ctor_get(x_202, 1); +lean_inc(x_204); +lean_dec(x_202); +x_205 = lean_box(0); +x_206 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_205, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_204); +x_18 = x_206; goto block_33; } else { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; -x_201 = lean_ctor_get(x_196, 1); -lean_inc(x_201); -lean_dec(x_196); -x_202 = lean_ctor_get(x_197, 0); -lean_inc(x_202); -lean_dec(x_197); -x_203 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_202, x_37); -x_204 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_203, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_201); -x_205 = lean_ctor_get(x_204, 0); -lean_inc(x_205); -x_206 = lean_ctor_get(x_204, 1); -lean_inc(x_206); -lean_dec(x_204); -x_207 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_205, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_206); -lean_dec(x_205); -x_18 = x_207; +lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_207 = lean_ctor_get(x_202, 1); +lean_inc(x_207); +lean_dec(x_202); +x_208 = lean_ctor_get(x_203, 0); +lean_inc(x_208); +lean_dec(x_203); +x_209 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_208, x_40); +x_210 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_209, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_207); +x_211 = lean_ctor_get(x_210, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_210, 1); +lean_inc(x_212); +lean_dec(x_210); +x_213 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_211, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_212); +lean_dec(x_211); +x_18 = x_213; goto block_33; } } else { -lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; -lean_dec(x_37); +lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; +lean_dec(x_40); lean_dec(x_6); -x_208 = lean_ctor_get(x_196, 0); -lean_inc(x_208); -x_209 = lean_ctor_get(x_196, 1); -lean_inc(x_209); -if (lean_is_exclusive(x_196)) { - lean_ctor_release(x_196, 0); - lean_ctor_release(x_196, 1); - x_210 = x_196; +x_214 = lean_ctor_get(x_202, 0); +lean_inc(x_214); +x_215 = lean_ctor_get(x_202, 1); +lean_inc(x_215); +if (lean_is_exclusive(x_202)) { + lean_ctor_release(x_202, 0); + lean_ctor_release(x_202, 1); + x_216 = x_202; } else { - lean_dec_ref(x_196); - x_210 = lean_box(0); + lean_dec_ref(x_202); + x_216 = lean_box(0); } -if (lean_is_scalar(x_210)) { - x_211 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_216)) { + x_217 = lean_alloc_ctor(1, 2, 0); } else { - x_211 = x_210; + x_217 = x_216; } -lean_ctor_set(x_211, 0, x_208); -lean_ctor_set(x_211, 1, x_209); -x_18 = x_211; +lean_ctor_set(x_217, 0, x_214); +lean_ctor_set(x_217, 1, x_215); +x_18 = x_217; goto block_33; } } else { -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; -lean_dec(x_190); -lean_dec(x_37); +lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +lean_dec(x_195); +lean_dec(x_40); lean_dec(x_6); -x_212 = lean_ctor_get(x_194, 0); -lean_inc(x_212); -x_213 = lean_ctor_get(x_194, 1); -lean_inc(x_213); -if (lean_is_exclusive(x_194)) { - lean_ctor_release(x_194, 0); - lean_ctor_release(x_194, 1); - x_214 = x_194; +x_218 = lean_ctor_get(x_200, 0); +lean_inc(x_218); +x_219 = lean_ctor_get(x_200, 1); +lean_inc(x_219); +if (lean_is_exclusive(x_200)) { + lean_ctor_release(x_200, 0); + lean_ctor_release(x_200, 1); + x_220 = x_200; } else { - lean_dec_ref(x_194); - x_214 = lean_box(0); + lean_dec_ref(x_200); + x_220 = lean_box(0); } -if (lean_is_scalar(x_214)) { - x_215 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_220)) { + x_221 = lean_alloc_ctor(1, 2, 0); } else { - x_215 = x_214; + x_221 = x_220; } -lean_ctor_set(x_215, 0, x_212); -lean_ctor_set(x_215, 1, x_213); -x_18 = x_215; +lean_ctor_set(x_221, 0, x_218); +lean_ctor_set(x_221, 1, x_219); +x_18 = x_221; goto block_33; } } else { -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; -lean_dec(x_37); +lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; +lean_dec(x_40); lean_dec(x_6); -x_216 = lean_ctor_get(x_186, 0); -lean_inc(x_216); -x_217 = lean_ctor_get(x_186, 1); -lean_inc(x_217); -if (lean_is_exclusive(x_186)) { - lean_ctor_release(x_186, 0); - lean_ctor_release(x_186, 1); - x_218 = x_186; +x_222 = lean_ctor_get(x_191, 0); +lean_inc(x_222); +x_223 = lean_ctor_get(x_191, 1); +lean_inc(x_223); +if (lean_is_exclusive(x_191)) { + lean_ctor_release(x_191, 0); + lean_ctor_release(x_191, 1); + x_224 = x_191; } else { - lean_dec_ref(x_186); - x_218 = lean_box(0); + lean_dec_ref(x_191); + x_224 = lean_box(0); } -if (lean_is_scalar(x_218)) { - x_219 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_224)) { + x_225 = lean_alloc_ctor(1, 2, 0); } else { - x_219 = x_218; + x_225 = x_224; } -lean_ctor_set(x_219, 0, x_216); -lean_ctor_set(x_219, 1, x_217); -x_18 = x_219; +lean_ctor_set(x_225, 0, x_222); +lean_ctor_set(x_225, 1, x_223); +x_18 = x_225; goto block_33; } } } else { -lean_object* x_220; -lean_dec(x_176); +lean_object* x_226; +lean_dec(x_181); lean_inc(x_16); lean_inc(x_15); lean_inc(x_14); @@ -3739,122 +3760,122 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_2); lean_inc(x_1); -x_220 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_175, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -if (lean_obj_tag(x_220) == 0) +x_226 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArg_x3f(x_1, x_2, x_180, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +if (lean_obj_tag(x_226) == 0) { -lean_object* x_221; -x_221 = lean_ctor_get(x_220, 0); -lean_inc(x_221); -if (lean_obj_tag(x_221) == 0) +lean_object* x_227; +x_227 = lean_ctor_get(x_226, 0); +lean_inc(x_227); +if (lean_obj_tag(x_227) == 0) { -lean_object* x_222; lean_object* x_223; lean_object* x_224; -lean_dec(x_37); -x_222 = lean_ctor_get(x_220, 1); -lean_inc(x_222); -lean_dec(x_220); -x_223 = lean_box(0); -x_224 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_223, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_222); -x_18 = x_224; +lean_object* x_228; lean_object* x_229; lean_object* x_230; +lean_dec(x_40); +x_228 = lean_ctor_get(x_226, 1); +lean_inc(x_228); +lean_dec(x_226); +x_229 = lean_box(0); +x_230 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_229, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_228); +x_18 = x_230; goto block_33; } else { -lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_225 = lean_ctor_get(x_220, 1); -lean_inc(x_225); -lean_dec(x_220); -x_226 = lean_ctor_get(x_221, 0); -lean_inc(x_226); -lean_dec(x_221); -x_227 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_226, x_37); -x_228 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_227, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_225); -x_229 = lean_ctor_get(x_228, 0); -lean_inc(x_229); -x_230 = lean_ctor_get(x_228, 1); -lean_inc(x_230); -lean_dec(x_228); -x_231 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_229, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_230); -lean_dec(x_229); -x_18 = x_231; +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; +x_231 = lean_ctor_get(x_226, 1); +lean_inc(x_231); +lean_dec(x_226); +x_232 = lean_ctor_get(x_227, 0); +lean_inc(x_232); +lean_dec(x_227); +x_233 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_232, x_40); +x_234 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_233, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_231); +x_235 = lean_ctor_get(x_234, 0); +lean_inc(x_235); +x_236 = lean_ctor_get(x_234, 1); +lean_inc(x_236); +lean_dec(x_234); +x_237 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_235, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_236); +lean_dec(x_235); +x_18 = x_237; goto block_33; } } else { -lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; -lean_dec(x_37); +lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +lean_dec(x_40); lean_dec(x_6); -x_232 = lean_ctor_get(x_220, 0); -lean_inc(x_232); -x_233 = lean_ctor_get(x_220, 1); -lean_inc(x_233); -if (lean_is_exclusive(x_220)) { - lean_ctor_release(x_220, 0); - lean_ctor_release(x_220, 1); - x_234 = x_220; +x_238 = lean_ctor_get(x_226, 0); +lean_inc(x_238); +x_239 = lean_ctor_get(x_226, 1); +lean_inc(x_239); +if (lean_is_exclusive(x_226)) { + lean_ctor_release(x_226, 0); + lean_ctor_release(x_226, 1); + x_240 = x_226; } else { - lean_dec_ref(x_220); - x_234 = lean_box(0); + lean_dec_ref(x_226); + x_240 = lean_box(0); } -if (lean_is_scalar(x_234)) { - x_235 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_240)) { + x_241 = lean_alloc_ctor(1, 2, 0); } else { - x_235 = x_234; + x_241 = x_240; } -lean_ctor_set(x_235, 0, x_232); -lean_ctor_set(x_235, 1, x_233); -x_18 = x_235; +lean_ctor_set(x_241, 0, x_238); +lean_ctor_set(x_241, 1, x_239); +x_18 = x_241; goto block_33; } } } else { -lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_inc(x_1); -x_236 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_1, x_37); -x_237 = lean_nat_sub(x_3, x_176); -lean_dec(x_176); +x_242 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_Choice_updateGen(x_1, x_40); +x_243 = lean_nat_sub(x_3, x_181); +lean_dec(x_181); lean_inc(x_2); -x_238 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_238, 0, x_2); -lean_ctor_set(x_238, 1, x_237); -lean_ctor_set(x_238, 2, x_175); -x_239 = lean_ctor_get(x_236, 0); -lean_inc(x_239); -x_240 = lean_ctor_get(x_236, 1); -lean_inc(x_240); -x_241 = lean_ctor_get(x_236, 2); -lean_inc(x_241); -if (lean_is_exclusive(x_236)) { - lean_ctor_release(x_236, 0); - lean_ctor_release(x_236, 1); - lean_ctor_release(x_236, 2); - x_242 = x_236; -} else { - lean_dec_ref(x_236); - x_242 = lean_box(0); -} -x_243 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_243, 0, x_238); -lean_ctor_set(x_243, 1, x_239); -if (lean_is_scalar(x_242)) { - x_244 = lean_alloc_ctor(0, 3, 0); -} else { - x_244 = x_242; -} -lean_ctor_set(x_244, 0, x_243); -lean_ctor_set(x_244, 1, x_240); -lean_ctor_set(x_244, 2, x_241); -x_245 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_244, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_95); -x_246 = lean_ctor_get(x_245, 0); +x_244 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_244, 0, x_2); +lean_ctor_set(x_244, 1, x_243); +lean_ctor_set(x_244, 2, x_180); +x_245 = lean_ctor_get(x_242, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_242, 1); lean_inc(x_246); -x_247 = lean_ctor_get(x_245, 1); +x_247 = lean_ctor_get(x_242, 2); lean_inc(x_247); -lean_dec(x_245); -x_248 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_246, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_247); -lean_dec(x_246); -x_18 = x_248; +if (lean_is_exclusive(x_242)) { + lean_ctor_release(x_242, 0); + lean_ctor_release(x_242, 1); + lean_ctor_release(x_242, 2); + x_248 = x_242; +} else { + lean_dec_ref(x_242); + x_248 = lean_box(0); +} +x_249 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_249, 0, x_244); +lean_ctor_set(x_249, 1, x_245); +if (lean_is_scalar(x_248)) { + x_250 = lean_alloc_ctor(0, 3, 0); +} else { + x_250 = x_248; +} +lean_ctor_set(x_250, 0, x_249); +lean_ctor_set(x_250, 1, x_246); +lean_ctor_set(x_250, 2, x_247); +x_251 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_pushChoice(x_250, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_99); +x_252 = lean_ctor_get(x_251, 0); +lean_inc(x_252); +x_253 = lean_ctor_get(x_251, 1); +lean_inc(x_253); +lean_dec(x_251); +x_254 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processMatch___spec__1___lambda__1(x_4, x_6, x_252, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_253); +lean_dec(x_252); +x_18 = x_254; goto block_33; } } @@ -3862,27 +3883,27 @@ goto block_33; } else { -uint8_t x_249; -lean_dec(x_37); +uint8_t x_255; +lean_dec(x_40); lean_dec(x_6); -x_249 = !lean_is_exclusive(x_41); -if (x_249 == 0) +x_255 = !lean_is_exclusive(x_44); +if (x_255 == 0) { -x_18 = x_41; +x_18 = x_44; goto block_33; } else { -lean_object* x_250; lean_object* x_251; lean_object* x_252; -x_250 = lean_ctor_get(x_41, 0); -x_251 = lean_ctor_get(x_41, 1); -lean_inc(x_251); -lean_inc(x_250); -lean_dec(x_41); -x_252 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_252, 0, x_250); -lean_ctor_set(x_252, 1, x_251); -x_18 = x_252; +lean_object* x_256; lean_object* x_257; lean_object* x_258; +x_256 = lean_ctor_get(x_44, 0); +x_257 = lean_ctor_get(x_44, 1); +lean_inc(x_257); +lean_inc(x_256); +lean_dec(x_44); +x_258 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_258, 0, x_256); +lean_ctor_set(x_258, 1, x_257); +x_18 = x_258; goto block_33; } } @@ -3890,26 +3911,26 @@ goto block_33; } else { -uint8_t x_253; +uint8_t x_259; lean_dec(x_6); -x_253 = !lean_is_exclusive(x_34); -if (x_253 == 0) +x_259 = !lean_is_exclusive(x_37); +if (x_259 == 0) { -x_18 = x_34; +x_18 = x_37; goto block_33; } else { -lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_254 = lean_ctor_get(x_34, 0); -x_255 = lean_ctor_get(x_34, 1); -lean_inc(x_255); -lean_inc(x_254); -lean_dec(x_34); -x_256 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_256, 0, x_254); -lean_ctor_set(x_256, 1, x_255); -x_18 = x_256; +lean_object* x_260; lean_object* x_261; lean_object* x_262; +x_260 = lean_ctor_get(x_37, 0); +x_261 = lean_ctor_get(x_37, 1); +lean_inc(x_261); +lean_inc(x_260); +lean_dec(x_37); +x_262 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_262, 0, x_260); +lean_ctor_set(x_262, 1, x_261); +x_18 = x_262; goto block_33; } } @@ -4146,7 +4167,7 @@ return x_21; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_30; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_dec(x_8); x_22 = lean_ctor_get(x_7, 0); lean_inc(x_22); @@ -4160,72 +4181,78 @@ if (lean_is_exclusive(x_7)) { lean_dec_ref(x_7); x_24 = lean_box(0); } -lean_inc(x_22); -x_30 = l_Lean_Meta_Grind_getENode(x_22, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_83; +x_30 = lean_st_ref_get(x_12, x_20); x_31 = lean_ctor_get(x_30, 0); lean_inc(x_31); x_32 = lean_ctor_get(x_30, 1); lean_inc(x_32); lean_dec(x_30); -x_33 = lean_ctor_get(x_31, 8); -lean_inc(x_33); -x_83 = lean_nat_dec_lt(x_33, x_4); -if (x_83 == 0) +lean_inc(x_22); +x_33 = l_Lean_Meta_Grind_Goal_getENode(x_31, x_22, x_18, x_19, x_32); +if (lean_obj_tag(x_33) == 0) { -lean_object* x_84; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_86; +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); lean_dec(x_33); -lean_dec(x_31); +x_36 = lean_ctor_get(x_34, 8); +lean_inc(x_36); +x_86 = lean_nat_dec_lt(x_36, x_4); +if (x_86 == 0) +{ +lean_object* x_87; +lean_dec(x_36); +lean_dec(x_34); lean_dec(x_24); lean_dec(x_22); -x_84 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_84; -x_26 = x_32; +x_87 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_87; +x_26 = x_35; goto block_29; } else { -uint8_t x_85; -x_85 = lean_ctor_get_uint8(x_31, sizeof(void*)*10 + 4); -if (x_85 == 0) +uint8_t x_88; +x_88 = lean_ctor_get_uint8(x_34, sizeof(void*)*11 + 4); +if (x_88 == 0) { -uint8_t x_86; -x_86 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_31); -lean_dec(x_31); -if (x_86 == 0) +uint8_t x_89; +x_89 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_34); +lean_dec(x_34); +if (x_89 == 0) { -lean_object* x_87; -lean_dec(x_33); +lean_object* x_90; +lean_dec(x_36); lean_dec(x_24); lean_dec(x_22); -x_87 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_87; -x_26 = x_32; +x_90 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_90; +x_26 = x_35; goto block_29; } else { -lean_object* x_88; -x_88 = lean_box(0); -x_34 = x_88; -goto block_82; +lean_object* x_91; +x_91 = lean_box(0); +x_37 = x_91; +goto block_85; } } else { -lean_object* x_89; -lean_dec(x_31); -x_89 = lean_box(0); -x_34 = x_89; -goto block_82; +lean_object* x_92; +lean_dec(x_34); +x_92 = lean_box(0); +x_37 = x_92; +goto block_85; } } -block_82: +block_85: { -lean_object* x_35; -lean_dec(x_34); +lean_object* x_38; +lean_dec(x_37); lean_inc(x_19); lean_inc(x_18); lean_inc(x_17); @@ -4235,164 +4262,164 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_1); -x_35 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_1, x_2, x_22, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_32); +x_38 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_1, x_2, x_22, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_35); lean_dec(x_22); -if (lean_obj_tag(x_35) == 0) +if (lean_obj_tag(x_38) == 0) { -lean_object* x_36; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -if (lean_obj_tag(x_36) == 0) +lean_object* x_39; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_37; lean_object* x_38; -lean_dec(x_33); +lean_object* x_40; lean_object* x_41; +lean_dec(x_36); lean_dec(x_24); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_38; -x_26 = x_37; +x_40 = lean_ctor_get(x_38, 1); +lean_inc(x_40); +lean_dec(x_38); +x_41 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_41; +x_26 = x_40; goto block_29; } else { -lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_39 = lean_ctor_get(x_36, 0); -lean_inc(x_39); -lean_dec(x_36); -x_40 = lean_ctor_get(x_35, 1); -lean_inc(x_40); -lean_dec(x_35); -x_41 = !lean_is_exclusive(x_39); -if (x_41 == 0) +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = lean_ctor_get(x_39, 0); +lean_inc(x_42); +lean_dec(x_39); +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_dec(x_38); +x_44 = !lean_is_exclusive(x_42); +if (x_44 == 0) { -lean_object* x_42; uint8_t x_43; -x_42 = lean_ctor_get(x_39, 1); -x_43 = lean_nat_dec_le(x_33, x_42); -if (x_43 == 0) +lean_object* x_45; uint8_t x_46; +x_45 = lean_ctor_get(x_42, 1); +x_46 = lean_nat_dec_le(x_36, x_45); +if (x_46 == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -lean_dec(x_42); -lean_ctor_set(x_39, 1, x_33); -x_44 = lean_st_ref_take(x_11, x_40); -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +lean_dec(x_45); +lean_ctor_set(x_42, 1, x_36); +x_47 = lean_st_ref_take(x_11, x_43); +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); if (lean_is_scalar(x_24)) { - x_47 = lean_alloc_ctor(1, 2, 0); + x_50 = lean_alloc_ctor(1, 2, 0); } else { - x_47 = x_24; + x_50 = x_24; } -lean_ctor_set(x_47, 0, x_39); -lean_ctor_set(x_47, 1, x_45); -x_48 = lean_st_ref_set(x_11, x_47, x_46); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -lean_dec(x_48); -x_50 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_50; -x_26 = x_49; +lean_ctor_set(x_50, 0, x_42); +lean_ctor_set(x_50, 1, x_48); +x_51 = lean_st_ref_set(x_11, x_50, x_49); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +lean_dec(x_51); +x_53 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_53; +x_26 = x_52; goto block_29; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -lean_dec(x_33); -x_51 = lean_st_ref_take(x_11, x_40); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +lean_dec(x_36); +x_54 = lean_st_ref_take(x_11, x_43); +x_55 = lean_ctor_get(x_54, 0); +lean_inc(x_55); +x_56 = lean_ctor_get(x_54, 1); +lean_inc(x_56); +lean_dec(x_54); if (lean_is_scalar(x_24)) { - x_54 = lean_alloc_ctor(1, 2, 0); + x_57 = lean_alloc_ctor(1, 2, 0); } else { - x_54 = x_24; + x_57 = x_24; } -lean_ctor_set(x_54, 0, x_39); -lean_ctor_set(x_54, 1, x_52); -x_55 = lean_st_ref_set(x_11, x_54, x_53); -x_56 = lean_ctor_get(x_55, 1); -lean_inc(x_56); -lean_dec(x_55); -x_57 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_57; -x_26 = x_56; +lean_ctor_set(x_57, 0, x_42); +lean_ctor_set(x_57, 1, x_55); +x_58 = lean_st_ref_set(x_11, x_57, x_56); +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +lean_dec(x_58); +x_60 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_60; +x_26 = x_59; goto block_29; } } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_58 = lean_ctor_get(x_39, 0); -x_59 = lean_ctor_get(x_39, 1); -x_60 = lean_ctor_get(x_39, 2); -lean_inc(x_60); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_39); -x_61 = lean_nat_dec_le(x_33, x_59); -if (x_61 == 0) +lean_object* x_61; lean_object* x_62; lean_object* x_63; uint8_t x_64; +x_61 = lean_ctor_get(x_42, 0); +x_62 = lean_ctor_get(x_42, 1); +x_63 = lean_ctor_get(x_42, 2); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_42); +x_64 = lean_nat_dec_le(x_36, x_62); +if (x_64 == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -lean_dec(x_59); -x_62 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_62, 0, x_58); -lean_ctor_set(x_62, 1, x_33); -lean_ctor_set(x_62, 2, x_60); -x_63 = lean_st_ref_take(x_11, x_40); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; +lean_dec(x_62); +x_65 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_65, 0, x_61); +lean_ctor_set(x_65, 1, x_36); +lean_ctor_set(x_65, 2, x_63); +x_66 = lean_st_ref_take(x_11, x_43); +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +lean_dec(x_66); if (lean_is_scalar(x_24)) { - x_66 = lean_alloc_ctor(1, 2, 0); + x_69 = lean_alloc_ctor(1, 2, 0); } else { - x_66 = x_24; + x_69 = x_24; } -lean_ctor_set(x_66, 0, x_62); -lean_ctor_set(x_66, 1, x_64); -x_67 = lean_st_ref_set(x_11, x_66, x_65); -x_68 = lean_ctor_get(x_67, 1); -lean_inc(x_68); -lean_dec(x_67); -x_69 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_69; -x_26 = x_68; +lean_ctor_set(x_69, 0, x_65); +lean_ctor_set(x_69, 1, x_67); +x_70 = lean_st_ref_set(x_11, x_69, x_68); +x_71 = lean_ctor_get(x_70, 1); +lean_inc(x_71); +lean_dec(x_70); +x_72 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_72; +x_26 = x_71; goto block_29; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -lean_dec(x_33); -x_70 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_70, 0, x_58); -lean_ctor_set(x_70, 1, x_59); -lean_ctor_set(x_70, 2, x_60); -x_71 = lean_st_ref_take(x_11, x_40); -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -lean_dec(x_71); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_dec(x_36); +x_73 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_73, 0, x_61); +lean_ctor_set(x_73, 1, x_62); +lean_ctor_set(x_73, 2, x_63); +x_74 = lean_st_ref_take(x_11, x_43); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); if (lean_is_scalar(x_24)) { - x_74 = lean_alloc_ctor(1, 2, 0); + x_77 = lean_alloc_ctor(1, 2, 0); } else { - x_74 = x_24; + x_77 = x_24; } -lean_ctor_set(x_74, 0, x_70); -lean_ctor_set(x_74, 1, x_72); -x_75 = lean_st_ref_set(x_11, x_74, x_73); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_77 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; -x_25 = x_77; -x_26 = x_76; +lean_ctor_set(x_77, 0, x_73); +lean_ctor_set(x_77, 1, x_75); +x_78 = lean_st_ref_set(x_11, x_77, x_76); +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processContinue___spec__1___closed__1; +x_25 = x_80; +x_26 = x_79; goto block_29; } } @@ -4400,8 +4427,8 @@ goto block_29; } else { -uint8_t x_78; -lean_dec(x_33); +uint8_t x_81; +lean_dec(x_36); lean_dec(x_24); lean_dec(x_23); lean_dec(x_19); @@ -4413,30 +4440,30 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_1); -x_78 = !lean_is_exclusive(x_35); -if (x_78 == 0) +x_81 = !lean_is_exclusive(x_38); +if (x_81 == 0) { -return x_35; +return x_38; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_35, 0); -x_80 = lean_ctor_get(x_35, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_35); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -return x_81; +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_38, 0); +x_83 = lean_ctor_get(x_38, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_38); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; } } } } else { -uint8_t x_90; +uint8_t x_93; lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); @@ -4449,23 +4476,23 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_1); -x_90 = !lean_is_exclusive(x_30); -if (x_90 == 0) +x_93 = !lean_is_exclusive(x_33); +if (x_93 == 0) { -return x_30; +return x_33; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_91 = lean_ctor_get(x_30, 0); -x_92 = lean_ctor_get(x_30, 1); -lean_inc(x_92); -lean_inc(x_91); -lean_dec(x_30); -x_93 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_93, 0, x_91); -lean_ctor_set(x_93, 1, x_92); -return x_93; +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_33, 0); +x_95 = lean_ctor_get(x_33, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_33); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +return x_96; } } block_29: @@ -4494,7 +4521,7 @@ if (x_15 == 0) lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_16, 4); +x_18 = lean_ctor_get(x_16, 5); lean_inc(x_18); lean_dec(x_16); lean_inc(x_2); @@ -4594,7 +4621,7 @@ x_38 = lean_ctor_get(x_14, 1); lean_inc(x_38); lean_inc(x_37); lean_dec(x_14); -x_39 = lean_ctor_get(x_37, 4); +x_39 = lean_ctor_get(x_37, 5); lean_inc(x_39); lean_dec(x_37); lean_inc(x_2); @@ -15848,27 +15875,33 @@ return x_15; LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_main___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19) { _start: { -lean_object* x_20; +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_20 = lean_st_ref_get(x_11, x_19); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); lean_inc(x_1); -x_20 = l_Lean_Meta_Grind_getENode(x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19); -if (lean_obj_tag(x_20) == 0) +x_23 = l_Lean_Meta_Grind_Goal_getENode(x_21, x_1, x_17, x_18, x_22); +if (lean_obj_tag(x_23) == 0) { -uint8_t x_21; -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_123; -x_22 = lean_ctor_get(x_20, 0); -x_23 = lean_ctor_get(x_20, 1); -x_123 = lean_ctor_get_uint8(x_22, sizeof(void*)*10 + 4); -if (x_123 == 0) +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_126; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +x_126 = lean_ctor_get_uint8(x_25, sizeof(void*)*11 + 4); +if (x_126 == 0) { -uint8_t x_124; -x_124 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_22); -if (x_124 == 0) +uint8_t x_127; +x_127 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_25); +if (x_127 == 0) { -lean_object* x_125; -lean_dec(x_22); +lean_object* x_128; +lean_dec(x_25); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -15882,32 +15915,32 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_125 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_125, 0, x_5); -lean_ctor_set(x_20, 0, x_125); -return x_20; +x_128 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_128, 0, x_5); +lean_ctor_set(x_23, 0, x_128); +return x_23; } else { if (x_6 == 0) { -lean_object* x_126; -lean_free_object(x_20); -x_126 = lean_box(0); -x_24 = x_126; -goto block_122; +lean_object* x_129; +lean_free_object(x_23); +x_129 = lean_box(0); +x_27 = x_129; +goto block_125; } else { -lean_object* x_127; uint8_t x_128; -x_127 = lean_ctor_get(x_22, 9); -lean_inc(x_127); -x_128 = lean_nat_dec_eq(x_127, x_7); -lean_dec(x_127); -if (x_128 == 0) +lean_object* x_130; uint8_t x_131; +x_130 = lean_ctor_get(x_25, 9); +lean_inc(x_130); +x_131 = lean_nat_dec_eq(x_130, x_7); +lean_dec(x_130); +if (x_131 == 0) { -lean_object* x_129; -lean_dec(x_22); +lean_object* x_132; +lean_dec(x_25); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -15921,18 +15954,18 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_129 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_129, 0, x_5); -lean_ctor_set(x_20, 0, x_129); -return x_20; +x_132 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_132, 0, x_5); +lean_ctor_set(x_23, 0, x_132); +return x_23; } else { -lean_object* x_130; -lean_free_object(x_20); -x_130 = lean_box(0); -x_24 = x_130; -goto block_122; +lean_object* x_133; +lean_free_object(x_23); +x_133 = lean_box(0); +x_27 = x_133; +goto block_125; } } } @@ -15941,23 +15974,23 @@ else { if (x_6 == 0) { -lean_object* x_131; -lean_free_object(x_20); -x_131 = lean_box(0); -x_24 = x_131; -goto block_122; +lean_object* x_134; +lean_free_object(x_23); +x_134 = lean_box(0); +x_27 = x_134; +goto block_125; } else { -lean_object* x_132; uint8_t x_133; -x_132 = lean_ctor_get(x_22, 9); -lean_inc(x_132); -x_133 = lean_nat_dec_eq(x_132, x_7); -lean_dec(x_132); -if (x_133 == 0) +lean_object* x_135; uint8_t x_136; +x_135 = lean_ctor_get(x_25, 9); +lean_inc(x_135); +x_136 = lean_nat_dec_eq(x_135, x_7); +lean_dec(x_135); +if (x_136 == 0) { -lean_object* x_134; -lean_dec(x_22); +lean_object* x_137; +lean_dec(x_25); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -15971,38 +16004,38 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_134 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_134, 0, x_5); -lean_ctor_set(x_20, 0, x_134); -return x_20; +x_137 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_137, 0, x_5); +lean_ctor_set(x_23, 0, x_137); +return x_23; } else { -lean_object* x_135; -lean_free_object(x_20); -x_135 = lean_box(0); -x_24 = x_135; -goto block_122; +lean_object* x_138; +lean_free_object(x_23); +x_138 = lean_box(0); +x_27 = x_138; +goto block_125; } } } -block_122: +block_125: { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -lean_dec(x_24); -x_25 = lean_ctor_get(x_22, 8); -lean_inc(x_25); -lean_dec(x_22); -x_26 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_26, 0, x_2); -lean_ctor_set(x_26, 1, x_25); -lean_ctor_set(x_26, 2, x_3); -x_27 = !lean_is_exclusive(x_9); -if (x_27 == 0) +lean_object* x_28; lean_object* x_29; uint8_t x_30; +lean_dec(x_27); +x_28 = lean_ctor_get(x_25, 8); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_29, 0, x_2); +lean_ctor_set(x_29, 1, x_28); +lean_ctor_set(x_29, 2, x_3); +x_30 = !lean_is_exclusive(x_9); +if (x_30 == 0) { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_9, 1); -lean_dec(x_28); +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_9, 1); +lean_dec(x_31); lean_inc(x_1); lean_ctor_set(x_9, 1, x_1); lean_inc(x_18); @@ -16013,16 +16046,16 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_29 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_26, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_23); +x_32 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_29, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_26); lean_dec(x_1); -if (lean_obj_tag(x_29) == 0) +if (lean_obj_tag(x_32) == 0) { -lean_object* x_30; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -if (lean_obj_tag(x_30) == 0) +lean_object* x_33; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +if (lean_obj_tag(x_33) == 0) { -uint8_t x_31; +uint8_t x_34; lean_dec(x_9); lean_dec(x_18); lean_dec(x_17); @@ -16033,262 +16066,262 @@ lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_31 = !lean_is_exclusive(x_29); -if (x_31 == 0) +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_33, 0, x_5); -lean_ctor_set(x_29, 0, x_33); -return x_29; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_32, 0); +lean_dec(x_35); +x_36 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_36, 0, x_5); +lean_ctor_set(x_32, 0, x_36); +return x_32; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_29, 1); -lean_inc(x_34); -lean_dec(x_29); -x_35 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_35, 0, x_5); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -return x_36; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_32, 1); +lean_inc(x_37); +lean_dec(x_32); +x_38 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_38, 0, x_5); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +return x_39; } } else { -lean_object* x_37; uint8_t x_38; -x_37 = lean_ctor_get(x_29, 1); -lean_inc(x_37); -lean_dec(x_29); -x_38 = !lean_is_exclusive(x_30); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; uint8_t x_41; -x_39 = lean_ctor_get(x_30, 0); -x_40 = lean_st_ref_take(x_10, x_37); -x_41 = !lean_is_exclusive(x_40); +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_32, 1); +lean_inc(x_40); +lean_dec(x_32); +x_41 = !lean_is_exclusive(x_33); if (x_41 == 0) { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_42 = lean_ctor_get(x_40, 1); -x_43 = lean_ctor_get(x_40, 0); -lean_dec(x_43); -x_44 = lean_box(0); -lean_ctor_set_tag(x_40, 1); -lean_ctor_set(x_40, 1, x_44); -lean_ctor_set(x_40, 0, x_39); -x_45 = lean_st_ref_set(x_10, x_40, x_42); -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -lean_dec(x_45); -x_47 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_46); -if (lean_obj_tag(x_47) == 0) +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = lean_ctor_get(x_33, 0); +x_43 = lean_st_ref_take(x_10, x_40); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_45 = lean_ctor_get(x_43, 1); +x_46 = lean_ctor_get(x_43, 0); +lean_dec(x_46); +x_47 = lean_box(0); +lean_ctor_set_tag(x_43, 1); +lean_ctor_set(x_43, 1, x_47); +lean_ctor_set(x_43, 0, x_42); +x_48 = lean_st_ref_set(x_10, x_43, x_45); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_49); +if (lean_obj_tag(x_50) == 0) { -uint8_t x_48; -x_48 = !lean_is_exclusive(x_47); -if (x_48 == 0) +uint8_t x_51; +x_51 = !lean_is_exclusive(x_50); +if (x_51 == 0) { -lean_object* x_49; -x_49 = lean_ctor_get(x_47, 0); -lean_dec(x_49); -lean_ctor_set(x_30, 0, x_5); -lean_ctor_set(x_47, 0, x_30); -return x_47; +lean_object* x_52; +x_52 = lean_ctor_get(x_50, 0); +lean_dec(x_52); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_50, 0, x_33); +return x_50; } else { -lean_object* x_50; lean_object* x_51; -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_dec(x_47); -lean_ctor_set(x_30, 0, x_5); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_30); -lean_ctor_set(x_51, 1, x_50); -return x_51; +lean_object* x_53; lean_object* x_54; +x_53 = lean_ctor_get(x_50, 1); +lean_inc(x_53); +lean_dec(x_50); +lean_ctor_set(x_33, 0, x_5); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_33); +lean_ctor_set(x_54, 1, x_53); +return x_54; } } else { -uint8_t x_52; -lean_free_object(x_30); +uint8_t x_55; +lean_free_object(x_33); lean_dec(x_5); -x_52 = !lean_is_exclusive(x_47); -if (x_52 == 0) +x_55 = !lean_is_exclusive(x_50); +if (x_55 == 0) { -return x_47; +return x_50; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_47, 0); -x_54 = lean_ctor_get(x_47, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_47); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_50, 0); +x_57 = lean_ctor_get(x_50, 1); +lean_inc(x_57); +lean_inc(x_56); +lean_dec(x_50); +x_58 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +return x_58; } } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_56 = lean_ctor_get(x_40, 1); -lean_inc(x_56); -lean_dec(x_40); -x_57 = lean_box(0); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_39); -lean_ctor_set(x_58, 1, x_57); -x_59 = lean_st_ref_set(x_10, x_58, x_56); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_60); -if (lean_obj_tag(x_61) == 0) +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_59 = lean_ctor_get(x_43, 1); +lean_inc(x_59); +lean_dec(x_43); +x_60 = lean_box(0); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_42); +lean_ctor_set(x_61, 1, x_60); +x_62 = lean_st_ref_set(x_10, x_61, x_59); +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +lean_dec(x_62); +x_64 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_63); +if (lean_obj_tag(x_64) == 0) { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_63 = x_61; +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_64, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_66 = x_64; } else { - lean_dec_ref(x_61); - x_63 = lean_box(0); + lean_dec_ref(x_64); + x_66 = lean_box(0); } -lean_ctor_set(x_30, 0, x_5); -if (lean_is_scalar(x_63)) { - x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_5); +if (lean_is_scalar(x_66)) { + x_67 = lean_alloc_ctor(0, 2, 0); } else { - x_64 = x_63; + x_67 = x_66; } -lean_ctor_set(x_64, 0, x_30); -lean_ctor_set(x_64, 1, x_62); -return x_64; +lean_ctor_set(x_67, 0, x_33); +lean_ctor_set(x_67, 1, x_65); +return x_67; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -lean_free_object(x_30); +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_free_object(x_33); lean_dec(x_5); -x_65 = lean_ctor_get(x_61, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_61, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_67 = x_61; +x_68 = lean_ctor_get(x_64, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_64, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_64)) { + lean_ctor_release(x_64, 0); + lean_ctor_release(x_64, 1); + x_70 = x_64; } else { - lean_dec_ref(x_61); - x_67 = lean_box(0); + lean_dec_ref(x_64); + x_70 = lean_box(0); } -if (lean_is_scalar(x_67)) { - x_68 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_70)) { + x_71 = lean_alloc_ctor(1, 2, 0); } else { - x_68 = x_67; + x_71 = x_70; } -lean_ctor_set(x_68, 0, x_65); -lean_ctor_set(x_68, 1, x_66); -return x_68; +lean_ctor_set(x_71, 0, x_68); +lean_ctor_set(x_71, 1, x_69); +return x_71; } } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_69 = lean_ctor_get(x_30, 0); -lean_inc(x_69); -lean_dec(x_30); -x_70 = lean_st_ref_take(x_10, x_37); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_72 = x_70; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_72 = lean_ctor_get(x_33, 0); +lean_inc(x_72); +lean_dec(x_33); +x_73 = lean_st_ref_take(x_10, x_40); +x_74 = lean_ctor_get(x_73, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_75 = x_73; } else { - lean_dec_ref(x_70); - x_72 = lean_box(0); + lean_dec_ref(x_73); + x_75 = lean_box(0); } -x_73 = lean_box(0); -if (lean_is_scalar(x_72)) { - x_74 = lean_alloc_ctor(1, 2, 0); +x_76 = lean_box(0); +if (lean_is_scalar(x_75)) { + x_77 = lean_alloc_ctor(1, 2, 0); } else { - x_74 = x_72; - lean_ctor_set_tag(x_74, 1); + x_77 = x_75; + lean_ctor_set_tag(x_77, 1); } -lean_ctor_set(x_74, 0, x_69); -lean_ctor_set(x_74, 1, x_73); -x_75 = lean_st_ref_set(x_10, x_74, x_71); -x_76 = lean_ctor_get(x_75, 1); -lean_inc(x_76); -lean_dec(x_75); -x_77 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_76); -if (lean_obj_tag(x_77) == 0) +lean_ctor_set(x_77, 0, x_72); +lean_ctor_set(x_77, 1, x_76); +x_78 = lean_st_ref_set(x_10, x_77, x_74); +x_79 = lean_ctor_get(x_78, 1); +lean_inc(x_79); +lean_dec(x_78); +x_80 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_79); +if (lean_obj_tag(x_80) == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_78 = lean_ctor_get(x_77, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_79 = x_77; +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_82 = x_80; } else { - lean_dec_ref(x_77); - x_79 = lean_box(0); + lean_dec_ref(x_80); + x_82 = lean_box(0); } -x_80 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_80, 0, x_5); -if (lean_is_scalar(x_79)) { - x_81 = lean_alloc_ctor(0, 2, 0); +x_83 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_83, 0, x_5); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); } else { - x_81 = x_79; + x_84 = x_82; } -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_78); -return x_81; +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_dec(x_5); -x_82 = lean_ctor_get(x_77, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_77, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_84 = x_77; +x_85 = lean_ctor_get(x_80, 0); +lean_inc(x_85); +x_86 = lean_ctor_get(x_80, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_87 = x_80; } else { - lean_dec_ref(x_77); - x_84 = lean_box(0); + lean_dec_ref(x_80); + x_87 = lean_box(0); } -if (lean_is_scalar(x_84)) { - x_85 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_87)) { + x_88 = lean_alloc_ctor(1, 2, 0); } else { - x_85 = x_84; + x_88 = x_87; } -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; +lean_ctor_set(x_88, 0, x_85); +lean_ctor_set(x_88, 1, x_86); +return x_88; } } } } else { -uint8_t x_86; +uint8_t x_89; lean_dec(x_9); lean_dec(x_18); lean_dec(x_17); @@ -16300,38 +16333,38 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); -x_86 = !lean_is_exclusive(x_29); -if (x_86 == 0) +x_89 = !lean_is_exclusive(x_32); +if (x_89 == 0) { -return x_29; +return x_32; } else { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_29, 0); -x_88 = lean_ctor_get(x_29, 1); -lean_inc(x_88); -lean_inc(x_87); -lean_dec(x_29); -x_89 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_89, 0, x_87); -lean_ctor_set(x_89, 1, x_88); -return x_89; +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_32, 0); +x_91 = lean_ctor_get(x_32, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_32); +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; } } } else { -uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -x_90 = lean_ctor_get_uint8(x_9, sizeof(void*)*2); -x_91 = lean_ctor_get(x_9, 0); -lean_inc(x_91); +uint8_t x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_93 = lean_ctor_get_uint8(x_9, sizeof(void*)*2); +x_94 = lean_ctor_get(x_9, 0); +lean_inc(x_94); lean_dec(x_9); lean_inc(x_1); -x_92 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_1); -lean_ctor_set_uint8(x_92, sizeof(void*)*2, x_90); +x_95 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_95, 1, x_1); +lean_ctor_set_uint8(x_95, sizeof(void*)*2, x_93); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); @@ -16340,17 +16373,17 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_93 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_26, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_23); +x_96 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_29, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_26); lean_dec(x_1); -if (lean_obj_tag(x_93) == 0) +if (lean_obj_tag(x_96) == 0) { -lean_object* x_94; -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -if (lean_obj_tag(x_94) == 0) +lean_object* x_97; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +if (lean_obj_tag(x_97) == 0) { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; -lean_dec(x_92); +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16360,127 +16393,127 @@ lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - x_96 = x_93; +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_99 = x_96; } else { - lean_dec_ref(x_93); - x_96 = lean_box(0); + lean_dec_ref(x_96); + x_99 = lean_box(0); } -x_97 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_97, 0, x_5); -if (lean_is_scalar(x_96)) { - x_98 = lean_alloc_ctor(0, 2, 0); +x_100 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_100, 0, x_5); +if (lean_is_scalar(x_99)) { + x_101 = lean_alloc_ctor(0, 2, 0); } else { - x_98 = x_96; + x_101 = x_99; } -lean_ctor_set(x_98, 0, x_97); -lean_ctor_set(x_98, 1, x_95); -return x_98; +lean_ctor_set(x_101, 0, x_100); +lean_ctor_set(x_101, 1, x_98); +return x_101; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_99 = lean_ctor_get(x_93, 1); -lean_inc(x_99); -lean_dec(x_93); -x_100 = lean_ctor_get(x_94, 0); -lean_inc(x_100); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - x_101 = x_94; -} else { - lean_dec_ref(x_94); - x_101 = lean_box(0); -} -x_102 = lean_st_ref_take(x_10, x_99); -x_103 = lean_ctor_get(x_102, 1); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_102 = lean_ctor_get(x_96, 1); +lean_inc(x_102); +lean_dec(x_96); +x_103 = lean_ctor_get(x_97, 0); lean_inc(x_103); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_104 = x_102; +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + x_104 = x_97; } else { - lean_dec_ref(x_102); + lean_dec_ref(x_97); x_104 = lean_box(0); } -x_105 = lean_box(0); -if (lean_is_scalar(x_104)) { - x_106 = lean_alloc_ctor(1, 2, 0); +x_105 = lean_st_ref_take(x_10, x_102); +x_106 = lean_ctor_get(x_105, 1); +lean_inc(x_106); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_107 = x_105; } else { - x_106 = x_104; - lean_ctor_set_tag(x_106, 1); + lean_dec_ref(x_105); + x_107 = lean_box(0); } -lean_ctor_set(x_106, 0, x_100); -lean_ctor_set(x_106, 1, x_105); -x_107 = lean_st_ref_set(x_10, x_106, x_103); -x_108 = lean_ctor_get(x_107, 1); -lean_inc(x_108); -lean_dec(x_107); -x_109 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_92, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_108); -if (lean_obj_tag(x_109) == 0) +x_108 = lean_box(0); +if (lean_is_scalar(x_107)) { + x_109 = lean_alloc_ctor(1, 2, 0); +} else { + x_109 = x_107; + lean_ctor_set_tag(x_109, 1); +} +lean_ctor_set(x_109, 0, x_103); +lean_ctor_set(x_109, 1, x_108); +x_110 = lean_st_ref_set(x_10, x_109, x_106); +x_111 = lean_ctor_get(x_110, 1); +lean_inc(x_111); +lean_dec(x_110); +x_112 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_95, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_111); +if (lean_obj_tag(x_112) == 0) { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_110 = lean_ctor_get(x_109, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_111 = x_109; +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_113 = lean_ctor_get(x_112, 1); +lean_inc(x_113); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_114 = x_112; } else { - lean_dec_ref(x_109); - x_111 = lean_box(0); + lean_dec_ref(x_112); + x_114 = lean_box(0); } -if (lean_is_scalar(x_101)) { - x_112 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_104)) { + x_115 = lean_alloc_ctor(1, 1, 0); } else { - x_112 = x_101; + x_115 = x_104; } -lean_ctor_set(x_112, 0, x_5); -if (lean_is_scalar(x_111)) { - x_113 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_115, 0, x_5); +if (lean_is_scalar(x_114)) { + x_116 = lean_alloc_ctor(0, 2, 0); } else { - x_113 = x_111; + x_116 = x_114; } -lean_ctor_set(x_113, 0, x_112); -lean_ctor_set(x_113, 1, x_110); -return x_113; +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_113); +return x_116; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -lean_dec(x_101); +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +lean_dec(x_104); lean_dec(x_5); -x_114 = lean_ctor_get(x_109, 0); -lean_inc(x_114); -x_115 = lean_ctor_get(x_109, 1); -lean_inc(x_115); -if (lean_is_exclusive(x_109)) { - lean_ctor_release(x_109, 0); - lean_ctor_release(x_109, 1); - x_116 = x_109; +x_117 = lean_ctor_get(x_112, 0); +lean_inc(x_117); +x_118 = lean_ctor_get(x_112, 1); +lean_inc(x_118); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_119 = x_112; } else { - lean_dec_ref(x_109); - x_116 = lean_box(0); + lean_dec_ref(x_112); + x_119 = lean_box(0); } -if (lean_is_scalar(x_116)) { - x_117 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_119)) { + x_120 = lean_alloc_ctor(1, 2, 0); } else { - x_117 = x_116; + x_120 = x_119; } -lean_ctor_set(x_117, 0, x_114); -lean_ctor_set(x_117, 1, x_115); -return x_117; +lean_ctor_set(x_120, 0, x_117); +lean_ctor_set(x_120, 1, x_118); +return x_120; } } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; -lean_dec(x_92); +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +lean_dec(x_95); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16491,47 +16524,47 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); -x_118 = lean_ctor_get(x_93, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_93, 1); -lean_inc(x_119); -if (lean_is_exclusive(x_93)) { - lean_ctor_release(x_93, 0); - lean_ctor_release(x_93, 1); - x_120 = x_93; +x_121 = lean_ctor_get(x_96, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_96, 1); +lean_inc(x_122); +if (lean_is_exclusive(x_96)) { + lean_ctor_release(x_96, 0); + lean_ctor_release(x_96, 1); + x_123 = x_96; } else { - lean_dec_ref(x_93); - x_120 = lean_box(0); + lean_dec_ref(x_96); + x_123 = lean_box(0); } -if (lean_is_scalar(x_120)) { - x_121 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_123)) { + x_124 = lean_alloc_ctor(1, 2, 0); } else { - x_121 = x_120; + x_124 = x_123; } -lean_ctor_set(x_121, 0, x_118); -lean_ctor_set(x_121, 1, x_119); -return x_121; +lean_ctor_set(x_124, 0, x_121); +lean_ctor_set(x_124, 1, x_122); +return x_124; } } } } else { -lean_object* x_136; lean_object* x_137; lean_object* x_138; uint8_t x_175; -x_136 = lean_ctor_get(x_20, 0); -x_137 = lean_ctor_get(x_20, 1); -lean_inc(x_137); -lean_inc(x_136); -lean_dec(x_20); -x_175 = lean_ctor_get_uint8(x_136, sizeof(void*)*10 + 4); -if (x_175 == 0) +lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_178; +x_139 = lean_ctor_get(x_23, 0); +x_140 = lean_ctor_get(x_23, 1); +lean_inc(x_140); +lean_inc(x_139); +lean_dec(x_23); +x_178 = lean_ctor_get_uint8(x_139, sizeof(void*)*11 + 4); +if (x_178 == 0) { -uint8_t x_176; -x_176 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_136); -if (x_176 == 0) +uint8_t x_179; +x_179 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_139); +if (x_179 == 0) { -lean_object* x_177; lean_object* x_178; -lean_dec(x_136); +lean_object* x_180; lean_object* x_181; +lean_dec(x_139); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16545,33 +16578,33 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_177 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_177, 0, x_5); -x_178 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_178, 0, x_177); -lean_ctor_set(x_178, 1, x_137); -return x_178; +x_180 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_180, 0, x_5); +x_181 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_181, 0, x_180); +lean_ctor_set(x_181, 1, x_140); +return x_181; } else { if (x_6 == 0) { -lean_object* x_179; -x_179 = lean_box(0); -x_138 = x_179; -goto block_174; +lean_object* x_182; +x_182 = lean_box(0); +x_141 = x_182; +goto block_177; } else { -lean_object* x_180; uint8_t x_181; -x_180 = lean_ctor_get(x_136, 9); -lean_inc(x_180); -x_181 = lean_nat_dec_eq(x_180, x_7); -lean_dec(x_180); -if (x_181 == 0) +lean_object* x_183; uint8_t x_184; +x_183 = lean_ctor_get(x_139, 9); +lean_inc(x_183); +x_184 = lean_nat_dec_eq(x_183, x_7); +lean_dec(x_183); +if (x_184 == 0) { -lean_object* x_182; lean_object* x_183; -lean_dec(x_136); +lean_object* x_185; lean_object* x_186; +lean_dec(x_139); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16585,19 +16618,19 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_182 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_182, 0, x_5); -x_183 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_183, 0, x_182); -lean_ctor_set(x_183, 1, x_137); -return x_183; +x_185 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_185, 0, x_5); +x_186 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_186, 0, x_185); +lean_ctor_set(x_186, 1, x_140); +return x_186; } else { -lean_object* x_184; -x_184 = lean_box(0); -x_138 = x_184; -goto block_174; +lean_object* x_187; +x_187 = lean_box(0); +x_141 = x_187; +goto block_177; } } } @@ -16606,22 +16639,22 @@ else { if (x_6 == 0) { -lean_object* x_185; -x_185 = lean_box(0); -x_138 = x_185; -goto block_174; +lean_object* x_188; +x_188 = lean_box(0); +x_141 = x_188; +goto block_177; } else { -lean_object* x_186; uint8_t x_187; -x_186 = lean_ctor_get(x_136, 9); -lean_inc(x_186); -x_187 = lean_nat_dec_eq(x_186, x_7); -lean_dec(x_186); -if (x_187 == 0) +lean_object* x_189; uint8_t x_190; +x_189 = lean_ctor_get(x_139, 9); +lean_inc(x_189); +x_190 = lean_nat_dec_eq(x_189, x_7); +lean_dec(x_189); +if (x_190 == 0) { -lean_object* x_188; lean_object* x_189; -lean_dec(x_136); +lean_object* x_191; lean_object* x_192; +lean_dec(x_139); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16635,53 +16668,53 @@ lean_dec(x_9); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_188 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_188, 0, x_5); -x_189 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_189, 0, x_188); -lean_ctor_set(x_189, 1, x_137); -return x_189; +x_191 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_191, 0, x_5); +x_192 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_192, 0, x_191); +lean_ctor_set(x_192, 1, x_140); +return x_192; } else { -lean_object* x_190; -x_190 = lean_box(0); -x_138 = x_190; -goto block_174; +lean_object* x_193; +x_193 = lean_box(0); +x_141 = x_193; +goto block_177; } } } -block_174: +block_177: { -lean_object* x_139; lean_object* x_140; uint8_t x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_138); -x_139 = lean_ctor_get(x_136, 8); -lean_inc(x_139); -lean_dec(x_136); -x_140 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_140, 0, x_2); -lean_ctor_set(x_140, 1, x_139); -lean_ctor_set(x_140, 2, x_3); -x_141 = lean_ctor_get_uint8(x_9, sizeof(void*)*2); -x_142 = lean_ctor_get(x_9, 0); +lean_object* x_142; lean_object* x_143; uint8_t x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +lean_dec(x_141); +x_142 = lean_ctor_get(x_139, 8); lean_inc(x_142); +lean_dec(x_139); +x_143 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_143, 0, x_2); +lean_ctor_set(x_143, 1, x_142); +lean_ctor_set(x_143, 2, x_3); +x_144 = lean_ctor_get_uint8(x_9, sizeof(void*)*2); +x_145 = lean_ctor_get(x_9, 0); +lean_inc(x_145); if (lean_is_exclusive(x_9)) { lean_ctor_release(x_9, 0); lean_ctor_release(x_9, 1); - x_143 = x_9; + x_146 = x_9; } else { lean_dec_ref(x_9); - x_143 = lean_box(0); + x_146 = lean_box(0); } lean_inc(x_1); -if (lean_is_scalar(x_143)) { - x_144 = lean_alloc_ctor(0, 2, 1); +if (lean_is_scalar(x_146)) { + x_147 = lean_alloc_ctor(0, 2, 1); } else { - x_144 = x_143; + x_147 = x_146; } -lean_ctor_set(x_144, 0, x_142); -lean_ctor_set(x_144, 1, x_1); -lean_ctor_set_uint8(x_144, sizeof(void*)*2, x_141); +lean_ctor_set(x_147, 0, x_145); +lean_ctor_set(x_147, 1, x_1); +lean_ctor_set_uint8(x_147, sizeof(void*)*2, x_144); lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); @@ -16690,17 +16723,17 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -x_145 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_140, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_137); +x_148 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_matchArgs_x3f(x_143, x_4, x_1, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_140); lean_dec(x_1); -if (lean_obj_tag(x_145) == 0) +if (lean_obj_tag(x_148) == 0) { -lean_object* x_146; -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -if (lean_obj_tag(x_146) == 0) +lean_object* x_149; +x_149 = lean_ctor_get(x_148, 0); +lean_inc(x_149); +if (lean_obj_tag(x_149) == 0) { -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -lean_dec(x_144); +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; +lean_dec(x_147); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16710,127 +16743,127 @@ lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_147 = lean_ctor_get(x_145, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_145)) { - lean_ctor_release(x_145, 0); - lean_ctor_release(x_145, 1); - x_148 = x_145; +x_150 = lean_ctor_get(x_148, 1); +lean_inc(x_150); +if (lean_is_exclusive(x_148)) { + lean_ctor_release(x_148, 0); + lean_ctor_release(x_148, 1); + x_151 = x_148; } else { - lean_dec_ref(x_145); - x_148 = lean_box(0); + lean_dec_ref(x_148); + x_151 = lean_box(0); } -x_149 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_149, 0, x_5); -if (lean_is_scalar(x_148)) { - x_150 = lean_alloc_ctor(0, 2, 0); +x_152 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_152, 0, x_5); +if (lean_is_scalar(x_151)) { + x_153 = lean_alloc_ctor(0, 2, 0); } else { - x_150 = x_148; + x_153 = x_151; } -lean_ctor_set(x_150, 0, x_149); -lean_ctor_set(x_150, 1, x_147); -return x_150; +lean_ctor_set(x_153, 0, x_152); +lean_ctor_set(x_153, 1, x_150); +return x_153; } else { -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; -x_151 = lean_ctor_get(x_145, 1); -lean_inc(x_151); -lean_dec(x_145); -x_152 = lean_ctor_get(x_146, 0); -lean_inc(x_152); -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - x_153 = x_146; -} else { - lean_dec_ref(x_146); - x_153 = lean_box(0); -} -x_154 = lean_st_ref_take(x_10, x_151); -x_155 = lean_ctor_get(x_154, 1); +lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_154 = lean_ctor_get(x_148, 1); +lean_inc(x_154); +lean_dec(x_148); +x_155 = lean_ctor_get(x_149, 0); lean_inc(x_155); -if (lean_is_exclusive(x_154)) { - lean_ctor_release(x_154, 0); - lean_ctor_release(x_154, 1); - x_156 = x_154; +if (lean_is_exclusive(x_149)) { + lean_ctor_release(x_149, 0); + x_156 = x_149; } else { - lean_dec_ref(x_154); + lean_dec_ref(x_149); x_156 = lean_box(0); } -x_157 = lean_box(0); -if (lean_is_scalar(x_156)) { - x_158 = lean_alloc_ctor(1, 2, 0); +x_157 = lean_st_ref_take(x_10, x_154); +x_158 = lean_ctor_get(x_157, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_159 = x_157; } else { - x_158 = x_156; - lean_ctor_set_tag(x_158, 1); + lean_dec_ref(x_157); + x_159 = lean_box(0); } -lean_ctor_set(x_158, 0, x_152); -lean_ctor_set(x_158, 1, x_157); -x_159 = lean_st_ref_set(x_10, x_158, x_155); -x_160 = lean_ctor_get(x_159, 1); -lean_inc(x_160); -lean_dec(x_159); -x_161 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_144, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_160); -if (lean_obj_tag(x_161) == 0) +x_160 = lean_box(0); +if (lean_is_scalar(x_159)) { + x_161 = lean_alloc_ctor(1, 2, 0); +} else { + x_161 = x_159; + lean_ctor_set_tag(x_161, 1); +} +lean_ctor_set(x_161, 0, x_155); +lean_ctor_set(x_161, 1, x_160); +x_162 = lean_st_ref_set(x_10, x_161, x_158); +x_163 = lean_ctor_get(x_162, 1); +lean_inc(x_163); +lean_dec(x_162); +x_164 = l___private_Lean_Meta_Tactic_Grind_EMatch_0__Lean_Meta_Grind_EMatch_processChoices(x_147, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_163); +if (lean_obj_tag(x_164) == 0) { -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_162 = lean_ctor_get(x_161, 1); -lean_inc(x_162); -if (lean_is_exclusive(x_161)) { - lean_ctor_release(x_161, 0); - lean_ctor_release(x_161, 1); - x_163 = x_161; +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_165 = lean_ctor_get(x_164, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_164)) { + lean_ctor_release(x_164, 0); + lean_ctor_release(x_164, 1); + x_166 = x_164; } else { - lean_dec_ref(x_161); - x_163 = lean_box(0); + lean_dec_ref(x_164); + x_166 = lean_box(0); } -if (lean_is_scalar(x_153)) { - x_164 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_156)) { + x_167 = lean_alloc_ctor(1, 1, 0); } else { - x_164 = x_153; + x_167 = x_156; } -lean_ctor_set(x_164, 0, x_5); -if (lean_is_scalar(x_163)) { - x_165 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_167, 0, x_5); +if (lean_is_scalar(x_166)) { + x_168 = lean_alloc_ctor(0, 2, 0); } else { - x_165 = x_163; + x_168 = x_166; } -lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_162); -return x_165; +lean_ctor_set(x_168, 0, x_167); +lean_ctor_set(x_168, 1, x_165); +return x_168; } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; -lean_dec(x_153); +lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; +lean_dec(x_156); lean_dec(x_5); -x_166 = lean_ctor_get(x_161, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_161, 1); -lean_inc(x_167); -if (lean_is_exclusive(x_161)) { - lean_ctor_release(x_161, 0); - lean_ctor_release(x_161, 1); - x_168 = x_161; +x_169 = lean_ctor_get(x_164, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_164, 1); +lean_inc(x_170); +if (lean_is_exclusive(x_164)) { + lean_ctor_release(x_164, 0); + lean_ctor_release(x_164, 1); + x_171 = x_164; } else { - lean_dec_ref(x_161); - x_168 = lean_box(0); + lean_dec_ref(x_164); + x_171 = lean_box(0); } -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_171)) { + x_172 = lean_alloc_ctor(1, 2, 0); } else { - x_169 = x_168; + x_172 = x_171; } -lean_ctor_set(x_169, 0, x_166); -lean_ctor_set(x_169, 1, x_167); -return x_169; +lean_ctor_set(x_172, 0, x_169); +lean_ctor_set(x_172, 1, x_170); +return x_172; } } } else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -lean_dec(x_144); +lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; +lean_dec(x_147); lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16841,33 +16874,33 @@ lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_5); -x_170 = lean_ctor_get(x_145, 0); -lean_inc(x_170); -x_171 = lean_ctor_get(x_145, 1); -lean_inc(x_171); -if (lean_is_exclusive(x_145)) { - lean_ctor_release(x_145, 0); - lean_ctor_release(x_145, 1); - x_172 = x_145; +x_173 = lean_ctor_get(x_148, 0); +lean_inc(x_173); +x_174 = lean_ctor_get(x_148, 1); +lean_inc(x_174); +if (lean_is_exclusive(x_148)) { + lean_ctor_release(x_148, 0); + lean_ctor_release(x_148, 1); + x_175 = x_148; } else { - lean_dec_ref(x_145); - x_172 = lean_box(0); + lean_dec_ref(x_148); + x_175 = lean_box(0); } -if (lean_is_scalar(x_172)) { - x_173 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_175)) { + x_176 = lean_alloc_ctor(1, 2, 0); } else { - x_173 = x_172; + x_176 = x_175; } -lean_ctor_set(x_173, 0, x_170); -lean_ctor_set(x_173, 1, x_171); -return x_173; +lean_ctor_set(x_176, 0, x_173); +lean_ctor_set(x_176, 1, x_174); +return x_176; } } } } else { -uint8_t x_191; +uint8_t x_194; lean_dec(x_18); lean_dec(x_17); lean_dec(x_16); @@ -16882,23 +16915,23 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_191 = !lean_is_exclusive(x_20); -if (x_191 == 0) +x_194 = !lean_is_exclusive(x_23); +if (x_194 == 0) { -return x_20; +return x_23; } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; -x_192 = lean_ctor_get(x_20, 0); -x_193 = lean_ctor_get(x_20, 1); -lean_inc(x_193); -lean_inc(x_192); -lean_dec(x_20); -x_194 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_194, 0, x_192); -lean_ctor_set(x_194, 1, x_193); -return x_194; +lean_object* x_195; lean_object* x_196; lean_object* x_197; +x_195 = lean_ctor_get(x_23, 0); +x_196 = lean_ctor_get(x_23, 1); +lean_inc(x_196); +lean_inc(x_195); +lean_dec(x_23); +x_197 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_197, 0, x_195); +lean_ctor_set(x_197, 1, x_196); +return x_197; } } } @@ -17119,7 +17152,7 @@ if (x_15 == 0) lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_16 = lean_ctor_get(x_14, 0); x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_16, 4); +x_18 = lean_ctor_get(x_16, 5); lean_inc(x_18); lean_dec(x_16); lean_inc(x_1); @@ -17166,7 +17199,7 @@ lean_inc(x_29); x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); lean_dec(x_28); -x_31 = lean_ctor_get(x_29, 6); +x_31 = lean_ctor_get(x_29, 7); lean_inc(x_31); lean_dec(x_29); x_32 = lean_box(0); @@ -17273,7 +17306,7 @@ x_54 = lean_ctor_get(x_14, 1); lean_inc(x_54); lean_inc(x_53); lean_dec(x_14); -x_55 = lean_ctor_get(x_53, 4); +x_55 = lean_ctor_get(x_53, 5); lean_inc(x_55); lean_dec(x_53); lean_inc(x_1); @@ -17321,7 +17354,7 @@ lean_inc(x_67); x_68 = lean_ctor_get(x_66, 1); lean_inc(x_68); lean_dec(x_66); -x_69 = lean_ctor_get(x_67, 6); +x_69 = lean_ctor_get(x_67, 7); lean_inc(x_69); lean_dec(x_67); x_70 = lean_box(0); @@ -18589,43 +18622,43 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematch(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -uint8_t x_10; lean_object* x_11; lean_object* x_84; lean_object* x_85; uint8_t x_86; -x_84 = l_Lean_Meta_Grind_checkMaxInstancesExceeded(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_unbox(x_85); -if (x_86 == 0) +uint8_t x_10; lean_object* x_11; lean_object* x_87; lean_object* x_88; uint8_t x_89; +x_87 = l_Lean_Meta_Grind_checkMaxInstancesExceeded(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_88 = lean_ctor_get(x_87, 0); +lean_inc(x_88); +x_89 = lean_unbox(x_88); +if (x_89 == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; -lean_dec(x_85); -x_87 = lean_ctor_get(x_84, 1); -lean_inc(x_87); -lean_dec(x_84); -x_88 = l_Lean_Meta_Grind_checkMaxEmatchExceeded(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_87); -x_89 = lean_ctor_get(x_88, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_88, 1); -lean_inc(x_90); +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; lean_dec(x_88); -x_91 = lean_unbox(x_89); -lean_dec(x_89); -x_10 = x_91; -x_11 = x_90; -goto block_83; +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = l_Lean_Meta_Grind_checkMaxEmatchExceeded(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_90); +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_91, 1); +lean_inc(x_93); +lean_dec(x_91); +x_94 = lean_unbox(x_92); +lean_dec(x_92); +x_10 = x_94; +x_11 = x_93; +goto block_86; } else { -lean_object* x_92; uint8_t x_93; -x_92 = lean_ctor_get(x_84, 1); -lean_inc(x_92); -lean_dec(x_84); -x_93 = lean_unbox(x_85); -lean_dec(x_85); -x_10 = x_93; -x_11 = x_92; -goto block_83; +lean_object* x_95; uint8_t x_96; +x_95 = lean_ctor_get(x_87, 1); +lean_inc(x_95); +lean_dec(x_87); +x_96 = lean_unbox(x_88); +lean_dec(x_88); +x_10 = x_96; +x_11 = x_95; +goto block_86; } -block_83: +block_86: { if (x_10 == 0) { @@ -18642,10 +18675,10 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = lean_ctor_get(x_13, 8); +x_18 = lean_ctor_get(x_13, 10); lean_inc(x_18); lean_dec(x_13); -x_19 = lean_ctor_get(x_16, 9); +x_19 = lean_ctor_get(x_16, 11); lean_inc(x_19); lean_dec(x_16); x_20 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_ematch___lambda__1___boxed), 12, 1); @@ -18673,10 +18706,10 @@ x_28 = !lean_is_exclusive(x_26); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_29 = lean_ctor_get(x_26, 6); -x_30 = lean_ctor_get(x_26, 8); -x_31 = lean_ctor_get(x_26, 9); -x_32 = lean_ctor_get(x_26, 12); +x_29 = lean_ctor_get(x_26, 7); +x_30 = lean_ctor_get(x_26, 10); +x_31 = lean_ctor_get(x_26, 11); +x_32 = lean_ctor_get(x_26, 14); x_33 = lean_unsigned_to_nat(1u); x_34 = lean_nat_add(x_29, x_33); lean_dec(x_29); @@ -18685,10 +18718,10 @@ lean_dec(x_31); x_36 = lean_nat_add(x_32, x_33); lean_dec(x_32); x_37 = l_Lean_Meta_Grind_ematch___closed__3; -lean_ctor_set(x_26, 12, x_36); -lean_ctor_set(x_26, 9, x_37); -lean_ctor_set(x_26, 8, x_35); -lean_ctor_set(x_26, 6, x_34); +lean_ctor_set(x_26, 14, x_36); +lean_ctor_set(x_26, 11, x_37); +lean_ctor_set(x_26, 10, x_35); +lean_ctor_set(x_26, 7, x_34); x_38 = lean_st_ref_set(x_1, x_26, x_27); lean_dec(x_1); x_39 = !lean_is_exclusive(x_38); @@ -18716,15 +18749,15 @@ return x_44; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; x_45 = lean_ctor_get(x_26, 0); x_46 = lean_ctor_get(x_26, 1); x_47 = lean_ctor_get(x_26, 2); x_48 = lean_ctor_get(x_26, 3); x_49 = lean_ctor_get(x_26, 4); x_50 = lean_ctor_get(x_26, 5); -x_51 = lean_ctor_get_uint8(x_26, sizeof(void*)*20); -x_52 = lean_ctor_get(x_26, 6); +x_51 = lean_ctor_get(x_26, 6); +x_52 = lean_ctor_get_uint8(x_26, sizeof(void*)*23); x_53 = lean_ctor_get(x_26, 7); x_54 = lean_ctor_get(x_26, 8); x_55 = lean_ctor_get(x_26, 9); @@ -18738,6 +18771,12 @@ x_62 = lean_ctor_get(x_26, 16); x_63 = lean_ctor_get(x_26, 17); x_64 = lean_ctor_get(x_26, 18); x_65 = lean_ctor_get(x_26, 19); +x_66 = lean_ctor_get(x_26, 20); +x_67 = lean_ctor_get(x_26, 21); +x_68 = lean_ctor_get(x_26, 22); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); @@ -18751,7 +18790,7 @@ lean_inc(x_56); lean_inc(x_55); lean_inc(x_54); lean_inc(x_53); -lean_inc(x_52); +lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); lean_inc(x_48); @@ -18759,86 +18798,89 @@ lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_dec(x_26); -x_66 = lean_unsigned_to_nat(1u); -x_67 = lean_nat_add(x_52, x_66); -lean_dec(x_52); -x_68 = l_Lean_PersistentArray_append___rarg(x_54, x_55); -lean_dec(x_55); -x_69 = lean_nat_add(x_58, x_66); -lean_dec(x_58); -x_70 = l_Lean_Meta_Grind_ematch___closed__3; -x_71 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_71, 0, x_45); -lean_ctor_set(x_71, 1, x_46); -lean_ctor_set(x_71, 2, x_47); -lean_ctor_set(x_71, 3, x_48); -lean_ctor_set(x_71, 4, x_49); -lean_ctor_set(x_71, 5, x_50); -lean_ctor_set(x_71, 6, x_67); -lean_ctor_set(x_71, 7, x_53); -lean_ctor_set(x_71, 8, x_68); -lean_ctor_set(x_71, 9, x_70); -lean_ctor_set(x_71, 10, x_56); -lean_ctor_set(x_71, 11, x_57); -lean_ctor_set(x_71, 12, x_69); -lean_ctor_set(x_71, 13, x_59); -lean_ctor_set(x_71, 14, x_60); -lean_ctor_set(x_71, 15, x_61); -lean_ctor_set(x_71, 16, x_62); -lean_ctor_set(x_71, 17, x_63); -lean_ctor_set(x_71, 18, x_64); -lean_ctor_set(x_71, 19, x_65); -lean_ctor_set_uint8(x_71, sizeof(void*)*20, x_51); -x_72 = lean_st_ref_set(x_1, x_71, x_27); +x_69 = lean_unsigned_to_nat(1u); +x_70 = lean_nat_add(x_53, x_69); +lean_dec(x_53); +x_71 = l_Lean_PersistentArray_append___rarg(x_56, x_57); +lean_dec(x_57); +x_72 = lean_nat_add(x_60, x_69); +lean_dec(x_60); +x_73 = l_Lean_Meta_Grind_ematch___closed__3; +x_74 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_74, 0, x_45); +lean_ctor_set(x_74, 1, x_46); +lean_ctor_set(x_74, 2, x_47); +lean_ctor_set(x_74, 3, x_48); +lean_ctor_set(x_74, 4, x_49); +lean_ctor_set(x_74, 5, x_50); +lean_ctor_set(x_74, 6, x_51); +lean_ctor_set(x_74, 7, x_70); +lean_ctor_set(x_74, 8, x_54); +lean_ctor_set(x_74, 9, x_55); +lean_ctor_set(x_74, 10, x_71); +lean_ctor_set(x_74, 11, x_73); +lean_ctor_set(x_74, 12, x_58); +lean_ctor_set(x_74, 13, x_59); +lean_ctor_set(x_74, 14, x_72); +lean_ctor_set(x_74, 15, x_61); +lean_ctor_set(x_74, 16, x_62); +lean_ctor_set(x_74, 17, x_63); +lean_ctor_set(x_74, 18, x_64); +lean_ctor_set(x_74, 19, x_65); +lean_ctor_set(x_74, 20, x_66); +lean_ctor_set(x_74, 21, x_67); +lean_ctor_set(x_74, 22, x_68); +lean_ctor_set_uint8(x_74, sizeof(void*)*23, x_52); +x_75 = lean_st_ref_set(x_1, x_74, x_27); lean_dec(x_1); -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_74 = x_72; +x_76 = lean_ctor_get(x_75, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_77 = x_75; } else { - lean_dec_ref(x_72); - x_74 = lean_box(0); + lean_dec_ref(x_75); + x_77 = lean_box(0); } -x_75 = lean_box(0); -if (lean_is_scalar(x_74)) { - x_76 = lean_alloc_ctor(0, 2, 0); +x_78 = lean_box(0); +if (lean_is_scalar(x_77)) { + x_79 = lean_alloc_ctor(0, 2, 0); } else { - x_76 = x_74; + x_79 = x_77; } -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_73); -return x_76; +lean_ctor_set(x_79, 0, x_78); +lean_ctor_set(x_79, 1, x_76); +return x_79; } } else { -uint8_t x_77; +uint8_t x_80; lean_dec(x_1); -x_77 = !lean_is_exclusive(x_23); -if (x_77 == 0) +x_80 = !lean_is_exclusive(x_23); +if (x_80 == 0) { return x_23; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_23, 0); -x_79 = lean_ctor_get(x_23, 1); -lean_inc(x_79); -lean_inc(x_78); +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_23, 0); +x_82 = lean_ctor_get(x_23, 1); +lean_inc(x_82); +lean_inc(x_81); lean_dec(x_23); -x_80 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_80, 0, x_78); -lean_ctor_set(x_80, 1, x_79); -return x_80; +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_81); +lean_ctor_set(x_83, 1, x_82); +return x_83; } } } else { -lean_object* x_81; lean_object* x_82; +lean_object* x_84; lean_object* x_85; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -18847,11 +18889,11 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_81 = lean_box(0); -x_82 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_11); -return x_82; +x_84 = lean_box(0); +x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_85, 0, x_84); +lean_ctor_set(x_85, 1, x_11); +return x_85; } } } @@ -19067,7 +19109,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ematchAndAssert(lean_object* x_1, lea _start: { lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_10 = lean_ctor_get(x_1, 11); +x_10 = lean_ctor_get(x_1, 13); lean_inc(x_10); x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); @@ -19098,7 +19140,7 @@ if (x_18 == 0) lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; x_19 = lean_ctor_get(x_17, 0); x_20 = lean_ctor_get(x_17, 1); -x_21 = lean_ctor_get(x_19, 11); +x_21 = lean_ctor_get(x_19, 13); lean_inc(x_21); x_22 = lean_nat_dec_eq(x_21, x_10); lean_dec(x_10); @@ -19135,7 +19177,7 @@ x_27 = lean_ctor_get(x_17, 1); lean_inc(x_27); lean_inc(x_26); lean_dec(x_17); -x_28 = lean_ctor_get(x_26, 11); +x_28 = lean_ctor_get(x_26, 13); lean_inc(x_28); x_29 = lean_nat_dec_eq(x_28, x_10); lean_dec(x_10); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatchTheorem.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatchTheorem.c index f05bbee30afe..74e52acfbf09 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatchTheorem.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/EMatchTheorem.c @@ -16,24 +16,24 @@ extern "C" { LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ematchTheoremsExt; static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__1; lean_object* l___private_Init_Meta_0__Lean_Syntax_reprSyntax____x40_Init_Meta___hyg_2170_(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21; lean_object* l_Lean_Name_reprPrec(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__10(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collectPatterns_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getProofFor___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__12; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_dontCare; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__15; static lean_object* l_Lean_Meta_Grind_preprocessPattern___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableOrigin___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__3; @@ -52,13 +52,11 @@ static lean_object* l_Lean_Meta_Grind_mkGroundPattern___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_pp___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_detectOffsets(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__2___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__4___closed__1; @@ -75,6 +73,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_NormalizePattern_getPatternSupportMas static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___lambda__1___closed__2; static lean_object* l_Lean_Meta_Grind_isOffsetPattern_x3f___closed__1; LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkTypeFVars___spec__1___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkTypeFVars___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__19; uint8_t lean_usize_dec_le(size_t, size_t); @@ -116,6 +115,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__3___closed__1; lean_object* l_Lean_Expr_sort___override(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1(lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); @@ -124,10 +124,10 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met lean_object* lean_array_push(lean_object*, lean_object*); lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__19; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__5; size_t lean_usize_mul(size_t, size_t); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___closed__3; lean_object* l_Lean_RBNode_fold___at_Lean_RBMap_size___spec__1___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute___closed__3; @@ -141,9 +141,9 @@ static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatc uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__10; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_toCtorIdx___boxed(lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__1___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_saveSymbol___spec__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279_(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqOrigin__1___boxed(lean_object*, lean_object*); @@ -154,20 +154,18 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea static lean_object* l_Lean_Meta_Grind_instInhabitedOrigin___closed__1; lean_object* l_Lean_Expr_bvar___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___lambda__1(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17; lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17; static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__1___closed__2; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Expr_fvarId_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_NormalizePattern_getPatternSupportMask___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkConstWithLevelParams___at_Lean_Meta_registerCoercion___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkTypeFVars___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t); @@ -175,6 +173,7 @@ LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Meta_Tactic_Grin LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__9(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Meta_forallTelescopeReducing___at_Lean_Meta_getParamNames___spec__2___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_EMatchTheorems_contains___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedEMatchTheorems; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -191,6 +190,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda_ lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__7; lean_object* l_Lean_stringToMessageData(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___spec__2(uint8_t, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_NormalizePattern_main___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instReprOrigin; @@ -205,44 +205,52 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea static lean_object* l_Lean_Meta_Grind_instInhabitedEMatchTheorem___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedEMatchTheorem; lean_object* l_Lean_throwError___at_Lean_Meta_setInlineAttribute___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__1; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_EMatchTheorems_isErased(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_NormalizePattern_getPatternSupportMask___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getPropTypes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__7; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__3; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isPatternDontCare___boxed(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__5; uint8_t l_Lean_Expr_isBVar(lean_object*); lean_object* l_List_mapTR_loop___at_Lean_mkConstWithLevelParams___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__15(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__4; static lean_object* l_Lean_Meta_Grind_mkOffsetPattern___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkGroundPattern___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_saveSymbol___spec__2(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18; uint8_t l_Lean_Expr_hasMVar(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatchTheorem_getProofWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_key___boxed(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_dontCare___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatchTheorems_insert(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_explainFailure___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853____boxed(lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_pp___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__20(lean_object*, size_t, size_t, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__6; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__20; @@ -250,7 +258,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_NormalizePattern_main___closed__3; static lean_object* l_Lean_Meta_Grind_NormalizePattern_main___closed__4; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3___closed__3; static lean_object* l_Lean_Meta_Grind_mkOffsetPattern___closed__2; size_t lean_usize_of_nat(lean_object*); @@ -260,6 +267,7 @@ lean_object* l_Lean_PersistentHashMap_isUnaryNode___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_preprocessPattern___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_expr_abstract(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_811_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__14___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -268,8 +276,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__6___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__7(lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_preprocessPattern(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -278,8 +285,10 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_M uint8_t l_Lean_ConstantInfo_isTheorem(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldrM___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__2___boxed(lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_mkEMatchEqTheoremCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at___private_Lean_Compiler_InlineAttrs_0__Lean_Compiler_isValidMacroInline___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getProofFor___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -292,7 +301,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea lean_object* l_Lean_Meta_forallBoundedTelescope___at_Lean_Meta_arrowDomainsN___spec__6___rarg(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___lambda__1___closed__3; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_saveBVar___spec__2(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofSyntax(lean_object*); @@ -300,9 +308,9 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_T static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__7; lean_object* lean_nat_div(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_NormalizePattern_main___closed__5; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go_goArg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__10; static lean_object* l_Lean_Meta_Grind_preprocessPattern___closed__2; @@ -321,7 +329,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_explainFailure___closed__1; static lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -334,7 +341,6 @@ lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__7___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___closed__1; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1; LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -342,32 +348,32 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEMatchTheorems(lean_object*); lean_object* l_Lean_Meta_getEqnsFor_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__8; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_reprOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_614____closed__8; static lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___lambda__2___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9; static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__3___closed__2; static lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1___closed__1; lean_object* l_Lean_RBNode_findCore___at_Lean_Meta_Closure_process___spec__1(lean_object*, lean_object*); uint8_t l_List_isEmpty___rarg(lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__16; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitWhileForbidden(lean_object*); static lean_object* l_Lean_Meta_Grind_preprocessPattern___lambda__1___closed__2; LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_isForbidden(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_explainFailure___closed__6; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540____boxed(lean_object*, lean_object*); lean_object* l_Lean_ScopedEnvExtension_modifyState___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt___spec__1___closed__3; uint8_t l_List_elem___at_Lean_Meta_Occurrences_contains___spec__1(lean_object*, lean_object*); @@ -376,7 +382,6 @@ static lean_object* l_Lean_Meta_Grind_ppPattern___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute___closed__6; lean_object* l_Lean_Expr_toHeadIndex(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__13; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__9___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__6___closed__2; @@ -388,11 +393,11 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met lean_object* l_panic___at_String_fromUTF8_x21___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_NormalizePattern_main(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__11; +static lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1; static lean_object* l_Lean_Meta_Grind_mkOffsetPattern___closed__4; lean_object* l_Lean_mkConstWithLevelParams___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9; lean_object* l_Lean_Expr_constName_x21(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg(uint8_t, uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__6___closed__1; @@ -402,16 +407,16 @@ static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___closed__5; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_saveSymbol___spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute___closed__1; lean_object* l_Lean_MessageData_ofConst(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEMatchTheorems___boxed(lean_object*); lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_grind_normalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__6; lean_object* l_Lean_mkAnnotation(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__13; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_dontCare___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_foundBVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkTypeFVars(lean_object*, lean_object*, lean_object*); @@ -420,6 +425,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_reprOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_614____closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_reprOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_614____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_toCtorIdx(uint8_t); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); @@ -443,6 +449,7 @@ lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_ lean_object* l_Lean_Meta_Grind_foldProjs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_NormalizePattern_getPatternSupportMask___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__2; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__14; static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__6; @@ -460,6 +467,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__2(lea static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__1___closed__1; lean_object* l_Lean_CollectFVars_main(lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instMonadMetaM; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_pp___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_indexOfAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__8___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); @@ -475,23 +483,22 @@ lean_object* lean_usize_to_nat(size_t); lean_object* l_Lean_Meta_instInhabitedMetaM___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__18(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__14; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_EMatchTheorems_insert___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkTypeFVars___closed__1; lean_object* l_Lean_MessageData_ofExpr(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__3(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__2___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___closed__1; static lean_object* l_Lean_Meta_Grind_mkOffsetPattern___closed__3; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4; LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_mkEMatchEqTheoremCore___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(uint8_t, uint8_t); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isOffsetPattern_x3f___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__12(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__4; @@ -501,21 +508,20 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f_go___lamb LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__14___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_pp___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatchTheorems_isErased___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12; LEAN_EXPORT lean_object* l_Array_indexOfAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__8(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collectPatterns_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_reprOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_614____closed__11; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getPropTypes___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_isForbidden___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20; LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableOrigin(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go_goArg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_explainFailure___closed__4; LEAN_EXPORT lean_object* l_Array_filterMapM___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getPropTypes___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -529,14 +535,13 @@ static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatc static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr(lean_object*, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3___closed__4; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_isAtomicPattern(lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__7(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__16; LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__1(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__10___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__11(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_NormalizePattern_normalizePattern(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -552,27 +557,23 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__3___closed__1; static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__3; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collectPatterns_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_isOffsetPattern_x3f___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_EMatchTheorems_contains(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10; lean_object* l_Lean_instantiateMVars___at___private_Lean_Meta_Basic_0__Lean_Meta_isClassApp_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute___closed__2; lean_object* l_Lean_mkRawNatLit(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx(uint8_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collectPatterns_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_id___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2___closed__2; +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_indentExpr(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheorem___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1(lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntries(lean_object*, lean_object*); @@ -589,6 +590,7 @@ static lean_object* l_Lean_Meta_Grind_EMatchTheorems_insert___closed__1; LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_foundBVar___spec__1(lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___lambda__2___closed__2; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___closed__3; uint64_t l_Lean_Name_hash___override(lean_object*); @@ -610,7 +612,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met lean_object* l_Lean_annotation_x3f(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind___closed__2; LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instInhabitedTheoremKind; -static uint64_t l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__2; lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -619,6 +620,7 @@ lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__18; static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__3___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3; lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getPropTypes___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__11(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -631,12 +633,16 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__4; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__11; lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2___closed__6; +static uint64_t l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_collect___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592_(lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_eraseAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__7(lean_object*, size_t, lean_object*); @@ -646,14 +652,14 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Met static lean_object* l_Lean_Meta_Grind_NormalizePattern_main___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_EMatchTheorems_contains___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_EMatchTheorems_insert___closed__3; -static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1; lean_object* l_Lean_registerBuiltinAttribute(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__17; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__8; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_isPatternFnCandidate___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__3; @@ -679,6 +685,7 @@ size_t lean_usize_add(size_t, size_t); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___closed__3; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12; static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_reprOrigin____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_614____closed__7; LEAN_EXPORT lean_object* l_Lean_throwError___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_addTrace___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addNewPattern___spec__2___closed__1; @@ -690,15 +697,14 @@ lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Expr_fvar___override(lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___lambda__1___closed__1; size_t lean_array_size(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__10___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__1___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4; lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f(lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_processPostponed_loop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__6___boxed(lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); @@ -719,11 +725,11 @@ static lean_object* l_Lean_Meta_Grind_preprocessPattern___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__3(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instBEqTheoremKind___closed__1; lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__10; static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_canBeSynthesized___spec__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_processPostponed_loop___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqOrigin__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ScopedEnvExtension_add___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindEqAttr___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -738,7 +744,6 @@ static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toAttribute(uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkOffsetPattern(lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___closed__1; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Origin_key(lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -763,7 +768,6 @@ LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_G uint8_t l_Lean_Exception_isRuntime(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchEqTheoremCore___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__16___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addEMatchEqTheorem(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_HeadIndex_hash(lean_object*); @@ -772,6 +776,7 @@ static lean_object* l_Lean_Meta_Grind_EMatchTheorems_insert___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEMatchTheorems___rarg___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_ppPattern___closed__6; lean_object* l_Lean_Meta_mkConstWithFreshMVarLevels(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10; static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2___closed__5; static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__3___closed__2; uint64_t l___private_Lean_Meta_Basic_0__Lean_Meta_Config_toKey(lean_object*); @@ -779,19 +784,15 @@ lean_object* l_Lean_Meta_Grind_unfoldReducible___lambda__2(lean_object*, lean_ob static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_ppParamsAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__8(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_groundPattern_x3f___boxed(lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2(lean_object*, lean_object*, size_t, size_t); lean_object* l_Lean_MessageData_ofName(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__14(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppPattern___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_dontCare___closed__1; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__13(lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instInhabitedEMatchTheorem___closed__2; static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__5; @@ -802,6 +803,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); size_t lean_usize_land(size_t, size_t); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isOffsetPattern_x3f___lambda__2(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_saveSymbol___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__4; @@ -5873,6 +5875,188 @@ x_3 = lean_box(x_2); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitWhileForbidden(lean_object* x_1) { +_start: +{ +lean_object* x_2; uint8_t x_3; +lean_inc(x_1); +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) +{ +lean_object* x_4; lean_object* x_5; +lean_dec(x_2); +x_4 = lean_box(0); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_6 = l_Lean_Expr_appArg(x_2, lean_box(0)); +x_7 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_8 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__12; +x_9 = l_Lean_Expr_isConstOf(x_7, x_8); +if (x_9 == 0) +{ +uint8_t x_10; +x_10 = l_Lean_Expr_isApp(x_7); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; +lean_dec(x_7); +lean_dec(x_6); +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); +return x_12; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = l_Lean_Expr_appArg(x_7, lean_box(0)); +x_14 = l_Lean_Expr_appFnCleanup(x_7, lean_box(0)); +x_15 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__6; +x_16 = l_Lean_Expr_isConstOf(x_14, x_15); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__10; +x_18 = l_Lean_Expr_isConstOf(x_14, x_17); +if (x_18 == 0) +{ +lean_object* x_19; uint8_t x_20; +x_19 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__8; +x_20 = l_Lean_Expr_isConstOf(x_14, x_19); +if (x_20 == 0) +{ +uint8_t x_21; +x_21 = l_Lean_Expr_isApp(x_14); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_6); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_1); +lean_ctor_set(x_23, 1, x_22); +return x_23; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_24 = l_Lean_Expr_appArg(x_14, lean_box(0)); +x_25 = l_Lean_Expr_appFnCleanup(x_14, lean_box(0)); +x_26 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__2; +x_27 = l_Lean_Expr_isConstOf(x_25, x_26); +if (x_27 == 0) +{ +uint8_t x_28; +lean_dec(x_13); +x_28 = l_Lean_Expr_isApp(x_25); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_6); +x_29 = lean_box(0); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_1); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); +x_32 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_forbiddenDeclNames___closed__4; +x_33 = l_Lean_Expr_isConstOf(x_31, x_32); +lean_dec(x_31); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_24); +lean_dec(x_6); +x_34 = lean_box(0); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_1); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_1); +x_36 = l_Lean_Meta_Grind_splitWhileForbidden(x_24); +x_37 = l_Lean_Meta_Grind_splitWhileForbidden(x_6); +x_38 = l_List_appendTR___rarg(x_36, x_37); +return x_38; +} +} +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_1); +x_39 = l_Lean_Meta_Grind_splitWhileForbidden(x_13); +x_40 = l_Lean_Meta_Grind_splitWhileForbidden(x_6); +x_41 = l_List_appendTR___rarg(x_39, x_40); +return x_41; +} +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +lean_dec(x_14); +lean_dec(x_1); +x_42 = l_Lean_Meta_Grind_splitWhileForbidden(x_13); +x_43 = l_Lean_Meta_Grind_splitWhileForbidden(x_6); +x_44 = l_List_appendTR___rarg(x_42, x_43); +return x_44; +} +} +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +lean_dec(x_14); +lean_dec(x_1); +x_45 = l_Lean_Meta_Grind_splitWhileForbidden(x_13); +x_46 = l_Lean_Meta_Grind_splitWhileForbidden(x_6); +x_47 = l_List_appendTR___rarg(x_45, x_46); +return x_47; +} +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_dec(x_14); +lean_dec(x_1); +x_48 = l_Lean_Meta_Grind_splitWhileForbidden(x_13); +x_49 = l_Lean_Meta_Grind_splitWhileForbidden(x_6); +x_50 = l_List_appendTR___rarg(x_48, x_49); +return x_50; +} +} +} +else +{ +lean_dec(x_7); +lean_dec(x_1); +x_1 = x_6; +goto _start; +} +} +} +} static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_dontCare___closed__1() { _start: { @@ -10218,7 +10402,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Le lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__1; x_2 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__6; -x_3 = lean_unsigned_to_nat(267u); +x_3 = lean_unsigned_to_nat(299u); x_4 = lean_unsigned_to_nat(2u); x_5 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_NormalizePattern_go___lambda__1___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -18722,7 +18906,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Le lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__1; x_2 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3___closed__3; -x_3 = lean_unsigned_to_nat(358u); +x_3 = lean_unsigned_to_nat(390u); x_4 = lean_unsigned_to_nat(4u); x_5 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_checkCoverage___lambda__3___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -21286,276 +21470,258 @@ uint8_t x_14; x_14 = !lean_is_exclusive(x_13); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_array_get_size(x_3); -x_17 = lean_expr_abstract(x_15, x_3); +x_16 = lean_expr_abstract(x_15, x_3); lean_dec(x_15); -x_18 = lean_box(0); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -lean_ctor_set(x_4, 1, x_19); -lean_ctor_set(x_4, 0, x_16); +x_17 = l_Lean_Meta_Grind_splitWhileForbidden(x_16); +x_18 = lean_array_get_size(x_3); +lean_ctor_set(x_4, 1, x_17); +lean_ctor_set(x_4, 0, x_18); lean_ctor_set(x_13, 0, x_4); return x_13; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_20 = lean_ctor_get(x_13, 0); -x_21 = lean_ctor_get(x_13, 1); -lean_inc(x_21); +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_19 = lean_ctor_get(x_13, 0); +x_20 = lean_ctor_get(x_13, 1); lean_inc(x_20); +lean_inc(x_19); lean_dec(x_13); -x_22 = lean_array_get_size(x_3); -x_23 = lean_expr_abstract(x_20, x_3); -lean_dec(x_20); -x_24 = lean_box(0); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -lean_ctor_set(x_4, 1, x_25); -lean_ctor_set(x_4, 0, x_22); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_4); -lean_ctor_set(x_26, 1, x_21); -return x_26; +x_21 = lean_expr_abstract(x_19, x_3); +lean_dec(x_19); +x_22 = l_Lean_Meta_Grind_splitWhileForbidden(x_21); +x_23 = lean_array_get_size(x_3); +lean_ctor_set(x_4, 1, x_22); +lean_ctor_set(x_4, 0, x_23); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_4); +lean_ctor_set(x_24, 1, x_20); +return x_24; } } else { -uint8_t x_27; +uint8_t x_25; lean_free_object(x_4); -x_27 = !lean_is_exclusive(x_13); -if (x_27 == 0) +x_25 = !lean_is_exclusive(x_13); +if (x_25 == 0) { return x_13; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_13, 0); -x_29 = lean_ctor_get(x_13, 1); -lean_inc(x_29); -lean_inc(x_28); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_13, 0); +x_27 = lean_ctor_get(x_13, 1); +lean_inc(x_27); +lean_inc(x_26); lean_dec(x_13); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } else { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_4, 1); -lean_inc(x_31); +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_4, 1); +lean_inc(x_29); lean_dec(x_4); -x_32 = l_Lean_Meta_Grind_preprocessPattern(x_31, x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_32) == 0) +x_30 = l_Lean_Meta_Grind_preprocessPattern(x_29, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_30) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_35 = x_32; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_33 = x_30; } else { - lean_dec_ref(x_32); - x_35 = lean_box(0); + lean_dec_ref(x_30); + x_33 = lean_box(0); } +x_34 = lean_expr_abstract(x_31, x_3); +lean_dec(x_31); +x_35 = l_Lean_Meta_Grind_splitWhileForbidden(x_34); x_36 = lean_array_get_size(x_3); -x_37 = lean_expr_abstract(x_33, x_3); -lean_dec(x_33); -x_38 = lean_box(0); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_36); -lean_ctor_set(x_40, 1, x_39); -if (lean_is_scalar(x_35)) { - x_41 = lean_alloc_ctor(0, 2, 0); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_35); +if (lean_is_scalar(x_33)) { + x_38 = lean_alloc_ctor(0, 2, 0); } else { - x_41 = x_35; + x_38 = x_33; } -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_34); -return x_41; +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_32); +return x_38; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_42 = lean_ctor_get(x_32, 0); -lean_inc(x_42); -x_43 = lean_ctor_get(x_32, 1); -lean_inc(x_43); -if (lean_is_exclusive(x_32)) { - lean_ctor_release(x_32, 0); - lean_ctor_release(x_32, 1); - x_44 = x_32; +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_39 = lean_ctor_get(x_30, 0); +lean_inc(x_39); +x_40 = lean_ctor_get(x_30, 1); +lean_inc(x_40); +if (lean_is_exclusive(x_30)) { + lean_ctor_release(x_30, 0); + lean_ctor_release(x_30, 1); + x_41 = x_30; } else { - lean_dec_ref(x_32); - x_44 = lean_box(0); + lean_dec_ref(x_30); + x_41 = lean_box(0); } -if (lean_is_scalar(x_44)) { - x_45 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_41)) { + x_42 = lean_alloc_ctor(1, 2, 0); } else { - x_45 = x_44; + x_42 = x_41; } -lean_ctor_set(x_45, 0, x_42); -lean_ctor_set(x_45, 1, x_43); -return x_45; +lean_ctor_set(x_42, 0, x_39); +lean_ctor_set(x_42, 1, x_40); +return x_42; } } } else { -uint8_t x_46; -x_46 = !lean_is_exclusive(x_4); -if (x_46 == 0) +uint8_t x_43; +x_43 = !lean_is_exclusive(x_4); +if (x_43 == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_4, 0); -x_48 = lean_ctor_get(x_4, 1); -lean_dec(x_48); -x_49 = l_Lean_Meta_Grind_preprocessPattern(x_47, x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_49) == 0) +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_4, 0); +x_45 = lean_ctor_get(x_4, 1); +lean_dec(x_45); +x_46 = l_Lean_Meta_Grind_preprocessPattern(x_44, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_46) == 0) { -uint8_t x_50; -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) +uint8_t x_47; +x_47 = !lean_is_exclusive(x_46); +if (x_47 == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_51 = lean_ctor_get(x_49, 0); -x_52 = lean_array_get_size(x_3); -x_53 = lean_expr_abstract(x_51, x_3); -lean_dec(x_51); -x_54 = lean_box(0); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -lean_ctor_set(x_4, 1, x_55); -lean_ctor_set(x_4, 0, x_52); -lean_ctor_set(x_49, 0, x_4); -return x_49; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_48 = lean_ctor_get(x_46, 0); +x_49 = lean_expr_abstract(x_48, x_3); +lean_dec(x_48); +x_50 = l_Lean_Meta_Grind_splitWhileForbidden(x_49); +x_51 = lean_array_get_size(x_3); +lean_ctor_set(x_4, 1, x_50); +lean_ctor_set(x_4, 0, x_51); +lean_ctor_set(x_46, 0, x_4); +return x_46; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_56 = lean_ctor_get(x_49, 0); -x_57 = lean_ctor_get(x_49, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_49); -x_58 = lean_array_get_size(x_3); -x_59 = lean_expr_abstract(x_56, x_3); -lean_dec(x_56); -x_60 = lean_box(0); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set(x_4, 1, x_61); -lean_ctor_set(x_4, 0, x_58); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_4); -lean_ctor_set(x_62, 1, x_57); -return x_62; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_52 = lean_ctor_get(x_46, 0); +x_53 = lean_ctor_get(x_46, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_46); +x_54 = lean_expr_abstract(x_52, x_3); +lean_dec(x_52); +x_55 = l_Lean_Meta_Grind_splitWhileForbidden(x_54); +x_56 = lean_array_get_size(x_3); +lean_ctor_set(x_4, 1, x_55); +lean_ctor_set(x_4, 0, x_56); +x_57 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_4); +lean_ctor_set(x_57, 1, x_53); +return x_57; } } else { -uint8_t x_63; +uint8_t x_58; lean_free_object(x_4); -x_63 = !lean_is_exclusive(x_49); -if (x_63 == 0) +x_58 = !lean_is_exclusive(x_46); +if (x_58 == 0) { -return x_49; +return x_46; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_49, 0); -x_65 = lean_ctor_get(x_49, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_49); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_46, 0); +x_60 = lean_ctor_get(x_46, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_46); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } else { -lean_object* x_67; lean_object* x_68; -x_67 = lean_ctor_get(x_4, 0); -lean_inc(x_67); +lean_object* x_62; lean_object* x_63; +x_62 = lean_ctor_get(x_4, 0); +lean_inc(x_62); lean_dec(x_4); -x_68 = l_Lean_Meta_Grind_preprocessPattern(x_67, x_2, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_68) == 0) +x_63 = l_Lean_Meta_Grind_preprocessPattern(x_62, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_63) == 0) { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_71 = x_68; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +x_65 = lean_ctor_get(x_63, 1); +lean_inc(x_65); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_66 = x_63; } else { - lean_dec_ref(x_68); - x_71 = lean_box(0); + lean_dec_ref(x_63); + x_66 = lean_box(0); } -x_72 = lean_array_get_size(x_3); -x_73 = lean_expr_abstract(x_69, x_3); -lean_dec(x_69); -x_74 = lean_box(0); -x_75 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_72); -lean_ctor_set(x_76, 1, x_75); -if (lean_is_scalar(x_71)) { - x_77 = lean_alloc_ctor(0, 2, 0); +x_67 = lean_expr_abstract(x_64, x_3); +lean_dec(x_64); +x_68 = l_Lean_Meta_Grind_splitWhileForbidden(x_67); +x_69 = lean_array_get_size(x_3); +x_70 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_68); +if (lean_is_scalar(x_66)) { + x_71 = lean_alloc_ctor(0, 2, 0); } else { - x_77 = x_71; + x_71 = x_66; } -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_70); -return x_77; +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_65); +return x_71; } else { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_78 = lean_ctor_get(x_68, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_68, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_80 = x_68; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_72 = lean_ctor_get(x_63, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_63, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_74 = x_63; } else { - lean_dec_ref(x_68); - x_80 = lean_box(0); + lean_dec_ref(x_63); + x_74 = lean_box(0); } -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(1, 2, 0); } else { - x_81 = x_80; + x_75 = x_74; } -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_79); -return x_81; +lean_ctor_set(x_75, 0, x_72); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } } @@ -22432,7 +22598,7 @@ lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx(uint8_t x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_toCtorIdx(uint8_t x_1) { _start: { switch (x_1) { @@ -22475,57 +22641,57 @@ return x_7; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_toCtorIdx___boxed(lean_object* x_1) { _start: { uint8_t x_2; lean_object* x_3; x_2 = lean_unbox(x_1); lean_dec(x_1); -x_3 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx(x_2); +x_3 = l_Lean_Meta_Grind_TheoremKind_toCtorIdx(x_2); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(lean_object* x_1) { _start: { lean_inc(x_1); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed), 1, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed), 1, 0); return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1; +x_4 = l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1; return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed), 3, 0); +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed), 3, 0); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(x_1); +x_2 = l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___lambda__1(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -22533,7 +22699,7 @@ x_4 = lean_unbox(x_1); lean_dec(x_1); x_5 = lean_unbox(x_2); lean_dec(x_2); -x_6 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg(x_4, x_5, x_3); +x_6 = l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg(x_4, x_5, x_3); return x_6; } } @@ -22545,19 +22711,19 @@ x_1 = 0; return x_1; } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(uint8_t x_1, uint8_t x_2) { +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(uint8_t x_1, uint8_t x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx(x_1); -x_4 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_toCtorIdx(x_2); +x_3 = l_Lean_Meta_Grind_TheoremKind_toCtorIdx(x_1); +x_4 = l_Lean_Meta_Grind_TheoremKind_toCtorIdx(x_2); x_5 = lean_nat_dec_eq(x_3, x_4); lean_dec(x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853____boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -22565,7 +22731,7 @@ x_3 = lean_unbox(x_1); lean_dec(x_1); x_4 = lean_unbox(x_2); lean_dec(x_2); -x_5 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_3, x_4); +x_5 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_3, x_4); x_6 = lean_box(x_5); return x_6; } @@ -22574,7 +22740,7 @@ static lean_object* _init_l_Lean_Meta_Grind_instBEqTheoremKind___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853____boxed), 2, 0); return x_1; } } @@ -22717,7 +22883,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Le lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__1; x_2 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_explainFailure___closed__3; -x_3 = lean_unsigned_to_nat(517u); +x_3 = lean_unsigned_to_nat(550u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -26380,7 +26546,7 @@ static lean_object* _init_l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__1; x_2 = l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f___lambda__2___closed__1; -x_3 = lean_unsigned_to_nat(617u); +x_3 = lean_unsigned_to_nat(650u); x_4 = lean_unsigned_to_nat(13u); x_5 = l_Lean_Meta_Grind_EMatchTheorems_insert___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -26751,12 +26917,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(lean_obje { uint8_t x_10; uint8_t x_11; x_10 = 0; -x_11 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_4, x_10); +x_11 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_4, x_10); if (x_11 == 0) { uint8_t x_12; uint8_t x_13; x_12 = 1; -x_13 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_4, x_12); +x_13 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_4, x_12); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; @@ -27817,17 +27983,17 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lea { uint8_t x_9; uint8_t x_10; x_9 = 0; -x_10 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_3, x_9); +x_10 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_3, x_9); if (x_10 == 0) { uint8_t x_11; uint8_t x_12; x_11 = 1; -x_12 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_3, x_11); +x_12 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_3, x_11); if (x_12 == 0) { uint8_t x_13; uint8_t x_14; x_13 = 2; -x_14 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6540_(x_3, x_13); +x_14 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_beqTheoremKind____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_6853_(x_3, x_13); if (x_14 == 0) { lean_object* x_15; @@ -28100,7 +28266,7 @@ x_11 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGr return x_11; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -28124,7 +28290,7 @@ return x_4; } } } -LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { +LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4) { _start: { uint8_t x_5; @@ -28163,7 +28329,7 @@ return x_13; } } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1() { _start: { uint8_t x_1; uint8_t x_2; uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; @@ -28193,16 +28359,16 @@ lean_ctor_set_uint8(x_6, 16, x_2); return x_6; } } -static uint64_t _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__2() { +static uint64_t _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__2() { _start: { lean_object* x_1; uint64_t x_2; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1; x_2 = l___private_Lean_Meta_Basic_0__Lean_Meta_Config_toKey(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -28211,23 +28377,23 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5() { _start: { size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 5; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3; x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_2); @@ -28238,28 +28404,28 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1___closed__2; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint64_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_1 = lean_box(0); x_2 = lean_box(0); -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__2; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__2; x_5 = 0; -x_6 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6; +x_6 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6; x_7 = l_Lean_Meta_Grind_NormalizePattern_main___closed__1; x_8 = lean_unsigned_to_nat(0u); x_9 = lean_alloc_ctor(0, 7, 11); @@ -28277,7 +28443,7 @@ lean_ctor_set_uint8(x_9, sizeof(void*)*7 + 10, x_5); return x_9; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -28296,7 +28462,7 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; @@ -28309,15 +28475,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8; x_3 = l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5; -x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5; +x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -28327,19 +28493,19 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_7 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_getKind(x_2); -x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10; +x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10; x_9 = lean_st_mk_ref(x_8, x_6); x_10 = lean_ctor_get(x_9, 0); lean_inc(x_10); x_11 = lean_ctor_get(x_9, 1); lean_inc(x_11); lean_dec(x_9); -x_12 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7; +x_12 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7; lean_inc(x_10); x_13 = l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr(x_1, x_3, x_7, x_12, x_10, x_4, x_5, x_11); if (lean_obj_tag(x_13) == 0) @@ -28398,7 +28564,7 @@ return x_24; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint8_t x_5; @@ -28425,13 +28591,13 @@ size_t x_7; size_t x_8; lean_object* x_9; x_7 = 0; x_8 = lean_usize_of_nat(x_3); lean_dec(x_3); -x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1(x_1, x_7, x_8, x_2); +x_9 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1(x_1, x_7, x_8, x_2); return x_9; } } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -28449,7 +28615,7 @@ x_14 = lean_ctor_get(x_10, 1); x_15 = lean_ctor_get(x_12, 0); x_16 = lean_ctor_get(x_12, 4); lean_dec(x_16); -x_17 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2___boxed), 2, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2___boxed), 2, 1); lean_closure_set(x_17, 0, x_1); x_18 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_19 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_18, x_15, x_17); @@ -28558,7 +28724,7 @@ lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_dec(x_12); -x_52 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2___boxed), 2, 1); +x_52 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2___boxed), 2, 1); lean_closure_set(x_52, 0, x_1); x_53 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_54 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_53, x_45, x_52); @@ -28671,7 +28837,7 @@ if (lean_is_exclusive(x_72)) { lean_dec_ref(x_72); x_81 = lean_box(0); } -x_82 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2___boxed), 2, 1); +x_82 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2___boxed), 2, 1); lean_closure_set(x_82, 0, x_1); x_83 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_84 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_83, x_74, x_82); @@ -28754,7 +28920,7 @@ return x_102; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__4(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__4(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; @@ -28764,7 +28930,7 @@ x_4 = l_Lean_Meta_Grind_EMatchTheorems_erase(x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; uint8_t x_11; @@ -28782,7 +28948,7 @@ x_14 = lean_ctor_get(x_10, 1); x_15 = lean_ctor_get(x_12, 0); x_16 = lean_ctor_get(x_12, 4); lean_dec(x_16); -x_17 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__4), 2, 1); +x_17 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__4), 2, 1); lean_closure_set(x_17, 0, x_1); x_18 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_19 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_18, x_15, x_17); @@ -28891,7 +29057,7 @@ lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_dec(x_12); -x_52 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__4), 2, 1); +x_52 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__4), 2, 1); lean_closure_set(x_52, 0, x_1); x_53 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_54 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_53, x_45, x_52); @@ -29004,7 +29170,7 @@ if (lean_is_exclusive(x_72)) { lean_dec_ref(x_72); x_81 = lean_box(0); } -x_82 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__4), 2, 1); +x_82 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__4), 2, 1); lean_closure_set(x_82, 0, x_1); x_83 = l_Lean_Meta_Grind_addEMatchTheorem___closed__1; x_84 = l_Lean_ScopedEnvExtension_modifyState___rarg(x_83, x_74, x_82); @@ -29087,7 +29253,7 @@ return x_102; } } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1() { _start: { lean_object* x_1; @@ -29095,16 +29261,16 @@ x_1 = lean_mk_string_unchecked("` is not marked with the `[grind]` attribute", 4 return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_27; lean_object* x_28; @@ -29114,18 +29280,18 @@ x_6 = l_Lean_Meta_Grind_mkEMatchTheoremCore___lambda__2___closed__4; x_7 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); -x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2; +x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2; x_9 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_9, 0, x_7); lean_ctor_set(x_9, 1, x_8); -x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10; +x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10; x_11 = lean_st_mk_ref(x_10, x_4); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_27 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7; +x_27 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7; lean_inc(x_1); x_28 = l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(x_1, x_27, x_12, x_2, x_3, x_13); if (lean_obj_tag(x_28) == 0) @@ -29213,7 +29379,7 @@ lean_dec(x_9); x_52 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1___closed__2; x_53 = l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2; x_54 = lean_box(0); -x_55 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3(x_41, x_52, x_53, x_54, x_27, x_12, x_2, x_3, x_44); +x_55 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3(x_41, x_52, x_53, x_54, x_27, x_12, x_2, x_3, x_44); lean_dec(x_3); lean_dec(x_2); x_14 = x_55; @@ -29225,7 +29391,7 @@ size_t x_56; size_t x_57; uint8_t x_58; x_56 = 0; x_57 = lean_usize_of_nat(x_49); lean_dec(x_49); -x_58 = l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2(x_48, x_41, x_56, x_57); +x_58 = l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2(x_48, x_41, x_56, x_57); if (x_58 == 0) { lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; @@ -29233,7 +29399,7 @@ lean_dec(x_9); x_59 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1___closed__2; x_60 = l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2; x_61 = lean_box(0); -x_62 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3(x_41, x_59, x_60, x_61, x_27, x_12, x_2, x_3, x_44); +x_62 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3(x_41, x_59, x_60, x_61, x_27, x_12, x_2, x_3, x_44); lean_dec(x_3); lean_dec(x_2); x_14 = x_62; @@ -29352,7 +29518,7 @@ lean_dec(x_9); x_86 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1___closed__2; x_87 = l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2; x_88 = lean_box(0); -x_89 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5(x_1, x_86, x_87, x_88, x_27, x_12, x_2, x_3, x_74); +x_89 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5(x_1, x_86, x_87, x_88, x_27, x_12, x_2, x_3, x_74); lean_dec(x_3); lean_dec(x_2); x_90 = lean_ctor_get(x_89, 0); @@ -29471,7 +29637,7 @@ return x_25; } } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29481,27 +29647,27 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1; x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2; x_2 = l_Lean_Meta_Grind_mkOffsetPattern___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4() { _start: { lean_object* x_1; @@ -29509,17 +29675,17 @@ x_1 = lean_mk_string_unchecked("initFn", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6() { _start: { lean_object* x_1; @@ -29527,67 +29693,67 @@ x_1 = lean_mk_string_unchecked("_@", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7; x_2 = l_Lean_Meta_Grind_mkOffsetPattern___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8; x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__4; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9; x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10; x_2 = l_Lean_Meta_Grind_mkOffsetPattern___closed__2; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11; x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_1666____closed__9; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13() { _start: { lean_object* x_1; @@ -29595,27 +29761,27 @@ x_1 = lean_mk_string_unchecked("_hyg", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14; -x_2 = lean_unsigned_to_nat(10279u); +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14; +x_2 = lean_unsigned_to_nat(10592u); x_3 = l_Lean_Name_num___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; @@ -29625,7 +29791,7 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17() { _start: { lean_object* x_1; @@ -29633,13 +29799,13 @@ x_1 = lean_mk_string_unchecked("The `[grind]` attribute is used to annotate decl return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint8_t x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17; x_4 = 1; x_5 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_5, 0, x_1); @@ -29649,29 +29815,29 @@ lean_ctor_set_uint8(x_5, sizeof(void*)*3, x_4); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___boxed), 6, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___boxed), 6, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6), 4, 0); +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6), 4, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20; x_4 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -29679,16 +29845,16 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21; x_3 = l_Lean_registerBuiltinAttribute(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -29696,12 +29862,12 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__1(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__1(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; uint8_t x_7; lean_object* x_8; @@ -29709,37 +29875,37 @@ x_5 = lean_unbox_usize(x_3); lean_dec(x_3); x_6 = lean_unbox_usize(x_4); lean_dec(x_4); -x_7 = l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____spec__2(x_1, x_2, x_5, x_6); +x_7 = l_Array_anyMUnsafe_any___at_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____spec__2(x_1, x_2, x_5, x_6); lean_dec(x_2); x_8 = lean_box(x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); -x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); +x_8 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); lean_dec(x_2); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__2(x_1, x_2); +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__2(x_1, x_2); lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -29748,11 +29914,11 @@ lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { lean_object* x_10; -x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_10 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -30149,8 +30315,8 @@ l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___ lean_mark_persistent(l_Lean_ScopedEnvExtension_add___at_Lean_Meta_Grind_addEMatchTheorem___spec__1___closed__2); l_Lean_Meta_Grind_addEMatchTheorem___closed__1 = _init_l_Lean_Meta_Grind_addEMatchTheorem___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_addEMatchTheorem___closed__1); -l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1); +l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1 = _init_l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_TheoremKind_noConfusion___rarg___closed__1); l_Lean_Meta_Grind_instInhabitedTheoremKind = _init_l_Lean_Meta_Grind_instInhabitedTheoremKind(); l_Lean_Meta_Grind_instBEqTheoremKind___closed__1 = _init_l_Lean_Meta_Grind_instBEqTheoremKind___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_instBEqTheoremKind___closed__1); @@ -30271,72 +30437,72 @@ l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__7); l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__8(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_EMatchTheorem_0__Lean_Meta_Grind_addGrindAttr___closed__8); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__1); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__2(); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__3); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__4); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__5); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__6); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__7); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__8); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__9); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__1___closed__10); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__1); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____lambda__6___closed__2); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__1); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__2); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__3); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__4); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__5); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__6); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__7); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__8); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__9); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__10); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__11); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__12); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__13); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__14); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__15); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__16); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__17); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__18); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__19); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__20); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279____closed__21); -if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10279_(lean_io_mk_world()); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__1); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__2(); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__3); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__4); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__5); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__6); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__7); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__8); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__9); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__1___closed__10); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__1); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____lambda__6___closed__2); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__1); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__2); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__3); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__4); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__5); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__6); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__7); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__8); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__9); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__10); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__11); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__12); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__13); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__14); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__15); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__16); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__17); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__18); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__19); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__20); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592____closed__21); +if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_EMatchTheorem___hyg_10592_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/ENodeKey.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/ENodeKey.c new file mode 100644 index 000000000000..275c75d38c92 --- /dev/null +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/ENodeKey.c @@ -0,0 +1,138 @@ +// Lean compiler output +// Module: Lean.Meta.Tactic.Grind.ENodeKey +// Imports: Lean.Expr +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqENodeKey(lean_object*, lean_object*); +uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr_unsafe__1___boxed(lean_object*, lean_object*); +size_t lean_ptr_addr(lean_object*); +uint64_t lean_usize_to_uint64(size_t); +LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqENodeKey___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1___boxed(lean_object*); +LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey___boxed(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +size_t x_3; size_t x_4; uint8_t x_5; +x_3 = lean_ptr_addr(x_1); +x_4 = lean_ptr_addr(x_2); +x_5 = lean_usize_dec_eq(x_3, x_4); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr_unsafe__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_Meta_Grind_isSameExpr(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object* x_1) { +_start: +{ +size_t x_2; uint64_t x_3; +x_2 = lean_ptr_addr(x_1); +x_3 = lean_usize_to_uint64(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1___boxed(lean_object* x_1) { +_start: +{ +uint64_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_1); +lean_dec(x_1); +x_3 = lean_box_uint64(x_2); +return x_3; +} +} +LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey(lean_object* x_1) { +_start: +{ +uint64_t x_2; +x_2 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey___boxed(lean_object* x_1) { +_start: +{ +uint64_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_instHashableENodeKey(x_1); +lean_dec(x_1); +x_3 = lean_box_uint64(x_2); +return x_3; +} +} +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqENodeKey(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; +x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqENodeKey___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +uint8_t x_3; lean_object* x_4; +x_3 = l_Lean_Meta_Grind_instBEqENodeKey(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; +} +} +lean_object* initialize_Lean_Expr(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_ENodeKey(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Lean_Expr(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/ForallProp.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/ForallProp.c index 05ee49a5c60f..2d626b9d699e 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/ForallProp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/ForallProp.c @@ -22,7 +22,8 @@ static lean_object* l_Lean_Meta_Grind_propagateForallPropDown___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___lambda__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Exception_isInterrupt(lean_object*); lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); @@ -31,25 +32,27 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_G static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1; lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__2; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___closed__4; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__6; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2; -lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_activateTheorem(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropDown___closed__3; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__2; @@ -76,8 +79,9 @@ lean_object* l_Lean_mkNot(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__3; lean_object* l_Lean_Meta_Grind_updateLastTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__8; +static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__7; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropDown___closed__8; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__10; lean_object* l_Lean_MessageData_ofExpr(lean_object*); @@ -88,11 +92,9 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_M static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3; lean_object* l_Lean_Meta_Grind_addNewFact(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7; uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8; lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__4; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); @@ -105,11 +107,11 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_M static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1; uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_mkOfEqTrueCore(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__2; static lean_object* l_Lean_Meta_Grind_propagateForallPropDown___closed__9; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___closed__2; lean_object* lean_array_mk(lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; lean_object* l_Lean_Meta_Grind_isEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_pushEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -125,14 +127,15 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_M static lean_object* l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__1; lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Exception_isRuntime(lean_object*); lean_object* l_Lean_Expr_lam___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_Lean_mkApp5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__2; static lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5; lean_object* lean_expr_instantiate1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateForallPropDown___closed__10; static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp_propagateImpliesUp___lambda__1___closed__1() { _start: @@ -724,65 +727,73 @@ x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3() { _start: { -lean_object* x_18; -lean_inc(x_16); +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +lean_object* x_17; lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); -x_18 = l_Lean_Meta_Simp_Result_getProof(x_1, x_13, x_14, x_15, x_16, x_17); -if (lean_obj_tag(x_18) == 0) +lean_inc(x_12); +x_17 = l_Lean_Meta_Simp_Result_getProof(x_1, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_19 = lean_ctor_get(x_18, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2; -x_22 = l_Lean_Expr_const___override(x_21, x_2); -lean_inc(x_5); -x_23 = l_Lean_mkApp5(x_22, x_3, x_4, x_5, x_6, x_19); -x_24 = 0; -x_25 = l_Lean_Meta_Grind_pushEqCore(x_7, x_5, x_23, x_24, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_20); -lean_dec(x_16); +lean_dec(x_17); +x_20 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3; +lean_inc(x_4); +x_21 = l_Lean_mkApp5(x_20, x_2, x_3, x_4, x_5, x_18); +x_22 = 0; +x_23 = l_Lean_Meta_Grind_pushEqCore(x_6, x_4, x_21, x_22, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -return x_25; +lean_dec(x_12); +return x_23; } else { -uint8_t x_26; -lean_dec(x_16); +uint8_t x_24; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); -lean_dec(x_7); +lean_dec(x_12); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_26 = !lean_is_exclusive(x_18); -if (x_26 == 0) +x_24 = !lean_is_exclusive(x_17); +if (x_24 == 0) { -return x_18; +return x_17; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_18, 0); -x_28 = lean_ctor_get(x_18, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_18); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_17, 0); +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_17); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } } } @@ -791,48 +802,20 @@ static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("of_eq_true", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__4() { -_start: -{ -lean_object* x_1; x_1 = lean_mk_string_unchecked("q': ", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__4; +x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -840,16 +823,16 @@ x_1 = lean_mk_string_unchecked(" for", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7() { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; +x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8() { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5() { _start: { lean_object* x_1; @@ -857,11 +840,11 @@ x_1 = lean_mk_string_unchecked("", 0, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9() { +static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8; +x_1 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } @@ -882,47 +865,46 @@ lean_inc(x_1); x_17 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); if (lean_obj_tag(x_17) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); lean_dec(x_17); -x_20 = lean_box(0); -x_21 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3; lean_inc(x_18); lean_inc(x_1); -x_22 = l_Lean_mkAppB(x_21, x_1, x_18); -x_23 = lean_expr_instantiate1(x_2, x_22); -lean_dec(x_22); +x_20 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_18); +x_21 = lean_expr_instantiate1(x_2, x_20); +lean_dec(x_20); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_10); -x_24 = l_Lean_Meta_Grind_simp(x_23, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); -if (lean_obj_tag(x_24) == 0) +x_22 = l_Lean_Meta_Grind_simp(x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); lean_inc(x_1); -x_27 = l_Lean_Expr_lam___override(x_3, x_1, x_2, x_4); -x_28 = lean_ctor_get(x_25, 0); -lean_inc(x_28); +x_25 = l_Lean_Expr_lam___override(x_3, x_1, x_2, x_4); +x_26 = lean_ctor_get(x_23, 0); +lean_inc(x_26); lean_inc(x_5); -x_29 = l_Lean_Meta_Grind_getGeneration(x_5, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_26); -if (lean_obj_tag(x_29) == 0) +x_27 = l_Lean_Meta_Grind_getGeneration(x_5, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_24); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_box(0); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -931,92 +913,92 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_28); -x_32 = l_Lean_Meta_Grind_internalize(x_28, x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_31); -if (lean_obj_tag(x_32) == 0) +lean_inc(x_26); +x_31 = l_Lean_Meta_Grind_internalize(x_26, x_28, x_30, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_29); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = lean_ctor_get(x_32, 1); -lean_inc(x_33); -lean_dec(x_32); +lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_32 = lean_ctor_get(x_31, 1); +lean_inc(x_32); +lean_dec(x_31); lean_inc(x_6); -x_34 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_33); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_unbox(x_35); -lean_dec(x_35); -if (x_36 == 0) +x_33 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_32); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_unbox(x_34); +lean_dec(x_34); +if (x_35 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_dec(x_6); -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -lean_dec(x_34); -x_38 = lean_box(0); -x_39 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_25, x_20, x_1, x_27, x_28, x_18, x_5, x_38, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_37); +x_36 = lean_ctor_get(x_33, 1); +lean_inc(x_36); +lean_dec(x_33); +x_37 = lean_box(0); +x_38 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_23, x_1, x_25, x_26, x_18, x_5, x_37, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_36); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_39; +return x_38; } else { -uint8_t x_40; -x_40 = !lean_is_exclusive(x_34); -if (x_40 == 0) +uint8_t x_39; +x_39 = !lean_is_exclusive(x_33); +if (x_39 == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_34, 1); -x_42 = lean_ctor_get(x_34, 0); -lean_dec(x_42); -x_43 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_41); -if (lean_obj_tag(x_43) == 0) +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_33, 1); +x_41 = lean_ctor_get(x_33, 0); +lean_dec(x_41); +x_42 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_40); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_44 = lean_ctor_get(x_43, 1); -lean_inc(x_44); -lean_dec(x_43); -lean_inc(x_28); -x_45 = l_Lean_MessageData_ofExpr(x_28); -x_46 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5; -lean_ctor_set_tag(x_34, 7); -lean_ctor_set(x_34, 1, x_45); -lean_ctor_set(x_34, 0, x_46); -x_47 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7; -x_48 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_48, 0, x_34); -lean_ctor_set(x_48, 1, x_47); +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_43 = lean_ctor_get(x_42, 1); +lean_inc(x_43); +lean_dec(x_42); +lean_inc(x_26); +x_44 = l_Lean_MessageData_ofExpr(x_26); +x_45 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2; +lean_ctor_set_tag(x_33, 7); +lean_ctor_set(x_33, 1, x_44); +lean_ctor_set(x_33, 0, x_45); +x_46 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__4; +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_33); +lean_ctor_set(x_47, 1, x_46); lean_inc(x_5); -x_49 = l_Lean_indentExpr(x_5); -x_50 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -x_51 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; -x_52 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -x_53 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_6, x_52, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_44); -x_54 = lean_ctor_get(x_53, 0); +x_48 = l_Lean_indentExpr(x_5); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +x_50 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +x_52 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_6, x_51, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); +x_53 = lean_ctor_get(x_52, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_52, 1); lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_25, x_20, x_1, x_27, x_28, x_18, x_5, x_54, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_55); +lean_dec(x_52); +x_55 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_23, x_1, x_25, x_26, x_18, x_5, x_53, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_54); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_54); -return x_56; +lean_dec(x_53); +return x_55; } else { -uint8_t x_57; -lean_free_object(x_34); -lean_dec(x_28); -lean_dec(x_27); +uint8_t x_56; +lean_free_object(x_33); +lean_dec(x_26); lean_dec(x_25); +lean_dec(x_23); lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -1029,78 +1011,78 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_57 = !lean_is_exclusive(x_43); -if (x_57 == 0) +x_56 = !lean_is_exclusive(x_42); +if (x_56 == 0) { -return x_43; +return x_42; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_43, 0); -x_59 = lean_ctor_get(x_43, 1); -lean_inc(x_59); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_42, 0); +x_58 = lean_ctor_get(x_42, 1); lean_inc(x_58); -lean_dec(x_43); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +lean_inc(x_57); +lean_dec(x_42); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } else { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_34, 1); -lean_inc(x_61); -lean_dec(x_34); -x_62 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_61); -if (lean_obj_tag(x_62) == 0) +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_33, 1); +lean_inc(x_60); +lean_dec(x_33); +x_61 = l_Lean_Meta_Grind_updateLastTag(x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_60); +if (lean_obj_tag(x_61) == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_63 = lean_ctor_get(x_62, 1); -lean_inc(x_63); -lean_dec(x_62); -lean_inc(x_28); -x_64 = l_Lean_MessageData_ofExpr(x_28); -x_65 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5; -x_66 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_66, 0, x_65); -lean_ctor_set(x_66, 1, x_64); -x_67 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7; -x_68 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); +lean_dec(x_61); +lean_inc(x_26); +x_63 = l_Lean_MessageData_ofExpr(x_26); +x_64 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2; +x_65 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +x_66 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__4; +x_67 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); lean_inc(x_5); -x_69 = l_Lean_indentExpr(x_5); -x_70 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -x_71 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; -x_72 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -x_73 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_6, x_72, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_63); -x_74 = lean_ctor_get(x_73, 0); +x_68 = l_Lean_indentExpr(x_5); +x_69 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +x_70 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; +x_71 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +x_72 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_6, x_71, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_62); +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); lean_inc(x_74); -x_75 = lean_ctor_get(x_73, 1); -lean_inc(x_75); -lean_dec(x_73); -x_76 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_25, x_20, x_1, x_27, x_28, x_18, x_5, x_74, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_75); +lean_dec(x_72); +x_75 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_23, x_1, x_25, x_26, x_18, x_5, x_73, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_74); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_74); -return x_76; +lean_dec(x_73); +return x_75; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_28); -lean_dec(x_27); +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_26); lean_dec(x_25); +lean_dec(x_23); lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -1113,36 +1095,36 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_77 = lean_ctor_get(x_62, 0); +x_76 = lean_ctor_get(x_61, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_61, 1); lean_inc(x_77); -x_78 = lean_ctor_get(x_62, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_62)) { - lean_ctor_release(x_62, 0); - lean_ctor_release(x_62, 1); - x_79 = x_62; +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_78 = x_61; } else { - lean_dec_ref(x_62); - x_79 = lean_box(0); + lean_dec_ref(x_61); + x_78 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_78)) { + x_79 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_79; + x_79 = x_78; } -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_79, 0, x_76); +lean_ctor_set(x_79, 1, x_77); +return x_79; } } } } else { -uint8_t x_81; -lean_dec(x_28); -lean_dec(x_27); +uint8_t x_80; +lean_dec(x_26); lean_dec(x_25); +lean_dec(x_23); lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -1155,32 +1137,32 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_81 = !lean_is_exclusive(x_32); -if (x_81 == 0) +x_80 = !lean_is_exclusive(x_31); +if (x_80 == 0) { -return x_32; +return x_31; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_82 = lean_ctor_get(x_32, 0); -x_83 = lean_ctor_get(x_32, 1); -lean_inc(x_83); +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_31, 0); +x_82 = lean_ctor_get(x_31, 1); lean_inc(x_82); -lean_dec(x_32); -x_84 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_84, 0, x_82); -lean_ctor_set(x_84, 1, x_83); -return x_84; +lean_inc(x_81); +lean_dec(x_31); +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_81); +lean_ctor_set(x_83, 1, x_82); +return x_83; } } } else { -uint8_t x_85; -lean_dec(x_28); -lean_dec(x_27); +uint8_t x_84; +lean_dec(x_26); lean_dec(x_25); +lean_dec(x_23); lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -1193,29 +1175,29 @@ lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_85 = !lean_is_exclusive(x_29); -if (x_85 == 0) +x_84 = !lean_is_exclusive(x_27); +if (x_84 == 0) { -return x_29; +return x_27; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_29, 0); -x_87 = lean_ctor_get(x_29, 1); -lean_inc(x_87); +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_27, 0); +x_86 = lean_ctor_get(x_27, 1); lean_inc(x_86); -lean_dec(x_29); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; +lean_inc(x_85); +lean_dec(x_27); +x_87 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_87, 0, x_85); +lean_ctor_set(x_87, 1, x_86); +return x_87; } } } else { -uint8_t x_89; +uint8_t x_88; lean_dec(x_18); lean_dec(x_15); lean_dec(x_14); @@ -1230,29 +1212,29 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_89 = !lean_is_exclusive(x_24); -if (x_89 == 0) +x_88 = !lean_is_exclusive(x_22); +if (x_88 == 0) { -return x_24; +return x_22; } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_90 = lean_ctor_get(x_24, 0); -x_91 = lean_ctor_get(x_24, 1); -lean_inc(x_91); +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_22, 0); +x_90 = lean_ctor_get(x_22, 1); lean_inc(x_90); -lean_dec(x_24); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_90); -lean_ctor_set(x_92, 1, x_91); -return x_92; +lean_inc(x_89); +lean_dec(x_22); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +return x_91; } } } else { -uint8_t x_93; +uint8_t x_92; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -1266,23 +1248,23 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_93 = !lean_is_exclusive(x_17); -if (x_93 == 0) +x_92 = !lean_is_exclusive(x_17); +if (x_92 == 0) { return x_17; } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_94 = lean_ctor_get(x_17, 0); -x_95 = lean_ctor_get(x_17, 1); -lean_inc(x_95); +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_17, 0); +x_94 = lean_ctor_get(x_17, 1); lean_inc(x_94); +lean_inc(x_93); lean_dec(x_17); -x_96 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -return x_96; +x_95 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +return x_95; } } } @@ -1347,7 +1329,7 @@ x_29 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__2; lean_ctor_set_tag(x_17, 7); lean_ctor_set(x_17, 1, x_28); lean_ctor_set(x_17, 0, x_29); -x_30 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_30 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; x_31 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_31, 0, x_17); lean_ctor_set(x_31, 1, x_30); @@ -1418,7 +1400,7 @@ x_44 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__2; x_45 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_45, 0, x_44); lean_ctor_set(x_45, 1, x_43); -x_46 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_46 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; x_47 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_47, 0, x_45); lean_ctor_set(x_47, 1, x_46); @@ -1670,7 +1652,7 @@ lean_inc(x_26); lean_dec(x_25); lean_inc(x_1); x_27 = l_Lean_MessageData_ofExpr(x_1); -x_28 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_28 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; lean_ctor_set_tag(x_16, 7); lean_ctor_set(x_16, 1, x_27); lean_ctor_set(x_16, 0, x_28); @@ -1738,7 +1720,7 @@ lean_inc(x_40); lean_dec(x_39); lean_inc(x_1); x_41 = l_Lean_MessageData_ofExpr(x_1); -x_42 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_42 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; x_43 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_41); @@ -1814,34 +1796,17 @@ return x_54; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_18; -x_18 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_12); +lean_object* x_17; +x_17 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_18; +lean_dec(x_7); +return x_17; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { @@ -2019,37 +1984,160 @@ lean_dec(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("issues", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__2() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_propagateForallPropUp___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} +lean_object* x_9; lean_object* x_10; +x_9 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1; +x_10 = l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(x_1, x_9, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_10) == 0) +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +return x_10; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("failed to create E-match local theorem for", 42, 42); -return x_1; +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3; +uint8_t x_15; +x_15 = !lean_is_exclusive(x_10); +if (x_15 == 0) +{ +lean_object* x_16; uint8_t x_17; +x_16 = lean_ctor_get(x_10, 0); +x_17 = l_Lean_Exception_isInterrupt(x_16); +if (x_17 == 0) +{ +uint8_t x_18; +x_18 = l_Lean_Exception_isRuntime(x_16); +if (x_18 == 0) +{ +lean_object* x_19; +lean_dec(x_16); +x_19 = lean_box(0); +lean_ctor_set_tag(x_10, 0); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +return x_10; +} +} +else +{ +return x_10; +} +} +else +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_10, 0); +x_21 = lean_ctor_get(x_10, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_10); +x_22 = l_Lean_Exception_isInterrupt(x_20); +if (x_22 == 0) +{ +uint8_t x_23; +x_23 = l_Lean_Exception_isRuntime(x_20); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +lean_dec(x_20); +x_24 = lean_box(0); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_21); +return x_25; +} +else +{ +lean_object* x_26; +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_20); +lean_ctor_set(x_26, 1, x_21); +return x_26; +} +} +else +{ +lean_object* x_27; +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_20); +lean_ctor_set(x_27, 1, x_21); +return x_27; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; lean_object* x_10; +x_9 = lean_unbox(x_3); +lean_dec(x_3); +x_10 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(x_1, x_2, x_9, x_4, x_5, x_6, x_7, x_8); +return x_10; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("issues", 6, 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_propagateForallPropUp___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("failed to create E-match local theorem for", 42, 42); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } @@ -2065,7 +2153,7 @@ if (x_14 == 0) lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_ctor_get(x_15, 9); +x_17 = lean_ctor_get(x_15, 11); lean_inc(x_17); lean_dec(x_15); x_18 = lean_ctor_get(x_17, 2); @@ -2129,7 +2217,7 @@ x_33 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocal x_34 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_34, 0, x_33); lean_ctor_set(x_34, 1, x_32); -x_35 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_35 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; x_36 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_36, 0, x_34); lean_ctor_set(x_36, 1, x_35); @@ -2146,7 +2234,7 @@ x_39 = lean_ctor_get(x_13, 1); lean_inc(x_39); lean_inc(x_38); lean_dec(x_13); -x_40 = lean_ctor_get(x_38, 9); +x_40 = lean_ctor_get(x_38, 11); lean_inc(x_40); lean_dec(x_38); x_41 = lean_ctor_get(x_40, 2); @@ -2208,7 +2296,7 @@ x_55 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocal x_56 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_56, 0, x_55); lean_ctor_set(x_56, 1, x_54); -x_57 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9; +x_57 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6; x_58 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_58, 0, x_56); lean_ctor_set(x_58, 1, x_57); @@ -2219,34 +2307,32 @@ return x_59; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_17 = lean_st_ref_get(x_8, x_16); -x_18 = lean_ctor_get(x_17, 0); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_16 = lean_st_ref_get(x_7, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); +lean_dec(x_16); +x_19 = lean_ctor_get(x_17, 11); lean_inc(x_19); lean_dec(x_17); -x_20 = lean_ctor_get(x_18, 9); +x_20 = lean_ctor_get(x_19, 2); lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_20, 2); -lean_inc(x_21); +lean_dec(x_19); +x_21 = lean_nat_dec_eq(x_20, x_1); lean_dec(x_20); -x_22 = lean_nat_dec_eq(x_21, x_1); -lean_dec(x_21); -if (x_22 == 0) +if (x_21 == 0) { -lean_object* x_23; lean_object* x_24; -lean_dec(x_6); +lean_object* x_22; lean_object* x_23; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_23 = lean_box(0); -x_24 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_23, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_19); -lean_dec(x_15); +x_22 = lean_box(0); +x_23 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_18); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2254,32 +2340,32 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_24; +lean_dec(x_7); +return x_23; } else { -uint8_t x_25; lean_object* x_26; -x_25 = 5; -lean_inc(x_15); +uint8_t x_24; lean_object* x_25; +x_24 = 5; lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_26 = l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(x_3, x_4, x_5, x_25, x_12, x_13, x_14, x_15, x_19); +lean_inc(x_11); +x_25 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(x_3, x_4, x_24, x_11, x_12, x_13, x_14, x_18); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); if (lean_obj_tag(x_26) == 0) { -lean_object* x_27; -x_27 = lean_ctor_get(x_26, 0); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_dec(x_5); +x_27 = lean_ctor_get(x_25, 1); lean_inc(x_27); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; -lean_dec(x_6); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = lean_box(0); -x_30 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_29, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_28); -lean_dec(x_15); +lean_dec(x_25); +x_28 = lean_box(0); +x_29 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_27); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2287,18 +2373,18 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_30; +lean_dec(x_7); +return x_29; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); +lean_dec(x_25); +x_31 = lean_ctor_get(x_26, 0); lean_inc(x_31); lean_dec(x_26); -x_32 = lean_ctor_get(x_27, 0); -lean_inc(x_32); -lean_dec(x_27); -lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -2306,17 +2392,17 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_33 = l_Lean_Meta_Grind_activateTheorem(x_32, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_31); -if (lean_obj_tag(x_33) == 0) +lean_inc(x_7); +x_32 = l_Lean_Meta_Grind_activateTheorem(x_31, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_30); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_33, 0); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_34, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_35); -lean_dec(x_15); +lean_dec(x_32); +x_35 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1(x_1, x_2, x_33, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_34); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2324,13 +2410,13 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_34); -return x_36; +lean_dec(x_7); +lean_dec(x_33); +return x_35; } else { -uint8_t x_37; -lean_dec(x_15); +uint8_t x_36; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2338,32 +2424,32 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_2); -x_37 = !lean_is_exclusive(x_33); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_32); +if (x_36 == 0) { -return x_33; +return x_32; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_33, 0); -x_39 = lean_ctor_get(x_33, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_32, 0); +x_38 = lean_ctor_get(x_32, 1); lean_inc(x_38); -lean_dec(x_33); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_inc(x_37); +lean_dec(x_32); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } } else { -uint8_t x_41; -lean_dec(x_15); +uint8_t x_40; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2371,68 +2457,67 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); +lean_dec(x_5); lean_dec(x_2); -x_41 = !lean_is_exclusive(x_26); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_25); +if (x_40 == 0) { -return x_26; +return x_25; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_26, 0); -x_43 = lean_ctor_get(x_26, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_25, 0); +x_42 = lean_ctor_get(x_25, 1); lean_inc(x_42); -lean_dec(x_26); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_inc(x_41); +lean_dec(x_25); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -uint8_t x_17; lean_object* x_18; -x_17 = 4; -lean_inc(x_15); +uint8_t x_16; lean_object* x_17; +x_16 = 4; lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_3); +lean_inc(x_11); lean_inc(x_2); lean_inc(x_1); -x_18 = l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(x_1, x_2, x_3, x_17, x_12, x_13, x_14, x_15, x_16); +x_17 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(x_1, x_2, x_16, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); if (lean_obj_tag(x_18) == 0) { -lean_object* x_19; -x_19 = lean_ctor_get(x_18, 0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_17, 1); lean_inc(x_19); -if (lean_obj_tag(x_19) == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_box(0); -x_22 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_4, x_5, x_1, x_2, x_3, x_6, x_21, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_20); -return x_22; +lean_dec(x_17); +x_20 = lean_box(0); +x_21 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_3, x_4, x_1, x_2, x_5, x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); +return x_21; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_18, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_dec(x_17); +x_23 = lean_ctor_get(x_18, 0); lean_inc(x_23); lean_dec(x_18); -x_24 = lean_ctor_get(x_19, 0); -lean_inc(x_24); -lean_dec(x_19); -lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); @@ -2440,24 +2525,24 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_6); -x_25 = l_Lean_Meta_Grind_activateTheorem(x_24, x_6, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_23); -if (lean_obj_tag(x_25) == 0) +lean_inc(x_7); +lean_inc(x_5); +x_24 = l_Lean_Meta_Grind_activateTheorem(x_23, x_5, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_22); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_25, 0); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); +lean_dec(x_24); +x_27 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_3, x_4, x_1, x_2, x_5, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_26); lean_dec(x_25); -x_28 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_4, x_5, x_1, x_2, x_3, x_6, x_26, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_27); -lean_dec(x_26); -return x_28; +return x_27; } else { -uint8_t x_29; -lean_dec(x_15); +uint8_t x_28; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2465,36 +2550,35 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); lean_dec(x_5); -lean_dec(x_3); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_29 = !lean_is_exclusive(x_25); -if (x_29 == 0) +x_28 = !lean_is_exclusive(x_24); +if (x_28 == 0) { -return x_25; +return x_24; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_25, 0); -x_31 = lean_ctor_get(x_25, 1); -lean_inc(x_31); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_24, 0); +x_30 = lean_ctor_get(x_24, 1); lean_inc(x_30); -lean_dec(x_25); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_inc(x_29); +lean_dec(x_24); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } } } else { -uint8_t x_33; -lean_dec(x_15); +uint8_t x_32; lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); @@ -2502,104 +2586,93 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_6); +lean_dec(x_7); lean_dec(x_5); -lean_dec(x_3); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_33 = !lean_is_exclusive(x_18); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_17); +if (x_32 == 0) { -return x_18; +return x_17; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_18, 0); -x_35 = lean_ctor_get(x_18, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_17, 0); +x_34 = lean_ctor_get(x_17, 1); lean_inc(x_34); -lean_dec(x_18); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} +lean_inc(x_33); +lean_dec(x_17); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_13 = l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__3; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_inc(x_1); -x_14 = l_Lean_mkAppB(x_13, x_1, x_2); -x_15 = lean_st_ref_get(x_4, x_12); -x_16 = lean_ctor_get(x_15, 0); +x_13 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_2); +x_14 = lean_st_ref_get(x_4, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); +lean_dec(x_14); +x_17 = lean_ctor_get(x_15, 11); lean_inc(x_17); lean_dec(x_15); -x_18 = lean_ctor_get(x_16, 9); +x_18 = lean_ctor_get(x_17, 2); lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_18, 2); -lean_inc(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_inc(x_1); -x_20 = l_Lean_Meta_Grind_getGeneration(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -if (lean_obj_tag(x_20) == 0) +x_19 = l_Lean_Meta_Grind_getGeneration(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +if (lean_obj_tag(x_19) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; lean_object* x_25; -x_21 = lean_ctor_get(x_20, 0); +lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1; -x_24 = 3; +lean_dec(x_19); +x_22 = 3; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_14); +lean_inc(x_13); lean_inc(x_3); -x_25 = l_Lean_Meta_Grind_mkEMatchTheoremWithKind_x3f(x_3, x_23, x_14, x_24, x_8, x_9, x_10, x_11, x_22); -if (lean_obj_tag(x_25) == 0) +x_23 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f(x_3, x_13, x_22, x_8, x_9, x_10, x_11, x_21); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_26; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -if (lean_obj_tag(x_26) == 0) +lean_object* x_24; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_box(0); -x_29 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_3, x_23, x_14, x_19, x_1, x_21, x_28, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); -lean_dec(x_19); -return x_29; +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +x_27 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_3, x_13, x_18, x_1, x_20, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +lean_dec(x_18); +return x_27; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_25, 1); -lean_inc(x_30); -lean_dec(x_25); -x_31 = lean_ctor_get(x_26, 0); -lean_inc(x_31); -lean_dec(x_26); +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_23, 1); +lean_inc(x_28); +lean_dec(x_23); +x_29 = lean_ctor_get(x_24, 0); +lean_inc(x_29); +lean_dec(x_24); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -2608,27 +2681,27 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_21); -x_32 = l_Lean_Meta_Grind_activateTheorem(x_31, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); -if (lean_obj_tag(x_32) == 0) +lean_inc(x_20); +x_30 = l_Lean_Meta_Grind_activateTheorem(x_29, x_20, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); +if (lean_obj_tag(x_30) == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_32, 1); -lean_inc(x_34); -lean_dec(x_32); -x_35 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_3, x_23, x_14, x_19, x_1, x_21, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_34); -lean_dec(x_33); -lean_dec(x_19); -return x_35; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_3, x_13, x_18, x_1, x_20, x_31, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +lean_dec(x_31); +lean_dec(x_18); +return x_33; } else { -uint8_t x_36; -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_14); +uint8_t x_34; +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2639,33 +2712,33 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_32); -if (x_36 == 0) +x_34 = !lean_is_exclusive(x_30); +if (x_34 == 0) { -return x_32; +return x_30; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_32, 0); -x_38 = lean_ctor_get(x_32, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_32); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_30, 0); +x_36 = lean_ctor_get(x_30, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_30); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } } else { -uint8_t x_40; -lean_dec(x_21); -lean_dec(x_19); -lean_dec(x_14); +uint8_t x_38; +lean_dec(x_20); +lean_dec(x_18); +lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2676,31 +2749,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_40 = !lean_is_exclusive(x_25); -if (x_40 == 0) +x_38 = !lean_is_exclusive(x_23); +if (x_38 == 0) { -return x_25; +return x_23; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_25, 0); -x_42 = lean_ctor_get(x_25, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_25); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_23, 0); +x_40 = lean_ctor_get(x_23, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_23); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } else { -uint8_t x_44; -lean_dec(x_19); -lean_dec(x_14); +uint8_t x_42; +lean_dec(x_18); +lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2711,23 +2784,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_44 = !lean_is_exclusive(x_20); -if (x_44 == 0) +x_42 = !lean_is_exclusive(x_19); +if (x_42 == 0) { -return x_20; +return x_19; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_20, 0); -x_46 = lean_ctor_get(x_20, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_20); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_19, 0); +x_44 = lean_ctor_get(x_19, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_19); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } } @@ -2787,10 +2860,10 @@ x_18 = !lean_is_exclusive(x_16); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_19 = lean_ctor_get(x_16, 19); +x_19 = lean_ctor_get(x_16, 21); x_20 = lean_unsigned_to_nat(1u); x_21 = lean_nat_add(x_19, x_20); -lean_ctor_set(x_16, 19, x_21); +lean_ctor_set(x_16, 21, x_21); x_22 = lean_st_ref_set(x_2, x_16, x_17); x_23 = lean_ctor_get(x_22, 1); lean_inc(x_23); @@ -2804,15 +2877,15 @@ return x_27; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; x_28 = lean_ctor_get(x_16, 0); x_29 = lean_ctor_get(x_16, 1); x_30 = lean_ctor_get(x_16, 2); x_31 = lean_ctor_get(x_16, 3); x_32 = lean_ctor_get(x_16, 4); x_33 = lean_ctor_get(x_16, 5); -x_34 = lean_ctor_get_uint8(x_16, sizeof(void*)*20); -x_35 = lean_ctor_get(x_16, 6); +x_34 = lean_ctor_get(x_16, 6); +x_35 = lean_ctor_get_uint8(x_16, sizeof(void*)*23); x_36 = lean_ctor_get(x_16, 7); x_37 = lean_ctor_get(x_16, 8); x_38 = lean_ctor_get(x_16, 9); @@ -2826,6 +2899,12 @@ x_45 = lean_ctor_get(x_16, 16); x_46 = lean_ctor_get(x_16, 17); x_47 = lean_ctor_get(x_16, 18); x_48 = lean_ctor_get(x_16, 19); +x_49 = lean_ctor_get(x_16, 20); +x_50 = lean_ctor_get(x_16, 21); +x_51 = lean_ctor_get(x_16, 22); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); @@ -2839,7 +2918,7 @@ lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); lean_inc(x_36); -lean_inc(x_35); +lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); @@ -2847,68 +2926,71 @@ lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_dec(x_16); -x_49 = lean_unsigned_to_nat(1u); -x_50 = lean_nat_add(x_48, x_49); -x_51 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_51, 0, x_28); -lean_ctor_set(x_51, 1, x_29); -lean_ctor_set(x_51, 2, x_30); -lean_ctor_set(x_51, 3, x_31); -lean_ctor_set(x_51, 4, x_32); -lean_ctor_set(x_51, 5, x_33); -lean_ctor_set(x_51, 6, x_35); -lean_ctor_set(x_51, 7, x_36); -lean_ctor_set(x_51, 8, x_37); -lean_ctor_set(x_51, 9, x_38); -lean_ctor_set(x_51, 10, x_39); -lean_ctor_set(x_51, 11, x_40); -lean_ctor_set(x_51, 12, x_41); -lean_ctor_set(x_51, 13, x_42); -lean_ctor_set(x_51, 14, x_43); -lean_ctor_set(x_51, 15, x_44); -lean_ctor_set(x_51, 16, x_45); -lean_ctor_set(x_51, 17, x_46); -lean_ctor_set(x_51, 18, x_47); -lean_ctor_set(x_51, 19, x_50); -lean_ctor_set_uint8(x_51, sizeof(void*)*20, x_34); -x_52 = lean_st_ref_set(x_2, x_51, x_17); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_54 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__2; -x_55 = lean_name_append_index_after(x_54, x_48); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_55); -x_57 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_56, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_53); -return x_57; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_add(x_50, x_52); +x_54 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_54, 0, x_28); +lean_ctor_set(x_54, 1, x_29); +lean_ctor_set(x_54, 2, x_30); +lean_ctor_set(x_54, 3, x_31); +lean_ctor_set(x_54, 4, x_32); +lean_ctor_set(x_54, 5, x_33); +lean_ctor_set(x_54, 6, x_34); +lean_ctor_set(x_54, 7, x_36); +lean_ctor_set(x_54, 8, x_37); +lean_ctor_set(x_54, 9, x_38); +lean_ctor_set(x_54, 10, x_39); +lean_ctor_set(x_54, 11, x_40); +lean_ctor_set(x_54, 12, x_41); +lean_ctor_set(x_54, 13, x_42); +lean_ctor_set(x_54, 14, x_43); +lean_ctor_set(x_54, 15, x_44); +lean_ctor_set(x_54, 16, x_45); +lean_ctor_set(x_54, 17, x_46); +lean_ctor_set(x_54, 18, x_47); +lean_ctor_set(x_54, 19, x_48); +lean_ctor_set(x_54, 20, x_49); +lean_ctor_set(x_54, 21, x_53); +lean_ctor_set(x_54, 22, x_51); +lean_ctor_set_uint8(x_54, sizeof(void*)*23, x_35); +x_55 = lean_st_ref_set(x_2, x_54, x_17); +x_56 = lean_ctor_get(x_55, 1); +lean_inc(x_56); +lean_dec(x_55); +x_57 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__2; +x_58 = lean_name_append_index_after(x_57, x_50); +x_59 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_59, 0, x_58); +x_60 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_59, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_56); +return x_60; } } else { -uint8_t x_58; -x_58 = !lean_is_exclusive(x_14); -if (x_58 == 0) +uint8_t x_61; +x_61 = !lean_is_exclusive(x_14); +if (x_61 == 0) { -lean_object* x_59; -x_59 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_59; +lean_object* x_62; +x_62 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_62; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_14, 0); -lean_inc(x_60); +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_14, 0); +lean_inc(x_63); lean_dec(x_14); -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_60); -x_62 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_61, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_62; +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_63); +x_65 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4(x_1, x_12, x_64, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_65; } } } else { -uint8_t x_63; +uint8_t x_66; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2918,23 +3000,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_11); -if (x_63 == 0) +x_66 = !lean_is_exclusive(x_11); +if (x_66 == 0) { return x_11; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_11, 0); -x_65 = lean_ctor_get(x_11, 1); -lean_inc(x_65); -lean_inc(x_64); +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_11, 0); +x_68 = lean_ctor_get(x_11, 1); +lean_inc(x_68); +lean_inc(x_67); lean_dec(x_11); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; } } } @@ -2957,24 +3039,24 @@ lean_dec(x_1); return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; -x_17 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); +lean_object* x_16; +x_16 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_6); lean_dec(x_1); -return x_17; +return x_16; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -lean_object* x_17; -x_17 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -lean_dec(x_4); -return x_17; +lean_object* x_16; +x_16 = l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +lean_dec(x_6); +lean_dec(x_3); +return x_16; } } static lean_object* _init_l_Lean_Meta_Grind_propagateForallPropDown___closed__1() { @@ -3619,6 +3701,8 @@ l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__1 = _init_l_Lean_M lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__1); l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__2); +l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__1___closed__3); l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__1); l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__2(); @@ -3631,12 +3715,6 @@ l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5 = _init_l_Lean_M lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__5); l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6(); lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__6); -l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__7); -l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__8); -l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__2___closed__9); l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__1 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__1); l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__2 = _init_l_Lean_Meta_Grind_propagateForallPropUp___lambda__3___closed__2(); @@ -3659,6 +3737,8 @@ l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___closed__4); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___closed__5(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_isEqTrueHyp_x3f___closed__5); +l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_mkEMatchTheoremWithKind_x27_x3f___closed__1); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__1); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__2(); @@ -3667,8 +3747,6 @@ l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchT lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__3); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__1___closed__4); -l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___lambda__4___closed__1); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__1); l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_ForallProp_0__Lean_Meta_Grind_addLocalEMatchTheorems___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Internalize.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Internalize.c index 3a1b248b6ded..d0f815369c67 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Internalize.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Internalize.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind.Internalize -// Imports: Init.Grind.Util Init.Grind.Lemmas Lean.Meta.LitValues Lean.Meta.Match.MatcherInfo Lean.Meta.Match.MatchEqsExt Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Util +// Imports: Init.Grind.Util Init.Grind.Lemmas Lean.Meta.LitValues Lean.Meta.Match.MatcherInfo Lean.Meta.Match.MatchEqsExt Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Util Lean.Meta.Tactic.Grind.Arith.Internalize #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -14,6 +14,7 @@ extern "C" { #endif LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); uint8_t lean_is_matcher(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -41,8 +42,10 @@ lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, l LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__2; uint8_t l_Lean_Expr_isDIte(lean_object*); +lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__3; lean_object* l_Lean_Meta_Grind_eraseIrrelevantMData___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1; uint8_t lean_usize_dec_le(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__4; @@ -50,7 +53,6 @@ LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Gr lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_addCongrTable___spec__6(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__2___boxed(lean_object**); lean_object* l_Lean_Meta_Grind_unfoldReducible___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); @@ -65,7 +67,7 @@ uint8_t l_Lean_Meta_Grind_isCongruent(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__6(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofList(lean_object*); lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); @@ -76,8 +78,8 @@ static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__3; lean_object* l_Lean_PersistentHashMap_insert___at_Lean_NameSSet_insert___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___closed__1; -LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_activateTheorem___closed__2; @@ -93,6 +95,8 @@ lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_setENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); @@ -100,7 +104,7 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_ lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAtAux___at_Lean_Meta_Grind_addCongrTable___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_internalize___lambda__3___closed__1; uint8_t l_Lean_Meta_Grind_EMatchTheorems_isErased(lean_object*, lean_object*); @@ -109,7 +113,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate___closed__1; lean_object* l_Lean_Meta_Grind_propagateUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isBVar(lean_object*); -extern lean_object* l_instInhabitedPUnit; +lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__4; @@ -139,6 +143,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___closed__5; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -166,7 +171,6 @@ uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); lean_object* l_Lean_Expr_toHeadIndex(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2(lean_object*, lean_object*, size_t, lean_object*); static size_t l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_levelZero; static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__3___closed__2; @@ -176,6 +180,7 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_T LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__7; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__11; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_addCongrTable___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -189,7 +194,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_ static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__3___closed__1; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isIte(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__2(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__6; @@ -197,20 +201,18 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_ lean_object* l_Lean_Meta_Grind_mkEMatchEqTheorem(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_updateLastTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_addCongrTable___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -extern lean_object* l_Lean_Meta_instMonadMetaM; lean_object* l_Lean_Meta_Grind_hasSameType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_activateTheorem___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__1___closed__2; static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___closed__5; LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___boxed(lean_object**); static lean_object* l_Lean_Meta_Grind_internalize___lambda__4___closed__1; -static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -218,12 +220,10 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_M lean_object* l_Lean_Meta_Grind_mkGroundPattern(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAtAux___at_Lean_Meta_Grind_addCongrTable___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constLevels_x21(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__10; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__5; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_shareCommon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -243,28 +243,26 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__9; static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__4___closed__2; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5; lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___closed__7; static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__7; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__1; lean_object* lean_get_match_equations_for(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isProp(lean_object*); lean_object* l_Lean_PersistentHashMap_mkCollisionNode___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__1(lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isMorallyIff___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___spec__1(lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; lean_object* l_Lean_Meta_Grind_mkENodeCore(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2___boxed(lean_object**); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__2(lean_object*, size_t, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__3; lean_object* l_List_reverse___rarg(lean_object*); @@ -278,25 +276,25 @@ static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_ size_t lean_usize_add(size_t, size_t); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); -lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__1___boxed(lean_object**); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_isMatcher___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_HeadIndex_0__Lean_beqHeadIndex____x40_Lean_HeadIndex___hyg_69_(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__8; LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__2; static lean_object* l_Lean_Meta_Grind_internalize___lambda__3___closed__2; lean_object* l_Lean_Meta_Grind_Origin_key(lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isMorallyIff(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3; lean_object* lean_nat_add(lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Grind_congrPlaceholderProof; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -307,7 +305,6 @@ uint64_t l_Lean_HeadIndex_hash(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate___closed__2; static lean_object* l_Lean_Meta_Grind_addCongrTable___closed__3; static lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__8; -static lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; lean_object* l_Lean_Meta_Grind_unfoldReducible___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getConfig___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); @@ -315,18 +312,17 @@ LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_activateTheorem__ lean_object* l_Lean_MessageData_ofName(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isLitValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_ReaderT_instMonad___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Meta_isMatcherApp___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__5; -static lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAtAux___at_Lean_Meta_Grind_addCongrTable___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_1, 1); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); x_8 = lean_array_get_size(x_2); x_9 = lean_nat_dec_lt(x_5, x_8); @@ -407,7 +403,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_6 = lean_ctor_get(x_2, 0); -x_7 = lean_ctor_get(x_1, 1); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); x_8 = 5; x_9 = l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__2; @@ -509,7 +505,7 @@ lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; size_t x_32; lea x_28 = lean_ctor_get(x_2, 0); lean_inc(x_28); lean_dec(x_2); -x_29 = lean_ctor_get(x_1, 1); +x_29 = lean_ctor_get(x_1, 2); lean_inc(x_29); x_30 = 5; x_31 = l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__2; @@ -606,7 +602,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntry_x3f___at_Lean_Meta_G _start: { lean_object* x_4; uint64_t x_5; size_t x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); lean_inc(x_4); lean_inc(x_3); x_5 = l_Lean_Meta_Grind_congrHash(x_4, x_3); @@ -619,7 +615,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_M _start: { lean_object* x_8; lean_object* x_9; uint8_t x_10; -x_8 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_1, 2); lean_inc(x_8); x_9 = lean_array_get_size(x_3); x_10 = lean_nat_dec_lt(x_6, x_9); @@ -664,7 +660,7 @@ x_6 = lean_ctor_get(x_2, 0); lean_inc(x_6); x_7 = lean_ctor_get(x_2, 1); lean_inc(x_7); -x_8 = lean_ctor_get(x_1, 1); +x_8 = lean_ctor_get(x_1, 2); lean_inc(x_8); x_9 = lean_array_get_size(x_6); x_10 = lean_nat_dec_lt(x_3, x_9); @@ -772,7 +768,7 @@ if (x_7 == 0) { lean_object* x_8; lean_object* x_9; size_t x_10; size_t x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; x_8 = lean_ctor_get(x_2, 0); -x_9 = lean_ctor_get(x_1, 1); +x_9 = lean_ctor_get(x_1, 2); lean_inc(x_9); x_10 = 1; x_11 = 5; @@ -930,7 +926,7 @@ lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; size_t x_54; siz x_50 = lean_ctor_get(x_2, 0); lean_inc(x_50); lean_dec(x_2); -x_51 = lean_ctor_get(x_1, 1); +x_51 = lean_ctor_get(x_1, 2); lean_inc(x_51); x_52 = 1; x_53 = 5; @@ -1157,7 +1153,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_ad _start: { lean_object* x_5; uint64_t x_6; size_t x_7; size_t x_8; lean_object* x_9; -x_5 = lean_ctor_get(x_1, 1); +x_5 = lean_ctor_get(x_1, 2); lean_inc(x_5); lean_inc(x_3); x_6 = l_Lean_Meta_Grind_congrHash(x_5, x_3); @@ -1170,188 +1166,197 @@ return x_9; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addCongrTable___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_41; +lean_object* x_13; lean_object* x_45; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_2); lean_inc(x_1); -x_41 = l_Lean_Meta_Grind_hasSameType(x_1, x_2, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_41) == 0) +x_45 = l_Lean_Meta_Grind_hasSameType(x_1, x_2, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_42; uint8_t x_43; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_unbox(x_42); -lean_dec(x_42); -if (x_43 == 0) +lean_object* x_46; uint8_t x_47; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_unbox(x_46); +lean_dec(x_46); +if (x_47 == 0) { -lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; -x_44 = lean_ctor_get(x_41, 1); -lean_inc(x_44); -lean_dec(x_41); -x_45 = l_Lean_Meta_Grind_congrPlaceholderProof; -x_46 = 1; +lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; +x_48 = lean_ctor_get(x_45, 1); +lean_inc(x_48); +lean_dec(x_45); +x_49 = l_Lean_Meta_Grind_congrPlaceholderProof; +x_50 = 1; lean_inc(x_2); lean_inc(x_1); -x_47 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_45, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_44); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -x_13 = x_48; -goto block_40; +x_51 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_49, x_50, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_48); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +lean_dec(x_51); +x_13 = x_52; +goto block_44; } else { -lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; lean_object* x_53; -x_49 = lean_ctor_get(x_41, 1); -lean_inc(x_49); -lean_dec(x_41); -x_50 = l_Lean_Meta_Grind_congrPlaceholderProof; -x_51 = 0; +lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; +x_53 = lean_ctor_get(x_45, 1); +lean_inc(x_53); +lean_dec(x_45); +x_54 = l_Lean_Meta_Grind_congrPlaceholderProof; +x_55 = 0; lean_inc(x_2); lean_inc(x_1); -x_52 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_50, x_51, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_49); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -lean_dec(x_52); -x_13 = x_53; -goto block_40; +x_56 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_54, x_55, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_53); +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +lean_dec(x_56); +x_13 = x_57; +goto block_44; } } else { -uint8_t x_54; +uint8_t x_58; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_2); lean_dec(x_1); -x_54 = !lean_is_exclusive(x_41); -if (x_54 == 0) +x_58 = !lean_is_exclusive(x_45); +if (x_58 == 0) { -return x_41; +return x_45; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_41, 0); -x_56 = lean_ctor_get(x_41, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_41); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_45, 0); +x_60 = lean_ctor_get(x_45, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_45); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } -block_40: -{ -lean_object* x_14; -lean_inc(x_1); -x_14 = l_Lean_Meta_Grind_getENode(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_13); -if (lean_obj_tag(x_14) == 0) +block_44: { -lean_object* x_15; lean_object* x_16; uint8_t x_17; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_st_ref_get(x_4, x_13); x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); -x_17 = !lean_is_exclusive(x_15); -if (x_17 == 0) +lean_inc(x_1); +x_17 = l_Lean_Meta_Grind_Goal_getENode(x_15, x_1, x_10, x_11, x_16); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_15, 3); -lean_dec(x_18); -lean_ctor_set(x_15, 3, x_2); -x_19 = l_Lean_Meta_Grind_setENode(x_1, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = !lean_is_exclusive(x_18); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_18, 3); +lean_dec(x_21); +lean_ctor_set(x_18, 3, x_2); +x_22 = l_Lean_Meta_Grind_setENode(x_1, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_19; +return x_22; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; uint8_t x_27; uint8_t x_28; uint8_t x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_20 = lean_ctor_get(x_15, 0); -x_21 = lean_ctor_get(x_15, 1); -x_22 = lean_ctor_get(x_15, 2); -x_23 = lean_ctor_get(x_15, 4); -x_24 = lean_ctor_get(x_15, 5); -x_25 = lean_ctor_get_uint8(x_15, sizeof(void*)*10); -x_26 = lean_ctor_get(x_15, 6); -x_27 = lean_ctor_get_uint8(x_15, sizeof(void*)*10 + 1); -x_28 = lean_ctor_get_uint8(x_15, sizeof(void*)*10 + 2); -x_29 = lean_ctor_get_uint8(x_15, sizeof(void*)*10 + 3); -x_30 = lean_ctor_get_uint8(x_15, sizeof(void*)*10 + 4); -x_31 = lean_ctor_get(x_15, 7); -x_32 = lean_ctor_get(x_15, 8); -x_33 = lean_ctor_get(x_15, 9); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; uint8_t x_30; uint8_t x_31; uint8_t x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_23 = lean_ctor_get(x_18, 0); +x_24 = lean_ctor_get(x_18, 1); +x_25 = lean_ctor_get(x_18, 2); +x_26 = lean_ctor_get(x_18, 4); +x_27 = lean_ctor_get(x_18, 5); +x_28 = lean_ctor_get_uint8(x_18, sizeof(void*)*11); +x_29 = lean_ctor_get(x_18, 6); +x_30 = lean_ctor_get_uint8(x_18, sizeof(void*)*11 + 1); +x_31 = lean_ctor_get_uint8(x_18, sizeof(void*)*11 + 2); +x_32 = lean_ctor_get_uint8(x_18, sizeof(void*)*11 + 3); +x_33 = lean_ctor_get_uint8(x_18, sizeof(void*)*11 + 4); +x_34 = lean_ctor_get(x_18, 7); +x_35 = lean_ctor_get(x_18, 8); +x_36 = lean_ctor_get(x_18, 9); +x_37 = lean_ctor_get(x_18, 10); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_29); +lean_inc(x_27); lean_inc(x_26); +lean_inc(x_25); lean_inc(x_24); lean_inc(x_23); -lean_inc(x_22); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_15); -x_34 = lean_alloc_ctor(0, 10, 5); -lean_ctor_set(x_34, 0, x_20); -lean_ctor_set(x_34, 1, x_21); -lean_ctor_set(x_34, 2, x_22); -lean_ctor_set(x_34, 3, x_2); -lean_ctor_set(x_34, 4, x_23); -lean_ctor_set(x_34, 5, x_24); -lean_ctor_set(x_34, 6, x_26); -lean_ctor_set(x_34, 7, x_31); -lean_ctor_set(x_34, 8, x_32); -lean_ctor_set(x_34, 9, x_33); -lean_ctor_set_uint8(x_34, sizeof(void*)*10, x_25); -lean_ctor_set_uint8(x_34, sizeof(void*)*10 + 1, x_27); -lean_ctor_set_uint8(x_34, sizeof(void*)*10 + 2, x_28); -lean_ctor_set_uint8(x_34, sizeof(void*)*10 + 3, x_29); -lean_ctor_set_uint8(x_34, sizeof(void*)*10 + 4, x_30); -x_35 = l_Lean_Meta_Grind_setENode(x_1, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +lean_dec(x_18); +x_38 = lean_alloc_ctor(0, 11, 5); +lean_ctor_set(x_38, 0, x_23); +lean_ctor_set(x_38, 1, x_24); +lean_ctor_set(x_38, 2, x_25); +lean_ctor_set(x_38, 3, x_2); +lean_ctor_set(x_38, 4, x_26); +lean_ctor_set(x_38, 5, x_27); +lean_ctor_set(x_38, 6, x_29); +lean_ctor_set(x_38, 7, x_34); +lean_ctor_set(x_38, 8, x_35); +lean_ctor_set(x_38, 9, x_36); +lean_ctor_set(x_38, 10, x_37); +lean_ctor_set_uint8(x_38, sizeof(void*)*11, x_28); +lean_ctor_set_uint8(x_38, sizeof(void*)*11 + 1, x_30); +lean_ctor_set_uint8(x_38, sizeof(void*)*11 + 2, x_31); +lean_ctor_set_uint8(x_38, sizeof(void*)*11 + 3, x_32); +lean_ctor_set_uint8(x_38, sizeof(void*)*11 + 4, x_33); +x_39 = l_Lean_Meta_Grind_setENode(x_1, x_38, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_35; +return x_39; } } else { -uint8_t x_36; +uint8_t x_40; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_2); lean_dec(x_1); -x_36 = !lean_is_exclusive(x_14); -if (x_36 == 0) +x_40 = !lean_is_exclusive(x_17); +if (x_40 == 0) { -return x_14; +return x_17; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_14, 0); -x_38 = lean_ctor_get(x_14, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_14); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); -return x_39; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_17, 0); +x_42 = lean_ctor_get(x_17, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_17); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } @@ -1695,13 +1700,13 @@ if (x_12 == 0) lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_13 = lean_ctor_get(x_11, 0); x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_ctor_get(x_13, 3); +x_15 = lean_ctor_get(x_13, 4); lean_inc(x_15); lean_inc(x_1); x_16 = l_Lean_PersistentHashMap_findEntry_x3f___at_Lean_Meta_Grind_addCongrTable___spec__1(x_13, x_15, x_1); if (lean_obj_tag(x_16) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -1728,9 +1733,9 @@ x_24 = lean_ctor_get(x_18, 4); lean_inc(x_24); x_25 = lean_ctor_get(x_18, 5); lean_inc(x_25); -x_26 = lean_ctor_get_uint8(x_18, sizeof(void*)*20); -x_27 = lean_ctor_get(x_18, 6); -lean_inc(x_27); +x_26 = lean_ctor_get(x_18, 6); +lean_inc(x_26); +x_27 = lean_ctor_get_uint8(x_18, sizeof(void*)*23); x_28 = lean_ctor_get(x_18, 7); lean_inc(x_28); x_29 = lean_ctor_get(x_18, 8); @@ -1757,227 +1762,242 @@ x_39 = lean_ctor_get(x_18, 18); lean_inc(x_39); x_40 = lean_ctor_get(x_18, 19); lean_inc(x_40); -x_41 = lean_box(0); +x_41 = lean_ctor_get(x_18, 20); +lean_inc(x_41); +x_42 = lean_ctor_get(x_18, 21); +lean_inc(x_42); +x_43 = lean_ctor_get(x_18, 22); +lean_inc(x_43); +x_44 = lean_box(0); lean_inc(x_18); -x_42 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_addCongrTable___spec__4(x_18, x_23, x_1, x_41); -x_43 = !lean_is_exclusive(x_18); -if (x_43 == 0) +x_45 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_addCongrTable___spec__4(x_18, x_24, x_1, x_44); +x_46 = !lean_is_exclusive(x_18); +if (x_46 == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; -x_44 = lean_ctor_get(x_18, 19); -lean_dec(x_44); -x_45 = lean_ctor_get(x_18, 18); -lean_dec(x_45); -x_46 = lean_ctor_get(x_18, 17); -lean_dec(x_46); -x_47 = lean_ctor_get(x_18, 16); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; +x_47 = lean_ctor_get(x_18, 22); lean_dec(x_47); -x_48 = lean_ctor_get(x_18, 15); +x_48 = lean_ctor_get(x_18, 21); lean_dec(x_48); -x_49 = lean_ctor_get(x_18, 14); +x_49 = lean_ctor_get(x_18, 20); lean_dec(x_49); -x_50 = lean_ctor_get(x_18, 13); +x_50 = lean_ctor_get(x_18, 19); lean_dec(x_50); -x_51 = lean_ctor_get(x_18, 12); +x_51 = lean_ctor_get(x_18, 18); lean_dec(x_51); -x_52 = lean_ctor_get(x_18, 11); +x_52 = lean_ctor_get(x_18, 17); lean_dec(x_52); -x_53 = lean_ctor_get(x_18, 10); +x_53 = lean_ctor_get(x_18, 16); lean_dec(x_53); -x_54 = lean_ctor_get(x_18, 9); +x_54 = lean_ctor_get(x_18, 15); lean_dec(x_54); -x_55 = lean_ctor_get(x_18, 8); +x_55 = lean_ctor_get(x_18, 14); lean_dec(x_55); -x_56 = lean_ctor_get(x_18, 7); +x_56 = lean_ctor_get(x_18, 13); lean_dec(x_56); -x_57 = lean_ctor_get(x_18, 6); +x_57 = lean_ctor_get(x_18, 12); lean_dec(x_57); -x_58 = lean_ctor_get(x_18, 5); +x_58 = lean_ctor_get(x_18, 11); lean_dec(x_58); -x_59 = lean_ctor_get(x_18, 4); +x_59 = lean_ctor_get(x_18, 10); lean_dec(x_59); -x_60 = lean_ctor_get(x_18, 3); +x_60 = lean_ctor_get(x_18, 9); lean_dec(x_60); -x_61 = lean_ctor_get(x_18, 2); +x_61 = lean_ctor_get(x_18, 8); lean_dec(x_61); -x_62 = lean_ctor_get(x_18, 1); +x_62 = lean_ctor_get(x_18, 7); lean_dec(x_62); -x_63 = lean_ctor_get(x_18, 0); +x_63 = lean_ctor_get(x_18, 6); lean_dec(x_63); -lean_ctor_set(x_18, 3, x_42); -x_64 = lean_st_ref_set(x_2, x_18, x_19); +x_64 = lean_ctor_get(x_18, 5); +lean_dec(x_64); +x_65 = lean_ctor_get(x_18, 4); +lean_dec(x_65); +x_66 = lean_ctor_get(x_18, 3); +lean_dec(x_66); +x_67 = lean_ctor_get(x_18, 2); +lean_dec(x_67); +x_68 = lean_ctor_get(x_18, 1); +lean_dec(x_68); +x_69 = lean_ctor_get(x_18, 0); +lean_dec(x_69); +lean_ctor_set(x_18, 4, x_45); +x_70 = lean_st_ref_set(x_2, x_18, x_19); lean_dec(x_2); -x_65 = !lean_is_exclusive(x_64); -if (x_65 == 0) +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) { -lean_object* x_66; -x_66 = lean_ctor_get(x_64, 0); -lean_dec(x_66); -lean_ctor_set(x_64, 0, x_41); -return x_64; +lean_object* x_72; +x_72 = lean_ctor_get(x_70, 0); +lean_dec(x_72); +lean_ctor_set(x_70, 0, x_44); +return x_70; } else { -lean_object* x_67; lean_object* x_68; -x_67 = lean_ctor_get(x_64, 1); -lean_inc(x_67); -lean_dec(x_64); -x_68 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_68, 0, x_41); -lean_ctor_set(x_68, 1, x_67); -return x_68; +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_70, 1); +lean_inc(x_73); +lean_dec(x_70); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_44); +lean_ctor_set(x_74, 1, x_73); +return x_74; } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_dec(x_18); -x_69 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_69, 0, x_20); -lean_ctor_set(x_69, 1, x_21); -lean_ctor_set(x_69, 2, x_22); -lean_ctor_set(x_69, 3, x_42); -lean_ctor_set(x_69, 4, x_24); -lean_ctor_set(x_69, 5, x_25); -lean_ctor_set(x_69, 6, x_27); -lean_ctor_set(x_69, 7, x_28); -lean_ctor_set(x_69, 8, x_29); -lean_ctor_set(x_69, 9, x_30); -lean_ctor_set(x_69, 10, x_31); -lean_ctor_set(x_69, 11, x_32); -lean_ctor_set(x_69, 12, x_33); -lean_ctor_set(x_69, 13, x_34); -lean_ctor_set(x_69, 14, x_35); -lean_ctor_set(x_69, 15, x_36); -lean_ctor_set(x_69, 16, x_37); -lean_ctor_set(x_69, 17, x_38); -lean_ctor_set(x_69, 18, x_39); -lean_ctor_set(x_69, 19, x_40); -lean_ctor_set_uint8(x_69, sizeof(void*)*20, x_26); -x_70 = lean_st_ref_set(x_2, x_69, x_19); -lean_dec(x_2); -x_71 = lean_ctor_get(x_70, 1); -lean_inc(x_71); -if (lean_is_exclusive(x_70)) { - lean_ctor_release(x_70, 0); - lean_ctor_release(x_70, 1); - x_72 = x_70; +x_75 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_75, 0, x_20); +lean_ctor_set(x_75, 1, x_21); +lean_ctor_set(x_75, 2, x_22); +lean_ctor_set(x_75, 3, x_23); +lean_ctor_set(x_75, 4, x_45); +lean_ctor_set(x_75, 5, x_25); +lean_ctor_set(x_75, 6, x_26); +lean_ctor_set(x_75, 7, x_28); +lean_ctor_set(x_75, 8, x_29); +lean_ctor_set(x_75, 9, x_30); +lean_ctor_set(x_75, 10, x_31); +lean_ctor_set(x_75, 11, x_32); +lean_ctor_set(x_75, 12, x_33); +lean_ctor_set(x_75, 13, x_34); +lean_ctor_set(x_75, 14, x_35); +lean_ctor_set(x_75, 15, x_36); +lean_ctor_set(x_75, 16, x_37); +lean_ctor_set(x_75, 17, x_38); +lean_ctor_set(x_75, 18, x_39); +lean_ctor_set(x_75, 19, x_40); +lean_ctor_set(x_75, 20, x_41); +lean_ctor_set(x_75, 21, x_42); +lean_ctor_set(x_75, 22, x_43); +lean_ctor_set_uint8(x_75, sizeof(void*)*23, x_27); +x_76 = lean_st_ref_set(x_2, x_75, x_19); +lean_dec(x_2); +x_77 = lean_ctor_get(x_76, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_76)) { + lean_ctor_release(x_76, 0); + lean_ctor_release(x_76, 1); + x_78 = x_76; } else { - lean_dec_ref(x_70); - x_72 = lean_box(0); + lean_dec_ref(x_76); + x_78 = lean_box(0); } -if (lean_is_scalar(x_72)) { - x_73 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_78)) { + x_79 = lean_alloc_ctor(0, 2, 0); } else { - x_73 = x_72; + x_79 = x_78; } -lean_ctor_set(x_73, 0, x_41); -lean_ctor_set(x_73, 1, x_71); -return x_73; +lean_ctor_set(x_79, 0, x_44); +lean_ctor_set(x_79, 1, x_77); +return x_79; } } else { -lean_object* x_74; uint8_t x_75; -x_74 = lean_ctor_get(x_16, 0); -lean_inc(x_74); +lean_object* x_80; uint8_t x_81; +x_80 = lean_ctor_get(x_16, 0); +lean_inc(x_80); lean_dec(x_16); -x_75 = !lean_is_exclusive(x_74); -if (x_75 == 0) +x_81 = !lean_is_exclusive(x_80); +if (x_81 == 0) { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; -x_76 = lean_ctor_get(x_74, 0); -x_77 = lean_ctor_get(x_74, 1); -lean_dec(x_77); -x_78 = l_Lean_Expr_getAppFn(x_1); -x_79 = l_Lean_Expr_getAppFn(x_76); -x_80 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_78, x_79); -if (x_80 == 0) +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +x_82 = lean_ctor_get(x_80, 0); +x_83 = lean_ctor_get(x_80, 1); +lean_dec(x_83); +x_84 = l_Lean_Expr_getAppFn(x_1); +x_85 = l_Lean_Expr_getAppFn(x_82); +x_86 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_84, x_85); +if (x_86 == 0) { -lean_object* x_81; +lean_object* x_87; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_81 = l_Lean_Meta_Grind_hasSameType(x_78, x_79, x_6, x_7, x_8, x_9, x_14); -if (lean_obj_tag(x_81) == 0) -{ -lean_object* x_82; uint8_t x_83; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_unbox(x_82); -lean_dec(x_82); -if (x_83 == 0) +x_87 = l_Lean_Meta_Grind_hasSameType(x_84, x_85, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_87) == 0) { -lean_object* x_84; lean_object* x_85; lean_object* x_86; uint8_t x_87; -x_84 = lean_ctor_get(x_81, 1); -lean_inc(x_84); -lean_dec(x_81); -x_85 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_86 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_85, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_84); -x_87 = !lean_is_exclusive(x_86); -if (x_87 == 0) -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; -x_88 = lean_ctor_get(x_86, 0); -x_89 = lean_ctor_get(x_86, 1); -x_90 = l_Lean_Meta_Grind_addCongrTable___closed__3; -x_91 = lean_unbox(x_88); +lean_object* x_88; uint8_t x_89; +x_88 = lean_ctor_get(x_87, 0); +lean_inc(x_88); +x_89 = lean_unbox(x_88); lean_dec(x_88); -if (x_91 == 0) +if (x_89 == 0) { -lean_object* x_92; lean_object* x_93; -lean_free_object(x_86); -lean_free_object(x_74); -lean_dec(x_76); +lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +x_91 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_92 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_91, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_90); +x_93 = !lean_is_exclusive(x_92); +if (x_93 == 0) +{ +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_92, 0); +x_95 = lean_ctor_get(x_92, 1); +x_96 = l_Lean_Meta_Grind_addCongrTable___closed__3; +x_97 = lean_unbox(x_94); +lean_dec(x_94); +if (x_97 == 0) +{ +lean_object* x_98; lean_object* x_99; +lean_free_object(x_92); +lean_free_object(x_80); +lean_dec(x_82); lean_free_object(x_11); lean_dec(x_1); -x_92 = lean_box(0); -x_93 = lean_apply_10(x_90, x_92, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_89); -return x_93; +x_98 = lean_box(0); +x_99 = lean_apply_10(x_96, x_98, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_95); +return x_99; } else { -lean_object* x_94; -x_94 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_89); -if (lean_obj_tag(x_94) == 0) +lean_object* x_100; +x_100 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_95); +if (lean_obj_tag(x_100) == 0) { -lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_95 = lean_ctor_get(x_94, 1); -lean_inc(x_95); -lean_dec(x_94); -x_96 = l_Lean_indentExpr(x_1); -x_97 = l_Lean_Meta_Grind_addCongrTable___closed__5; -lean_ctor_set_tag(x_86, 7); -lean_ctor_set(x_86, 1, x_96); -lean_ctor_set(x_86, 0, x_97); -x_98 = l_Lean_Meta_Grind_addCongrTable___closed__7; -lean_ctor_set_tag(x_74, 7); -lean_ctor_set(x_74, 1, x_98); -lean_ctor_set(x_74, 0, x_86); -x_99 = l_Lean_indentExpr(x_76); +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +x_102 = l_Lean_indentExpr(x_1); +x_103 = l_Lean_Meta_Grind_addCongrTable___closed__5; +lean_ctor_set_tag(x_92, 7); +lean_ctor_set(x_92, 1, x_102); +lean_ctor_set(x_92, 0, x_103); +x_104 = l_Lean_Meta_Grind_addCongrTable___closed__7; +lean_ctor_set_tag(x_80, 7); +lean_ctor_set(x_80, 1, x_104); +lean_ctor_set(x_80, 0, x_92); +x_105 = l_Lean_indentExpr(x_82); lean_ctor_set_tag(x_11, 7); -lean_ctor_set(x_11, 1, x_99); -lean_ctor_set(x_11, 0, x_74); -x_100 = l_Lean_Meta_Grind_addCongrTable___closed__9; -x_101 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_101, 0, x_11); -lean_ctor_set(x_101, 1, x_100); -x_102 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_85, x_101, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_95); -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -lean_dec(x_102); -x_105 = lean_apply_10(x_90, x_103, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_104); -return x_105; +lean_ctor_set(x_11, 1, x_105); +lean_ctor_set(x_11, 0, x_80); +x_106 = l_Lean_Meta_Grind_addCongrTable___closed__9; +x_107 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_107, 0, x_11); +lean_ctor_set(x_107, 1, x_106); +x_108 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_91, x_107, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_101); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_apply_10(x_96, x_109, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_110); +return x_111; } else { -uint8_t x_106; -lean_free_object(x_86); -lean_free_object(x_74); -lean_dec(x_76); +uint8_t x_112; +lean_free_object(x_92); +lean_free_object(x_80); +lean_dec(x_82); lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -1988,90 +2008,90 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_106 = !lean_is_exclusive(x_94); -if (x_106 == 0) +x_112 = !lean_is_exclusive(x_100); +if (x_112 == 0) { -return x_94; +return x_100; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_94, 0); -x_108 = lean_ctor_get(x_94, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_94); -x_109 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_108); -return x_109; +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_100, 0); +x_114 = lean_ctor_get(x_100, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_100); +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +return x_115; } } } } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; uint8_t x_113; -x_110 = lean_ctor_get(x_86, 0); -x_111 = lean_ctor_get(x_86, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_86); -x_112 = l_Lean_Meta_Grind_addCongrTable___closed__3; -x_113 = lean_unbox(x_110); -lean_dec(x_110); -if (x_113 == 0) -{ -lean_object* x_114; lean_object* x_115; -lean_free_object(x_74); -lean_dec(x_76); +lean_object* x_116; lean_object* x_117; lean_object* x_118; uint8_t x_119; +x_116 = lean_ctor_get(x_92, 0); +x_117 = lean_ctor_get(x_92, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_92); +x_118 = l_Lean_Meta_Grind_addCongrTable___closed__3; +x_119 = lean_unbox(x_116); +lean_dec(x_116); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; +lean_free_object(x_80); +lean_dec(x_82); lean_free_object(x_11); lean_dec(x_1); -x_114 = lean_box(0); -x_115 = lean_apply_10(x_112, x_114, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_111); -return x_115; +x_120 = lean_box(0); +x_121 = lean_apply_10(x_118, x_120, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_117); +return x_121; } else { -lean_object* x_116; -x_116 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_111); -if (lean_obj_tag(x_116) == 0) +lean_object* x_122; +x_122 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_117); +if (lean_obj_tag(x_122) == 0) { -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_117 = lean_ctor_get(x_116, 1); -lean_inc(x_117); -lean_dec(x_116); -x_118 = l_Lean_indentExpr(x_1); -x_119 = l_Lean_Meta_Grind_addCongrTable___closed__5; -x_120 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_120, 0, x_119); -lean_ctor_set(x_120, 1, x_118); -x_121 = l_Lean_Meta_Grind_addCongrTable___closed__7; -lean_ctor_set_tag(x_74, 7); -lean_ctor_set(x_74, 1, x_121); -lean_ctor_set(x_74, 0, x_120); -x_122 = l_Lean_indentExpr(x_76); +lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_123 = lean_ctor_get(x_122, 1); +lean_inc(x_123); +lean_dec(x_122); +x_124 = l_Lean_indentExpr(x_1); +x_125 = l_Lean_Meta_Grind_addCongrTable___closed__5; +x_126 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_124); +x_127 = l_Lean_Meta_Grind_addCongrTable___closed__7; +lean_ctor_set_tag(x_80, 7); +lean_ctor_set(x_80, 1, x_127); +lean_ctor_set(x_80, 0, x_126); +x_128 = l_Lean_indentExpr(x_82); lean_ctor_set_tag(x_11, 7); -lean_ctor_set(x_11, 1, x_122); -lean_ctor_set(x_11, 0, x_74); -x_123 = l_Lean_Meta_Grind_addCongrTable___closed__9; -x_124 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_124, 0, x_11); -lean_ctor_set(x_124, 1, x_123); -x_125 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_85, x_124, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_117); -x_126 = lean_ctor_get(x_125, 0); -lean_inc(x_126); -x_127 = lean_ctor_get(x_125, 1); -lean_inc(x_127); -lean_dec(x_125); -x_128 = lean_apply_10(x_112, x_126, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_127); -return x_128; +lean_ctor_set(x_11, 1, x_128); +lean_ctor_set(x_11, 0, x_80); +x_129 = l_Lean_Meta_Grind_addCongrTable___closed__9; +x_130 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_130, 0, x_11); +lean_ctor_set(x_130, 1, x_129); +x_131 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_91, x_130, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_123); +x_132 = lean_ctor_get(x_131, 0); +lean_inc(x_132); +x_133 = lean_ctor_get(x_131, 1); +lean_inc(x_133); +lean_dec(x_131); +x_134 = lean_apply_10(x_118, x_132, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_133); +return x_134; } else { -lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -lean_free_object(x_74); -lean_dec(x_76); +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_free_object(x_80); +lean_dec(x_82); lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -2082,52 +2102,52 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_129 = lean_ctor_get(x_116, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_116, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_116)) { - lean_ctor_release(x_116, 0); - lean_ctor_release(x_116, 1); - x_131 = x_116; +x_135 = lean_ctor_get(x_122, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_122, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_122)) { + lean_ctor_release(x_122, 0); + lean_ctor_release(x_122, 1); + x_137 = x_122; } else { - lean_dec_ref(x_116); - x_131 = lean_box(0); + lean_dec_ref(x_122); + x_137 = lean_box(0); } -if (lean_is_scalar(x_131)) { - x_132 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); } else { - x_132 = x_131; + x_138 = x_137; } -lean_ctor_set(x_132, 0, x_129); -lean_ctor_set(x_132, 1, x_130); -return x_132; +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; } } } } else { -lean_object* x_133; lean_object* x_134; lean_object* x_135; -lean_free_object(x_74); +lean_object* x_139; lean_object* x_140; lean_object* x_141; +lean_free_object(x_80); lean_free_object(x_11); -x_133 = lean_ctor_get(x_81, 1); -lean_inc(x_133); -lean_dec(x_81); -x_134 = lean_box(0); -x_135 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_76, x_134, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_133); +x_139 = lean_ctor_get(x_87, 1); +lean_inc(x_139); +lean_dec(x_87); +x_140 = lean_box(0); +x_141 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_82, x_140, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_139); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_135; +return x_141; } } else { -uint8_t x_136; -lean_free_object(x_74); -lean_dec(x_76); +uint8_t x_142; +lean_free_object(x_80); +lean_dec(x_82); lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -2138,146 +2158,146 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_136 = !lean_is_exclusive(x_81); -if (x_136 == 0) +x_142 = !lean_is_exclusive(x_87); +if (x_142 == 0) { -return x_81; +return x_87; } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_137 = lean_ctor_get(x_81, 0); -x_138 = lean_ctor_get(x_81, 1); -lean_inc(x_138); -lean_inc(x_137); -lean_dec(x_81); -x_139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -return x_139; +lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_143 = lean_ctor_get(x_87, 0); +x_144 = lean_ctor_get(x_87, 1); +lean_inc(x_144); +lean_inc(x_143); +lean_dec(x_87); +x_145 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_145, 0, x_143); +lean_ctor_set(x_145, 1, x_144); +return x_145; } } } else { -lean_object* x_140; lean_object* x_141; -lean_dec(x_79); -lean_dec(x_78); -lean_free_object(x_74); +lean_object* x_146; lean_object* x_147; +lean_dec(x_85); +lean_dec(x_84); +lean_free_object(x_80); lean_free_object(x_11); -x_140 = lean_box(0); -x_141 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_76, x_140, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +x_146 = lean_box(0); +x_147 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_82, x_146, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_141; +return x_147; } } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; uint8_t x_145; -x_142 = lean_ctor_get(x_74, 0); -lean_inc(x_142); -lean_dec(x_74); -x_143 = l_Lean_Expr_getAppFn(x_1); -x_144 = l_Lean_Expr_getAppFn(x_142); -x_145 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_143, x_144); -if (x_145 == 0) +lean_object* x_148; lean_object* x_149; lean_object* x_150; uint8_t x_151; +x_148 = lean_ctor_get(x_80, 0); +lean_inc(x_148); +lean_dec(x_80); +x_149 = l_Lean_Expr_getAppFn(x_1); +x_150 = l_Lean_Expr_getAppFn(x_148); +x_151 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_149, x_150); +if (x_151 == 0) { -lean_object* x_146; +lean_object* x_152; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_146 = l_Lean_Meta_Grind_hasSameType(x_143, x_144, x_6, x_7, x_8, x_9, x_14); -if (lean_obj_tag(x_146) == 0) -{ -lean_object* x_147; uint8_t x_148; -x_147 = lean_ctor_get(x_146, 0); -lean_inc(x_147); -x_148 = lean_unbox(x_147); -lean_dec(x_147); -if (x_148 == 0) +x_152 = l_Lean_Meta_Grind_hasSameType(x_149, x_150, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_152) == 0) { -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; -x_149 = lean_ctor_get(x_146, 1); -lean_inc(x_149); -lean_dec(x_146); -x_150 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_151 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_150, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_149); -x_152 = lean_ctor_get(x_151, 0); -lean_inc(x_152); -x_153 = lean_ctor_get(x_151, 1); +lean_object* x_153; uint8_t x_154; +x_153 = lean_ctor_get(x_152, 0); lean_inc(x_153); -if (lean_is_exclusive(x_151)) { - lean_ctor_release(x_151, 0); - lean_ctor_release(x_151, 1); - x_154 = x_151; +x_154 = lean_unbox(x_153); +lean_dec(x_153); +if (x_154 == 0) +{ +lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; uint8_t x_162; +x_155 = lean_ctor_get(x_152, 1); +lean_inc(x_155); +lean_dec(x_152); +x_156 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_157 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_156, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_155); +x_158 = lean_ctor_get(x_157, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_157, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_160 = x_157; } else { - lean_dec_ref(x_151); - x_154 = lean_box(0); + lean_dec_ref(x_157); + x_160 = lean_box(0); } -x_155 = l_Lean_Meta_Grind_addCongrTable___closed__3; -x_156 = lean_unbox(x_152); -lean_dec(x_152); -if (x_156 == 0) +x_161 = l_Lean_Meta_Grind_addCongrTable___closed__3; +x_162 = lean_unbox(x_158); +lean_dec(x_158); +if (x_162 == 0) { -lean_object* x_157; lean_object* x_158; -lean_dec(x_154); -lean_dec(x_142); +lean_object* x_163; lean_object* x_164; +lean_dec(x_160); +lean_dec(x_148); lean_free_object(x_11); lean_dec(x_1); -x_157 = lean_box(0); -x_158 = lean_apply_10(x_155, x_157, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_153); -return x_158; +x_163 = lean_box(0); +x_164 = lean_apply_10(x_161, x_163, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_159); +return x_164; } else { -lean_object* x_159; -x_159 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_153); -if (lean_obj_tag(x_159) == 0) +lean_object* x_165; +x_165 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_159); +if (lean_obj_tag(x_165) == 0) { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; -x_160 = lean_ctor_get(x_159, 1); -lean_inc(x_160); -lean_dec(x_159); -x_161 = l_Lean_indentExpr(x_1); -x_162 = l_Lean_Meta_Grind_addCongrTable___closed__5; -if (lean_is_scalar(x_154)) { - x_163 = lean_alloc_ctor(7, 2, 0); +lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; +x_166 = lean_ctor_get(x_165, 1); +lean_inc(x_166); +lean_dec(x_165); +x_167 = l_Lean_indentExpr(x_1); +x_168 = l_Lean_Meta_Grind_addCongrTable___closed__5; +if (lean_is_scalar(x_160)) { + x_169 = lean_alloc_ctor(7, 2, 0); } else { - x_163 = x_154; - lean_ctor_set_tag(x_163, 7); -} -lean_ctor_set(x_163, 0, x_162); -lean_ctor_set(x_163, 1, x_161); -x_164 = l_Lean_Meta_Grind_addCongrTable___closed__7; -x_165 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_165, 0, x_163); -lean_ctor_set(x_165, 1, x_164); -x_166 = l_Lean_indentExpr(x_142); + x_169 = x_160; + lean_ctor_set_tag(x_169, 7); +} +lean_ctor_set(x_169, 0, x_168); +lean_ctor_set(x_169, 1, x_167); +x_170 = l_Lean_Meta_Grind_addCongrTable___closed__7; +x_171 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_171, 0, x_169); +lean_ctor_set(x_171, 1, x_170); +x_172 = l_Lean_indentExpr(x_148); lean_ctor_set_tag(x_11, 7); -lean_ctor_set(x_11, 1, x_166); -lean_ctor_set(x_11, 0, x_165); -x_167 = l_Lean_Meta_Grind_addCongrTable___closed__9; -x_168 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_168, 0, x_11); -lean_ctor_set(x_168, 1, x_167); -x_169 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_150, x_168, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_160); -x_170 = lean_ctor_get(x_169, 0); -lean_inc(x_170); -x_171 = lean_ctor_get(x_169, 1); -lean_inc(x_171); -lean_dec(x_169); -x_172 = lean_apply_10(x_155, x_170, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_171); -return x_172; +lean_ctor_set(x_11, 1, x_172); +lean_ctor_set(x_11, 0, x_171); +x_173 = l_Lean_Meta_Grind_addCongrTable___closed__9; +x_174 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_174, 0, x_11); +lean_ctor_set(x_174, 1, x_173); +x_175 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_156, x_174, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_166); +x_176 = lean_ctor_get(x_175, 0); +lean_inc(x_176); +x_177 = lean_ctor_get(x_175, 1); +lean_inc(x_177); +lean_dec(x_175); +x_178 = lean_apply_10(x_161, x_176, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_177); +return x_178; } else { -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -lean_dec(x_154); -lean_dec(x_142); +lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +lean_dec(x_160); +lean_dec(x_148); lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -2288,49 +2308,49 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_173 = lean_ctor_get(x_159, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_159, 1); -lean_inc(x_174); -if (lean_is_exclusive(x_159)) { - lean_ctor_release(x_159, 0); - lean_ctor_release(x_159, 1); - x_175 = x_159; +x_179 = lean_ctor_get(x_165, 0); +lean_inc(x_179); +x_180 = lean_ctor_get(x_165, 1); +lean_inc(x_180); +if (lean_is_exclusive(x_165)) { + lean_ctor_release(x_165, 0); + lean_ctor_release(x_165, 1); + x_181 = x_165; } else { - lean_dec_ref(x_159); - x_175 = lean_box(0); + lean_dec_ref(x_165); + x_181 = lean_box(0); } -if (lean_is_scalar(x_175)) { - x_176 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_181)) { + x_182 = lean_alloc_ctor(1, 2, 0); } else { - x_176 = x_175; + x_182 = x_181; } -lean_ctor_set(x_176, 0, x_173); -lean_ctor_set(x_176, 1, x_174); -return x_176; +lean_ctor_set(x_182, 0, x_179); +lean_ctor_set(x_182, 1, x_180); +return x_182; } } } else { -lean_object* x_177; lean_object* x_178; lean_object* x_179; +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_free_object(x_11); -x_177 = lean_ctor_get(x_146, 1); -lean_inc(x_177); -lean_dec(x_146); -x_178 = lean_box(0); -x_179 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_142, x_178, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_177); +x_183 = lean_ctor_get(x_152, 1); +lean_inc(x_183); +lean_dec(x_152); +x_184 = lean_box(0); +x_185 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_148, x_184, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_183); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_179; +return x_185; } } else { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; -lean_dec(x_142); +lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; +lean_dec(x_148); lean_free_object(x_11); lean_dec(x_9); lean_dec(x_8); @@ -2341,60 +2361,60 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_180 = lean_ctor_get(x_146, 0); -lean_inc(x_180); -x_181 = lean_ctor_get(x_146, 1); -lean_inc(x_181); -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - lean_ctor_release(x_146, 1); - x_182 = x_146; +x_186 = lean_ctor_get(x_152, 0); +lean_inc(x_186); +x_187 = lean_ctor_get(x_152, 1); +lean_inc(x_187); +if (lean_is_exclusive(x_152)) { + lean_ctor_release(x_152, 0); + lean_ctor_release(x_152, 1); + x_188 = x_152; } else { - lean_dec_ref(x_146); - x_182 = lean_box(0); + lean_dec_ref(x_152); + x_188 = lean_box(0); } -if (lean_is_scalar(x_182)) { - x_183 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_188)) { + x_189 = lean_alloc_ctor(1, 2, 0); } else { - x_183 = x_182; + x_189 = x_188; } -lean_ctor_set(x_183, 0, x_180); -lean_ctor_set(x_183, 1, x_181); -return x_183; +lean_ctor_set(x_189, 0, x_186); +lean_ctor_set(x_189, 1, x_187); +return x_189; } } else { -lean_object* x_184; lean_object* x_185; -lean_dec(x_144); -lean_dec(x_143); +lean_object* x_190; lean_object* x_191; +lean_dec(x_150); +lean_dec(x_149); lean_free_object(x_11); -x_184 = lean_box(0); -x_185 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_142, x_184, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +x_190 = lean_box(0); +x_191 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_148, x_190, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_185; +return x_191; } } } } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; -x_186 = lean_ctor_get(x_11, 0); -x_187 = lean_ctor_get(x_11, 1); -lean_inc(x_187); -lean_inc(x_186); +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_192 = lean_ctor_get(x_11, 0); +x_193 = lean_ctor_get(x_11, 1); +lean_inc(x_193); +lean_inc(x_192); lean_dec(x_11); -x_188 = lean_ctor_get(x_186, 3); -lean_inc(x_188); +x_194 = lean_ctor_get(x_192, 4); +lean_inc(x_194); lean_inc(x_1); -x_189 = l_Lean_PersistentHashMap_findEntry_x3f___at_Lean_Meta_Grind_addCongrTable___spec__1(x_186, x_188, x_1); -if (lean_obj_tag(x_189) == 0) +x_195 = l_Lean_PersistentHashMap_findEntry_x3f___at_Lean_Meta_Grind_addCongrTable___spec__1(x_192, x_194, x_1); +if (lean_obj_tag(x_195) == 0) { -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; uint8_t x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; lean_object* x_230; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2402,249 +2422,261 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_190 = lean_st_ref_take(x_2, x_187); -x_191 = lean_ctor_get(x_190, 0); -lean_inc(x_191); -x_192 = lean_ctor_get(x_190, 1); -lean_inc(x_192); -lean_dec(x_190); -x_193 = lean_ctor_get(x_191, 0); -lean_inc(x_193); -x_194 = lean_ctor_get(x_191, 1); -lean_inc(x_194); -x_195 = lean_ctor_get(x_191, 2); -lean_inc(x_195); -x_196 = lean_ctor_get(x_191, 3); -lean_inc(x_196); -x_197 = lean_ctor_get(x_191, 4); +x_196 = lean_st_ref_take(x_2, x_193); +x_197 = lean_ctor_get(x_196, 0); lean_inc(x_197); -x_198 = lean_ctor_get(x_191, 5); +x_198 = lean_ctor_get(x_196, 1); lean_inc(x_198); -x_199 = lean_ctor_get_uint8(x_191, sizeof(void*)*20); -x_200 = lean_ctor_get(x_191, 6); +lean_dec(x_196); +x_199 = lean_ctor_get(x_197, 0); +lean_inc(x_199); +x_200 = lean_ctor_get(x_197, 1); lean_inc(x_200); -x_201 = lean_ctor_get(x_191, 7); +x_201 = lean_ctor_get(x_197, 2); lean_inc(x_201); -x_202 = lean_ctor_get(x_191, 8); +x_202 = lean_ctor_get(x_197, 3); lean_inc(x_202); -x_203 = lean_ctor_get(x_191, 9); +x_203 = lean_ctor_get(x_197, 4); lean_inc(x_203); -x_204 = lean_ctor_get(x_191, 10); +x_204 = lean_ctor_get(x_197, 5); lean_inc(x_204); -x_205 = lean_ctor_get(x_191, 11); +x_205 = lean_ctor_get(x_197, 6); lean_inc(x_205); -x_206 = lean_ctor_get(x_191, 12); -lean_inc(x_206); -x_207 = lean_ctor_get(x_191, 13); +x_206 = lean_ctor_get_uint8(x_197, sizeof(void*)*23); +x_207 = lean_ctor_get(x_197, 7); lean_inc(x_207); -x_208 = lean_ctor_get(x_191, 14); +x_208 = lean_ctor_get(x_197, 8); lean_inc(x_208); -x_209 = lean_ctor_get(x_191, 15); +x_209 = lean_ctor_get(x_197, 9); lean_inc(x_209); -x_210 = lean_ctor_get(x_191, 16); +x_210 = lean_ctor_get(x_197, 10); lean_inc(x_210); -x_211 = lean_ctor_get(x_191, 17); +x_211 = lean_ctor_get(x_197, 11); lean_inc(x_211); -x_212 = lean_ctor_get(x_191, 18); +x_212 = lean_ctor_get(x_197, 12); lean_inc(x_212); -x_213 = lean_ctor_get(x_191, 19); +x_213 = lean_ctor_get(x_197, 13); lean_inc(x_213); -x_214 = lean_box(0); -lean_inc(x_191); -x_215 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_addCongrTable___spec__4(x_191, x_196, x_1, x_214); -if (lean_is_exclusive(x_191)) { - lean_ctor_release(x_191, 0); - lean_ctor_release(x_191, 1); - lean_ctor_release(x_191, 2); - lean_ctor_release(x_191, 3); - lean_ctor_release(x_191, 4); - lean_ctor_release(x_191, 5); - lean_ctor_release(x_191, 6); - lean_ctor_release(x_191, 7); - lean_ctor_release(x_191, 8); - lean_ctor_release(x_191, 9); - lean_ctor_release(x_191, 10); - lean_ctor_release(x_191, 11); - lean_ctor_release(x_191, 12); - lean_ctor_release(x_191, 13); - lean_ctor_release(x_191, 14); - lean_ctor_release(x_191, 15); - lean_ctor_release(x_191, 16); - lean_ctor_release(x_191, 17); - lean_ctor_release(x_191, 18); - lean_ctor_release(x_191, 19); - x_216 = x_191; +x_214 = lean_ctor_get(x_197, 14); +lean_inc(x_214); +x_215 = lean_ctor_get(x_197, 15); +lean_inc(x_215); +x_216 = lean_ctor_get(x_197, 16); +lean_inc(x_216); +x_217 = lean_ctor_get(x_197, 17); +lean_inc(x_217); +x_218 = lean_ctor_get(x_197, 18); +lean_inc(x_218); +x_219 = lean_ctor_get(x_197, 19); +lean_inc(x_219); +x_220 = lean_ctor_get(x_197, 20); +lean_inc(x_220); +x_221 = lean_ctor_get(x_197, 21); +lean_inc(x_221); +x_222 = lean_ctor_get(x_197, 22); +lean_inc(x_222); +x_223 = lean_box(0); +lean_inc(x_197); +x_224 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_addCongrTable___spec__4(x_197, x_203, x_1, x_223); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + lean_ctor_release(x_197, 2); + lean_ctor_release(x_197, 3); + lean_ctor_release(x_197, 4); + lean_ctor_release(x_197, 5); + lean_ctor_release(x_197, 6); + lean_ctor_release(x_197, 7); + lean_ctor_release(x_197, 8); + lean_ctor_release(x_197, 9); + lean_ctor_release(x_197, 10); + lean_ctor_release(x_197, 11); + lean_ctor_release(x_197, 12); + lean_ctor_release(x_197, 13); + lean_ctor_release(x_197, 14); + lean_ctor_release(x_197, 15); + lean_ctor_release(x_197, 16); + lean_ctor_release(x_197, 17); + lean_ctor_release(x_197, 18); + lean_ctor_release(x_197, 19); + lean_ctor_release(x_197, 20); + lean_ctor_release(x_197, 21); + lean_ctor_release(x_197, 22); + x_225 = x_197; } else { - lean_dec_ref(x_191); - x_216 = lean_box(0); + lean_dec_ref(x_197); + x_225 = lean_box(0); } -if (lean_is_scalar(x_216)) { - x_217 = lean_alloc_ctor(0, 20, 1); +if (lean_is_scalar(x_225)) { + x_226 = lean_alloc_ctor(0, 23, 1); } else { - x_217 = x_216; -} -lean_ctor_set(x_217, 0, x_193); -lean_ctor_set(x_217, 1, x_194); -lean_ctor_set(x_217, 2, x_195); -lean_ctor_set(x_217, 3, x_215); -lean_ctor_set(x_217, 4, x_197); -lean_ctor_set(x_217, 5, x_198); -lean_ctor_set(x_217, 6, x_200); -lean_ctor_set(x_217, 7, x_201); -lean_ctor_set(x_217, 8, x_202); -lean_ctor_set(x_217, 9, x_203); -lean_ctor_set(x_217, 10, x_204); -lean_ctor_set(x_217, 11, x_205); -lean_ctor_set(x_217, 12, x_206); -lean_ctor_set(x_217, 13, x_207); -lean_ctor_set(x_217, 14, x_208); -lean_ctor_set(x_217, 15, x_209); -lean_ctor_set(x_217, 16, x_210); -lean_ctor_set(x_217, 17, x_211); -lean_ctor_set(x_217, 18, x_212); -lean_ctor_set(x_217, 19, x_213); -lean_ctor_set_uint8(x_217, sizeof(void*)*20, x_199); -x_218 = lean_st_ref_set(x_2, x_217, x_192); -lean_dec(x_2); -x_219 = lean_ctor_get(x_218, 1); -lean_inc(x_219); -if (lean_is_exclusive(x_218)) { - lean_ctor_release(x_218, 0); - lean_ctor_release(x_218, 1); - x_220 = x_218; + x_226 = x_225; +} +lean_ctor_set(x_226, 0, x_199); +lean_ctor_set(x_226, 1, x_200); +lean_ctor_set(x_226, 2, x_201); +lean_ctor_set(x_226, 3, x_202); +lean_ctor_set(x_226, 4, x_224); +lean_ctor_set(x_226, 5, x_204); +lean_ctor_set(x_226, 6, x_205); +lean_ctor_set(x_226, 7, x_207); +lean_ctor_set(x_226, 8, x_208); +lean_ctor_set(x_226, 9, x_209); +lean_ctor_set(x_226, 10, x_210); +lean_ctor_set(x_226, 11, x_211); +lean_ctor_set(x_226, 12, x_212); +lean_ctor_set(x_226, 13, x_213); +lean_ctor_set(x_226, 14, x_214); +lean_ctor_set(x_226, 15, x_215); +lean_ctor_set(x_226, 16, x_216); +lean_ctor_set(x_226, 17, x_217); +lean_ctor_set(x_226, 18, x_218); +lean_ctor_set(x_226, 19, x_219); +lean_ctor_set(x_226, 20, x_220); +lean_ctor_set(x_226, 21, x_221); +lean_ctor_set(x_226, 22, x_222); +lean_ctor_set_uint8(x_226, sizeof(void*)*23, x_206); +x_227 = lean_st_ref_set(x_2, x_226, x_198); +lean_dec(x_2); +x_228 = lean_ctor_get(x_227, 1); +lean_inc(x_228); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_229 = x_227; } else { - lean_dec_ref(x_218); - x_220 = lean_box(0); + lean_dec_ref(x_227); + x_229 = lean_box(0); } -if (lean_is_scalar(x_220)) { - x_221 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_229)) { + x_230 = lean_alloc_ctor(0, 2, 0); } else { - x_221 = x_220; + x_230 = x_229; } -lean_ctor_set(x_221, 0, x_214); -lean_ctor_set(x_221, 1, x_219); -return x_221; +lean_ctor_set(x_230, 0, x_223); +lean_ctor_set(x_230, 1, x_228); +return x_230; } else { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; uint8_t x_227; -x_222 = lean_ctor_get(x_189, 0); -lean_inc(x_222); -lean_dec(x_189); -x_223 = lean_ctor_get(x_222, 0); -lean_inc(x_223); -if (lean_is_exclusive(x_222)) { - lean_ctor_release(x_222, 0); - lean_ctor_release(x_222, 1); - x_224 = x_222; +lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; uint8_t x_236; +x_231 = lean_ctor_get(x_195, 0); +lean_inc(x_231); +lean_dec(x_195); +x_232 = lean_ctor_get(x_231, 0); +lean_inc(x_232); +if (lean_is_exclusive(x_231)) { + lean_ctor_release(x_231, 0); + lean_ctor_release(x_231, 1); + x_233 = x_231; } else { - lean_dec_ref(x_222); - x_224 = lean_box(0); + lean_dec_ref(x_231); + x_233 = lean_box(0); } -x_225 = l_Lean_Expr_getAppFn(x_1); -x_226 = l_Lean_Expr_getAppFn(x_223); -x_227 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_225, x_226); -if (x_227 == 0) +x_234 = l_Lean_Expr_getAppFn(x_1); +x_235 = l_Lean_Expr_getAppFn(x_232); +x_236 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_234, x_235); +if (x_236 == 0) { -lean_object* x_228; +lean_object* x_237; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_228 = l_Lean_Meta_Grind_hasSameType(x_225, x_226, x_6, x_7, x_8, x_9, x_187); -if (lean_obj_tag(x_228) == 0) -{ -lean_object* x_229; uint8_t x_230; -x_229 = lean_ctor_get(x_228, 0); -lean_inc(x_229); -x_230 = lean_unbox(x_229); -lean_dec(x_229); -if (x_230 == 0) -{ -lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; uint8_t x_238; -x_231 = lean_ctor_get(x_228, 1); -lean_inc(x_231); -lean_dec(x_228); -x_232 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_233 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_232, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_231); -x_234 = lean_ctor_get(x_233, 0); -lean_inc(x_234); -x_235 = lean_ctor_get(x_233, 1); -lean_inc(x_235); -if (lean_is_exclusive(x_233)) { - lean_ctor_release(x_233, 0); - lean_ctor_release(x_233, 1); - x_236 = x_233; +x_237 = l_Lean_Meta_Grind_hasSameType(x_234, x_235, x_6, x_7, x_8, x_9, x_193); +if (lean_obj_tag(x_237) == 0) +{ +lean_object* x_238; uint8_t x_239; +x_238 = lean_ctor_get(x_237, 0); +lean_inc(x_238); +x_239 = lean_unbox(x_238); +lean_dec(x_238); +if (x_239 == 0) +{ +lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; uint8_t x_247; +x_240 = lean_ctor_get(x_237, 1); +lean_inc(x_240); +lean_dec(x_237); +x_241 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_242 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_241, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_240); +x_243 = lean_ctor_get(x_242, 0); +lean_inc(x_243); +x_244 = lean_ctor_get(x_242, 1); +lean_inc(x_244); +if (lean_is_exclusive(x_242)) { + lean_ctor_release(x_242, 0); + lean_ctor_release(x_242, 1); + x_245 = x_242; } else { - lean_dec_ref(x_233); - x_236 = lean_box(0); + lean_dec_ref(x_242); + x_245 = lean_box(0); } -x_237 = l_Lean_Meta_Grind_addCongrTable___closed__3; -x_238 = lean_unbox(x_234); -lean_dec(x_234); -if (x_238 == 0) +x_246 = l_Lean_Meta_Grind_addCongrTable___closed__3; +x_247 = lean_unbox(x_243); +lean_dec(x_243); +if (x_247 == 0) { -lean_object* x_239; lean_object* x_240; -lean_dec(x_236); -lean_dec(x_224); -lean_dec(x_223); +lean_object* x_248; lean_object* x_249; +lean_dec(x_245); +lean_dec(x_233); +lean_dec(x_232); lean_dec(x_1); -x_239 = lean_box(0); -x_240 = lean_apply_10(x_237, x_239, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_235); -return x_240; +x_248 = lean_box(0); +x_249 = lean_apply_10(x_246, x_248, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_244); +return x_249; } else { -lean_object* x_241; -x_241 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_235); -if (lean_obj_tag(x_241) == 0) +lean_object* x_250; +x_250 = l_Lean_Meta_Grind_updateLastTag(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_244); +if (lean_obj_tag(x_250) == 0) { -lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; -x_242 = lean_ctor_get(x_241, 1); -lean_inc(x_242); -lean_dec(x_241); -x_243 = l_Lean_indentExpr(x_1); -x_244 = l_Lean_Meta_Grind_addCongrTable___closed__5; -if (lean_is_scalar(x_236)) { - x_245 = lean_alloc_ctor(7, 2, 0); +lean_object* x_251; lean_object* x_252; lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; +x_251 = lean_ctor_get(x_250, 1); +lean_inc(x_251); +lean_dec(x_250); +x_252 = l_Lean_indentExpr(x_1); +x_253 = l_Lean_Meta_Grind_addCongrTable___closed__5; +if (lean_is_scalar(x_245)) { + x_254 = lean_alloc_ctor(7, 2, 0); } else { - x_245 = x_236; - lean_ctor_set_tag(x_245, 7); -} -lean_ctor_set(x_245, 0, x_244); -lean_ctor_set(x_245, 1, x_243); -x_246 = l_Lean_Meta_Grind_addCongrTable___closed__7; -if (lean_is_scalar(x_224)) { - x_247 = lean_alloc_ctor(7, 2, 0); + x_254 = x_245; + lean_ctor_set_tag(x_254, 7); +} +lean_ctor_set(x_254, 0, x_253); +lean_ctor_set(x_254, 1, x_252); +x_255 = l_Lean_Meta_Grind_addCongrTable___closed__7; +if (lean_is_scalar(x_233)) { + x_256 = lean_alloc_ctor(7, 2, 0); } else { - x_247 = x_224; - lean_ctor_set_tag(x_247, 7); -} -lean_ctor_set(x_247, 0, x_245); -lean_ctor_set(x_247, 1, x_246); -x_248 = l_Lean_indentExpr(x_223); -x_249 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_249, 0, x_247); -lean_ctor_set(x_249, 1, x_248); -x_250 = l_Lean_Meta_Grind_addCongrTable___closed__9; -x_251 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_251, 0, x_249); -lean_ctor_set(x_251, 1, x_250); -x_252 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_232, x_251, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_242); -x_253 = lean_ctor_get(x_252, 0); -lean_inc(x_253); -x_254 = lean_ctor_get(x_252, 1); -lean_inc(x_254); -lean_dec(x_252); -x_255 = lean_apply_10(x_237, x_253, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_254); -return x_255; + x_256 = x_233; + lean_ctor_set_tag(x_256, 7); +} +lean_ctor_set(x_256, 0, x_254); +lean_ctor_set(x_256, 1, x_255); +x_257 = l_Lean_indentExpr(x_232); +x_258 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_258, 0, x_256); +lean_ctor_set(x_258, 1, x_257); +x_259 = l_Lean_Meta_Grind_addCongrTable___closed__9; +x_260 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_260, 0, x_258); +lean_ctor_set(x_260, 1, x_259); +x_261 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_241, x_260, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_251); +x_262 = lean_ctor_get(x_261, 0); +lean_inc(x_262); +x_263 = lean_ctor_get(x_261, 1); +lean_inc(x_263); +lean_dec(x_261); +x_264 = lean_apply_10(x_246, x_262, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_263); +return x_264; } else { -lean_object* x_256; lean_object* x_257; lean_object* x_258; lean_object* x_259; -lean_dec(x_236); -lean_dec(x_224); -lean_dec(x_223); +lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +lean_dec(x_245); +lean_dec(x_233); +lean_dec(x_232); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2654,50 +2686,50 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_256 = lean_ctor_get(x_241, 0); -lean_inc(x_256); -x_257 = lean_ctor_get(x_241, 1); -lean_inc(x_257); -if (lean_is_exclusive(x_241)) { - lean_ctor_release(x_241, 0); - lean_ctor_release(x_241, 1); - x_258 = x_241; +x_265 = lean_ctor_get(x_250, 0); +lean_inc(x_265); +x_266 = lean_ctor_get(x_250, 1); +lean_inc(x_266); +if (lean_is_exclusive(x_250)) { + lean_ctor_release(x_250, 0); + lean_ctor_release(x_250, 1); + x_267 = x_250; } else { - lean_dec_ref(x_241); - x_258 = lean_box(0); + lean_dec_ref(x_250); + x_267 = lean_box(0); } -if (lean_is_scalar(x_258)) { - x_259 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_267)) { + x_268 = lean_alloc_ctor(1, 2, 0); } else { - x_259 = x_258; + x_268 = x_267; } -lean_ctor_set(x_259, 0, x_256); -lean_ctor_set(x_259, 1, x_257); -return x_259; +lean_ctor_set(x_268, 0, x_265); +lean_ctor_set(x_268, 1, x_266); +return x_268; } } } else { -lean_object* x_260; lean_object* x_261; lean_object* x_262; -lean_dec(x_224); -x_260 = lean_ctor_get(x_228, 1); -lean_inc(x_260); -lean_dec(x_228); -x_261 = lean_box(0); -x_262 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_223, x_261, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_260); +lean_object* x_269; lean_object* x_270; lean_object* x_271; +lean_dec(x_233); +x_269 = lean_ctor_get(x_237, 1); +lean_inc(x_269); +lean_dec(x_237); +x_270 = lean_box(0); +x_271 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_232, x_270, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_269); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_262; +return x_271; } } else { -lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; -lean_dec(x_224); -lean_dec(x_223); +lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; +lean_dec(x_233); +lean_dec(x_232); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2707,41 +2739,41 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_263 = lean_ctor_get(x_228, 0); -lean_inc(x_263); -x_264 = lean_ctor_get(x_228, 1); -lean_inc(x_264); -if (lean_is_exclusive(x_228)) { - lean_ctor_release(x_228, 0); - lean_ctor_release(x_228, 1); - x_265 = x_228; +x_272 = lean_ctor_get(x_237, 0); +lean_inc(x_272); +x_273 = lean_ctor_get(x_237, 1); +lean_inc(x_273); +if (lean_is_exclusive(x_237)) { + lean_ctor_release(x_237, 0); + lean_ctor_release(x_237, 1); + x_274 = x_237; } else { - lean_dec_ref(x_228); - x_265 = lean_box(0); + lean_dec_ref(x_237); + x_274 = lean_box(0); } -if (lean_is_scalar(x_265)) { - x_266 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_274)) { + x_275 = lean_alloc_ctor(1, 2, 0); } else { - x_266 = x_265; + x_275 = x_274; } -lean_ctor_set(x_266, 0, x_263); -lean_ctor_set(x_266, 1, x_264); -return x_266; +lean_ctor_set(x_275, 0, x_272); +lean_ctor_set(x_275, 1, x_273); +return x_275; } } else { -lean_object* x_267; lean_object* x_268; -lean_dec(x_226); -lean_dec(x_225); -lean_dec(x_224); -x_267 = lean_box(0); -x_268 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_223, x_267, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_187); +lean_object* x_276; lean_object* x_277; +lean_dec(x_235); +lean_dec(x_234); +lean_dec(x_233); +x_276 = lean_box(0); +x_277 = l_Lean_Meta_Grind_addCongrTable___lambda__2(x_1, x_232, x_276, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_193); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_268; +return x_277; } } } @@ -3547,7 +3579,7 @@ if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; x_16 = lean_ctor_get(x_12, 1); -x_17 = lean_ctor_get(x_14, 4); +x_17 = lean_ctor_get(x_14, 5); lean_inc(x_17); x_18 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__1(x_17, x_11); if (lean_obj_tag(x_18) == 0) @@ -3558,7 +3590,7 @@ lean_ctor_set_tag(x_12, 1); lean_ctor_set(x_12, 1, x_19); lean_ctor_set(x_12, 0, x_1); x_20 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_17, x_11, x_12); -lean_ctor_set(x_14, 4, x_20); +lean_ctor_set(x_14, 5, x_20); x_21 = lean_st_ref_set(x_2, x_14, x_16); x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) @@ -3593,7 +3625,7 @@ lean_ctor_set_tag(x_12, 1); lean_ctor_set(x_12, 1, x_28); lean_ctor_set(x_12, 0, x_1); x_29 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_17, x_11, x_12); -lean_ctor_set(x_14, 4, x_29); +lean_ctor_set(x_14, 5, x_29); x_30 = lean_st_ref_set(x_2, x_14, x_16); x_31 = !lean_is_exclusive(x_30); if (x_31 == 0) @@ -3621,7 +3653,7 @@ return x_36; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; x_37 = lean_ctor_get(x_12, 1); x_38 = lean_ctor_get(x_14, 0); x_39 = lean_ctor_get(x_14, 1); @@ -3629,8 +3661,8 @@ x_40 = lean_ctor_get(x_14, 2); x_41 = lean_ctor_get(x_14, 3); x_42 = lean_ctor_get(x_14, 4); x_43 = lean_ctor_get(x_14, 5); -x_44 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); -x_45 = lean_ctor_get(x_14, 6); +x_44 = lean_ctor_get(x_14, 6); +x_45 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); x_46 = lean_ctor_get(x_14, 7); x_47 = lean_ctor_get(x_14, 8); x_48 = lean_ctor_get(x_14, 9); @@ -3644,6 +3676,12 @@ x_55 = lean_ctor_get(x_14, 16); x_56 = lean_ctor_get(x_14, 17); x_57 = lean_ctor_get(x_14, 18); x_58 = lean_ctor_get(x_14, 19); +x_59 = lean_ctor_get(x_14, 20); +x_60 = lean_ctor_get(x_14, 21); +x_61 = lean_ctor_get(x_14, 22); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); @@ -3657,7 +3695,7 @@ lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); -lean_inc(x_45); +lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); lean_inc(x_41); @@ -3665,302 +3703,323 @@ lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); lean_dec(x_14); -lean_inc(x_42); -x_59 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__1(x_42, x_11); -if (lean_obj_tag(x_59) == 0) +lean_inc(x_43); +x_62 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__1(x_43, x_11); +if (lean_obj_tag(x_62) == 0) { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_60 = lean_box(0); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_63 = lean_box(0); lean_ctor_set_tag(x_12, 1); -lean_ctor_set(x_12, 1, x_60); +lean_ctor_set(x_12, 1, x_63); lean_ctor_set(x_12, 0, x_1); -x_61 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_42, x_11, x_12); -x_62 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_62, 0, x_38); -lean_ctor_set(x_62, 1, x_39); -lean_ctor_set(x_62, 2, x_40); -lean_ctor_set(x_62, 3, x_41); -lean_ctor_set(x_62, 4, x_61); -lean_ctor_set(x_62, 5, x_43); -lean_ctor_set(x_62, 6, x_45); -lean_ctor_set(x_62, 7, x_46); -lean_ctor_set(x_62, 8, x_47); -lean_ctor_set(x_62, 9, x_48); -lean_ctor_set(x_62, 10, x_49); -lean_ctor_set(x_62, 11, x_50); -lean_ctor_set(x_62, 12, x_51); -lean_ctor_set(x_62, 13, x_52); -lean_ctor_set(x_62, 14, x_53); -lean_ctor_set(x_62, 15, x_54); -lean_ctor_set(x_62, 16, x_55); -lean_ctor_set(x_62, 17, x_56); -lean_ctor_set(x_62, 18, x_57); -lean_ctor_set(x_62, 19, x_58); -lean_ctor_set_uint8(x_62, sizeof(void*)*20, x_44); -x_63 = lean_st_ref_set(x_2, x_62, x_37); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +x_64 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_43, x_11, x_12); +x_65 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_65, 0, x_38); +lean_ctor_set(x_65, 1, x_39); +lean_ctor_set(x_65, 2, x_40); +lean_ctor_set(x_65, 3, x_41); +lean_ctor_set(x_65, 4, x_42); +lean_ctor_set(x_65, 5, x_64); +lean_ctor_set(x_65, 6, x_44); +lean_ctor_set(x_65, 7, x_46); +lean_ctor_set(x_65, 8, x_47); +lean_ctor_set(x_65, 9, x_48); +lean_ctor_set(x_65, 10, x_49); +lean_ctor_set(x_65, 11, x_50); +lean_ctor_set(x_65, 12, x_51); +lean_ctor_set(x_65, 13, x_52); +lean_ctor_set(x_65, 14, x_53); +lean_ctor_set(x_65, 15, x_54); +lean_ctor_set(x_65, 16, x_55); +lean_ctor_set(x_65, 17, x_56); +lean_ctor_set(x_65, 18, x_57); +lean_ctor_set(x_65, 19, x_58); +lean_ctor_set(x_65, 20, x_59); +lean_ctor_set(x_65, 21, x_60); +lean_ctor_set(x_65, 22, x_61); +lean_ctor_set_uint8(x_65, sizeof(void*)*23, x_45); +x_66 = lean_st_ref_set(x_2, x_65, x_37); +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_68 = x_66; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_66); + x_68 = lean_box(0); } -x_66 = lean_box(0); -if (lean_is_scalar(x_65)) { - x_67 = lean_alloc_ctor(0, 2, 0); +x_69 = lean_box(0); +if (lean_is_scalar(x_68)) { + x_70 = lean_alloc_ctor(0, 2, 0); } else { - x_67 = x_65; + x_70 = x_68; } -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_64); -return x_67; +lean_ctor_set(x_70, 0, x_69); +lean_ctor_set(x_70, 1, x_67); +return x_70; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; -x_68 = lean_ctor_get(x_59, 0); -lean_inc(x_68); -lean_dec(x_59); +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_71 = lean_ctor_get(x_62, 0); +lean_inc(x_71); +lean_dec(x_62); lean_ctor_set_tag(x_12, 1); -lean_ctor_set(x_12, 1, x_68); +lean_ctor_set(x_12, 1, x_71); lean_ctor_set(x_12, 0, x_1); -x_69 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_42, x_11, x_12); -x_70 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_70, 0, x_38); -lean_ctor_set(x_70, 1, x_39); -lean_ctor_set(x_70, 2, x_40); -lean_ctor_set(x_70, 3, x_41); -lean_ctor_set(x_70, 4, x_69); -lean_ctor_set(x_70, 5, x_43); -lean_ctor_set(x_70, 6, x_45); -lean_ctor_set(x_70, 7, x_46); -lean_ctor_set(x_70, 8, x_47); -lean_ctor_set(x_70, 9, x_48); -lean_ctor_set(x_70, 10, x_49); -lean_ctor_set(x_70, 11, x_50); -lean_ctor_set(x_70, 12, x_51); -lean_ctor_set(x_70, 13, x_52); -lean_ctor_set(x_70, 14, x_53); -lean_ctor_set(x_70, 15, x_54); -lean_ctor_set(x_70, 16, x_55); -lean_ctor_set(x_70, 17, x_56); -lean_ctor_set(x_70, 18, x_57); -lean_ctor_set(x_70, 19, x_58); -lean_ctor_set_uint8(x_70, sizeof(void*)*20, x_44); -x_71 = lean_st_ref_set(x_2, x_70, x_37); -x_72 = lean_ctor_get(x_71, 1); -lean_inc(x_72); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_73 = x_71; +x_72 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_43, x_11, x_12); +x_73 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_73, 0, x_38); +lean_ctor_set(x_73, 1, x_39); +lean_ctor_set(x_73, 2, x_40); +lean_ctor_set(x_73, 3, x_41); +lean_ctor_set(x_73, 4, x_42); +lean_ctor_set(x_73, 5, x_72); +lean_ctor_set(x_73, 6, x_44); +lean_ctor_set(x_73, 7, x_46); +lean_ctor_set(x_73, 8, x_47); +lean_ctor_set(x_73, 9, x_48); +lean_ctor_set(x_73, 10, x_49); +lean_ctor_set(x_73, 11, x_50); +lean_ctor_set(x_73, 12, x_51); +lean_ctor_set(x_73, 13, x_52); +lean_ctor_set(x_73, 14, x_53); +lean_ctor_set(x_73, 15, x_54); +lean_ctor_set(x_73, 16, x_55); +lean_ctor_set(x_73, 17, x_56); +lean_ctor_set(x_73, 18, x_57); +lean_ctor_set(x_73, 19, x_58); +lean_ctor_set(x_73, 20, x_59); +lean_ctor_set(x_73, 21, x_60); +lean_ctor_set(x_73, 22, x_61); +lean_ctor_set_uint8(x_73, sizeof(void*)*23, x_45); +x_74 = lean_st_ref_set(x_2, x_73, x_37); +x_75 = lean_ctor_get(x_74, 1); +lean_inc(x_75); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_76 = x_74; } else { - lean_dec_ref(x_71); - x_73 = lean_box(0); + lean_dec_ref(x_74); + x_76 = lean_box(0); } -x_74 = lean_box(0); -if (lean_is_scalar(x_73)) { - x_75 = lean_alloc_ctor(0, 2, 0); +x_77 = lean_box(0); +if (lean_is_scalar(x_76)) { + x_78 = lean_alloc_ctor(0, 2, 0); } else { - x_75 = x_73; + x_78 = x_76; } -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_72); -return x_75; +lean_ctor_set(x_78, 0, x_77); +lean_ctor_set(x_78, 1, x_75); +return x_78; } } } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_76 = lean_ctor_get(x_12, 0); -x_77 = lean_ctor_get(x_12, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_12); -x_78 = lean_ctor_get(x_76, 0); -lean_inc(x_78); -x_79 = lean_ctor_get(x_76, 1); -lean_inc(x_79); -x_80 = lean_ctor_get(x_76, 2); +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_79 = lean_ctor_get(x_12, 0); +x_80 = lean_ctor_get(x_12, 1); lean_inc(x_80); -x_81 = lean_ctor_get(x_76, 3); +lean_inc(x_79); +lean_dec(x_12); +x_81 = lean_ctor_get(x_79, 0); lean_inc(x_81); -x_82 = lean_ctor_get(x_76, 4); +x_82 = lean_ctor_get(x_79, 1); lean_inc(x_82); -x_83 = lean_ctor_get(x_76, 5); +x_83 = lean_ctor_get(x_79, 2); lean_inc(x_83); -x_84 = lean_ctor_get_uint8(x_76, sizeof(void*)*20); -x_85 = lean_ctor_get(x_76, 6); +x_84 = lean_ctor_get(x_79, 3); +lean_inc(x_84); +x_85 = lean_ctor_get(x_79, 4); lean_inc(x_85); -x_86 = lean_ctor_get(x_76, 7); +x_86 = lean_ctor_get(x_79, 5); lean_inc(x_86); -x_87 = lean_ctor_get(x_76, 8); +x_87 = lean_ctor_get(x_79, 6); lean_inc(x_87); -x_88 = lean_ctor_get(x_76, 9); -lean_inc(x_88); -x_89 = lean_ctor_get(x_76, 10); +x_88 = lean_ctor_get_uint8(x_79, sizeof(void*)*23); +x_89 = lean_ctor_get(x_79, 7); lean_inc(x_89); -x_90 = lean_ctor_get(x_76, 11); +x_90 = lean_ctor_get(x_79, 8); lean_inc(x_90); -x_91 = lean_ctor_get(x_76, 12); +x_91 = lean_ctor_get(x_79, 9); lean_inc(x_91); -x_92 = lean_ctor_get(x_76, 13); +x_92 = lean_ctor_get(x_79, 10); lean_inc(x_92); -x_93 = lean_ctor_get(x_76, 14); +x_93 = lean_ctor_get(x_79, 11); lean_inc(x_93); -x_94 = lean_ctor_get(x_76, 15); +x_94 = lean_ctor_get(x_79, 12); lean_inc(x_94); -x_95 = lean_ctor_get(x_76, 16); +x_95 = lean_ctor_get(x_79, 13); lean_inc(x_95); -x_96 = lean_ctor_get(x_76, 17); +x_96 = lean_ctor_get(x_79, 14); lean_inc(x_96); -x_97 = lean_ctor_get(x_76, 18); +x_97 = lean_ctor_get(x_79, 15); lean_inc(x_97); -x_98 = lean_ctor_get(x_76, 19); +x_98 = lean_ctor_get(x_79, 16); lean_inc(x_98); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - lean_ctor_release(x_76, 2); - lean_ctor_release(x_76, 3); - lean_ctor_release(x_76, 4); - lean_ctor_release(x_76, 5); - lean_ctor_release(x_76, 6); - lean_ctor_release(x_76, 7); - lean_ctor_release(x_76, 8); - lean_ctor_release(x_76, 9); - lean_ctor_release(x_76, 10); - lean_ctor_release(x_76, 11); - lean_ctor_release(x_76, 12); - lean_ctor_release(x_76, 13); - lean_ctor_release(x_76, 14); - lean_ctor_release(x_76, 15); - lean_ctor_release(x_76, 16); - lean_ctor_release(x_76, 17); - lean_ctor_release(x_76, 18); - lean_ctor_release(x_76, 19); - x_99 = x_76; +x_99 = lean_ctor_get(x_79, 17); +lean_inc(x_99); +x_100 = lean_ctor_get(x_79, 18); +lean_inc(x_100); +x_101 = lean_ctor_get(x_79, 19); +lean_inc(x_101); +x_102 = lean_ctor_get(x_79, 20); +lean_inc(x_102); +x_103 = lean_ctor_get(x_79, 21); +lean_inc(x_103); +x_104 = lean_ctor_get(x_79, 22); +lean_inc(x_104); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + lean_ctor_release(x_79, 2); + lean_ctor_release(x_79, 3); + lean_ctor_release(x_79, 4); + lean_ctor_release(x_79, 5); + lean_ctor_release(x_79, 6); + lean_ctor_release(x_79, 7); + lean_ctor_release(x_79, 8); + lean_ctor_release(x_79, 9); + lean_ctor_release(x_79, 10); + lean_ctor_release(x_79, 11); + lean_ctor_release(x_79, 12); + lean_ctor_release(x_79, 13); + lean_ctor_release(x_79, 14); + lean_ctor_release(x_79, 15); + lean_ctor_release(x_79, 16); + lean_ctor_release(x_79, 17); + lean_ctor_release(x_79, 18); + lean_ctor_release(x_79, 19); + lean_ctor_release(x_79, 20); + lean_ctor_release(x_79, 21); + lean_ctor_release(x_79, 22); + x_105 = x_79; } else { - lean_dec_ref(x_76); - x_99 = lean_box(0); + lean_dec_ref(x_79); + x_105 = lean_box(0); } -lean_inc(x_82); -x_100 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__1(x_82, x_11); -if (lean_obj_tag(x_100) == 0) -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_101 = lean_box(0); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_1); -lean_ctor_set(x_102, 1, x_101); -x_103 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_82, x_11, x_102); -if (lean_is_scalar(x_99)) { - x_104 = lean_alloc_ctor(0, 20, 1); +lean_inc(x_86); +x_106 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__1(x_86, x_11); +if (lean_obj_tag(x_106) == 0) +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_107 = lean_box(0); +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_1); +lean_ctor_set(x_108, 1, x_107); +x_109 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_86, x_11, x_108); +if (lean_is_scalar(x_105)) { + x_110 = lean_alloc_ctor(0, 23, 1); } else { - x_104 = x_99; -} -lean_ctor_set(x_104, 0, x_78); -lean_ctor_set(x_104, 1, x_79); -lean_ctor_set(x_104, 2, x_80); -lean_ctor_set(x_104, 3, x_81); -lean_ctor_set(x_104, 4, x_103); -lean_ctor_set(x_104, 5, x_83); -lean_ctor_set(x_104, 6, x_85); -lean_ctor_set(x_104, 7, x_86); -lean_ctor_set(x_104, 8, x_87); -lean_ctor_set(x_104, 9, x_88); -lean_ctor_set(x_104, 10, x_89); -lean_ctor_set(x_104, 11, x_90); -lean_ctor_set(x_104, 12, x_91); -lean_ctor_set(x_104, 13, x_92); -lean_ctor_set(x_104, 14, x_93); -lean_ctor_set(x_104, 15, x_94); -lean_ctor_set(x_104, 16, x_95); -lean_ctor_set(x_104, 17, x_96); -lean_ctor_set(x_104, 18, x_97); -lean_ctor_set(x_104, 19, x_98); -lean_ctor_set_uint8(x_104, sizeof(void*)*20, x_84); -x_105 = lean_st_ref_set(x_2, x_104, x_77); -x_106 = lean_ctor_get(x_105, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_105)) { - lean_ctor_release(x_105, 0); - lean_ctor_release(x_105, 1); - x_107 = x_105; + x_110 = x_105; +} +lean_ctor_set(x_110, 0, x_81); +lean_ctor_set(x_110, 1, x_82); +lean_ctor_set(x_110, 2, x_83); +lean_ctor_set(x_110, 3, x_84); +lean_ctor_set(x_110, 4, x_85); +lean_ctor_set(x_110, 5, x_109); +lean_ctor_set(x_110, 6, x_87); +lean_ctor_set(x_110, 7, x_89); +lean_ctor_set(x_110, 8, x_90); +lean_ctor_set(x_110, 9, x_91); +lean_ctor_set(x_110, 10, x_92); +lean_ctor_set(x_110, 11, x_93); +lean_ctor_set(x_110, 12, x_94); +lean_ctor_set(x_110, 13, x_95); +lean_ctor_set(x_110, 14, x_96); +lean_ctor_set(x_110, 15, x_97); +lean_ctor_set(x_110, 16, x_98); +lean_ctor_set(x_110, 17, x_99); +lean_ctor_set(x_110, 18, x_100); +lean_ctor_set(x_110, 19, x_101); +lean_ctor_set(x_110, 20, x_102); +lean_ctor_set(x_110, 21, x_103); +lean_ctor_set(x_110, 22, x_104); +lean_ctor_set_uint8(x_110, sizeof(void*)*23, x_88); +x_111 = lean_st_ref_set(x_2, x_110, x_80); +x_112 = lean_ctor_get(x_111, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_111)) { + lean_ctor_release(x_111, 0); + lean_ctor_release(x_111, 1); + x_113 = x_111; } else { - lean_dec_ref(x_105); - x_107 = lean_box(0); + lean_dec_ref(x_111); + x_113 = lean_box(0); } -x_108 = lean_box(0); -if (lean_is_scalar(x_107)) { - x_109 = lean_alloc_ctor(0, 2, 0); +x_114 = lean_box(0); +if (lean_is_scalar(x_113)) { + x_115 = lean_alloc_ctor(0, 2, 0); } else { - x_109 = x_107; + x_115 = x_113; } -lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_106); -return x_109; +lean_ctor_set(x_115, 0, x_114); +lean_ctor_set(x_115, 1, x_112); +return x_115; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_110 = lean_ctor_get(x_100, 0); -lean_inc(x_110); -lean_dec(x_100); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_1); -lean_ctor_set(x_111, 1, x_110); -x_112 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_82, x_11, x_111); -if (lean_is_scalar(x_99)) { - x_113 = lean_alloc_ctor(0, 20, 1); +lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_116 = lean_ctor_get(x_106, 0); +lean_inc(x_116); +lean_dec(x_106); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_1); +lean_ctor_set(x_117, 1, x_116); +x_118 = l_Lean_PersistentHashMap_insert___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap___spec__4(x_86, x_11, x_117); +if (lean_is_scalar(x_105)) { + x_119 = lean_alloc_ctor(0, 23, 1); } else { - x_113 = x_99; -} -lean_ctor_set(x_113, 0, x_78); -lean_ctor_set(x_113, 1, x_79); -lean_ctor_set(x_113, 2, x_80); -lean_ctor_set(x_113, 3, x_81); -lean_ctor_set(x_113, 4, x_112); -lean_ctor_set(x_113, 5, x_83); -lean_ctor_set(x_113, 6, x_85); -lean_ctor_set(x_113, 7, x_86); -lean_ctor_set(x_113, 8, x_87); -lean_ctor_set(x_113, 9, x_88); -lean_ctor_set(x_113, 10, x_89); -lean_ctor_set(x_113, 11, x_90); -lean_ctor_set(x_113, 12, x_91); -lean_ctor_set(x_113, 13, x_92); -lean_ctor_set(x_113, 14, x_93); -lean_ctor_set(x_113, 15, x_94); -lean_ctor_set(x_113, 16, x_95); -lean_ctor_set(x_113, 17, x_96); -lean_ctor_set(x_113, 18, x_97); -lean_ctor_set(x_113, 19, x_98); -lean_ctor_set_uint8(x_113, sizeof(void*)*20, x_84); -x_114 = lean_st_ref_set(x_2, x_113, x_77); -x_115 = lean_ctor_get(x_114, 1); -lean_inc(x_115); -if (lean_is_exclusive(x_114)) { - lean_ctor_release(x_114, 0); - lean_ctor_release(x_114, 1); - x_116 = x_114; + x_119 = x_105; +} +lean_ctor_set(x_119, 0, x_81); +lean_ctor_set(x_119, 1, x_82); +lean_ctor_set(x_119, 2, x_83); +lean_ctor_set(x_119, 3, x_84); +lean_ctor_set(x_119, 4, x_85); +lean_ctor_set(x_119, 5, x_118); +lean_ctor_set(x_119, 6, x_87); +lean_ctor_set(x_119, 7, x_89); +lean_ctor_set(x_119, 8, x_90); +lean_ctor_set(x_119, 9, x_91); +lean_ctor_set(x_119, 10, x_92); +lean_ctor_set(x_119, 11, x_93); +lean_ctor_set(x_119, 12, x_94); +lean_ctor_set(x_119, 13, x_95); +lean_ctor_set(x_119, 14, x_96); +lean_ctor_set(x_119, 15, x_97); +lean_ctor_set(x_119, 16, x_98); +lean_ctor_set(x_119, 17, x_99); +lean_ctor_set(x_119, 18, x_100); +lean_ctor_set(x_119, 19, x_101); +lean_ctor_set(x_119, 20, x_102); +lean_ctor_set(x_119, 21, x_103); +lean_ctor_set(x_119, 22, x_104); +lean_ctor_set_uint8(x_119, sizeof(void*)*23, x_88); +x_120 = lean_st_ref_set(x_2, x_119, x_80); +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +if (lean_is_exclusive(x_120)) { + lean_ctor_release(x_120, 0); + lean_ctor_release(x_120, 1); + x_122 = x_120; } else { - lean_dec_ref(x_114); - x_116 = lean_box(0); + lean_dec_ref(x_120); + x_122 = lean_box(0); } -x_117 = lean_box(0); -if (lean_is_scalar(x_116)) { - x_118 = lean_alloc_ctor(0, 2, 0); +x_123 = lean_box(0); +if (lean_is_scalar(x_122)) { + x_124 = lean_alloc_ctor(0, 2, 0); } else { - x_118 = x_116; + x_124 = x_122; } -lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_115); -return x_118; +lean_ctor_set(x_124, 0, x_123); +lean_ctor_set(x_124, 1, x_121); +return x_124; } } } @@ -4051,11 +4110,11 @@ if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; x_16 = lean_ctor_get(x_12, 1); -x_17 = lean_ctor_get(x_14, 16); +x_17 = lean_ctor_get(x_14, 18); lean_ctor_set_tag(x_12, 1); lean_ctor_set(x_12, 1, x_17); lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_14, 16, x_12); +lean_ctor_set(x_14, 18, x_12); x_18 = lean_st_ref_set(x_3, x_14, x_16); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) @@ -4082,7 +4141,7 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_25 = lean_ctor_get(x_12, 1); x_26 = lean_ctor_get(x_14, 0); x_27 = lean_ctor_get(x_14, 1); @@ -4090,8 +4149,8 @@ x_28 = lean_ctor_get(x_14, 2); x_29 = lean_ctor_get(x_14, 3); x_30 = lean_ctor_get(x_14, 4); x_31 = lean_ctor_get(x_14, 5); -x_32 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); -x_33 = lean_ctor_get(x_14, 6); +x_32 = lean_ctor_get(x_14, 6); +x_33 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); x_34 = lean_ctor_get(x_14, 7); x_35 = lean_ctor_get(x_14, 8); x_36 = lean_ctor_get(x_14, 9); @@ -4105,6 +4164,12 @@ x_43 = lean_ctor_get(x_14, 16); x_44 = lean_ctor_get(x_14, 17); x_45 = lean_ctor_get(x_14, 18); x_46 = lean_ctor_get(x_14, 19); +x_47 = lean_ctor_get(x_14, 20); +x_48 = lean_ctor_get(x_14, 21); +x_49 = lean_ctor_get(x_14, 22); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); @@ -4118,7 +4183,7 @@ lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); -lean_inc(x_33); +lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); @@ -4127,176 +4192,191 @@ lean_inc(x_27); lean_inc(x_26); lean_dec(x_14); lean_ctor_set_tag(x_12, 1); -lean_ctor_set(x_12, 1, x_43); +lean_ctor_set(x_12, 1, x_45); lean_ctor_set(x_12, 0, x_1); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_26); -lean_ctor_set(x_47, 1, x_27); -lean_ctor_set(x_47, 2, x_28); -lean_ctor_set(x_47, 3, x_29); -lean_ctor_set(x_47, 4, x_30); -lean_ctor_set(x_47, 5, x_31); -lean_ctor_set(x_47, 6, x_33); -lean_ctor_set(x_47, 7, x_34); -lean_ctor_set(x_47, 8, x_35); -lean_ctor_set(x_47, 9, x_36); -lean_ctor_set(x_47, 10, x_37); -lean_ctor_set(x_47, 11, x_38); -lean_ctor_set(x_47, 12, x_39); -lean_ctor_set(x_47, 13, x_40); -lean_ctor_set(x_47, 14, x_41); -lean_ctor_set(x_47, 15, x_42); -lean_ctor_set(x_47, 16, x_12); -lean_ctor_set(x_47, 17, x_44); -lean_ctor_set(x_47, 18, x_45); -lean_ctor_set(x_47, 19, x_46); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_32); -x_48 = lean_st_ref_set(x_3, x_47, x_25); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_26); +lean_ctor_set(x_50, 1, x_27); +lean_ctor_set(x_50, 2, x_28); +lean_ctor_set(x_50, 3, x_29); +lean_ctor_set(x_50, 4, x_30); +lean_ctor_set(x_50, 5, x_31); +lean_ctor_set(x_50, 6, x_32); +lean_ctor_set(x_50, 7, x_34); +lean_ctor_set(x_50, 8, x_35); +lean_ctor_set(x_50, 9, x_36); +lean_ctor_set(x_50, 10, x_37); +lean_ctor_set(x_50, 11, x_38); +lean_ctor_set(x_50, 12, x_39); +lean_ctor_set(x_50, 13, x_40); +lean_ctor_set(x_50, 14, x_41); +lean_ctor_set(x_50, 15, x_42); +lean_ctor_set(x_50, 16, x_43); +lean_ctor_set(x_50, 17, x_44); +lean_ctor_set(x_50, 18, x_12); +lean_ctor_set(x_50, 19, x_46); +lean_ctor_set(x_50, 20, x_47); +lean_ctor_set(x_50, 21, x_48); +lean_ctor_set(x_50, 22, x_49); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_33); +x_51 = lean_st_ref_set(x_3, x_50, x_25); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -x_51 = lean_box(0); -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); +x_54 = lean_box(0); +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_50; + x_55 = x_53; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_53 = lean_ctor_get(x_12, 0); -x_54 = lean_ctor_get(x_12, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_12); -x_55 = lean_ctor_get(x_53, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_53, 1); -lean_inc(x_56); -x_57 = lean_ctor_get(x_53, 2); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_56 = lean_ctor_get(x_12, 0); +x_57 = lean_ctor_get(x_12, 1); lean_inc(x_57); -x_58 = lean_ctor_get(x_53, 3); +lean_inc(x_56); +lean_dec(x_12); +x_58 = lean_ctor_get(x_56, 0); lean_inc(x_58); -x_59 = lean_ctor_get(x_53, 4); +x_59 = lean_ctor_get(x_56, 1); lean_inc(x_59); -x_60 = lean_ctor_get(x_53, 5); +x_60 = lean_ctor_get(x_56, 2); lean_inc(x_60); -x_61 = lean_ctor_get_uint8(x_53, sizeof(void*)*20); -x_62 = lean_ctor_get(x_53, 6); +x_61 = lean_ctor_get(x_56, 3); +lean_inc(x_61); +x_62 = lean_ctor_get(x_56, 4); lean_inc(x_62); -x_63 = lean_ctor_get(x_53, 7); +x_63 = lean_ctor_get(x_56, 5); lean_inc(x_63); -x_64 = lean_ctor_get(x_53, 8); +x_64 = lean_ctor_get(x_56, 6); lean_inc(x_64); -x_65 = lean_ctor_get(x_53, 9); -lean_inc(x_65); -x_66 = lean_ctor_get(x_53, 10); +x_65 = lean_ctor_get_uint8(x_56, sizeof(void*)*23); +x_66 = lean_ctor_get(x_56, 7); lean_inc(x_66); -x_67 = lean_ctor_get(x_53, 11); +x_67 = lean_ctor_get(x_56, 8); lean_inc(x_67); -x_68 = lean_ctor_get(x_53, 12); +x_68 = lean_ctor_get(x_56, 9); lean_inc(x_68); -x_69 = lean_ctor_get(x_53, 13); +x_69 = lean_ctor_get(x_56, 10); lean_inc(x_69); -x_70 = lean_ctor_get(x_53, 14); +x_70 = lean_ctor_get(x_56, 11); lean_inc(x_70); -x_71 = lean_ctor_get(x_53, 15); +x_71 = lean_ctor_get(x_56, 12); lean_inc(x_71); -x_72 = lean_ctor_get(x_53, 16); +x_72 = lean_ctor_get(x_56, 13); lean_inc(x_72); -x_73 = lean_ctor_get(x_53, 17); +x_73 = lean_ctor_get(x_56, 14); lean_inc(x_73); -x_74 = lean_ctor_get(x_53, 18); +x_74 = lean_ctor_get(x_56, 15); lean_inc(x_74); -x_75 = lean_ctor_get(x_53, 19); +x_75 = lean_ctor_get(x_56, 16); lean_inc(x_75); -if (lean_is_exclusive(x_53)) { - lean_ctor_release(x_53, 0); - lean_ctor_release(x_53, 1); - lean_ctor_release(x_53, 2); - lean_ctor_release(x_53, 3); - lean_ctor_release(x_53, 4); - lean_ctor_release(x_53, 5); - lean_ctor_release(x_53, 6); - lean_ctor_release(x_53, 7); - lean_ctor_release(x_53, 8); - lean_ctor_release(x_53, 9); - lean_ctor_release(x_53, 10); - lean_ctor_release(x_53, 11); - lean_ctor_release(x_53, 12); - lean_ctor_release(x_53, 13); - lean_ctor_release(x_53, 14); - lean_ctor_release(x_53, 15); - lean_ctor_release(x_53, 16); - lean_ctor_release(x_53, 17); - lean_ctor_release(x_53, 18); - lean_ctor_release(x_53, 19); - x_76 = x_53; +x_76 = lean_ctor_get(x_56, 17); +lean_inc(x_76); +x_77 = lean_ctor_get(x_56, 18); +lean_inc(x_77); +x_78 = lean_ctor_get(x_56, 19); +lean_inc(x_78); +x_79 = lean_ctor_get(x_56, 20); +lean_inc(x_79); +x_80 = lean_ctor_get(x_56, 21); +lean_inc(x_80); +x_81 = lean_ctor_get(x_56, 22); +lean_inc(x_81); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + lean_ctor_release(x_56, 2); + lean_ctor_release(x_56, 3); + lean_ctor_release(x_56, 4); + lean_ctor_release(x_56, 5); + lean_ctor_release(x_56, 6); + lean_ctor_release(x_56, 7); + lean_ctor_release(x_56, 8); + lean_ctor_release(x_56, 9); + lean_ctor_release(x_56, 10); + lean_ctor_release(x_56, 11); + lean_ctor_release(x_56, 12); + lean_ctor_release(x_56, 13); + lean_ctor_release(x_56, 14); + lean_ctor_release(x_56, 15); + lean_ctor_release(x_56, 16); + lean_ctor_release(x_56, 17); + lean_ctor_release(x_56, 18); + lean_ctor_release(x_56, 19); + lean_ctor_release(x_56, 20); + lean_ctor_release(x_56, 21); + lean_ctor_release(x_56, 22); + x_82 = x_56; } else { - lean_dec_ref(x_53); - x_76 = lean_box(0); -} -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_1); -lean_ctor_set(x_77, 1, x_72); -if (lean_is_scalar(x_76)) { - x_78 = lean_alloc_ctor(0, 20, 1); + lean_dec_ref(x_56); + x_82 = lean_box(0); +} +x_83 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_83, 0, x_1); +lean_ctor_set(x_83, 1, x_77); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 23, 1); } else { - x_78 = x_76; -} -lean_ctor_set(x_78, 0, x_55); -lean_ctor_set(x_78, 1, x_56); -lean_ctor_set(x_78, 2, x_57); -lean_ctor_set(x_78, 3, x_58); -lean_ctor_set(x_78, 4, x_59); -lean_ctor_set(x_78, 5, x_60); -lean_ctor_set(x_78, 6, x_62); -lean_ctor_set(x_78, 7, x_63); -lean_ctor_set(x_78, 8, x_64); -lean_ctor_set(x_78, 9, x_65); -lean_ctor_set(x_78, 10, x_66); -lean_ctor_set(x_78, 11, x_67); -lean_ctor_set(x_78, 12, x_68); -lean_ctor_set(x_78, 13, x_69); -lean_ctor_set(x_78, 14, x_70); -lean_ctor_set(x_78, 15, x_71); -lean_ctor_set(x_78, 16, x_77); -lean_ctor_set(x_78, 17, x_73); -lean_ctor_set(x_78, 18, x_74); -lean_ctor_set(x_78, 19, x_75); -lean_ctor_set_uint8(x_78, sizeof(void*)*20, x_61); -x_79 = lean_st_ref_set(x_3, x_78, x_54); -x_80 = lean_ctor_get(x_79, 1); -lean_inc(x_80); -if (lean_is_exclusive(x_79)) { - lean_ctor_release(x_79, 0); - lean_ctor_release(x_79, 1); - x_81 = x_79; + x_84 = x_82; +} +lean_ctor_set(x_84, 0, x_58); +lean_ctor_set(x_84, 1, x_59); +lean_ctor_set(x_84, 2, x_60); +lean_ctor_set(x_84, 3, x_61); +lean_ctor_set(x_84, 4, x_62); +lean_ctor_set(x_84, 5, x_63); +lean_ctor_set(x_84, 6, x_64); +lean_ctor_set(x_84, 7, x_66); +lean_ctor_set(x_84, 8, x_67); +lean_ctor_set(x_84, 9, x_68); +lean_ctor_set(x_84, 10, x_69); +lean_ctor_set(x_84, 11, x_70); +lean_ctor_set(x_84, 12, x_71); +lean_ctor_set(x_84, 13, x_72); +lean_ctor_set(x_84, 14, x_73); +lean_ctor_set(x_84, 15, x_74); +lean_ctor_set(x_84, 16, x_75); +lean_ctor_set(x_84, 17, x_76); +lean_ctor_set(x_84, 18, x_83); +lean_ctor_set(x_84, 19, x_78); +lean_ctor_set(x_84, 20, x_79); +lean_ctor_set(x_84, 21, x_80); +lean_ctor_set(x_84, 22, x_81); +lean_ctor_set_uint8(x_84, sizeof(void*)*23, x_65); +x_85 = lean_st_ref_set(x_3, x_84, x_57); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_87 = x_85; } else { - lean_dec_ref(x_79); - x_81 = lean_box(0); + lean_dec_ref(x_85); + x_87 = lean_box(0); } -x_82 = lean_box(0); -if (lean_is_scalar(x_81)) { - x_83 = lean_alloc_ctor(0, 2, 0); +x_88 = lean_box(0); +if (lean_is_scalar(x_87)) { + x_89 = lean_alloc_ctor(0, 2, 0); } else { - x_83 = x_81; + x_89 = x_87; } -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_80); -return x_83; +lean_ctor_set(x_89, 0, x_88); +lean_ctor_set(x_89, 1, x_86); +return x_89; } } } @@ -4630,16 +4710,89 @@ x_1 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbidde return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_isMatcherApp___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isMorallyIff(lean_object* x_1) { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = lean_st_ref_get(x_9, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) { -lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_11, 0); +uint8_t x_4; +lean_dec(x_2); +x_4 = 0; +return x_4; +} +else +{ +lean_object* x_5; uint8_t x_6; +x_5 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_6 = l_Lean_Expr_isApp(x_5); +if (x_6 == 0) +{ +uint8_t x_7; +lean_dec(x_5); +x_7 = 0; +return x_7; +} +else +{ +lean_object* x_8; uint8_t x_9; +x_8 = l_Lean_Expr_appFnCleanup(x_5, lean_box(0)); +x_9 = l_Lean_Expr_isApp(x_8); +if (x_9 == 0) +{ +uint8_t x_10; +lean_dec(x_8); +x_10 = 0; +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = l_Lean_Expr_appArg(x_8, lean_box(0)); +x_12 = l_Lean_Expr_appFnCleanup(x_8, lean_box(0)); +x_13 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_forbiddenSplitTypes___closed__2; +x_14 = l_Lean_Expr_isConstOf(x_12, x_13); +lean_dec(x_12); +if (x_14 == 0) +{ +uint8_t x_15; +lean_dec(x_11); +x_15 = 0; +return x_15; +} +else +{ +uint8_t x_16; +x_16 = l_Lean_Expr_isProp(x_11); +lean_dec(x_11); +return x_16; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isMorallyIff___boxed(lean_object* x_1) { +_start: +{ +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_isMorallyIff(x_1); +x_3 = lean_box(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_isMatcherApp___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_11, 0); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); lean_dec(x_13); @@ -5042,6 +5195,78 @@ return x_49; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { +uint8_t x_12; +lean_inc(x_1); +x_12 = l_Lean_Meta_Grind_isMorallyIff(x_1); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__3(x_1, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_14; +} +else +{ +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addSplitCandidate(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +if (lean_obj_tag(x_15) == 0) +{ +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_15, 0); +lean_dec(x_17); +x_18 = lean_box(0); +lean_ctor_set(x_15, 0, x_18); +return x_15; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_15, 1); +lean_inc(x_19); +lean_dec(x_15); +x_20 = lean_box(0); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; +} +} +else +{ +uint8_t x_22; +x_22 = !lean_is_exclusive(x_15); +if (x_22 == 0) +{ +return x_15; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_15, 0); +x_24 = lean_ctor_get(x_15, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_15); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ lean_object* x_12; lean_object* x_13; uint8_t x_14; x_12 = l_Lean_Meta_Grind_getConfig___rarg(x_5, x_6, x_7, x_8, x_9, x_10, x_11); x_13 = lean_ctor_get(x_12, 0); @@ -5055,7 +5280,7 @@ x_15 = lean_ctor_get(x_12, 1); lean_inc(x_15); lean_dec(x_12); x_16 = lean_box(0); -x_17 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__3(x_1, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +x_17 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__4(x_1, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); return x_17; } else @@ -5073,7 +5298,7 @@ if (x_20 == 0) { lean_object* x_21; lean_object* x_22; x_21 = lean_box(0); -x_22 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__3(x_1, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_22 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__4(x_1, x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); return x_22; } else @@ -5217,7 +5442,7 @@ else { lean_object* x_14; lean_object* x_15; x_14 = lean_box(0); -x_15 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__4(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_15 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); return x_15; } } @@ -5291,6 +5516,19 @@ lean_dec(x_2); return x_12; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -6328,10 +6566,10 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -x_34 = l_Lean_Meta_Grind_canon(x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_33); +x_34 = l_Lean_Meta_Grind_canon(x_32, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_33); if (lean_obj_tag(x_34) == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); x_36 = lean_ctor_get(x_34, 1); @@ -6343,61 +6581,62 @@ lean_inc(x_38); x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); lean_dec(x_37); +x_40 = lean_box(0); lean_inc(x_38); -x_40 = l_Lean_Meta_Grind_internalize(x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_39); -if (lean_obj_tag(x_40) == 0) +x_41 = l_Lean_Meta_Grind_internalize(x_38, x_2, x_40, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_39); +if (lean_obj_tag(x_41) == 0) { -uint8_t x_41; -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +uint8_t x_42; +x_42 = !lean_is_exclusive(x_41); +if (x_42 == 0) { -lean_object* x_42; lean_object* x_43; -x_42 = lean_ctor_get(x_40, 0); -lean_dec(x_42); -x_43 = l_Lean_Meta_Grind_mkGroundPattern(x_38); -lean_ctor_set(x_40, 0, x_43); -return x_40; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_41, 0); +lean_dec(x_43); +x_44 = l_Lean_Meta_Grind_mkGroundPattern(x_38); +lean_ctor_set(x_41, 0, x_44); +return x_41; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_40, 1); -lean_inc(x_44); -lean_dec(x_40); -x_45 = l_Lean_Meta_Grind_mkGroundPattern(x_38); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_44); -return x_46; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_41, 1); +lean_inc(x_45); +lean_dec(x_41); +x_46 = l_Lean_Meta_Grind_mkGroundPattern(x_38); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +return x_47; } } else { -uint8_t x_47; +uint8_t x_48; lean_dec(x_38); -x_47 = !lean_is_exclusive(x_40); -if (x_47 == 0) +x_48 = !lean_is_exclusive(x_41); +if (x_48 == 0) { -return x_40; +return x_41; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_40, 0); -x_49 = lean_ctor_get(x_40, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_41, 0); +x_50 = lean_ctor_get(x_41, 1); +lean_inc(x_50); lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_40); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_dec(x_41); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } else { -uint8_t x_51; +uint8_t x_52; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6407,29 +6646,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_51 = !lean_is_exclusive(x_34); -if (x_51 == 0) +x_52 = !lean_is_exclusive(x_34); +if (x_52 == 0) { return x_34; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_34, 0); -x_53 = lean_ctor_get(x_34, 1); +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_34, 0); +x_54 = lean_ctor_get(x_34, 1); +lean_inc(x_54); lean_inc(x_53); -lean_inc(x_52); lean_dec(x_34); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } else { -uint8_t x_55; +uint8_t x_56; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6439,29 +6678,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_55 = !lean_is_exclusive(x_31); -if (x_55 == 0) +x_56 = !lean_is_exclusive(x_31); +if (x_56 == 0) { return x_31; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_31, 0); -x_57 = lean_ctor_get(x_31, 1); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_31, 0); +x_58 = lean_ctor_get(x_31, 1); +lean_inc(x_58); lean_inc(x_57); -lean_inc(x_56); lean_dec(x_31); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } else { -uint8_t x_59; +uint8_t x_60; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6471,30 +6710,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_59 = !lean_is_exclusive(x_26); -if (x_59 == 0) +x_60 = !lean_is_exclusive(x_26); +if (x_60 == 0) { return x_26; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_26, 0); -x_61 = lean_ctor_get(x_26, 1); +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_26, 0); +x_62 = lean_ctor_get(x_26, 1); +lean_inc(x_62); lean_inc(x_61); -lean_inc(x_60); lean_dec(x_26); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; } } } } else { -lean_object* x_63; +lean_object* x_64; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6504,15 +6743,15 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_1); -lean_ctor_set(x_63, 1, x_11); -return x_63; +x_64 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_64, 0, x_1); +lean_ctor_set(x_64, 1, x_11); +return x_64; } } else { -lean_object* x_64; +lean_object* x_65; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -6522,70 +6761,14 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_64 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_64, 0, x_1); -lean_ctor_set(x_64, 1, x_11); -return x_64; -} -} -} -static lean_object* _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_instMonadMetaM; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4; -x_2 = l_instInhabitedPUnit; -x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); -return x_3; -} +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_1); +lean_ctor_set(x_65, 1, x_11); +return x_65; } -LEAN_EXPORT lean_object* l_panic___at_Lean_Meta_Grind_internalize___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5; -x_12 = lean_panic_fn(x_11, x_1); -x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { _start: { lean_object* x_19; uint8_t x_20; @@ -6612,9 +6795,12 @@ return x_21; } else { -lean_object* x_22; lean_object* x_23; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_dec(x_6); x_22 = lean_array_fget(x_3, x_7); +lean_inc(x_1); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_1); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); @@ -6625,33 +6811,33 @@ lean_inc(x_11); lean_inc(x_10); lean_inc(x_2); lean_inc(x_22); -x_23 = l_Lean_Meta_Grind_internalize(x_22, x_2, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); -if (lean_obj_tag(x_23) == 0) +x_24 = l_Lean_Meta_Grind_internalize(x_22, x_2, x_23, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); lean_inc(x_1); -x_25 = l_Lean_Meta_Grind_registerParent(x_1, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_24); +x_26 = l_Lean_Meta_Grind_registerParent(x_1, x_22, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_25); lean_dec(x_22); -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); -lean_dec(x_25); -x_27 = lean_ctor_get(x_5, 2); -x_28 = lean_nat_add(x_7, x_27); +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); +x_28 = lean_ctor_get(x_5, 2); +x_29 = lean_nat_add(x_7, x_28); lean_dec(x_7); -x_29 = lean_box(0); -x_6 = x_29; -x_7 = x_28; +x_30 = lean_box(0); +x_6 = x_30; +x_7 = x_29; x_8 = lean_box(0); x_9 = lean_box(0); -x_18 = x_26; +x_18 = x_27; goto _start; } else { -uint8_t x_31; +uint8_t x_32; lean_dec(x_22); lean_dec(x_17); lean_dec(x_16); @@ -6664,44 +6850,45 @@ lean_dec(x_10); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_31 = !lean_is_exclusive(x_23); -if (x_31 == 0) +x_32 = !lean_is_exclusive(x_24); +if (x_32 == 0) { -return x_23; +return x_24; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_23, 0); -x_33 = lean_ctor_get(x_23, 1); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_24, 0); +x_34 = lean_ctor_get(x_24, 1); +lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_23); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +lean_dec(x_24); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; +lean_object* x_14; +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); lean_inc(x_1); -x_13 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) +x_14 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +lean_dec(x_14); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -6709,26 +6896,42 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); lean_inc(x_1); -x_15 = l_Lean_Meta_Grind_addCongrTable(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_14); -if (lean_obj_tag(x_15) == 0) +x_16 = l_Lean_Meta_Grind_addCongrTable(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); lean_inc(x_1); -x_17 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = l_Lean_Meta_Grind_propagateUp(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_18); -return x_19; +x_18 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_updateAppMap(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_20 = l_Lean_Meta_Grind_Arith_Offset_internalize(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_Meta_Grind_propagateUp(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_21); +return x_22; } else { -uint8_t x_20; +uint8_t x_23; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -6736,31 +6939,31 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) { -return x_15; +return x_20; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_15, 0); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_15); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_20, 0); +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_20); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; } } } else { -uint8_t x_24; +uint8_t x_27; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -6768,30 +6971,63 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_1); -x_24 = !lean_is_exclusive(x_13); -if (x_24 == 0) +x_27 = !lean_is_exclusive(x_16); +if (x_27 == 0) { -return x_13; +return x_16; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_13, 0); -x_26 = lean_ctor_get(x_13, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_13); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_16, 0); +x_29 = lean_ctor_get(x_16, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_16); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } } +else +{ +uint8_t x_31; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_31 = !lean_is_exclusive(x_14); +if (x_31 == 0) +{ +return x_14; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_14, 0); +x_33 = lean_ctor_get(x_14, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_14); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; +} } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +} +} +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; @@ -6811,7 +7047,7 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2(x_2, x_3, x_1, x_18, x_18, x_19, x_16, lean_box(0), lean_box(0), x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1(x_2, x_3, x_1, x_18, x_18, x_19, x_16, lean_box(0), lean_box(0), x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_18); if (lean_obj_tag(x_20) == 0) { @@ -6855,7 +7091,7 @@ return x_26; } } } -static lean_object* _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1() { +static lean_object* _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1() { _start: { lean_object* x_1; @@ -6863,42 +7099,43 @@ x_1 = lean_mk_string_unchecked("nestedProof", 11, 11); return x_1; } } -static lean_object* _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2() { +static lean_object* _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__1___closed__1; x_2 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs___lambda__1___closed__2; -x_3 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1; +x_3 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { _start: { -switch (lean_obj_tag(x_3)) { +switch (lean_obj_tag(x_4)) { case 0: { -lean_object* x_15; -lean_dec(x_5); +lean_object* x_16; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_15 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) +x_16 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); lean_inc(x_1); -x_17 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_16); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); +x_18 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_17); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6906,58 +7143,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_19 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); -if (lean_obj_tag(x_19) == 0) +lean_inc(x_4); +x_20 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_19); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_34; uint8_t x_35; -x_20 = lean_ctor_get(x_19, 1); -lean_inc(x_20); -lean_dec(x_19); +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_36; uint8_t x_37; +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_21, 0, x_1); -lean_closure_set(x_21, 1, x_2); -x_34 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_35 = l_Lean_Expr_isConstOf(x_3, x_34); -if (x_35 == 0) +x_22 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_22, 0, x_1); +lean_closure_set(x_22, 1, x_2); +lean_closure_set(x_22, 2, x_3); +x_36 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_37 = l_Lean_Expr_isConstOf(x_4, x_36); +if (x_37 == 0) { -lean_object* x_36; -x_36 = lean_box(0); -x_22 = x_36; -goto block_33; +lean_object* x_38; +lean_dec(x_3); +x_38 = lean_box(0); +x_23 = x_38; +goto block_35; } else { -lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = lean_array_get_size(x_4); -x_38 = lean_unsigned_to_nat(2u); -x_39 = lean_nat_dec_eq(x_37, x_38); -if (x_39 == 0) +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = lean_array_get_size(x_5); +x_40 = lean_unsigned_to_nat(2u); +x_41 = lean_nat_dec_eq(x_39, x_40); +if (x_41 == 0) { -lean_object* x_40; -lean_dec(x_37); -x_40 = lean_box(0); -x_22 = x_40; -goto block_33; +lean_object* x_42; +lean_dec(x_39); +lean_dec(x_3); +x_42 = lean_box(0); +x_23 = x_42; +goto block_35; } else { -lean_object* x_41; uint8_t x_42; -lean_dec(x_21); -lean_dec(x_3); -x_41 = lean_unsigned_to_nat(0u); -x_42 = lean_nat_dec_lt(x_41, x_37); -lean_dec(x_37); -if (x_42 == 0) -{ -lean_object* x_43; lean_object* x_44; lean_object* x_45; +lean_object* x_43; uint8_t x_44; lean_object* x_45; +lean_dec(x_22); lean_dec(x_4); -x_43 = l_Lean_instInhabitedExpr; -x_44 = l_outOfBounds___rarg(x_43); +x_43 = lean_unsigned_to_nat(0u); +x_44 = lean_nat_dec_lt(x_43, x_39); +lean_dec(x_39); +lean_inc(x_1); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_1); +if (x_44 == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +lean_dec(x_5); +x_46 = l_Lean_instInhabitedExpr; +x_47 = l_outOfBounds___rarg(x_46); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6965,32 +7209,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_44); -x_45 = l_Lean_Meta_Grind_internalize(x_44, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); -if (lean_obj_tag(x_45) == 0) +lean_inc(x_47); +x_48 = l_Lean_Meta_Grind_internalize(x_47, x_2, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_21); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -lean_dec(x_45); -lean_inc(x_1); -x_47 = l_Lean_Meta_Grind_registerParent(x_1, x_44, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_46); -lean_dec(x_44); -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_49 = lean_ctor_get(x_48, 1); lean_inc(x_49); -lean_dec(x_47); -x_50 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_48, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_49); lean_dec(x_48); -return x_50; +lean_inc(x_1); +x_50 = l_Lean_Meta_Grind_registerParent(x_1, x_47, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_49); +lean_dec(x_47); +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +lean_dec(x_50); +x_53 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_51, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_52); +lean_dec(x_51); +return x_53; } else { -uint8_t x_51; -lean_dec(x_44); +uint8_t x_54; +lean_dec(x_47); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6998,34 +7242,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_51 = !lean_is_exclusive(x_45); -if (x_51 == 0) +x_54 = !lean_is_exclusive(x_48); +if (x_54 == 0) { -return x_45; +return x_48; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_45, 0); -x_53 = lean_ctor_get(x_45, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_45); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_48, 0); +x_56 = lean_ctor_get(x_48, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_48); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } else { -lean_object* x_55; lean_object* x_56; -x_55 = lean_array_fget(x_4, x_41); -lean_dec(x_4); +lean_object* x_58; lean_object* x_59; +x_58 = lean_array_fget(x_5, x_43); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7033,32 +7278,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_55); -x_56 = l_Lean_Meta_Grind_internalize(x_55, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); -if (lean_obj_tag(x_56) == 0) +lean_inc(x_58); +x_59 = l_Lean_Meta_Grind_internalize(x_58, x_2, x_45, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_21); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_57 = lean_ctor_get(x_56, 1); -lean_inc(x_57); -lean_dec(x_56); -lean_inc(x_1); -x_58 = l_Lean_Meta_Grind_registerParent(x_1, x_55, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_57); -lean_dec(x_55); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_60 = lean_ctor_get(x_59, 1); lean_inc(x_60); -lean_dec(x_58); -x_61 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_59, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_60); lean_dec(x_59); -return x_61; +lean_inc(x_1); +x_61 = l_Lean_Meta_Grind_registerParent(x_1, x_58, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_60); +lean_dec(x_58); +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_61, 1); +lean_inc(x_63); +lean_dec(x_61); +x_64 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_62, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_63); +lean_dec(x_62); +return x_64; } else { -uint8_t x_62; -lean_dec(x_55); +uint8_t x_65; +lean_dec(x_58); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7066,35 +7311,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_62 = !lean_is_exclusive(x_56); -if (x_62 == 0) +x_65 = !lean_is_exclusive(x_59); +if (x_65 == 0) { -return x_56; +return x_59; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_63 = lean_ctor_get(x_56, 0); -x_64 = lean_ctor_get(x_56, 1); -lean_inc(x_64); -lean_inc(x_63); -lean_dec(x_56); -x_65 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_65, 0, x_63); -lean_ctor_set(x_65, 1, x_64); -return x_65; +lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_66 = lean_ctor_get(x_59, 0); +x_67 = lean_ctor_get(x_59, 1); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_59); +x_68 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_68, 0, x_66); +lean_ctor_set(x_68, 1, x_67); +return x_68; } } } } } -block_33: +block_35: { -lean_object* x_23; -lean_dec(x_22); +lean_object* x_24; lean_object* x_25; +lean_dec(x_23); +lean_inc(x_1); +x_24 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_24, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7102,33 +7351,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_23 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); -if (lean_obj_tag(x_23) == 0) +lean_inc(x_4); +x_25 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_24, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_21); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); -lean_dec(x_23); -lean_inc(x_1); -x_25 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_24); -lean_dec(x_3); -x_26 = lean_ctor_get(x_25, 0); +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_26 = lean_ctor_get(x_25, 1); lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); lean_dec(x_25); -x_28 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_21, x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_27); -lean_dec(x_26); +lean_inc(x_1); +x_27 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_26); lean_dec(x_4); -return x_28; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_22, x_28, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_29); +lean_dec(x_28); +lean_dec(x_5); +return x_30; } else { -uint8_t x_29; -lean_dec(x_21); +uint8_t x_31; +lean_dec(x_22); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7136,35 +7385,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_29 = !lean_is_exclusive(x_23); -if (x_29 == 0) +x_31 = !lean_is_exclusive(x_25); +if (x_31 == 0) { -return x_23; +return x_25; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_23, 0); -x_31 = lean_ctor_get(x_23, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_23); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_25, 0); +x_33 = lean_ctor_get(x_25, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_25); +x_34 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_34, 0, x_32); +lean_ctor_set(x_34, 1, x_33); +return x_34; } } } } else { -uint8_t x_66; +uint8_t x_69; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7172,34 +7421,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_66 = !lean_is_exclusive(x_19); -if (x_66 == 0) +x_69 = !lean_is_exclusive(x_20); +if (x_69 == 0) { -return x_19; +return x_20; } else { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_19, 0); -x_68 = lean_ctor_get(x_19, 1); -lean_inc(x_68); -lean_inc(x_67); -lean_dec(x_19); -x_69 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -return x_69; +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_ctor_get(x_20, 0); +x_71 = lean_ctor_get(x_20, 1); +lean_inc(x_71); +lean_inc(x_70); +lean_dec(x_20); +x_72 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_72, 0, x_70); +lean_ctor_set(x_72, 1, x_71); +return x_72; } } } else { -uint8_t x_70; +uint8_t x_73; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7207,52 +7457,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_70 = !lean_is_exclusive(x_15); -if (x_70 == 0) +x_73 = !lean_is_exclusive(x_16); +if (x_73 == 0) { -return x_15; +return x_16; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_15, 0); -x_72 = lean_ctor_get(x_15, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_15); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_74; lean_object* x_75; lean_object* x_76; +x_74 = lean_ctor_get(x_16, 0); +x_75 = lean_ctor_get(x_16, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_16); +x_76 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_76, 0, x_74); +lean_ctor_set(x_76, 1, x_75); +return x_76; } } } case 1: { -lean_object* x_74; -lean_dec(x_5); +lean_object* x_77; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_74 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_74) == 0) +x_77 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_75 = lean_ctor_get(x_74, 1); -lean_inc(x_75); -lean_dec(x_74); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_78 = lean_ctor_get(x_77, 1); +lean_inc(x_78); +lean_dec(x_77); lean_inc(x_1); -x_76 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_75); -x_77 = lean_ctor_get(x_76, 1); -lean_inc(x_77); -lean_dec(x_76); +x_79 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_78); +x_80 = lean_ctor_get(x_79, 1); +lean_inc(x_80); +lean_dec(x_79); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7260,58 +7511,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_78 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_77); -if (lean_obj_tag(x_78) == 0) +lean_inc(x_4); +x_81 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_80); +if (lean_obj_tag(x_81) == 0) { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_93; uint8_t x_94; -x_79 = lean_ctor_get(x_78, 1); -lean_inc(x_79); -lean_dec(x_78); +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_97; uint8_t x_98; +x_82 = lean_ctor_get(x_81, 1); +lean_inc(x_82); +lean_dec(x_81); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_80 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_80, 0, x_1); -lean_closure_set(x_80, 1, x_2); -x_93 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_94 = l_Lean_Expr_isConstOf(x_3, x_93); -if (x_94 == 0) -{ -lean_object* x_95; -x_95 = lean_box(0); -x_81 = x_95; -goto block_92; -} -else -{ -lean_object* x_96; lean_object* x_97; uint8_t x_98; -x_96 = lean_array_get_size(x_4); -x_97 = lean_unsigned_to_nat(2u); -x_98 = lean_nat_dec_eq(x_96, x_97); +x_83 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_83, 0, x_1); +lean_closure_set(x_83, 1, x_2); +lean_closure_set(x_83, 2, x_3); +x_97 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_98 = l_Lean_Expr_isConstOf(x_4, x_97); if (x_98 == 0) { lean_object* x_99; -lean_dec(x_96); +lean_dec(x_3); x_99 = lean_box(0); -x_81 = x_99; -goto block_92; +x_84 = x_99; +goto block_96; } else { -lean_object* x_100; uint8_t x_101; -lean_dec(x_80); +lean_object* x_100; lean_object* x_101; uint8_t x_102; +x_100 = lean_array_get_size(x_5); +x_101 = lean_unsigned_to_nat(2u); +x_102 = lean_nat_dec_eq(x_100, x_101); +if (x_102 == 0) +{ +lean_object* x_103; +lean_dec(x_100); lean_dec(x_3); -x_100 = lean_unsigned_to_nat(0u); -x_101 = lean_nat_dec_lt(x_100, x_96); -lean_dec(x_96); -if (x_101 == 0) +x_103 = lean_box(0); +x_84 = x_103; +goto block_96; +} +else { -lean_object* x_102; lean_object* x_103; lean_object* x_104; +lean_object* x_104; uint8_t x_105; lean_object* x_106; +lean_dec(x_83); lean_dec(x_4); -x_102 = l_Lean_instInhabitedExpr; -x_103 = l_outOfBounds___rarg(x_102); +x_104 = lean_unsigned_to_nat(0u); +x_105 = lean_nat_dec_lt(x_104, x_100); +lean_dec(x_100); +lean_inc(x_1); +x_106 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_106, 0, x_1); +if (x_105 == 0) +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +lean_dec(x_5); +x_107 = l_Lean_instInhabitedExpr; +x_108 = l_outOfBounds___rarg(x_107); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7319,32 +7577,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_103); -x_104 = l_Lean_Meta_Grind_internalize(x_103, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_79); -if (lean_obj_tag(x_104) == 0) +lean_inc(x_108); +x_109 = l_Lean_Meta_Grind_internalize(x_108, x_2, x_106, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_82); +if (lean_obj_tag(x_109) == 0) { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_105 = lean_ctor_get(x_104, 1); -lean_inc(x_105); -lean_dec(x_104); +lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_110 = lean_ctor_get(x_109, 1); +lean_inc(x_110); +lean_dec(x_109); lean_inc(x_1); -x_106 = l_Lean_Meta_Grind_registerParent(x_1, x_103, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_105); -lean_dec(x_103); -x_107 = lean_ctor_get(x_106, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_106, 1); -lean_inc(x_108); -lean_dec(x_106); -x_109 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_107, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_108); -lean_dec(x_107); -return x_109; +x_111 = l_Lean_Meta_Grind_registerParent(x_1, x_108, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_110); +lean_dec(x_108); +x_112 = lean_ctor_get(x_111, 0); +lean_inc(x_112); +x_113 = lean_ctor_get(x_111, 1); +lean_inc(x_113); +lean_dec(x_111); +x_114 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_112, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_113); +lean_dec(x_112); +return x_114; } else { -uint8_t x_110; -lean_dec(x_103); +uint8_t x_115; +lean_dec(x_108); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7352,34 +7610,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_110 = !lean_is_exclusive(x_104); -if (x_110 == 0) +x_115 = !lean_is_exclusive(x_109); +if (x_115 == 0) { -return x_104; +return x_109; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_111 = lean_ctor_get(x_104, 0); -x_112 = lean_ctor_get(x_104, 1); -lean_inc(x_112); -lean_inc(x_111); -lean_dec(x_104); -x_113 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -return x_113; +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_109, 0); +x_117 = lean_ctor_get(x_109, 1); +lean_inc(x_117); +lean_inc(x_116); +lean_dec(x_109); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } } } else { -lean_object* x_114; lean_object* x_115; -x_114 = lean_array_fget(x_4, x_100); -lean_dec(x_4); +lean_object* x_119; lean_object* x_120; +x_119 = lean_array_fget(x_5, x_104); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7387,32 +7646,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_114); -x_115 = l_Lean_Meta_Grind_internalize(x_114, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_79); -if (lean_obj_tag(x_115) == 0) +lean_inc(x_119); +x_120 = l_Lean_Meta_Grind_internalize(x_119, x_2, x_106, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_82); +if (lean_obj_tag(x_120) == 0) { -lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_116 = lean_ctor_get(x_115, 1); -lean_inc(x_116); -lean_dec(x_115); +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_121 = lean_ctor_get(x_120, 1); +lean_inc(x_121); +lean_dec(x_120); lean_inc(x_1); -x_117 = l_Lean_Meta_Grind_registerParent(x_1, x_114, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_116); -lean_dec(x_114); -x_118 = lean_ctor_get(x_117, 0); -lean_inc(x_118); -x_119 = lean_ctor_get(x_117, 1); -lean_inc(x_119); -lean_dec(x_117); -x_120 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_118, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_119); -lean_dec(x_118); -return x_120; +x_122 = l_Lean_Meta_Grind_registerParent(x_1, x_119, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_121); +lean_dec(x_119); +x_123 = lean_ctor_get(x_122, 0); +lean_inc(x_123); +x_124 = lean_ctor_get(x_122, 1); +lean_inc(x_124); +lean_dec(x_122); +x_125 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_123, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_124); +lean_dec(x_123); +return x_125; } else { -uint8_t x_121; -lean_dec(x_114); +uint8_t x_126; +lean_dec(x_119); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7420,35 +7679,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_121 = !lean_is_exclusive(x_115); -if (x_121 == 0) +x_126 = !lean_is_exclusive(x_120); +if (x_126 == 0) { -return x_115; +return x_120; } else { -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_115, 0); -x_123 = lean_ctor_get(x_115, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_115); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -return x_124; +lean_object* x_127; lean_object* x_128; lean_object* x_129; +x_127 = lean_ctor_get(x_120, 0); +x_128 = lean_ctor_get(x_120, 1); +lean_inc(x_128); +lean_inc(x_127); +lean_dec(x_120); +x_129 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_129, 0, x_127); +lean_ctor_set(x_129, 1, x_128); +return x_129; } } } } } -block_92: +block_96: { -lean_object* x_82; -lean_dec(x_81); +lean_object* x_85; lean_object* x_86; +lean_dec(x_84); +lean_inc(x_1); +x_85 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_85, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7456,33 +7719,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_82 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_79); -if (lean_obj_tag(x_82) == 0) +lean_inc(x_4); +x_86 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_85, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_82); +if (lean_obj_tag(x_86) == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_83 = lean_ctor_get(x_82, 1); -lean_inc(x_83); -lean_dec(x_82); +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_87 = lean_ctor_get(x_86, 1); +lean_inc(x_87); +lean_dec(x_86); lean_inc(x_1); -x_84 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_83); -lean_dec(x_3); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_80, x_85, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_86); -lean_dec(x_85); +x_88 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_87); lean_dec(x_4); -return x_87; +x_89 = lean_ctor_get(x_88, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_88, 1); +lean_inc(x_90); +lean_dec(x_88); +x_91 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_83, x_89, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_90); +lean_dec(x_89); +lean_dec(x_5); +return x_91; } else { -uint8_t x_88; -lean_dec(x_80); +uint8_t x_92; +lean_dec(x_83); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7490,35 +7753,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_88 = !lean_is_exclusive(x_82); -if (x_88 == 0) +x_92 = !lean_is_exclusive(x_86); +if (x_92 == 0) { -return x_82; +return x_86; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_82, 0); -x_90 = lean_ctor_get(x_82, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_82); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_86, 0); +x_94 = lean_ctor_get(x_86, 1); +lean_inc(x_94); +lean_inc(x_93); +lean_dec(x_86); +x_95 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_94); +return x_95; } } } } else { -uint8_t x_125; +uint8_t x_130; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7526,34 +7789,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_125 = !lean_is_exclusive(x_78); -if (x_125 == 0) +x_130 = !lean_is_exclusive(x_81); +if (x_130 == 0) { -return x_78; +return x_81; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_126 = lean_ctor_get(x_78, 0); -x_127 = lean_ctor_get(x_78, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_78); -x_128 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_128, 0, x_126); -lean_ctor_set(x_128, 1, x_127); -return x_128; +lean_object* x_131; lean_object* x_132; lean_object* x_133; +x_131 = lean_ctor_get(x_81, 0); +x_132 = lean_ctor_get(x_81, 1); +lean_inc(x_132); +lean_inc(x_131); +lean_dec(x_81); +x_133 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_133, 0, x_131); +lean_ctor_set(x_133, 1, x_132); +return x_133; } } } else { -uint8_t x_129; +uint8_t x_134; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7561,52 +7825,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_129 = !lean_is_exclusive(x_74); -if (x_129 == 0) +x_134 = !lean_is_exclusive(x_77); +if (x_134 == 0) { -return x_74; +return x_77; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_130 = lean_ctor_get(x_74, 0); -x_131 = lean_ctor_get(x_74, 1); -lean_inc(x_131); -lean_inc(x_130); -lean_dec(x_74); -x_132 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_132, 0, x_130); -lean_ctor_set(x_132, 1, x_131); -return x_132; +lean_object* x_135; lean_object* x_136; lean_object* x_137; +x_135 = lean_ctor_get(x_77, 0); +x_136 = lean_ctor_get(x_77, 1); +lean_inc(x_136); +lean_inc(x_135); +lean_dec(x_77); +x_137 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +return x_137; } } } case 2: { -lean_object* x_133; -lean_dec(x_5); +lean_object* x_138; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_133 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_133) == 0) +x_138 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_138) == 0) { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_134 = lean_ctor_get(x_133, 1); -lean_inc(x_134); -lean_dec(x_133); +lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_139 = lean_ctor_get(x_138, 1); +lean_inc(x_139); +lean_dec(x_138); lean_inc(x_1); -x_135 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_134); -x_136 = lean_ctor_get(x_135, 1); -lean_inc(x_136); -lean_dec(x_135); +x_140 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_139); +x_141 = lean_ctor_get(x_140, 1); +lean_inc(x_141); +lean_dec(x_140); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7614,58 +7879,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_137 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_136); -if (lean_obj_tag(x_137) == 0) +lean_inc(x_4); +x_142 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_141); +if (lean_obj_tag(x_142) == 0) { -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_152; uint8_t x_153; -x_138 = lean_ctor_get(x_137, 1); -lean_inc(x_138); -lean_dec(x_137); +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_158; uint8_t x_159; +x_143 = lean_ctor_get(x_142, 1); +lean_inc(x_143); +lean_dec(x_142); +lean_inc(x_3); lean_inc(x_2); -lean_inc(x_1); -x_139 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_139, 0, x_1); -lean_closure_set(x_139, 1, x_2); -x_152 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_153 = l_Lean_Expr_isConstOf(x_3, x_152); -if (x_153 == 0) -{ -lean_object* x_154; -x_154 = lean_box(0); -x_140 = x_154; -goto block_151; +lean_inc(x_1); +x_144 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_144, 0, x_1); +lean_closure_set(x_144, 1, x_2); +lean_closure_set(x_144, 2, x_3); +x_158 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_159 = l_Lean_Expr_isConstOf(x_4, x_158); +if (x_159 == 0) +{ +lean_object* x_160; +lean_dec(x_3); +x_160 = lean_box(0); +x_145 = x_160; +goto block_157; } else { -lean_object* x_155; lean_object* x_156; uint8_t x_157; -x_155 = lean_array_get_size(x_4); -x_156 = lean_unsigned_to_nat(2u); -x_157 = lean_nat_dec_eq(x_155, x_156); -if (x_157 == 0) +lean_object* x_161; lean_object* x_162; uint8_t x_163; +x_161 = lean_array_get_size(x_5); +x_162 = lean_unsigned_to_nat(2u); +x_163 = lean_nat_dec_eq(x_161, x_162); +if (x_163 == 0) { -lean_object* x_158; -lean_dec(x_155); -x_158 = lean_box(0); -x_140 = x_158; -goto block_151; +lean_object* x_164; +lean_dec(x_161); +lean_dec(x_3); +x_164 = lean_box(0); +x_145 = x_164; +goto block_157; } else { -lean_object* x_159; uint8_t x_160; -lean_dec(x_139); -lean_dec(x_3); -x_159 = lean_unsigned_to_nat(0u); -x_160 = lean_nat_dec_lt(x_159, x_155); -lean_dec(x_155); -if (x_160 == 0) -{ -lean_object* x_161; lean_object* x_162; lean_object* x_163; +lean_object* x_165; uint8_t x_166; lean_object* x_167; +lean_dec(x_144); lean_dec(x_4); -x_161 = l_Lean_instInhabitedExpr; -x_162 = l_outOfBounds___rarg(x_161); +x_165 = lean_unsigned_to_nat(0u); +x_166 = lean_nat_dec_lt(x_165, x_161); +lean_dec(x_161); +lean_inc(x_1); +x_167 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_167, 0, x_1); +if (x_166 == 0) +{ +lean_object* x_168; lean_object* x_169; lean_object* x_170; +lean_dec(x_5); +x_168 = l_Lean_instInhabitedExpr; +x_169 = l_outOfBounds___rarg(x_168); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7673,32 +7945,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_162); -x_163 = l_Lean_Meta_Grind_internalize(x_162, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_138); -if (lean_obj_tag(x_163) == 0) +lean_inc(x_169); +x_170 = l_Lean_Meta_Grind_internalize(x_169, x_2, x_167, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_143); +if (lean_obj_tag(x_170) == 0) { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_164 = lean_ctor_get(x_163, 1); -lean_inc(x_164); -lean_dec(x_163); +lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; +x_171 = lean_ctor_get(x_170, 1); +lean_inc(x_171); +lean_dec(x_170); lean_inc(x_1); -x_165 = l_Lean_Meta_Grind_registerParent(x_1, x_162, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_164); -lean_dec(x_162); -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -x_167 = lean_ctor_get(x_165, 1); -lean_inc(x_167); -lean_dec(x_165); -x_168 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_166, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_167); -lean_dec(x_166); -return x_168; +x_172 = l_Lean_Meta_Grind_registerParent(x_1, x_169, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_171); +lean_dec(x_169); +x_173 = lean_ctor_get(x_172, 0); +lean_inc(x_173); +x_174 = lean_ctor_get(x_172, 1); +lean_inc(x_174); +lean_dec(x_172); +x_175 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_173, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_174); +lean_dec(x_173); +return x_175; } else { -uint8_t x_169; -lean_dec(x_162); +uint8_t x_176; +lean_dec(x_169); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7706,34 +7978,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_169 = !lean_is_exclusive(x_163); -if (x_169 == 0) +x_176 = !lean_is_exclusive(x_170); +if (x_176 == 0) { -return x_163; +return x_170; } else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; -x_170 = lean_ctor_get(x_163, 0); -x_171 = lean_ctor_get(x_163, 1); -lean_inc(x_171); -lean_inc(x_170); -lean_dec(x_163); -x_172 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_172, 0, x_170); -lean_ctor_set(x_172, 1, x_171); -return x_172; +lean_object* x_177; lean_object* x_178; lean_object* x_179; +x_177 = lean_ctor_get(x_170, 0); +x_178 = lean_ctor_get(x_170, 1); +lean_inc(x_178); +lean_inc(x_177); +lean_dec(x_170); +x_179 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_179, 0, x_177); +lean_ctor_set(x_179, 1, x_178); +return x_179; } } } else { -lean_object* x_173; lean_object* x_174; -x_173 = lean_array_fget(x_4, x_159); -lean_dec(x_4); +lean_object* x_180; lean_object* x_181; +x_180 = lean_array_fget(x_5, x_165); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7741,32 +8014,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_173); -x_174 = l_Lean_Meta_Grind_internalize(x_173, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_138); -if (lean_obj_tag(x_174) == 0) +lean_inc(x_180); +x_181 = l_Lean_Meta_Grind_internalize(x_180, x_2, x_167, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_143); +if (lean_obj_tag(x_181) == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_175 = lean_ctor_get(x_174, 1); -lean_inc(x_175); -lean_dec(x_174); +lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_182 = lean_ctor_get(x_181, 1); +lean_inc(x_182); +lean_dec(x_181); lean_inc(x_1); -x_176 = l_Lean_Meta_Grind_registerParent(x_1, x_173, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_175); -lean_dec(x_173); -x_177 = lean_ctor_get(x_176, 0); -lean_inc(x_177); -x_178 = lean_ctor_get(x_176, 1); -lean_inc(x_178); -lean_dec(x_176); -x_179 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_177, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_178); -lean_dec(x_177); -return x_179; +x_183 = l_Lean_Meta_Grind_registerParent(x_1, x_180, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_182); +lean_dec(x_180); +x_184 = lean_ctor_get(x_183, 0); +lean_inc(x_184); +x_185 = lean_ctor_get(x_183, 1); +lean_inc(x_185); +lean_dec(x_183); +x_186 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_184, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_185); +lean_dec(x_184); +return x_186; } else { -uint8_t x_180; -lean_dec(x_173); +uint8_t x_187; +lean_dec(x_180); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7774,35 +8047,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_180 = !lean_is_exclusive(x_174); -if (x_180 == 0) +x_187 = !lean_is_exclusive(x_181); +if (x_187 == 0) { -return x_174; +return x_181; } else { -lean_object* x_181; lean_object* x_182; lean_object* x_183; -x_181 = lean_ctor_get(x_174, 0); -x_182 = lean_ctor_get(x_174, 1); -lean_inc(x_182); -lean_inc(x_181); -lean_dec(x_174); -x_183 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_183, 0, x_181); -lean_ctor_set(x_183, 1, x_182); -return x_183; +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_ctor_get(x_181, 0); +x_189 = lean_ctor_get(x_181, 1); +lean_inc(x_189); +lean_inc(x_188); +lean_dec(x_181); +x_190 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_190, 0, x_188); +lean_ctor_set(x_190, 1, x_189); +return x_190; } } } } } -block_151: +block_157: { -lean_object* x_141; -lean_dec(x_140); +lean_object* x_146; lean_object* x_147; +lean_dec(x_145); +lean_inc(x_1); +x_146 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_146, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7810,33 +8087,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_141 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_138); -if (lean_obj_tag(x_141) == 0) +lean_inc(x_4); +x_147 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_146, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_143); +if (lean_obj_tag(x_147) == 0) { -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_142 = lean_ctor_get(x_141, 1); -lean_inc(x_142); -lean_dec(x_141); +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_148 = lean_ctor_get(x_147, 1); +lean_inc(x_148); +lean_dec(x_147); lean_inc(x_1); -x_143 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_142); -lean_dec(x_3); -x_144 = lean_ctor_get(x_143, 0); -lean_inc(x_144); -x_145 = lean_ctor_get(x_143, 1); -lean_inc(x_145); -lean_dec(x_143); -x_146 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_139, x_144, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_145); -lean_dec(x_144); +x_149 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_148); lean_dec(x_4); -return x_146; +x_150 = lean_ctor_get(x_149, 0); +lean_inc(x_150); +x_151 = lean_ctor_get(x_149, 1); +lean_inc(x_151); +lean_dec(x_149); +x_152 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_144, x_150, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_151); +lean_dec(x_150); +lean_dec(x_5); +return x_152; } else { -uint8_t x_147; -lean_dec(x_139); +uint8_t x_153; +lean_dec(x_144); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7844,35 +8121,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_147 = !lean_is_exclusive(x_141); -if (x_147 == 0) +x_153 = !lean_is_exclusive(x_147); +if (x_153 == 0) { -return x_141; +return x_147; } else { -lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_148 = lean_ctor_get(x_141, 0); -x_149 = lean_ctor_get(x_141, 1); -lean_inc(x_149); -lean_inc(x_148); -lean_dec(x_141); -x_150 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_150, 0, x_148); -lean_ctor_set(x_150, 1, x_149); -return x_150; +lean_object* x_154; lean_object* x_155; lean_object* x_156; +x_154 = lean_ctor_get(x_147, 0); +x_155 = lean_ctor_get(x_147, 1); +lean_inc(x_155); +lean_inc(x_154); +lean_dec(x_147); +x_156 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_156, 0, x_154); +lean_ctor_set(x_156, 1, x_155); +return x_156; } } } } else { -uint8_t x_184; +uint8_t x_191; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7880,34 +8157,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_184 = !lean_is_exclusive(x_137); -if (x_184 == 0) +x_191 = !lean_is_exclusive(x_142); +if (x_191 == 0) { -return x_137; +return x_142; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_137, 0); -x_186 = lean_ctor_get(x_137, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_137); -x_187 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -return x_187; +lean_object* x_192; lean_object* x_193; lean_object* x_194; +x_192 = lean_ctor_get(x_142, 0); +x_193 = lean_ctor_get(x_142, 1); +lean_inc(x_193); +lean_inc(x_192); +lean_dec(x_142); +x_194 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_194, 0, x_192); +lean_ctor_set(x_194, 1, x_193); +return x_194; } } } else { -uint8_t x_188; +uint8_t x_195; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -7915,52 +8193,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_188 = !lean_is_exclusive(x_133); -if (x_188 == 0) +x_195 = !lean_is_exclusive(x_138); +if (x_195 == 0) { -return x_133; +return x_138; } else { -lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_189 = lean_ctor_get(x_133, 0); -x_190 = lean_ctor_get(x_133, 1); -lean_inc(x_190); -lean_inc(x_189); -lean_dec(x_133); -x_191 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_191, 0, x_189); -lean_ctor_set(x_191, 1, x_190); -return x_191; +lean_object* x_196; lean_object* x_197; lean_object* x_198; +x_196 = lean_ctor_get(x_138, 0); +x_197 = lean_ctor_get(x_138, 1); +lean_inc(x_197); +lean_inc(x_196); +lean_dec(x_138); +x_198 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_198, 0, x_196); +lean_ctor_set(x_198, 1, x_197); +return x_198; } } } case 3: { -lean_object* x_192; -lean_dec(x_5); +lean_object* x_199; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_192 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_192) == 0) +x_199 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_199) == 0) { -lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; -x_193 = lean_ctor_get(x_192, 1); -lean_inc(x_193); -lean_dec(x_192); +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +x_200 = lean_ctor_get(x_199, 1); +lean_inc(x_200); +lean_dec(x_199); lean_inc(x_1); -x_194 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_193); -x_195 = lean_ctor_get(x_194, 1); -lean_inc(x_195); -lean_dec(x_194); +x_201 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_200); +x_202 = lean_ctor_get(x_201, 1); +lean_inc(x_202); +lean_dec(x_201); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -7968,58 +8247,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_196 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_195); -if (lean_obj_tag(x_196) == 0) +lean_inc(x_4); +x_203 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_202); +if (lean_obj_tag(x_203) == 0) { -lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_211; uint8_t x_212; -x_197 = lean_ctor_get(x_196, 1); -lean_inc(x_197); -lean_dec(x_196); +lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_219; uint8_t x_220; +x_204 = lean_ctor_get(x_203, 1); +lean_inc(x_204); +lean_dec(x_203); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_198 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_198, 0, x_1); -lean_closure_set(x_198, 1, x_2); -x_211 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_212 = l_Lean_Expr_isConstOf(x_3, x_211); -if (x_212 == 0) -{ -lean_object* x_213; -x_213 = lean_box(0); -x_199 = x_213; -goto block_210; +x_205 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_205, 0, x_1); +lean_closure_set(x_205, 1, x_2); +lean_closure_set(x_205, 2, x_3); +x_219 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_220 = l_Lean_Expr_isConstOf(x_4, x_219); +if (x_220 == 0) +{ +lean_object* x_221; +lean_dec(x_3); +x_221 = lean_box(0); +x_206 = x_221; +goto block_218; } else { -lean_object* x_214; lean_object* x_215; uint8_t x_216; -x_214 = lean_array_get_size(x_4); -x_215 = lean_unsigned_to_nat(2u); -x_216 = lean_nat_dec_eq(x_214, x_215); -if (x_216 == 0) +lean_object* x_222; lean_object* x_223; uint8_t x_224; +x_222 = lean_array_get_size(x_5); +x_223 = lean_unsigned_to_nat(2u); +x_224 = lean_nat_dec_eq(x_222, x_223); +if (x_224 == 0) { -lean_object* x_217; -lean_dec(x_214); -x_217 = lean_box(0); -x_199 = x_217; -goto block_210; +lean_object* x_225; +lean_dec(x_222); +lean_dec(x_3); +x_225 = lean_box(0); +x_206 = x_225; +goto block_218; } else { -lean_object* x_218; uint8_t x_219; -lean_dec(x_198); -lean_dec(x_3); -x_218 = lean_unsigned_to_nat(0u); -x_219 = lean_nat_dec_lt(x_218, x_214); -lean_dec(x_214); -if (x_219 == 0) -{ -lean_object* x_220; lean_object* x_221; lean_object* x_222; +lean_object* x_226; uint8_t x_227; lean_object* x_228; +lean_dec(x_205); lean_dec(x_4); -x_220 = l_Lean_instInhabitedExpr; -x_221 = l_outOfBounds___rarg(x_220); +x_226 = lean_unsigned_to_nat(0u); +x_227 = lean_nat_dec_lt(x_226, x_222); +lean_dec(x_222); +lean_inc(x_1); +x_228 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_228, 0, x_1); +if (x_227 == 0) +{ +lean_object* x_229; lean_object* x_230; lean_object* x_231; +lean_dec(x_5); +x_229 = l_Lean_instInhabitedExpr; +x_230 = l_outOfBounds___rarg(x_229); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8027,32 +8313,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_221); -x_222 = l_Lean_Meta_Grind_internalize(x_221, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_197); -if (lean_obj_tag(x_222) == 0) +lean_inc(x_230); +x_231 = l_Lean_Meta_Grind_internalize(x_230, x_2, x_228, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_204); +if (lean_obj_tag(x_231) == 0) { -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; -x_223 = lean_ctor_get(x_222, 1); -lean_inc(x_223); -lean_dec(x_222); +lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_232 = lean_ctor_get(x_231, 1); +lean_inc(x_232); +lean_dec(x_231); lean_inc(x_1); -x_224 = l_Lean_Meta_Grind_registerParent(x_1, x_221, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_223); -lean_dec(x_221); -x_225 = lean_ctor_get(x_224, 0); -lean_inc(x_225); -x_226 = lean_ctor_get(x_224, 1); -lean_inc(x_226); -lean_dec(x_224); -x_227 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_225, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_226); -lean_dec(x_225); -return x_227; +x_233 = l_Lean_Meta_Grind_registerParent(x_1, x_230, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_232); +lean_dec(x_230); +x_234 = lean_ctor_get(x_233, 0); +lean_inc(x_234); +x_235 = lean_ctor_get(x_233, 1); +lean_inc(x_235); +lean_dec(x_233); +x_236 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_234, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_235); +lean_dec(x_234); +return x_236; } else { -uint8_t x_228; -lean_dec(x_221); +uint8_t x_237; +lean_dec(x_230); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8060,34 +8346,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_228 = !lean_is_exclusive(x_222); -if (x_228 == 0) +x_237 = !lean_is_exclusive(x_231); +if (x_237 == 0) { -return x_222; +return x_231; } else { -lean_object* x_229; lean_object* x_230; lean_object* x_231; -x_229 = lean_ctor_get(x_222, 0); -x_230 = lean_ctor_get(x_222, 1); -lean_inc(x_230); -lean_inc(x_229); -lean_dec(x_222); -x_231 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_231, 0, x_229); -lean_ctor_set(x_231, 1, x_230); -return x_231; +lean_object* x_238; lean_object* x_239; lean_object* x_240; +x_238 = lean_ctor_get(x_231, 0); +x_239 = lean_ctor_get(x_231, 1); +lean_inc(x_239); +lean_inc(x_238); +lean_dec(x_231); +x_240 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_240, 0, x_238); +lean_ctor_set(x_240, 1, x_239); +return x_240; } } } else { -lean_object* x_232; lean_object* x_233; -x_232 = lean_array_fget(x_4, x_218); -lean_dec(x_4); +lean_object* x_241; lean_object* x_242; +x_241 = lean_array_fget(x_5, x_226); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8095,32 +8382,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_232); -x_233 = l_Lean_Meta_Grind_internalize(x_232, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_197); -if (lean_obj_tag(x_233) == 0) +lean_inc(x_241); +x_242 = l_Lean_Meta_Grind_internalize(x_241, x_2, x_228, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_204); +if (lean_obj_tag(x_242) == 0) { -lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; -x_234 = lean_ctor_get(x_233, 1); -lean_inc(x_234); -lean_dec(x_233); +lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; +x_243 = lean_ctor_get(x_242, 1); +lean_inc(x_243); +lean_dec(x_242); lean_inc(x_1); -x_235 = l_Lean_Meta_Grind_registerParent(x_1, x_232, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_234); -lean_dec(x_232); -x_236 = lean_ctor_get(x_235, 0); -lean_inc(x_236); -x_237 = lean_ctor_get(x_235, 1); -lean_inc(x_237); -lean_dec(x_235); -x_238 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_236, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_237); -lean_dec(x_236); -return x_238; +x_244 = l_Lean_Meta_Grind_registerParent(x_1, x_241, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_243); +lean_dec(x_241); +x_245 = lean_ctor_get(x_244, 0); +lean_inc(x_245); +x_246 = lean_ctor_get(x_244, 1); +lean_inc(x_246); +lean_dec(x_244); +x_247 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_245, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_246); +lean_dec(x_245); +return x_247; } else { -uint8_t x_239; -lean_dec(x_232); +uint8_t x_248; +lean_dec(x_241); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8128,35 +8415,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_239 = !lean_is_exclusive(x_233); -if (x_239 == 0) +x_248 = !lean_is_exclusive(x_242); +if (x_248 == 0) { -return x_233; +return x_242; } else { -lean_object* x_240; lean_object* x_241; lean_object* x_242; -x_240 = lean_ctor_get(x_233, 0); -x_241 = lean_ctor_get(x_233, 1); -lean_inc(x_241); -lean_inc(x_240); -lean_dec(x_233); -x_242 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_242, 0, x_240); -lean_ctor_set(x_242, 1, x_241); -return x_242; +lean_object* x_249; lean_object* x_250; lean_object* x_251; +x_249 = lean_ctor_get(x_242, 0); +x_250 = lean_ctor_get(x_242, 1); +lean_inc(x_250); +lean_inc(x_249); +lean_dec(x_242); +x_251 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_251, 0, x_249); +lean_ctor_set(x_251, 1, x_250); +return x_251; } } } } } -block_210: +block_218: { -lean_object* x_200; -lean_dec(x_199); +lean_object* x_207; lean_object* x_208; +lean_dec(x_206); +lean_inc(x_1); +x_207 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_207, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8164,33 +8455,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_200 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_197); -if (lean_obj_tag(x_200) == 0) +lean_inc(x_4); +x_208 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_207, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_204); +if (lean_obj_tag(x_208) == 0) { -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; -x_201 = lean_ctor_get(x_200, 1); -lean_inc(x_201); -lean_dec(x_200); +lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_209 = lean_ctor_get(x_208, 1); +lean_inc(x_209); +lean_dec(x_208); lean_inc(x_1); -x_202 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_201); -lean_dec(x_3); -x_203 = lean_ctor_get(x_202, 0); -lean_inc(x_203); -x_204 = lean_ctor_get(x_202, 1); -lean_inc(x_204); -lean_dec(x_202); -x_205 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_198, x_203, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_204); -lean_dec(x_203); +x_210 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_209); lean_dec(x_4); -return x_205; +x_211 = lean_ctor_get(x_210, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_210, 1); +lean_inc(x_212); +lean_dec(x_210); +x_213 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_205, x_211, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_212); +lean_dec(x_211); +lean_dec(x_5); +return x_213; } else { -uint8_t x_206; -lean_dec(x_198); +uint8_t x_214; +lean_dec(x_205); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8198,35 +8489,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_206 = !lean_is_exclusive(x_200); -if (x_206 == 0) +x_214 = !lean_is_exclusive(x_208); +if (x_214 == 0) { -return x_200; +return x_208; } else { -lean_object* x_207; lean_object* x_208; lean_object* x_209; -x_207 = lean_ctor_get(x_200, 0); -x_208 = lean_ctor_get(x_200, 1); -lean_inc(x_208); -lean_inc(x_207); -lean_dec(x_200); -x_209 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_209, 0, x_207); -lean_ctor_set(x_209, 1, x_208); -return x_209; +lean_object* x_215; lean_object* x_216; lean_object* x_217; +x_215 = lean_ctor_get(x_208, 0); +x_216 = lean_ctor_get(x_208, 1); +lean_inc(x_216); +lean_inc(x_215); +lean_dec(x_208); +x_217 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_217, 0, x_215); +lean_ctor_set(x_217, 1, x_216); +return x_217; } } } } else { -uint8_t x_243; +uint8_t x_252; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8234,34 +8525,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_243 = !lean_is_exclusive(x_196); -if (x_243 == 0) +x_252 = !lean_is_exclusive(x_203); +if (x_252 == 0) { -return x_196; +return x_203; } else { -lean_object* x_244; lean_object* x_245; lean_object* x_246; -x_244 = lean_ctor_get(x_196, 0); -x_245 = lean_ctor_get(x_196, 1); -lean_inc(x_245); -lean_inc(x_244); -lean_dec(x_196); -x_246 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_246, 0, x_244); -lean_ctor_set(x_246, 1, x_245); -return x_246; +lean_object* x_253; lean_object* x_254; lean_object* x_255; +x_253 = lean_ctor_get(x_203, 0); +x_254 = lean_ctor_get(x_203, 1); +lean_inc(x_254); +lean_inc(x_253); +lean_dec(x_203); +x_255 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_255, 0, x_253); +lean_ctor_set(x_255, 1, x_254); +return x_255; } } } else { -uint8_t x_247; +uint8_t x_256; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8269,54 +8561,55 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_247 = !lean_is_exclusive(x_192); -if (x_247 == 0) +x_256 = !lean_is_exclusive(x_199); +if (x_256 == 0) { -return x_192; +return x_199; } else { -lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_248 = lean_ctor_get(x_192, 0); -x_249 = lean_ctor_get(x_192, 1); -lean_inc(x_249); -lean_inc(x_248); -lean_dec(x_192); -x_250 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_250, 0, x_248); -lean_ctor_set(x_250, 1, x_249); -return x_250; +lean_object* x_257; lean_object* x_258; lean_object* x_259; +x_257 = lean_ctor_get(x_199, 0); +x_258 = lean_ctor_get(x_199, 1); +lean_inc(x_258); +lean_inc(x_257); +lean_dec(x_199); +x_259 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_259, 0, x_257); +lean_ctor_set(x_259, 1, x_258); +return x_259; } } } case 4: { -lean_object* x_251; lean_object* x_252; -lean_dec(x_5); -x_251 = lean_ctor_get(x_3, 0); -lean_inc(x_251); +lean_object* x_260; lean_object* x_261; +lean_dec(x_6); +x_260 = lean_ctor_get(x_4, 0); +lean_inc(x_260); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_252 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_252) == 0) +x_261 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_261) == 0) { -lean_object* x_253; lean_object* x_254; lean_object* x_255; lean_object* x_256; -x_253 = lean_ctor_get(x_252, 1); -lean_inc(x_253); -lean_dec(x_252); +lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; +x_262 = lean_ctor_get(x_261, 1); +lean_inc(x_262); +lean_dec(x_261); lean_inc(x_1); -x_254 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_253); -x_255 = lean_ctor_get(x_254, 1); -lean_inc(x_255); -lean_dec(x_254); +x_263 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_262); +x_264 = lean_ctor_get(x_263, 1); +lean_inc(x_264); +lean_dec(x_263); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8324,59 +8617,66 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_256 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_255); -if (lean_obj_tag(x_256) == 0) +lean_inc(x_4); +x_265 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_264); +if (lean_obj_tag(x_265) == 0) { -lean_object* x_257; lean_object* x_258; lean_object* x_259; lean_object* x_269; uint8_t x_270; -x_257 = lean_ctor_get(x_256, 1); -lean_inc(x_257); -lean_dec(x_256); +lean_object* x_266; lean_object* x_267; lean_object* x_268; lean_object* x_278; uint8_t x_279; +x_266 = lean_ctor_get(x_265, 1); +lean_inc(x_266); +lean_dec(x_265); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_258 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_258, 0, x_1); -lean_closure_set(x_258, 1, x_2); -x_269 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_270 = l_Lean_Expr_isConstOf(x_3, x_269); -lean_dec(x_3); -if (x_270 == 0) +x_267 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_267, 0, x_1); +lean_closure_set(x_267, 1, x_2); +lean_closure_set(x_267, 2, x_3); +x_278 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_279 = l_Lean_Expr_isConstOf(x_4, x_278); +lean_dec(x_4); +if (x_279 == 0) { -lean_object* x_271; -x_271 = lean_box(0); -x_259 = x_271; -goto block_268; +lean_object* x_280; +lean_dec(x_3); +x_280 = lean_box(0); +x_268 = x_280; +goto block_277; } else { -lean_object* x_272; lean_object* x_273; uint8_t x_274; -x_272 = lean_array_get_size(x_4); -x_273 = lean_unsigned_to_nat(2u); -x_274 = lean_nat_dec_eq(x_272, x_273); -if (x_274 == 0) +lean_object* x_281; lean_object* x_282; uint8_t x_283; +x_281 = lean_array_get_size(x_5); +x_282 = lean_unsigned_to_nat(2u); +x_283 = lean_nat_dec_eq(x_281, x_282); +if (x_283 == 0) { -lean_object* x_275; -lean_dec(x_272); -x_275 = lean_box(0); -x_259 = x_275; -goto block_268; +lean_object* x_284; +lean_dec(x_281); +lean_dec(x_3); +x_284 = lean_box(0); +x_268 = x_284; +goto block_277; } else { -lean_object* x_276; uint8_t x_277; -lean_dec(x_258); -lean_dec(x_251); -x_276 = lean_unsigned_to_nat(0u); -x_277 = lean_nat_dec_lt(x_276, x_272); -lean_dec(x_272); -if (x_277 == 0) +lean_object* x_285; uint8_t x_286; lean_object* x_287; +lean_dec(x_267); +lean_dec(x_260); +x_285 = lean_unsigned_to_nat(0u); +x_286 = lean_nat_dec_lt(x_285, x_281); +lean_dec(x_281); +lean_inc(x_1); +x_287 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_287, 0, x_1); +if (x_286 == 0) { -lean_object* x_278; lean_object* x_279; lean_object* x_280; -lean_dec(x_4); -x_278 = l_Lean_instInhabitedExpr; -x_279 = l_outOfBounds___rarg(x_278); +lean_object* x_288; lean_object* x_289; lean_object* x_290; +lean_dec(x_5); +x_288 = l_Lean_instInhabitedExpr; +x_289 = l_outOfBounds___rarg(x_288); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8384,32 +8684,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_279); -x_280 = l_Lean_Meta_Grind_internalize(x_279, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_257); -if (lean_obj_tag(x_280) == 0) -{ -lean_object* x_281; lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; -x_281 = lean_ctor_get(x_280, 1); -lean_inc(x_281); -lean_dec(x_280); -lean_inc(x_1); -x_282 = l_Lean_Meta_Grind_registerParent(x_1, x_279, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_281); -lean_dec(x_279); -x_283 = lean_ctor_get(x_282, 0); -lean_inc(x_283); -x_284 = lean_ctor_get(x_282, 1); -lean_inc(x_284); -lean_dec(x_282); -x_285 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_283, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_284); -lean_dec(x_283); -return x_285; -} -else -{ -uint8_t x_286; -lean_dec(x_279); +lean_inc(x_289); +x_290 = l_Lean_Meta_Grind_internalize(x_289, x_2, x_287, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_266); +if (lean_obj_tag(x_290) == 0) +{ +lean_object* x_291; lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; +x_291 = lean_ctor_get(x_290, 1); +lean_inc(x_291); +lean_dec(x_290); +lean_inc(x_1); +x_292 = l_Lean_Meta_Grind_registerParent(x_1, x_289, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_291); +lean_dec(x_289); +x_293 = lean_ctor_get(x_292, 0); +lean_inc(x_293); +x_294 = lean_ctor_get(x_292, 1); +lean_inc(x_294); +lean_dec(x_292); +x_295 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_293, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_294); +lean_dec(x_293); +return x_295; +} +else +{ +uint8_t x_296; +lean_dec(x_289); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8417,34 +8717,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_286 = !lean_is_exclusive(x_280); -if (x_286 == 0) +x_296 = !lean_is_exclusive(x_290); +if (x_296 == 0) { -return x_280; +return x_290; } else { -lean_object* x_287; lean_object* x_288; lean_object* x_289; -x_287 = lean_ctor_get(x_280, 0); -x_288 = lean_ctor_get(x_280, 1); -lean_inc(x_288); -lean_inc(x_287); -lean_dec(x_280); -x_289 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_289, 0, x_287); -lean_ctor_set(x_289, 1, x_288); -return x_289; +lean_object* x_297; lean_object* x_298; lean_object* x_299; +x_297 = lean_ctor_get(x_290, 0); +x_298 = lean_ctor_get(x_290, 1); +lean_inc(x_298); +lean_inc(x_297); +lean_dec(x_290); +x_299 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_299, 0, x_297); +lean_ctor_set(x_299, 1, x_298); +return x_299; } } } else { -lean_object* x_290; lean_object* x_291; -x_290 = lean_array_fget(x_4, x_276); -lean_dec(x_4); +lean_object* x_300; lean_object* x_301; +x_300 = lean_array_fget(x_5, x_285); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8452,32 +8753,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_290); -x_291 = l_Lean_Meta_Grind_internalize(x_290, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_257); -if (lean_obj_tag(x_291) == 0) +lean_inc(x_300); +x_301 = l_Lean_Meta_Grind_internalize(x_300, x_2, x_287, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_266); +if (lean_obj_tag(x_301) == 0) { -lean_object* x_292; lean_object* x_293; lean_object* x_294; lean_object* x_295; lean_object* x_296; -x_292 = lean_ctor_get(x_291, 1); -lean_inc(x_292); -lean_dec(x_291); +lean_object* x_302; lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +x_302 = lean_ctor_get(x_301, 1); +lean_inc(x_302); +lean_dec(x_301); lean_inc(x_1); -x_293 = l_Lean_Meta_Grind_registerParent(x_1, x_290, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_292); -lean_dec(x_290); -x_294 = lean_ctor_get(x_293, 0); -lean_inc(x_294); -x_295 = lean_ctor_get(x_293, 1); -lean_inc(x_295); -lean_dec(x_293); -x_296 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_294, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_295); -lean_dec(x_294); -return x_296; +x_303 = l_Lean_Meta_Grind_registerParent(x_1, x_300, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_302); +lean_dec(x_300); +x_304 = lean_ctor_get(x_303, 0); +lean_inc(x_304); +x_305 = lean_ctor_get(x_303, 1); +lean_inc(x_305); +lean_dec(x_303); +x_306 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_304, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_305); +lean_dec(x_304); +return x_306; } else { -uint8_t x_297; -lean_dec(x_290); +uint8_t x_307; +lean_dec(x_300); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8485,35 +8786,36 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_297 = !lean_is_exclusive(x_291); -if (x_297 == 0) +x_307 = !lean_is_exclusive(x_301); +if (x_307 == 0) { -return x_291; +return x_301; } else { -lean_object* x_298; lean_object* x_299; lean_object* x_300; -x_298 = lean_ctor_get(x_291, 0); -x_299 = lean_ctor_get(x_291, 1); -lean_inc(x_299); -lean_inc(x_298); -lean_dec(x_291); -x_300 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_300, 0, x_298); -lean_ctor_set(x_300, 1, x_299); -return x_300; +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_301, 0); +x_309 = lean_ctor_get(x_301, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_301); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; } } } } } -block_268: +block_277: { -lean_object* x_260; -lean_dec(x_259); +lean_object* x_269; +lean_dec(x_268); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8521,27 +8823,27 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -x_260 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns(x_251, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_257); -lean_dec(x_251); -if (lean_obj_tag(x_260) == 0) -{ -lean_object* x_261; lean_object* x_262; lean_object* x_263; -x_261 = lean_ctor_get(x_260, 0); -lean_inc(x_261); -x_262 = lean_ctor_get(x_260, 1); -lean_inc(x_262); +x_269 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns(x_260, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_266); lean_dec(x_260); -x_263 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_258, x_261, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_262); -lean_dec(x_261); -lean_dec(x_4); -return x_263; +if (lean_obj_tag(x_269) == 0) +{ +lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +x_271 = lean_ctor_get(x_269, 1); +lean_inc(x_271); +lean_dec(x_269); +x_272 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_267, x_270, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_271); +lean_dec(x_270); +lean_dec(x_5); +return x_272; } else { -uint8_t x_264; -lean_dec(x_258); +uint8_t x_273; +lean_dec(x_267); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8549,35 +8851,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_4); +lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_264 = !lean_is_exclusive(x_260); -if (x_264 == 0) +x_273 = !lean_is_exclusive(x_269); +if (x_273 == 0) { -return x_260; +return x_269; } else { -lean_object* x_265; lean_object* x_266; lean_object* x_267; -x_265 = lean_ctor_get(x_260, 0); -x_266 = lean_ctor_get(x_260, 1); -lean_inc(x_266); -lean_inc(x_265); -lean_dec(x_260); -x_267 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_267, 0, x_265); -lean_ctor_set(x_267, 1, x_266); -return x_267; +lean_object* x_274; lean_object* x_275; lean_object* x_276; +x_274 = lean_ctor_get(x_269, 0); +x_275 = lean_ctor_get(x_269, 1); +lean_inc(x_275); +lean_inc(x_274); +lean_dec(x_269); +x_276 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_276, 0, x_274); +lean_ctor_set(x_276, 1, x_275); +return x_276; } } } } else { -uint8_t x_301; -lean_dec(x_251); +uint8_t x_311; +lean_dec(x_260); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8585,35 +8887,36 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_301 = !lean_is_exclusive(x_256); -if (x_301 == 0) +x_311 = !lean_is_exclusive(x_265); +if (x_311 == 0) { -return x_256; +return x_265; } else { -lean_object* x_302; lean_object* x_303; lean_object* x_304; -x_302 = lean_ctor_get(x_256, 0); -x_303 = lean_ctor_get(x_256, 1); -lean_inc(x_303); -lean_inc(x_302); -lean_dec(x_256); -x_304 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_304, 0, x_302); -lean_ctor_set(x_304, 1, x_303); -return x_304; +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_265, 0); +x_313 = lean_ctor_get(x_265, 1); +lean_inc(x_313); +lean_inc(x_312); +lean_dec(x_265); +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_305; -lean_dec(x_251); +uint8_t x_315; +lean_dec(x_260); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8621,69 +8924,70 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_305 = !lean_is_exclusive(x_252); -if (x_305 == 0) +x_315 = !lean_is_exclusive(x_261); +if (x_315 == 0) { -return x_252; +return x_261; } else { -lean_object* x_306; lean_object* x_307; lean_object* x_308; -x_306 = lean_ctor_get(x_252, 0); -x_307 = lean_ctor_get(x_252, 1); -lean_inc(x_307); -lean_inc(x_306); -lean_dec(x_252); -x_308 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_308, 0, x_306); -lean_ctor_set(x_308, 1, x_307); -return x_308; +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_261, 0); +x_317 = lean_ctor_get(x_261, 1); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_261); +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } case 5: { -lean_object* x_309; lean_object* x_310; lean_object* x_311; lean_object* x_312; lean_object* x_313; -x_309 = lean_ctor_get(x_3, 0); -lean_inc(x_309); -x_310 = lean_ctor_get(x_3, 1); -lean_inc(x_310); -lean_dec(x_3); -x_311 = lean_array_set(x_4, x_5, x_310); -x_312 = lean_unsigned_to_nat(1u); -x_313 = lean_nat_sub(x_5, x_312); -lean_dec(x_5); -x_3 = x_309; -x_4 = x_311; -x_5 = x_313; +lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_323; +x_319 = lean_ctor_get(x_4, 0); +lean_inc(x_319); +x_320 = lean_ctor_get(x_4, 1); +lean_inc(x_320); +lean_dec(x_4); +x_321 = lean_array_set(x_5, x_6, x_320); +x_322 = lean_unsigned_to_nat(1u); +x_323 = lean_nat_sub(x_6, x_322); +lean_dec(x_6); +x_4 = x_319; +x_5 = x_321; +x_6 = x_323; goto _start; } case 6: { -lean_object* x_315; -lean_dec(x_5); +lean_object* x_325; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_315 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_315) == 0) +x_325 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_325) == 0) { -lean_object* x_316; lean_object* x_317; lean_object* x_318; lean_object* x_319; -x_316 = lean_ctor_get(x_315, 1); -lean_inc(x_316); -lean_dec(x_315); +lean_object* x_326; lean_object* x_327; lean_object* x_328; lean_object* x_329; +x_326 = lean_ctor_get(x_325, 1); +lean_inc(x_326); +lean_dec(x_325); lean_inc(x_1); -x_317 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_316); -x_318 = lean_ctor_get(x_317, 1); -lean_inc(x_318); -lean_dec(x_317); +x_327 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_326); +x_328 = lean_ctor_get(x_327, 1); +lean_inc(x_328); +lean_dec(x_327); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8691,58 +8995,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_319 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_318); -if (lean_obj_tag(x_319) == 0) +lean_inc(x_4); +x_329 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_328); +if (lean_obj_tag(x_329) == 0) { -lean_object* x_320; lean_object* x_321; lean_object* x_322; lean_object* x_334; uint8_t x_335; -x_320 = lean_ctor_get(x_319, 1); -lean_inc(x_320); -lean_dec(x_319); +lean_object* x_330; lean_object* x_331; lean_object* x_332; lean_object* x_345; uint8_t x_346; +x_330 = lean_ctor_get(x_329, 1); +lean_inc(x_330); +lean_dec(x_329); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_321 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_321, 0, x_1); -lean_closure_set(x_321, 1, x_2); -x_334 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_335 = l_Lean_Expr_isConstOf(x_3, x_334); -if (x_335 == 0) -{ -lean_object* x_336; -x_336 = lean_box(0); -x_322 = x_336; -goto block_333; +x_331 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_331, 0, x_1); +lean_closure_set(x_331, 1, x_2); +lean_closure_set(x_331, 2, x_3); +x_345 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_346 = l_Lean_Expr_isConstOf(x_4, x_345); +if (x_346 == 0) +{ +lean_object* x_347; +lean_dec(x_3); +x_347 = lean_box(0); +x_332 = x_347; +goto block_344; } else { -lean_object* x_337; lean_object* x_338; uint8_t x_339; -x_337 = lean_array_get_size(x_4); -x_338 = lean_unsigned_to_nat(2u); -x_339 = lean_nat_dec_eq(x_337, x_338); -if (x_339 == 0) +lean_object* x_348; lean_object* x_349; uint8_t x_350; +x_348 = lean_array_get_size(x_5); +x_349 = lean_unsigned_to_nat(2u); +x_350 = lean_nat_dec_eq(x_348, x_349); +if (x_350 == 0) { -lean_object* x_340; -lean_dec(x_337); -x_340 = lean_box(0); -x_322 = x_340; -goto block_333; +lean_object* x_351; +lean_dec(x_348); +lean_dec(x_3); +x_351 = lean_box(0); +x_332 = x_351; +goto block_344; } else { -lean_object* x_341; uint8_t x_342; -lean_dec(x_321); -lean_dec(x_3); -x_341 = lean_unsigned_to_nat(0u); -x_342 = lean_nat_dec_lt(x_341, x_337); -lean_dec(x_337); -if (x_342 == 0) -{ -lean_object* x_343; lean_object* x_344; lean_object* x_345; +lean_object* x_352; uint8_t x_353; lean_object* x_354; +lean_dec(x_331); lean_dec(x_4); -x_343 = l_Lean_instInhabitedExpr; -x_344 = l_outOfBounds___rarg(x_343); +x_352 = lean_unsigned_to_nat(0u); +x_353 = lean_nat_dec_lt(x_352, x_348); +lean_dec(x_348); +lean_inc(x_1); +x_354 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_354, 0, x_1); +if (x_353 == 0) +{ +lean_object* x_355; lean_object* x_356; lean_object* x_357; +lean_dec(x_5); +x_355 = l_Lean_instInhabitedExpr; +x_356 = l_outOfBounds___rarg(x_355); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8750,32 +9061,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_344); -x_345 = l_Lean_Meta_Grind_internalize(x_344, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_320); -if (lean_obj_tag(x_345) == 0) -{ -lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; lean_object* x_350; -x_346 = lean_ctor_get(x_345, 1); -lean_inc(x_346); -lean_dec(x_345); -lean_inc(x_1); -x_347 = l_Lean_Meta_Grind_registerParent(x_1, x_344, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_346); -lean_dec(x_344); -x_348 = lean_ctor_get(x_347, 0); -lean_inc(x_348); -x_349 = lean_ctor_get(x_347, 1); -lean_inc(x_349); -lean_dec(x_347); -x_350 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_348, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_349); -lean_dec(x_348); -return x_350; +lean_inc(x_356); +x_357 = l_Lean_Meta_Grind_internalize(x_356, x_2, x_354, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_330); +if (lean_obj_tag(x_357) == 0) +{ +lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; lean_object* x_362; +x_358 = lean_ctor_get(x_357, 1); +lean_inc(x_358); +lean_dec(x_357); +lean_inc(x_1); +x_359 = l_Lean_Meta_Grind_registerParent(x_1, x_356, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_358); +lean_dec(x_356); +x_360 = lean_ctor_get(x_359, 0); +lean_inc(x_360); +x_361 = lean_ctor_get(x_359, 1); +lean_inc(x_361); +lean_dec(x_359); +x_362 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_360, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_361); +lean_dec(x_360); +return x_362; } else { -uint8_t x_351; -lean_dec(x_344); +uint8_t x_363; +lean_dec(x_356); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8783,34 +9094,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_351 = !lean_is_exclusive(x_345); -if (x_351 == 0) +x_363 = !lean_is_exclusive(x_357); +if (x_363 == 0) { -return x_345; +return x_357; } else { -lean_object* x_352; lean_object* x_353; lean_object* x_354; -x_352 = lean_ctor_get(x_345, 0); -x_353 = lean_ctor_get(x_345, 1); -lean_inc(x_353); -lean_inc(x_352); -lean_dec(x_345); -x_354 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_354, 0, x_352); -lean_ctor_set(x_354, 1, x_353); -return x_354; +lean_object* x_364; lean_object* x_365; lean_object* x_366; +x_364 = lean_ctor_get(x_357, 0); +x_365 = lean_ctor_get(x_357, 1); +lean_inc(x_365); +lean_inc(x_364); +lean_dec(x_357); +x_366 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_366, 0, x_364); +lean_ctor_set(x_366, 1, x_365); +return x_366; } } } else { -lean_object* x_355; lean_object* x_356; -x_355 = lean_array_fget(x_4, x_341); -lean_dec(x_4); +lean_object* x_367; lean_object* x_368; +x_367 = lean_array_fget(x_5, x_352); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8818,32 +9130,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_355); -x_356 = l_Lean_Meta_Grind_internalize(x_355, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_320); -if (lean_obj_tag(x_356) == 0) +lean_inc(x_367); +x_368 = l_Lean_Meta_Grind_internalize(x_367, x_2, x_354, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_330); +if (lean_obj_tag(x_368) == 0) { -lean_object* x_357; lean_object* x_358; lean_object* x_359; lean_object* x_360; lean_object* x_361; -x_357 = lean_ctor_get(x_356, 1); -lean_inc(x_357); -lean_dec(x_356); +lean_object* x_369; lean_object* x_370; lean_object* x_371; lean_object* x_372; lean_object* x_373; +x_369 = lean_ctor_get(x_368, 1); +lean_inc(x_369); +lean_dec(x_368); lean_inc(x_1); -x_358 = l_Lean_Meta_Grind_registerParent(x_1, x_355, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_357); -lean_dec(x_355); -x_359 = lean_ctor_get(x_358, 0); -lean_inc(x_359); -x_360 = lean_ctor_get(x_358, 1); -lean_inc(x_360); -lean_dec(x_358); -x_361 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_359, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_360); -lean_dec(x_359); -return x_361; +x_370 = l_Lean_Meta_Grind_registerParent(x_1, x_367, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_369); +lean_dec(x_367); +x_371 = lean_ctor_get(x_370, 0); +lean_inc(x_371); +x_372 = lean_ctor_get(x_370, 1); +lean_inc(x_372); +lean_dec(x_370); +x_373 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_371, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_372); +lean_dec(x_371); +return x_373; } else { -uint8_t x_362; -lean_dec(x_355); +uint8_t x_374; +lean_dec(x_367); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8851,35 +9163,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_362 = !lean_is_exclusive(x_356); -if (x_362 == 0) +x_374 = !lean_is_exclusive(x_368); +if (x_374 == 0) { -return x_356; +return x_368; } else { -lean_object* x_363; lean_object* x_364; lean_object* x_365; -x_363 = lean_ctor_get(x_356, 0); -x_364 = lean_ctor_get(x_356, 1); -lean_inc(x_364); -lean_inc(x_363); -lean_dec(x_356); -x_365 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_365, 0, x_363); -lean_ctor_set(x_365, 1, x_364); -return x_365; +lean_object* x_375; lean_object* x_376; lean_object* x_377; +x_375 = lean_ctor_get(x_368, 0); +x_376 = lean_ctor_get(x_368, 1); +lean_inc(x_376); +lean_inc(x_375); +lean_dec(x_368); +x_377 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_377, 0, x_375); +lean_ctor_set(x_377, 1, x_376); +return x_377; } } } } } -block_333: +block_344: { -lean_object* x_323; -lean_dec(x_322); +lean_object* x_333; lean_object* x_334; +lean_dec(x_332); +lean_inc(x_1); +x_333 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_333, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -8887,33 +9203,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_323 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_320); -if (lean_obj_tag(x_323) == 0) +lean_inc(x_4); +x_334 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_333, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_330); +if (lean_obj_tag(x_334) == 0) { -lean_object* x_324; lean_object* x_325; lean_object* x_326; lean_object* x_327; lean_object* x_328; -x_324 = lean_ctor_get(x_323, 1); -lean_inc(x_324); -lean_dec(x_323); +lean_object* x_335; lean_object* x_336; lean_object* x_337; lean_object* x_338; lean_object* x_339; +x_335 = lean_ctor_get(x_334, 1); +lean_inc(x_335); +lean_dec(x_334); lean_inc(x_1); -x_325 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_324); -lean_dec(x_3); -x_326 = lean_ctor_get(x_325, 0); -lean_inc(x_326); -x_327 = lean_ctor_get(x_325, 1); -lean_inc(x_327); -lean_dec(x_325); -x_328 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_321, x_326, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_327); -lean_dec(x_326); +x_336 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_335); lean_dec(x_4); -return x_328; +x_337 = lean_ctor_get(x_336, 0); +lean_inc(x_337); +x_338 = lean_ctor_get(x_336, 1); +lean_inc(x_338); +lean_dec(x_336); +x_339 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_331, x_337, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_338); +lean_dec(x_337); +lean_dec(x_5); +return x_339; } else { -uint8_t x_329; -lean_dec(x_321); +uint8_t x_340; +lean_dec(x_331); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8921,35 +9237,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_329 = !lean_is_exclusive(x_323); -if (x_329 == 0) +x_340 = !lean_is_exclusive(x_334); +if (x_340 == 0) { -return x_323; +return x_334; } else { -lean_object* x_330; lean_object* x_331; lean_object* x_332; -x_330 = lean_ctor_get(x_323, 0); -x_331 = lean_ctor_get(x_323, 1); -lean_inc(x_331); -lean_inc(x_330); -lean_dec(x_323); -x_332 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_332, 0, x_330); -lean_ctor_set(x_332, 1, x_331); -return x_332; +lean_object* x_341; lean_object* x_342; lean_object* x_343; +x_341 = lean_ctor_get(x_334, 0); +x_342 = lean_ctor_get(x_334, 1); +lean_inc(x_342); +lean_inc(x_341); +lean_dec(x_334); +x_343 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_343, 0, x_341); +lean_ctor_set(x_343, 1, x_342); +return x_343; } } } } else { -uint8_t x_366; +uint8_t x_378; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8957,34 +9273,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_366 = !lean_is_exclusive(x_319); -if (x_366 == 0) +x_378 = !lean_is_exclusive(x_329); +if (x_378 == 0) { -return x_319; +return x_329; } else { -lean_object* x_367; lean_object* x_368; lean_object* x_369; -x_367 = lean_ctor_get(x_319, 0); -x_368 = lean_ctor_get(x_319, 1); -lean_inc(x_368); -lean_inc(x_367); -lean_dec(x_319); -x_369 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_369, 0, x_367); -lean_ctor_set(x_369, 1, x_368); -return x_369; +lean_object* x_379; lean_object* x_380; lean_object* x_381; +x_379 = lean_ctor_get(x_329, 0); +x_380 = lean_ctor_get(x_329, 1); +lean_inc(x_380); +lean_inc(x_379); +lean_dec(x_329); +x_381 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_381, 0, x_379); +lean_ctor_set(x_381, 1, x_380); +return x_381; } } } else { -uint8_t x_370; +uint8_t x_382; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -8992,52 +9309,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_370 = !lean_is_exclusive(x_315); -if (x_370 == 0) +x_382 = !lean_is_exclusive(x_325); +if (x_382 == 0) { -return x_315; +return x_325; } else { -lean_object* x_371; lean_object* x_372; lean_object* x_373; -x_371 = lean_ctor_get(x_315, 0); -x_372 = lean_ctor_get(x_315, 1); -lean_inc(x_372); -lean_inc(x_371); -lean_dec(x_315); -x_373 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_373, 0, x_371); -lean_ctor_set(x_373, 1, x_372); -return x_373; +lean_object* x_383; lean_object* x_384; lean_object* x_385; +x_383 = lean_ctor_get(x_325, 0); +x_384 = lean_ctor_get(x_325, 1); +lean_inc(x_384); +lean_inc(x_383); +lean_dec(x_325); +x_385 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_385, 0, x_383); +lean_ctor_set(x_385, 1, x_384); +return x_385; } } } case 7: { -lean_object* x_374; -lean_dec(x_5); +lean_object* x_386; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_374 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_374) == 0) +x_386 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_386) == 0) { -lean_object* x_375; lean_object* x_376; lean_object* x_377; lean_object* x_378; -x_375 = lean_ctor_get(x_374, 1); -lean_inc(x_375); -lean_dec(x_374); +lean_object* x_387; lean_object* x_388; lean_object* x_389; lean_object* x_390; +x_387 = lean_ctor_get(x_386, 1); +lean_inc(x_387); +lean_dec(x_386); lean_inc(x_1); -x_376 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_375); -x_377 = lean_ctor_get(x_376, 1); -lean_inc(x_377); -lean_dec(x_376); +x_388 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_387); +x_389 = lean_ctor_get(x_388, 1); +lean_inc(x_389); +lean_dec(x_388); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9045,58 +9363,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_378 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_377); -if (lean_obj_tag(x_378) == 0) +lean_inc(x_4); +x_390 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_389); +if (lean_obj_tag(x_390) == 0) { -lean_object* x_379; lean_object* x_380; lean_object* x_381; lean_object* x_393; uint8_t x_394; -x_379 = lean_ctor_get(x_378, 1); -lean_inc(x_379); -lean_dec(x_378); +lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_406; uint8_t x_407; +x_391 = lean_ctor_get(x_390, 1); +lean_inc(x_391); +lean_dec(x_390); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_380 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_380, 0, x_1); -lean_closure_set(x_380, 1, x_2); -x_393 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_394 = l_Lean_Expr_isConstOf(x_3, x_393); -if (x_394 == 0) -{ -lean_object* x_395; -x_395 = lean_box(0); -x_381 = x_395; -goto block_392; +x_392 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_392, 0, x_1); +lean_closure_set(x_392, 1, x_2); +lean_closure_set(x_392, 2, x_3); +x_406 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_407 = l_Lean_Expr_isConstOf(x_4, x_406); +if (x_407 == 0) +{ +lean_object* x_408; +lean_dec(x_3); +x_408 = lean_box(0); +x_393 = x_408; +goto block_405; } else { -lean_object* x_396; lean_object* x_397; uint8_t x_398; -x_396 = lean_array_get_size(x_4); -x_397 = lean_unsigned_to_nat(2u); -x_398 = lean_nat_dec_eq(x_396, x_397); -if (x_398 == 0) +lean_object* x_409; lean_object* x_410; uint8_t x_411; +x_409 = lean_array_get_size(x_5); +x_410 = lean_unsigned_to_nat(2u); +x_411 = lean_nat_dec_eq(x_409, x_410); +if (x_411 == 0) { -lean_object* x_399; -lean_dec(x_396); -x_399 = lean_box(0); -x_381 = x_399; -goto block_392; +lean_object* x_412; +lean_dec(x_409); +lean_dec(x_3); +x_412 = lean_box(0); +x_393 = x_412; +goto block_405; } else { -lean_object* x_400; uint8_t x_401; -lean_dec(x_380); -lean_dec(x_3); -x_400 = lean_unsigned_to_nat(0u); -x_401 = lean_nat_dec_lt(x_400, x_396); -lean_dec(x_396); -if (x_401 == 0) -{ -lean_object* x_402; lean_object* x_403; lean_object* x_404; +lean_object* x_413; uint8_t x_414; lean_object* x_415; +lean_dec(x_392); lean_dec(x_4); -x_402 = l_Lean_instInhabitedExpr; -x_403 = l_outOfBounds___rarg(x_402); +x_413 = lean_unsigned_to_nat(0u); +x_414 = lean_nat_dec_lt(x_413, x_409); +lean_dec(x_409); +lean_inc(x_1); +x_415 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_415, 0, x_1); +if (x_414 == 0) +{ +lean_object* x_416; lean_object* x_417; lean_object* x_418; +lean_dec(x_5); +x_416 = l_Lean_instInhabitedExpr; +x_417 = l_outOfBounds___rarg(x_416); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9104,32 +9429,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_403); -x_404 = l_Lean_Meta_Grind_internalize(x_403, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_379); -if (lean_obj_tag(x_404) == 0) +lean_inc(x_417); +x_418 = l_Lean_Meta_Grind_internalize(x_417, x_2, x_415, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_391); +if (lean_obj_tag(x_418) == 0) { -lean_object* x_405; lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; -x_405 = lean_ctor_get(x_404, 1); -lean_inc(x_405); -lean_dec(x_404); +lean_object* x_419; lean_object* x_420; lean_object* x_421; lean_object* x_422; lean_object* x_423; +x_419 = lean_ctor_get(x_418, 1); +lean_inc(x_419); +lean_dec(x_418); lean_inc(x_1); -x_406 = l_Lean_Meta_Grind_registerParent(x_1, x_403, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_405); -lean_dec(x_403); -x_407 = lean_ctor_get(x_406, 0); -lean_inc(x_407); -x_408 = lean_ctor_get(x_406, 1); -lean_inc(x_408); -lean_dec(x_406); -x_409 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_407, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_408); -lean_dec(x_407); -return x_409; +x_420 = l_Lean_Meta_Grind_registerParent(x_1, x_417, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_419); +lean_dec(x_417); +x_421 = lean_ctor_get(x_420, 0); +lean_inc(x_421); +x_422 = lean_ctor_get(x_420, 1); +lean_inc(x_422); +lean_dec(x_420); +x_423 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_421, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_422); +lean_dec(x_421); +return x_423; } else { -uint8_t x_410; -lean_dec(x_403); +uint8_t x_424; +lean_dec(x_417); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9137,34 +9462,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_410 = !lean_is_exclusive(x_404); -if (x_410 == 0) +x_424 = !lean_is_exclusive(x_418); +if (x_424 == 0) { -return x_404; +return x_418; } else { -lean_object* x_411; lean_object* x_412; lean_object* x_413; -x_411 = lean_ctor_get(x_404, 0); -x_412 = lean_ctor_get(x_404, 1); -lean_inc(x_412); -lean_inc(x_411); -lean_dec(x_404); -x_413 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_413, 0, x_411); -lean_ctor_set(x_413, 1, x_412); -return x_413; +lean_object* x_425; lean_object* x_426; lean_object* x_427; +x_425 = lean_ctor_get(x_418, 0); +x_426 = lean_ctor_get(x_418, 1); +lean_inc(x_426); +lean_inc(x_425); +lean_dec(x_418); +x_427 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_427, 0, x_425); +lean_ctor_set(x_427, 1, x_426); +return x_427; } } } else { -lean_object* x_414; lean_object* x_415; -x_414 = lean_array_fget(x_4, x_400); -lean_dec(x_4); +lean_object* x_428; lean_object* x_429; +x_428 = lean_array_fget(x_5, x_413); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9172,32 +9498,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_414); -x_415 = l_Lean_Meta_Grind_internalize(x_414, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_379); -if (lean_obj_tag(x_415) == 0) -{ -lean_object* x_416; lean_object* x_417; lean_object* x_418; lean_object* x_419; lean_object* x_420; -x_416 = lean_ctor_get(x_415, 1); -lean_inc(x_416); -lean_dec(x_415); -lean_inc(x_1); -x_417 = l_Lean_Meta_Grind_registerParent(x_1, x_414, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_416); -lean_dec(x_414); -x_418 = lean_ctor_get(x_417, 0); -lean_inc(x_418); -x_419 = lean_ctor_get(x_417, 1); -lean_inc(x_419); -lean_dec(x_417); -x_420 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_418, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_419); -lean_dec(x_418); -return x_420; +lean_inc(x_428); +x_429 = l_Lean_Meta_Grind_internalize(x_428, x_2, x_415, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_391); +if (lean_obj_tag(x_429) == 0) +{ +lean_object* x_430; lean_object* x_431; lean_object* x_432; lean_object* x_433; lean_object* x_434; +x_430 = lean_ctor_get(x_429, 1); +lean_inc(x_430); +lean_dec(x_429); +lean_inc(x_1); +x_431 = l_Lean_Meta_Grind_registerParent(x_1, x_428, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_430); +lean_dec(x_428); +x_432 = lean_ctor_get(x_431, 0); +lean_inc(x_432); +x_433 = lean_ctor_get(x_431, 1); +lean_inc(x_433); +lean_dec(x_431); +x_434 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_432, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_433); +lean_dec(x_432); +return x_434; } else { -uint8_t x_421; -lean_dec(x_414); +uint8_t x_435; +lean_dec(x_428); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9205,35 +9531,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_421 = !lean_is_exclusive(x_415); -if (x_421 == 0) +x_435 = !lean_is_exclusive(x_429); +if (x_435 == 0) { -return x_415; +return x_429; } else { -lean_object* x_422; lean_object* x_423; lean_object* x_424; -x_422 = lean_ctor_get(x_415, 0); -x_423 = lean_ctor_get(x_415, 1); -lean_inc(x_423); -lean_inc(x_422); -lean_dec(x_415); -x_424 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_424, 0, x_422); -lean_ctor_set(x_424, 1, x_423); -return x_424; +lean_object* x_436; lean_object* x_437; lean_object* x_438; +x_436 = lean_ctor_get(x_429, 0); +x_437 = lean_ctor_get(x_429, 1); +lean_inc(x_437); +lean_inc(x_436); +lean_dec(x_429); +x_438 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_438, 0, x_436); +lean_ctor_set(x_438, 1, x_437); +return x_438; } } } } } -block_392: +block_405: { -lean_object* x_382; -lean_dec(x_381); +lean_object* x_394; lean_object* x_395; +lean_dec(x_393); +lean_inc(x_1); +x_394 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_394, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9241,33 +9571,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_382 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_379); -if (lean_obj_tag(x_382) == 0) +lean_inc(x_4); +x_395 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_394, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_391); +if (lean_obj_tag(x_395) == 0) { -lean_object* x_383; lean_object* x_384; lean_object* x_385; lean_object* x_386; lean_object* x_387; -x_383 = lean_ctor_get(x_382, 1); -lean_inc(x_383); -lean_dec(x_382); +lean_object* x_396; lean_object* x_397; lean_object* x_398; lean_object* x_399; lean_object* x_400; +x_396 = lean_ctor_get(x_395, 1); +lean_inc(x_396); +lean_dec(x_395); lean_inc(x_1); -x_384 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_383); -lean_dec(x_3); -x_385 = lean_ctor_get(x_384, 0); -lean_inc(x_385); -x_386 = lean_ctor_get(x_384, 1); -lean_inc(x_386); -lean_dec(x_384); -x_387 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_380, x_385, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_386); -lean_dec(x_385); +x_397 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_396); lean_dec(x_4); -return x_387; +x_398 = lean_ctor_get(x_397, 0); +lean_inc(x_398); +x_399 = lean_ctor_get(x_397, 1); +lean_inc(x_399); +lean_dec(x_397); +x_400 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_392, x_398, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_399); +lean_dec(x_398); +lean_dec(x_5); +return x_400; } else { -uint8_t x_388; -lean_dec(x_380); +uint8_t x_401; +lean_dec(x_392); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9275,35 +9605,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_388 = !lean_is_exclusive(x_382); -if (x_388 == 0) +x_401 = !lean_is_exclusive(x_395); +if (x_401 == 0) { -return x_382; +return x_395; } else { -lean_object* x_389; lean_object* x_390; lean_object* x_391; -x_389 = lean_ctor_get(x_382, 0); -x_390 = lean_ctor_get(x_382, 1); -lean_inc(x_390); -lean_inc(x_389); -lean_dec(x_382); -x_391 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_391, 0, x_389); -lean_ctor_set(x_391, 1, x_390); -return x_391; +lean_object* x_402; lean_object* x_403; lean_object* x_404; +x_402 = lean_ctor_get(x_395, 0); +x_403 = lean_ctor_get(x_395, 1); +lean_inc(x_403); +lean_inc(x_402); +lean_dec(x_395); +x_404 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_404, 0, x_402); +lean_ctor_set(x_404, 1, x_403); +return x_404; } } } } else { -uint8_t x_425; +uint8_t x_439; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9311,34 +9641,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_425 = !lean_is_exclusive(x_378); -if (x_425 == 0) +x_439 = !lean_is_exclusive(x_390); +if (x_439 == 0) { -return x_378; +return x_390; } else { -lean_object* x_426; lean_object* x_427; lean_object* x_428; -x_426 = lean_ctor_get(x_378, 0); -x_427 = lean_ctor_get(x_378, 1); -lean_inc(x_427); -lean_inc(x_426); -lean_dec(x_378); -x_428 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_428, 0, x_426); -lean_ctor_set(x_428, 1, x_427); -return x_428; +lean_object* x_440; lean_object* x_441; lean_object* x_442; +x_440 = lean_ctor_get(x_390, 0); +x_441 = lean_ctor_get(x_390, 1); +lean_inc(x_441); +lean_inc(x_440); +lean_dec(x_390); +x_442 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_442, 0, x_440); +lean_ctor_set(x_442, 1, x_441); +return x_442; } } } else { -uint8_t x_429; +uint8_t x_443; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9346,52 +9677,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_429 = !lean_is_exclusive(x_374); -if (x_429 == 0) +x_443 = !lean_is_exclusive(x_386); +if (x_443 == 0) { -return x_374; +return x_386; } else { -lean_object* x_430; lean_object* x_431; lean_object* x_432; -x_430 = lean_ctor_get(x_374, 0); -x_431 = lean_ctor_get(x_374, 1); -lean_inc(x_431); -lean_inc(x_430); -lean_dec(x_374); -x_432 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_432, 0, x_430); -lean_ctor_set(x_432, 1, x_431); -return x_432; +lean_object* x_444; lean_object* x_445; lean_object* x_446; +x_444 = lean_ctor_get(x_386, 0); +x_445 = lean_ctor_get(x_386, 1); +lean_inc(x_445); +lean_inc(x_444); +lean_dec(x_386); +x_446 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_446, 0, x_444); +lean_ctor_set(x_446, 1, x_445); +return x_446; } } } case 8: { -lean_object* x_433; -lean_dec(x_5); +lean_object* x_447; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_433 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_433) == 0) +x_447 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_447) == 0) { -lean_object* x_434; lean_object* x_435; lean_object* x_436; lean_object* x_437; -x_434 = lean_ctor_get(x_433, 1); -lean_inc(x_434); -lean_dec(x_433); +lean_object* x_448; lean_object* x_449; lean_object* x_450; lean_object* x_451; +x_448 = lean_ctor_get(x_447, 1); +lean_inc(x_448); +lean_dec(x_447); lean_inc(x_1); -x_435 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_434); -x_436 = lean_ctor_get(x_435, 1); -lean_inc(x_436); -lean_dec(x_435); +x_449 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_448); +x_450 = lean_ctor_get(x_449, 1); +lean_inc(x_450); +lean_dec(x_449); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9399,58 +9731,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_437 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_436); -if (lean_obj_tag(x_437) == 0) +lean_inc(x_4); +x_451 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_450); +if (lean_obj_tag(x_451) == 0) { -lean_object* x_438; lean_object* x_439; lean_object* x_440; lean_object* x_452; uint8_t x_453; -x_438 = lean_ctor_get(x_437, 1); -lean_inc(x_438); -lean_dec(x_437); +lean_object* x_452; lean_object* x_453; lean_object* x_454; lean_object* x_467; uint8_t x_468; +x_452 = lean_ctor_get(x_451, 1); +lean_inc(x_452); +lean_dec(x_451); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_439 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_439, 0, x_1); -lean_closure_set(x_439, 1, x_2); -x_452 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_453 = l_Lean_Expr_isConstOf(x_3, x_452); -if (x_453 == 0) -{ -lean_object* x_454; -x_454 = lean_box(0); -x_440 = x_454; -goto block_451; +x_453 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_453, 0, x_1); +lean_closure_set(x_453, 1, x_2); +lean_closure_set(x_453, 2, x_3); +x_467 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_468 = l_Lean_Expr_isConstOf(x_4, x_467); +if (x_468 == 0) +{ +lean_object* x_469; +lean_dec(x_3); +x_469 = lean_box(0); +x_454 = x_469; +goto block_466; } else { -lean_object* x_455; lean_object* x_456; uint8_t x_457; -x_455 = lean_array_get_size(x_4); -x_456 = lean_unsigned_to_nat(2u); -x_457 = lean_nat_dec_eq(x_455, x_456); -if (x_457 == 0) +lean_object* x_470; lean_object* x_471; uint8_t x_472; +x_470 = lean_array_get_size(x_5); +x_471 = lean_unsigned_to_nat(2u); +x_472 = lean_nat_dec_eq(x_470, x_471); +if (x_472 == 0) { -lean_object* x_458; -lean_dec(x_455); -x_458 = lean_box(0); -x_440 = x_458; -goto block_451; +lean_object* x_473; +lean_dec(x_470); +lean_dec(x_3); +x_473 = lean_box(0); +x_454 = x_473; +goto block_466; } else { -lean_object* x_459; uint8_t x_460; -lean_dec(x_439); -lean_dec(x_3); -x_459 = lean_unsigned_to_nat(0u); -x_460 = lean_nat_dec_lt(x_459, x_455); -lean_dec(x_455); -if (x_460 == 0) +lean_object* x_474; uint8_t x_475; lean_object* x_476; +lean_dec(x_453); +lean_dec(x_4); +x_474 = lean_unsigned_to_nat(0u); +x_475 = lean_nat_dec_lt(x_474, x_470); +lean_dec(x_470); +lean_inc(x_1); +x_476 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_476, 0, x_1); +if (x_475 == 0) { -lean_object* x_461; lean_object* x_462; lean_object* x_463; -lean_dec(x_4); -x_461 = l_Lean_instInhabitedExpr; -x_462 = l_outOfBounds___rarg(x_461); +lean_object* x_477; lean_object* x_478; lean_object* x_479; +lean_dec(x_5); +x_477 = l_Lean_instInhabitedExpr; +x_478 = l_outOfBounds___rarg(x_477); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9458,32 +9797,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_462); -x_463 = l_Lean_Meta_Grind_internalize(x_462, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_438); -if (lean_obj_tag(x_463) == 0) +lean_inc(x_478); +x_479 = l_Lean_Meta_Grind_internalize(x_478, x_2, x_476, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_452); +if (lean_obj_tag(x_479) == 0) { -lean_object* x_464; lean_object* x_465; lean_object* x_466; lean_object* x_467; lean_object* x_468; -x_464 = lean_ctor_get(x_463, 1); -lean_inc(x_464); -lean_dec(x_463); +lean_object* x_480; lean_object* x_481; lean_object* x_482; lean_object* x_483; lean_object* x_484; +x_480 = lean_ctor_get(x_479, 1); +lean_inc(x_480); +lean_dec(x_479); lean_inc(x_1); -x_465 = l_Lean_Meta_Grind_registerParent(x_1, x_462, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_464); -lean_dec(x_462); -x_466 = lean_ctor_get(x_465, 0); -lean_inc(x_466); -x_467 = lean_ctor_get(x_465, 1); -lean_inc(x_467); -lean_dec(x_465); -x_468 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_466, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_467); -lean_dec(x_466); -return x_468; +x_481 = l_Lean_Meta_Grind_registerParent(x_1, x_478, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_480); +lean_dec(x_478); +x_482 = lean_ctor_get(x_481, 0); +lean_inc(x_482); +x_483 = lean_ctor_get(x_481, 1); +lean_inc(x_483); +lean_dec(x_481); +x_484 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_482, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_483); +lean_dec(x_482); +return x_484; } else { -uint8_t x_469; -lean_dec(x_462); +uint8_t x_485; +lean_dec(x_478); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9491,34 +9830,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_469 = !lean_is_exclusive(x_463); -if (x_469 == 0) +x_485 = !lean_is_exclusive(x_479); +if (x_485 == 0) { -return x_463; +return x_479; } else { -lean_object* x_470; lean_object* x_471; lean_object* x_472; -x_470 = lean_ctor_get(x_463, 0); -x_471 = lean_ctor_get(x_463, 1); -lean_inc(x_471); -lean_inc(x_470); -lean_dec(x_463); -x_472 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_472, 0, x_470); -lean_ctor_set(x_472, 1, x_471); -return x_472; +lean_object* x_486; lean_object* x_487; lean_object* x_488; +x_486 = lean_ctor_get(x_479, 0); +x_487 = lean_ctor_get(x_479, 1); +lean_inc(x_487); +lean_inc(x_486); +lean_dec(x_479); +x_488 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_488, 0, x_486); +lean_ctor_set(x_488, 1, x_487); +return x_488; } } } else { -lean_object* x_473; lean_object* x_474; -x_473 = lean_array_fget(x_4, x_459); -lean_dec(x_4); +lean_object* x_489; lean_object* x_490; +x_489 = lean_array_fget(x_5, x_474); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9526,32 +9866,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_473); -x_474 = l_Lean_Meta_Grind_internalize(x_473, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_438); -if (lean_obj_tag(x_474) == 0) -{ -lean_object* x_475; lean_object* x_476; lean_object* x_477; lean_object* x_478; lean_object* x_479; -x_475 = lean_ctor_get(x_474, 1); -lean_inc(x_475); -lean_dec(x_474); -lean_inc(x_1); -x_476 = l_Lean_Meta_Grind_registerParent(x_1, x_473, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_475); -lean_dec(x_473); -x_477 = lean_ctor_get(x_476, 0); -lean_inc(x_477); -x_478 = lean_ctor_get(x_476, 1); -lean_inc(x_478); -lean_dec(x_476); -x_479 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_477, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_478); -lean_dec(x_477); -return x_479; +lean_inc(x_489); +x_490 = l_Lean_Meta_Grind_internalize(x_489, x_2, x_476, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_452); +if (lean_obj_tag(x_490) == 0) +{ +lean_object* x_491; lean_object* x_492; lean_object* x_493; lean_object* x_494; lean_object* x_495; +x_491 = lean_ctor_get(x_490, 1); +lean_inc(x_491); +lean_dec(x_490); +lean_inc(x_1); +x_492 = l_Lean_Meta_Grind_registerParent(x_1, x_489, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_491); +lean_dec(x_489); +x_493 = lean_ctor_get(x_492, 0); +lean_inc(x_493); +x_494 = lean_ctor_get(x_492, 1); +lean_inc(x_494); +lean_dec(x_492); +x_495 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_493, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_494); +lean_dec(x_493); +return x_495; } else { -uint8_t x_480; -lean_dec(x_473); +uint8_t x_496; +lean_dec(x_489); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9559,35 +9899,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_480 = !lean_is_exclusive(x_474); -if (x_480 == 0) +x_496 = !lean_is_exclusive(x_490); +if (x_496 == 0) { -return x_474; +return x_490; } else { -lean_object* x_481; lean_object* x_482; lean_object* x_483; -x_481 = lean_ctor_get(x_474, 0); -x_482 = lean_ctor_get(x_474, 1); -lean_inc(x_482); -lean_inc(x_481); -lean_dec(x_474); -x_483 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_483, 0, x_481); -lean_ctor_set(x_483, 1, x_482); -return x_483; +lean_object* x_497; lean_object* x_498; lean_object* x_499; +x_497 = lean_ctor_get(x_490, 0); +x_498 = lean_ctor_get(x_490, 1); +lean_inc(x_498); +lean_inc(x_497); +lean_dec(x_490); +x_499 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_499, 0, x_497); +lean_ctor_set(x_499, 1, x_498); +return x_499; } } } } } -block_451: +block_466: { -lean_object* x_441; -lean_dec(x_440); +lean_object* x_455; lean_object* x_456; +lean_dec(x_454); +lean_inc(x_1); +x_455 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_455, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9595,33 +9939,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_441 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_438); -if (lean_obj_tag(x_441) == 0) +lean_inc(x_4); +x_456 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_455, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_452); +if (lean_obj_tag(x_456) == 0) { -lean_object* x_442; lean_object* x_443; lean_object* x_444; lean_object* x_445; lean_object* x_446; -x_442 = lean_ctor_get(x_441, 1); -lean_inc(x_442); -lean_dec(x_441); +lean_object* x_457; lean_object* x_458; lean_object* x_459; lean_object* x_460; lean_object* x_461; +x_457 = lean_ctor_get(x_456, 1); +lean_inc(x_457); +lean_dec(x_456); lean_inc(x_1); -x_443 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_442); -lean_dec(x_3); -x_444 = lean_ctor_get(x_443, 0); -lean_inc(x_444); -x_445 = lean_ctor_get(x_443, 1); -lean_inc(x_445); -lean_dec(x_443); -x_446 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_439, x_444, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_445); -lean_dec(x_444); +x_458 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_457); lean_dec(x_4); -return x_446; +x_459 = lean_ctor_get(x_458, 0); +lean_inc(x_459); +x_460 = lean_ctor_get(x_458, 1); +lean_inc(x_460); +lean_dec(x_458); +x_461 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_453, x_459, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_460); +lean_dec(x_459); +lean_dec(x_5); +return x_461; } else { -uint8_t x_447; -lean_dec(x_439); +uint8_t x_462; +lean_dec(x_453); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9629,35 +9973,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_447 = !lean_is_exclusive(x_441); -if (x_447 == 0) +x_462 = !lean_is_exclusive(x_456); +if (x_462 == 0) { -return x_441; +return x_456; } else { -lean_object* x_448; lean_object* x_449; lean_object* x_450; -x_448 = lean_ctor_get(x_441, 0); -x_449 = lean_ctor_get(x_441, 1); -lean_inc(x_449); -lean_inc(x_448); -lean_dec(x_441); -x_450 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_450, 0, x_448); -lean_ctor_set(x_450, 1, x_449); -return x_450; +lean_object* x_463; lean_object* x_464; lean_object* x_465; +x_463 = lean_ctor_get(x_456, 0); +x_464 = lean_ctor_get(x_456, 1); +lean_inc(x_464); +lean_inc(x_463); +lean_dec(x_456); +x_465 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_465, 0, x_463); +lean_ctor_set(x_465, 1, x_464); +return x_465; } } } } else { -uint8_t x_484; +uint8_t x_500; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9665,34 +10009,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_484 = !lean_is_exclusive(x_437); -if (x_484 == 0) +x_500 = !lean_is_exclusive(x_451); +if (x_500 == 0) { -return x_437; +return x_451; } else { -lean_object* x_485; lean_object* x_486; lean_object* x_487; -x_485 = lean_ctor_get(x_437, 0); -x_486 = lean_ctor_get(x_437, 1); -lean_inc(x_486); -lean_inc(x_485); -lean_dec(x_437); -x_487 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_487, 0, x_485); -lean_ctor_set(x_487, 1, x_486); -return x_487; +lean_object* x_501; lean_object* x_502; lean_object* x_503; +x_501 = lean_ctor_get(x_451, 0); +x_502 = lean_ctor_get(x_451, 1); +lean_inc(x_502); +lean_inc(x_501); +lean_dec(x_451); +x_503 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_503, 0, x_501); +lean_ctor_set(x_503, 1, x_502); +return x_503; } } } else { -uint8_t x_488; +uint8_t x_504; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9700,52 +10045,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_488 = !lean_is_exclusive(x_433); -if (x_488 == 0) +x_504 = !lean_is_exclusive(x_447); +if (x_504 == 0) { -return x_433; +return x_447; } else { -lean_object* x_489; lean_object* x_490; lean_object* x_491; -x_489 = lean_ctor_get(x_433, 0); -x_490 = lean_ctor_get(x_433, 1); -lean_inc(x_490); -lean_inc(x_489); -lean_dec(x_433); -x_491 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_491, 0, x_489); -lean_ctor_set(x_491, 1, x_490); -return x_491; +lean_object* x_505; lean_object* x_506; lean_object* x_507; +x_505 = lean_ctor_get(x_447, 0); +x_506 = lean_ctor_get(x_447, 1); +lean_inc(x_506); +lean_inc(x_505); +lean_dec(x_447); +x_507 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_507, 0, x_505); +lean_ctor_set(x_507, 1, x_506); +return x_507; } } } case 9: { -lean_object* x_492; -lean_dec(x_5); +lean_object* x_508; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_492 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_492) == 0) +x_508 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_508) == 0) { -lean_object* x_493; lean_object* x_494; lean_object* x_495; lean_object* x_496; -x_493 = lean_ctor_get(x_492, 1); -lean_inc(x_493); -lean_dec(x_492); +lean_object* x_509; lean_object* x_510; lean_object* x_511; lean_object* x_512; +x_509 = lean_ctor_get(x_508, 1); +lean_inc(x_509); +lean_dec(x_508); lean_inc(x_1); -x_494 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_493); -x_495 = lean_ctor_get(x_494, 1); -lean_inc(x_495); -lean_dec(x_494); +x_510 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_509); +x_511 = lean_ctor_get(x_510, 1); +lean_inc(x_511); +lean_dec(x_510); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9753,58 +10099,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_496 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_495); -if (lean_obj_tag(x_496) == 0) +lean_inc(x_4); +x_512 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_511); +if (lean_obj_tag(x_512) == 0) { -lean_object* x_497; lean_object* x_498; lean_object* x_499; lean_object* x_511; uint8_t x_512; -x_497 = lean_ctor_get(x_496, 1); -lean_inc(x_497); -lean_dec(x_496); +lean_object* x_513; lean_object* x_514; lean_object* x_515; lean_object* x_528; uint8_t x_529; +x_513 = lean_ctor_get(x_512, 1); +lean_inc(x_513); +lean_dec(x_512); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_498 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_498, 0, x_1); -lean_closure_set(x_498, 1, x_2); -x_511 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_512 = l_Lean_Expr_isConstOf(x_3, x_511); -if (x_512 == 0) -{ -lean_object* x_513; -x_513 = lean_box(0); -x_499 = x_513; -goto block_510; +x_514 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_514, 0, x_1); +lean_closure_set(x_514, 1, x_2); +lean_closure_set(x_514, 2, x_3); +x_528 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_529 = l_Lean_Expr_isConstOf(x_4, x_528); +if (x_529 == 0) +{ +lean_object* x_530; +lean_dec(x_3); +x_530 = lean_box(0); +x_515 = x_530; +goto block_527; } else { -lean_object* x_514; lean_object* x_515; uint8_t x_516; -x_514 = lean_array_get_size(x_4); -x_515 = lean_unsigned_to_nat(2u); -x_516 = lean_nat_dec_eq(x_514, x_515); -if (x_516 == 0) +lean_object* x_531; lean_object* x_532; uint8_t x_533; +x_531 = lean_array_get_size(x_5); +x_532 = lean_unsigned_to_nat(2u); +x_533 = lean_nat_dec_eq(x_531, x_532); +if (x_533 == 0) { -lean_object* x_517; -lean_dec(x_514); -x_517 = lean_box(0); -x_499 = x_517; -goto block_510; +lean_object* x_534; +lean_dec(x_531); +lean_dec(x_3); +x_534 = lean_box(0); +x_515 = x_534; +goto block_527; } else { -lean_object* x_518; uint8_t x_519; -lean_dec(x_498); -lean_dec(x_3); -x_518 = lean_unsigned_to_nat(0u); -x_519 = lean_nat_dec_lt(x_518, x_514); +lean_object* x_535; uint8_t x_536; lean_object* x_537; lean_dec(x_514); -if (x_519 == 0) -{ -lean_object* x_520; lean_object* x_521; lean_object* x_522; lean_dec(x_4); -x_520 = l_Lean_instInhabitedExpr; -x_521 = l_outOfBounds___rarg(x_520); +x_535 = lean_unsigned_to_nat(0u); +x_536 = lean_nat_dec_lt(x_535, x_531); +lean_dec(x_531); +lean_inc(x_1); +x_537 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_537, 0, x_1); +if (x_536 == 0) +{ +lean_object* x_538; lean_object* x_539; lean_object* x_540; +lean_dec(x_5); +x_538 = l_Lean_instInhabitedExpr; +x_539 = l_outOfBounds___rarg(x_538); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9812,32 +10165,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_521); -x_522 = l_Lean_Meta_Grind_internalize(x_521, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_497); -if (lean_obj_tag(x_522) == 0) +lean_inc(x_539); +x_540 = l_Lean_Meta_Grind_internalize(x_539, x_2, x_537, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_513); +if (lean_obj_tag(x_540) == 0) { -lean_object* x_523; lean_object* x_524; lean_object* x_525; lean_object* x_526; lean_object* x_527; -x_523 = lean_ctor_get(x_522, 1); -lean_inc(x_523); -lean_dec(x_522); +lean_object* x_541; lean_object* x_542; lean_object* x_543; lean_object* x_544; lean_object* x_545; +x_541 = lean_ctor_get(x_540, 1); +lean_inc(x_541); +lean_dec(x_540); lean_inc(x_1); -x_524 = l_Lean_Meta_Grind_registerParent(x_1, x_521, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_523); -lean_dec(x_521); -x_525 = lean_ctor_get(x_524, 0); -lean_inc(x_525); -x_526 = lean_ctor_get(x_524, 1); -lean_inc(x_526); -lean_dec(x_524); -x_527 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_525, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_526); -lean_dec(x_525); -return x_527; +x_542 = l_Lean_Meta_Grind_registerParent(x_1, x_539, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_541); +lean_dec(x_539); +x_543 = lean_ctor_get(x_542, 0); +lean_inc(x_543); +x_544 = lean_ctor_get(x_542, 1); +lean_inc(x_544); +lean_dec(x_542); +x_545 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_543, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_544); +lean_dec(x_543); +return x_545; } else { -uint8_t x_528; -lean_dec(x_521); +uint8_t x_546; +lean_dec(x_539); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9845,34 +10198,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_528 = !lean_is_exclusive(x_522); -if (x_528 == 0) +x_546 = !lean_is_exclusive(x_540); +if (x_546 == 0) { -return x_522; +return x_540; } else { -lean_object* x_529; lean_object* x_530; lean_object* x_531; -x_529 = lean_ctor_get(x_522, 0); -x_530 = lean_ctor_get(x_522, 1); -lean_inc(x_530); -lean_inc(x_529); -lean_dec(x_522); -x_531 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_531, 0, x_529); -lean_ctor_set(x_531, 1, x_530); -return x_531; +lean_object* x_547; lean_object* x_548; lean_object* x_549; +x_547 = lean_ctor_get(x_540, 0); +x_548 = lean_ctor_get(x_540, 1); +lean_inc(x_548); +lean_inc(x_547); +lean_dec(x_540); +x_549 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_549, 0, x_547); +lean_ctor_set(x_549, 1, x_548); +return x_549; } } } else { -lean_object* x_532; lean_object* x_533; -x_532 = lean_array_fget(x_4, x_518); -lean_dec(x_4); +lean_object* x_550; lean_object* x_551; +x_550 = lean_array_fget(x_5, x_535); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9880,32 +10234,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_532); -x_533 = l_Lean_Meta_Grind_internalize(x_532, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_497); -if (lean_obj_tag(x_533) == 0) -{ -lean_object* x_534; lean_object* x_535; lean_object* x_536; lean_object* x_537; lean_object* x_538; -x_534 = lean_ctor_get(x_533, 1); -lean_inc(x_534); -lean_dec(x_533); -lean_inc(x_1); -x_535 = l_Lean_Meta_Grind_registerParent(x_1, x_532, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_534); -lean_dec(x_532); -x_536 = lean_ctor_get(x_535, 0); -lean_inc(x_536); -x_537 = lean_ctor_get(x_535, 1); -lean_inc(x_537); -lean_dec(x_535); -x_538 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_536, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_537); -lean_dec(x_536); -return x_538; -} -else -{ -uint8_t x_539; -lean_dec(x_532); +lean_inc(x_550); +x_551 = l_Lean_Meta_Grind_internalize(x_550, x_2, x_537, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_513); +if (lean_obj_tag(x_551) == 0) +{ +lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; lean_object* x_556; +x_552 = lean_ctor_get(x_551, 1); +lean_inc(x_552); +lean_dec(x_551); +lean_inc(x_1); +x_553 = l_Lean_Meta_Grind_registerParent(x_1, x_550, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_552); +lean_dec(x_550); +x_554 = lean_ctor_get(x_553, 0); +lean_inc(x_554); +x_555 = lean_ctor_get(x_553, 1); +lean_inc(x_555); +lean_dec(x_553); +x_556 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_554, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_555); +lean_dec(x_554); +return x_556; +} +else +{ +uint8_t x_557; +lean_dec(x_550); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9913,35 +10267,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_539 = !lean_is_exclusive(x_533); -if (x_539 == 0) +x_557 = !lean_is_exclusive(x_551); +if (x_557 == 0) { -return x_533; +return x_551; } else { -lean_object* x_540; lean_object* x_541; lean_object* x_542; -x_540 = lean_ctor_get(x_533, 0); -x_541 = lean_ctor_get(x_533, 1); -lean_inc(x_541); -lean_inc(x_540); -lean_dec(x_533); -x_542 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_542, 0, x_540); -lean_ctor_set(x_542, 1, x_541); -return x_542; +lean_object* x_558; lean_object* x_559; lean_object* x_560; +x_558 = lean_ctor_get(x_551, 0); +x_559 = lean_ctor_get(x_551, 1); +lean_inc(x_559); +lean_inc(x_558); +lean_dec(x_551); +x_560 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_560, 0, x_558); +lean_ctor_set(x_560, 1, x_559); +return x_560; } } } } } -block_510: +block_527: { -lean_object* x_500; -lean_dec(x_499); +lean_object* x_516; lean_object* x_517; +lean_dec(x_515); +lean_inc(x_1); +x_516 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_516, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9949,33 +10307,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_500 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_497); -if (lean_obj_tag(x_500) == 0) +lean_inc(x_4); +x_517 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_516, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_513); +if (lean_obj_tag(x_517) == 0) { -lean_object* x_501; lean_object* x_502; lean_object* x_503; lean_object* x_504; lean_object* x_505; -x_501 = lean_ctor_get(x_500, 1); -lean_inc(x_501); -lean_dec(x_500); +lean_object* x_518; lean_object* x_519; lean_object* x_520; lean_object* x_521; lean_object* x_522; +x_518 = lean_ctor_get(x_517, 1); +lean_inc(x_518); +lean_dec(x_517); lean_inc(x_1); -x_502 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_501); -lean_dec(x_3); -x_503 = lean_ctor_get(x_502, 0); -lean_inc(x_503); -x_504 = lean_ctor_get(x_502, 1); -lean_inc(x_504); -lean_dec(x_502); -x_505 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_498, x_503, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_504); -lean_dec(x_503); +x_519 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_518); lean_dec(x_4); -return x_505; +x_520 = lean_ctor_get(x_519, 0); +lean_inc(x_520); +x_521 = lean_ctor_get(x_519, 1); +lean_inc(x_521); +lean_dec(x_519); +x_522 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_514, x_520, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_521); +lean_dec(x_520); +lean_dec(x_5); +return x_522; } else { -uint8_t x_506; -lean_dec(x_498); +uint8_t x_523; +lean_dec(x_514); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9983,35 +10341,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_506 = !lean_is_exclusive(x_500); -if (x_506 == 0) +x_523 = !lean_is_exclusive(x_517); +if (x_523 == 0) { -return x_500; +return x_517; } else { -lean_object* x_507; lean_object* x_508; lean_object* x_509; -x_507 = lean_ctor_get(x_500, 0); -x_508 = lean_ctor_get(x_500, 1); -lean_inc(x_508); -lean_inc(x_507); -lean_dec(x_500); -x_509 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_509, 0, x_507); -lean_ctor_set(x_509, 1, x_508); -return x_509; +lean_object* x_524; lean_object* x_525; lean_object* x_526; +x_524 = lean_ctor_get(x_517, 0); +x_525 = lean_ctor_get(x_517, 1); +lean_inc(x_525); +lean_inc(x_524); +lean_dec(x_517); +x_526 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_526, 0, x_524); +lean_ctor_set(x_526, 1, x_525); +return x_526; } } } } else { -uint8_t x_543; +uint8_t x_561; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10019,34 +10377,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_543 = !lean_is_exclusive(x_496); -if (x_543 == 0) +x_561 = !lean_is_exclusive(x_512); +if (x_561 == 0) { -return x_496; +return x_512; } else { -lean_object* x_544; lean_object* x_545; lean_object* x_546; -x_544 = lean_ctor_get(x_496, 0); -x_545 = lean_ctor_get(x_496, 1); -lean_inc(x_545); -lean_inc(x_544); -lean_dec(x_496); -x_546 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_546, 0, x_544); -lean_ctor_set(x_546, 1, x_545); -return x_546; +lean_object* x_562; lean_object* x_563; lean_object* x_564; +x_562 = lean_ctor_get(x_512, 0); +x_563 = lean_ctor_get(x_512, 1); +lean_inc(x_563); +lean_inc(x_562); +lean_dec(x_512); +x_564 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_564, 0, x_562); +lean_ctor_set(x_564, 1, x_563); +return x_564; } } } else { -uint8_t x_547; +uint8_t x_565; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10054,52 +10413,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_547 = !lean_is_exclusive(x_492); -if (x_547 == 0) +x_565 = !lean_is_exclusive(x_508); +if (x_565 == 0) { -return x_492; +return x_508; } else { -lean_object* x_548; lean_object* x_549; lean_object* x_550; -x_548 = lean_ctor_get(x_492, 0); -x_549 = lean_ctor_get(x_492, 1); -lean_inc(x_549); -lean_inc(x_548); -lean_dec(x_492); -x_550 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_550, 0, x_548); -lean_ctor_set(x_550, 1, x_549); -return x_550; +lean_object* x_566; lean_object* x_567; lean_object* x_568; +x_566 = lean_ctor_get(x_508, 0); +x_567 = lean_ctor_get(x_508, 1); +lean_inc(x_567); +lean_inc(x_566); +lean_dec(x_508); +x_568 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_568, 0, x_566); +lean_ctor_set(x_568, 1, x_567); +return x_568; } } } case 10: { -lean_object* x_551; -lean_dec(x_5); +lean_object* x_569; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_551 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_551) == 0) +x_569 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_569) == 0) { -lean_object* x_552; lean_object* x_553; lean_object* x_554; lean_object* x_555; -x_552 = lean_ctor_get(x_551, 1); -lean_inc(x_552); -lean_dec(x_551); +lean_object* x_570; lean_object* x_571; lean_object* x_572; lean_object* x_573; +x_570 = lean_ctor_get(x_569, 1); +lean_inc(x_570); +lean_dec(x_569); lean_inc(x_1); -x_553 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_552); -x_554 = lean_ctor_get(x_553, 1); -lean_inc(x_554); -lean_dec(x_553); +x_571 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_570); +x_572 = lean_ctor_get(x_571, 1); +lean_inc(x_572); +lean_dec(x_571); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10107,58 +10467,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_555 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_554); -if (lean_obj_tag(x_555) == 0) +lean_inc(x_4); +x_573 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_572); +if (lean_obj_tag(x_573) == 0) { -lean_object* x_556; lean_object* x_557; lean_object* x_558; lean_object* x_570; uint8_t x_571; -x_556 = lean_ctor_get(x_555, 1); -lean_inc(x_556); -lean_dec(x_555); +lean_object* x_574; lean_object* x_575; lean_object* x_576; lean_object* x_589; uint8_t x_590; +x_574 = lean_ctor_get(x_573, 1); +lean_inc(x_574); +lean_dec(x_573); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_557 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_557, 0, x_1); -lean_closure_set(x_557, 1, x_2); -x_570 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_571 = l_Lean_Expr_isConstOf(x_3, x_570); -if (x_571 == 0) -{ -lean_object* x_572; -x_572 = lean_box(0); -x_558 = x_572; -goto block_569; +x_575 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_575, 0, x_1); +lean_closure_set(x_575, 1, x_2); +lean_closure_set(x_575, 2, x_3); +x_589 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_590 = l_Lean_Expr_isConstOf(x_4, x_589); +if (x_590 == 0) +{ +lean_object* x_591; +lean_dec(x_3); +x_591 = lean_box(0); +x_576 = x_591; +goto block_588; } else { -lean_object* x_573; lean_object* x_574; uint8_t x_575; -x_573 = lean_array_get_size(x_4); -x_574 = lean_unsigned_to_nat(2u); -x_575 = lean_nat_dec_eq(x_573, x_574); -if (x_575 == 0) +lean_object* x_592; lean_object* x_593; uint8_t x_594; +x_592 = lean_array_get_size(x_5); +x_593 = lean_unsigned_to_nat(2u); +x_594 = lean_nat_dec_eq(x_592, x_593); +if (x_594 == 0) { -lean_object* x_576; -lean_dec(x_573); -x_576 = lean_box(0); -x_558 = x_576; -goto block_569; +lean_object* x_595; +lean_dec(x_592); +lean_dec(x_3); +x_595 = lean_box(0); +x_576 = x_595; +goto block_588; } else { -lean_object* x_577; uint8_t x_578; -lean_dec(x_557); -lean_dec(x_3); -x_577 = lean_unsigned_to_nat(0u); -x_578 = lean_nat_dec_lt(x_577, x_573); -lean_dec(x_573); -if (x_578 == 0) -{ -lean_object* x_579; lean_object* x_580; lean_object* x_581; +lean_object* x_596; uint8_t x_597; lean_object* x_598; +lean_dec(x_575); lean_dec(x_4); -x_579 = l_Lean_instInhabitedExpr; -x_580 = l_outOfBounds___rarg(x_579); +x_596 = lean_unsigned_to_nat(0u); +x_597 = lean_nat_dec_lt(x_596, x_592); +lean_dec(x_592); +lean_inc(x_1); +x_598 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_598, 0, x_1); +if (x_597 == 0) +{ +lean_object* x_599; lean_object* x_600; lean_object* x_601; +lean_dec(x_5); +x_599 = l_Lean_instInhabitedExpr; +x_600 = l_outOfBounds___rarg(x_599); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10166,32 +10533,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_580); -x_581 = l_Lean_Meta_Grind_internalize(x_580, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_556); -if (lean_obj_tag(x_581) == 0) +lean_inc(x_600); +x_601 = l_Lean_Meta_Grind_internalize(x_600, x_2, x_598, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_574); +if (lean_obj_tag(x_601) == 0) { -lean_object* x_582; lean_object* x_583; lean_object* x_584; lean_object* x_585; lean_object* x_586; -x_582 = lean_ctor_get(x_581, 1); -lean_inc(x_582); -lean_dec(x_581); +lean_object* x_602; lean_object* x_603; lean_object* x_604; lean_object* x_605; lean_object* x_606; +x_602 = lean_ctor_get(x_601, 1); +lean_inc(x_602); +lean_dec(x_601); lean_inc(x_1); -x_583 = l_Lean_Meta_Grind_registerParent(x_1, x_580, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_582); -lean_dec(x_580); -x_584 = lean_ctor_get(x_583, 0); -lean_inc(x_584); -x_585 = lean_ctor_get(x_583, 1); -lean_inc(x_585); -lean_dec(x_583); -x_586 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_584, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_585); -lean_dec(x_584); -return x_586; +x_603 = l_Lean_Meta_Grind_registerParent(x_1, x_600, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_602); +lean_dec(x_600); +x_604 = lean_ctor_get(x_603, 0); +lean_inc(x_604); +x_605 = lean_ctor_get(x_603, 1); +lean_inc(x_605); +lean_dec(x_603); +x_606 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_604, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_605); +lean_dec(x_604); +return x_606; } else { -uint8_t x_587; -lean_dec(x_580); +uint8_t x_607; +lean_dec(x_600); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10199,34 +10566,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_587 = !lean_is_exclusive(x_581); -if (x_587 == 0) +x_607 = !lean_is_exclusive(x_601); +if (x_607 == 0) { -return x_581; +return x_601; } else { -lean_object* x_588; lean_object* x_589; lean_object* x_590; -x_588 = lean_ctor_get(x_581, 0); -x_589 = lean_ctor_get(x_581, 1); -lean_inc(x_589); -lean_inc(x_588); -lean_dec(x_581); -x_590 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_590, 0, x_588); -lean_ctor_set(x_590, 1, x_589); -return x_590; +lean_object* x_608; lean_object* x_609; lean_object* x_610; +x_608 = lean_ctor_get(x_601, 0); +x_609 = lean_ctor_get(x_601, 1); +lean_inc(x_609); +lean_inc(x_608); +lean_dec(x_601); +x_610 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_610, 0, x_608); +lean_ctor_set(x_610, 1, x_609); +return x_610; } } } else { -lean_object* x_591; lean_object* x_592; -x_591 = lean_array_fget(x_4, x_577); -lean_dec(x_4); +lean_object* x_611; lean_object* x_612; +x_611 = lean_array_fget(x_5, x_596); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10234,32 +10602,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_591); -x_592 = l_Lean_Meta_Grind_internalize(x_591, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_556); -if (lean_obj_tag(x_592) == 0) +lean_inc(x_611); +x_612 = l_Lean_Meta_Grind_internalize(x_611, x_2, x_598, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_574); +if (lean_obj_tag(x_612) == 0) { -lean_object* x_593; lean_object* x_594; lean_object* x_595; lean_object* x_596; lean_object* x_597; -x_593 = lean_ctor_get(x_592, 1); -lean_inc(x_593); -lean_dec(x_592); +lean_object* x_613; lean_object* x_614; lean_object* x_615; lean_object* x_616; lean_object* x_617; +x_613 = lean_ctor_get(x_612, 1); +lean_inc(x_613); +lean_dec(x_612); lean_inc(x_1); -x_594 = l_Lean_Meta_Grind_registerParent(x_1, x_591, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_593); -lean_dec(x_591); -x_595 = lean_ctor_get(x_594, 0); -lean_inc(x_595); -x_596 = lean_ctor_get(x_594, 1); -lean_inc(x_596); -lean_dec(x_594); -x_597 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_595, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_596); -lean_dec(x_595); -return x_597; +x_614 = l_Lean_Meta_Grind_registerParent(x_1, x_611, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_613); +lean_dec(x_611); +x_615 = lean_ctor_get(x_614, 0); +lean_inc(x_615); +x_616 = lean_ctor_get(x_614, 1); +lean_inc(x_616); +lean_dec(x_614); +x_617 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_615, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_616); +lean_dec(x_615); +return x_617; } else { -uint8_t x_598; -lean_dec(x_591); +uint8_t x_618; +lean_dec(x_611); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10267,35 +10635,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_598 = !lean_is_exclusive(x_592); -if (x_598 == 0) +x_618 = !lean_is_exclusive(x_612); +if (x_618 == 0) { -return x_592; +return x_612; } else { -lean_object* x_599; lean_object* x_600; lean_object* x_601; -x_599 = lean_ctor_get(x_592, 0); -x_600 = lean_ctor_get(x_592, 1); -lean_inc(x_600); -lean_inc(x_599); -lean_dec(x_592); -x_601 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_601, 0, x_599); -lean_ctor_set(x_601, 1, x_600); -return x_601; +lean_object* x_619; lean_object* x_620; lean_object* x_621; +x_619 = lean_ctor_get(x_612, 0); +x_620 = lean_ctor_get(x_612, 1); +lean_inc(x_620); +lean_inc(x_619); +lean_dec(x_612); +x_621 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_621, 0, x_619); +lean_ctor_set(x_621, 1, x_620); +return x_621; } } } } } -block_569: +block_588: { -lean_object* x_559; -lean_dec(x_558); +lean_object* x_577; lean_object* x_578; +lean_dec(x_576); +lean_inc(x_1); +x_577 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_577, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10303,33 +10675,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_559 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_556); -if (lean_obj_tag(x_559) == 0) +lean_inc(x_4); +x_578 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_577, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_574); +if (lean_obj_tag(x_578) == 0) { -lean_object* x_560; lean_object* x_561; lean_object* x_562; lean_object* x_563; lean_object* x_564; -x_560 = lean_ctor_get(x_559, 1); -lean_inc(x_560); -lean_dec(x_559); +lean_object* x_579; lean_object* x_580; lean_object* x_581; lean_object* x_582; lean_object* x_583; +x_579 = lean_ctor_get(x_578, 1); +lean_inc(x_579); +lean_dec(x_578); lean_inc(x_1); -x_561 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_560); -lean_dec(x_3); -x_562 = lean_ctor_get(x_561, 0); -lean_inc(x_562); -x_563 = lean_ctor_get(x_561, 1); -lean_inc(x_563); -lean_dec(x_561); -x_564 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_557, x_562, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_563); -lean_dec(x_562); +x_580 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_579); lean_dec(x_4); -return x_564; +x_581 = lean_ctor_get(x_580, 0); +lean_inc(x_581); +x_582 = lean_ctor_get(x_580, 1); +lean_inc(x_582); +lean_dec(x_580); +x_583 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_575, x_581, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_582); +lean_dec(x_581); +lean_dec(x_5); +return x_583; } else { -uint8_t x_565; -lean_dec(x_557); +uint8_t x_584; +lean_dec(x_575); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10337,35 +10709,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_565 = !lean_is_exclusive(x_559); -if (x_565 == 0) +x_584 = !lean_is_exclusive(x_578); +if (x_584 == 0) { -return x_559; +return x_578; } else { -lean_object* x_566; lean_object* x_567; lean_object* x_568; -x_566 = lean_ctor_get(x_559, 0); -x_567 = lean_ctor_get(x_559, 1); -lean_inc(x_567); -lean_inc(x_566); -lean_dec(x_559); -x_568 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_568, 0, x_566); -lean_ctor_set(x_568, 1, x_567); -return x_568; +lean_object* x_585; lean_object* x_586; lean_object* x_587; +x_585 = lean_ctor_get(x_578, 0); +x_586 = lean_ctor_get(x_578, 1); +lean_inc(x_586); +lean_inc(x_585); +lean_dec(x_578); +x_587 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_587, 0, x_585); +lean_ctor_set(x_587, 1, x_586); +return x_587; } } } } else { -uint8_t x_602; +uint8_t x_622; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10373,34 +10745,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_602 = !lean_is_exclusive(x_555); -if (x_602 == 0) +x_622 = !lean_is_exclusive(x_573); +if (x_622 == 0) { -return x_555; +return x_573; } else { -lean_object* x_603; lean_object* x_604; lean_object* x_605; -x_603 = lean_ctor_get(x_555, 0); -x_604 = lean_ctor_get(x_555, 1); -lean_inc(x_604); -lean_inc(x_603); -lean_dec(x_555); -x_605 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_605, 0, x_603); -lean_ctor_set(x_605, 1, x_604); -return x_605; +lean_object* x_623; lean_object* x_624; lean_object* x_625; +x_623 = lean_ctor_get(x_573, 0); +x_624 = lean_ctor_get(x_573, 1); +lean_inc(x_624); +lean_inc(x_623); +lean_dec(x_573); +x_625 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_625, 0, x_623); +lean_ctor_set(x_625, 1, x_624); +return x_625; } } } else { -uint8_t x_606; +uint8_t x_626; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10408,52 +10781,53 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_606 = !lean_is_exclusive(x_551); -if (x_606 == 0) +x_626 = !lean_is_exclusive(x_569); +if (x_626 == 0) { -return x_551; +return x_569; } else { -lean_object* x_607; lean_object* x_608; lean_object* x_609; -x_607 = lean_ctor_get(x_551, 0); -x_608 = lean_ctor_get(x_551, 1); -lean_inc(x_608); -lean_inc(x_607); -lean_dec(x_551); -x_609 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_609, 0, x_607); -lean_ctor_set(x_609, 1, x_608); -return x_609; +lean_object* x_627; lean_object* x_628; lean_object* x_629; +x_627 = lean_ctor_get(x_569, 0); +x_628 = lean_ctor_get(x_569, 1); +lean_inc(x_628); +lean_inc(x_627); +lean_dec(x_569); +x_629 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_629, 0, x_627); +lean_ctor_set(x_629, 1, x_628); +return x_629; } } } default: { -lean_object* x_610; -lean_dec(x_5); +lean_object* x_630; +lean_dec(x_6); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); -lean_inc(x_10); lean_inc(x_1); -x_610 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_610) == 0) +x_630 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +if (lean_obj_tag(x_630) == 0) { -lean_object* x_611; lean_object* x_612; lean_object* x_613; lean_object* x_614; -x_611 = lean_ctor_get(x_610, 1); -lean_inc(x_611); -lean_dec(x_610); +lean_object* x_631; lean_object* x_632; lean_object* x_633; lean_object* x_634; +x_631 = lean_ctor_get(x_630, 1); +lean_inc(x_631); +lean_dec(x_630); lean_inc(x_1); -x_612 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_611); -x_613 = lean_ctor_get(x_612, 1); -lean_inc(x_613); -lean_dec(x_612); +x_632 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_pushCastHEqs(x_1, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_631); +x_633 = lean_ctor_get(x_632, 1); +lean_inc(x_633); +lean_dec(x_632); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10461,58 +10835,65 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_614 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_613); -if (lean_obj_tag(x_614) == 0) +lean_inc(x_4); +x_634 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns(x_4, x_2, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_633); +if (lean_obj_tag(x_634) == 0) { -lean_object* x_615; lean_object* x_616; lean_object* x_617; lean_object* x_629; uint8_t x_630; -x_615 = lean_ctor_get(x_614, 1); -lean_inc(x_615); -lean_dec(x_614); +lean_object* x_635; lean_object* x_636; lean_object* x_637; lean_object* x_650; uint8_t x_651; +x_635 = lean_ctor_get(x_634, 1); +lean_inc(x_635); +lean_dec(x_634); +lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_616 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed), 12, 2); -lean_closure_set(x_616, 0, x_1); -lean_closure_set(x_616, 1, x_2); -x_629 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2; -x_630 = l_Lean_Expr_isConstOf(x_3, x_629); -if (x_630 == 0) -{ -lean_object* x_631; -x_631 = lean_box(0); -x_617 = x_631; -goto block_628; +x_636 = lean_alloc_closure((void*)(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed), 13, 3); +lean_closure_set(x_636, 0, x_1); +lean_closure_set(x_636, 1, x_2); +lean_closure_set(x_636, 2, x_3); +x_650 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2; +x_651 = l_Lean_Expr_isConstOf(x_4, x_650); +if (x_651 == 0) +{ +lean_object* x_652; +lean_dec(x_3); +x_652 = lean_box(0); +x_637 = x_652; +goto block_649; } else { -lean_object* x_632; lean_object* x_633; uint8_t x_634; -x_632 = lean_array_get_size(x_4); -x_633 = lean_unsigned_to_nat(2u); -x_634 = lean_nat_dec_eq(x_632, x_633); -if (x_634 == 0) +lean_object* x_653; lean_object* x_654; uint8_t x_655; +x_653 = lean_array_get_size(x_5); +x_654 = lean_unsigned_to_nat(2u); +x_655 = lean_nat_dec_eq(x_653, x_654); +if (x_655 == 0) { -lean_object* x_635; -lean_dec(x_632); -x_635 = lean_box(0); -x_617 = x_635; -goto block_628; +lean_object* x_656; +lean_dec(x_653); +lean_dec(x_3); +x_656 = lean_box(0); +x_637 = x_656; +goto block_649; } else { -lean_object* x_636; uint8_t x_637; -lean_dec(x_616); -lean_dec(x_3); -x_636 = lean_unsigned_to_nat(0u); -x_637 = lean_nat_dec_lt(x_636, x_632); -lean_dec(x_632); -if (x_637 == 0) -{ -lean_object* x_638; lean_object* x_639; lean_object* x_640; +lean_object* x_657; uint8_t x_658; lean_object* x_659; +lean_dec(x_636); lean_dec(x_4); -x_638 = l_Lean_instInhabitedExpr; -x_639 = l_outOfBounds___rarg(x_638); +x_657 = lean_unsigned_to_nat(0u); +x_658 = lean_nat_dec_lt(x_657, x_653); +lean_dec(x_653); +lean_inc(x_1); +x_659 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_659, 0, x_1); +if (x_658 == 0) +{ +lean_object* x_660; lean_object* x_661; lean_object* x_662; +lean_dec(x_5); +x_660 = l_Lean_instInhabitedExpr; +x_661 = l_outOfBounds___rarg(x_660); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10520,32 +10901,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_639); -x_640 = l_Lean_Meta_Grind_internalize(x_639, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_615); -if (lean_obj_tag(x_640) == 0) +lean_inc(x_661); +x_662 = l_Lean_Meta_Grind_internalize(x_661, x_2, x_659, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_635); +if (lean_obj_tag(x_662) == 0) { -lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; lean_object* x_645; -x_641 = lean_ctor_get(x_640, 1); -lean_inc(x_641); -lean_dec(x_640); +lean_object* x_663; lean_object* x_664; lean_object* x_665; lean_object* x_666; lean_object* x_667; +x_663 = lean_ctor_get(x_662, 1); +lean_inc(x_663); +lean_dec(x_662); lean_inc(x_1); -x_642 = l_Lean_Meta_Grind_registerParent(x_1, x_639, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_641); -lean_dec(x_639); -x_643 = lean_ctor_get(x_642, 0); -lean_inc(x_643); -x_644 = lean_ctor_get(x_642, 1); -lean_inc(x_644); -lean_dec(x_642); -x_645 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_643, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_644); -lean_dec(x_643); -return x_645; +x_664 = l_Lean_Meta_Grind_registerParent(x_1, x_661, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_663); +lean_dec(x_661); +x_665 = lean_ctor_get(x_664, 0); +lean_inc(x_665); +x_666 = lean_ctor_get(x_664, 1); +lean_inc(x_666); +lean_dec(x_664); +x_667 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_665, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_666); +lean_dec(x_665); +return x_667; } else { -uint8_t x_646; -lean_dec(x_639); +uint8_t x_668; +lean_dec(x_661); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10553,34 +10934,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_646 = !lean_is_exclusive(x_640); -if (x_646 == 0) +x_668 = !lean_is_exclusive(x_662); +if (x_668 == 0) { -return x_640; +return x_662; } else { -lean_object* x_647; lean_object* x_648; lean_object* x_649; -x_647 = lean_ctor_get(x_640, 0); -x_648 = lean_ctor_get(x_640, 1); -lean_inc(x_648); -lean_inc(x_647); -lean_dec(x_640); -x_649 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_649, 0, x_647); -lean_ctor_set(x_649, 1, x_648); -return x_649; +lean_object* x_669; lean_object* x_670; lean_object* x_671; +x_669 = lean_ctor_get(x_662, 0); +x_670 = lean_ctor_get(x_662, 1); +lean_inc(x_670); +lean_inc(x_669); +lean_dec(x_662); +x_671 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_671, 0, x_669); +lean_ctor_set(x_671, 1, x_670); +return x_671; } } } else { -lean_object* x_650; lean_object* x_651; -x_650 = lean_array_fget(x_4, x_636); -lean_dec(x_4); +lean_object* x_672; lean_object* x_673; +x_672 = lean_array_fget(x_5, x_657); +lean_dec(x_5); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10588,32 +10970,32 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_650); -x_651 = l_Lean_Meta_Grind_internalize(x_650, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_615); -if (lean_obj_tag(x_651) == 0) -{ -lean_object* x_652; lean_object* x_653; lean_object* x_654; lean_object* x_655; lean_object* x_656; -x_652 = lean_ctor_get(x_651, 1); -lean_inc(x_652); -lean_dec(x_651); -lean_inc(x_1); -x_653 = l_Lean_Meta_Grind_registerParent(x_1, x_650, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_652); -lean_dec(x_650); -x_654 = lean_ctor_get(x_653, 0); -lean_inc(x_654); -x_655 = lean_ctor_get(x_653, 1); -lean_inc(x_655); -lean_dec(x_653); -x_656 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_654, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_655); -lean_dec(x_654); -return x_656; +lean_inc(x_672); +x_673 = l_Lean_Meta_Grind_internalize(x_672, x_2, x_659, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_635); +if (lean_obj_tag(x_673) == 0) +{ +lean_object* x_674; lean_object* x_675; lean_object* x_676; lean_object* x_677; lean_object* x_678; +x_674 = lean_ctor_get(x_673, 1); +lean_inc(x_674); +lean_dec(x_673); +lean_inc(x_1); +x_675 = l_Lean_Meta_Grind_registerParent(x_1, x_672, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_674); +lean_dec(x_672); +x_676 = lean_ctor_get(x_675, 0); +lean_inc(x_676); +x_677 = lean_ctor_get(x_675, 1); +lean_inc(x_677); +lean_dec(x_675); +x_678 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_676, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_677); +lean_dec(x_676); +return x_678; } else { -uint8_t x_657; -lean_dec(x_650); +uint8_t x_679; +lean_dec(x_672); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10621,35 +11003,39 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_657 = !lean_is_exclusive(x_651); -if (x_657 == 0) +x_679 = !lean_is_exclusive(x_673); +if (x_679 == 0) { -return x_651; +return x_673; } else { -lean_object* x_658; lean_object* x_659; lean_object* x_660; -x_658 = lean_ctor_get(x_651, 0); -x_659 = lean_ctor_get(x_651, 1); -lean_inc(x_659); -lean_inc(x_658); -lean_dec(x_651); -x_660 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_660, 0, x_658); -lean_ctor_set(x_660, 1, x_659); -return x_660; +lean_object* x_680; lean_object* x_681; lean_object* x_682; +x_680 = lean_ctor_get(x_673, 0); +x_681 = lean_ctor_get(x_673, 1); +lean_inc(x_681); +lean_inc(x_680); +lean_dec(x_673); +x_682 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_682, 0, x_680); +lean_ctor_set(x_682, 1, x_681); +return x_682; } } } } } -block_628: +block_649: { -lean_object* x_618; -lean_dec(x_617); +lean_object* x_638; lean_object* x_639; +lean_dec(x_637); +lean_inc(x_1); +x_638 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_638, 0, x_1); +lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -10657,33 +11043,33 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); -lean_inc(x_6); lean_inc(x_2); -lean_inc(x_3); -x_618 = l_Lean_Meta_Grind_internalize(x_3, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_615); -if (lean_obj_tag(x_618) == 0) +lean_inc(x_4); +x_639 = l_Lean_Meta_Grind_internalize(x_4, x_2, x_638, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_635); +if (lean_obj_tag(x_639) == 0) { -lean_object* x_619; lean_object* x_620; lean_object* x_621; lean_object* x_622; lean_object* x_623; -x_619 = lean_ctor_get(x_618, 1); -lean_inc(x_619); -lean_dec(x_618); +lean_object* x_640; lean_object* x_641; lean_object* x_642; lean_object* x_643; lean_object* x_644; +x_640 = lean_ctor_get(x_639, 1); +lean_inc(x_640); +lean_dec(x_639); lean_inc(x_1); -x_620 = l_Lean_Meta_Grind_registerParent(x_1, x_3, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_619); -lean_dec(x_3); -x_621 = lean_ctor_get(x_620, 0); -lean_inc(x_621); -x_622 = lean_ctor_get(x_620, 1); -lean_inc(x_622); -lean_dec(x_620); -x_623 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_4, x_1, x_2, x_616, x_621, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_622); -lean_dec(x_621); +x_641 = l_Lean_Meta_Grind_registerParent(x_1, x_4, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_640); lean_dec(x_4); -return x_623; +x_642 = lean_ctor_get(x_641, 0); +lean_inc(x_642); +x_643 = lean_ctor_get(x_641, 1); +lean_inc(x_643); +lean_dec(x_641); +x_644 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_5, x_1, x_2, x_636, x_642, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_643); +lean_dec(x_642); +lean_dec(x_5); +return x_644; } else { -uint8_t x_624; -lean_dec(x_616); +uint8_t x_645; +lean_dec(x_636); +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10691,35 +11077,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_624 = !lean_is_exclusive(x_618); -if (x_624 == 0) +x_645 = !lean_is_exclusive(x_639); +if (x_645 == 0) { -return x_618; +return x_639; } else { -lean_object* x_625; lean_object* x_626; lean_object* x_627; -x_625 = lean_ctor_get(x_618, 0); -x_626 = lean_ctor_get(x_618, 1); -lean_inc(x_626); -lean_inc(x_625); -lean_dec(x_618); -x_627 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_627, 0, x_625); -lean_ctor_set(x_627, 1, x_626); -return x_627; +lean_object* x_646; lean_object* x_647; lean_object* x_648; +x_646 = lean_ctor_get(x_639, 0); +x_647 = lean_ctor_get(x_639, 1); +lean_inc(x_647); +lean_inc(x_646); +lean_dec(x_639); +x_648 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_648, 0, x_646); +lean_ctor_set(x_648, 1, x_647); +return x_648; } } } } else { -uint8_t x_661; +uint8_t x_683; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10727,34 +11113,35 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_661 = !lean_is_exclusive(x_614); -if (x_661 == 0) +x_683 = !lean_is_exclusive(x_634); +if (x_683 == 0) { -return x_614; +return x_634; } else { -lean_object* x_662; lean_object* x_663; lean_object* x_664; -x_662 = lean_ctor_get(x_614, 0); -x_663 = lean_ctor_get(x_614, 1); -lean_inc(x_663); -lean_inc(x_662); -lean_dec(x_614); -x_664 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_664, 0, x_662); -lean_ctor_set(x_664, 1, x_663); -return x_664; +lean_object* x_684; lean_object* x_685; lean_object* x_686; +x_684 = lean_ctor_get(x_634, 0); +x_685 = lean_ctor_get(x_634, 1); +lean_inc(x_685); +lean_inc(x_684); +lean_dec(x_634); +x_686 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_686, 0, x_684); +lean_ctor_set(x_686, 1, x_685); +return x_686; } } } else { -uint8_t x_665; +uint8_t x_687; +lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -10762,28 +11149,28 @@ lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); +lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_665 = !lean_is_exclusive(x_610); -if (x_665 == 0) +x_687 = !lean_is_exclusive(x_630); +if (x_687 == 0) { -return x_610; +return x_630; } else { -lean_object* x_666; lean_object* x_667; lean_object* x_668; -x_666 = lean_ctor_get(x_610, 0); -x_667 = lean_ctor_get(x_610, 1); -lean_inc(x_667); -lean_inc(x_666); -lean_dec(x_610); -x_668 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_668, 0, x_666); -lean_ctor_set(x_668, 1, x_667); -return x_668; +lean_object* x_688; lean_object* x_689; lean_object* x_690; +x_688 = lean_ctor_get(x_630, 0); +x_689 = lean_ctor_get(x_630, 1); +lean_inc(x_689); +lean_inc(x_688); +lean_dec(x_630); +x_690 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_690, 0, x_688); +lean_ctor_set(x_690, 1, x_689); +return x_690; } } } @@ -10837,7 +11224,7 @@ static lean_object* _init_l_Lean_Meta_Grind_internalize___lambda__3___closed__4( lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Meta_Grind_internalize___lambda__3___closed__1; x_2 = l_Lean_Meta_Grind_internalize___lambda__3___closed__2; -x_3 = lean_unsigned_to_nat(144u); +x_3 = lean_unsigned_to_nat(153u); x_4 = lean_unsigned_to_nat(16u); x_5 = l_Lean_Meta_Grind_internalize___lambda__3___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -10861,36 +11248,39 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_13; lean_object* x_14; +lean_object* x_14; lean_object* x_15; +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_13 = l_Lean_Meta_Grind_internalize___lambda__3___closed__4; -x_14 = l_panic___at_Lean_Meta_Grind_internalize___spec__1(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -return x_14; +x_14 = l_Lean_Meta_Grind_internalize___lambda__3___closed__4; +x_15 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +return x_15; } case 2: { -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_15 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_16 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_unbox(x_17); -lean_dec(x_17); -if (x_18 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +lean_dec(x_3); +x_16 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_17 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_16, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) { -lean_object* x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_16, 1); -lean_inc(x_19); -lean_dec(x_16); -x_20 = 0; -x_21 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_20, x_20, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); +lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +x_21 = 0; +x_22 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_21, x_21, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10898,42 +11288,42 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_21; +return x_22; } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_16); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_16, 1); -x_24 = lean_ctor_get(x_16, 0); -lean_dec(x_24); -x_25 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23); -if (lean_obj_tag(x_25) == 0) +uint8_t x_23; +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; -x_26 = lean_ctor_get(x_25, 1); -lean_inc(x_26); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_17, 1); +x_25 = lean_ctor_get(x_17, 0); lean_dec(x_25); +x_26 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_24); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; +x_27 = lean_ctor_get(x_26, 1); +lean_inc(x_27); +lean_dec(x_26); lean_inc(x_1); -x_27 = l_Lean_indentExpr(x_1); -x_28 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -lean_ctor_set_tag(x_16, 7); -lean_ctor_set(x_16, 1, x_27); -lean_ctor_set(x_16, 0, x_28); -x_29 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_16); -lean_ctor_set(x_30, 1, x_29); -x_31 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_15, x_30, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); -x_32 = lean_ctor_get(x_31, 1); -lean_inc(x_32); -lean_dec(x_31); -x_33 = 0; -x_34 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_33, x_33, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_32); +x_28 = l_Lean_indentExpr(x_1); +x_29 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +lean_ctor_set_tag(x_17, 7); +lean_ctor_set(x_17, 1, x_28); +lean_ctor_set(x_17, 0, x_29); +x_30 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_17); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_16, x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_27); +x_33 = lean_ctor_get(x_32, 1); +lean_inc(x_33); +lean_dec(x_32); +x_34 = 0; +x_35 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_34, x_34, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_33); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10941,13 +11331,13 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_34; +return x_35; } else { -uint8_t x_35; -lean_free_object(x_16); +uint8_t x_36; +lean_free_object(x_17); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -10955,58 +11345,58 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_35 = !lean_is_exclusive(x_25); -if (x_35 == 0) +x_36 = !lean_is_exclusive(x_26); +if (x_36 == 0) { -return x_25; +return x_26; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_25, 0); -x_37 = lean_ctor_get(x_25, 1); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_26, 0); +x_38 = lean_ctor_get(x_26, 1); +lean_inc(x_38); lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_25); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_dec(x_26); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_16, 1); -lean_inc(x_39); -lean_dec(x_16); -x_40 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_39); -if (lean_obj_tag(x_40) == 0) +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_17, 1); +lean_inc(x_40); +lean_dec(x_17); +x_41 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_40); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; -x_41 = lean_ctor_get(x_40, 1); -lean_inc(x_41); -lean_dec(x_40); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +x_42 = lean_ctor_get(x_41, 1); +lean_inc(x_42); +lean_dec(x_41); lean_inc(x_1); -x_42 = l_Lean_indentExpr(x_1); -x_43 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -x_44 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -x_45 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_46 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_15, x_46, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_41); -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -x_49 = 0; -x_50 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_49, x_49, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_48); +x_43 = l_Lean_indentExpr(x_1); +x_44 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +x_46 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_47 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +x_48 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_16, x_47, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_42); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = 0; +x_51 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_50, x_50, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_49); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11014,12 +11404,12 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_50; +return x_51; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11027,36 +11417,36 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_51 = lean_ctor_get(x_40, 0); -lean_inc(x_51); -x_52 = lean_ctor_get(x_40, 1); +x_52 = lean_ctor_get(x_41, 0); lean_inc(x_52); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_53 = x_40; +x_53 = lean_ctor_get(x_41, 1); +lean_inc(x_53); +if (lean_is_exclusive(x_41)) { + lean_ctor_release(x_41, 0); + lean_ctor_release(x_41, 1); + x_54 = x_41; } else { - lean_dec_ref(x_40); - x_53 = lean_box(0); + lean_dec_ref(x_41); + x_54 = lean_box(0); } -if (lean_is_scalar(x_53)) { - x_54 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_54)) { + x_55 = lean_alloc_ctor(1, 2, 0); } else { - x_54 = x_53; + x_55 = x_54; } -lean_ctor_set(x_54, 0, x_51); -lean_ctor_set(x_54, 1, x_52); -return x_54; +lean_ctor_set(x_55, 0, x_52); +lean_ctor_set(x_55, 1, x_53); +return x_55; } } } } case 3: { -lean_object* x_55; lean_object* x_56; +lean_object* x_56; lean_object* x_57; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11064,76 +11454,119 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_55 = lean_box(0); -x_56 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_12); -return x_56; +x_56 = lean_box(0); +x_57 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_13); +return x_57; } case 4: { -lean_object* x_57; -x_57 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_58; +lean_dec(x_3); +x_58 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_57; +return x_58; } case 5: { -lean_object* x_58; +lean_object* x_59; +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); lean_inc(x_1); -x_58 = l_Lean_Meta_isLitValue(x_1, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_58) == 0) +x_59 = l_Lean_Meta_isLitValue(x_1, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_59) == 0) { -lean_object* x_59; uint8_t x_60; -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_unbox(x_59); +lean_object* x_60; uint8_t x_61; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_unbox(x_60); +lean_dec(x_60); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_62 = lean_ctor_get(x_59, 1); +lean_inc(x_62); lean_dec(x_59); -if (x_60 == 0) +x_63 = lean_unsigned_to_nat(0u); +x_64 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_63); +x_65 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__1; +lean_inc(x_64); +x_66 = lean_mk_array(x_64, x_65); +x_67 = lean_unsigned_to_nat(1u); +x_68 = lean_nat_sub(x_64, x_67); +lean_dec(x_64); +lean_inc(x_1); +x_69 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2(x_1, x_2, x_3, x_1, x_66, x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_62); +return x_69; +} +else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_61 = lean_ctor_get(x_58, 1); -lean_inc(x_61); -lean_dec(x_58); -x_62 = lean_unsigned_to_nat(0u); -x_63 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_62); -x_64 = l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__1; -lean_inc(x_63); -x_65 = lean_mk_array(x_63, x_64); -x_66 = lean_unsigned_to_nat(1u); -x_67 = lean_nat_sub(x_63, x_66); -lean_dec(x_63); +lean_object* x_70; lean_object* x_71; +x_70 = lean_ctor_get(x_59, 1); +lean_inc(x_70); +lean_dec(x_59); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); lean_inc(x_1); -x_68 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3(x_1, x_2, x_1, x_65, x_67, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_61); -return x_68; +x_71 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_70); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_71, 1); +lean_inc(x_72); +lean_dec(x_71); +x_73 = l_Lean_Meta_Grind_Arith_Offset_internalize(x_1, x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_72); +return x_73; } else { -lean_object* x_69; lean_object* x_70; -x_69 = lean_ctor_get(x_58, 1); -lean_inc(x_69); -lean_dec(x_58); -x_70 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_69); +uint8_t x_74; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_70; +lean_dec(x_3); +lean_dec(x_1); +x_74 = !lean_is_exclusive(x_71); +if (x_74 == 0) +{ +return x_71; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_75 = lean_ctor_get(x_71, 0); +x_76 = lean_ctor_get(x_71, 1); +lean_inc(x_76); +lean_inc(x_75); +lean_dec(x_71); +x_77 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_77, 0, x_75); +lean_ctor_set(x_77, 1, x_76); +return x_77; +} +} } } else { -uint8_t x_71; +uint8_t x_78; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11141,107 +11574,109 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_71 = !lean_is_exclusive(x_58); -if (x_71 == 0) +x_78 = !lean_is_exclusive(x_59); +if (x_78 == 0) { -return x_58; +return x_59; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_58, 0); -x_73 = lean_ctor_get(x_58, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_58); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_59, 0); +x_80 = lean_ctor_get(x_59, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_59); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; } } } case 7: { -lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; uint8_t x_81; lean_object* x_82; lean_object* x_105; -x_75 = lean_ctor_get(x_1, 1); -lean_inc(x_75); -x_76 = lean_ctor_get(x_1, 2); -lean_inc(x_76); -x_77 = 0; +lean_object* x_82; lean_object* x_83; uint8_t x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; lean_object* x_89; lean_object* x_113; +lean_dec(x_3); +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_1, 2); +lean_inc(x_83); +x_84 = 0; lean_inc(x_2); lean_inc(x_1); -x_78 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_77, x_77, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_79 = lean_ctor_get(x_78, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_80 = x_78; +x_85 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_84, x_84, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_86 = lean_ctor_get(x_85, 1); +lean_inc(x_86); +if (lean_is_exclusive(x_85)) { + lean_ctor_release(x_85, 0); + lean_ctor_release(x_85, 1); + x_87 = x_85; } else { - lean_dec_ref(x_78); - x_80 = lean_box(0); + lean_dec_ref(x_85); + x_87 = lean_box(0); } +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_75); -x_105 = l_Lean_Meta_isProp(x_75, x_8, x_9, x_10, x_11, x_79); -if (lean_obj_tag(x_105) == 0) +lean_inc(x_82); +x_113 = l_Lean_Meta_isProp(x_82, x_9, x_10, x_11, x_12, x_86); +if (lean_obj_tag(x_113) == 0) { -lean_object* x_106; uint8_t x_107; -x_106 = lean_ctor_get(x_105, 0); -lean_inc(x_106); -x_107 = lean_unbox(x_106); -if (x_107 == 0) +lean_object* x_114; uint8_t x_115; +x_114 = lean_ctor_get(x_113, 0); +lean_inc(x_114); +x_115 = lean_unbox(x_114); +if (x_115 == 0) { -lean_object* x_108; uint8_t x_109; -x_108 = lean_ctor_get(x_105, 1); -lean_inc(x_108); -lean_dec(x_105); -x_109 = lean_unbox(x_106); -lean_dec(x_106); -x_81 = x_109; -x_82 = x_108; -goto block_104; +lean_object* x_116; uint8_t x_117; +x_116 = lean_ctor_get(x_113, 1); +lean_inc(x_116); +lean_dec(x_113); +x_117 = lean_unbox(x_114); +lean_dec(x_114); +x_88 = x_117; +x_89 = x_116; +goto block_112; } else { -lean_object* x_110; lean_object* x_111; -lean_dec(x_106); -x_110 = lean_ctor_get(x_105, 1); -lean_inc(x_110); -lean_dec(x_105); +lean_object* x_118; lean_object* x_119; +lean_dec(x_114); +x_118 = lean_ctor_get(x_113, 1); +lean_inc(x_118); +lean_dec(x_113); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); -lean_inc(x_8); lean_inc(x_1); -x_111 = l_Lean_Meta_isProp(x_1, x_8, x_9, x_10, x_11, x_110); -if (lean_obj_tag(x_111) == 0) +x_119 = l_Lean_Meta_isProp(x_1, x_9, x_10, x_11, x_12, x_118); +if (lean_obj_tag(x_119) == 0) { -lean_object* x_112; lean_object* x_113; uint8_t x_114; -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -lean_dec(x_111); -x_114 = lean_unbox(x_112); -lean_dec(x_112); -x_81 = x_114; -x_82 = x_113; -goto block_104; +lean_object* x_120; lean_object* x_121; uint8_t x_122; +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_119, 1); +lean_inc(x_121); +lean_dec(x_119); +x_122 = lean_unbox(x_120); +lean_dec(x_120); +x_88 = x_122; +x_89 = x_121; +goto block_112; } else { -uint8_t x_115; -lean_dec(x_80); -lean_dec(x_76); -lean_dec(x_75); +uint8_t x_123; +lean_dec(x_87); +lean_dec(x_83); +lean_dec(x_82); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11249,36 +11684,36 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_115 = !lean_is_exclusive(x_111); -if (x_115 == 0) +x_123 = !lean_is_exclusive(x_119); +if (x_123 == 0) { -return x_111; +return x_119; } else { -lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_116 = lean_ctor_get(x_111, 0); -x_117 = lean_ctor_get(x_111, 1); -lean_inc(x_117); -lean_inc(x_116); -lean_dec(x_111); -x_118 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_118, 0, x_116); -lean_ctor_set(x_118, 1, x_117); -return x_118; +lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_124 = lean_ctor_get(x_119, 0); +x_125 = lean_ctor_get(x_119, 1); +lean_inc(x_125); +lean_inc(x_124); +lean_dec(x_119); +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; } } } } else { -uint8_t x_119; -lean_dec(x_80); -lean_dec(x_76); -lean_dec(x_75); +uint8_t x_127; +lean_dec(x_87); +lean_dec(x_83); +lean_dec(x_82); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11286,35 +11721,35 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_119 = !lean_is_exclusive(x_105); -if (x_119 == 0) +x_127 = !lean_is_exclusive(x_113); +if (x_127 == 0) { -return x_105; +return x_113; } else { -lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_120 = lean_ctor_get(x_105, 0); -x_121 = lean_ctor_get(x_105, 1); -lean_inc(x_121); -lean_inc(x_120); -lean_dec(x_105); -x_122 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_122, 0, x_120); -lean_ctor_set(x_122, 1, x_121); -return x_122; +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_113, 0); +x_129 = lean_ctor_get(x_113, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_113); +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; } } -block_104: +block_112: { -if (x_81 == 0) +if (x_88 == 0) { -lean_object* x_83; lean_object* x_84; -lean_dec(x_76); -lean_dec(x_75); +lean_object* x_90; lean_object* x_91; +lean_dec(x_83); +lean_dec(x_82); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11322,23 +11757,26 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_83 = lean_box(0); -if (lean_is_scalar(x_80)) { - x_84 = lean_alloc_ctor(0, 2, 0); +x_90 = lean_box(0); +if (lean_is_scalar(x_87)) { + x_91 = lean_alloc_ctor(0, 2, 0); } else { - x_84 = x_80; + x_91 = x_87; } -lean_ctor_set(x_84, 0, x_83); -lean_ctor_set(x_84, 1, x_82); -return x_84; +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_89); +return x_91; } else { -lean_object* x_85; -lean_dec(x_80); +lean_object* x_92; lean_object* x_93; +lean_dec(x_87); +lean_inc(x_1); +x_92 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_92, 0, x_1); +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -11346,26 +11784,27 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); +lean_inc(x_92); lean_inc(x_2); -lean_inc(x_75); -x_85 = l_Lean_Meta_Grind_internalize(x_75, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_82); -if (lean_obj_tag(x_85) == 0) +lean_inc(x_82); +x_93 = l_Lean_Meta_Grind_internalize(x_82, x_2, x_92, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_89); +if (lean_obj_tag(x_93) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; -x_86 = lean_ctor_get(x_85, 1); -lean_inc(x_86); -lean_dec(x_85); +lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; +x_94 = lean_ctor_get(x_93, 1); +lean_inc(x_94); +lean_dec(x_93); lean_inc(x_1); -x_87 = l_Lean_Meta_Grind_registerParent(x_1, x_75, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_86); -lean_dec(x_75); -x_88 = lean_ctor_get(x_87, 1); -lean_inc(x_88); -lean_dec(x_87); -x_89 = l_Lean_Expr_hasLooseBVars(x_76); -if (x_89 == 0) +x_95 = l_Lean_Meta_Grind_registerParent(x_1, x_82, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_94); +lean_dec(x_82); +x_96 = lean_ctor_get(x_95, 1); +lean_inc(x_96); +lean_dec(x_95); +x_97 = l_Lean_Expr_hasLooseBVars(x_83); +if (x_97 == 0) { -lean_object* x_90; +lean_object* x_98; +lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -11373,28 +11812,28 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_76); -x_90 = l_Lean_Meta_Grind_internalize(x_76, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_88); -if (lean_obj_tag(x_90) == 0) +lean_inc(x_83); +x_98 = l_Lean_Meta_Grind_internalize(x_83, x_2, x_92, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_96); +if (lean_obj_tag(x_98) == 0) { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_91 = lean_ctor_get(x_90, 1); -lean_inc(x_91); -lean_dec(x_90); +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +x_99 = lean_ctor_get(x_98, 1); +lean_inc(x_99); +lean_dec(x_98); lean_inc(x_1); -x_92 = l_Lean_Meta_Grind_registerParent(x_1, x_76, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_91); -lean_dec(x_76); -x_93 = lean_ctor_get(x_92, 1); -lean_inc(x_93); -lean_dec(x_92); -x_94 = l_Lean_Meta_Grind_propagateUp(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_93); -return x_94; +x_100 = l_Lean_Meta_Grind_registerParent(x_1, x_83, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_99); +lean_dec(x_83); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +lean_dec(x_100); +x_102 = l_Lean_Meta_Grind_propagateUp(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_101); +return x_102; } else { -uint8_t x_95; -lean_dec(x_76); +uint8_t x_103; +lean_dec(x_83); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11402,42 +11841,44 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_1); -x_95 = !lean_is_exclusive(x_90); -if (x_95 == 0) +x_103 = !lean_is_exclusive(x_98); +if (x_103 == 0) { -return x_90; +return x_98; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_90, 0); -x_97 = lean_ctor_get(x_90, 1); -lean_inc(x_97); -lean_inc(x_96); -lean_dec(x_90); -x_98 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_104 = lean_ctor_get(x_98, 0); +x_105 = lean_ctor_get(x_98, 1); +lean_inc(x_105); +lean_inc(x_104); +lean_dec(x_98); +x_106 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_106, 0, x_104); +lean_ctor_set(x_106, 1, x_105); +return x_106; } } } else { -lean_object* x_99; -lean_dec(x_76); +lean_object* x_107; +lean_dec(x_92); +lean_dec(x_83); lean_dec(x_2); -x_99 = l_Lean_Meta_Grind_propagateUp(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_88); -return x_99; +x_107 = l_Lean_Meta_Grind_propagateUp(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_96); +return x_107; } } else { -uint8_t x_100; -lean_dec(x_76); -lean_dec(x_75); +uint8_t x_108; +lean_dec(x_92); +lean_dec(x_83); +lean_dec(x_82); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11445,26 +11886,25 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_100 = !lean_is_exclusive(x_85); -if (x_100 == 0) +x_108 = !lean_is_exclusive(x_93); +if (x_108 == 0) { -return x_85; +return x_93; } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_101 = lean_ctor_get(x_85, 0); -x_102 = lean_ctor_get(x_85, 1); -lean_inc(x_102); -lean_inc(x_101); -lean_dec(x_85); -x_103 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -return x_103; +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_93, 0); +x_110 = lean_ctor_get(x_93, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_93); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +return x_111; } } } @@ -11472,31 +11912,34 @@ return x_103; } case 9: { -lean_object* x_123; -x_123 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_object* x_131; +lean_dec(x_3); +x_131 = l_Lean_Meta_Grind_mkENode(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_123; +return x_131; } case 10: { -lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; -x_124 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_125 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_124, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_126 = lean_ctor_get(x_125, 0); -lean_inc(x_126); -x_127 = lean_unbox(x_126); -lean_dec(x_126); -if (x_127 == 0) +lean_object* x_132; lean_object* x_133; lean_object* x_134; uint8_t x_135; +lean_dec(x_3); +x_132 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_133 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_132, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_134 = lean_ctor_get(x_133, 0); +lean_inc(x_134); +x_135 = lean_unbox(x_134); +lean_dec(x_134); +if (x_135 == 0) { -lean_object* x_128; uint8_t x_129; lean_object* x_130; -x_128 = lean_ctor_get(x_125, 1); -lean_inc(x_128); -lean_dec(x_125); -x_129 = 0; -x_130 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_129, x_129, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_128); +lean_object* x_136; uint8_t x_137; lean_object* x_138; +x_136 = lean_ctor_get(x_133, 1); +lean_inc(x_136); +lean_dec(x_133); +x_137 = 0; +x_138 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_137, x_137, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_136); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11504,42 +11947,42 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_130; +return x_138; } else { -uint8_t x_131; -x_131 = !lean_is_exclusive(x_125); -if (x_131 == 0) +uint8_t x_139; +x_139 = !lean_is_exclusive(x_133); +if (x_139 == 0) { -lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_132 = lean_ctor_get(x_125, 1); -x_133 = lean_ctor_get(x_125, 0); -lean_dec(x_133); -x_134 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_132); -if (lean_obj_tag(x_134) == 0) +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_133, 1); +x_141 = lean_ctor_get(x_133, 0); +lean_dec(x_141); +x_142 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_140); +if (lean_obj_tag(x_142) == 0) { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; uint8_t x_142; lean_object* x_143; -x_135 = lean_ctor_get(x_134, 1); -lean_inc(x_135); -lean_dec(x_134); +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; uint8_t x_150; lean_object* x_151; +x_143 = lean_ctor_get(x_142, 1); +lean_inc(x_143); +lean_dec(x_142); lean_inc(x_1); -x_136 = l_Lean_indentExpr(x_1); -x_137 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -lean_ctor_set_tag(x_125, 7); -lean_ctor_set(x_125, 1, x_136); -lean_ctor_set(x_125, 0, x_137); -x_138 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_139 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_139, 0, x_125); -lean_ctor_set(x_139, 1, x_138); -x_140 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_124, x_139, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_135); -x_141 = lean_ctor_get(x_140, 1); -lean_inc(x_141); -lean_dec(x_140); -x_142 = 0; -x_143 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_142, x_142, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_141); +x_144 = l_Lean_indentExpr(x_1); +x_145 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +lean_ctor_set_tag(x_133, 7); +lean_ctor_set(x_133, 1, x_144); +lean_ctor_set(x_133, 0, x_145); +x_146 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_147 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_147, 0, x_133); +lean_ctor_set(x_147, 1, x_146); +x_148 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_132, x_147, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_143); +x_149 = lean_ctor_get(x_148, 1); +lean_inc(x_149); +lean_dec(x_148); +x_150 = 0; +x_151 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_150, x_150, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_149); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11547,13 +11990,13 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_143; +return x_151; } else { -uint8_t x_144; -lean_free_object(x_125); +uint8_t x_152; +lean_free_object(x_133); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11561,58 +12004,58 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_144 = !lean_is_exclusive(x_134); -if (x_144 == 0) +x_152 = !lean_is_exclusive(x_142); +if (x_152 == 0) { -return x_134; +return x_142; } else { -lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_145 = lean_ctor_get(x_134, 0); -x_146 = lean_ctor_get(x_134, 1); -lean_inc(x_146); -lean_inc(x_145); -lean_dec(x_134); -x_147 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_147, 0, x_145); -lean_ctor_set(x_147, 1, x_146); -return x_147; +lean_object* x_153; lean_object* x_154; lean_object* x_155; +x_153 = lean_ctor_get(x_142, 0); +x_154 = lean_ctor_get(x_142, 1); +lean_inc(x_154); +lean_inc(x_153); +lean_dec(x_142); +x_155 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_155, 0, x_153); +lean_ctor_set(x_155, 1, x_154); +return x_155; } } } else { -lean_object* x_148; lean_object* x_149; -x_148 = lean_ctor_get(x_125, 1); -lean_inc(x_148); -lean_dec(x_125); -x_149 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_148); -if (lean_obj_tag(x_149) == 0) +lean_object* x_156; lean_object* x_157; +x_156 = lean_ctor_get(x_133, 1); +lean_inc(x_156); +lean_dec(x_133); +x_157 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_156); +if (lean_obj_tag(x_157) == 0) { -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; lean_object* x_159; -x_150 = lean_ctor_get(x_149, 1); -lean_inc(x_150); -lean_dec(x_149); +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; uint8_t x_166; lean_object* x_167; +x_158 = lean_ctor_get(x_157, 1); +lean_inc(x_158); +lean_dec(x_157); lean_inc(x_1); -x_151 = l_Lean_indentExpr(x_1); -x_152 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -x_153 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_153, 0, x_152); -lean_ctor_set(x_153, 1, x_151); -x_154 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_155 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_155, 0, x_153); -lean_ctor_set(x_155, 1, x_154); -x_156 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_124, x_155, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_150); -x_157 = lean_ctor_get(x_156, 1); -lean_inc(x_157); -lean_dec(x_156); -x_158 = 0; -x_159 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_158, x_158, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_157); +x_159 = l_Lean_indentExpr(x_1); +x_160 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +x_161 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_161, 0, x_160); +lean_ctor_set(x_161, 1, x_159); +x_162 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_163 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_163, 0, x_161); +lean_ctor_set(x_163, 1, x_162); +x_164 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_132, x_163, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_158); +x_165 = lean_ctor_get(x_164, 1); +lean_inc(x_165); +lean_dec(x_164); +x_166 = 0; +x_167 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_166, x_166, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_165); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11620,12 +12063,12 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_159; +return x_167; } else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11633,50 +12076,51 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_160 = lean_ctor_get(x_149, 0); -lean_inc(x_160); -x_161 = lean_ctor_get(x_149, 1); -lean_inc(x_161); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_162 = x_149; +x_168 = lean_ctor_get(x_157, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_157, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_170 = x_157; } else { - lean_dec_ref(x_149); - x_162 = lean_box(0); + lean_dec_ref(x_157); + x_170 = lean_box(0); } -if (lean_is_scalar(x_162)) { - x_163 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_163 = x_162; + x_171 = x_170; } -lean_ctor_set(x_163, 0, x_160); -lean_ctor_set(x_163, 1, x_161); -return x_163; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } case 11: { -lean_object* x_164; lean_object* x_165; lean_object* x_166; uint8_t x_167; -x_164 = l_Lean_Meta_Grind_addCongrTable___closed__2; -x_165 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_164, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_166 = lean_ctor_get(x_165, 0); -lean_inc(x_166); -x_167 = lean_unbox(x_166); -lean_dec(x_166); -if (x_167 == 0) +lean_object* x_172; lean_object* x_173; lean_object* x_174; uint8_t x_175; +lean_dec(x_3); +x_172 = l_Lean_Meta_Grind_addCongrTable___closed__2; +x_173 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_172, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_174 = lean_ctor_get(x_173, 0); +lean_inc(x_174); +x_175 = lean_unbox(x_174); +lean_dec(x_174); +if (x_175 == 0) { -lean_object* x_168; uint8_t x_169; lean_object* x_170; -x_168 = lean_ctor_get(x_165, 1); -lean_inc(x_168); -lean_dec(x_165); -x_169 = 0; -x_170 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_169, x_169, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_168); +lean_object* x_176; uint8_t x_177; lean_object* x_178; +x_176 = lean_ctor_get(x_173, 1); +lean_inc(x_176); +lean_dec(x_173); +x_177 = 0; +x_178 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_177, x_177, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_176); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11684,42 +12128,42 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_170; +return x_178; } else { -uint8_t x_171; -x_171 = !lean_is_exclusive(x_165); -if (x_171 == 0) +uint8_t x_179; +x_179 = !lean_is_exclusive(x_173); +if (x_179 == 0) { -lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_172 = lean_ctor_get(x_165, 1); -x_173 = lean_ctor_get(x_165, 0); -lean_dec(x_173); -x_174 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_172); -if (lean_obj_tag(x_174) == 0) +lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_180 = lean_ctor_get(x_173, 1); +x_181 = lean_ctor_get(x_173, 0); +lean_dec(x_181); +x_182 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_180); +if (lean_obj_tag(x_182) == 0) { -lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; uint8_t x_182; lean_object* x_183; -x_175 = lean_ctor_get(x_174, 1); -lean_inc(x_175); -lean_dec(x_174); +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; uint8_t x_190; lean_object* x_191; +x_183 = lean_ctor_get(x_182, 1); +lean_inc(x_183); +lean_dec(x_182); lean_inc(x_1); -x_176 = l_Lean_indentExpr(x_1); -x_177 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -lean_ctor_set_tag(x_165, 7); -lean_ctor_set(x_165, 1, x_176); -lean_ctor_set(x_165, 0, x_177); -x_178 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_179 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_179, 0, x_165); -lean_ctor_set(x_179, 1, x_178); -x_180 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_164, x_179, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_175); -x_181 = lean_ctor_get(x_180, 1); -lean_inc(x_181); -lean_dec(x_180); -x_182 = 0; -x_183 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_182, x_182, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_181); +x_184 = l_Lean_indentExpr(x_1); +x_185 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +lean_ctor_set_tag(x_173, 7); +lean_ctor_set(x_173, 1, x_184); +lean_ctor_set(x_173, 0, x_185); +x_186 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_187 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_187, 0, x_173); +lean_ctor_set(x_187, 1, x_186); +x_188 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_172, x_187, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_183); +x_189 = lean_ctor_get(x_188, 1); +lean_inc(x_189); +lean_dec(x_188); +x_190 = 0; +x_191 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_190, x_190, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_189); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11727,13 +12171,13 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_183; +return x_191; } else { -uint8_t x_184; -lean_free_object(x_165); +uint8_t x_192; +lean_free_object(x_173); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11741,58 +12185,58 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_184 = !lean_is_exclusive(x_174); -if (x_184 == 0) +x_192 = !lean_is_exclusive(x_182); +if (x_192 == 0) { -return x_174; +return x_182; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; -x_185 = lean_ctor_get(x_174, 0); -x_186 = lean_ctor_get(x_174, 1); -lean_inc(x_186); -lean_inc(x_185); -lean_dec(x_174); -x_187 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_187, 0, x_185); -lean_ctor_set(x_187, 1, x_186); -return x_187; +lean_object* x_193; lean_object* x_194; lean_object* x_195; +x_193 = lean_ctor_get(x_182, 0); +x_194 = lean_ctor_get(x_182, 1); +lean_inc(x_194); +lean_inc(x_193); +lean_dec(x_182); +x_195 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_195, 0, x_193); +lean_ctor_set(x_195, 1, x_194); +return x_195; } } } else { -lean_object* x_188; lean_object* x_189; -x_188 = lean_ctor_get(x_165, 1); -lean_inc(x_188); -lean_dec(x_165); -x_189 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_188); -if (lean_obj_tag(x_189) == 0) -{ -lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; uint8_t x_198; lean_object* x_199; -x_190 = lean_ctor_get(x_189, 1); -lean_inc(x_190); -lean_dec(x_189); -lean_inc(x_1); -x_191 = l_Lean_indentExpr(x_1); -x_192 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; -x_193 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_193, 0, x_192); -lean_ctor_set(x_193, 1, x_191); -x_194 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_195 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_195, 0, x_193); -lean_ctor_set(x_195, 1, x_194); -x_196 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_164, x_195, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_190); -x_197 = lean_ctor_get(x_196, 1); -lean_inc(x_197); -lean_dec(x_196); -x_198 = 0; -x_199 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_198, x_198, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_197); +lean_object* x_196; lean_object* x_197; +x_196 = lean_ctor_get(x_173, 1); +lean_inc(x_196); +lean_dec(x_173); +x_197 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_196); +if (lean_obj_tag(x_197) == 0) +{ +lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; uint8_t x_206; lean_object* x_207; +x_198 = lean_ctor_get(x_197, 1); +lean_inc(x_198); +lean_dec(x_197); +lean_inc(x_1); +x_199 = l_Lean_indentExpr(x_1); +x_200 = l_Lean_Meta_Grind_internalize___lambda__3___closed__6; +x_201 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_201, 0, x_200); +lean_ctor_set(x_201, 1, x_199); +x_202 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +x_203 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_203, 0, x_201); +lean_ctor_set(x_203, 1, x_202); +x_204 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_172, x_203, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_198); +x_205 = lean_ctor_get(x_204, 1); +lean_inc(x_205); +lean_dec(x_204); +x_206 = 0; +x_207 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_206, x_206, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_205); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11800,12 +12244,12 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_199; +return x_207; } else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; +lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11813,38 +12257,39 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_200 = lean_ctor_get(x_189, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_189, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_189)) { - lean_ctor_release(x_189, 0); - lean_ctor_release(x_189, 1); - x_202 = x_189; +x_208 = lean_ctor_get(x_197, 0); +lean_inc(x_208); +x_209 = lean_ctor_get(x_197, 1); +lean_inc(x_209); +if (lean_is_exclusive(x_197)) { + lean_ctor_release(x_197, 0); + lean_ctor_release(x_197, 1); + x_210 = x_197; } else { - lean_dec_ref(x_189); - x_202 = lean_box(0); + lean_dec_ref(x_197); + x_210 = lean_box(0); } -if (lean_is_scalar(x_202)) { - x_203 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_210)) { + x_211 = lean_alloc_ctor(1, 2, 0); } else { - x_203 = x_202; + x_211 = x_210; } -lean_ctor_set(x_203, 0, x_200); -lean_ctor_set(x_203, 1, x_201); -return x_203; +lean_ctor_set(x_211, 0, x_208); +lean_ctor_set(x_211, 1, x_209); +return x_211; } } } } default: { -uint8_t x_204; lean_object* x_205; -x_204 = 0; -x_205 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_204, x_204, x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +uint8_t x_212; lean_object* x_213; +lean_dec(x_3); +x_212 = 0; +x_213 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_212, x_212, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11852,8 +12297,7 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); -return x_205; +return x_213; } } } @@ -11876,66 +12320,67 @@ x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = l_Lean_Meta_Grind_internalize___lambda__4___closed__2; -x_14 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_unbox(x_15); -lean_dec(x_15); -if (x_16 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_14 = l_Lean_Meta_Grind_internalize___lambda__4___closed__2; +x_15 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = lean_box(0); -x_19 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); -return x_19; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_15, 1); +lean_inc(x_18); +lean_dec(x_15); +x_19 = lean_box(0); +x_20 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_3, x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +return x_20; } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_14); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_14, 1); -x_22 = lean_ctor_get(x_14, 0); -lean_dec(x_22); -x_23 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_21); -if (lean_obj_tag(x_23) == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_15); +if (x_21 == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_ctor_get(x_23, 1); -lean_inc(x_24); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_15, 1); +x_23 = lean_ctor_get(x_15, 0); lean_dec(x_23); +x_24 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); lean_inc(x_1); -x_25 = l_Lean_MessageData_ofExpr(x_1); -x_26 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -lean_ctor_set_tag(x_14, 7); -lean_ctor_set(x_14, 1, x_25); -lean_ctor_set(x_14, 0, x_26); -x_27 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_27, 0, x_14); -lean_ctor_set(x_27, 1, x_26); -x_28 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24); -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); +x_26 = l_Lean_MessageData_ofExpr(x_1); +x_27 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_26); +lean_ctor_set(x_15, 0, x_27); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_15); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); lean_dec(x_29); -return x_31; +x_32 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_3, x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_31); +lean_dec(x_30); +return x_32; } else { -uint8_t x_32; -lean_free_object(x_14); +uint8_t x_33; +lean_free_object(x_15); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -11943,64 +12388,65 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_23); -if (x_32 == 0) +x_33 = !lean_is_exclusive(x_24); +if (x_33 == 0) { -return x_23; +return x_24; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_23, 0); -x_34 = lean_ctor_get(x_23, 1); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_24, 0); +x_35 = lean_ctor_get(x_24, 1); +lean_inc(x_35); lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_23); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_dec(x_24); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } else { -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_14, 1); -lean_inc(x_36); -lean_dec(x_14); -x_37 = l_Lean_Meta_Grind_updateLastTag(x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_36); -if (lean_obj_tag(x_37) == 0) +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_15, 1); +lean_inc(x_37); +lean_dec(x_15); +x_38 = l_Lean_Meta_Grind_updateLastTag(x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_38 = lean_ctor_get(x_37, 1); -lean_inc(x_38); -lean_dec(x_37); +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_39 = lean_ctor_get(x_38, 1); +lean_inc(x_39); +lean_dec(x_38); lean_inc(x_1); -x_39 = l_Lean_MessageData_ofExpr(x_1); -x_40 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; -x_41 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_39); +x_40 = l_Lean_MessageData_ofExpr(x_1); +x_41 = l_Lean_Meta_Grind_addCongrTable___lambda__2___closed__6; x_42 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_42, 0, x_41); lean_ctor_set(x_42, 1, x_40); -x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_13, x_42, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); +x_43 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +x_44 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_43, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); +x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); -lean_dec(x_43); -x_46 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_44, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); lean_dec(x_44); -return x_46; +x_47 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_3, x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_46); +lean_dec(x_45); +return x_47; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -12008,56 +12454,57 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); +lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_47 = lean_ctor_get(x_37, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_37, 1); +x_48 = lean_ctor_get(x_38, 0); lean_inc(x_48); -if (lean_is_exclusive(x_37)) { - lean_ctor_release(x_37, 0); - lean_ctor_release(x_37, 1); - x_49 = x_37; +x_49 = lean_ctor_get(x_38, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_38)) { + lean_ctor_release(x_38, 0); + lean_ctor_release(x_38, 1); + x_50 = x_38; } else { - lean_dec_ref(x_37); - x_49 = lean_box(0); + lean_dec_ref(x_38); + x_50 = lean_box(0); } -if (lean_is_scalar(x_49)) { - x_50 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_50)) { + x_51 = lean_alloc_ctor(1, 2, 0); } else { - x_50 = x_49; + x_51 = x_50; } -lean_ctor_set(x_50, 0, x_47); -lean_ctor_set(x_50, 1, x_48); -return x_50; +lean_ctor_set(x_51, 0, x_48); +lean_ctor_set(x_51, 1, x_49); +return x_51; } } } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = l_Lean_Meta_Grind_alreadyInternalized(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_unbox(x_13); -lean_dec(x_13); -if (x_14 == 0) +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Meta_Grind_alreadyInternalized(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = lean_box(0); -x_17 = l_Lean_Meta_Grind_internalize___lambda__4(x_1, x_2, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -return x_17; +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = lean_box(0); +x_18 = l_Lean_Meta_Grind_internalize___lambda__4(x_1, x_2, x_3, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +return x_18; } else { -uint8_t x_18; +uint8_t x_19; +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -12068,27 +12515,27 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_18 = !lean_is_exclusive(x_12); -if (x_18 == 0) +x_19 = !lean_is_exclusive(x_13); +if (x_19 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_12, 0); -lean_dec(x_19); -x_20 = lean_box(0); -lean_ctor_set(x_12, 0, x_20); -return x_12; +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_13, 0); +lean_dec(x_20); +x_21 = lean_box(0); +lean_ctor_set(x_13, 0, x_21); +return x_13; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_12, 1); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_box(0); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_13, 1); +lean_inc(x_22); +lean_dec(x_13); +x_23 = lean_box(0); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } } } @@ -12300,9 +12747,9 @@ x_15 = !lean_is_exclusive(x_13); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_13, 10); +x_16 = lean_ctor_get(x_13, 12); x_17 = l_Lean_Meta_Grind_EMatchTheorems_insert(x_16, x_1); -lean_ctor_set(x_13, 10, x_17); +lean_ctor_set(x_13, 12, x_17); x_18 = lean_st_ref_set(x_3, x_13, x_14); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) @@ -12329,15 +12776,15 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_25 = lean_ctor_get(x_13, 0); x_26 = lean_ctor_get(x_13, 1); x_27 = lean_ctor_get(x_13, 2); x_28 = lean_ctor_get(x_13, 3); x_29 = lean_ctor_get(x_13, 4); x_30 = lean_ctor_get(x_13, 5); -x_31 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_32 = lean_ctor_get(x_13, 6); +x_31 = lean_ctor_get(x_13, 6); +x_32 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_33 = lean_ctor_get(x_13, 7); x_34 = lean_ctor_get(x_13, 8); x_35 = lean_ctor_get(x_13, 9); @@ -12351,6 +12798,12 @@ x_42 = lean_ctor_get(x_13, 16); x_43 = lean_ctor_get(x_13, 17); x_44 = lean_ctor_get(x_13, 18); x_45 = lean_ctor_get(x_13, 19); +x_46 = lean_ctor_get(x_13, 20); +x_47 = lean_ctor_get(x_13, 21); +x_48 = lean_ctor_get(x_13, 22); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); @@ -12364,7 +12817,7 @@ lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); +lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); @@ -12372,49 +12825,52 @@ lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_dec(x_13); -x_46 = l_Lean_Meta_Grind_EMatchTheorems_insert(x_36, x_1); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_25); -lean_ctor_set(x_47, 1, x_26); -lean_ctor_set(x_47, 2, x_27); -lean_ctor_set(x_47, 3, x_28); -lean_ctor_set(x_47, 4, x_29); -lean_ctor_set(x_47, 5, x_30); -lean_ctor_set(x_47, 6, x_32); -lean_ctor_set(x_47, 7, x_33); -lean_ctor_set(x_47, 8, x_34); -lean_ctor_set(x_47, 9, x_35); -lean_ctor_set(x_47, 10, x_46); -lean_ctor_set(x_47, 11, x_37); -lean_ctor_set(x_47, 12, x_38); -lean_ctor_set(x_47, 13, x_39); -lean_ctor_set(x_47, 14, x_40); -lean_ctor_set(x_47, 15, x_41); -lean_ctor_set(x_47, 16, x_42); -lean_ctor_set(x_47, 17, x_43); -lean_ctor_set(x_47, 18, x_44); -lean_ctor_set(x_47, 19, x_45); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_31); -x_48 = lean_st_ref_set(x_3, x_47, x_14); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_49 = l_Lean_Meta_Grind_EMatchTheorems_insert(x_38, x_1); +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_25); +lean_ctor_set(x_50, 1, x_26); +lean_ctor_set(x_50, 2, x_27); +lean_ctor_set(x_50, 3, x_28); +lean_ctor_set(x_50, 4, x_29); +lean_ctor_set(x_50, 5, x_30); +lean_ctor_set(x_50, 6, x_31); +lean_ctor_set(x_50, 7, x_33); +lean_ctor_set(x_50, 8, x_34); +lean_ctor_set(x_50, 9, x_35); +lean_ctor_set(x_50, 10, x_36); +lean_ctor_set(x_50, 11, x_37); +lean_ctor_set(x_50, 12, x_49); +lean_ctor_set(x_50, 13, x_39); +lean_ctor_set(x_50, 14, x_40); +lean_ctor_set(x_50, 15, x_41); +lean_ctor_set(x_50, 16, x_42); +lean_ctor_set(x_50, 17, x_43); +lean_ctor_set(x_50, 18, x_44); +lean_ctor_set(x_50, 19, x_45); +lean_ctor_set(x_50, 20, x_46); +lean_ctor_set(x_50, 21, x_47); +lean_ctor_set(x_50, 22, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_32); +x_51 = lean_st_ref_set(x_3, x_50, x_14); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -x_51 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___lambda__1___closed__1; -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); +x_54 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5___lambda__1___closed__1; +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_50; + x_55 = x_53; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } } } @@ -12506,7 +12962,7 @@ lean_inc(x_27); x_28 = lean_ctor_get(x_26, 1); lean_inc(x_28); lean_dec(x_26); -x_29 = lean_ctor_get(x_27, 10); +x_29 = lean_ctor_get(x_27, 12); lean_inc(x_29); lean_dec(x_27); x_30 = !lean_is_exclusive(x_19); @@ -13194,7 +13650,7 @@ lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; x_12 = lean_st_ref_get(x_3, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); -x_14 = lean_ctor_get(x_13, 10); +x_14 = lean_ctor_get(x_13, 12); lean_inc(x_14); lean_dec(x_13); x_15 = !lean_is_exclusive(x_12); @@ -13252,9 +13708,9 @@ x_29 = !lean_is_exclusive(x_27); if (x_29 == 0) { lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_30 = lean_ctor_get(x_27, 10); +x_30 = lean_ctor_get(x_27, 12); lean_dec(x_30); -lean_ctor_set(x_27, 10, x_14); +lean_ctor_set(x_27, 12, x_14); x_31 = lean_st_ref_set(x_3, x_27, x_28); x_32 = lean_ctor_get(x_31, 1); lean_inc(x_32); @@ -13265,7 +13721,7 @@ lean_inc(x_34); x_35 = lean_ctor_get(x_33, 1); lean_inc(x_35); lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 4); +x_36 = lean_ctor_get(x_34, 5); lean_inc(x_36); lean_dec(x_34); x_37 = lean_box(0); @@ -13322,20 +13778,20 @@ return x_47; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; x_48 = lean_ctor_get(x_27, 0); x_49 = lean_ctor_get(x_27, 1); x_50 = lean_ctor_get(x_27, 2); x_51 = lean_ctor_get(x_27, 3); x_52 = lean_ctor_get(x_27, 4); x_53 = lean_ctor_get(x_27, 5); -x_54 = lean_ctor_get_uint8(x_27, sizeof(void*)*20); -x_55 = lean_ctor_get(x_27, 6); +x_54 = lean_ctor_get(x_27, 6); +x_55 = lean_ctor_get_uint8(x_27, sizeof(void*)*23); x_56 = lean_ctor_get(x_27, 7); x_57 = lean_ctor_get(x_27, 8); x_58 = lean_ctor_get(x_27, 9); -x_59 = lean_ctor_get(x_27, 11); -x_60 = lean_ctor_get(x_27, 12); +x_59 = lean_ctor_get(x_27, 10); +x_60 = lean_ctor_get(x_27, 11); x_61 = lean_ctor_get(x_27, 13); x_62 = lean_ctor_get(x_27, 14); x_63 = lean_ctor_get(x_27, 15); @@ -13343,6 +13799,12 @@ x_64 = lean_ctor_get(x_27, 16); x_65 = lean_ctor_get(x_27, 17); x_66 = lean_ctor_get(x_27, 18); x_67 = lean_ctor_get(x_27, 19); +x_68 = lean_ctor_get(x_27, 20); +x_69 = lean_ctor_get(x_27, 21); +x_70 = lean_ctor_get(x_27, 22); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); lean_inc(x_67); lean_inc(x_66); lean_inc(x_65); @@ -13355,7 +13817,7 @@ lean_inc(x_59); lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); -lean_inc(x_55); +lean_inc(x_54); lean_inc(x_53); lean_inc(x_52); lean_inc(x_51); @@ -13363,113 +13825,116 @@ lean_inc(x_50); lean_inc(x_49); lean_inc(x_48); lean_dec(x_27); -x_68 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_68, 0, x_48); -lean_ctor_set(x_68, 1, x_49); -lean_ctor_set(x_68, 2, x_50); -lean_ctor_set(x_68, 3, x_51); -lean_ctor_set(x_68, 4, x_52); -lean_ctor_set(x_68, 5, x_53); -lean_ctor_set(x_68, 6, x_55); -lean_ctor_set(x_68, 7, x_56); -lean_ctor_set(x_68, 8, x_57); -lean_ctor_set(x_68, 9, x_58); -lean_ctor_set(x_68, 10, x_14); -lean_ctor_set(x_68, 11, x_59); -lean_ctor_set(x_68, 12, x_60); -lean_ctor_set(x_68, 13, x_61); -lean_ctor_set(x_68, 14, x_62); -lean_ctor_set(x_68, 15, x_63); -lean_ctor_set(x_68, 16, x_64); -lean_ctor_set(x_68, 17, x_65); -lean_ctor_set(x_68, 18, x_66); -lean_ctor_set(x_68, 19, x_67); -lean_ctor_set_uint8(x_68, sizeof(void*)*20, x_54); -x_69 = lean_st_ref_set(x_3, x_68, x_28); -x_70 = lean_ctor_get(x_69, 1); -lean_inc(x_70); -lean_dec(x_69); -x_71 = lean_st_ref_get(x_3, x_70); -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); +x_71 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_71, 0, x_48); +lean_ctor_set(x_71, 1, x_49); +lean_ctor_set(x_71, 2, x_50); +lean_ctor_set(x_71, 3, x_51); +lean_ctor_set(x_71, 4, x_52); +lean_ctor_set(x_71, 5, x_53); +lean_ctor_set(x_71, 6, x_54); +lean_ctor_set(x_71, 7, x_56); +lean_ctor_set(x_71, 8, x_57); +lean_ctor_set(x_71, 9, x_58); +lean_ctor_set(x_71, 10, x_59); +lean_ctor_set(x_71, 11, x_60); +lean_ctor_set(x_71, 12, x_14); +lean_ctor_set(x_71, 13, x_61); +lean_ctor_set(x_71, 14, x_62); +lean_ctor_set(x_71, 15, x_63); +lean_ctor_set(x_71, 16, x_64); +lean_ctor_set(x_71, 17, x_65); +lean_ctor_set(x_71, 18, x_66); +lean_ctor_set(x_71, 19, x_67); +lean_ctor_set(x_71, 20, x_68); +lean_ctor_set(x_71, 21, x_69); +lean_ctor_set(x_71, 22, x_70); +lean_ctor_set_uint8(x_71, sizeof(void*)*23, x_55); +x_72 = lean_st_ref_set(x_3, x_71, x_28); +x_73 = lean_ctor_get(x_72, 1); lean_inc(x_73); -lean_dec(x_71); -x_74 = lean_ctor_get(x_72, 4); -lean_inc(x_74); lean_dec(x_72); -x_75 = lean_box(0); -x_76 = lean_box(0); +x_74 = lean_st_ref_get(x_3, x_73); +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = lean_ctor_get(x_75, 5); +lean_inc(x_77); +lean_dec(x_75); +x_78 = lean_box(0); +x_79 = lean_box(0); lean_inc(x_24); -x_77 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_24, x_74, x_75, x_24, x_24, x_76, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_73); +x_80 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_24, x_77, x_78, x_24, x_24, x_79, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_76); lean_dec(x_24); -if (lean_obj_tag(x_77) == 0) +if (lean_obj_tag(x_80) == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_78 = lean_ctor_get(x_77, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_79 = x_77; +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_80, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_82 = x_80; } else { - lean_dec_ref(x_77); - x_79 = lean_box(0); + lean_dec_ref(x_80); + x_82 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(0, 2, 0); } else { - x_80 = x_79; + x_83 = x_82; } -lean_ctor_set(x_80, 0, x_76); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_83, 0, x_79); +lean_ctor_set(x_83, 1, x_81); +return x_83; } else -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_81 = lean_ctor_get(x_77, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_77, 1); -lean_inc(x_82); -if (lean_is_exclusive(x_77)) { - lean_ctor_release(x_77, 0); - lean_ctor_release(x_77, 1); - x_83 = x_77; +{ +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_84 = lean_ctor_get(x_80, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_80, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + lean_ctor_release(x_80, 1); + x_86 = x_80; } else { - lean_dec_ref(x_77); - x_83 = lean_box(0); + lean_dec_ref(x_80); + x_86 = lean_box(0); } -if (lean_is_scalar(x_83)) { - x_84 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_86)) { + x_87 = lean_alloc_ctor(1, 2, 0); } else { - x_84 = x_83; + x_87 = x_86; } -lean_ctor_set(x_84, 0, x_81); -lean_ctor_set(x_84, 1, x_82); -return x_84; +lean_ctor_set(x_87, 0, x_84); +lean_ctor_set(x_87, 1, x_85); +return x_87; } } } } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_85 = lean_ctor_get(x_14, 0); -x_86 = lean_ctor_get(x_14, 1); -x_87 = lean_ctor_get(x_14, 2); -lean_inc(x_87); -lean_inc(x_86); -lean_inc(x_85); +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_88 = lean_ctor_get(x_14, 0); +x_89 = lean_ctor_get(x_14, 1); +x_90 = lean_ctor_get(x_14, 2); +lean_inc(x_90); +lean_inc(x_89); +lean_inc(x_88); lean_dec(x_14); -lean_inc(x_85); -x_88 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__9(x_85, x_1); -if (lean_obj_tag(x_88) == 0) +lean_inc(x_88); +x_91 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__9(x_88, x_1); +if (lean_obj_tag(x_91) == 0) { -lean_object* x_89; -lean_dec(x_87); -lean_dec(x_86); -lean_dec(x_85); +lean_object* x_92; +lean_dec(x_90); +lean_dec(x_89); +lean_dec(x_88); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -13479,216 +13944,228 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_89 = lean_box(0); -lean_ctor_set(x_12, 0, x_89); +x_92 = lean_box(0); +lean_ctor_set(x_12, 0, x_92); return x_12; } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_free_object(x_12); -x_90 = lean_ctor_get(x_88, 0); -lean_inc(x_90); -lean_dec(x_88); -x_91 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1(x_85, x_1); -x_92 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_86); -lean_ctor_set(x_92, 2, x_87); -x_93 = lean_st_ref_take(x_3, x_16); -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -lean_dec(x_93); -x_96 = lean_ctor_get(x_94, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_94, 1); +x_93 = lean_ctor_get(x_91, 0); +lean_inc(x_93); +lean_dec(x_91); +x_94 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1(x_88, x_1); +x_95 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_95, 0, x_94); +lean_ctor_set(x_95, 1, x_89); +lean_ctor_set(x_95, 2, x_90); +x_96 = lean_st_ref_take(x_3, x_16); +x_97 = lean_ctor_get(x_96, 0); lean_inc(x_97); -x_98 = lean_ctor_get(x_94, 2); +x_98 = lean_ctor_get(x_96, 1); lean_inc(x_98); -x_99 = lean_ctor_get(x_94, 3); +lean_dec(x_96); +x_99 = lean_ctor_get(x_97, 0); lean_inc(x_99); -x_100 = lean_ctor_get(x_94, 4); +x_100 = lean_ctor_get(x_97, 1); lean_inc(x_100); -x_101 = lean_ctor_get(x_94, 5); +x_101 = lean_ctor_get(x_97, 2); lean_inc(x_101); -x_102 = lean_ctor_get_uint8(x_94, sizeof(void*)*20); -x_103 = lean_ctor_get(x_94, 6); +x_102 = lean_ctor_get(x_97, 3); +lean_inc(x_102); +x_103 = lean_ctor_get(x_97, 4); lean_inc(x_103); -x_104 = lean_ctor_get(x_94, 7); +x_104 = lean_ctor_get(x_97, 5); lean_inc(x_104); -x_105 = lean_ctor_get(x_94, 8); +x_105 = lean_ctor_get(x_97, 6); lean_inc(x_105); -x_106 = lean_ctor_get(x_94, 9); -lean_inc(x_106); -x_107 = lean_ctor_get(x_94, 11); +x_106 = lean_ctor_get_uint8(x_97, sizeof(void*)*23); +x_107 = lean_ctor_get(x_97, 7); lean_inc(x_107); -x_108 = lean_ctor_get(x_94, 12); +x_108 = lean_ctor_get(x_97, 8); lean_inc(x_108); -x_109 = lean_ctor_get(x_94, 13); +x_109 = lean_ctor_get(x_97, 9); lean_inc(x_109); -x_110 = lean_ctor_get(x_94, 14); +x_110 = lean_ctor_get(x_97, 10); lean_inc(x_110); -x_111 = lean_ctor_get(x_94, 15); +x_111 = lean_ctor_get(x_97, 11); lean_inc(x_111); -x_112 = lean_ctor_get(x_94, 16); +x_112 = lean_ctor_get(x_97, 13); lean_inc(x_112); -x_113 = lean_ctor_get(x_94, 17); +x_113 = lean_ctor_get(x_97, 14); lean_inc(x_113); -x_114 = lean_ctor_get(x_94, 18); +x_114 = lean_ctor_get(x_97, 15); lean_inc(x_114); -x_115 = lean_ctor_get(x_94, 19); +x_115 = lean_ctor_get(x_97, 16); lean_inc(x_115); -if (lean_is_exclusive(x_94)) { - lean_ctor_release(x_94, 0); - lean_ctor_release(x_94, 1); - lean_ctor_release(x_94, 2); - lean_ctor_release(x_94, 3); - lean_ctor_release(x_94, 4); - lean_ctor_release(x_94, 5); - lean_ctor_release(x_94, 6); - lean_ctor_release(x_94, 7); - lean_ctor_release(x_94, 8); - lean_ctor_release(x_94, 9); - lean_ctor_release(x_94, 10); - lean_ctor_release(x_94, 11); - lean_ctor_release(x_94, 12); - lean_ctor_release(x_94, 13); - lean_ctor_release(x_94, 14); - lean_ctor_release(x_94, 15); - lean_ctor_release(x_94, 16); - lean_ctor_release(x_94, 17); - lean_ctor_release(x_94, 18); - lean_ctor_release(x_94, 19); - x_116 = x_94; +x_116 = lean_ctor_get(x_97, 17); +lean_inc(x_116); +x_117 = lean_ctor_get(x_97, 18); +lean_inc(x_117); +x_118 = lean_ctor_get(x_97, 19); +lean_inc(x_118); +x_119 = lean_ctor_get(x_97, 20); +lean_inc(x_119); +x_120 = lean_ctor_get(x_97, 21); +lean_inc(x_120); +x_121 = lean_ctor_get(x_97, 22); +lean_inc(x_121); +if (lean_is_exclusive(x_97)) { + lean_ctor_release(x_97, 0); + lean_ctor_release(x_97, 1); + lean_ctor_release(x_97, 2); + lean_ctor_release(x_97, 3); + lean_ctor_release(x_97, 4); + lean_ctor_release(x_97, 5); + lean_ctor_release(x_97, 6); + lean_ctor_release(x_97, 7); + lean_ctor_release(x_97, 8); + lean_ctor_release(x_97, 9); + lean_ctor_release(x_97, 10); + lean_ctor_release(x_97, 11); + lean_ctor_release(x_97, 12); + lean_ctor_release(x_97, 13); + lean_ctor_release(x_97, 14); + lean_ctor_release(x_97, 15); + lean_ctor_release(x_97, 16); + lean_ctor_release(x_97, 17); + lean_ctor_release(x_97, 18); + lean_ctor_release(x_97, 19); + lean_ctor_release(x_97, 20); + lean_ctor_release(x_97, 21); + lean_ctor_release(x_97, 22); + x_122 = x_97; } else { - lean_dec_ref(x_94); - x_116 = lean_box(0); + lean_dec_ref(x_97); + x_122 = lean_box(0); } -if (lean_is_scalar(x_116)) { - x_117 = lean_alloc_ctor(0, 20, 1); +if (lean_is_scalar(x_122)) { + x_123 = lean_alloc_ctor(0, 23, 1); } else { - x_117 = x_116; -} -lean_ctor_set(x_117, 0, x_96); -lean_ctor_set(x_117, 1, x_97); -lean_ctor_set(x_117, 2, x_98); -lean_ctor_set(x_117, 3, x_99); -lean_ctor_set(x_117, 4, x_100); -lean_ctor_set(x_117, 5, x_101); -lean_ctor_set(x_117, 6, x_103); -lean_ctor_set(x_117, 7, x_104); -lean_ctor_set(x_117, 8, x_105); -lean_ctor_set(x_117, 9, x_106); -lean_ctor_set(x_117, 10, x_92); -lean_ctor_set(x_117, 11, x_107); -lean_ctor_set(x_117, 12, x_108); -lean_ctor_set(x_117, 13, x_109); -lean_ctor_set(x_117, 14, x_110); -lean_ctor_set(x_117, 15, x_111); -lean_ctor_set(x_117, 16, x_112); -lean_ctor_set(x_117, 17, x_113); -lean_ctor_set(x_117, 18, x_114); -lean_ctor_set(x_117, 19, x_115); -lean_ctor_set_uint8(x_117, sizeof(void*)*20, x_102); -x_118 = lean_st_ref_set(x_3, x_117, x_95); -x_119 = lean_ctor_get(x_118, 1); -lean_inc(x_119); -lean_dec(x_118); -x_120 = lean_st_ref_get(x_3, x_119); -x_121 = lean_ctor_get(x_120, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -lean_dec(x_120); -x_123 = lean_ctor_get(x_121, 4); -lean_inc(x_123); -lean_dec(x_121); -x_124 = lean_box(0); -x_125 = lean_box(0); -lean_inc(x_90); -x_126 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_90, x_123, x_124, x_90, x_90, x_125, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_122); -lean_dec(x_90); -if (lean_obj_tag(x_126) == 0) -{ -lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_127 = lean_ctor_get(x_126, 1); + x_123 = x_122; +} +lean_ctor_set(x_123, 0, x_99); +lean_ctor_set(x_123, 1, x_100); +lean_ctor_set(x_123, 2, x_101); +lean_ctor_set(x_123, 3, x_102); +lean_ctor_set(x_123, 4, x_103); +lean_ctor_set(x_123, 5, x_104); +lean_ctor_set(x_123, 6, x_105); +lean_ctor_set(x_123, 7, x_107); +lean_ctor_set(x_123, 8, x_108); +lean_ctor_set(x_123, 9, x_109); +lean_ctor_set(x_123, 10, x_110); +lean_ctor_set(x_123, 11, x_111); +lean_ctor_set(x_123, 12, x_95); +lean_ctor_set(x_123, 13, x_112); +lean_ctor_set(x_123, 14, x_113); +lean_ctor_set(x_123, 15, x_114); +lean_ctor_set(x_123, 16, x_115); +lean_ctor_set(x_123, 17, x_116); +lean_ctor_set(x_123, 18, x_117); +lean_ctor_set(x_123, 19, x_118); +lean_ctor_set(x_123, 20, x_119); +lean_ctor_set(x_123, 21, x_120); +lean_ctor_set(x_123, 22, x_121); +lean_ctor_set_uint8(x_123, sizeof(void*)*23, x_106); +x_124 = lean_st_ref_set(x_3, x_123, x_98); +x_125 = lean_ctor_get(x_124, 1); +lean_inc(x_125); +lean_dec(x_124); +x_126 = lean_st_ref_get(x_3, x_125); +x_127 = lean_ctor_get(x_126, 0); lean_inc(x_127); -if (lean_is_exclusive(x_126)) { - lean_ctor_release(x_126, 0); - lean_ctor_release(x_126, 1); - x_128 = x_126; +x_128 = lean_ctor_get(x_126, 1); +lean_inc(x_128); +lean_dec(x_126); +x_129 = lean_ctor_get(x_127, 5); +lean_inc(x_129); +lean_dec(x_127); +x_130 = lean_box(0); +x_131 = lean_box(0); +lean_inc(x_93); +x_132 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_93, x_129, x_130, x_93, x_93, x_131, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_128); +lean_dec(x_93); +if (lean_obj_tag(x_132) == 0) +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_133 = lean_ctor_get(x_132, 1); +lean_inc(x_133); +if (lean_is_exclusive(x_132)) { + lean_ctor_release(x_132, 0); + lean_ctor_release(x_132, 1); + x_134 = x_132; } else { - lean_dec_ref(x_126); - x_128 = lean_box(0); + lean_dec_ref(x_132); + x_134 = lean_box(0); } -if (lean_is_scalar(x_128)) { - x_129 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_134)) { + x_135 = lean_alloc_ctor(0, 2, 0); } else { - x_129 = x_128; + x_135 = x_134; } -lean_ctor_set(x_129, 0, x_125); -lean_ctor_set(x_129, 1, x_127); -return x_129; +lean_ctor_set(x_135, 0, x_131); +lean_ctor_set(x_135, 1, x_133); +return x_135; } else { -lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_130 = lean_ctor_get(x_126, 0); -lean_inc(x_130); -x_131 = lean_ctor_get(x_126, 1); -lean_inc(x_131); -if (lean_is_exclusive(x_126)) { - lean_ctor_release(x_126, 0); - lean_ctor_release(x_126, 1); - x_132 = x_126; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_136 = lean_ctor_get(x_132, 0); +lean_inc(x_136); +x_137 = lean_ctor_get(x_132, 1); +lean_inc(x_137); +if (lean_is_exclusive(x_132)) { + lean_ctor_release(x_132, 0); + lean_ctor_release(x_132, 1); + x_138 = x_132; } else { - lean_dec_ref(x_126); - x_132 = lean_box(0); + lean_dec_ref(x_132); + x_138 = lean_box(0); } -if (lean_is_scalar(x_132)) { - x_133 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_138)) { + x_139 = lean_alloc_ctor(1, 2, 0); } else { - x_133 = x_132; + x_139 = x_138; } -lean_ctor_set(x_133, 0, x_130); -lean_ctor_set(x_133, 1, x_131); -return x_133; +lean_ctor_set(x_139, 0, x_136); +lean_ctor_set(x_139, 1, x_137); +return x_139; } } } } else { -lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_134 = lean_ctor_get(x_12, 1); -lean_inc(x_134); +lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_140 = lean_ctor_get(x_12, 1); +lean_inc(x_140); lean_dec(x_12); -x_135 = lean_ctor_get(x_14, 0); -lean_inc(x_135); -x_136 = lean_ctor_get(x_14, 1); -lean_inc(x_136); -x_137 = lean_ctor_get(x_14, 2); -lean_inc(x_137); +x_141 = lean_ctor_get(x_14, 0); +lean_inc(x_141); +x_142 = lean_ctor_get(x_14, 1); +lean_inc(x_142); +x_143 = lean_ctor_get(x_14, 2); +lean_inc(x_143); if (lean_is_exclusive(x_14)) { lean_ctor_release(x_14, 0); lean_ctor_release(x_14, 1); lean_ctor_release(x_14, 2); - x_138 = x_14; + x_144 = x_14; } else { lean_dec_ref(x_14); - x_138 = lean_box(0); + x_144 = lean_box(0); } -lean_inc(x_135); -x_139 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__9(x_135, x_1); -if (lean_obj_tag(x_139) == 0) +lean_inc(x_141); +x_145 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_EMatchTheorems_insert___spec__9(x_141, x_1); +if (lean_obj_tag(x_145) == 0) { -lean_object* x_140; lean_object* x_141; -lean_dec(x_138); -lean_dec(x_137); -lean_dec(x_136); -lean_dec(x_135); +lean_object* x_146; lean_object* x_147; +lean_dec(x_144); +lean_dec(x_143); +lean_dec(x_142); +lean_dec(x_141); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -13698,187 +14175,199 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_140 = lean_box(0); -x_141 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_141, 0, x_140); -lean_ctor_set(x_141, 1, x_134); -return x_141; +x_146 = lean_box(0); +x_147 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_140); +return x_147; } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; -x_142 = lean_ctor_get(x_139, 0); -lean_inc(x_142); -lean_dec(x_139); -x_143 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1(x_135, x_1); -if (lean_is_scalar(x_138)) { - x_144 = lean_alloc_ctor(0, 3, 0); +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; uint8_t x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; +x_148 = lean_ctor_get(x_145, 0); +lean_inc(x_148); +lean_dec(x_145); +x_149 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_EMatchTheorems_retrieve_x3f___spec__1(x_141, x_1); +if (lean_is_scalar(x_144)) { + x_150 = lean_alloc_ctor(0, 3, 0); } else { - x_144 = x_138; + x_150 = x_144; } -lean_ctor_set(x_144, 0, x_143); -lean_ctor_set(x_144, 1, x_136); -lean_ctor_set(x_144, 2, x_137); -x_145 = lean_st_ref_take(x_3, x_134); -x_146 = lean_ctor_get(x_145, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_145, 1); -lean_inc(x_147); -lean_dec(x_145); -x_148 = lean_ctor_get(x_146, 0); -lean_inc(x_148); -x_149 = lean_ctor_get(x_146, 1); -lean_inc(x_149); -x_150 = lean_ctor_get(x_146, 2); -lean_inc(x_150); -x_151 = lean_ctor_get(x_146, 3); -lean_inc(x_151); -x_152 = lean_ctor_get(x_146, 4); +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_142); +lean_ctor_set(x_150, 2, x_143); +x_151 = lean_st_ref_take(x_3, x_140); +x_152 = lean_ctor_get(x_151, 0); lean_inc(x_152); -x_153 = lean_ctor_get(x_146, 5); +x_153 = lean_ctor_get(x_151, 1); lean_inc(x_153); -x_154 = lean_ctor_get_uint8(x_146, sizeof(void*)*20); -x_155 = lean_ctor_get(x_146, 6); +lean_dec(x_151); +x_154 = lean_ctor_get(x_152, 0); +lean_inc(x_154); +x_155 = lean_ctor_get(x_152, 1); lean_inc(x_155); -x_156 = lean_ctor_get(x_146, 7); +x_156 = lean_ctor_get(x_152, 2); lean_inc(x_156); -x_157 = lean_ctor_get(x_146, 8); +x_157 = lean_ctor_get(x_152, 3); lean_inc(x_157); -x_158 = lean_ctor_get(x_146, 9); +x_158 = lean_ctor_get(x_152, 4); lean_inc(x_158); -x_159 = lean_ctor_get(x_146, 11); +x_159 = lean_ctor_get(x_152, 5); lean_inc(x_159); -x_160 = lean_ctor_get(x_146, 12); +x_160 = lean_ctor_get(x_152, 6); lean_inc(x_160); -x_161 = lean_ctor_get(x_146, 13); -lean_inc(x_161); -x_162 = lean_ctor_get(x_146, 14); +x_161 = lean_ctor_get_uint8(x_152, sizeof(void*)*23); +x_162 = lean_ctor_get(x_152, 7); lean_inc(x_162); -x_163 = lean_ctor_get(x_146, 15); +x_163 = lean_ctor_get(x_152, 8); lean_inc(x_163); -x_164 = lean_ctor_get(x_146, 16); +x_164 = lean_ctor_get(x_152, 9); lean_inc(x_164); -x_165 = lean_ctor_get(x_146, 17); +x_165 = lean_ctor_get(x_152, 10); lean_inc(x_165); -x_166 = lean_ctor_get(x_146, 18); +x_166 = lean_ctor_get(x_152, 11); lean_inc(x_166); -x_167 = lean_ctor_get(x_146, 19); +x_167 = lean_ctor_get(x_152, 13); lean_inc(x_167); -if (lean_is_exclusive(x_146)) { - lean_ctor_release(x_146, 0); - lean_ctor_release(x_146, 1); - lean_ctor_release(x_146, 2); - lean_ctor_release(x_146, 3); - lean_ctor_release(x_146, 4); - lean_ctor_release(x_146, 5); - lean_ctor_release(x_146, 6); - lean_ctor_release(x_146, 7); - lean_ctor_release(x_146, 8); - lean_ctor_release(x_146, 9); - lean_ctor_release(x_146, 10); - lean_ctor_release(x_146, 11); - lean_ctor_release(x_146, 12); - lean_ctor_release(x_146, 13); - lean_ctor_release(x_146, 14); - lean_ctor_release(x_146, 15); - lean_ctor_release(x_146, 16); - lean_ctor_release(x_146, 17); - lean_ctor_release(x_146, 18); - lean_ctor_release(x_146, 19); - x_168 = x_146; -} else { - lean_dec_ref(x_146); - x_168 = lean_box(0); -} -if (lean_is_scalar(x_168)) { - x_169 = lean_alloc_ctor(0, 20, 1); -} else { - x_169 = x_168; -} -lean_ctor_set(x_169, 0, x_148); -lean_ctor_set(x_169, 1, x_149); -lean_ctor_set(x_169, 2, x_150); -lean_ctor_set(x_169, 3, x_151); -lean_ctor_set(x_169, 4, x_152); -lean_ctor_set(x_169, 5, x_153); -lean_ctor_set(x_169, 6, x_155); -lean_ctor_set(x_169, 7, x_156); -lean_ctor_set(x_169, 8, x_157); -lean_ctor_set(x_169, 9, x_158); -lean_ctor_set(x_169, 10, x_144); -lean_ctor_set(x_169, 11, x_159); -lean_ctor_set(x_169, 12, x_160); -lean_ctor_set(x_169, 13, x_161); -lean_ctor_set(x_169, 14, x_162); -lean_ctor_set(x_169, 15, x_163); -lean_ctor_set(x_169, 16, x_164); -lean_ctor_set(x_169, 17, x_165); -lean_ctor_set(x_169, 18, x_166); -lean_ctor_set(x_169, 19, x_167); -lean_ctor_set_uint8(x_169, sizeof(void*)*20, x_154); -x_170 = lean_st_ref_set(x_3, x_169, x_147); -x_171 = lean_ctor_get(x_170, 1); +x_168 = lean_ctor_get(x_152, 14); +lean_inc(x_168); +x_169 = lean_ctor_get(x_152, 15); +lean_inc(x_169); +x_170 = lean_ctor_get(x_152, 16); +lean_inc(x_170); +x_171 = lean_ctor_get(x_152, 17); lean_inc(x_171); -lean_dec(x_170); -x_172 = lean_st_ref_get(x_3, x_171); -x_173 = lean_ctor_get(x_172, 0); +x_172 = lean_ctor_get(x_152, 18); +lean_inc(x_172); +x_173 = lean_ctor_get(x_152, 19); lean_inc(x_173); -x_174 = lean_ctor_get(x_172, 1); +x_174 = lean_ctor_get(x_152, 20); lean_inc(x_174); -lean_dec(x_172); -x_175 = lean_ctor_get(x_173, 4); +x_175 = lean_ctor_get(x_152, 21); lean_inc(x_175); -lean_dec(x_173); -x_176 = lean_box(0); -x_177 = lean_box(0); -lean_inc(x_142); -x_178 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_142, x_175, x_176, x_142, x_142, x_177, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_174); -lean_dec(x_142); -if (lean_obj_tag(x_178) == 0) +x_176 = lean_ctor_get(x_152, 22); +lean_inc(x_176); +if (lean_is_exclusive(x_152)) { + lean_ctor_release(x_152, 0); + lean_ctor_release(x_152, 1); + lean_ctor_release(x_152, 2); + lean_ctor_release(x_152, 3); + lean_ctor_release(x_152, 4); + lean_ctor_release(x_152, 5); + lean_ctor_release(x_152, 6); + lean_ctor_release(x_152, 7); + lean_ctor_release(x_152, 8); + lean_ctor_release(x_152, 9); + lean_ctor_release(x_152, 10); + lean_ctor_release(x_152, 11); + lean_ctor_release(x_152, 12); + lean_ctor_release(x_152, 13); + lean_ctor_release(x_152, 14); + lean_ctor_release(x_152, 15); + lean_ctor_release(x_152, 16); + lean_ctor_release(x_152, 17); + lean_ctor_release(x_152, 18); + lean_ctor_release(x_152, 19); + lean_ctor_release(x_152, 20); + lean_ctor_release(x_152, 21); + lean_ctor_release(x_152, 22); + x_177 = x_152; +} else { + lean_dec_ref(x_152); + x_177 = lean_box(0); +} +if (lean_is_scalar(x_177)) { + x_178 = lean_alloc_ctor(0, 23, 1); +} else { + x_178 = x_177; +} +lean_ctor_set(x_178, 0, x_154); +lean_ctor_set(x_178, 1, x_155); +lean_ctor_set(x_178, 2, x_156); +lean_ctor_set(x_178, 3, x_157); +lean_ctor_set(x_178, 4, x_158); +lean_ctor_set(x_178, 5, x_159); +lean_ctor_set(x_178, 6, x_160); +lean_ctor_set(x_178, 7, x_162); +lean_ctor_set(x_178, 8, x_163); +lean_ctor_set(x_178, 9, x_164); +lean_ctor_set(x_178, 10, x_165); +lean_ctor_set(x_178, 11, x_166); +lean_ctor_set(x_178, 12, x_150); +lean_ctor_set(x_178, 13, x_167); +lean_ctor_set(x_178, 14, x_168); +lean_ctor_set(x_178, 15, x_169); +lean_ctor_set(x_178, 16, x_170); +lean_ctor_set(x_178, 17, x_171); +lean_ctor_set(x_178, 18, x_172); +lean_ctor_set(x_178, 19, x_173); +lean_ctor_set(x_178, 20, x_174); +lean_ctor_set(x_178, 21, x_175); +lean_ctor_set(x_178, 22, x_176); +lean_ctor_set_uint8(x_178, sizeof(void*)*23, x_161); +x_179 = lean_st_ref_set(x_3, x_178, x_153); +x_180 = lean_ctor_get(x_179, 1); +lean_inc(x_180); +lean_dec(x_179); +x_181 = lean_st_ref_get(x_3, x_180); +x_182 = lean_ctor_get(x_181, 0); +lean_inc(x_182); +x_183 = lean_ctor_get(x_181, 1); +lean_inc(x_183); +lean_dec(x_181); +x_184 = lean_ctor_get(x_182, 5); +lean_inc(x_184); +lean_dec(x_182); +x_185 = lean_box(0); +x_186 = lean_box(0); +lean_inc(x_148); +x_187 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__5(x_2, x_148, x_184, x_185, x_148, x_148, x_186, lean_box(0), x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_183); +lean_dec(x_148); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_179; lean_object* x_180; lean_object* x_181; -x_179 = lean_ctor_get(x_178, 1); -lean_inc(x_179); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_180 = x_178; +lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_188 = lean_ctor_get(x_187, 1); +lean_inc(x_188); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_189 = x_187; } else { - lean_dec_ref(x_178); - x_180 = lean_box(0); + lean_dec_ref(x_187); + x_189 = lean_box(0); } -if (lean_is_scalar(x_180)) { - x_181 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_189)) { + x_190 = lean_alloc_ctor(0, 2, 0); } else { - x_181 = x_180; + x_190 = x_189; } -lean_ctor_set(x_181, 0, x_177); -lean_ctor_set(x_181, 1, x_179); -return x_181; +lean_ctor_set(x_190, 0, x_186); +lean_ctor_set(x_190, 1, x_188); +return x_190; } else { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_182 = lean_ctor_get(x_178, 0); -lean_inc(x_182); -x_183 = lean_ctor_get(x_178, 1); -lean_inc(x_183); -if (lean_is_exclusive(x_178)) { - lean_ctor_release(x_178, 0); - lean_ctor_release(x_178, 1); - x_184 = x_178; +lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; +x_191 = lean_ctor_get(x_187, 0); +lean_inc(x_191); +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_193 = x_187; } else { - lean_dec_ref(x_178); - x_184 = lean_box(0); + lean_dec_ref(x_187); + x_193 = lean_box(0); } -if (lean_is_scalar(x_184)) { - x_185 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_193)) { + x_194 = lean_alloc_ctor(1, 2, 0); } else { - x_185 = x_184; + x_194 = x_193; } -lean_ctor_set(x_185, 0, x_182); -lean_ctor_set(x_185, 1, x_183); -return x_185; +lean_ctor_set(x_194, 0, x_191); +lean_ctor_set(x_194, 1, x_192); +return x_194; } } } @@ -14066,9 +14555,9 @@ x_15 = !lean_is_exclusive(x_13); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_13, 9); +x_16 = lean_ctor_get(x_13, 11); x_17 = l_Lean_PersistentArray_push___rarg(x_16, x_1); -lean_ctor_set(x_13, 9, x_17); +lean_ctor_set(x_13, 11, x_17); x_18 = lean_st_ref_set(x_3, x_13, x_14); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) @@ -14095,15 +14584,15 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_25 = lean_ctor_get(x_13, 0); x_26 = lean_ctor_get(x_13, 1); x_27 = lean_ctor_get(x_13, 2); x_28 = lean_ctor_get(x_13, 3); x_29 = lean_ctor_get(x_13, 4); x_30 = lean_ctor_get(x_13, 5); -x_31 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_32 = lean_ctor_get(x_13, 6); +x_31 = lean_ctor_get(x_13, 6); +x_32 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_33 = lean_ctor_get(x_13, 7); x_34 = lean_ctor_get(x_13, 8); x_35 = lean_ctor_get(x_13, 9); @@ -14117,6 +14606,12 @@ x_42 = lean_ctor_get(x_13, 16); x_43 = lean_ctor_get(x_13, 17); x_44 = lean_ctor_get(x_13, 18); x_45 = lean_ctor_get(x_13, 19); +x_46 = lean_ctor_get(x_13, 20); +x_47 = lean_ctor_get(x_13, 21); +x_48 = lean_ctor_get(x_13, 22); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); @@ -14130,7 +14625,7 @@ lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); +lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); @@ -14138,49 +14633,52 @@ lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_dec(x_13); -x_46 = l_Lean_PersistentArray_push___rarg(x_35, x_1); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_25); -lean_ctor_set(x_47, 1, x_26); -lean_ctor_set(x_47, 2, x_27); -lean_ctor_set(x_47, 3, x_28); -lean_ctor_set(x_47, 4, x_29); -lean_ctor_set(x_47, 5, x_30); -lean_ctor_set(x_47, 6, x_32); -lean_ctor_set(x_47, 7, x_33); -lean_ctor_set(x_47, 8, x_34); -lean_ctor_set(x_47, 9, x_46); -lean_ctor_set(x_47, 10, x_36); -lean_ctor_set(x_47, 11, x_37); -lean_ctor_set(x_47, 12, x_38); -lean_ctor_set(x_47, 13, x_39); -lean_ctor_set(x_47, 14, x_40); -lean_ctor_set(x_47, 15, x_41); -lean_ctor_set(x_47, 16, x_42); -lean_ctor_set(x_47, 17, x_43); -lean_ctor_set(x_47, 18, x_44); -lean_ctor_set(x_47, 19, x_45); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_31); -x_48 = lean_st_ref_set(x_3, x_47, x_14); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_49 = l_Lean_PersistentArray_push___rarg(x_37, x_1); +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_25); +lean_ctor_set(x_50, 1, x_26); +lean_ctor_set(x_50, 2, x_27); +lean_ctor_set(x_50, 3, x_28); +lean_ctor_set(x_50, 4, x_29); +lean_ctor_set(x_50, 5, x_30); +lean_ctor_set(x_50, 6, x_31); +lean_ctor_set(x_50, 7, x_33); +lean_ctor_set(x_50, 8, x_34); +lean_ctor_set(x_50, 9, x_35); +lean_ctor_set(x_50, 10, x_36); +lean_ctor_set(x_50, 11, x_49); +lean_ctor_set(x_50, 12, x_38); +lean_ctor_set(x_50, 13, x_39); +lean_ctor_set(x_50, 14, x_40); +lean_ctor_set(x_50, 15, x_41); +lean_ctor_set(x_50, 16, x_42); +lean_ctor_set(x_50, 17, x_43); +lean_ctor_set(x_50, 18, x_44); +lean_ctor_set(x_50, 19, x_45); +lean_ctor_set(x_50, 20, x_46); +lean_ctor_set(x_50, 21, x_47); +lean_ctor_set(x_50, 22, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_32); +x_51 = lean_st_ref_set(x_3, x_50, x_14); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -x_51 = lean_box(0); -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); +x_54 = lean_box(0); +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_50; + x_55 = x_53; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } } } @@ -15112,7 +15610,7 @@ return x_38; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; x_13 = lean_st_ref_take(x_4, x_12); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); @@ -15131,9 +15629,9 @@ x_20 = lean_ctor_get(x_14, 4); lean_inc(x_20); x_21 = lean_ctor_get(x_14, 5); lean_inc(x_21); -x_22 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); -x_23 = lean_ctor_get(x_14, 6); -lean_inc(x_23); +x_22 = lean_ctor_get(x_14, 6); +lean_inc(x_22); +x_23 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); x_24 = lean_ctor_get(x_14, 7); lean_inc(x_24); x_25 = lean_ctor_get(x_14, 8); @@ -15152,115 +15650,124 @@ x_31 = lean_ctor_get(x_14, 14); lean_inc(x_31); x_32 = lean_ctor_get(x_14, 15); lean_inc(x_32); -x_33 = lean_box(0); +x_33 = lean_ctor_get(x_14, 16); +lean_inc(x_33); +x_34 = lean_ctor_get(x_14, 17); +lean_inc(x_34); +x_35 = lean_box(0); lean_inc(x_1); -x_34 = l_Lean_PersistentHashMap_insert___at_Lean_NameSSet_insert___spec__2(x_32, x_1, x_33); -x_35 = lean_ctor_get(x_14, 16); -lean_inc(x_35); -x_36 = lean_ctor_get(x_14, 17); -lean_inc(x_36); +x_36 = l_Lean_PersistentHashMap_insert___at_Lean_NameSSet_insert___spec__2(x_34, x_1, x_35); x_37 = lean_ctor_get(x_14, 18); lean_inc(x_37); x_38 = lean_ctor_get(x_14, 19); lean_inc(x_38); -lean_dec(x_14); -x_39 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_39, 0, x_16); -lean_ctor_set(x_39, 1, x_17); -lean_ctor_set(x_39, 2, x_18); -lean_ctor_set(x_39, 3, x_19); -lean_ctor_set(x_39, 4, x_20); -lean_ctor_set(x_39, 5, x_21); -lean_ctor_set(x_39, 6, x_23); -lean_ctor_set(x_39, 7, x_24); -lean_ctor_set(x_39, 8, x_25); -lean_ctor_set(x_39, 9, x_26); -lean_ctor_set(x_39, 10, x_27); -lean_ctor_set(x_39, 11, x_28); -lean_ctor_set(x_39, 12, x_29); -lean_ctor_set(x_39, 13, x_30); -lean_ctor_set(x_39, 14, x_31); -lean_ctor_set(x_39, 15, x_34); -lean_ctor_set(x_39, 16, x_35); -lean_ctor_set(x_39, 17, x_36); -lean_ctor_set(x_39, 18, x_37); -lean_ctor_set(x_39, 19, x_38); -lean_ctor_set_uint8(x_39, sizeof(void*)*20, x_22); -x_40 = lean_st_ref_set(x_4, x_39, x_15); -x_41 = lean_ctor_get(x_40, 1); +x_39 = lean_ctor_get(x_14, 20); +lean_inc(x_39); +x_40 = lean_ctor_get(x_14, 21); +lean_inc(x_40); +x_41 = lean_ctor_get(x_14, 22); lean_inc(x_41); -lean_dec(x_40); +lean_dec(x_14); +x_42 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_42, 0, x_16); +lean_ctor_set(x_42, 1, x_17); +lean_ctor_set(x_42, 2, x_18); +lean_ctor_set(x_42, 3, x_19); +lean_ctor_set(x_42, 4, x_20); +lean_ctor_set(x_42, 5, x_21); +lean_ctor_set(x_42, 6, x_22); +lean_ctor_set(x_42, 7, x_24); +lean_ctor_set(x_42, 8, x_25); +lean_ctor_set(x_42, 9, x_26); +lean_ctor_set(x_42, 10, x_27); +lean_ctor_set(x_42, 11, x_28); +lean_ctor_set(x_42, 12, x_29); +lean_ctor_set(x_42, 13, x_30); +lean_ctor_set(x_42, 14, x_31); +lean_ctor_set(x_42, 15, x_32); +lean_ctor_set(x_42, 16, x_33); +lean_ctor_set(x_42, 17, x_36); +lean_ctor_set(x_42, 18, x_37); +lean_ctor_set(x_42, 19, x_38); +lean_ctor_set(x_42, 20, x_39); +lean_ctor_set(x_42, 21, x_40); +lean_ctor_set(x_42, 22, x_41); +lean_ctor_set_uint8(x_42, sizeof(void*)*23, x_23); +x_43 = lean_st_ref_set(x_4, x_42, x_15); +x_44 = lean_ctor_get(x_43, 1); +lean_inc(x_44); +lean_dec(x_43); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_42 = lean_get_match_equations_for(x_1, x_8, x_9, x_10, x_11, x_41); -if (lean_obj_tag(x_42) == 0) +x_45 = lean_get_match_equations_for(x_1, x_8, x_9, x_10, x_11, x_44); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; size_t x_47; size_t x_48; lean_object* x_49; -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_ctor_get(x_43, 0); -lean_inc(x_45); -lean_dec(x_43); -x_46 = lean_box(0); -x_47 = lean_array_size(x_45); -x_48 = 0; -x_49 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___spec__2(x_2, x_45, x_46, x_45, x_47, x_48, x_33, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_44); +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; size_t x_50; size_t x_51; lean_object* x_52; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); lean_dec(x_45); -if (lean_obj_tag(x_49) == 0) +x_48 = lean_ctor_get(x_46, 0); +lean_inc(x_48); +lean_dec(x_46); +x_49 = lean_box(0); +x_50 = lean_array_size(x_48); +x_51 = 0; +x_52 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_addMatchEqns___spec__2(x_2, x_48, x_49, x_48, x_50, x_51, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +lean_dec(x_48); +if (lean_obj_tag(x_52) == 0) { -uint8_t x_50; -x_50 = !lean_is_exclusive(x_49); -if (x_50 == 0) +uint8_t x_53; +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) { -lean_object* x_51; -x_51 = lean_ctor_get(x_49, 0); -lean_dec(x_51); -lean_ctor_set(x_49, 0, x_33); -return x_49; +lean_object* x_54; +x_54 = lean_ctor_get(x_52, 0); +lean_dec(x_54); +lean_ctor_set(x_52, 0, x_35); +return x_52; } else { -lean_object* x_52; lean_object* x_53; -x_52 = lean_ctor_get(x_49, 1); -lean_inc(x_52); -lean_dec(x_49); -x_53 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_53, 0, x_33); -lean_ctor_set(x_53, 1, x_52); -return x_53; +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_52, 1); +lean_inc(x_55); +lean_dec(x_52); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_35); +lean_ctor_set(x_56, 1, x_55); +return x_56; } } else { -uint8_t x_54; -x_54 = !lean_is_exclusive(x_49); -if (x_54 == 0) +uint8_t x_57; +x_57 = !lean_is_exclusive(x_52); +if (x_57 == 0) { -return x_49; +return x_52; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_49, 0); -x_56 = lean_ctor_get(x_49, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_49); -x_57 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_57, 0, x_55); -lean_ctor_set(x_57, 1, x_56); -return x_57; +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_52, 0); +x_59 = lean_ctor_get(x_52, 1); +lean_inc(x_59); +lean_inc(x_58); +lean_dec(x_52); +x_60 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_60, 0, x_58); +lean_ctor_set(x_60, 1, x_59); +return x_60; } } } else { -uint8_t x_58; +uint8_t x_61; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -15270,23 +15777,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_58 = !lean_is_exclusive(x_42); -if (x_58 == 0) +x_61 = !lean_is_exclusive(x_45); +if (x_61 == 0) { -return x_42; +return x_45; } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_42, 0); -x_60 = lean_ctor_get(x_42, 1); -lean_inc(x_60); -lean_inc(x_59); -lean_dec(x_42); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_61, 1, x_60); -return x_61; +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_45, 0); +x_63 = lean_ctor_get(x_45, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_45); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +return x_64; } } } @@ -15302,7 +15809,7 @@ if (x_14 == 0) lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_ctor_get(x_15, 15); +x_17 = lean_ctor_get(x_15, 17); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_PersistentHashMap_contains___at_Lean_NameSSet_contains___spec__2(x_17, x_1); @@ -15340,7 +15847,7 @@ x_23 = lean_ctor_get(x_13, 1); lean_inc(x_23); lean_inc(x_22); lean_dec(x_13); -x_24 = lean_ctor_get(x_22, 15); +x_24 = lean_ctor_get(x_22, 17); lean_inc(x_24); lean_dec(x_22); x_25 = l_Lean_PersistentHashMap_contains___at_Lean_NameSSet_contains___spec__2(x_24, x_1); @@ -15525,7 +16032,7 @@ x_16 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_Internalize_ return x_16; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -15547,27 +16054,27 @@ lean_object* x_18 = _args[17]; _start: { lean_object* x_19; -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_Meta_Grind_internalize___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; -x_13 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_3); -return x_13; +lean_object* x_14; +x_14 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { lean_object* x_15; -x_15 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +x_15 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_5); lean_dec(x_1); return x_15; @@ -15599,22 +16106,22 @@ lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; -x_13 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_3); -return x_13; +lean_object* x_14; +x_14 = l_Lean_Meta_Grind_internalize___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_internalize___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; -x_13 = l_Lean_Meta_Grind_internalize___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_3); -return x_13; +lean_object* x_14; +x_14 = l_Lean_Meta_Grind_internalize___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_4); +return x_14; } } LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_activateTheoremPatterns___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { @@ -15787,6 +16294,7 @@ lean_object* initialize_Lean_Meta_Match_MatcherInfo(uint8_t builtin, lean_object lean_object* initialize_Lean_Meta_Match_MatchEqsExt(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Util(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Internalize(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Internalize(uint8_t builtin, lean_object* w) { lean_object * res; @@ -15813,6 +16321,9 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Util(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Internalize(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__1 = _init_l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__1(); l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__2 = _init_l_Lean_PersistentHashMap_findEntryAux___at_Lean_Meta_Grind_addCongrTable___spec__2___closed__2(); l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_addCongrTable___spec__5___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_addCongrTable___spec__5___closed__1(); @@ -15929,20 +16440,10 @@ l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePat lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__4); l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__5(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_internalizePattern___closed__5); -l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1 = _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1(); -lean_mark_persistent(l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__1); -l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2 = _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2(); -lean_mark_persistent(l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__2); -l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3 = _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3(); -lean_mark_persistent(l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__3); -l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4 = _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4(); -lean_mark_persistent(l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__4); -l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5 = _init_l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5(); -lean_mark_persistent(l_panic___at_Lean_Meta_Grind_internalize___spec__1___closed__5); -l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__1); -l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2(); -lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__3___closed__2); +l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__1); +l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2 = _init_l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2(); +lean_mark_persistent(l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_internalize___spec__2___closed__2); l_Lean_Meta_Grind_internalize___lambda__3___closed__1 = _init_l_Lean_Meta_Grind_internalize___lambda__3___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_internalize___lambda__3___closed__1); l_Lean_Meta_Grind_internalize___lambda__3___closed__2 = _init_l_Lean_Meta_Grind_internalize___lambda__3___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Intro.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Intro.c index 424e7a401187..3de49b4ce7a6 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Intro.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Intro.c @@ -16,12 +16,11 @@ extern "C" { lean_object* l_Lean_Expr_bindingName_x21(lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_Simp_Result_getProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_injection_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedIntroResult; lean_object* l_Lean_mkAppN(lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFreshExprMVarAt(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_isProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isLet(lean_object*); @@ -31,10 +30,10 @@ LEAN_EXPORT lean_object* l_List_forM___at_Lean_Meta_Grind_intros_go___spec__2(le lean_object* l_Lean_MVarId_getTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isLetFun(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_assertAt(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_isCasesCandidate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkEqMP(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -46,85 +45,88 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_G LEAN_EXPORT lean_object* l_List_forM___at_Lean_Meta_Grind_intros_go___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_StateRefT_x27_lift___rarg___boxed(lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_addNewEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_assertAll___closed__1; lean_object* l_Lean_LocalDecl_value(lean_object*); lean_object* l_Lean_FVarId_getDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_intros___closed__1; lean_object* lean_st_ref_get(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); +lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_num___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_assertAt___closed__1; lean_object* l_Lean_Meta_Grind_isGrindCasesTarget(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3; LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f___spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9___boxed(lean_object**); lean_object* l_Lean_FVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Queue_dequeue_x3f___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__2___boxed(lean_object**); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); uint8_t l_Lean_Expr_isArrow(lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_GrindTactic_iterate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_assertAt___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1; lean_object* l_Lean_MVarId_assert(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2; lean_object* l_Lean_LocalContext_mkLocalDecl(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_isCasesCandidate___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_userName(lean_object*); lean_object* l_Lean_Meta_Grind_addHypothesis(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2; lean_object* l_Lean_Expr_bindingDomain_x21(lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_assertAt___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_shareCommon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_getLocalInstances(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___boxed(lean_object**); lean_object* l_Lean_LocalDecl_type(lean_object*); LEAN_EXPORT lean_object* l_List_forM___at_Lean_Meta_Grind_intros_go___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); lean_object* l_List_reverse___rarg(lean_object*); lean_object* l_Lean_MVarId_byContra_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_assertAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3; lean_object* l_Lean_Expr_fvar___override(lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed(lean_object**); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingBody_x21(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_cases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_intro1Core(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_bindingInfo_x21(lean_object*); uint8_t l_Lean_Expr_isForall(lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_mvarId_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_assertNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -331,231 +333,162 @@ return x_56; } } } -LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_7; -x_7 = lean_alloc_closure((void*)(l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg___boxed), 2, 0); -return x_7; +lean_object* x_8; +x_8 = lean_alloc_closure((void*)(l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg___boxed), 2, 0); +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_9; uint8_t x_10; -x_9 = l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg(x_7, x_8); -x_10 = !lean_is_exclusive(x_9); -if (x_10 == 0) +lean_object* x_10; uint8_t x_11; +x_10 = l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___rarg(x_8, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -return x_9; +return x_10; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = lean_ctor_get(x_9, 0); -x_12 = lean_ctor_get(x_9, 1); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_9); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_11); -lean_ctor_set(x_13, 1, x_12); -return x_13; +lean_dec(x_10); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; } } } -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_11 = lean_st_ref_take(x_7, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_12 = lean_apply_9(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); -x_14 = lean_ctor_get(x_11, 1); +x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); -lean_dec(x_11); -x_15 = !lean_is_exclusive(x_12); -if (x_15 == 0) +lean_dec(x_12); +x_15 = lean_apply_10(x_2, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_15; +} +else { -lean_object* x_16; uint8_t x_17; -x_16 = lean_ctor_get(x_12, 0); -lean_dec(x_16); -x_17 = !lean_is_exclusive(x_13); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_13, 7); -x_19 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_18, x_1, x_2); -lean_ctor_set(x_13, 7, x_19); -x_20 = lean_st_ref_set(x_7, x_12, x_14); -x_21 = !lean_is_exclusive(x_20); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_20, 0); -lean_dec(x_22); -x_23 = lean_box(0); -lean_ctor_set(x_20, 0, x_23); -return x_20; +uint8_t x_16; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) +{ +return x_12; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_20, 1); -lean_inc(x_24); -lean_dec(x_20); -x_25 = lean_box(0); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 0); +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_12); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} +LEAN_EXPORT lean_object* l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___rarg), 11, 0); +return x_3; +} } +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_apply_4(x_2, x_3, x_4, x_5, x_6); +x_13 = l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(x_1, x_12, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_27 = lean_ctor_get(x_13, 0); -x_28 = lean_ctor_get(x_13, 1); -x_29 = lean_ctor_get(x_13, 2); -x_30 = lean_ctor_get(x_13, 3); -x_31 = lean_ctor_get(x_13, 4); -x_32 = lean_ctor_get(x_13, 5); -x_33 = lean_ctor_get(x_13, 6); -x_34 = lean_ctor_get(x_13, 7); -x_35 = lean_ctor_get(x_13, 8); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); lean_dec(x_13); -x_36 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_34, x_1, x_2); -x_37 = lean_alloc_ctor(0, 9, 0); -lean_ctor_set(x_37, 0, x_27); -lean_ctor_set(x_37, 1, x_28); -lean_ctor_set(x_37, 2, x_29); -lean_ctor_set(x_37, 3, x_30); -lean_ctor_set(x_37, 4, x_31); -lean_ctor_set(x_37, 5, x_32); -lean_ctor_set(x_37, 6, x_33); -lean_ctor_set(x_37, 7, x_36); -lean_ctor_set(x_37, 8, x_35); -lean_ctor_set(x_12, 0, x_37); -x_38 = lean_st_ref_set(x_7, x_12, x_14); -x_39 = lean_ctor_get(x_38, 1); -lean_inc(x_39); -if (lean_is_exclusive(x_38)) { - lean_ctor_release(x_38, 0); - lean_ctor_release(x_38, 1); - x_40 = x_38; -} else { - lean_dec_ref(x_38); - x_40 = lean_box(0); -} -x_41 = lean_box(0); -if (lean_is_scalar(x_40)) { - x_42 = lean_alloc_ctor(0, 2, 0); -} else { - x_42 = x_40; +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; } -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_39); -return x_42; } +else +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) +{ +return x_13; } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_43 = lean_ctor_get(x_12, 1); -x_44 = lean_ctor_get(x_12, 2); -x_45 = lean_ctor_get(x_12, 3); -x_46 = lean_ctor_get(x_12, 4); -lean_inc(x_46); -lean_inc(x_45); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_12); -x_47 = lean_ctor_get(x_13, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_13, 1); -lean_inc(x_48); -x_49 = lean_ctor_get(x_13, 2); -lean_inc(x_49); -x_50 = lean_ctor_get(x_13, 3); -lean_inc(x_50); -x_51 = lean_ctor_get(x_13, 4); -lean_inc(x_51); -x_52 = lean_ctor_get(x_13, 5); -lean_inc(x_52); -x_53 = lean_ctor_get(x_13, 6); -lean_inc(x_53); -x_54 = lean_ctor_get(x_13, 7); -lean_inc(x_54); -x_55 = lean_ctor_get(x_13, 8); -lean_inc(x_55); -if (lean_is_exclusive(x_13)) { - lean_ctor_release(x_13, 0); - lean_ctor_release(x_13, 1); - lean_ctor_release(x_13, 2); - lean_ctor_release(x_13, 3); - lean_ctor_release(x_13, 4); - lean_ctor_release(x_13, 5); - lean_ctor_release(x_13, 6); - lean_ctor_release(x_13, 7); - lean_ctor_release(x_13, 8); - x_56 = x_13; -} else { - lean_dec_ref(x_13); - x_56 = lean_box(0); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_13, 0); +x_20 = lean_ctor_get(x_13, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_13); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } -x_57 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_54, x_1, x_2); -if (lean_is_scalar(x_56)) { - x_58 = lean_alloc_ctor(0, 9, 0); -} else { - x_58 = x_56; -} -lean_ctor_set(x_58, 0, x_47); -lean_ctor_set(x_58, 1, x_48); -lean_ctor_set(x_58, 2, x_49); -lean_ctor_set(x_58, 3, x_50); -lean_ctor_set(x_58, 4, x_51); -lean_ctor_set(x_58, 5, x_52); -lean_ctor_set(x_58, 6, x_53); -lean_ctor_set(x_58, 7, x_57); -lean_ctor_set(x_58, 8, x_55); -x_59 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_43); -lean_ctor_set(x_59, 2, x_44); -lean_ctor_set(x_59, 3, x_45); -lean_ctor_set(x_59, 4, x_46); -x_60 = lean_st_ref_set(x_7, x_59, x_14); -x_61 = lean_ctor_get(x_60, 1); -lean_inc(x_61); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_62 = x_60; -} else { - lean_dec_ref(x_60); - x_62 = lean_box(0); } -x_63 = lean_box(0); -if (lean_is_scalar(x_62)) { - x_64 = lean_alloc_ctor(0, 2, 0); -} else { - x_64 = x_62; } -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_61); -return x_64; } +LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4___rarg), 11, 0); +return x_2; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -591,130 +524,281 @@ return x_14; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_14; -lean_inc(x_5); -x_14 = l_Lean_Meta_Grind_addNewEq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_14) == 0) +lean_object* x_12; +lean_inc(x_7); +lean_inc(x_1); +x_12 = l_Lean_FVarId_getDecl(x_1, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_15 = lean_ctor_get(x_14, 1); -lean_inc(x_15); -lean_dec(x_14); -x_16 = lean_st_ref_get(x_5, x_15); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = l_Lean_LocalDecl_value(x_13); +lean_dec(x_13); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_5); +x_16 = l_Lean_Meta_Grind_simp(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_18; lean_object* x_19; uint8_t x_20; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); -x_19 = lean_st_ref_get(x_5, x_18); -lean_dec(x_5); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_Expr_fvar___override(x_1); +x_20 = l_Lean_Meta_Grind_shareCommon(x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_18); +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_17); +x_23 = l_Lean_Meta_Simp_Result_getProof(x_17, x_7, x_8, x_9, x_10, x_22); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_21; -x_21 = lean_ctor_get(x_19, 0); -lean_ctor_set(x_16, 1, x_21); -lean_ctor_set(x_19, 0, x_16); -return x_19; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_ctor_get(x_17, 0); +lean_inc(x_26); +lean_dec(x_17); +lean_inc(x_3); +x_27 = l_Lean_Meta_Grind_addNewEq(x_21, x_26, x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_ctor_get(x_27, 1); +lean_inc(x_28); +lean_dec(x_27); +x_29 = lean_st_ref_get(x_3, x_28); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_ctor_get(x_29, 1); +x_32 = lean_st_ref_get(x_3, x_31); +lean_dec(x_3); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; +x_34 = lean_ctor_get(x_32, 0); +lean_ctor_set(x_29, 1, x_34); +lean_ctor_set(x_32, 0, x_29); +return x_32; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_19, 0); -x_23 = lean_ctor_get(x_19, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_19); -lean_ctor_set(x_16, 1, x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_16); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_32, 0); +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_32); +lean_ctor_set(x_29, 1, x_35); +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_29); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_25 = lean_ctor_get(x_16, 0); -x_26 = lean_ctor_get(x_16, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_16); -x_27 = lean_st_ref_get(x_5, x_26); -lean_dec(x_5); -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -if (lean_is_exclusive(x_27)) { - lean_ctor_release(x_27, 0); - lean_ctor_release(x_27, 1); - x_30 = x_27; +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_38 = lean_ctor_get(x_29, 0); +x_39 = lean_ctor_get(x_29, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_29); +x_40 = lean_st_ref_get(x_3, x_39); +lean_dec(x_3); +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +if (lean_is_exclusive(x_40)) { + lean_ctor_release(x_40, 0); + lean_ctor_release(x_40, 1); + x_43 = x_40; } else { - lean_dec_ref(x_27); - x_30 = lean_box(0); -} -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_25); -lean_ctor_set(x_31, 1, x_28); -if (lean_is_scalar(x_30)) { - x_32 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_40); + x_43 = lean_box(0); +} +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_38); +lean_ctor_set(x_44, 1, x_41); +if (lean_is_scalar(x_43)) { + x_45 = lean_alloc_ctor(0, 2, 0); } else { - x_32 = x_30; + x_45 = x_43; } -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_29); -return x_32; +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_42); +return x_45; } } else { -uint8_t x_33; -lean_dec(x_5); -x_33 = !lean_is_exclusive(x_14); -if (x_33 == 0) +uint8_t x_46; +lean_dec(x_3); +x_46 = !lean_is_exclusive(x_27); +if (x_46 == 0) { -return x_14; +return x_27; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_14, 0); -x_35 = lean_ctor_get(x_14, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_14); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; -} -} +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_27, 0); +x_48 = lean_ctor_get(x_27, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_27); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_1); -if (x_10 == 0) -{ -lean_object* x_11; -x_11 = lean_ctor_get(x_1, 1); -lean_dec(x_11); -lean_ctor_set(x_1, 1, x_9); -return x_1; } else { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_1, 0); -lean_inc(x_12); -lean_dec(x_1); -x_13 = lean_alloc_ctor(0, 2, 0); +uint8_t x_50; +lean_dec(x_21); +lean_dec(x_17); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_50 = !lean_is_exclusive(x_23); +if (x_50 == 0) +{ +return x_23; +} +else +{ +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_23, 0); +x_52 = lean_ctor_get(x_23, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_23); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; +} +} +} +else +{ +uint8_t x_54; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_54 = !lean_is_exclusive(x_16); +if (x_54 == 0) +{ +return x_16; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_16, 0); +x_56 = lean_ctor_get(x_16, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_16); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +} +else +{ +uint8_t x_58; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_58 = !lean_is_exclusive(x_12); +if (x_58 == 0) +{ +return x_12; +} +else +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_12, 0); +x_60 = lean_ctor_get(x_12, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_12); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_1); +if (x_10 == 0) +{ +lean_object* x_11; +x_11 = lean_ctor_get(x_1, 1); +lean_dec(x_11); +lean_ctor_set(x_1, 1, x_9); +return x_1; +} +else +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_1, 0); +lean_inc(x_12); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_13, 0, x_12); lean_ctor_set(x_13, 1, x_9); return x_13; @@ -729,1665 +813,2080 @@ x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lea return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, uint8_t x_24, lean_object* x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32, lean_object* x_33, lean_object* x_34) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24, uint8_t x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32, lean_object* x_33, lean_object* x_34, lean_object* x_35, lean_object* x_36, lean_object* x_37) { _start: { -lean_object* x_35; lean_object* x_36; -x_35 = l_Lean_LocalDecl_type(x_26); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_38; lean_object* x_39; +x_38 = l_Lean_LocalDecl_type(x_29); +lean_inc(x_36); lean_inc(x_35); -x_36 = l_Lean_Meta_isProp(x_35, x_30, x_31, x_32, x_33, x_34); -if (lean_obj_tag(x_36) == 0) +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_38); +x_39 = l_Lean_Meta_isProp(x_38, x_33, x_34, x_35, x_36, x_37); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_37; uint8_t x_38; -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -x_38 = lean_unbox(x_37); -lean_dec(x_37); -if (x_38 == 0) +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_unbox(x_40); +lean_dec(x_40); +if (x_41 == 0) { -uint8_t x_39; -lean_dec(x_35); -x_39 = !lean_is_exclusive(x_36); -if (x_39 == 0) +uint8_t x_42; +lean_dec(x_38); +x_42 = !lean_is_exclusive(x_39); +if (x_42 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_36, 1); -x_41 = lean_ctor_get(x_36, 0); -lean_dec(x_41); +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 1); +x_44 = lean_ctor_get(x_39, 0); +lean_dec(x_44); lean_inc(x_1); -x_42 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_42, 0, x_1); -lean_ctor_set(x_42, 1, x_2); -lean_ctor_set(x_42, 2, x_3); -lean_ctor_set(x_42, 3, x_4); -lean_ctor_set(x_42, 4, x_5); -lean_ctor_set(x_42, 5, x_6); -lean_ctor_set(x_42, 6, x_8); -lean_ctor_set(x_42, 7, x_9); -lean_ctor_set(x_42, 8, x_10); -lean_ctor_set(x_42, 9, x_11); -lean_ctor_set(x_42, 10, x_12); -lean_ctor_set(x_42, 11, x_13); -lean_ctor_set(x_42, 12, x_14); -lean_ctor_set(x_42, 13, x_15); -lean_ctor_set(x_42, 14, x_16); -lean_ctor_set(x_42, 15, x_17); -lean_ctor_set(x_42, 16, x_18); -lean_ctor_set(x_42, 17, x_19); -lean_ctor_set(x_42, 18, x_20); -lean_ctor_set(x_42, 19, x_21); -lean_ctor_set_uint8(x_42, sizeof(void*)*20, x_7); -if (x_24 == 0) +x_45 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_45, 0, x_1); +lean_ctor_set(x_45, 1, x_2); +lean_ctor_set(x_45, 2, x_3); +lean_ctor_set(x_45, 3, x_4); +lean_ctor_set(x_45, 4, x_5); +lean_ctor_set(x_45, 5, x_6); +lean_ctor_set(x_45, 6, x_7); +lean_ctor_set(x_45, 7, x_9); +lean_ctor_set(x_45, 8, x_10); +lean_ctor_set(x_45, 9, x_11); +lean_ctor_set(x_45, 10, x_12); +lean_ctor_set(x_45, 11, x_13); +lean_ctor_set(x_45, 12, x_14); +lean_ctor_set(x_45, 13, x_15); +lean_ctor_set(x_45, 14, x_16); +lean_ctor_set(x_45, 15, x_17); +lean_ctor_set(x_45, 16, x_18); +lean_ctor_set(x_45, 17, x_19); +lean_ctor_set(x_45, 18, x_20); +lean_ctor_set(x_45, 19, x_21); +lean_ctor_set(x_45, 20, x_22); +lean_ctor_set(x_45, 21, x_23); +lean_ctor_set(x_45, 22, x_24); +lean_ctor_set_uint8(x_45, sizeof(void*)*23, x_8); +if (x_25 == 0) { -uint8_t x_113; -x_113 = l_Lean_Expr_isLetFun(x_25); -if (x_113 == 0) +uint8_t x_46; +x_46 = l_Lean_Expr_isLetFun(x_26); +if (x_46 == 0) { -lean_object* x_114; +lean_object* x_47; +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_34); lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); lean_dec(x_1); -x_114 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_114, 0, x_22); -lean_ctor_set(x_114, 1, x_42); -lean_ctor_set(x_36, 0, x_114); -return x_36; +x_47 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_47, 0, x_27); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_39, 0, x_47); +return x_39; } else { -lean_object* x_115; -lean_free_object(x_36); -x_115 = lean_box(0); -x_43 = x_115; -goto block_112; -} +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +lean_free_object(x_39); +x_48 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_48, 0, x_45); +lean_inc(x_27); +x_49 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 11, 2); +lean_closure_set(x_49, 0, x_27); +lean_closure_set(x_49, 1, x_28); +x_50 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_50, 0, x_48); +lean_closure_set(x_50, 1, x_49); +x_51 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_52, 0, x_50); +lean_closure_set(x_52, 1, x_51); +x_53 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_52, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_43); +if (lean_obj_tag(x_53) == 0) +{ +uint8_t x_54; +x_54 = !lean_is_exclusive(x_53); +if (x_54 == 0) +{ +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_53, 0); +x_56 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_56, 0, x_27); +lean_ctor_set(x_56, 1, x_55); +lean_ctor_set(x_53, 0, x_56); +return x_53; } else { -lean_object* x_116; -lean_free_object(x_36); -x_116 = lean_box(0); -x_43 = x_116; -goto block_112; +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_57 = lean_ctor_get(x_53, 0); +x_58 = lean_ctor_get(x_53, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_53); +x_59 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_59, 0, x_27); +lean_ctor_set(x_59, 1, x_57); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_58); +return x_60; } -block_112: -{ -lean_object* x_44; -lean_dec(x_43); -lean_inc(x_30); -lean_inc(x_22); -x_44 = l_Lean_FVarId_getDecl(x_22, x_30, x_31, x_32, x_33, x_40); -if (lean_obj_tag(x_44) == 0) +} +else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = l_Lean_LocalDecl_value(x_45); -lean_dec(x_45); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_28); -x_48 = l_Lean_Meta_Grind_simp(x_47, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_46); -if (lean_obj_tag(x_48) == 0) +uint8_t x_61; +lean_dec(x_27); +x_61 = !lean_is_exclusive(x_53); +if (x_61 == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); -lean_inc(x_50); -lean_dec(x_48); -lean_inc(x_22); -x_51 = l_Lean_Expr_fvar___override(x_22); -x_52 = l_Lean_Meta_Grind_shareCommon(x_51, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_50); -x_53 = !lean_is_exclusive(x_52); -if (x_53 == 0) +return x_53; +} +else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_52, 0); -x_55 = lean_ctor_get(x_52, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_49); -x_56 = l_Lean_Meta_Simp_Result_getProof(x_49, x_30, x_31, x_32, x_33, x_55); -if (lean_obj_tag(x_56) == 0) +lean_object* x_62; lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_53, 0); +x_63 = lean_ctor_get(x_53, 1); +lean_inc(x_63); +lean_inc(x_62); +lean_dec(x_53); +x_64 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_64, 1, x_63); +return x_64; +} +} +} +} +else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = lean_ctor_get(x_49, 0); -lean_inc(x_59); -lean_dec(x_49); -x_60 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); -lean_closure_set(x_60, 0, x_42); -x_61 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 13, 4); -lean_closure_set(x_61, 0, x_54); -lean_closure_set(x_61, 1, x_59); -lean_closure_set(x_61, 2, x_57); -lean_closure_set(x_61, 3, x_23); -x_62 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_62, 0, x_60); -lean_closure_set(x_62, 1, x_61); -x_63 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; -x_64 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_64, 0, x_62); -lean_closure_set(x_64, 1, x_63); -x_65 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_64, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_58); -if (lean_obj_tag(x_65) == 0) +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; +lean_free_object(x_39); +x_65 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_65, 0, x_45); +lean_inc(x_27); +x_66 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 11, 2); +lean_closure_set(x_66, 0, x_27); +lean_closure_set(x_66, 1, x_28); +x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_67, 0, x_65); +lean_closure_set(x_67, 1, x_66); +x_68 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +x_69 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_69, 0, x_67); +lean_closure_set(x_69, 1, x_68); +x_70 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_69, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_43); +if (lean_obj_tag(x_70) == 0) { -uint8_t x_66; -x_66 = !lean_is_exclusive(x_65); -if (x_66 == 0) +uint8_t x_71; +x_71 = !lean_is_exclusive(x_70); +if (x_71 == 0) { -lean_object* x_67; -x_67 = lean_ctor_get(x_65, 0); -lean_ctor_set_tag(x_52, 3); -lean_ctor_set(x_52, 1, x_67); -lean_ctor_set(x_52, 0, x_22); -lean_ctor_set(x_65, 0, x_52); -return x_65; +lean_object* x_72; lean_object* x_73; +x_72 = lean_ctor_get(x_70, 0); +x_73 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_73, 0, x_27); +lean_ctor_set(x_73, 1, x_72); +lean_ctor_set(x_70, 0, x_73); +return x_70; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_65, 0); -x_69 = lean_ctor_get(x_65, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_65); -lean_ctor_set_tag(x_52, 3); -lean_ctor_set(x_52, 1, x_68); -lean_ctor_set(x_52, 0, x_22); -x_70 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_70, 0, x_52); -lean_ctor_set(x_70, 1, x_69); -return x_70; +lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_74 = lean_ctor_get(x_70, 0); +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_inc(x_74); +lean_dec(x_70); +x_76 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_76, 0, x_27); +lean_ctor_set(x_76, 1, x_74); +x_77 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_75); +return x_77; } } else { -uint8_t x_71; -lean_free_object(x_52); -lean_dec(x_22); -x_71 = !lean_is_exclusive(x_65); -if (x_71 == 0) +uint8_t x_78; +lean_dec(x_27); +x_78 = !lean_is_exclusive(x_70); +if (x_78 == 0) { -return x_65; +return x_70; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_65, 0); -x_73 = lean_ctor_get(x_65, 1); -lean_inc(x_73); -lean_inc(x_72); -lean_dec(x_65); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; +lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_79 = lean_ctor_get(x_70, 0); +x_80 = lean_ctor_get(x_70, 1); +lean_inc(x_80); +lean_inc(x_79); +lean_dec(x_70); +x_81 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +return x_81; +} } } } else { -uint8_t x_75; -lean_free_object(x_52); -lean_dec(x_54); -lean_dec(x_49); -lean_dec(x_42); +lean_object* x_82; lean_object* x_83; +x_82 = lean_ctor_get(x_39, 1); +lean_inc(x_82); +lean_dec(x_39); +lean_inc(x_1); +x_83 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_83, 0, x_1); +lean_ctor_set(x_83, 1, x_2); +lean_ctor_set(x_83, 2, x_3); +lean_ctor_set(x_83, 3, x_4); +lean_ctor_set(x_83, 4, x_5); +lean_ctor_set(x_83, 5, x_6); +lean_ctor_set(x_83, 6, x_7); +lean_ctor_set(x_83, 7, x_9); +lean_ctor_set(x_83, 8, x_10); +lean_ctor_set(x_83, 9, x_11); +lean_ctor_set(x_83, 10, x_12); +lean_ctor_set(x_83, 11, x_13); +lean_ctor_set(x_83, 12, x_14); +lean_ctor_set(x_83, 13, x_15); +lean_ctor_set(x_83, 14, x_16); +lean_ctor_set(x_83, 15, x_17); +lean_ctor_set(x_83, 16, x_18); +lean_ctor_set(x_83, 17, x_19); +lean_ctor_set(x_83, 18, x_20); +lean_ctor_set(x_83, 19, x_21); +lean_ctor_set(x_83, 20, x_22); +lean_ctor_set(x_83, 21, x_23); +lean_ctor_set(x_83, 22, x_24); +lean_ctor_set_uint8(x_83, sizeof(void*)*23, x_8); +if (x_25 == 0) +{ +uint8_t x_84; +x_84 = l_Lean_Expr_isLetFun(x_26); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_34); lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_56); -if (x_75 == 0) -{ -return x_56; +x_85 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_85, 0, x_27); +lean_ctor_set(x_85, 1, x_83); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_82); +return x_86; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_56, 0); -x_77 = lean_ctor_get(x_56, 1); -lean_inc(x_77); -lean_inc(x_76); -lean_dec(x_56); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; -} -} -} -else -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_52, 0); -x_80 = lean_ctor_get(x_52, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_52); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_49); -x_81 = l_Lean_Meta_Simp_Result_getProof(x_49, x_30, x_31, x_32, x_33, x_80); -if (lean_obj_tag(x_81) == 0) -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_ctor_get(x_49, 0); -lean_inc(x_84); -lean_dec(x_49); -x_85 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); -lean_closure_set(x_85, 0, x_42); -x_86 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 13, 4); -lean_closure_set(x_86, 0, x_79); -lean_closure_set(x_86, 1, x_84); -lean_closure_set(x_86, 2, x_82); -lean_closure_set(x_86, 3, x_23); -x_87 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_87, 0, x_85); -lean_closure_set(x_87, 1, x_86); -x_88 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_87 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_87, 0, x_83); +lean_inc(x_27); +x_88 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 11, 2); +lean_closure_set(x_88, 0, x_27); +lean_closure_set(x_88, 1, x_28); x_89 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); lean_closure_set(x_89, 0, x_87); lean_closure_set(x_89, 1, x_88); -x_90 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_89, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_83); -if (lean_obj_tag(x_90) == 0) -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_91 = lean_ctor_get(x_90, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_90, 1); -lean_inc(x_92); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_93 = x_90; +x_90 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +x_91 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_91, 0, x_89); +lean_closure_set(x_91, 1, x_90); +x_92 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_91, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_82); +if (lean_obj_tag(x_92) == 0) +{ +lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_95 = x_92; } else { - lean_dec_ref(x_90); - x_93 = lean_box(0); -} -x_94 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_94, 0, x_22); -lean_ctor_set(x_94, 1, x_91); -if (lean_is_scalar(x_93)) { - x_95 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_92); + x_95 = lean_box(0); +} +x_96 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_96, 0, x_27); +lean_ctor_set(x_96, 1, x_93); +if (lean_is_scalar(x_95)) { + x_97 = lean_alloc_ctor(0, 2, 0); } else { - x_95 = x_93; + x_97 = x_95; } -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_92); -return x_95; +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); +return x_97; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -lean_dec(x_22); -x_96 = lean_ctor_get(x_90, 0); -lean_inc(x_96); -x_97 = lean_ctor_get(x_90, 1); -lean_inc(x_97); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_98 = x_90; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_dec(x_27); +x_98 = lean_ctor_get(x_92, 0); +lean_inc(x_98); +x_99 = lean_ctor_get(x_92, 1); +lean_inc(x_99); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_100 = x_92; } else { - lean_dec_ref(x_90); - x_98 = lean_box(0); + lean_dec_ref(x_92); + x_100 = lean_box(0); } -if (lean_is_scalar(x_98)) { - x_99 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_100)) { + x_101 = lean_alloc_ctor(1, 2, 0); } else { - x_99 = x_98; + x_101 = x_100; +} +lean_ctor_set(x_101, 0, x_98); +lean_ctor_set(x_101, 1, x_99); +return x_101; } -lean_ctor_set(x_99, 0, x_96); -lean_ctor_set(x_99, 1, x_97); -return x_99; } } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_79); -lean_dec(x_49); -lean_dec(x_42); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; +x_102 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_102, 0, x_83); +lean_inc(x_27); +x_103 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 11, 2); +lean_closure_set(x_103, 0, x_27); +lean_closure_set(x_103, 1, x_28); +x_104 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_104, 0, x_102); +lean_closure_set(x_104, 1, x_103); +x_105 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +x_106 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_106, 0, x_104); +lean_closure_set(x_106, 1, x_105); +x_107 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_106, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_82); +if (lean_obj_tag(x_107) == 0) +{ +lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_108 = lean_ctor_get(x_107, 0); +lean_inc(x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_110 = x_107; +} else { + lean_dec_ref(x_107); + x_110 = lean_box(0); +} +x_111 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_111, 0, x_27); +lean_ctor_set(x_111, 1, x_108); +if (lean_is_scalar(x_110)) { + x_112 = lean_alloc_ctor(0, 2, 0); +} else { + x_112 = x_110; +} +lean_ctor_set(x_112, 0, x_111); +lean_ctor_set(x_112, 1, x_109); +return x_112; +} +else +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_1); -x_100 = lean_ctor_get(x_81, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_81, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_81)) { - lean_ctor_release(x_81, 0); - lean_ctor_release(x_81, 1); - x_102 = x_81; +x_113 = lean_ctor_get(x_107, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_107, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_107)) { + lean_ctor_release(x_107, 0); + lean_ctor_release(x_107, 1); + x_115 = x_107; } else { - lean_dec_ref(x_81); - x_102 = lean_box(0); + lean_dec_ref(x_107); + x_115 = lean_box(0); } -if (lean_is_scalar(x_102)) { - x_103 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_115)) { + x_116 = lean_alloc_ctor(1, 2, 0); } else { - x_103 = x_102; + x_116 = x_115; +} +lean_ctor_set(x_116, 0, x_113); +lean_ctor_set(x_116, 1, x_114); +return x_116; } -lean_ctor_set(x_103, 0, x_100); -lean_ctor_set(x_103, 1, x_101); -return x_103; } } } else { -uint8_t x_104; -lean_dec(x_42); -lean_dec(x_33); +lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); +x_117 = lean_ctor_get(x_39, 1); +lean_inc(x_117); +lean_dec(x_39); +x_118 = l_Lean_LocalDecl_userName(x_29); +x_119 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_118, x_35, x_36, x_117); +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_119, 1); +lean_inc(x_121); +lean_dec(x_119); +x_122 = l_Lean_Expr_fvar___override(x_27); +x_123 = l_Lean_MVarId_assert(x_1, x_120, x_38, x_122, x_33, x_34, x_35, x_36, x_121); +if (lean_obj_tag(x_123) == 0) +{ +uint8_t x_124; +x_124 = !lean_is_exclusive(x_123); +if (x_124 == 0) +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +x_125 = lean_ctor_get(x_123, 0); +x_126 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_2); +lean_ctor_set(x_126, 2, x_3); +lean_ctor_set(x_126, 3, x_4); +lean_ctor_set(x_126, 4, x_5); +lean_ctor_set(x_126, 5, x_6); +lean_ctor_set(x_126, 6, x_7); +lean_ctor_set(x_126, 7, x_9); +lean_ctor_set(x_126, 8, x_10); +lean_ctor_set(x_126, 9, x_11); +lean_ctor_set(x_126, 10, x_12); +lean_ctor_set(x_126, 11, x_13); +lean_ctor_set(x_126, 12, x_14); +lean_ctor_set(x_126, 13, x_15); +lean_ctor_set(x_126, 14, x_16); +lean_ctor_set(x_126, 15, x_17); +lean_ctor_set(x_126, 16, x_18); +lean_ctor_set(x_126, 17, x_19); +lean_ctor_set(x_126, 18, x_20); +lean_ctor_set(x_126, 19, x_21); +lean_ctor_set(x_126, 20, x_22); +lean_ctor_set(x_126, 21, x_23); +lean_ctor_set(x_126, 22, x_24); +lean_ctor_set_uint8(x_126, sizeof(void*)*23, x_8); +x_127 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_127, 0, x_126); +lean_ctor_set(x_123, 0, x_127); +return x_123; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_128 = lean_ctor_get(x_123, 0); +x_129 = lean_ctor_get(x_123, 1); +lean_inc(x_129); +lean_inc(x_128); +lean_dec(x_123); +x_130 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_2); +lean_ctor_set(x_130, 2, x_3); +lean_ctor_set(x_130, 3, x_4); +lean_ctor_set(x_130, 4, x_5); +lean_ctor_set(x_130, 5, x_6); +lean_ctor_set(x_130, 6, x_7); +lean_ctor_set(x_130, 7, x_9); +lean_ctor_set(x_130, 8, x_10); +lean_ctor_set(x_130, 9, x_11); +lean_ctor_set(x_130, 10, x_12); +lean_ctor_set(x_130, 11, x_13); +lean_ctor_set(x_130, 12, x_14); +lean_ctor_set(x_130, 13, x_15); +lean_ctor_set(x_130, 14, x_16); +lean_ctor_set(x_130, 15, x_17); +lean_ctor_set(x_130, 16, x_18); +lean_ctor_set(x_130, 17, x_19); +lean_ctor_set(x_130, 18, x_20); +lean_ctor_set(x_130, 19, x_21); +lean_ctor_set(x_130, 20, x_22); +lean_ctor_set(x_130, 21, x_23); +lean_ctor_set(x_130, 22, x_24); +lean_ctor_set_uint8(x_130, sizeof(void*)*23, x_8); +x_131 = lean_alloc_ctor(2, 1, 0); +lean_ctor_set(x_131, 0, x_130); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_131); +lean_ctor_set(x_132, 1, x_129); +return x_132; +} +} +else +{ +uint8_t x_133; +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); -lean_dec(x_1); -x_104 = !lean_is_exclusive(x_48); -if (x_104 == 0) +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_133 = !lean_is_exclusive(x_123); +if (x_133 == 0) { -return x_48; +return x_123; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_48, 0); -x_106 = lean_ctor_get(x_48, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_48); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_134 = lean_ctor_get(x_123, 0); +x_135 = lean_ctor_get(x_123, 1); +lean_inc(x_135); +lean_inc(x_134); +lean_dec(x_123); +x_136 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_136, 0, x_134); +lean_ctor_set(x_136, 1, x_135); +return x_136; +} } } } else { -uint8_t x_108; -lean_dec(x_42); +uint8_t x_137; +lean_dec(x_38); +lean_dec(x_36); +lean_dec(x_35); +lean_dec(x_34); lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); -lean_dec(x_29); lean_dec(x_28); lean_dec(x_27); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_108 = !lean_is_exclusive(x_44); -if (x_108 == 0) +x_137 = !lean_is_exclusive(x_39); +if (x_137 == 0) { -return x_44; +return x_39; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_44, 0); -x_110 = lean_ctor_get(x_44, 1); -lean_inc(x_110); -lean_inc(x_109); -lean_dec(x_44); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +lean_object* x_138; lean_object* x_139; lean_object* x_140; +x_138 = lean_ctor_get(x_39, 0); +x_139 = lean_ctor_get(x_39, 1); +lean_inc(x_139); +lean_inc(x_138); +lean_dec(x_39); +x_140 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_140, 0, x_138); +lean_ctor_set(x_140, 1, x_139); +return x_140; } } } } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_ctor_get(x_36, 1); -lean_inc(x_117); -lean_dec(x_36); -lean_inc(x_1); -x_118 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_118, 0, x_1); -lean_ctor_set(x_118, 1, x_2); -lean_ctor_set(x_118, 2, x_3); -lean_ctor_set(x_118, 3, x_4); -lean_ctor_set(x_118, 4, x_5); -lean_ctor_set(x_118, 5, x_6); -lean_ctor_set(x_118, 6, x_8); -lean_ctor_set(x_118, 7, x_9); -lean_ctor_set(x_118, 8, x_10); -lean_ctor_set(x_118, 9, x_11); -lean_ctor_set(x_118, 10, x_12); -lean_ctor_set(x_118, 11, x_13); -lean_ctor_set(x_118, 12, x_14); -lean_ctor_set(x_118, 13, x_15); -lean_ctor_set(x_118, 14, x_16); -lean_ctor_set(x_118, 15, x_17); -lean_ctor_set(x_118, 16, x_18); -lean_ctor_set(x_118, 17, x_19); -lean_ctor_set(x_118, 18, x_20); -lean_ctor_set(x_118, 19, x_21); -lean_ctor_set_uint8(x_118, sizeof(void*)*20, x_7); -if (x_24 == 0) +uint8_t x_11; uint8_t x_12; uint8_t x_13; lean_object* x_14; +x_11 = 0; +x_12 = 1; +x_13 = 1; +x_14 = l_Lean_Meta_mkLambdaFVars(x_1, x_2, x_11, x_12, x_11, x_13, x_6, x_7, x_8, x_9, x_10); +return x_14; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1() { +_start: { -uint8_t x_164; -x_164 = l_Lean_Expr_isLetFun(x_25); -if (x_164 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2() { +_start: { -lean_object* x_165; lean_object* x_166; -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_1); -x_165 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_165, 0, x_22); -lean_ctor_set(x_165, 1, x_118); -x_166 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_166, 0, x_165); -lean_ctor_set(x_166, 1, x_117); -return x_166; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Grind", 5, 5); +return x_1; } -else +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3() { +_start: { -lean_object* x_167; -x_167 = lean_box(0); -x_119 = x_167; -goto block_163; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("intro_with_eq", 13, 13); +return x_1; } } -else +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4() { +_start: { -lean_object* x_168; -x_168 = lean_box(0); -x_119 = x_168; -goto block_163; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; } -block_163: +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18) { +_start: { -lean_object* x_120; -lean_dec(x_119); -lean_inc(x_30); -lean_inc(x_22); -x_120 = l_Lean_FVarId_getDecl(x_22, x_30, x_31, x_32, x_33, x_117); -if (lean_obj_tag(x_120) == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_121 = lean_ctor_get(x_120, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -lean_dec(x_120); -x_123 = l_Lean_LocalDecl_value(x_121); -lean_dec(x_121); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_28); -x_124 = l_Lean_Meta_Grind_simp(x_123, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_122); -if (lean_obj_tag(x_124) == 0) +lean_object* x_19; uint8_t x_20; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +x_19 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_2, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) { -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -lean_inc(x_22); -x_127 = l_Lean_Expr_fvar___override(x_22); -x_128 = l_Lean_Meta_Grind_shareCommon(x_127, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_126); -x_129 = lean_ctor_get(x_128, 0); -lean_inc(x_129); -x_130 = lean_ctor_get(x_128, 1); -lean_inc(x_130); -if (lean_is_exclusive(x_128)) { - lean_ctor_release(x_128, 0); - lean_ctor_release(x_128, 1); - x_131 = x_128; -} else { - lean_dec_ref(x_128); - x_131 = lean_box(0); +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_19, 1); +x_22 = lean_ctor_get(x_19, 0); +lean_dec(x_22); +x_23 = lean_st_ref_get(x_10, x_21); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_23, 0); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +lean_ctor_set(x_25, 0, x_3); +lean_ctor_set_tag(x_19, 1); +lean_ctor_set(x_19, 1, x_25); +lean_ctor_set(x_19, 0, x_4); +lean_ctor_set(x_23, 0, x_19); +return x_23; } +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_28 = lean_ctor_get(x_25, 1); +x_29 = lean_ctor_get(x_25, 2); +x_30 = lean_ctor_get(x_25, 3); +x_31 = lean_ctor_get(x_25, 4); +x_32 = lean_ctor_get(x_25, 5); +x_33 = lean_ctor_get(x_25, 6); +x_34 = lean_ctor_get_uint8(x_25, sizeof(void*)*23); +x_35 = lean_ctor_get(x_25, 7); +x_36 = lean_ctor_get(x_25, 8); +x_37 = lean_ctor_get(x_25, 9); +x_38 = lean_ctor_get(x_25, 10); +x_39 = lean_ctor_get(x_25, 11); +x_40 = lean_ctor_get(x_25, 12); +x_41 = lean_ctor_get(x_25, 13); +x_42 = lean_ctor_get(x_25, 14); +x_43 = lean_ctor_get(x_25, 15); +x_44 = lean_ctor_get(x_25, 16); +x_45 = lean_ctor_get(x_25, 17); +x_46 = lean_ctor_get(x_25, 18); +x_47 = lean_ctor_get(x_25, 19); +x_48 = lean_ctor_get(x_25, 20); +x_49 = lean_ctor_get(x_25, 21); +x_50 = lean_ctor_get(x_25, 22); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); -lean_inc(x_125); -x_132 = l_Lean_Meta_Simp_Result_getProof(x_125, x_30, x_31, x_32, x_33, x_130); -if (lean_obj_tag(x_132) == 0) -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -lean_dec(x_132); -x_135 = lean_ctor_get(x_125, 0); -lean_inc(x_135); -lean_dec(x_125); -x_136 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); -lean_closure_set(x_136, 0, x_118); -x_137 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__3), 13, 4); -lean_closure_set(x_137, 0, x_129); -lean_closure_set(x_137, 1, x_135); -lean_closure_set(x_137, 2, x_133); -lean_closure_set(x_137, 3, x_23); -x_138 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_138, 0, x_136); -lean_closure_set(x_138, 1, x_137); -x_139 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; -x_140 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_140, 0, x_138); -lean_closure_set(x_140, 1, x_139); -x_141 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_140, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_134); -if (lean_obj_tag(x_141) == 0) -{ -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; -x_142 = lean_ctor_get(x_141, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_141, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_141)) { - lean_ctor_release(x_141, 0); - lean_ctor_release(x_141, 1); - x_144 = x_141; -} else { - lean_dec_ref(x_141); - x_144 = lean_box(0); -} -if (lean_is_scalar(x_131)) { - x_145 = lean_alloc_ctor(3, 2, 0); -} else { - x_145 = x_131; - lean_ctor_set_tag(x_145, 3); -} -lean_ctor_set(x_145, 0, x_22); -lean_ctor_set(x_145, 1, x_142); -if (lean_is_scalar(x_144)) { - x_146 = lean_alloc_ctor(0, 2, 0); -} else { - x_146 = x_144; +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_25); +x_51 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_51, 0, x_3); +lean_ctor_set(x_51, 1, x_28); +lean_ctor_set(x_51, 2, x_29); +lean_ctor_set(x_51, 3, x_30); +lean_ctor_set(x_51, 4, x_31); +lean_ctor_set(x_51, 5, x_32); +lean_ctor_set(x_51, 6, x_33); +lean_ctor_set(x_51, 7, x_35); +lean_ctor_set(x_51, 8, x_36); +lean_ctor_set(x_51, 9, x_37); +lean_ctor_set(x_51, 10, x_38); +lean_ctor_set(x_51, 11, x_39); +lean_ctor_set(x_51, 12, x_40); +lean_ctor_set(x_51, 13, x_41); +lean_ctor_set(x_51, 14, x_42); +lean_ctor_set(x_51, 15, x_43); +lean_ctor_set(x_51, 16, x_44); +lean_ctor_set(x_51, 17, x_45); +lean_ctor_set(x_51, 18, x_46); +lean_ctor_set(x_51, 19, x_47); +lean_ctor_set(x_51, 20, x_48); +lean_ctor_set(x_51, 21, x_49); +lean_ctor_set(x_51, 22, x_50); +lean_ctor_set_uint8(x_51, sizeof(void*)*23, x_34); +lean_ctor_set_tag(x_19, 1); +lean_ctor_set(x_19, 1, x_51); +lean_ctor_set(x_19, 0, x_4); +lean_ctor_set(x_23, 0, x_19); +return x_23; } -lean_ctor_set(x_146, 0, x_145); -lean_ctor_set(x_146, 1, x_143); -return x_146; } else { -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -lean_dec(x_131); -lean_dec(x_22); -x_147 = lean_ctor_get(x_141, 0); -lean_inc(x_147); -x_148 = lean_ctor_get(x_141, 1); -lean_inc(x_148); -if (lean_is_exclusive(x_141)) { - lean_ctor_release(x_141, 0); - lean_ctor_release(x_141, 1); - x_149 = x_141; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint8_t x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_52 = lean_ctor_get(x_23, 0); +x_53 = lean_ctor_get(x_23, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_23); +x_54 = lean_ctor_get(x_52, 1); +lean_inc(x_54); +x_55 = lean_ctor_get(x_52, 2); +lean_inc(x_55); +x_56 = lean_ctor_get(x_52, 3); +lean_inc(x_56); +x_57 = lean_ctor_get(x_52, 4); +lean_inc(x_57); +x_58 = lean_ctor_get(x_52, 5); +lean_inc(x_58); +x_59 = lean_ctor_get(x_52, 6); +lean_inc(x_59); +x_60 = lean_ctor_get_uint8(x_52, sizeof(void*)*23); +x_61 = lean_ctor_get(x_52, 7); +lean_inc(x_61); +x_62 = lean_ctor_get(x_52, 8); +lean_inc(x_62); +x_63 = lean_ctor_get(x_52, 9); +lean_inc(x_63); +x_64 = lean_ctor_get(x_52, 10); +lean_inc(x_64); +x_65 = lean_ctor_get(x_52, 11); +lean_inc(x_65); +x_66 = lean_ctor_get(x_52, 12); +lean_inc(x_66); +x_67 = lean_ctor_get(x_52, 13); +lean_inc(x_67); +x_68 = lean_ctor_get(x_52, 14); +lean_inc(x_68); +x_69 = lean_ctor_get(x_52, 15); +lean_inc(x_69); +x_70 = lean_ctor_get(x_52, 16); +lean_inc(x_70); +x_71 = lean_ctor_get(x_52, 17); +lean_inc(x_71); +x_72 = lean_ctor_get(x_52, 18); +lean_inc(x_72); +x_73 = lean_ctor_get(x_52, 19); +lean_inc(x_73); +x_74 = lean_ctor_get(x_52, 20); +lean_inc(x_74); +x_75 = lean_ctor_get(x_52, 21); +lean_inc(x_75); +x_76 = lean_ctor_get(x_52, 22); +lean_inc(x_76); +if (lean_is_exclusive(x_52)) { + lean_ctor_release(x_52, 0); + lean_ctor_release(x_52, 1); + lean_ctor_release(x_52, 2); + lean_ctor_release(x_52, 3); + lean_ctor_release(x_52, 4); + lean_ctor_release(x_52, 5); + lean_ctor_release(x_52, 6); + lean_ctor_release(x_52, 7); + lean_ctor_release(x_52, 8); + lean_ctor_release(x_52, 9); + lean_ctor_release(x_52, 10); + lean_ctor_release(x_52, 11); + lean_ctor_release(x_52, 12); + lean_ctor_release(x_52, 13); + lean_ctor_release(x_52, 14); + lean_ctor_release(x_52, 15); + lean_ctor_release(x_52, 16); + lean_ctor_release(x_52, 17); + lean_ctor_release(x_52, 18); + lean_ctor_release(x_52, 19); + lean_ctor_release(x_52, 20); + lean_ctor_release(x_52, 21); + lean_ctor_release(x_52, 22); + x_77 = x_52; } else { - lean_dec_ref(x_141); - x_149 = lean_box(0); + lean_dec_ref(x_52); + x_77 = lean_box(0); } -if (lean_is_scalar(x_149)) { - x_150 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_77)) { + x_78 = lean_alloc_ctor(0, 23, 1); } else { - x_150 = x_149; -} -lean_ctor_set(x_150, 0, x_147); -lean_ctor_set(x_150, 1, x_148); -return x_150; -} + x_78 = x_77; +} +lean_ctor_set(x_78, 0, x_3); +lean_ctor_set(x_78, 1, x_54); +lean_ctor_set(x_78, 2, x_55); +lean_ctor_set(x_78, 3, x_56); +lean_ctor_set(x_78, 4, x_57); +lean_ctor_set(x_78, 5, x_58); +lean_ctor_set(x_78, 6, x_59); +lean_ctor_set(x_78, 7, x_61); +lean_ctor_set(x_78, 8, x_62); +lean_ctor_set(x_78, 9, x_63); +lean_ctor_set(x_78, 10, x_64); +lean_ctor_set(x_78, 11, x_65); +lean_ctor_set(x_78, 12, x_66); +lean_ctor_set(x_78, 13, x_67); +lean_ctor_set(x_78, 14, x_68); +lean_ctor_set(x_78, 15, x_69); +lean_ctor_set(x_78, 16, x_70); +lean_ctor_set(x_78, 17, x_71); +lean_ctor_set(x_78, 18, x_72); +lean_ctor_set(x_78, 19, x_73); +lean_ctor_set(x_78, 20, x_74); +lean_ctor_set(x_78, 21, x_75); +lean_ctor_set(x_78, 22, x_76); +lean_ctor_set_uint8(x_78, sizeof(void*)*23, x_60); +lean_ctor_set_tag(x_19, 1); +lean_ctor_set(x_19, 1, x_78); +lean_ctor_set(x_19, 0, x_4); +x_79 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_79, 0, x_19); +lean_ctor_set(x_79, 1, x_53); +return x_79; +} +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_80 = lean_ctor_get(x_19, 1); +lean_inc(x_80); +lean_dec(x_19); +x_81 = lean_st_ref_get(x_10, x_80); +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_84 = x_81; +} else { + lean_dec_ref(x_81); + x_84 = lean_box(0); } -else -{ -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; -lean_dec(x_131); -lean_dec(x_129); -lean_dec(x_125); -lean_dec(x_118); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_1); -x_151 = lean_ctor_get(x_132, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_132, 1); -lean_inc(x_152); -if (lean_is_exclusive(x_132)) { - lean_ctor_release(x_132, 0); - lean_ctor_release(x_132, 1); - x_153 = x_132; +x_85 = lean_ctor_get(x_82, 1); +lean_inc(x_85); +x_86 = lean_ctor_get(x_82, 2); +lean_inc(x_86); +x_87 = lean_ctor_get(x_82, 3); +lean_inc(x_87); +x_88 = lean_ctor_get(x_82, 4); +lean_inc(x_88); +x_89 = lean_ctor_get(x_82, 5); +lean_inc(x_89); +x_90 = lean_ctor_get(x_82, 6); +lean_inc(x_90); +x_91 = lean_ctor_get_uint8(x_82, sizeof(void*)*23); +x_92 = lean_ctor_get(x_82, 7); +lean_inc(x_92); +x_93 = lean_ctor_get(x_82, 8); +lean_inc(x_93); +x_94 = lean_ctor_get(x_82, 9); +lean_inc(x_94); +x_95 = lean_ctor_get(x_82, 10); +lean_inc(x_95); +x_96 = lean_ctor_get(x_82, 11); +lean_inc(x_96); +x_97 = lean_ctor_get(x_82, 12); +lean_inc(x_97); +x_98 = lean_ctor_get(x_82, 13); +lean_inc(x_98); +x_99 = lean_ctor_get(x_82, 14); +lean_inc(x_99); +x_100 = lean_ctor_get(x_82, 15); +lean_inc(x_100); +x_101 = lean_ctor_get(x_82, 16); +lean_inc(x_101); +x_102 = lean_ctor_get(x_82, 17); +lean_inc(x_102); +x_103 = lean_ctor_get(x_82, 18); +lean_inc(x_103); +x_104 = lean_ctor_get(x_82, 19); +lean_inc(x_104); +x_105 = lean_ctor_get(x_82, 20); +lean_inc(x_105); +x_106 = lean_ctor_get(x_82, 21); +lean_inc(x_106); +x_107 = lean_ctor_get(x_82, 22); +lean_inc(x_107); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + lean_ctor_release(x_82, 2); + lean_ctor_release(x_82, 3); + lean_ctor_release(x_82, 4); + lean_ctor_release(x_82, 5); + lean_ctor_release(x_82, 6); + lean_ctor_release(x_82, 7); + lean_ctor_release(x_82, 8); + lean_ctor_release(x_82, 9); + lean_ctor_release(x_82, 10); + lean_ctor_release(x_82, 11); + lean_ctor_release(x_82, 12); + lean_ctor_release(x_82, 13); + lean_ctor_release(x_82, 14); + lean_ctor_release(x_82, 15); + lean_ctor_release(x_82, 16); + lean_ctor_release(x_82, 17); + lean_ctor_release(x_82, 18); + lean_ctor_release(x_82, 19); + lean_ctor_release(x_82, 20); + lean_ctor_release(x_82, 21); + lean_ctor_release(x_82, 22); + x_108 = x_82; } else { - lean_dec_ref(x_132); - x_153 = lean_box(0); + lean_dec_ref(x_82); + x_108 = lean_box(0); } -if (lean_is_scalar(x_153)) { - x_154 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_108)) { + x_109 = lean_alloc_ctor(0, 23, 1); +} else { + x_109 = x_108; +} +lean_ctor_set(x_109, 0, x_3); +lean_ctor_set(x_109, 1, x_85); +lean_ctor_set(x_109, 2, x_86); +lean_ctor_set(x_109, 3, x_87); +lean_ctor_set(x_109, 4, x_88); +lean_ctor_set(x_109, 5, x_89); +lean_ctor_set(x_109, 6, x_90); +lean_ctor_set(x_109, 7, x_92); +lean_ctor_set(x_109, 8, x_93); +lean_ctor_set(x_109, 9, x_94); +lean_ctor_set(x_109, 10, x_95); +lean_ctor_set(x_109, 11, x_96); +lean_ctor_set(x_109, 12, x_97); +lean_ctor_set(x_109, 13, x_98); +lean_ctor_set(x_109, 14, x_99); +lean_ctor_set(x_109, 15, x_100); +lean_ctor_set(x_109, 16, x_101); +lean_ctor_set(x_109, 17, x_102); +lean_ctor_set(x_109, 18, x_103); +lean_ctor_set(x_109, 19, x_104); +lean_ctor_set(x_109, 20, x_105); +lean_ctor_set(x_109, 21, x_106); +lean_ctor_set(x_109, 22, x_107); +lean_ctor_set_uint8(x_109, sizeof(void*)*23, x_91); +x_110 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_110, 0, x_4); +lean_ctor_set(x_110, 1, x_109); +if (lean_is_scalar(x_84)) { + x_111 = lean_alloc_ctor(0, 2, 0); } else { - x_154 = x_153; + x_111 = x_84; } -lean_ctor_set(x_154, 0, x_151); -lean_ctor_set(x_154, 1, x_152); -return x_154; +lean_ctor_set(x_111, 0, x_110); +lean_ctor_set(x_111, 1, x_83); +return x_111; } } else { -lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -lean_dec(x_118); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_1); -x_155 = lean_ctor_get(x_124, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_124, 1); -lean_inc(x_156); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_157 = x_124; -} else { - lean_dec_ref(x_124); - x_157 = lean_box(0); -} -if (lean_is_scalar(x_157)) { - x_158 = lean_alloc_ctor(1, 2, 0); -} else { - x_158 = x_157; +lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; +x_112 = lean_ctor_get(x_1, 0); +x_113 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4; +lean_inc(x_5); +x_114 = l_Lean_Expr_const___override(x_113, x_5); +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_9); +lean_ctor_set(x_115, 1, x_5); +lean_inc(x_112); +x_116 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_116, 0, x_112); +lean_ctor_set(x_116, 1, x_115); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_6); +lean_ctor_set(x_117, 1, x_116); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_7); +lean_ctor_set(x_118, 1, x_117); +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_8); +lean_ctor_set(x_119, 1, x_118); +x_120 = lean_array_mk(x_119); +x_121 = l_Lean_mkAppN(x_114, x_120); +lean_dec(x_120); +x_122 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_2, x_121, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +x_123 = !lean_is_exclusive(x_122); +if (x_123 == 0) +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; uint8_t x_127; +x_124 = lean_ctor_get(x_122, 1); +x_125 = lean_ctor_get(x_122, 0); +lean_dec(x_125); +x_126 = lean_st_ref_get(x_10, x_124); +x_127 = !lean_is_exclusive(x_126); +if (x_127 == 0) +{ +lean_object* x_128; uint8_t x_129; +x_128 = lean_ctor_get(x_126, 0); +x_129 = !lean_is_exclusive(x_128); +if (x_129 == 0) +{ +lean_object* x_130; +x_130 = lean_ctor_get(x_128, 0); +lean_dec(x_130); +lean_ctor_set(x_128, 0, x_3); +lean_ctor_set_tag(x_122, 1); +lean_ctor_set(x_122, 1, x_128); +lean_ctor_set(x_122, 0, x_4); +lean_ctor_set(x_126, 0, x_122); +return x_126; } -lean_ctor_set(x_158, 0, x_155); -lean_ctor_set(x_158, 1, x_156); -return x_158; +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; uint8_t x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_131 = lean_ctor_get(x_128, 1); +x_132 = lean_ctor_get(x_128, 2); +x_133 = lean_ctor_get(x_128, 3); +x_134 = lean_ctor_get(x_128, 4); +x_135 = lean_ctor_get(x_128, 5); +x_136 = lean_ctor_get(x_128, 6); +x_137 = lean_ctor_get_uint8(x_128, sizeof(void*)*23); +x_138 = lean_ctor_get(x_128, 7); +x_139 = lean_ctor_get(x_128, 8); +x_140 = lean_ctor_get(x_128, 9); +x_141 = lean_ctor_get(x_128, 10); +x_142 = lean_ctor_get(x_128, 11); +x_143 = lean_ctor_get(x_128, 12); +x_144 = lean_ctor_get(x_128, 13); +x_145 = lean_ctor_get(x_128, 14); +x_146 = lean_ctor_get(x_128, 15); +x_147 = lean_ctor_get(x_128, 16); +x_148 = lean_ctor_get(x_128, 17); +x_149 = lean_ctor_get(x_128, 18); +x_150 = lean_ctor_get(x_128, 19); +x_151 = lean_ctor_get(x_128, 20); +x_152 = lean_ctor_get(x_128, 21); +x_153 = lean_ctor_get(x_128, 22); +lean_inc(x_153); +lean_inc(x_152); +lean_inc(x_151); +lean_inc(x_150); +lean_inc(x_149); +lean_inc(x_148); +lean_inc(x_147); +lean_inc(x_146); +lean_inc(x_145); +lean_inc(x_144); +lean_inc(x_143); +lean_inc(x_142); +lean_inc(x_141); +lean_inc(x_140); +lean_inc(x_139); +lean_inc(x_138); +lean_inc(x_136); +lean_inc(x_135); +lean_inc(x_134); +lean_inc(x_133); +lean_inc(x_132); +lean_inc(x_131); +lean_dec(x_128); +x_154 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_154, 0, x_3); +lean_ctor_set(x_154, 1, x_131); +lean_ctor_set(x_154, 2, x_132); +lean_ctor_set(x_154, 3, x_133); +lean_ctor_set(x_154, 4, x_134); +lean_ctor_set(x_154, 5, x_135); +lean_ctor_set(x_154, 6, x_136); +lean_ctor_set(x_154, 7, x_138); +lean_ctor_set(x_154, 8, x_139); +lean_ctor_set(x_154, 9, x_140); +lean_ctor_set(x_154, 10, x_141); +lean_ctor_set(x_154, 11, x_142); +lean_ctor_set(x_154, 12, x_143); +lean_ctor_set(x_154, 13, x_144); +lean_ctor_set(x_154, 14, x_145); +lean_ctor_set(x_154, 15, x_146); +lean_ctor_set(x_154, 16, x_147); +lean_ctor_set(x_154, 17, x_148); +lean_ctor_set(x_154, 18, x_149); +lean_ctor_set(x_154, 19, x_150); +lean_ctor_set(x_154, 20, x_151); +lean_ctor_set(x_154, 21, x_152); +lean_ctor_set(x_154, 22, x_153); +lean_ctor_set_uint8(x_154, sizeof(void*)*23, x_137); +lean_ctor_set_tag(x_122, 1); +lean_ctor_set(x_122, 1, x_154); +lean_ctor_set(x_122, 0, x_4); +lean_ctor_set(x_126, 0, x_122); +return x_126; } } else { -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; -lean_dec(x_118); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_1); -x_159 = lean_ctor_get(x_120, 0); +lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; +x_155 = lean_ctor_get(x_126, 0); +x_156 = lean_ctor_get(x_126, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_126); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +x_158 = lean_ctor_get(x_155, 2); +lean_inc(x_158); +x_159 = lean_ctor_get(x_155, 3); lean_inc(x_159); -x_160 = lean_ctor_get(x_120, 1); +x_160 = lean_ctor_get(x_155, 4); lean_inc(x_160); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_161 = x_120; +x_161 = lean_ctor_get(x_155, 5); +lean_inc(x_161); +x_162 = lean_ctor_get(x_155, 6); +lean_inc(x_162); +x_163 = lean_ctor_get_uint8(x_155, sizeof(void*)*23); +x_164 = lean_ctor_get(x_155, 7); +lean_inc(x_164); +x_165 = lean_ctor_get(x_155, 8); +lean_inc(x_165); +x_166 = lean_ctor_get(x_155, 9); +lean_inc(x_166); +x_167 = lean_ctor_get(x_155, 10); +lean_inc(x_167); +x_168 = lean_ctor_get(x_155, 11); +lean_inc(x_168); +x_169 = lean_ctor_get(x_155, 12); +lean_inc(x_169); +x_170 = lean_ctor_get(x_155, 13); +lean_inc(x_170); +x_171 = lean_ctor_get(x_155, 14); +lean_inc(x_171); +x_172 = lean_ctor_get(x_155, 15); +lean_inc(x_172); +x_173 = lean_ctor_get(x_155, 16); +lean_inc(x_173); +x_174 = lean_ctor_get(x_155, 17); +lean_inc(x_174); +x_175 = lean_ctor_get(x_155, 18); +lean_inc(x_175); +x_176 = lean_ctor_get(x_155, 19); +lean_inc(x_176); +x_177 = lean_ctor_get(x_155, 20); +lean_inc(x_177); +x_178 = lean_ctor_get(x_155, 21); +lean_inc(x_178); +x_179 = lean_ctor_get(x_155, 22); +lean_inc(x_179); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + lean_ctor_release(x_155, 2); + lean_ctor_release(x_155, 3); + lean_ctor_release(x_155, 4); + lean_ctor_release(x_155, 5); + lean_ctor_release(x_155, 6); + lean_ctor_release(x_155, 7); + lean_ctor_release(x_155, 8); + lean_ctor_release(x_155, 9); + lean_ctor_release(x_155, 10); + lean_ctor_release(x_155, 11); + lean_ctor_release(x_155, 12); + lean_ctor_release(x_155, 13); + lean_ctor_release(x_155, 14); + lean_ctor_release(x_155, 15); + lean_ctor_release(x_155, 16); + lean_ctor_release(x_155, 17); + lean_ctor_release(x_155, 18); + lean_ctor_release(x_155, 19); + lean_ctor_release(x_155, 20); + lean_ctor_release(x_155, 21); + lean_ctor_release(x_155, 22); + x_180 = x_155; } else { - lean_dec_ref(x_120); - x_161 = lean_box(0); + lean_dec_ref(x_155); + x_180 = lean_box(0); } -if (lean_is_scalar(x_161)) { - x_162 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_180)) { + x_181 = lean_alloc_ctor(0, 23, 1); } else { - x_162 = x_161; + x_181 = x_180; +} +lean_ctor_set(x_181, 0, x_3); +lean_ctor_set(x_181, 1, x_157); +lean_ctor_set(x_181, 2, x_158); +lean_ctor_set(x_181, 3, x_159); +lean_ctor_set(x_181, 4, x_160); +lean_ctor_set(x_181, 5, x_161); +lean_ctor_set(x_181, 6, x_162); +lean_ctor_set(x_181, 7, x_164); +lean_ctor_set(x_181, 8, x_165); +lean_ctor_set(x_181, 9, x_166); +lean_ctor_set(x_181, 10, x_167); +lean_ctor_set(x_181, 11, x_168); +lean_ctor_set(x_181, 12, x_169); +lean_ctor_set(x_181, 13, x_170); +lean_ctor_set(x_181, 14, x_171); +lean_ctor_set(x_181, 15, x_172); +lean_ctor_set(x_181, 16, x_173); +lean_ctor_set(x_181, 17, x_174); +lean_ctor_set(x_181, 18, x_175); +lean_ctor_set(x_181, 19, x_176); +lean_ctor_set(x_181, 20, x_177); +lean_ctor_set(x_181, 21, x_178); +lean_ctor_set(x_181, 22, x_179); +lean_ctor_set_uint8(x_181, sizeof(void*)*23, x_163); +lean_ctor_set_tag(x_122, 1); +lean_ctor_set(x_122, 1, x_181); +lean_ctor_set(x_122, 0, x_4); +x_182 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_182, 0, x_122); +lean_ctor_set(x_182, 1, x_156); +return x_182; +} +} +else +{ +lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; uint8_t x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +x_183 = lean_ctor_get(x_122, 1); +lean_inc(x_183); +lean_dec(x_122); +x_184 = lean_st_ref_get(x_10, x_183); +x_185 = lean_ctor_get(x_184, 0); +lean_inc(x_185); +x_186 = lean_ctor_get(x_184, 1); +lean_inc(x_186); +if (lean_is_exclusive(x_184)) { + lean_ctor_release(x_184, 0); + lean_ctor_release(x_184, 1); + x_187 = x_184; +} else { + lean_dec_ref(x_184); + x_187 = lean_box(0); +} +x_188 = lean_ctor_get(x_185, 1); +lean_inc(x_188); +x_189 = lean_ctor_get(x_185, 2); +lean_inc(x_189); +x_190 = lean_ctor_get(x_185, 3); +lean_inc(x_190); +x_191 = lean_ctor_get(x_185, 4); +lean_inc(x_191); +x_192 = lean_ctor_get(x_185, 5); +lean_inc(x_192); +x_193 = lean_ctor_get(x_185, 6); +lean_inc(x_193); +x_194 = lean_ctor_get_uint8(x_185, sizeof(void*)*23); +x_195 = lean_ctor_get(x_185, 7); +lean_inc(x_195); +x_196 = lean_ctor_get(x_185, 8); +lean_inc(x_196); +x_197 = lean_ctor_get(x_185, 9); +lean_inc(x_197); +x_198 = lean_ctor_get(x_185, 10); +lean_inc(x_198); +x_199 = lean_ctor_get(x_185, 11); +lean_inc(x_199); +x_200 = lean_ctor_get(x_185, 12); +lean_inc(x_200); +x_201 = lean_ctor_get(x_185, 13); +lean_inc(x_201); +x_202 = lean_ctor_get(x_185, 14); +lean_inc(x_202); +x_203 = lean_ctor_get(x_185, 15); +lean_inc(x_203); +x_204 = lean_ctor_get(x_185, 16); +lean_inc(x_204); +x_205 = lean_ctor_get(x_185, 17); +lean_inc(x_205); +x_206 = lean_ctor_get(x_185, 18); +lean_inc(x_206); +x_207 = lean_ctor_get(x_185, 19); +lean_inc(x_207); +x_208 = lean_ctor_get(x_185, 20); +lean_inc(x_208); +x_209 = lean_ctor_get(x_185, 21); +lean_inc(x_209); +x_210 = lean_ctor_get(x_185, 22); +lean_inc(x_210); +if (lean_is_exclusive(x_185)) { + lean_ctor_release(x_185, 0); + lean_ctor_release(x_185, 1); + lean_ctor_release(x_185, 2); + lean_ctor_release(x_185, 3); + lean_ctor_release(x_185, 4); + lean_ctor_release(x_185, 5); + lean_ctor_release(x_185, 6); + lean_ctor_release(x_185, 7); + lean_ctor_release(x_185, 8); + lean_ctor_release(x_185, 9); + lean_ctor_release(x_185, 10); + lean_ctor_release(x_185, 11); + lean_ctor_release(x_185, 12); + lean_ctor_release(x_185, 13); + lean_ctor_release(x_185, 14); + lean_ctor_release(x_185, 15); + lean_ctor_release(x_185, 16); + lean_ctor_release(x_185, 17); + lean_ctor_release(x_185, 18); + lean_ctor_release(x_185, 19); + lean_ctor_release(x_185, 20); + lean_ctor_release(x_185, 21); + lean_ctor_release(x_185, 22); + x_211 = x_185; +} else { + lean_dec_ref(x_185); + x_211 = lean_box(0); } -lean_ctor_set(x_162, 0, x_159); -lean_ctor_set(x_162, 1, x_160); -return x_162; +if (lean_is_scalar(x_211)) { + x_212 = lean_alloc_ctor(0, 23, 1); +} else { + x_212 = x_211; +} +lean_ctor_set(x_212, 0, x_3); +lean_ctor_set(x_212, 1, x_188); +lean_ctor_set(x_212, 2, x_189); +lean_ctor_set(x_212, 3, x_190); +lean_ctor_set(x_212, 4, x_191); +lean_ctor_set(x_212, 5, x_192); +lean_ctor_set(x_212, 6, x_193); +lean_ctor_set(x_212, 7, x_195); +lean_ctor_set(x_212, 8, x_196); +lean_ctor_set(x_212, 9, x_197); +lean_ctor_set(x_212, 10, x_198); +lean_ctor_set(x_212, 11, x_199); +lean_ctor_set(x_212, 12, x_200); +lean_ctor_set(x_212, 13, x_201); +lean_ctor_set(x_212, 14, x_202); +lean_ctor_set(x_212, 15, x_203); +lean_ctor_set(x_212, 16, x_204); +lean_ctor_set(x_212, 17, x_205); +lean_ctor_set(x_212, 18, x_206); +lean_ctor_set(x_212, 19, x_207); +lean_ctor_set(x_212, 20, x_208); +lean_ctor_set(x_212, 21, x_209); +lean_ctor_set(x_212, 22, x_210); +lean_ctor_set_uint8(x_212, sizeof(void*)*23, x_194); +x_213 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_213, 0, x_4); +lean_ctor_set(x_213, 1, x_212); +if (lean_is_scalar(x_187)) { + x_214 = lean_alloc_ctor(0, 2, 0); +} else { + x_214 = x_187; } +lean_ctor_set(x_214, 0, x_213); +lean_ctor_set(x_214, 1, x_186); +return x_214; } } } -else -{ -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -x_169 = lean_ctor_get(x_36, 1); -lean_inc(x_169); -lean_dec(x_36); -x_170 = l_Lean_LocalDecl_userName(x_26); -x_171 = l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(x_170, x_32, x_33, x_169); -x_172 = lean_ctor_get(x_171, 0); -lean_inc(x_172); -x_173 = lean_ctor_get(x_171, 1); -lean_inc(x_173); -lean_dec(x_171); -x_174 = l_Lean_Expr_fvar___override(x_22); -x_175 = l_Lean_MVarId_assert(x_1, x_172, x_35, x_174, x_30, x_31, x_32, x_33, x_173); -if (lean_obj_tag(x_175) == 0) -{ -uint8_t x_176; -x_176 = !lean_is_exclusive(x_175); -if (x_176 == 0) -{ -lean_object* x_177; lean_object* x_178; lean_object* x_179; -x_177 = lean_ctor_get(x_175, 0); -x_178 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_178, 0, x_177); -lean_ctor_set(x_178, 1, x_2); -lean_ctor_set(x_178, 2, x_3); -lean_ctor_set(x_178, 3, x_4); -lean_ctor_set(x_178, 4, x_5); -lean_ctor_set(x_178, 5, x_6); -lean_ctor_set(x_178, 6, x_8); -lean_ctor_set(x_178, 7, x_9); -lean_ctor_set(x_178, 8, x_10); -lean_ctor_set(x_178, 9, x_11); -lean_ctor_set(x_178, 10, x_12); -lean_ctor_set(x_178, 11, x_13); -lean_ctor_set(x_178, 12, x_14); -lean_ctor_set(x_178, 13, x_15); -lean_ctor_set(x_178, 14, x_16); -lean_ctor_set(x_178, 15, x_17); -lean_ctor_set(x_178, 16, x_18); -lean_ctor_set(x_178, 17, x_19); -lean_ctor_set(x_178, 18, x_20); -lean_ctor_set(x_178, 19, x_21); -lean_ctor_set_uint8(x_178, sizeof(void*)*20, x_7); -x_179 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_179, 0, x_178); -lean_ctor_set(x_175, 0, x_179); -return x_175; -} -else -{ -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_180 = lean_ctor_get(x_175, 0); -x_181 = lean_ctor_get(x_175, 1); -lean_inc(x_181); -lean_inc(x_180); -lean_dec(x_175); -x_182 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_182, 0, x_180); -lean_ctor_set(x_182, 1, x_2); -lean_ctor_set(x_182, 2, x_3); -lean_ctor_set(x_182, 3, x_4); -lean_ctor_set(x_182, 4, x_5); -lean_ctor_set(x_182, 5, x_6); -lean_ctor_set(x_182, 6, x_8); -lean_ctor_set(x_182, 7, x_9); -lean_ctor_set(x_182, 8, x_10); -lean_ctor_set(x_182, 9, x_11); -lean_ctor_set(x_182, 10, x_12); -lean_ctor_set(x_182, 11, x_13); -lean_ctor_set(x_182, 12, x_14); -lean_ctor_set(x_182, 13, x_15); -lean_ctor_set(x_182, 14, x_16); -lean_ctor_set(x_182, 15, x_17); -lean_ctor_set(x_182, 16, x_18); -lean_ctor_set(x_182, 17, x_19); -lean_ctor_set(x_182, 18, x_20); -lean_ctor_set(x_182, 19, x_21); -lean_ctor_set_uint8(x_182, sizeof(void*)*20, x_7); -x_183 = lean_alloc_ctor(2, 1, 0); -lean_ctor_set(x_183, 0, x_182); -x_184 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_184, 0, x_183); -lean_ctor_set(x_184, 1, x_181); -return x_184; -} -} -else -{ -uint8_t x_185; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_185 = !lean_is_exclusive(x_175); -if (x_185 == 0) -{ -return x_175; } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_186 = lean_ctor_get(x_175, 0); -x_187 = lean_ctor_get(x_175, 1); -lean_inc(x_187); -lean_inc(x_186); -lean_dec(x_175); -x_188 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_188, 0, x_186); -lean_ctor_set(x_188, 1, x_187); -return x_188; -} -} -} -} -else +lean_object* x_11; lean_object* x_12; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_22 = lean_st_ref_get(x_2, x_10); +x_23 = lean_ctor_get(x_22, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Lean_Expr_bindingDomain_x21(x_1); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_26); +x_27 = l_Lean_Meta_isProp(x_26, x_6, x_7, x_8, x_9, x_24); +if (lean_obj_tag(x_27) == 0) { -uint8_t x_189; -lean_dec(x_35); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_unbox(x_28); lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_23); -lean_dec(x_22); -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_6); +if (x_29 == 0) +{ +lean_object* x_30; uint8_t x_31; lean_object* x_32; +lean_dec(x_26); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_189 = !lean_is_exclusive(x_36); -if (x_189 == 0) +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = 1; +x_32 = l_Lean_Meta_intro1Core(x_25, x_31, x_6, x_7, x_8, x_9, x_30); +if (lean_obj_tag(x_32) == 0) { -return x_36; -} -else +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +x_34 = lean_ctor_get(x_32, 1); +lean_inc(x_34); +lean_dec(x_32); +x_35 = lean_ctor_get(x_33, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_33, 1); +lean_inc(x_36); +lean_dec(x_33); +x_37 = lean_st_ref_get(x_2, x_34); +x_38 = !lean_is_exclusive(x_37); +if (x_38 == 0) { -lean_object* x_190; lean_object* x_191; lean_object* x_192; -x_190 = lean_ctor_get(x_36, 0); -x_191 = lean_ctor_get(x_36, 1); -lean_inc(x_191); -lean_inc(x_190); -lean_dec(x_36); -x_192 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_192, 0, x_190); -lean_ctor_set(x_192, 1, x_191); -return x_192; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +lean_object* x_39; uint8_t x_40; +x_39 = lean_ctor_get(x_37, 0); +x_40 = !lean_is_exclusive(x_39); +if (x_40 == 0) { -lean_object* x_10; -x_10 = l_Lean_Meta_isProp(x_1, x_5, x_6, x_7, x_8, x_9); -return x_10; -} +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_37, 1); +x_42 = lean_ctor_get(x_39, 0); +lean_dec(x_42); +lean_ctor_set(x_39, 0, x_36); +lean_ctor_set_tag(x_37, 3); +lean_ctor_set(x_37, 1, x_39); +lean_ctor_set(x_37, 0, x_35); +x_11 = x_37; +x_12 = x_41; +goto block_21; +} +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_43 = lean_ctor_get(x_37, 1); +x_44 = lean_ctor_get(x_39, 1); +x_45 = lean_ctor_get(x_39, 2); +x_46 = lean_ctor_get(x_39, 3); +x_47 = lean_ctor_get(x_39, 4); +x_48 = lean_ctor_get(x_39, 5); +x_49 = lean_ctor_get(x_39, 6); +x_50 = lean_ctor_get_uint8(x_39, sizeof(void*)*23); +x_51 = lean_ctor_get(x_39, 7); +x_52 = lean_ctor_get(x_39, 8); +x_53 = lean_ctor_get(x_39, 9); +x_54 = lean_ctor_get(x_39, 10); +x_55 = lean_ctor_get(x_39, 11); +x_56 = lean_ctor_get(x_39, 12); +x_57 = lean_ctor_get(x_39, 13); +x_58 = lean_ctor_get(x_39, 14); +x_59 = lean_ctor_get(x_39, 15); +x_60 = lean_ctor_get(x_39, 16); +x_61 = lean_ctor_get(x_39, 17); +x_62 = lean_ctor_get(x_39, 18); +x_63 = lean_ctor_get(x_39, 19); +x_64 = lean_ctor_get(x_39, 20); +x_65 = lean_ctor_get(x_39, 21); +x_66 = lean_ctor_get(x_39, 22); +lean_inc(x_66); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_39); +x_67 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_67, 0, x_36); +lean_ctor_set(x_67, 1, x_44); +lean_ctor_set(x_67, 2, x_45); +lean_ctor_set(x_67, 3, x_46); +lean_ctor_set(x_67, 4, x_47); +lean_ctor_set(x_67, 5, x_48); +lean_ctor_set(x_67, 6, x_49); +lean_ctor_set(x_67, 7, x_51); +lean_ctor_set(x_67, 8, x_52); +lean_ctor_set(x_67, 9, x_53); +lean_ctor_set(x_67, 10, x_54); +lean_ctor_set(x_67, 11, x_55); +lean_ctor_set(x_67, 12, x_56); +lean_ctor_set(x_67, 13, x_57); +lean_ctor_set(x_67, 14, x_58); +lean_ctor_set(x_67, 15, x_59); +lean_ctor_set(x_67, 16, x_60); +lean_ctor_set(x_67, 17, x_61); +lean_ctor_set(x_67, 18, x_62); +lean_ctor_set(x_67, 19, x_63); +lean_ctor_set(x_67, 20, x_64); +lean_ctor_set(x_67, 21, x_65); +lean_ctor_set(x_67, 22, x_66); +lean_ctor_set_uint8(x_67, sizeof(void*)*23, x_50); +lean_ctor_set_tag(x_37, 3); +lean_ctor_set(x_37, 1, x_67); +lean_ctor_set(x_37, 0, x_35); +x_11 = x_37; +x_12 = x_43; +goto block_21; +} +} +else +{ +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_68 = lean_ctor_get(x_37, 0); +x_69 = lean_ctor_get(x_37, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_37); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +x_71 = lean_ctor_get(x_68, 2); +lean_inc(x_71); +x_72 = lean_ctor_get(x_68, 3); +lean_inc(x_72); +x_73 = lean_ctor_get(x_68, 4); +lean_inc(x_73); +x_74 = lean_ctor_get(x_68, 5); +lean_inc(x_74); +x_75 = lean_ctor_get(x_68, 6); +lean_inc(x_75); +x_76 = lean_ctor_get_uint8(x_68, sizeof(void*)*23); +x_77 = lean_ctor_get(x_68, 7); +lean_inc(x_77); +x_78 = lean_ctor_get(x_68, 8); +lean_inc(x_78); +x_79 = lean_ctor_get(x_68, 9); +lean_inc(x_79); +x_80 = lean_ctor_get(x_68, 10); +lean_inc(x_80); +x_81 = lean_ctor_get(x_68, 11); +lean_inc(x_81); +x_82 = lean_ctor_get(x_68, 12); +lean_inc(x_82); +x_83 = lean_ctor_get(x_68, 13); +lean_inc(x_83); +x_84 = lean_ctor_get(x_68, 14); +lean_inc(x_84); +x_85 = lean_ctor_get(x_68, 15); +lean_inc(x_85); +x_86 = lean_ctor_get(x_68, 16); +lean_inc(x_86); +x_87 = lean_ctor_get(x_68, 17); +lean_inc(x_87); +x_88 = lean_ctor_get(x_68, 18); +lean_inc(x_88); +x_89 = lean_ctor_get(x_68, 19); +lean_inc(x_89); +x_90 = lean_ctor_get(x_68, 20); +lean_inc(x_90); +x_91 = lean_ctor_get(x_68, 21); +lean_inc(x_91); +x_92 = lean_ctor_get(x_68, 22); +lean_inc(x_92); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + lean_ctor_release(x_68, 2); + lean_ctor_release(x_68, 3); + lean_ctor_release(x_68, 4); + lean_ctor_release(x_68, 5); + lean_ctor_release(x_68, 6); + lean_ctor_release(x_68, 7); + lean_ctor_release(x_68, 8); + lean_ctor_release(x_68, 9); + lean_ctor_release(x_68, 10); + lean_ctor_release(x_68, 11); + lean_ctor_release(x_68, 12); + lean_ctor_release(x_68, 13); + lean_ctor_release(x_68, 14); + lean_ctor_release(x_68, 15); + lean_ctor_release(x_68, 16); + lean_ctor_release(x_68, 17); + lean_ctor_release(x_68, 18); + lean_ctor_release(x_68, 19); + lean_ctor_release(x_68, 20); + lean_ctor_release(x_68, 21); + lean_ctor_release(x_68, 22); + x_93 = x_68; +} else { + lean_dec_ref(x_68); + x_93 = lean_box(0); } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; uint8_t x_12; uint8_t x_13; lean_object* x_14; -x_11 = 0; -x_12 = 1; -x_13 = 1; -x_14 = l_Lean_Meta_mkLambdaFVars(x_1, x_2, x_11, x_12, x_11, x_13, x_6, x_7, x_8, x_9, x_10); -return x_14; +if (lean_is_scalar(x_93)) { + x_94 = lean_alloc_ctor(0, 23, 1); +} else { + x_94 = x_93; +} +lean_ctor_set(x_94, 0, x_36); +lean_ctor_set(x_94, 1, x_70); +lean_ctor_set(x_94, 2, x_71); +lean_ctor_set(x_94, 3, x_72); +lean_ctor_set(x_94, 4, x_73); +lean_ctor_set(x_94, 5, x_74); +lean_ctor_set(x_94, 6, x_75); +lean_ctor_set(x_94, 7, x_77); +lean_ctor_set(x_94, 8, x_78); +lean_ctor_set(x_94, 9, x_79); +lean_ctor_set(x_94, 10, x_80); +lean_ctor_set(x_94, 11, x_81); +lean_ctor_set(x_94, 12, x_82); +lean_ctor_set(x_94, 13, x_83); +lean_ctor_set(x_94, 14, x_84); +lean_ctor_set(x_94, 15, x_85); +lean_ctor_set(x_94, 16, x_86); +lean_ctor_set(x_94, 17, x_87); +lean_ctor_set(x_94, 18, x_88); +lean_ctor_set(x_94, 19, x_89); +lean_ctor_set(x_94, 20, x_90); +lean_ctor_set(x_94, 21, x_91); +lean_ctor_set(x_94, 22, x_92); +lean_ctor_set_uint8(x_94, sizeof(void*)*23, x_76); +x_95 = lean_alloc_ctor(3, 2, 0); +lean_ctor_set(x_95, 0, x_35); +lean_ctor_set(x_95, 1, x_94); +x_11 = x_95; +x_12 = x_69; +goto block_21; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2() { -_start: +uint8_t x_96; +lean_dec(x_2); +x_96 = !lean_is_exclusive(x_32); +if (x_96 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Grind", 5, 5); -return x_1; -} +return x_32; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("intro_with_eq", 13, 13); -return x_1; -} +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_32, 0); +x_98 = lean_ctor_get(x_32, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_32); +x_99 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_99, 0, x_97); +lean_ctor_set(x_99, 1, x_98); +return x_99; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2; -x_3 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24, lean_object* x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32, lean_object* x_33, lean_object* x_34, lean_object* x_35, lean_object* x_36, lean_object* x_37) { -_start: -{ -if (lean_obj_tag(x_1) == 0) +else { -lean_object* x_38; uint8_t x_39; -lean_dec(x_28); +lean_object* x_100; lean_object* x_101; +x_100 = lean_ctor_get(x_27, 1); +lean_inc(x_100); lean_dec(x_27); -lean_dec(x_26); -lean_dec(x_25); -x_38 = l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(x_2, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_37); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +lean_inc(x_25); +x_101 = l_Lean_MVarId_getTag(x_25, x_6, x_7, x_8, x_9, x_100); +if (lean_obj_tag(x_101) == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_38, 0); -lean_dec(x_40); -x_41 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_41, 0, x_3); -lean_ctor_set(x_41, 1, x_4); -lean_ctor_set(x_41, 2, x_5); -lean_ctor_set(x_41, 3, x_6); -lean_ctor_set(x_41, 4, x_7); -lean_ctor_set(x_41, 5, x_8); -lean_ctor_set(x_41, 6, x_10); -lean_ctor_set(x_41, 7, x_11); -lean_ctor_set(x_41, 8, x_12); -lean_ctor_set(x_41, 9, x_13); -lean_ctor_set(x_41, 10, x_14); -lean_ctor_set(x_41, 11, x_15); -lean_ctor_set(x_41, 12, x_16); -lean_ctor_set(x_41, 13, x_17); -lean_ctor_set(x_41, 14, x_18); -lean_ctor_set(x_41, 15, x_19); -lean_ctor_set(x_41, 16, x_20); -lean_ctor_set(x_41, 17, x_21); -lean_ctor_set(x_41, 18, x_22); -lean_ctor_set(x_41, 19, x_23); -lean_ctor_set_uint8(x_41, sizeof(void*)*20, x_9); -x_42 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_42, 0, x_24); -lean_ctor_set(x_42, 1, x_41); -lean_ctor_set(x_38, 0, x_42); -return x_38; -} -else +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_102 = lean_ctor_get(x_101, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_101, 1); +lean_inc(x_103); +lean_dec(x_101); +x_104 = l_Lean_Expr_bindingBody_x21(x_1); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_4); +lean_inc(x_26); +x_105 = l_Lean_Meta_Grind_simp(x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_103); +if (lean_obj_tag(x_105) == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_43 = lean_ctor_get(x_38, 1); -lean_inc(x_43); -lean_dec(x_38); -x_44 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_44, 0, x_3); -lean_ctor_set(x_44, 1, x_4); -lean_ctor_set(x_44, 2, x_5); -lean_ctor_set(x_44, 3, x_6); -lean_ctor_set(x_44, 4, x_7); -lean_ctor_set(x_44, 5, x_8); -lean_ctor_set(x_44, 6, x_10); -lean_ctor_set(x_44, 7, x_11); -lean_ctor_set(x_44, 8, x_12); -lean_ctor_set(x_44, 9, x_13); -lean_ctor_set(x_44, 10, x_14); -lean_ctor_set(x_44, 11, x_15); -lean_ctor_set(x_44, 12, x_16); -lean_ctor_set(x_44, 13, x_17); -lean_ctor_set(x_44, 14, x_18); -lean_ctor_set(x_44, 15, x_19); -lean_ctor_set(x_44, 16, x_20); -lean_ctor_set(x_44, 17, x_21); -lean_ctor_set(x_44, 18, x_22); -lean_ctor_set(x_44, 19, x_23); -lean_ctor_set_uint8(x_44, sizeof(void*)*20, x_9); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_24); -lean_ctor_set(x_45, 1, x_44); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_45); -lean_ctor_set(x_46, 1, x_43); -return x_46; -} +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; uint8_t x_116; uint8_t x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +lean_dec(x_105); +x_108 = l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_107); +x_109 = lean_ctor_get(x_108, 0); +lean_inc(x_109); +x_110 = lean_ctor_get(x_108, 1); +lean_inc(x_110); +lean_dec(x_108); +x_111 = lean_ctor_get(x_6, 2); +lean_inc(x_111); +x_112 = l_Lean_Expr_bindingName_x21(x_1); +x_113 = lean_ctor_get(x_106, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_106, 1); +lean_inc(x_114); +lean_dec(x_106); +x_115 = l_Lean_Expr_bindingInfo_x21(x_1); +x_116 = lean_unbox(x_115); +lean_dec(x_115); +x_117 = 0; +lean_inc(x_113); +lean_inc(x_109); +x_118 = l_Lean_LocalContext_mkLocalDecl(x_111, x_109, x_112, x_113, x_116, x_117); +x_119 = l_Lean_Meta_getLocalInstances(x_6, x_7, x_8, x_9, x_110); +x_120 = lean_ctor_get(x_119, 0); +lean_inc(x_120); +x_121 = lean_ctor_get(x_119, 1); +lean_inc(x_121); +lean_dec(x_119); +x_122 = 2; +x_123 = lean_unsigned_to_nat(0u); +lean_inc(x_104); +x_124 = l_Lean_Meta_mkFreshExprMVarAt(x_118, x_120, x_104, x_122, x_102, x_123, x_6, x_7, x_8, x_9, x_121); +x_125 = !lean_is_exclusive(x_124); +if (x_125 == 0) +{ +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +x_126 = lean_ctor_get(x_124, 0); +x_127 = lean_ctor_get(x_124, 1); +x_128 = l_Lean_Expr_mvarId_x21(x_126); +lean_inc(x_109); +x_129 = l_Lean_Expr_fvar___override(x_109); +x_130 = lean_box(0); +lean_ctor_set_tag(x_124, 1); +lean_ctor_set(x_124, 1, x_130); +lean_ctor_set(x_124, 0, x_129); +x_131 = lean_array_mk(x_124); +x_132 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed), 10, 2); +lean_closure_set(x_132, 0, x_131); +lean_closure_set(x_132, 1, x_126); +x_133 = lean_alloc_closure((void*)(l_StateRefT_x27_lift___rarg___boxed), 2, 1); +lean_closure_set(x_133, 0, x_132); +lean_inc(x_128); +x_134 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed), 18, 8); +lean_closure_set(x_134, 0, x_114); +lean_closure_set(x_134, 1, x_25); +lean_closure_set(x_134, 2, x_128); +lean_closure_set(x_134, 3, x_109); +lean_closure_set(x_134, 4, x_130); +lean_closure_set(x_134, 5, x_104); +lean_closure_set(x_134, 6, x_113); +lean_closure_set(x_134, 7, x_26); +x_135 = lean_alloc_closure((void*)(l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___rarg), 11, 2); +lean_closure_set(x_135, 0, x_133); +lean_closure_set(x_135, 1, x_134); +lean_inc(x_2); +x_136 = l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4___rarg(x_128, x_135, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_127); +if (lean_obj_tag(x_136) == 0) +{ +lean_object* x_137; lean_object* x_138; +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +x_138 = lean_ctor_get(x_136, 1); +lean_inc(x_138); +lean_dec(x_136); +x_11 = x_137; +x_12 = x_138; +goto block_21; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; -x_47 = lean_ctor_get(x_1, 0); -x_48 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4; -lean_inc(x_25); -x_49 = l_Lean_Expr_const___override(x_48, x_25); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_29); -lean_ctor_set(x_50, 1, x_25); -lean_inc(x_47); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_47); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_26); -lean_ctor_set(x_52, 1, x_51); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_27); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_28); -lean_ctor_set(x_54, 1, x_53); -x_55 = lean_array_mk(x_54); -x_56 = l_Lean_mkAppN(x_49, x_55); -lean_dec(x_55); -x_57 = l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(x_2, x_56, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_37); -x_58 = !lean_is_exclusive(x_57); -if (x_58 == 0) +uint8_t x_139; +lean_dec(x_2); +x_139 = !lean_is_exclusive(x_136); +if (x_139 == 0) { -lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_59 = lean_ctor_get(x_57, 0); -lean_dec(x_59); -x_60 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_60, 0, x_3); -lean_ctor_set(x_60, 1, x_4); -lean_ctor_set(x_60, 2, x_5); -lean_ctor_set(x_60, 3, x_6); -lean_ctor_set(x_60, 4, x_7); -lean_ctor_set(x_60, 5, x_8); -lean_ctor_set(x_60, 6, x_10); -lean_ctor_set(x_60, 7, x_11); -lean_ctor_set(x_60, 8, x_12); -lean_ctor_set(x_60, 9, x_13); -lean_ctor_set(x_60, 10, x_14); -lean_ctor_set(x_60, 11, x_15); -lean_ctor_set(x_60, 12, x_16); -lean_ctor_set(x_60, 13, x_17); -lean_ctor_set(x_60, 14, x_18); -lean_ctor_set(x_60, 15, x_19); -lean_ctor_set(x_60, 16, x_20); -lean_ctor_set(x_60, 17, x_21); -lean_ctor_set(x_60, 18, x_22); -lean_ctor_set(x_60, 19, x_23); -lean_ctor_set_uint8(x_60, sizeof(void*)*20, x_9); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_24); -lean_ctor_set(x_61, 1, x_60); -lean_ctor_set(x_57, 0, x_61); -return x_57; +return x_136; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_62 = lean_ctor_get(x_57, 1); -lean_inc(x_62); -lean_dec(x_57); -x_63 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_63, 0, x_3); -lean_ctor_set(x_63, 1, x_4); -lean_ctor_set(x_63, 2, x_5); -lean_ctor_set(x_63, 3, x_6); -lean_ctor_set(x_63, 4, x_7); -lean_ctor_set(x_63, 5, x_8); -lean_ctor_set(x_63, 6, x_10); -lean_ctor_set(x_63, 7, x_11); -lean_ctor_set(x_63, 8, x_12); -lean_ctor_set(x_63, 9, x_13); -lean_ctor_set(x_63, 10, x_14); -lean_ctor_set(x_63, 11, x_15); -lean_ctor_set(x_63, 12, x_16); -lean_ctor_set(x_63, 13, x_17); -lean_ctor_set(x_63, 14, x_18); -lean_ctor_set(x_63, 15, x_19); -lean_ctor_set(x_63, 16, x_20); -lean_ctor_set(x_63, 17, x_21); -lean_ctor_set(x_63, 18, x_22); -lean_ctor_set(x_63, 19, x_23); -lean_ctor_set_uint8(x_63, sizeof(void*)*20, x_9); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_24); -lean_ctor_set(x_64, 1, x_63); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -return x_65; -} +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_136, 0); +x_141 = lean_ctor_get(x_136, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_136); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, uint8_t x_24, lean_object* x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32) { -_start: -{ -if (x_24 == 0) -{ -uint8_t x_33; lean_object* x_34; -lean_dec(x_27); -lean_dec(x_26); -lean_dec(x_25); -lean_dec(x_23); -x_33 = 1; -x_34 = l_Lean_Meta_intro1Core(x_1, x_33, x_28, x_29, x_30, x_31, x_32); -if (lean_obj_tag(x_34) == 0) -{ -uint8_t x_35; -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) -{ -lean_object* x_36; uint8_t x_37; -x_36 = lean_ctor_get(x_34, 0); -x_37 = !lean_is_exclusive(x_36); -if (x_37 == 0) -{ -lean_object* x_38; lean_object* x_39; -x_38 = lean_ctor_get(x_36, 1); -x_39 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_2); -lean_ctor_set(x_39, 2, x_3); -lean_ctor_set(x_39, 3, x_4); -lean_ctor_set(x_39, 4, x_5); -lean_ctor_set(x_39, 5, x_6); -lean_ctor_set(x_39, 6, x_8); -lean_ctor_set(x_39, 7, x_9); -lean_ctor_set(x_39, 8, x_10); -lean_ctor_set(x_39, 9, x_11); -lean_ctor_set(x_39, 10, x_12); -lean_ctor_set(x_39, 11, x_13); -lean_ctor_set(x_39, 12, x_14); -lean_ctor_set(x_39, 13, x_15); -lean_ctor_set(x_39, 14, x_16); -lean_ctor_set(x_39, 15, x_17); -lean_ctor_set(x_39, 16, x_18); -lean_ctor_set(x_39, 17, x_19); -lean_ctor_set(x_39, 18, x_20); -lean_ctor_set(x_39, 19, x_21); -lean_ctor_set_uint8(x_39, sizeof(void*)*20, x_7); -lean_ctor_set_tag(x_36, 3); -lean_ctor_set(x_36, 1, x_39); -return x_34; -} else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_36, 0); -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_36); -x_42 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_2); -lean_ctor_set(x_42, 2, x_3); -lean_ctor_set(x_42, 3, x_4); -lean_ctor_set(x_42, 4, x_5); -lean_ctor_set(x_42, 5, x_6); -lean_ctor_set(x_42, 6, x_8); -lean_ctor_set(x_42, 7, x_9); -lean_ctor_set(x_42, 8, x_10); -lean_ctor_set(x_42, 9, x_11); -lean_ctor_set(x_42, 10, x_12); -lean_ctor_set(x_42, 11, x_13); -lean_ctor_set(x_42, 12, x_14); -lean_ctor_set(x_42, 13, x_15); -lean_ctor_set(x_42, 14, x_16); -lean_ctor_set(x_42, 15, x_17); -lean_ctor_set(x_42, 16, x_18); -lean_ctor_set(x_42, 17, x_19); -lean_ctor_set(x_42, 18, x_20); -lean_ctor_set(x_42, 19, x_21); -lean_ctor_set_uint8(x_42, sizeof(void*)*20, x_7); -x_43 = lean_alloc_ctor(3, 2, 0); -lean_ctor_set(x_43, 0, x_40); -lean_ctor_set(x_43, 1, x_42); -lean_ctor_set(x_34, 0, x_43); -return x_34; -} +lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_143 = lean_ctor_get(x_124, 0); +x_144 = lean_ctor_get(x_124, 1); +lean_inc(x_144); +lean_inc(x_143); +lean_dec(x_124); +x_145 = l_Lean_Expr_mvarId_x21(x_143); +lean_inc(x_109); +x_146 = l_Lean_Expr_fvar___override(x_109); +x_147 = lean_box(0); +x_148 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_148, 0, x_146); +lean_ctor_set(x_148, 1, x_147); +x_149 = lean_array_mk(x_148); +x_150 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed), 10, 2); +lean_closure_set(x_150, 0, x_149); +lean_closure_set(x_150, 1, x_143); +x_151 = lean_alloc_closure((void*)(l_StateRefT_x27_lift___rarg___boxed), 2, 1); +lean_closure_set(x_151, 0, x_150); +lean_inc(x_145); +x_152 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed), 18, 8); +lean_closure_set(x_152, 0, x_114); +lean_closure_set(x_152, 1, x_25); +lean_closure_set(x_152, 2, x_145); +lean_closure_set(x_152, 3, x_109); +lean_closure_set(x_152, 4, x_147); +lean_closure_set(x_152, 5, x_104); +lean_closure_set(x_152, 6, x_113); +lean_closure_set(x_152, 7, x_26); +x_153 = lean_alloc_closure((void*)(l_ReaderT_bind___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___rarg), 11, 2); +lean_closure_set(x_153, 0, x_151); +lean_closure_set(x_153, 1, x_152); +lean_inc(x_2); +x_154 = l_Lean_MVarId_withContext___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__4___rarg(x_145, x_153, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_144); +if (lean_obj_tag(x_154) == 0) +{ +lean_object* x_155; lean_object* x_156; +x_155 = lean_ctor_get(x_154, 0); +lean_inc(x_155); +x_156 = lean_ctor_get(x_154, 1); +lean_inc(x_156); +lean_dec(x_154); +x_11 = x_155; +x_12 = x_156; +goto block_21; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_44 = lean_ctor_get(x_34, 0); -x_45 = lean_ctor_get(x_34, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_34); -x_46 = lean_ctor_get(x_44, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_44, 1); -lean_inc(x_47); -if (lean_is_exclusive(x_44)) { - lean_ctor_release(x_44, 0); - lean_ctor_release(x_44, 1); - x_48 = x_44; +lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; +lean_dec(x_2); +x_157 = lean_ctor_get(x_154, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_154, 1); +lean_inc(x_158); +if (lean_is_exclusive(x_154)) { + lean_ctor_release(x_154, 0); + lean_ctor_release(x_154, 1); + x_159 = x_154; } else { - lean_dec_ref(x_44); - x_48 = lean_box(0); -} -x_49 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_2); -lean_ctor_set(x_49, 2, x_3); -lean_ctor_set(x_49, 3, x_4); -lean_ctor_set(x_49, 4, x_5); -lean_ctor_set(x_49, 5, x_6); -lean_ctor_set(x_49, 6, x_8); -lean_ctor_set(x_49, 7, x_9); -lean_ctor_set(x_49, 8, x_10); -lean_ctor_set(x_49, 9, x_11); -lean_ctor_set(x_49, 10, x_12); -lean_ctor_set(x_49, 11, x_13); -lean_ctor_set(x_49, 12, x_14); -lean_ctor_set(x_49, 13, x_15); -lean_ctor_set(x_49, 14, x_16); -lean_ctor_set(x_49, 15, x_17); -lean_ctor_set(x_49, 16, x_18); -lean_ctor_set(x_49, 17, x_19); -lean_ctor_set(x_49, 18, x_20); -lean_ctor_set(x_49, 19, x_21); -lean_ctor_set_uint8(x_49, sizeof(void*)*20, x_7); -if (lean_is_scalar(x_48)) { - x_50 = lean_alloc_ctor(3, 2, 0); + lean_dec_ref(x_154); + x_159 = lean_box(0); +} +if (lean_is_scalar(x_159)) { + x_160 = lean_alloc_ctor(1, 2, 0); } else { - x_50 = x_48; - lean_ctor_set_tag(x_50, 3); + x_160 = x_159; +} +lean_ctor_set(x_160, 0, x_157); +lean_ctor_set(x_160, 1, x_158); +return x_160; } -lean_ctor_set(x_50, 0, x_46); -lean_ctor_set(x_50, 1, x_49); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_45); -return x_51; } } else { -uint8_t x_52; -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_161; +lean_dec(x_104); +lean_dec(x_102); +lean_dec(x_26); +lean_dec(x_25); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_52 = !lean_is_exclusive(x_34); -if (x_52 == 0) -{ -return x_34; -} -else +x_161 = !lean_is_exclusive(x_105); +if (x_161 == 0) { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_34, 0); -x_54 = lean_ctor_get(x_34, 1); -lean_inc(x_54); -lean_inc(x_53); -lean_dec(x_34); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); -return x_55; -} -} +return x_105; } else { -lean_object* x_56; -lean_inc(x_1); -x_56 = l_Lean_MVarId_getTag(x_1, x_28, x_29, x_30, x_31, x_32); -if (lean_obj_tag(x_56) == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = l_Lean_Expr_bindingBody_x21(x_22); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_26); -lean_inc(x_23); -x_60 = l_Lean_Meta_Grind_simp(x_23, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_58); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; uint8_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_63 = l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_62); -x_64 = lean_ctor_get(x_63, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_63, 1); -lean_inc(x_65); -lean_dec(x_63); -x_66 = lean_ctor_get(x_28, 2); -lean_inc(x_66); -x_67 = l_Lean_Expr_bindingName_x21(x_22); -x_68 = lean_ctor_get(x_61, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_61, 1); -lean_inc(x_69); -lean_dec(x_61); -x_70 = l_Lean_Expr_bindingInfo_x21(x_22); -x_71 = lean_unbox(x_70); -lean_dec(x_70); -x_72 = 0; -lean_inc(x_68); -lean_inc(x_64); -x_73 = l_Lean_LocalContext_mkLocalDecl(x_66, x_64, x_67, x_68, x_71, x_72); -x_74 = l_Lean_Meta_getLocalInstances(x_28, x_29, x_30, x_31, x_65); -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = 2; -x_78 = lean_unsigned_to_nat(0u); -lean_inc(x_59); -x_79 = l_Lean_Meta_mkFreshExprMVarAt(x_73, x_75, x_59, x_77, x_57, x_78, x_28, x_29, x_30, x_31, x_76); -x_80 = !lean_is_exclusive(x_79); -if (x_80 == 0) -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_81 = lean_ctor_get(x_79, 0); -x_82 = lean_ctor_get(x_79, 1); -x_83 = l_Lean_Expr_mvarId_x21(x_81); -lean_inc(x_64); -x_84 = l_Lean_Expr_fvar___override(x_64); -x_85 = lean_box(0); -lean_ctor_set_tag(x_79, 1); -lean_ctor_set(x_79, 1, x_85); -lean_ctor_set(x_79, 0, x_84); -x_86 = lean_array_mk(x_79); -x_87 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed), 10, 2); -lean_closure_set(x_87, 0, x_86); -lean_closure_set(x_87, 1, x_81); -x_88 = lean_box(x_7); -lean_inc(x_83); -x_89 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed), 37, 28); -lean_closure_set(x_89, 0, x_69); -lean_closure_set(x_89, 1, x_1); -lean_closure_set(x_89, 2, x_83); -lean_closure_set(x_89, 3, x_2); -lean_closure_set(x_89, 4, x_3); -lean_closure_set(x_89, 5, x_4); -lean_closure_set(x_89, 6, x_5); -lean_closure_set(x_89, 7, x_6); -lean_closure_set(x_89, 8, x_88); -lean_closure_set(x_89, 9, x_8); -lean_closure_set(x_89, 10, x_9); -lean_closure_set(x_89, 11, x_10); -lean_closure_set(x_89, 12, x_11); -lean_closure_set(x_89, 13, x_12); -lean_closure_set(x_89, 14, x_13); -lean_closure_set(x_89, 15, x_14); -lean_closure_set(x_89, 16, x_15); -lean_closure_set(x_89, 17, x_16); -lean_closure_set(x_89, 18, x_17); -lean_closure_set(x_89, 19, x_18); -lean_closure_set(x_89, 20, x_19); -lean_closure_set(x_89, 21, x_20); -lean_closure_set(x_89, 22, x_21); -lean_closure_set(x_89, 23, x_64); -lean_closure_set(x_89, 24, x_85); -lean_closure_set(x_89, 25, x_59); -lean_closure_set(x_89, 26, x_68); -lean_closure_set(x_89, 27, x_23); -x_90 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_90, 0, x_87); -lean_closure_set(x_90, 1, x_89); -x_91 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_83, x_90, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_82); -return x_91; +lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_162 = lean_ctor_get(x_105, 0); +x_163 = lean_ctor_get(x_105, 1); +lean_inc(x_163); +lean_inc(x_162); +lean_dec(x_105); +x_164 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_164, 0, x_162); +lean_ctor_set(x_164, 1, x_163); +return x_164; } -else -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_92 = lean_ctor_get(x_79, 0); -x_93 = lean_ctor_get(x_79, 1); -lean_inc(x_93); -lean_inc(x_92); -lean_dec(x_79); -x_94 = l_Lean_Expr_mvarId_x21(x_92); -lean_inc(x_64); -x_95 = l_Lean_Expr_fvar___override(x_64); -x_96 = lean_box(0); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -x_98 = lean_array_mk(x_97); -x_99 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed), 10, 2); -lean_closure_set(x_99, 0, x_98); -lean_closure_set(x_99, 1, x_92); -x_100 = lean_box(x_7); -lean_inc(x_94); -x_101 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed), 37, 28); -lean_closure_set(x_101, 0, x_69); -lean_closure_set(x_101, 1, x_1); -lean_closure_set(x_101, 2, x_94); -lean_closure_set(x_101, 3, x_2); -lean_closure_set(x_101, 4, x_3); -lean_closure_set(x_101, 5, x_4); -lean_closure_set(x_101, 6, x_5); -lean_closure_set(x_101, 7, x_6); -lean_closure_set(x_101, 8, x_100); -lean_closure_set(x_101, 9, x_8); -lean_closure_set(x_101, 10, x_9); -lean_closure_set(x_101, 11, x_10); -lean_closure_set(x_101, 12, x_11); -lean_closure_set(x_101, 13, x_12); -lean_closure_set(x_101, 14, x_13); -lean_closure_set(x_101, 15, x_14); -lean_closure_set(x_101, 16, x_15); -lean_closure_set(x_101, 17, x_16); -lean_closure_set(x_101, 18, x_17); -lean_closure_set(x_101, 19, x_18); -lean_closure_set(x_101, 20, x_19); -lean_closure_set(x_101, 21, x_20); -lean_closure_set(x_101, 22, x_21); -lean_closure_set(x_101, 23, x_64); -lean_closure_set(x_101, 24, x_96); -lean_closure_set(x_101, 25, x_59); -lean_closure_set(x_101, 26, x_68); -lean_closure_set(x_101, 27, x_23); -x_102 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_102, 0, x_99); -lean_closure_set(x_102, 1, x_101); -x_103 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_94, x_102, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_93); -return x_103; } } else { -uint8_t x_104; -lean_dec(x_59); -lean_dec(x_57); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); +uint8_t x_165; lean_dec(x_26); lean_dec(x_25); -lean_dec(x_23); -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_104 = !lean_is_exclusive(x_60); -if (x_104 == 0) +x_165 = !lean_is_exclusive(x_101); +if (x_165 == 0) { -return x_60; +return x_101; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_60, 0); -x_106 = lean_ctor_get(x_60, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_60); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_166 = lean_ctor_get(x_101, 0); +x_167 = lean_ctor_get(x_101, 1); +lean_inc(x_167); +lean_inc(x_166); +lean_dec(x_101); +x_168 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_168, 0, x_166); +lean_ctor_set(x_168, 1, x_167); +return x_168; +} } } } else { -uint8_t x_108; -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); +uint8_t x_169; lean_dec(x_26); lean_dec(x_25); -lean_dec(x_23); -lean_dec(x_21); -lean_dec(x_20); -lean_dec(x_19); -lean_dec(x_18); -lean_dec(x_17); -lean_dec(x_16); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); +lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_108 = !lean_is_exclusive(x_56); -if (x_108 == 0) +x_169 = !lean_is_exclusive(x_27); +if (x_169 == 0) { -return x_56; +return x_27; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_56, 0); -x_110 = lean_ctor_get(x_56, 1); -lean_inc(x_110); -lean_inc(x_109); -lean_dec(x_56); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +lean_object* x_170; lean_object* x_171; lean_object* x_172; +x_170 = lean_ctor_get(x_27, 0); +x_171 = lean_ctor_get(x_27, 1); +lean_inc(x_171); +lean_inc(x_170); +lean_dec(x_27); +x_172 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_172, 0, x_170); +lean_ctor_set(x_172, 1, x_171); +return x_172; +} +} +block_21: +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_st_ref_get(x_2, x_12); +lean_dec(x_2); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_11); +lean_ctor_set(x_16, 1, x_15); +lean_ctor_set(x_13, 0, x_16); +return x_13; } +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_13, 0); +x_18 = lean_ctor_get(x_13, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_13); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_11); +lean_ctor_set(x_19, 1, x_17); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +return x_20; } } } @@ -2395,7 +2894,7 @@ return x_111; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; x_11 = lean_ctor_get(x_1, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_1, 1); @@ -2408,9 +2907,9 @@ x_15 = lean_ctor_get(x_1, 4); lean_inc(x_15); x_16 = lean_ctor_get(x_1, 5); lean_inc(x_16); -x_17 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_18 = lean_ctor_get(x_1, 6); -lean_inc(x_18); +x_17 = lean_ctor_get(x_1, 6); +lean_inc(x_17); +x_18 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); x_19 = lean_ctor_get(x_1, 7); lean_inc(x_19); x_20 = lean_ctor_get(x_1, 8); @@ -2437,35 +2936,44 @@ x_30 = lean_ctor_get(x_1, 18); lean_inc(x_30); x_31 = lean_ctor_get(x_1, 19); lean_inc(x_31); -lean_dec(x_1); +x_32 = lean_ctor_get(x_1, 20); +lean_inc(x_32); +x_33 = lean_ctor_get(x_1, 21); +lean_inc(x_33); +x_34 = lean_ctor_get(x_1, 22); +lean_inc(x_34); lean_inc(x_11); -x_32 = l_Lean_MVarId_getType(x_11, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_32) == 0) -{ -uint8_t x_33; -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) +x_35 = l_Lean_MVarId_getType(x_11, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_34 = lean_ctor_get(x_32, 0); -x_35 = lean_ctor_get(x_32, 1); -x_36 = l_Lean_Expr_isArrow(x_34); +uint8_t x_36; +x_36 = !lean_is_exclusive(x_35); if (x_36 == 0) { -uint8_t x_37; lean_object* x_38; -x_37 = l_Lean_Expr_isLet(x_34); -if (x_37 == 0) +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = lean_ctor_get(x_35, 0); +x_38 = lean_ctor_get(x_35, 1); +x_39 = l_Lean_Expr_isArrow(x_37); +if (x_39 == 0) +{ +uint8_t x_40; lean_object* x_41; +lean_dec(x_1); +x_40 = l_Lean_Expr_isLet(x_37); +if (x_40 == 0) { -uint8_t x_56; -x_56 = l_Lean_Expr_isForall(x_34); -if (x_56 == 0) +uint8_t x_59; +x_59 = l_Lean_Expr_isForall(x_37); +if (x_59 == 0) { -uint8_t x_57; -x_57 = l_Lean_Expr_isLetFun(x_34); -if (x_57 == 0) +uint8_t x_60; +x_60 = l_Lean_Expr_isLetFun(x_37); +if (x_60 == 0) { -lean_object* x_58; +lean_object* x_61; +lean_dec(x_37); lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); @@ -2479,7 +2987,7 @@ lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2494,101 +3002,162 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_58 = lean_box(0); -lean_ctor_set(x_32, 0, x_58); -return x_32; +x_61 = lean_box(0); +lean_ctor_set(x_35, 0, x_61); +return x_35; } else { -lean_object* x_59; -lean_free_object(x_32); -x_59 = lean_box(0); -x_38 = x_59; -goto block_55; +lean_object* x_62; +lean_free_object(x_35); +x_62 = lean_box(0); +x_41 = x_62; +goto block_58; } } else { -lean_object* x_60; -lean_free_object(x_32); -x_60 = lean_box(0); -x_38 = x_60; -goto block_55; +lean_object* x_63; +lean_free_object(x_35); +x_63 = lean_box(0); +x_41 = x_63; +goto block_58; } } else { -lean_object* x_61; -lean_free_object(x_32); -x_61 = lean_box(0); -x_38 = x_61; -goto block_55; +lean_object* x_64; +lean_free_object(x_35); +x_64 = lean_box(0); +x_41 = x_64; +goto block_58; } -block_55: +block_58: { -uint8_t x_39; lean_object* x_40; -lean_dec(x_38); -x_39 = 1; +uint8_t x_42; lean_object* x_43; +lean_dec(x_41); +x_42 = 1; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_40 = l_Lean_Meta_intro1Core(x_11, x_39, x_6, x_7, x_8, x_9, x_35); -if (lean_obj_tag(x_40) == 0) +x_43 = l_Lean_Meta_intro1Core(x_11, x_42, x_6, x_7, x_8, x_9, x_38); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); -lean_inc(x_42); -lean_dec(x_40); -x_43 = lean_ctor_get(x_41, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_41, 1); -lean_inc(x_44); -lean_dec(x_41); -lean_inc(x_43); -x_45 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed), 9, 1); -lean_closure_set(x_45, 0, x_43); -x_46 = lean_box(x_17); -x_47 = lean_box(x_37); +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -x_48 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___boxed), 34, 25); -lean_closure_set(x_48, 0, x_44); -lean_closure_set(x_48, 1, x_12); -lean_closure_set(x_48, 2, x_13); -lean_closure_set(x_48, 3, x_14); -lean_closure_set(x_48, 4, x_15); -lean_closure_set(x_48, 5, x_16); -lean_closure_set(x_48, 6, x_46); -lean_closure_set(x_48, 7, x_18); -lean_closure_set(x_48, 8, x_19); -lean_closure_set(x_48, 9, x_20); -lean_closure_set(x_48, 10, x_21); -lean_closure_set(x_48, 11, x_22); -lean_closure_set(x_48, 12, x_23); -lean_closure_set(x_48, 13, x_24); -lean_closure_set(x_48, 14, x_25); -lean_closure_set(x_48, 15, x_26); -lean_closure_set(x_48, 16, x_27); -lean_closure_set(x_48, 17, x_28); -lean_closure_set(x_48, 18, x_29); -lean_closure_set(x_48, 19, x_30); -lean_closure_set(x_48, 20, x_31); -lean_closure_set(x_48, 21, x_43); -lean_closure_set(x_48, 22, x_2); -lean_closure_set(x_48, 23, x_47); -lean_closure_set(x_48, 24, x_34); -x_49 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_49, 0, x_45); -lean_closure_set(x_49, 1, x_48); -x_50 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_44, x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_42); -return x_50; +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = lean_ctor_get(x_44, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_44, 1); +lean_inc(x_47); +lean_dec(x_44); +lean_inc(x_46); +x_48 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed), 9, 1); +lean_closure_set(x_48, 0, x_46); +x_49 = lean_box(x_18); +x_50 = lean_box(x_40); +lean_inc(x_47); +x_51 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___boxed), 37, 28); +lean_closure_set(x_51, 0, x_47); +lean_closure_set(x_51, 1, x_12); +lean_closure_set(x_51, 2, x_13); +lean_closure_set(x_51, 3, x_14); +lean_closure_set(x_51, 4, x_15); +lean_closure_set(x_51, 5, x_16); +lean_closure_set(x_51, 6, x_17); +lean_closure_set(x_51, 7, x_49); +lean_closure_set(x_51, 8, x_19); +lean_closure_set(x_51, 9, x_20); +lean_closure_set(x_51, 10, x_21); +lean_closure_set(x_51, 11, x_22); +lean_closure_set(x_51, 12, x_23); +lean_closure_set(x_51, 13, x_24); +lean_closure_set(x_51, 14, x_25); +lean_closure_set(x_51, 15, x_26); +lean_closure_set(x_51, 16, x_27); +lean_closure_set(x_51, 17, x_28); +lean_closure_set(x_51, 18, x_29); +lean_closure_set(x_51, 19, x_30); +lean_closure_set(x_51, 20, x_31); +lean_closure_set(x_51, 21, x_32); +lean_closure_set(x_51, 22, x_33); +lean_closure_set(x_51, 23, x_34); +lean_closure_set(x_51, 24, x_50); +lean_closure_set(x_51, 25, x_37); +lean_closure_set(x_51, 26, x_46); +lean_closure_set(x_51, 27, x_2); +x_52 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_52, 0, x_48); +lean_closure_set(x_52, 1, x_51); +x_53 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_47, x_52, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_45); +return x_53; } else { -uint8_t x_51; +uint8_t x_54; +lean_dec(x_37); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_54 = !lean_is_exclusive(x_43); +if (x_54 == 0) +{ +return x_43; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_43, 0); +x_56 = lean_ctor_get(x_43, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_43); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +} +} +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_free_object(x_35); lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); @@ -2602,108 +3171,105 @@ lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); -x_51 = !lean_is_exclusive(x_40); -if (x_51 == 0) +x_65 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_65, 0, x_1); +x_66 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed), 10, 1); +lean_closure_set(x_66, 0, x_37); +x_67 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_67, 0, x_65); +lean_closure_set(x_67, 1, x_66); +x_68 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_11, x_67, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_38); +if (lean_obj_tag(x_68) == 0) +{ +uint8_t x_69; +x_69 = !lean_is_exclusive(x_68); +if (x_69 == 0) +{ +lean_object* x_70; lean_object* x_71; +x_70 = lean_ctor_get(x_68, 0); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +lean_dec(x_70); +lean_ctor_set(x_68, 0, x_71); +return x_68; +} +else { -return x_40; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_72 = lean_ctor_get(x_68, 0); +x_73 = lean_ctor_get(x_68, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_68); +x_74 = lean_ctor_get(x_72, 0); +lean_inc(x_74); +lean_dec(x_72); +x_75 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_73); +return x_75; +} } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_40, 0); -x_53 = lean_ctor_get(x_40, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_40); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +uint8_t x_76; +x_76 = !lean_is_exclusive(x_68); +if (x_76 == 0) +{ +return x_68; +} +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_68, 0); +x_78 = lean_ctor_get(x_68, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_68); +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -lean_free_object(x_32); -lean_dec(x_2); -x_62 = l_Lean_Expr_bindingDomain_x21(x_34); -lean_inc(x_62); -x_63 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed), 9, 1); -lean_closure_set(x_63, 0, x_62); -x_64 = lean_box(x_17); -lean_inc(x_11); -x_65 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9___boxed), 32, 23); -lean_closure_set(x_65, 0, x_11); -lean_closure_set(x_65, 1, x_12); -lean_closure_set(x_65, 2, x_13); -lean_closure_set(x_65, 3, x_14); -lean_closure_set(x_65, 4, x_15); -lean_closure_set(x_65, 5, x_16); -lean_closure_set(x_65, 6, x_64); -lean_closure_set(x_65, 7, x_18); -lean_closure_set(x_65, 8, x_19); -lean_closure_set(x_65, 9, x_20); -lean_closure_set(x_65, 10, x_21); -lean_closure_set(x_65, 11, x_22); -lean_closure_set(x_65, 12, x_23); -lean_closure_set(x_65, 13, x_24); -lean_closure_set(x_65, 14, x_25); -lean_closure_set(x_65, 15, x_26); -lean_closure_set(x_65, 16, x_27); -lean_closure_set(x_65, 17, x_28); -lean_closure_set(x_65, 18, x_29); -lean_closure_set(x_65, 19, x_30); -lean_closure_set(x_65, 20, x_31); -lean_closure_set(x_65, 21, x_34); -lean_closure_set(x_65, 22, x_62); -x_66 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_66, 0, x_63); -lean_closure_set(x_66, 1, x_65); -x_67 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_11, x_66, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_35); -return x_67; -} -} -else -{ -lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_68 = lean_ctor_get(x_32, 0); -x_69 = lean_ctor_get(x_32, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_32); -x_70 = l_Lean_Expr_isArrow(x_68); -if (x_70 == 0) +lean_object* x_80; lean_object* x_81; uint8_t x_82; +x_80 = lean_ctor_get(x_35, 0); +x_81 = lean_ctor_get(x_35, 1); +lean_inc(x_81); +lean_inc(x_80); +lean_dec(x_35); +x_82 = l_Lean_Expr_isArrow(x_80); +if (x_82 == 0) { -uint8_t x_71; lean_object* x_72; -x_71 = l_Lean_Expr_isLet(x_68); -if (x_71 == 0) +uint8_t x_83; lean_object* x_84; +lean_dec(x_1); +x_83 = l_Lean_Expr_isLet(x_80); +if (x_83 == 0) { -uint8_t x_90; -x_90 = l_Lean_Expr_isForall(x_68); -if (x_90 == 0) +uint8_t x_102; +x_102 = l_Lean_Expr_isForall(x_80); +if (x_102 == 0) { -uint8_t x_91; -x_91 = l_Lean_Expr_isLetFun(x_68); -if (x_91 == 0) +uint8_t x_103; +x_103 = l_Lean_Expr_isLetFun(x_80); +if (x_103 == 0) { -lean_object* x_92; lean_object* x_93; -lean_dec(x_68); +lean_object* x_104; lean_object* x_105; +lean_dec(x_80); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); @@ -2717,7 +3283,7 @@ lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2732,100 +3298,106 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_92 = lean_box(0); -x_93 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_69); -return x_93; +x_104 = lean_box(0); +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_104); +lean_ctor_set(x_105, 1, x_81); +return x_105; } else { -lean_object* x_94; -x_94 = lean_box(0); -x_72 = x_94; -goto block_89; +lean_object* x_106; +x_106 = lean_box(0); +x_84 = x_106; +goto block_101; } } else { -lean_object* x_95; -x_95 = lean_box(0); -x_72 = x_95; -goto block_89; +lean_object* x_107; +x_107 = lean_box(0); +x_84 = x_107; +goto block_101; } } else { -lean_object* x_96; -x_96 = lean_box(0); -x_72 = x_96; -goto block_89; +lean_object* x_108; +x_108 = lean_box(0); +x_84 = x_108; +goto block_101; } -block_89: +block_101: { -uint8_t x_73; lean_object* x_74; -lean_dec(x_72); -x_73 = 1; +uint8_t x_85; lean_object* x_86; +lean_dec(x_84); +x_85 = 1; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -x_74 = l_Lean_Meta_intro1Core(x_11, x_73, x_6, x_7, x_8, x_9, x_69); -if (lean_obj_tag(x_74) == 0) +x_86 = l_Lean_Meta_intro1Core(x_11, x_85, x_6, x_7, x_8, x_9, x_81); +if (lean_obj_tag(x_86) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = lean_ctor_get(x_75, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_75, 1); -lean_inc(x_78); -lean_dec(x_75); -lean_inc(x_77); -x_79 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed), 9, 1); -lean_closure_set(x_79, 0, x_77); -x_80 = lean_box(x_17); -x_81 = lean_box(x_71); -lean_inc(x_78); -x_82 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___boxed), 34, 25); -lean_closure_set(x_82, 0, x_78); -lean_closure_set(x_82, 1, x_12); -lean_closure_set(x_82, 2, x_13); -lean_closure_set(x_82, 3, x_14); -lean_closure_set(x_82, 4, x_15); -lean_closure_set(x_82, 5, x_16); -lean_closure_set(x_82, 6, x_80); -lean_closure_set(x_82, 7, x_18); -lean_closure_set(x_82, 8, x_19); -lean_closure_set(x_82, 9, x_20); -lean_closure_set(x_82, 10, x_21); -lean_closure_set(x_82, 11, x_22); -lean_closure_set(x_82, 12, x_23); -lean_closure_set(x_82, 13, x_24); -lean_closure_set(x_82, 14, x_25); -lean_closure_set(x_82, 15, x_26); -lean_closure_set(x_82, 16, x_27); -lean_closure_set(x_82, 17, x_28); -lean_closure_set(x_82, 18, x_29); -lean_closure_set(x_82, 19, x_30); -lean_closure_set(x_82, 20, x_31); -lean_closure_set(x_82, 21, x_77); -lean_closure_set(x_82, 22, x_2); -lean_closure_set(x_82, 23, x_81); -lean_closure_set(x_82, 24, x_68); -x_83 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_83, 0, x_79); -lean_closure_set(x_83, 1, x_82); -x_84 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_78, x_83, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_76); -return x_84; +lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_87 = lean_ctor_get(x_86, 0); +lean_inc(x_87); +x_88 = lean_ctor_get(x_86, 1); +lean_inc(x_88); +lean_dec(x_86); +x_89 = lean_ctor_get(x_87, 0); +lean_inc(x_89); +x_90 = lean_ctor_get(x_87, 1); +lean_inc(x_90); +lean_dec(x_87); +lean_inc(x_89); +x_91 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed), 9, 1); +lean_closure_set(x_91, 0, x_89); +x_92 = lean_box(x_18); +x_93 = lean_box(x_83); +lean_inc(x_90); +x_94 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___boxed), 37, 28); +lean_closure_set(x_94, 0, x_90); +lean_closure_set(x_94, 1, x_12); +lean_closure_set(x_94, 2, x_13); +lean_closure_set(x_94, 3, x_14); +lean_closure_set(x_94, 4, x_15); +lean_closure_set(x_94, 5, x_16); +lean_closure_set(x_94, 6, x_17); +lean_closure_set(x_94, 7, x_92); +lean_closure_set(x_94, 8, x_19); +lean_closure_set(x_94, 9, x_20); +lean_closure_set(x_94, 10, x_21); +lean_closure_set(x_94, 11, x_22); +lean_closure_set(x_94, 12, x_23); +lean_closure_set(x_94, 13, x_24); +lean_closure_set(x_94, 14, x_25); +lean_closure_set(x_94, 15, x_26); +lean_closure_set(x_94, 16, x_27); +lean_closure_set(x_94, 17, x_28); +lean_closure_set(x_94, 18, x_29); +lean_closure_set(x_94, 19, x_30); +lean_closure_set(x_94, 20, x_31); +lean_closure_set(x_94, 21, x_32); +lean_closure_set(x_94, 22, x_33); +lean_closure_set(x_94, 23, x_34); +lean_closure_set(x_94, 24, x_93); +lean_closure_set(x_94, 25, x_80); +lean_closure_set(x_94, 26, x_89); +lean_closure_set(x_94, 27, x_2); +x_95 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_95, 0, x_91); +lean_closure_set(x_95, 1, x_94); +x_96 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_90, x_95, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_88); +return x_96; } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -lean_dec(x_68); +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; +lean_dec(x_80); +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); @@ -2839,7 +3411,7 @@ lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2853,74 +3425,123 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_85 = lean_ctor_get(x_74, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_74, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - lean_ctor_release(x_74, 1); - x_87 = x_74; +x_97 = lean_ctor_get(x_86, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_86, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_86)) { + lean_ctor_release(x_86, 0); + lean_ctor_release(x_86, 1); + x_99 = x_86; } else { - lean_dec_ref(x_74); - x_87 = lean_box(0); + lean_dec_ref(x_86); + x_99 = lean_box(0); } -if (lean_is_scalar(x_87)) { - x_88 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_99)) { + x_100 = lean_alloc_ctor(1, 2, 0); } else { - x_88 = x_87; + x_100 = x_99; } -lean_ctor_set(x_88, 0, x_85); -lean_ctor_set(x_88, 1, x_86); -return x_88; +lean_ctor_set(x_100, 0, x_97); +lean_ctor_set(x_100, 1, x_98); +return x_100; } } } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_23); +lean_dec(x_22); +lean_dec(x_21); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_2); -x_97 = l_Lean_Expr_bindingDomain_x21(x_68); -lean_inc(x_97); -x_98 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed), 9, 1); -lean_closure_set(x_98, 0, x_97); -x_99 = lean_box(x_17); -lean_inc(x_11); -x_100 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9___boxed), 32, 23); -lean_closure_set(x_100, 0, x_11); -lean_closure_set(x_100, 1, x_12); -lean_closure_set(x_100, 2, x_13); -lean_closure_set(x_100, 3, x_14); -lean_closure_set(x_100, 4, x_15); -lean_closure_set(x_100, 5, x_16); -lean_closure_set(x_100, 6, x_99); -lean_closure_set(x_100, 7, x_18); -lean_closure_set(x_100, 8, x_19); -lean_closure_set(x_100, 9, x_20); -lean_closure_set(x_100, 10, x_21); -lean_closure_set(x_100, 11, x_22); -lean_closure_set(x_100, 12, x_23); -lean_closure_set(x_100, 13, x_24); -lean_closure_set(x_100, 14, x_25); -lean_closure_set(x_100, 15, x_26); -lean_closure_set(x_100, 16, x_27); -lean_closure_set(x_100, 17, x_28); -lean_closure_set(x_100, 18, x_29); -lean_closure_set(x_100, 19, x_30); -lean_closure_set(x_100, 20, x_31); -lean_closure_set(x_100, 21, x_68); -lean_closure_set(x_100, 22, x_97); -x_101 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_101, 0, x_98); -lean_closure_set(x_101, 1, x_100); -x_102 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_11, x_101, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_69); -return x_102; +x_109 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_109, 0, x_1); +x_110 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed), 10, 1); +lean_closure_set(x_110, 0, x_80); +x_111 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_111, 0, x_109); +lean_closure_set(x_111, 1, x_110); +x_112 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_11, x_111, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_81); +if (lean_obj_tag(x_112) == 0) +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_113 = lean_ctor_get(x_112, 0); +lean_inc(x_113); +x_114 = lean_ctor_get(x_112, 1); +lean_inc(x_114); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_115 = x_112; +} else { + lean_dec_ref(x_112); + x_115 = lean_box(0); } +x_116 = lean_ctor_get(x_113, 0); +lean_inc(x_116); +lean_dec(x_113); +if (lean_is_scalar(x_115)) { + x_117 = lean_alloc_ctor(0, 2, 0); +} else { + x_117 = x_115; } +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_114); +return x_117; } else { -uint8_t x_103; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; +x_118 = lean_ctor_get(x_112, 0); +lean_inc(x_118); +x_119 = lean_ctor_get(x_112, 1); +lean_inc(x_119); +if (lean_is_exclusive(x_112)) { + lean_ctor_release(x_112, 0); + lean_ctor_release(x_112, 1); + x_120 = x_112; +} else { + lean_dec_ref(x_112); + x_120 = lean_box(0); +} +if (lean_is_scalar(x_120)) { + x_121 = lean_alloc_ctor(1, 2, 0); +} else { + x_121 = x_120; +} +lean_ctor_set(x_121, 0, x_118); +lean_ctor_set(x_121, 1, x_119); +return x_121; +} +} +} +} +else +{ +uint8_t x_122; +lean_dec(x_34); +lean_dec(x_33); +lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); @@ -2934,7 +3555,7 @@ lean_dec(x_22); lean_dec(x_21); lean_dec(x_20); lean_dec(x_19); -lean_dec(x_18); +lean_dec(x_17); lean_dec(x_16); lean_dec(x_15); lean_dec(x_14); @@ -2949,23 +3570,24 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_103 = !lean_is_exclusive(x_32); -if (x_103 == 0) +lean_dec(x_1); +x_122 = !lean_is_exclusive(x_35); +if (x_122 == 0) { -return x_32; +return x_35; } else { -lean_object* x_104; lean_object* x_105; lean_object* x_106; -x_104 = lean_ctor_get(x_32, 0); -x_105 = lean_ctor_get(x_32, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_32); -x_106 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_106, 0, x_104); -lean_ctor_set(x_106, 1, x_105); -return x_106; +lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_123 = lean_ctor_get(x_35, 0); +x_124 = lean_ctor_get(x_35, 1); +lean_inc(x_124); +lean_inc(x_123); +lean_dec(x_35); +x_125 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_125, 0, x_123); +lean_ctor_set(x_125, 1, x_124); +return x_125; } } } @@ -2979,25 +3601,11 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_9; -x_9 = l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_object* x_8; +x_8 = l_Lean_mkFreshId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -3005,22 +3613,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_9; +return x_8; } } -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_11; -x_11 = l_Lean_MVarId_assign___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); +lean_object* x_10; +x_10 = l_Lean_mkFreshFVarId___at___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -return x_11; +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -3102,35 +3711,27 @@ lean_object* x_31 = _args[30]; lean_object* x_32 = _args[31]; lean_object* x_33 = _args[32]; lean_object* x_34 = _args[33]; +lean_object* x_35 = _args[34]; +lean_object* x_36 = _args[35]; +lean_object* x_37 = _args[36]; _start: { -uint8_t x_35; uint8_t x_36; lean_object* x_37; -x_35 = lean_unbox(x_7); -lean_dec(x_7); -x_36 = lean_unbox(x_24); -lean_dec(x_24); -x_37 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_35, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_36, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34); -lean_dec(x_26); +uint8_t x_38; uint8_t x_39; lean_object* x_40; +x_38 = lean_unbox(x_8); +lean_dec(x_8); +x_39 = lean_unbox(x_25); lean_dec(x_25); -return x_37; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +x_40 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_38, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_24, x_39, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_37); +lean_dec(x_29); +lean_dec(x_26); +return x_40; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3142,7 +3743,7 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -3161,85 +3762,29 @@ lean_object* x_15 = _args[14]; lean_object* x_16 = _args[15]; lean_object* x_17 = _args[16]; lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -lean_object* x_21 = _args[20]; -lean_object* x_22 = _args[21]; -lean_object* x_23 = _args[22]; -lean_object* x_24 = _args[23]; -lean_object* x_25 = _args[24]; -lean_object* x_26 = _args[25]; -lean_object* x_27 = _args[26]; -lean_object* x_28 = _args[27]; -lean_object* x_29 = _args[28]; -lean_object* x_30 = _args[29]; -lean_object* x_31 = _args[30]; -lean_object* x_32 = _args[31]; -lean_object* x_33 = _args[32]; -lean_object* x_34 = _args[33]; -lean_object* x_35 = _args[34]; -lean_object* x_36 = _args[35]; -lean_object* x_37 = _args[36]; _start: { -uint8_t x_38; lean_object* x_39; -x_38 = lean_unbox(x_9); -lean_dec(x_9); -x_39 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_38, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_24, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_37); -lean_dec(x_36); -lean_dec(x_35); -lean_dec(x_34); -lean_dec(x_33); -lean_dec(x_32); -lean_dec(x_31); -lean_dec(x_30); -lean_dec(x_1); -return x_39; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -lean_object* x_18 = _args[17]; -lean_object* x_19 = _args[18]; -lean_object* x_20 = _args[19]; -lean_object* x_21 = _args[20]; -lean_object* x_22 = _args[21]; -lean_object* x_23 = _args[22]; -lean_object* x_24 = _args[23]; -lean_object* x_25 = _args[24]; -lean_object* x_26 = _args[25]; -lean_object* x_27 = _args[26]; -lean_object* x_28 = _args[27]; -lean_object* x_29 = _args[28]; -lean_object* x_30 = _args[29]; -lean_object* x_31 = _args[30]; -lean_object* x_32 = _args[31]; +lean_object* x_19; +x_19 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18); +lean_dec(x_17); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_1); +return x_19; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_33; uint8_t x_34; lean_object* x_35; -x_33 = lean_unbox(x_7); -lean_dec(x_7); -x_34 = lean_unbox(x_24); -lean_dec(x_24); -x_35 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__9(x_1, x_2, x_3, x_4, x_5, x_6, x_33, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_34, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32); -lean_dec(x_22); -return x_35; +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_isCasesCandidate(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -3298,7 +3843,7 @@ uint8_t x_5; x_5 = !lean_is_exclusive(x_2); if (x_5 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); x_8 = lean_ctor_get(x_1, 1); @@ -3306,8 +3851,8 @@ x_9 = lean_ctor_get(x_1, 2); x_10 = lean_ctor_get(x_1, 3); x_11 = lean_ctor_get(x_1, 4); x_12 = lean_ctor_get(x_1, 5); -x_13 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_14 = lean_ctor_get(x_1, 6); +x_13 = lean_ctor_get(x_1, 6); +x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); x_15 = lean_ctor_get(x_1, 7); x_16 = lean_ctor_get(x_1, 8); x_17 = lean_ctor_get(x_1, 9); @@ -3321,6 +3866,12 @@ x_24 = lean_ctor_get(x_1, 16); x_25 = lean_ctor_get(x_1, 17); x_26 = lean_ctor_get(x_1, 18); x_27 = lean_ctor_get(x_1, 19); +x_28 = lean_ctor_get(x_1, 20); +x_29 = lean_ctor_get(x_1, 21); +x_30 = lean_ctor_get(x_1, 22); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); @@ -3334,36 +3885,39 @@ lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_28 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_8); -lean_ctor_set(x_28, 2, x_9); -lean_ctor_set(x_28, 3, x_10); -lean_ctor_set(x_28, 4, x_11); -lean_ctor_set(x_28, 5, x_12); -lean_ctor_set(x_28, 6, x_14); -lean_ctor_set(x_28, 7, x_15); -lean_ctor_set(x_28, 8, x_16); -lean_ctor_set(x_28, 9, x_17); -lean_ctor_set(x_28, 10, x_18); -lean_ctor_set(x_28, 11, x_19); -lean_ctor_set(x_28, 12, x_20); -lean_ctor_set(x_28, 13, x_21); -lean_ctor_set(x_28, 14, x_22); -lean_ctor_set(x_28, 15, x_23); -lean_ctor_set(x_28, 16, x_24); -lean_ctor_set(x_28, 17, x_25); -lean_ctor_set(x_28, 18, x_26); -lean_ctor_set(x_28, 19, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*20, x_13); +x_31 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_31, 0, x_6); +lean_ctor_set(x_31, 1, x_8); +lean_ctor_set(x_31, 2, x_9); +lean_ctor_set(x_31, 3, x_10); +lean_ctor_set(x_31, 4, x_11); +lean_ctor_set(x_31, 5, x_12); +lean_ctor_set(x_31, 6, x_13); +lean_ctor_set(x_31, 7, x_15); +lean_ctor_set(x_31, 8, x_16); +lean_ctor_set(x_31, 9, x_17); +lean_ctor_set(x_31, 10, x_18); +lean_ctor_set(x_31, 11, x_19); +lean_ctor_set(x_31, 12, x_20); +lean_ctor_set(x_31, 13, x_21); +lean_ctor_set(x_31, 14, x_22); +lean_ctor_set(x_31, 15, x_23); +lean_ctor_set(x_31, 16, x_24); +lean_ctor_set(x_31, 17, x_25); +lean_ctor_set(x_31, 18, x_26); +lean_ctor_set(x_31, 19, x_27); +lean_ctor_set(x_31, 20, x_28); +lean_ctor_set(x_31, 21, x_29); +lean_ctor_set(x_31, 22, x_30); +lean_ctor_set_uint8(x_31, sizeof(void*)*23, x_14); lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_28); +lean_ctor_set(x_2, 0, x_31); { lean_object* _tmp_1 = x_7; lean_object* _tmp_2 = x_2; @@ -3374,32 +3928,41 @@ goto _start; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_30 = lean_ctor_get(x_2, 0); -x_31 = lean_ctor_get(x_2, 1); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_33 = lean_ctor_get(x_2, 0); +x_34 = lean_ctor_get(x_2, 1); +lean_inc(x_34); +lean_inc(x_33); lean_dec(x_2); -x_32 = lean_ctor_get(x_1, 1); -x_33 = lean_ctor_get(x_1, 2); -x_34 = lean_ctor_get(x_1, 3); -x_35 = lean_ctor_get(x_1, 4); -x_36 = lean_ctor_get(x_1, 5); -x_37 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_38 = lean_ctor_get(x_1, 6); -x_39 = lean_ctor_get(x_1, 7); -x_40 = lean_ctor_get(x_1, 8); -x_41 = lean_ctor_get(x_1, 9); -x_42 = lean_ctor_get(x_1, 10); -x_43 = lean_ctor_get(x_1, 11); -x_44 = lean_ctor_get(x_1, 12); -x_45 = lean_ctor_get(x_1, 13); -x_46 = lean_ctor_get(x_1, 14); -x_47 = lean_ctor_get(x_1, 15); -x_48 = lean_ctor_get(x_1, 16); -x_49 = lean_ctor_get(x_1, 17); -x_50 = lean_ctor_get(x_1, 18); -x_51 = lean_ctor_get(x_1, 19); +x_35 = lean_ctor_get(x_1, 1); +x_36 = lean_ctor_get(x_1, 2); +x_37 = lean_ctor_get(x_1, 3); +x_38 = lean_ctor_get(x_1, 4); +x_39 = lean_ctor_get(x_1, 5); +x_40 = lean_ctor_get(x_1, 6); +x_41 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); +x_42 = lean_ctor_get(x_1, 7); +x_43 = lean_ctor_get(x_1, 8); +x_44 = lean_ctor_get(x_1, 9); +x_45 = lean_ctor_get(x_1, 10); +x_46 = lean_ctor_get(x_1, 11); +x_47 = lean_ctor_get(x_1, 12); +x_48 = lean_ctor_get(x_1, 13); +x_49 = lean_ctor_get(x_1, 14); +x_50 = lean_ctor_get(x_1, 15); +x_51 = lean_ctor_get(x_1, 16); +x_52 = lean_ctor_get(x_1, 17); +x_53 = lean_ctor_get(x_1, 18); +x_54 = lean_ctor_get(x_1, 19); +x_55 = lean_ctor_get(x_1, 20); +x_56 = lean_ctor_get(x_1, 21); +x_57 = lean_ctor_get(x_1, 22); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); @@ -3410,42 +3973,42 @@ lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); +lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -x_52 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_52, 0, x_30); -lean_ctor_set(x_52, 1, x_32); -lean_ctor_set(x_52, 2, x_33); -lean_ctor_set(x_52, 3, x_34); -lean_ctor_set(x_52, 4, x_35); -lean_ctor_set(x_52, 5, x_36); -lean_ctor_set(x_52, 6, x_38); -lean_ctor_set(x_52, 7, x_39); -lean_ctor_set(x_52, 8, x_40); -lean_ctor_set(x_52, 9, x_41); -lean_ctor_set(x_52, 10, x_42); -lean_ctor_set(x_52, 11, x_43); -lean_ctor_set(x_52, 12, x_44); -lean_ctor_set(x_52, 13, x_45); -lean_ctor_set(x_52, 14, x_46); -lean_ctor_set(x_52, 15, x_47); -lean_ctor_set(x_52, 16, x_48); -lean_ctor_set(x_52, 17, x_49); -lean_ctor_set(x_52, 18, x_50); -lean_ctor_set(x_52, 19, x_51); -lean_ctor_set_uint8(x_52, sizeof(void*)*20, x_37); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_3); -x_2 = x_31; -x_3 = x_53; +x_58 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_58, 0, x_33); +lean_ctor_set(x_58, 1, x_35); +lean_ctor_set(x_58, 2, x_36); +lean_ctor_set(x_58, 3, x_37); +lean_ctor_set(x_58, 4, x_38); +lean_ctor_set(x_58, 5, x_39); +lean_ctor_set(x_58, 6, x_40); +lean_ctor_set(x_58, 7, x_42); +lean_ctor_set(x_58, 8, x_43); +lean_ctor_set(x_58, 9, x_44); +lean_ctor_set(x_58, 10, x_45); +lean_ctor_set(x_58, 11, x_46); +lean_ctor_set(x_58, 12, x_47); +lean_ctor_set(x_58, 13, x_48); +lean_ctor_set(x_58, 14, x_49); +lean_ctor_set(x_58, 15, x_50); +lean_ctor_set(x_58, 16, x_51); +lean_ctor_set(x_58, 17, x_52); +lean_ctor_set(x_58, 18, x_53); +lean_ctor_set(x_58, 19, x_54); +lean_ctor_set(x_58, 20, x_55); +lean_ctor_set(x_58, 21, x_56); +lean_ctor_set(x_58, 22, x_57); +lean_ctor_set_uint8(x_58, sizeof(void*)*23, x_41); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_3); +x_2 = x_34; +x_3 = x_59; goto _start; } } @@ -3639,7 +4202,7 @@ uint8_t x_8; x_8 = !lean_is_exclusive(x_1); if (x_8 == 0) { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; x_9 = lean_ctor_get(x_1, 0); x_10 = lean_ctor_get(x_1, 1); x_11 = lean_ctor_get(x_1, 2); @@ -3660,16 +4223,22 @@ x_25 = lean_ctor_get(x_1, 16); x_26 = lean_ctor_get(x_1, 17); x_27 = lean_ctor_get(x_1, 18); x_28 = lean_ctor_get(x_1, 19); -x_29 = l_Lean_Meta_Grind_injection_x3f(x_9, x_2, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_29) == 0) +x_29 = lean_ctor_get(x_1, 20); +x_30 = lean_ctor_get(x_1, 21); +x_31 = lean_ctor_get(x_1, 22); +x_32 = l_Lean_Meta_Grind_injection_x3f(x_9, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_30; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -if (lean_obj_tag(x_30) == 0) +lean_object* x_33; +x_33 = lean_ctor_get(x_32, 0); +lean_inc(x_33); +if (lean_obj_tag(x_33) == 0) { -uint8_t x_31; +uint8_t x_34; lean_free_object(x_1); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_29); lean_dec(x_28); lean_dec(x_27); lean_dec(x_26); @@ -3689,93 +4258,96 @@ lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_31 = !lean_is_exclusive(x_29); -if (x_31 == 0) +x_34 = !lean_is_exclusive(x_32); +if (x_34 == 0) { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 0); -lean_dec(x_32); -x_33 = lean_box(0); -lean_ctor_set(x_29, 0, x_33); -return x_29; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_32, 0); +lean_dec(x_35); +x_36 = lean_box(0); +lean_ctor_set(x_32, 0, x_36); +return x_32; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_29, 1); -lean_inc(x_34); -lean_dec(x_29); -x_35 = lean_box(0); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_34); -return x_36; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_32, 1); +lean_inc(x_37); +lean_dec(x_32); +x_38 = lean_box(0); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +return x_39; } } else { -uint8_t x_37; -x_37 = !lean_is_exclusive(x_29); -if (x_37 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_32); +if (x_40 == 0) { -lean_object* x_38; uint8_t x_39; -x_38 = lean_ctor_get(x_29, 0); -lean_dec(x_38); -x_39 = !lean_is_exclusive(x_30); -if (x_39 == 0) +lean_object* x_41; uint8_t x_42; +x_41 = lean_ctor_get(x_32, 0); +lean_dec(x_41); +x_42 = !lean_is_exclusive(x_33); +if (x_42 == 0) { -lean_object* x_40; -x_40 = lean_ctor_get(x_30, 0); -lean_ctor_set(x_1, 0, x_40); -lean_ctor_set(x_30, 0, x_1); -return x_29; +lean_object* x_43; +x_43 = lean_ctor_get(x_33, 0); +lean_ctor_set(x_1, 0, x_43); +lean_ctor_set(x_33, 0, x_1); +return x_32; } else { -lean_object* x_41; lean_object* x_42; -x_41 = lean_ctor_get(x_30, 0); -lean_inc(x_41); -lean_dec(x_30); -lean_ctor_set(x_1, 0, x_41); -x_42 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_42, 0, x_1); -lean_ctor_set(x_29, 0, x_42); -return x_29; +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_33, 0); +lean_inc(x_44); +lean_dec(x_33); +lean_ctor_set(x_1, 0, x_44); +x_45 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_45, 0, x_1); +lean_ctor_set(x_32, 0, x_45); +return x_32; } } else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_43 = lean_ctor_get(x_29, 1); -lean_inc(x_43); -lean_dec(x_29); -x_44 = lean_ctor_get(x_30, 0); -lean_inc(x_44); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - x_45 = x_30; +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_46 = lean_ctor_get(x_32, 1); +lean_inc(x_46); +lean_dec(x_32); +x_47 = lean_ctor_get(x_33, 0); +lean_inc(x_47); +if (lean_is_exclusive(x_33)) { + lean_ctor_release(x_33, 0); + x_48 = x_33; } else { - lean_dec_ref(x_30); - x_45 = lean_box(0); + lean_dec_ref(x_33); + x_48 = lean_box(0); } -lean_ctor_set(x_1, 0, x_44); -if (lean_is_scalar(x_45)) { - x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_1, 0, x_47); +if (lean_is_scalar(x_48)) { + x_49 = lean_alloc_ctor(1, 1, 0); } else { - x_46 = x_45; + x_49 = x_48; } -lean_ctor_set(x_46, 0, x_1); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_43); -return x_47; +lean_ctor_set(x_49, 0, x_1); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_46); +return x_50; } } } else { -uint8_t x_48; +uint8_t x_51; lean_free_object(x_1); +lean_dec(x_31); +lean_dec(x_30); +lean_dec(x_29); lean_dec(x_28); lean_dec(x_27); lean_dec(x_26); @@ -3795,50 +4367,59 @@ lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_48 = !lean_is_exclusive(x_29); -if (x_48 == 0) +x_51 = !lean_is_exclusive(x_32); +if (x_51 == 0) { -return x_29; +return x_32; } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_29, 0); -x_50 = lean_ctor_get(x_29, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_29); -x_51 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_51, 0, x_49); -lean_ctor_set(x_51, 1, x_50); -return x_51; -} -} -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_52 = lean_ctor_get(x_1, 0); -x_53 = lean_ctor_get(x_1, 1); -x_54 = lean_ctor_get(x_1, 2); -x_55 = lean_ctor_get(x_1, 3); -x_56 = lean_ctor_get(x_1, 4); -x_57 = lean_ctor_get(x_1, 5); -x_58 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_59 = lean_ctor_get(x_1, 6); -x_60 = lean_ctor_get(x_1, 7); -x_61 = lean_ctor_get(x_1, 8); -x_62 = lean_ctor_get(x_1, 9); -x_63 = lean_ctor_get(x_1, 10); -x_64 = lean_ctor_get(x_1, 11); -x_65 = lean_ctor_get(x_1, 12); -x_66 = lean_ctor_get(x_1, 13); -x_67 = lean_ctor_get(x_1, 14); -x_68 = lean_ctor_get(x_1, 15); -x_69 = lean_ctor_get(x_1, 16); -x_70 = lean_ctor_get(x_1, 17); -x_71 = lean_ctor_get(x_1, 18); -x_72 = lean_ctor_get(x_1, 19); +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_32, 0); +x_53 = lean_ctor_get(x_32, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_32); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +} +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_55 = lean_ctor_get(x_1, 0); +x_56 = lean_ctor_get(x_1, 1); +x_57 = lean_ctor_get(x_1, 2); +x_58 = lean_ctor_get(x_1, 3); +x_59 = lean_ctor_get(x_1, 4); +x_60 = lean_ctor_get(x_1, 5); +x_61 = lean_ctor_get(x_1, 6); +x_62 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); +x_63 = lean_ctor_get(x_1, 7); +x_64 = lean_ctor_get(x_1, 8); +x_65 = lean_ctor_get(x_1, 9); +x_66 = lean_ctor_get(x_1, 10); +x_67 = lean_ctor_get(x_1, 11); +x_68 = lean_ctor_get(x_1, 12); +x_69 = lean_ctor_get(x_1, 13); +x_70 = lean_ctor_get(x_1, 14); +x_71 = lean_ctor_get(x_1, 15); +x_72 = lean_ctor_get(x_1, 16); +x_73 = lean_ctor_get(x_1, 17); +x_74 = lean_ctor_get(x_1, 18); +x_75 = lean_ctor_get(x_1, 19); +x_76 = lean_ctor_get(x_1, 20); +x_77 = lean_ctor_get(x_1, 21); +x_78 = lean_ctor_get(x_1, 22); +lean_inc(x_78); +lean_inc(x_77); +lean_inc(x_76); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_73); lean_inc(x_72); lean_inc(x_71); lean_inc(x_70); @@ -3849,26 +4430,29 @@ lean_inc(x_66); lean_inc(x_65); lean_inc(x_64); lean_inc(x_63); -lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); lean_inc(x_59); +lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); lean_dec(x_1); -x_73 = l_Lean_Meta_Grind_injection_x3f(x_52, x_2, x_3, x_4, x_5, x_6, x_7); -if (lean_obj_tag(x_73) == 0) +x_79 = l_Lean_Meta_Grind_injection_x3f(x_55, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_79) == 0) { -lean_object* x_74; -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -if (lean_obj_tag(x_74) == 0) +lean_object* x_80; +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +if (lean_obj_tag(x_80) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; +lean_dec(x_78); +lean_dec(x_77); +lean_dec(x_76); +lean_dec(x_75); +lean_dec(x_74); +lean_dec(x_73); lean_dec(x_72); lean_dec(x_71); lean_dec(x_70); @@ -3879,98 +4463,104 @@ lean_dec(x_66); lean_dec(x_65); lean_dec(x_64); lean_dec(x_63); -lean_dec(x_62); lean_dec(x_61); lean_dec(x_60); lean_dec(x_59); +lean_dec(x_58); lean_dec(x_57); lean_dec(x_56); -lean_dec(x_55); -lean_dec(x_54); -lean_dec(x_53); -x_75 = lean_ctor_get(x_73, 1); -lean_inc(x_75); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_76 = x_73; +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_82 = x_79; } else { - lean_dec_ref(x_73); - x_76 = lean_box(0); + lean_dec_ref(x_79); + x_82 = lean_box(0); } -x_77 = lean_box(0); -if (lean_is_scalar(x_76)) { - x_78 = lean_alloc_ctor(0, 2, 0); +x_83 = lean_box(0); +if (lean_is_scalar(x_82)) { + x_84 = lean_alloc_ctor(0, 2, 0); } else { - x_78 = x_76; + x_84 = x_82; } -lean_ctor_set(x_78, 0, x_77); -lean_ctor_set(x_78, 1, x_75); -return x_78; +lean_ctor_set(x_84, 0, x_83); +lean_ctor_set(x_84, 1, x_81); +return x_84; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_79 = lean_ctor_get(x_73, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_80 = x_73; +lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_85 = lean_ctor_get(x_79, 1); +lean_inc(x_85); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_86 = x_79; } else { - lean_dec_ref(x_73); - x_80 = lean_box(0); + lean_dec_ref(x_79); + x_86 = lean_box(0); } -x_81 = lean_ctor_get(x_74, 0); -lean_inc(x_81); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - x_82 = x_74; +x_87 = lean_ctor_get(x_80, 0); +lean_inc(x_87); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_88 = x_80; } else { - lean_dec_ref(x_74); - x_82 = lean_box(0); + lean_dec_ref(x_80); + x_88 = lean_box(0); } -x_83 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_53); -lean_ctor_set(x_83, 2, x_54); -lean_ctor_set(x_83, 3, x_55); -lean_ctor_set(x_83, 4, x_56); -lean_ctor_set(x_83, 5, x_57); -lean_ctor_set(x_83, 6, x_59); -lean_ctor_set(x_83, 7, x_60); -lean_ctor_set(x_83, 8, x_61); -lean_ctor_set(x_83, 9, x_62); -lean_ctor_set(x_83, 10, x_63); -lean_ctor_set(x_83, 11, x_64); -lean_ctor_set(x_83, 12, x_65); -lean_ctor_set(x_83, 13, x_66); -lean_ctor_set(x_83, 14, x_67); -lean_ctor_set(x_83, 15, x_68); -lean_ctor_set(x_83, 16, x_69); -lean_ctor_set(x_83, 17, x_70); -lean_ctor_set(x_83, 18, x_71); -lean_ctor_set(x_83, 19, x_72); -lean_ctor_set_uint8(x_83, sizeof(void*)*20, x_58); -if (lean_is_scalar(x_82)) { - x_84 = lean_alloc_ctor(1, 1, 0); +x_89 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_56); +lean_ctor_set(x_89, 2, x_57); +lean_ctor_set(x_89, 3, x_58); +lean_ctor_set(x_89, 4, x_59); +lean_ctor_set(x_89, 5, x_60); +lean_ctor_set(x_89, 6, x_61); +lean_ctor_set(x_89, 7, x_63); +lean_ctor_set(x_89, 8, x_64); +lean_ctor_set(x_89, 9, x_65); +lean_ctor_set(x_89, 10, x_66); +lean_ctor_set(x_89, 11, x_67); +lean_ctor_set(x_89, 12, x_68); +lean_ctor_set(x_89, 13, x_69); +lean_ctor_set(x_89, 14, x_70); +lean_ctor_set(x_89, 15, x_71); +lean_ctor_set(x_89, 16, x_72); +lean_ctor_set(x_89, 17, x_73); +lean_ctor_set(x_89, 18, x_74); +lean_ctor_set(x_89, 19, x_75); +lean_ctor_set(x_89, 20, x_76); +lean_ctor_set(x_89, 21, x_77); +lean_ctor_set(x_89, 22, x_78); +lean_ctor_set_uint8(x_89, sizeof(void*)*23, x_62); +if (lean_is_scalar(x_88)) { + x_90 = lean_alloc_ctor(1, 1, 0); } else { - x_84 = x_82; + x_90 = x_88; } -lean_ctor_set(x_84, 0, x_83); -if (lean_is_scalar(x_80)) { - x_85 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_89); +if (lean_is_scalar(x_86)) { + x_91 = lean_alloc_ctor(0, 2, 0); } else { - x_85 = x_80; + x_91 = x_86; } -lean_ctor_set(x_85, 0, x_84); -lean_ctor_set(x_85, 1, x_79); -return x_85; +lean_ctor_set(x_91, 0, x_90); +lean_ctor_set(x_91, 1, x_85); +return x_91; } } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_dec(x_78); +lean_dec(x_77); +lean_dec(x_76); +lean_dec(x_75); +lean_dec(x_74); +lean_dec(x_73); lean_dec(x_72); lean_dec(x_71); lean_dec(x_70); @@ -3981,35 +4571,32 @@ lean_dec(x_66); lean_dec(x_65); lean_dec(x_64); lean_dec(x_63); -lean_dec(x_62); lean_dec(x_61); lean_dec(x_60); lean_dec(x_59); +lean_dec(x_58); lean_dec(x_57); lean_dec(x_56); -lean_dec(x_55); -lean_dec(x_54); -lean_dec(x_53); -x_86 = lean_ctor_get(x_73, 0); -lean_inc(x_86); -x_87 = lean_ctor_get(x_73, 1); -lean_inc(x_87); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_88 = x_73; +x_92 = lean_ctor_get(x_79, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_79, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + lean_ctor_release(x_79, 1); + x_94 = x_79; } else { - lean_dec_ref(x_73); - x_88 = lean_box(0); + lean_dec_ref(x_79); + x_94 = lean_box(0); } -if (lean_is_scalar(x_88)) { - x_89 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(1, 2, 0); } else { - x_89 = x_88; + x_95 = x_94; } -lean_ctor_set(x_89, 0, x_86); -lean_ctor_set(x_89, 1, x_87); -return x_89; +lean_ctor_set(x_95, 0, x_92); +lean_ctor_set(x_95, 1, x_93); +return x_95; } } } @@ -4280,52 +4867,55 @@ return x_34; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, uint8_t x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24, lean_object* x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32, lean_object* x_33) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, uint8_t x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17, lean_object* x_18, lean_object* x_19, lean_object* x_20, lean_object* x_21, lean_object* x_22, lean_object* x_23, lean_object* x_24, lean_object* x_25, lean_object* x_26, lean_object* x_27, lean_object* x_28, lean_object* x_29, lean_object* x_30, lean_object* x_31, lean_object* x_32, lean_object* x_33, lean_object* x_34, lean_object* x_35, lean_object* x_36) { _start: { -lean_object* x_34; +lean_object* x_37; +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); lean_inc(x_2); lean_inc(x_1); -x_34 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext(x_1, x_2, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33); -if (lean_obj_tag(x_34) == 0) -{ -lean_object* x_35; -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -switch (lean_obj_tag(x_35)) { -case 0: -{ -lean_object* x_36; lean_object* x_37; -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -x_37 = l_Lean_MVarId_byContra_x3f(x_3, x_29, x_30, x_31, x_32, x_36); +x_37 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext(x_1, x_2, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); -if (lean_obj_tag(x_38) == 0) +switch (lean_obj_tag(x_38)) { +case 0: +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +x_40 = l_Lean_MVarId_byContra_x3f(x_3, x_32, x_33, x_34, x_35, x_39); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +if (lean_obj_tag(x_41) == 0) { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4339,93 +4929,99 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -lean_dec(x_37); -x_40 = lean_st_ref_take(x_25, x_39); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); x_42 = lean_ctor_get(x_40, 1); lean_inc(x_42); lean_dec(x_40); -x_43 = lean_array_push(x_41, x_1); -x_44 = lean_st_ref_set(x_25, x_43, x_42); -x_45 = !lean_is_exclusive(x_44); -if (x_45 == 0) +x_43 = lean_st_ref_take(x_28, x_42); +x_44 = lean_ctor_get(x_43, 0); +lean_inc(x_44); +x_45 = lean_ctor_get(x_43, 1); +lean_inc(x_45); +lean_dec(x_43); +x_46 = lean_array_push(x_44, x_1); +x_47 = lean_st_ref_set(x_28, x_46, x_45); +x_48 = !lean_is_exclusive(x_47); +if (x_48 == 0) { -lean_object* x_46; lean_object* x_47; -x_46 = lean_ctor_get(x_44, 0); -lean_dec(x_46); -x_47 = lean_box(0); -lean_ctor_set(x_44, 0, x_47); -return x_44; +lean_object* x_49; lean_object* x_50; +x_49 = lean_ctor_get(x_47, 0); +lean_dec(x_49); +x_50 = lean_box(0); +lean_ctor_set(x_47, 0, x_50); +return x_47; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_44, 1); -lean_inc(x_48); -lean_dec(x_44); -x_49 = lean_box(0); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -return x_50; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_47, 1); +lean_inc(x_51); +lean_dec(x_47); +x_52 = lean_box(0); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +return x_53; } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_dec(x_1); -x_51 = lean_ctor_get(x_37, 1); -lean_inc(x_51); -lean_dec(x_37); -x_52 = lean_ctor_get(x_38, 0); -lean_inc(x_52); -lean_dec(x_38); -x_53 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_4); -lean_ctor_set(x_53, 2, x_5); -lean_ctor_set(x_53, 3, x_6); -lean_ctor_set(x_53, 4, x_7); -lean_ctor_set(x_53, 5, x_8); -lean_ctor_set(x_53, 6, x_10); -lean_ctor_set(x_53, 7, x_11); -lean_ctor_set(x_53, 8, x_12); -lean_ctor_set(x_53, 9, x_13); -lean_ctor_set(x_53, 10, x_14); -lean_ctor_set(x_53, 11, x_15); -lean_ctor_set(x_53, 12, x_16); -lean_ctor_set(x_53, 13, x_17); -lean_ctor_set(x_53, 14, x_18); -lean_ctor_set(x_53, 15, x_19); -lean_ctor_set(x_53, 16, x_20); -lean_ctor_set(x_53, 17, x_21); -lean_ctor_set(x_53, 18, x_22); -lean_ctor_set(x_53, 19, x_23); -lean_ctor_set_uint8(x_53, sizeof(void*)*20, x_9); -x_54 = l_Lean_Meta_Grind_intros_go(x_2, x_53, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_51); -return x_54; +x_54 = lean_ctor_get(x_40, 1); +lean_inc(x_54); +lean_dec(x_40); +x_55 = lean_ctor_get(x_41, 0); +lean_inc(x_55); +lean_dec(x_41); +x_56 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_4); +lean_ctor_set(x_56, 2, x_5); +lean_ctor_set(x_56, 3, x_6); +lean_ctor_set(x_56, 4, x_7); +lean_ctor_set(x_56, 5, x_8); +lean_ctor_set(x_56, 6, x_9); +lean_ctor_set(x_56, 7, x_11); +lean_ctor_set(x_56, 8, x_12); +lean_ctor_set(x_56, 9, x_13); +lean_ctor_set(x_56, 10, x_14); +lean_ctor_set(x_56, 11, x_15); +lean_ctor_set(x_56, 12, x_16); +lean_ctor_set(x_56, 13, x_17); +lean_ctor_set(x_56, 14, x_18); +lean_ctor_set(x_56, 15, x_19); +lean_ctor_set(x_56, 16, x_20); +lean_ctor_set(x_56, 17, x_21); +lean_ctor_set(x_56, 18, x_22); +lean_ctor_set(x_56, 19, x_23); +lean_ctor_set(x_56, 20, x_24); +lean_ctor_set(x_56, 21, x_25); +lean_ctor_set(x_56, 22, x_26); +lean_ctor_set_uint8(x_56, sizeof(void*)*23, x_10); +x_57 = l_Lean_Meta_Grind_intros_go(x_2, x_56, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_54); +return x_57; } } else { -uint8_t x_55; +uint8_t x_58; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4439,7 +5035,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4447,29 +5043,32 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_55 = !lean_is_exclusive(x_37); -if (x_55 == 0) +x_58 = !lean_is_exclusive(x_40); +if (x_58 == 0) { -return x_37; +return x_40; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_37, 0); -x_57 = lean_ctor_get(x_37, 1); -lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_37); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_40, 0); +x_60 = lean_ctor_get(x_40, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_40); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; } } } case 1: { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4483,7 +5082,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4491,39 +5090,21 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_59 = lean_ctor_get(x_34, 1); -lean_inc(x_59); -lean_dec(x_34); -x_60 = lean_ctor_get(x_35, 0); -lean_inc(x_60); -x_61 = lean_ctor_get(x_35, 1); -lean_inc(x_61); -lean_dec(x_35); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_60); -lean_inc(x_61); -x_62 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f(x_61, x_60, x_29, x_30, x_31, x_32, x_59); -if (lean_obj_tag(x_62) == 0) -{ -lean_object* x_63; -x_63 = lean_ctor_get(x_62, 0); +x_62 = lean_ctor_get(x_37, 1); +lean_inc(x_62); +lean_dec(x_37); +x_63 = lean_ctor_get(x_38, 0); lean_inc(x_63); -if (lean_obj_tag(x_63) == 0) -{ -lean_object* x_64; lean_object* x_65; -x_64 = lean_ctor_get(x_62, 1); +x_64 = lean_ctor_get(x_38, 1); lean_inc(x_64); -lean_dec(x_62); +lean_dec(x_38); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_60); -lean_inc(x_61); -x_65 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyInjection_x3f(x_61, x_60, x_29, x_30, x_31, x_32, x_64); +lean_inc(x_63); +lean_inc(x_64); +x_65 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f(x_64, x_63, x_32, x_33, x_34, x_35, x_62); if (lean_obj_tag(x_65) == 0) { lean_object* x_66; @@ -4531,174 +5112,195 @@ x_66 = lean_ctor_get(x_65, 0); lean_inc(x_66); if (lean_obj_tag(x_66) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_object* x_67; lean_object* x_68; x_67 = lean_ctor_get(x_65, 1); lean_inc(x_67); lean_dec(x_65); -x_68 = lean_ctor_get(x_61, 0); -lean_inc(x_68); -x_69 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); -lean_closure_set(x_69, 0, x_61); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_63); +lean_inc(x_64); +x_68 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyInjection_x3f(x_64, x_63, x_32, x_33, x_34, x_35, x_67); +if (lean_obj_tag(x_68) == 0) +{ +lean_object* x_69; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +if (lean_obj_tag(x_69) == 0) +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_64, 0); +lean_inc(x_71); +x_72 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__2___boxed), 9, 1); +lean_closure_set(x_72, 0, x_64); lean_inc(x_2); -x_70 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_intros_go___lambda__1), 11, 2); -lean_closure_set(x_70, 0, x_60); -lean_closure_set(x_70, 1, x_2); -x_71 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_71, 0, x_69); -lean_closure_set(x_71, 1, x_70); -x_72 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; -x_73 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_73, 0, x_71); -lean_closure_set(x_73, 1, x_72); +x_73 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_intros_go___lambda__1), 11, 2); +lean_closure_set(x_73, 0, x_63); +lean_closure_set(x_73, 1, x_2); +x_74 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_74, 0, x_72); +lean_closure_set(x_74, 1, x_73); +x_75 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1; +x_76 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_76, 0, x_74); +lean_closure_set(x_76, 1, x_75); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); -lean_inc(x_26); -x_74 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_68, x_73, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_67); -if (lean_obj_tag(x_74) == 0) +x_77 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_71, x_76, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_70); +if (lean_obj_tag(x_77) == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = l_Lean_Meta_Grind_intros_go(x_2, x_75, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_76); -return x_77; +lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_78 = lean_ctor_get(x_77, 0); +lean_inc(x_78); +x_79 = lean_ctor_get(x_77, 1); +lean_inc(x_79); +lean_dec(x_77); +x_80 = l_Lean_Meta_Grind_intros_go(x_2, x_78, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_79); +return x_80; } else { -uint8_t x_78; +uint8_t x_81; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_26); lean_dec(x_2); -x_78 = !lean_is_exclusive(x_74); -if (x_78 == 0) +x_81 = !lean_is_exclusive(x_77); +if (x_81 == 0) { -return x_74; +return x_77; } else { -lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_79 = lean_ctor_get(x_74, 0); -x_80 = lean_ctor_get(x_74, 1); -lean_inc(x_80); -lean_inc(x_79); -lean_dec(x_74); -x_81 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_81, 0, x_79); -lean_ctor_set(x_81, 1, x_80); -return x_81; +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_77, 0); +x_83 = lean_ctor_get(x_77, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_77); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; } } } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; -lean_dec(x_61); -lean_dec(x_60); -x_82 = lean_ctor_get(x_65, 1); -lean_inc(x_82); -lean_dec(x_65); -x_83 = lean_ctor_get(x_66, 0); -lean_inc(x_83); -lean_dec(x_66); -x_84 = l_Lean_Meta_Grind_intros_go(x_2, x_83, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_82); -return x_84; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_dec(x_64); +lean_dec(x_63); +x_85 = lean_ctor_get(x_68, 1); +lean_inc(x_85); +lean_dec(x_68); +x_86 = lean_ctor_get(x_69, 0); +lean_inc(x_86); +lean_dec(x_69); +x_87 = l_Lean_Meta_Grind_intros_go(x_2, x_86, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_85); +return x_87; } } else { -uint8_t x_85; -lean_dec(x_61); -lean_dec(x_60); +uint8_t x_88; +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_26); lean_dec(x_2); -x_85 = !lean_is_exclusive(x_65); -if (x_85 == 0) +x_88 = !lean_is_exclusive(x_68); +if (x_88 == 0) { -return x_65; +return x_68; } else { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_65, 0); -x_87 = lean_ctor_get(x_65, 1); -lean_inc(x_87); -lean_inc(x_86); -lean_dec(x_65); -x_88 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_88, 0, x_86); -lean_ctor_set(x_88, 1, x_87); -return x_88; +lean_object* x_89; lean_object* x_90; lean_object* x_91; +x_89 = lean_ctor_get(x_68, 0); +x_90 = lean_ctor_get(x_68, 1); +lean_inc(x_90); +lean_inc(x_89); +lean_dec(x_68); +x_91 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_91, 0, x_89); +lean_ctor_set(x_91, 1, x_90); +return x_91; } } } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -lean_dec(x_61); -lean_dec(x_60); -x_89 = lean_ctor_get(x_62, 1); -lean_inc(x_89); -lean_dec(x_62); -x_90 = lean_ctor_get(x_63, 0); -lean_inc(x_90); +lean_object* x_92; lean_object* x_93; lean_object* x_94; +lean_dec(x_64); lean_dec(x_63); -x_91 = l_List_forM___at_Lean_Meta_Grind_intros_go___spec__1(x_2, x_90, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_89); -return x_91; +x_92 = lean_ctor_get(x_65, 1); +lean_inc(x_92); +lean_dec(x_65); +x_93 = lean_ctor_get(x_66, 0); +lean_inc(x_93); +lean_dec(x_66); +x_94 = l_List_forM___at_Lean_Meta_Grind_intros_go___spec__1(x_2, x_93, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_92); +return x_94; } } else { -uint8_t x_92; -lean_dec(x_61); -lean_dec(x_60); +uint8_t x_95; +lean_dec(x_64); +lean_dec(x_63); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_26); lean_dec(x_2); -x_92 = !lean_is_exclusive(x_62); -if (x_92 == 0) +x_95 = !lean_is_exclusive(x_65); +if (x_95 == 0) { -return x_62; +return x_65; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_62, 0); -x_94 = lean_ctor_get(x_62, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_62); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_object* x_96; lean_object* x_97; lean_object* x_98; +x_96 = lean_ctor_get(x_65, 0); +x_97 = lean_ctor_get(x_65, 1); +lean_inc(x_97); +lean_inc(x_96); +lean_dec(x_65); +x_98 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_98, 0, x_96); +lean_ctor_set(x_98, 1, x_97); +return x_98; } } } case 2: { -lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4712,7 +5314,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4720,18 +5322,21 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_96 = lean_ctor_get(x_34, 1); -lean_inc(x_96); -lean_dec(x_34); -x_97 = lean_ctor_get(x_35, 0); -lean_inc(x_97); -lean_dec(x_35); -x_98 = l_Lean_Meta_Grind_intros_go(x_2, x_97, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_96); -return x_98; +x_99 = lean_ctor_get(x_37, 1); +lean_inc(x_99); +lean_dec(x_37); +x_100 = lean_ctor_get(x_38, 0); +lean_inc(x_100); +lean_dec(x_38); +x_101 = l_Lean_Meta_Grind_intros_go(x_2, x_100, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_99); +return x_101; } default: { -lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4745,7 +5350,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4753,77 +5358,77 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_99 = lean_ctor_get(x_34, 1); -lean_inc(x_99); -lean_dec(x_34); -x_100 = lean_ctor_get(x_35, 0); -lean_inc(x_100); -x_101 = lean_ctor_get(x_35, 1); -lean_inc(x_101); -lean_dec(x_35); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_101); -x_102 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f(x_101, x_100, x_29, x_30, x_31, x_32, x_99); -if (lean_obj_tag(x_102) == 0) -{ -lean_object* x_103; -x_103 = lean_ctor_get(x_102, 0); +x_102 = lean_ctor_get(x_37, 1); +lean_inc(x_102); +lean_dec(x_37); +x_103 = lean_ctor_get(x_38, 0); lean_inc(x_103); -if (lean_obj_tag(x_103) == 0) -{ -lean_object* x_104; lean_object* x_105; -x_104 = lean_ctor_get(x_102, 1); +x_104 = lean_ctor_get(x_38, 1); lean_inc(x_104); -lean_dec(x_102); -x_105 = l_Lean_Meta_Grind_intros_go(x_2, x_101, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_104); -return x_105; -} -else +lean_dec(x_38); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_104); +x_105 = l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_applyCases_x3f(x_104, x_103, x_32, x_33, x_34, x_35, x_102); +if (lean_obj_tag(x_105) == 0) { -lean_object* x_106; lean_object* x_107; lean_object* x_108; -lean_dec(x_101); -x_106 = lean_ctor_get(x_102, 1); +lean_object* x_106; +x_106 = lean_ctor_get(x_105, 0); lean_inc(x_106); -lean_dec(x_102); -x_107 = lean_ctor_get(x_103, 0); +if (lean_obj_tag(x_106) == 0) +{ +lean_object* x_107; lean_object* x_108; +x_107 = lean_ctor_get(x_105, 1); lean_inc(x_107); -lean_dec(x_103); -x_108 = l_List_forM___at_Lean_Meta_Grind_intros_go___spec__2(x_2, x_107, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_106); +lean_dec(x_105); +x_108 = l_Lean_Meta_Grind_intros_go(x_2, x_104, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_107); return x_108; } +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; +lean_dec(x_104); +x_109 = lean_ctor_get(x_105, 1); +lean_inc(x_109); +lean_dec(x_105); +x_110 = lean_ctor_get(x_106, 0); +lean_inc(x_110); +lean_dec(x_106); +x_111 = l_List_forM___at_Lean_Meta_Grind_intros_go___spec__2(x_2, x_110, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_109); +return x_111; +} } else { -uint8_t x_109; -lean_dec(x_101); +uint8_t x_112; +lean_dec(x_104); +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); -lean_dec(x_26); lean_dec(x_2); -x_109 = !lean_is_exclusive(x_102); -if (x_109 == 0) +x_112 = !lean_is_exclusive(x_105); +if (x_112 == 0) { -return x_102; +return x_105; } else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_102, 0); -x_111 = lean_ctor_get(x_102, 1); -lean_inc(x_111); -lean_inc(x_110); -lean_dec(x_102); -x_112 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_112, 0, x_110); -lean_ctor_set(x_112, 1, x_111); -return x_112; +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_105, 0); +x_114 = lean_ctor_get(x_105, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_105); +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +return x_115; } } } @@ -4831,14 +5436,17 @@ return x_112; } else { -uint8_t x_113; +uint8_t x_116; +lean_dec(x_35); +lean_dec(x_34); +lean_dec(x_33); lean_dec(x_32); lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); -lean_dec(x_28); -lean_dec(x_27); lean_dec(x_26); +lean_dec(x_25); +lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); lean_dec(x_21); @@ -4852,7 +5460,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4861,23 +5469,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_113 = !lean_is_exclusive(x_34); -if (x_113 == 0) +x_116 = !lean_is_exclusive(x_37); +if (x_116 == 0) { -return x_34; +return x_37; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_114 = lean_ctor_get(x_34, 0); -x_115 = lean_ctor_get(x_34, 1); -lean_inc(x_115); -lean_inc(x_114); -lean_dec(x_34); -x_116 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_116, 0, x_114); -lean_ctor_set(x_116, 1, x_115); -return x_116; +lean_object* x_117; lean_object* x_118; lean_object* x_119; +x_117 = lean_ctor_get(x_37, 0); +x_118 = lean_ctor_get(x_37, 1); +lean_inc(x_118); +lean_inc(x_117); +lean_dec(x_37); +x_119 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_119, 0, x_117); +lean_ctor_set(x_119, 1, x_118); +return x_119; } } } @@ -4886,10 +5494,10 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go(lean_object* x_1, lean_obje _start: { uint8_t x_12; -x_12 = lean_ctor_get_uint8(x_2, sizeof(void*)*20); +x_12 = lean_ctor_get_uint8(x_2, sizeof(void*)*23); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; x_13 = lean_ctor_get(x_2, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_2, 1); @@ -4930,13 +5538,19 @@ x_31 = lean_ctor_get(x_2, 18); lean_inc(x_31); x_32 = lean_ctor_get(x_2, 19); lean_inc(x_32); -x_33 = lean_box(0); -x_34 = l_Lean_Meta_Grind_intros_go___lambda__2(x_2, x_1, x_13, x_14, x_15, x_16, x_17, x_18, x_12, x_19, x_20, x_21, x_22, x_23, x_24, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_34; +x_33 = lean_ctor_get(x_2, 20); +lean_inc(x_33); +x_34 = lean_ctor_get(x_2, 21); +lean_inc(x_34); +x_35 = lean_ctor_get(x_2, 22); +lean_inc(x_35); +x_36 = lean_box(0); +x_37 = l_Lean_Meta_Grind_intros_go___lambda__2(x_2, x_1, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_12, x_20, x_21, x_22, x_23, x_24, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_37; } else { -lean_object* x_35; lean_object* x_36; +lean_object* x_38; lean_object* x_39; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -4946,11 +5560,11 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_35 = lean_box(0); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_11); -return x_36; +x_38 = lean_box(0); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_11); +return x_39; } } } @@ -5006,15 +5620,18 @@ lean_object* x_30 = _args[29]; lean_object* x_31 = _args[30]; lean_object* x_32 = _args[31]; lean_object* x_33 = _args[32]; +lean_object* x_34 = _args[33]; +lean_object* x_35 = _args[34]; +lean_object* x_36 = _args[35]; _start: { -uint8_t x_34; lean_object* x_35; -x_34 = lean_unbox(x_9); -lean_dec(x_9); -x_35 = l_Lean_Meta_Grind_intros_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_34, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_24, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33); -lean_dec(x_25); -lean_dec(x_24); -return x_35; +uint8_t x_37; lean_object* x_38; +x_37 = lean_unbox(x_10); +lean_dec(x_10); +x_38 = l_Lean_Meta_Grind_intros_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_37, x_11, x_12, x_13, x_14, x_15, x_16, x_17, x_18, x_19, x_20, x_21, x_22, x_23, x_24, x_25, x_26, x_27, x_28, x_29, x_30, x_31, x_32, x_33, x_34, x_35, x_36); +lean_dec(x_28); +lean_dec(x_27); +return x_38; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_intros_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { @@ -5113,7 +5730,7 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_6); -x_13 = l_Lean_Meta_Grind_simp(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_13 = l_Lean_Meta_Grind_simp(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_13) == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; @@ -5408,7 +6025,7 @@ if (lean_obj_tag(x_25) == 0) lean_object* x_26; uint8_t x_27; x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); -x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*20); +x_27 = lean_ctor_get_uint8(x_26, sizeof(void*)*23); if (x_27 == 0) { uint8_t x_28; @@ -5521,7 +6138,7 @@ if (lean_obj_tag(x_51) == 0) lean_object* x_52; uint8_t x_53; x_52 = lean_ctor_get(x_51, 0); lean_inc(x_52); -x_53 = lean_ctor_get_uint8(x_52, sizeof(void*)*20); +x_53 = lean_ctor_get_uint8(x_52, sizeof(void*)*23); if (x_53 == 0) { lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; @@ -5615,7 +6232,7 @@ lean_dec(x_69); x_72 = !lean_is_exclusive(x_4); if (x_72 == 0) { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; x_73 = lean_ctor_get(x_4, 0); x_74 = lean_ctor_get(x_4, 1); x_75 = lean_ctor_get(x_4, 2); @@ -5636,27 +6253,33 @@ x_89 = lean_ctor_get(x_4, 16); x_90 = lean_ctor_get(x_4, 17); x_91 = lean_ctor_get(x_4, 18); x_92 = lean_ctor_get(x_4, 19); +x_93 = lean_ctor_get(x_4, 20); +x_94 = lean_ctor_get(x_4, 21); +x_95 = lean_ctor_get(x_4, 22); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_93 = l_Lean_MVarId_assert(x_73, x_70, x_2, x_1, x_8, x_9, x_10, x_11, x_71); -if (lean_obj_tag(x_93) == 0) +x_96 = l_Lean_MVarId_assert(x_73, x_70, x_2, x_1, x_8, x_9, x_10, x_11, x_71); +if (lean_obj_tag(x_96) == 0) { -lean_object* x_94; lean_object* x_95; lean_object* x_96; -x_94 = lean_ctor_get(x_93, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_93, 1); -lean_inc(x_95); -lean_dec(x_93); -lean_ctor_set(x_4, 0, x_94); -x_96 = l_Lean_Meta_Grind_intros(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_95); -return x_96; +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_96, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_96, 1); +lean_inc(x_98); +lean_dec(x_96); +lean_ctor_set(x_4, 0, x_97); +x_99 = l_Lean_Meta_Grind_intros(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_98); +return x_99; } else { -uint8_t x_97; +uint8_t x_100; lean_free_object(x_4); +lean_dec(x_95); +lean_dec(x_94); +lean_dec(x_93); lean_dec(x_92); lean_dec(x_91); lean_dec(x_90); @@ -5684,50 +6307,59 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_97 = !lean_is_exclusive(x_93); -if (x_97 == 0) +x_100 = !lean_is_exclusive(x_96); +if (x_100 == 0) { -return x_93; +return x_96; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_93, 0); -x_99 = lean_ctor_get(x_93, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_93); -x_100 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_100, 0, x_98); -lean_ctor_set(x_100, 1, x_99); -return x_100; +lean_object* x_101; lean_object* x_102; lean_object* x_103; +x_101 = lean_ctor_get(x_96, 0); +x_102 = lean_ctor_get(x_96, 1); +lean_inc(x_102); +lean_inc(x_101); +lean_dec(x_96); +x_103 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_103, 0, x_101); +lean_ctor_set(x_103, 1, x_102); +return x_103; } } } else { -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_101 = lean_ctor_get(x_4, 0); -x_102 = lean_ctor_get(x_4, 1); -x_103 = lean_ctor_get(x_4, 2); -x_104 = lean_ctor_get(x_4, 3); -x_105 = lean_ctor_get(x_4, 4); -x_106 = lean_ctor_get(x_4, 5); -x_107 = lean_ctor_get_uint8(x_4, sizeof(void*)*20); -x_108 = lean_ctor_get(x_4, 6); -x_109 = lean_ctor_get(x_4, 7); -x_110 = lean_ctor_get(x_4, 8); -x_111 = lean_ctor_get(x_4, 9); -x_112 = lean_ctor_get(x_4, 10); -x_113 = lean_ctor_get(x_4, 11); -x_114 = lean_ctor_get(x_4, 12); -x_115 = lean_ctor_get(x_4, 13); -x_116 = lean_ctor_get(x_4, 14); -x_117 = lean_ctor_get(x_4, 15); -x_118 = lean_ctor_get(x_4, 16); -x_119 = lean_ctor_get(x_4, 17); -x_120 = lean_ctor_get(x_4, 18); -x_121 = lean_ctor_get(x_4, 19); +lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; uint8_t x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_104 = lean_ctor_get(x_4, 0); +x_105 = lean_ctor_get(x_4, 1); +x_106 = lean_ctor_get(x_4, 2); +x_107 = lean_ctor_get(x_4, 3); +x_108 = lean_ctor_get(x_4, 4); +x_109 = lean_ctor_get(x_4, 5); +x_110 = lean_ctor_get(x_4, 6); +x_111 = lean_ctor_get_uint8(x_4, sizeof(void*)*23); +x_112 = lean_ctor_get(x_4, 7); +x_113 = lean_ctor_get(x_4, 8); +x_114 = lean_ctor_get(x_4, 9); +x_115 = lean_ctor_get(x_4, 10); +x_116 = lean_ctor_get(x_4, 11); +x_117 = lean_ctor_get(x_4, 12); +x_118 = lean_ctor_get(x_4, 13); +x_119 = lean_ctor_get(x_4, 14); +x_120 = lean_ctor_get(x_4, 15); +x_121 = lean_ctor_get(x_4, 16); +x_122 = lean_ctor_get(x_4, 17); +x_123 = lean_ctor_get(x_4, 18); +x_124 = lean_ctor_get(x_4, 19); +x_125 = lean_ctor_get(x_4, 20); +x_126 = lean_ctor_get(x_4, 21); +x_127 = lean_ctor_get(x_4, 22); +lean_inc(x_127); +lean_inc(x_126); +lean_inc(x_125); +lean_inc(x_124); +lean_inc(x_123); +lean_inc(x_122); lean_inc(x_121); lean_inc(x_120); lean_inc(x_119); @@ -5738,58 +6370,64 @@ lean_inc(x_115); lean_inc(x_114); lean_inc(x_113); lean_inc(x_112); -lean_inc(x_111); lean_inc(x_110); lean_inc(x_109); lean_inc(x_108); +lean_inc(x_107); lean_inc(x_106); lean_inc(x_105); lean_inc(x_104); -lean_inc(x_103); -lean_inc(x_102); -lean_inc(x_101); lean_dec(x_4); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_122 = l_Lean_MVarId_assert(x_101, x_70, x_2, x_1, x_8, x_9, x_10, x_11, x_71); -if (lean_obj_tag(x_122) == 0) +x_128 = l_Lean_MVarId_assert(x_104, x_70, x_2, x_1, x_8, x_9, x_10, x_11, x_71); +if (lean_obj_tag(x_128) == 0) { -lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_123 = lean_ctor_get(x_122, 0); -lean_inc(x_123); -x_124 = lean_ctor_get(x_122, 1); -lean_inc(x_124); +lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_129 = lean_ctor_get(x_128, 0); +lean_inc(x_129); +x_130 = lean_ctor_get(x_128, 1); +lean_inc(x_130); +lean_dec(x_128); +x_131 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_131, 0, x_129); +lean_ctor_set(x_131, 1, x_105); +lean_ctor_set(x_131, 2, x_106); +lean_ctor_set(x_131, 3, x_107); +lean_ctor_set(x_131, 4, x_108); +lean_ctor_set(x_131, 5, x_109); +lean_ctor_set(x_131, 6, x_110); +lean_ctor_set(x_131, 7, x_112); +lean_ctor_set(x_131, 8, x_113); +lean_ctor_set(x_131, 9, x_114); +lean_ctor_set(x_131, 10, x_115); +lean_ctor_set(x_131, 11, x_116); +lean_ctor_set(x_131, 12, x_117); +lean_ctor_set(x_131, 13, x_118); +lean_ctor_set(x_131, 14, x_119); +lean_ctor_set(x_131, 15, x_120); +lean_ctor_set(x_131, 16, x_121); +lean_ctor_set(x_131, 17, x_122); +lean_ctor_set(x_131, 18, x_123); +lean_ctor_set(x_131, 19, x_124); +lean_ctor_set(x_131, 20, x_125); +lean_ctor_set(x_131, 21, x_126); +lean_ctor_set(x_131, 22, x_127); +lean_ctor_set_uint8(x_131, sizeof(void*)*23, x_111); +x_132 = l_Lean_Meta_Grind_intros(x_3, x_131, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_130); +return x_132; +} +else +{ +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; +lean_dec(x_127); +lean_dec(x_126); +lean_dec(x_125); +lean_dec(x_124); +lean_dec(x_123); lean_dec(x_122); -x_125 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_102); -lean_ctor_set(x_125, 2, x_103); -lean_ctor_set(x_125, 3, x_104); -lean_ctor_set(x_125, 4, x_105); -lean_ctor_set(x_125, 5, x_106); -lean_ctor_set(x_125, 6, x_108); -lean_ctor_set(x_125, 7, x_109); -lean_ctor_set(x_125, 8, x_110); -lean_ctor_set(x_125, 9, x_111); -lean_ctor_set(x_125, 10, x_112); -lean_ctor_set(x_125, 11, x_113); -lean_ctor_set(x_125, 12, x_114); -lean_ctor_set(x_125, 13, x_115); -lean_ctor_set(x_125, 14, x_116); -lean_ctor_set(x_125, 15, x_117); -lean_ctor_set(x_125, 16, x_118); -lean_ctor_set(x_125, 17, x_119); -lean_ctor_set(x_125, 18, x_120); -lean_ctor_set(x_125, 19, x_121); -lean_ctor_set_uint8(x_125, sizeof(void*)*20, x_107); -x_126 = l_Lean_Meta_Grind_intros(x_3, x_125, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_124); -return x_126; -} -else -{ -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_dec(x_121); lean_dec(x_120); lean_dec(x_119); @@ -5800,15 +6438,12 @@ lean_dec(x_115); lean_dec(x_114); lean_dec(x_113); lean_dec(x_112); -lean_dec(x_111); lean_dec(x_110); lean_dec(x_109); lean_dec(x_108); +lean_dec(x_107); lean_dec(x_106); lean_dec(x_105); -lean_dec(x_104); -lean_dec(x_103); -lean_dec(x_102); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5817,26 +6452,26 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_127 = lean_ctor_get(x_122, 0); -lean_inc(x_127); -x_128 = lean_ctor_get(x_122, 1); -lean_inc(x_128); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_129 = x_122; +x_133 = lean_ctor_get(x_128, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_128, 1); +lean_inc(x_134); +if (lean_is_exclusive(x_128)) { + lean_ctor_release(x_128, 0); + lean_ctor_release(x_128, 1); + x_135 = x_128; } else { - lean_dec_ref(x_122); - x_129 = lean_box(0); + lean_dec_ref(x_128); + x_135 = lean_box(0); } -if (lean_is_scalar(x_129)) { - x_130 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_135)) { + x_136 = lean_alloc_ctor(1, 2, 0); } else { - x_130 = x_129; + x_136 = x_135; } -lean_ctor_set(x_130, 0, x_127); -lean_ctor_set(x_130, 1, x_128); -return x_130; +lean_ctor_set(x_136, 0, x_133); +lean_ctor_set(x_136, 1, x_134); +return x_136; } } } @@ -5849,7 +6484,7 @@ uint8_t x_10; x_10 = !lean_is_exclusive(x_1); if (x_10 == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; x_11 = lean_ctor_get(x_1, 0); x_12 = lean_ctor_get(x_1, 1); x_13 = lean_ctor_get(x_1, 2); @@ -5870,16 +6505,22 @@ x_27 = lean_ctor_get(x_1, 16); x_28 = lean_ctor_get(x_1, 17); x_29 = lean_ctor_get(x_1, 18); x_30 = lean_ctor_get(x_1, 19); -x_31 = l_Std_Queue_dequeue_x3f___rarg(x_25); -if (lean_obj_tag(x_31) == 0) +x_31 = lean_ctor_get(x_1, 20); +x_32 = lean_ctor_get(x_1, 21); +x_33 = lean_ctor_get(x_1, 22); +x_34 = l_Std_Queue_dequeue_x3f___rarg(x_27); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_32; lean_object* x_33; +lean_object* x_35; lean_object* x_36; lean_free_object(x_1); +lean_dec(x_33); +lean_dec(x_32); +lean_dec(x_31); lean_dec(x_30); lean_dec(x_29); lean_dec(x_28); -lean_dec(x_27); lean_dec(x_26); +lean_dec(x_25); lean_dec(x_24); lean_dec(x_23); lean_dec(x_22); @@ -5901,182 +6542,191 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_9); -return x_33; +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_9); +return x_36; } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_31); -if (x_34 == 0) +uint8_t x_37; +x_37 = !lean_is_exclusive(x_34); +if (x_37 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_35 = lean_ctor_get(x_31, 0); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_ctor_get(x_36, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_36, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_38 = lean_ctor_get(x_34, 0); +x_39 = lean_ctor_get(x_38, 0); lean_inc(x_39); -x_40 = lean_ctor_get(x_36, 2); +x_40 = lean_ctor_get(x_38, 1); lean_inc(x_40); -lean_dec(x_36); -lean_ctor_set(x_1, 14, x_37); -x_41 = l_Lean_Meta_Grind_assertAt(x_38, x_39, x_40, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_41) == 0) +lean_dec(x_38); +x_41 = lean_ctor_get(x_39, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +x_43 = lean_ctor_get(x_39, 2); +lean_inc(x_43); +lean_dec(x_39); +lean_ctor_set(x_1, 16, x_40); +x_44 = l_Lean_Meta_Grind_assertAt(x_41, x_42, x_43, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_44) == 0) { -uint8_t x_42; -x_42 = !lean_is_exclusive(x_41); -if (x_42 == 0) +uint8_t x_45; +x_45 = !lean_is_exclusive(x_44); +if (x_45 == 0) { -lean_object* x_43; -x_43 = lean_ctor_get(x_41, 0); -lean_ctor_set(x_31, 0, x_43); -lean_ctor_set(x_41, 0, x_31); -return x_41; +lean_object* x_46; +x_46 = lean_ctor_get(x_44, 0); +lean_ctor_set(x_34, 0, x_46); +lean_ctor_set(x_44, 0, x_34); +return x_44; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_41, 0); -x_45 = lean_ctor_get(x_41, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_41); -lean_ctor_set(x_31, 0, x_44); -x_46 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_46, 0, x_31); -lean_ctor_set(x_46, 1, x_45); -return x_46; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_44, 0); +x_48 = lean_ctor_get(x_44, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_44); +lean_ctor_set(x_34, 0, x_47); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_34); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } else { -uint8_t x_47; -lean_free_object(x_31); -x_47 = !lean_is_exclusive(x_41); -if (x_47 == 0) +uint8_t x_50; +lean_free_object(x_34); +x_50 = !lean_is_exclusive(x_44); +if (x_50 == 0) { -return x_41; +return x_44; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_41, 0); -x_49 = lean_ctor_get(x_41, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_41); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_44, 0); +x_52 = lean_ctor_get(x_44, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_44); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; } } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_51 = lean_ctor_get(x_31, 0); -lean_inc(x_51); -lean_dec(x_31); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = lean_ctor_get(x_52, 0); +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_54 = lean_ctor_get(x_34, 0); lean_inc(x_54); -x_55 = lean_ctor_get(x_52, 1); +lean_dec(x_34); +x_55 = lean_ctor_get(x_54, 0); lean_inc(x_55); -x_56 = lean_ctor_get(x_52, 2); +x_56 = lean_ctor_get(x_54, 1); lean_inc(x_56); -lean_dec(x_52); -lean_ctor_set(x_1, 14, x_53); -x_57 = l_Lean_Meta_Grind_assertAt(x_54, x_55, x_56, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_58 = lean_ctor_get(x_57, 0); +lean_dec(x_54); +x_57 = lean_ctor_get(x_55, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_55, 1); lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); +x_59 = lean_ctor_get(x_55, 2); lean_inc(x_59); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_60 = x_57; +lean_dec(x_55); +lean_ctor_set(x_1, 16, x_56); +x_60 = l_Lean_Meta_Grind_assertAt(x_57, x_58, x_59, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_60) == 0) +{ +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_ctor_get(x_60, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_63 = x_60; } else { - lean_dec_ref(x_57); - x_60 = lean_box(0); + lean_dec_ref(x_60); + x_63 = lean_box(0); } -x_61 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_61, 0, x_58); -if (lean_is_scalar(x_60)) { - x_62 = lean_alloc_ctor(0, 2, 0); +x_64 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_64, 0, x_61); +if (lean_is_scalar(x_63)) { + x_65 = lean_alloc_ctor(0, 2, 0); } else { - x_62 = x_60; + x_65 = x_63; } -lean_ctor_set(x_62, 0, x_61); -lean_ctor_set(x_62, 1, x_59); -return x_62; +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_62); +return x_65; } else { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_63 = lean_ctor_get(x_57, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_57, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_65 = x_57; +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_66 = lean_ctor_get(x_60, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_60, 1); +lean_inc(x_67); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_68 = x_60; } else { - lean_dec_ref(x_57); - x_65 = lean_box(0); + lean_dec_ref(x_60); + x_68 = lean_box(0); } -if (lean_is_scalar(x_65)) { - x_66 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_68)) { + x_69 = lean_alloc_ctor(1, 2, 0); } else { - x_66 = x_65; -} -lean_ctor_set(x_66, 0, x_63); -lean_ctor_set(x_66, 1, x_64); -return x_66; -} -} -} -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_67 = lean_ctor_get(x_1, 0); -x_68 = lean_ctor_get(x_1, 1); -x_69 = lean_ctor_get(x_1, 2); -x_70 = lean_ctor_get(x_1, 3); -x_71 = lean_ctor_get(x_1, 4); -x_72 = lean_ctor_get(x_1, 5); -x_73 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_74 = lean_ctor_get(x_1, 6); -x_75 = lean_ctor_get(x_1, 7); -x_76 = lean_ctor_get(x_1, 8); -x_77 = lean_ctor_get(x_1, 9); -x_78 = lean_ctor_get(x_1, 10); -x_79 = lean_ctor_get(x_1, 11); -x_80 = lean_ctor_get(x_1, 12); -x_81 = lean_ctor_get(x_1, 13); -x_82 = lean_ctor_get(x_1, 14); -x_83 = lean_ctor_get(x_1, 15); -x_84 = lean_ctor_get(x_1, 16); -x_85 = lean_ctor_get(x_1, 17); -x_86 = lean_ctor_get(x_1, 18); -x_87 = lean_ctor_get(x_1, 19); + x_69 = x_68; +} +lean_ctor_set(x_69, 0, x_66); +lean_ctor_set(x_69, 1, x_67); +return x_69; +} +} +} +} +else +{ +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_70 = lean_ctor_get(x_1, 0); +x_71 = lean_ctor_get(x_1, 1); +x_72 = lean_ctor_get(x_1, 2); +x_73 = lean_ctor_get(x_1, 3); +x_74 = lean_ctor_get(x_1, 4); +x_75 = lean_ctor_get(x_1, 5); +x_76 = lean_ctor_get(x_1, 6); +x_77 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); +x_78 = lean_ctor_get(x_1, 7); +x_79 = lean_ctor_get(x_1, 8); +x_80 = lean_ctor_get(x_1, 9); +x_81 = lean_ctor_get(x_1, 10); +x_82 = lean_ctor_get(x_1, 11); +x_83 = lean_ctor_get(x_1, 12); +x_84 = lean_ctor_get(x_1, 13); +x_85 = lean_ctor_get(x_1, 14); +x_86 = lean_ctor_get(x_1, 15); +x_87 = lean_ctor_get(x_1, 16); +x_88 = lean_ctor_get(x_1, 17); +x_89 = lean_ctor_get(x_1, 18); +x_90 = lean_ctor_get(x_1, 19); +x_91 = lean_ctor_get(x_1, 20); +x_92 = lean_ctor_get(x_1, 21); +x_93 = lean_ctor_get(x_1, 22); +lean_inc(x_93); +lean_inc(x_92); +lean_inc(x_91); +lean_inc(x_90); +lean_inc(x_89); +lean_inc(x_88); lean_inc(x_87); lean_inc(x_86); lean_inc(x_85); @@ -6087,40 +6737,40 @@ lean_inc(x_81); lean_inc(x_80); lean_inc(x_79); lean_inc(x_78); -lean_inc(x_77); lean_inc(x_76); lean_inc(x_75); lean_inc(x_74); +lean_inc(x_73); lean_inc(x_72); lean_inc(x_71); lean_inc(x_70); -lean_inc(x_69); -lean_inc(x_68); -lean_inc(x_67); lean_dec(x_1); -x_88 = l_Std_Queue_dequeue_x3f___rarg(x_82); -if (lean_obj_tag(x_88) == 0) +x_94 = l_Std_Queue_dequeue_x3f___rarg(x_87); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_89; lean_object* x_90; -lean_dec(x_87); +lean_object* x_95; lean_object* x_96; +lean_dec(x_93); +lean_dec(x_92); +lean_dec(x_91); +lean_dec(x_90); +lean_dec(x_89); +lean_dec(x_88); lean_dec(x_86); lean_dec(x_85); lean_dec(x_84); lean_dec(x_83); +lean_dec(x_82); lean_dec(x_81); lean_dec(x_80); lean_dec(x_79); lean_dec(x_78); -lean_dec(x_77); lean_dec(x_76); lean_dec(x_75); lean_dec(x_74); +lean_dec(x_73); lean_dec(x_72); lean_dec(x_71); lean_dec(x_70); -lean_dec(x_69); -lean_dec(x_68); -lean_dec(x_67); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -6128,113 +6778,116 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_89 = lean_box(0); -x_90 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_90, 0, x_89); -lean_ctor_set(x_90, 1, x_9); -return x_90; +x_95 = lean_box(0); +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_95); +lean_ctor_set(x_96, 1, x_9); +return x_96; } else { -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; -x_91 = lean_ctor_get(x_88, 0); -lean_inc(x_91); -if (lean_is_exclusive(x_88)) { - lean_ctor_release(x_88, 0); - x_92 = x_88; +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; +x_97 = lean_ctor_get(x_94, 0); +lean_inc(x_97); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + x_98 = x_94; } else { - lean_dec_ref(x_88); - x_92 = lean_box(0); + lean_dec_ref(x_94); + x_98 = lean_box(0); } -x_93 = lean_ctor_get(x_91, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_91, 1); -lean_inc(x_94); -lean_dec(x_91); -x_95 = lean_ctor_get(x_93, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_93, 1); -lean_inc(x_96); -x_97 = lean_ctor_get(x_93, 2); -lean_inc(x_97); -lean_dec(x_93); -x_98 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_98, 0, x_67); -lean_ctor_set(x_98, 1, x_68); -lean_ctor_set(x_98, 2, x_69); -lean_ctor_set(x_98, 3, x_70); -lean_ctor_set(x_98, 4, x_71); -lean_ctor_set(x_98, 5, x_72); -lean_ctor_set(x_98, 6, x_74); -lean_ctor_set(x_98, 7, x_75); -lean_ctor_set(x_98, 8, x_76); -lean_ctor_set(x_98, 9, x_77); -lean_ctor_set(x_98, 10, x_78); -lean_ctor_set(x_98, 11, x_79); -lean_ctor_set(x_98, 12, x_80); -lean_ctor_set(x_98, 13, x_81); -lean_ctor_set(x_98, 14, x_94); -lean_ctor_set(x_98, 15, x_83); -lean_ctor_set(x_98, 16, x_84); -lean_ctor_set(x_98, 17, x_85); -lean_ctor_set(x_98, 18, x_86); -lean_ctor_set(x_98, 19, x_87); -lean_ctor_set_uint8(x_98, sizeof(void*)*20, x_73); -x_99 = l_Lean_Meta_Grind_assertAt(x_95, x_96, x_97, x_98, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_99) == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_100 = lean_ctor_get(x_99, 0); +x_99 = lean_ctor_get(x_97, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_97, 1); lean_inc(x_100); -x_101 = lean_ctor_get(x_99, 1); +lean_dec(x_97); +x_101 = lean_ctor_get(x_99, 0); lean_inc(x_101); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_102 = x_99; +x_102 = lean_ctor_get(x_99, 1); +lean_inc(x_102); +x_103 = lean_ctor_get(x_99, 2); +lean_inc(x_103); +lean_dec(x_99); +x_104 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_104, 0, x_70); +lean_ctor_set(x_104, 1, x_71); +lean_ctor_set(x_104, 2, x_72); +lean_ctor_set(x_104, 3, x_73); +lean_ctor_set(x_104, 4, x_74); +lean_ctor_set(x_104, 5, x_75); +lean_ctor_set(x_104, 6, x_76); +lean_ctor_set(x_104, 7, x_78); +lean_ctor_set(x_104, 8, x_79); +lean_ctor_set(x_104, 9, x_80); +lean_ctor_set(x_104, 10, x_81); +lean_ctor_set(x_104, 11, x_82); +lean_ctor_set(x_104, 12, x_83); +lean_ctor_set(x_104, 13, x_84); +lean_ctor_set(x_104, 14, x_85); +lean_ctor_set(x_104, 15, x_86); +lean_ctor_set(x_104, 16, x_100); +lean_ctor_set(x_104, 17, x_88); +lean_ctor_set(x_104, 18, x_89); +lean_ctor_set(x_104, 19, x_90); +lean_ctor_set(x_104, 20, x_91); +lean_ctor_set(x_104, 21, x_92); +lean_ctor_set(x_104, 22, x_93); +lean_ctor_set_uint8(x_104, sizeof(void*)*23, x_77); +x_105 = l_Lean_Meta_Grind_assertAt(x_101, x_102, x_103, x_104, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_105) == 0) +{ +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_106 = lean_ctor_get(x_105, 0); +lean_inc(x_106); +x_107 = lean_ctor_get(x_105, 1); +lean_inc(x_107); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_108 = x_105; } else { - lean_dec_ref(x_99); - x_102 = lean_box(0); + lean_dec_ref(x_105); + x_108 = lean_box(0); } -if (lean_is_scalar(x_92)) { - x_103 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_98)) { + x_109 = lean_alloc_ctor(1, 1, 0); } else { - x_103 = x_92; + x_109 = x_98; } -lean_ctor_set(x_103, 0, x_100); -if (lean_is_scalar(x_102)) { - x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_109, 0, x_106); +if (lean_is_scalar(x_108)) { + x_110 = lean_alloc_ctor(0, 2, 0); } else { - x_104 = x_102; + x_110 = x_108; } -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_101); -return x_104; +lean_ctor_set(x_110, 0, x_109); +lean_ctor_set(x_110, 1, x_107); +return x_110; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -lean_dec(x_92); -x_105 = lean_ctor_get(x_99, 0); -lean_inc(x_105); -x_106 = lean_ctor_get(x_99, 1); -lean_inc(x_106); -if (lean_is_exclusive(x_99)) { - lean_ctor_release(x_99, 0); - lean_ctor_release(x_99, 1); - x_107 = x_99; +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_dec(x_98); +x_111 = lean_ctor_get(x_105, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_105, 1); +lean_inc(x_112); +if (lean_is_exclusive(x_105)) { + lean_ctor_release(x_105, 0); + lean_ctor_release(x_105, 1); + x_113 = x_105; } else { - lean_dec_ref(x_99); - x_107 = lean_box(0); + lean_dec_ref(x_105); + x_113 = lean_box(0); } -if (lean_is_scalar(x_107)) { - x_108 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_113)) { + x_114 = lean_alloc_ctor(1, 2, 0); } else { - x_108 = x_107; + x_114 = x_113; } -lean_ctor_set(x_108, 0, x_105); -lean_ctor_set(x_108, 1, x_106); -return x_108; +lean_ctor_set(x_114, 0, x_111); +lean_ctor_set(x_114, 1, x_112); +return x_114; } } } @@ -6298,14 +6951,14 @@ l_Lean_Meta_Grind_instInhabitedIntroResult = _init_l_Lean_Meta_Grind_instInhabit lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedIntroResult); l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__5___closed__1); -l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__1); -l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__2); -l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__3); -l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__8___closed__4); +l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__1); +l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__2); +l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__3); +l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Intro_0__Lean_Meta_Grind_introNext___lambda__7___closed__4); l_Lean_Meta_Grind_intros___closed__1 = _init_l_Lean_Meta_Grind_intros___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_intros___closed__1); l_Lean_Meta_Grind_assertAt___closed__1 = _init_l_Lean_Meta_Grind_assertAt___closed__1(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Inv.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Inv.c index 7b27280575ef..c6617ed68746 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Inv.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Inv.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind.Inv -// Imports: Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Proof +// Imports: Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Proof Lean.Meta.Tactic.Grind.Arith.Inv #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -25,12 +25,14 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_ch LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___boxed(lean_object**); static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__1___closed__4; size_t lean_usize_shift_right(size_t, size_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2___closed__1; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__3; static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__3; +lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_checkInvariants___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux___at_Lean_Meta_Grind_checkInvariants___spec__3(lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); @@ -43,7 +45,6 @@ lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAux___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__5(lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_Meta_Grind_checkInvariants___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___closed__2; uint64_t l_Lean_Meta_Grind_congrHash(lean_object*, lean_object*); @@ -51,13 +52,16 @@ lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_checkInvariants___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Grind_grind_debug_proofs; +lean_object* l_Lean_Meta_Grind_Goal_getNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__6; -lean_object* l_Lean_Meta_Grind_getEqcs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_checkInvariants___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_checkInvariants(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Grind_grind_debug; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__8; @@ -66,14 +70,12 @@ static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_ extern lean_object* l_instInhabitedNat; extern lean_object* l_instInhabitedPUnit; static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__3; -lean_object* l_Lean_Meta_Grind_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__1___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___closed__1; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__5; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__3; -lean_object* l_Lean_Meta_Grind_getTarget_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__3; @@ -90,6 +92,7 @@ static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Gr LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getCongrRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEqHEqProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f(lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__2; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__5; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -101,6 +104,7 @@ lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__4; static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__1___lambda__1___closed__1; +uint8_t l_Lean_Expr_hasLooseBVars(lean_object*); static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_checkInvariants___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAux___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -111,7 +115,6 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux_traverse___at_Lean_M LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_checkInvariants___closed__1; static size_t l_Lean_PersistentHashMap_findEntryAux___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__5___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__7; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__3___boxed(lean_object**); @@ -119,7 +122,6 @@ uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); uint8_t lean_expr_equal(lean_object*, lean_object*); uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__1; -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getParents(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,12 +139,12 @@ lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__1; lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__1___closed__5; static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__7; static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__1___closed__6; lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getEqcs(lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -152,6 +154,7 @@ LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_G lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__1___closed__1; static lean_object* l_Lean_Meta_Grind_Goal_checkInvariants___closed__1; +lean_object* l_Lean_Meta_Grind_Goal_getRoot_x3f(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntry_x3f___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__4(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); @@ -187,8 +190,8 @@ lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1; lean_object* lean_array_get_size(lean_object*); +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -202,12 +205,12 @@ LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_G static lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_checkInvariants___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Meta_Grind_checkInvariants___spec__4(lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getRoot_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* l_ReaderT_instMonad___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlMAux___at_Lean_Meta_Grind_checkInvariants___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__1; static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__1() { _start: @@ -290,50 +293,64 @@ return x_13; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Meta_Grind_getTarget_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_13, x_1); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_14; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); lean_ctor_set(x_11, 0, x_1); return x_11; } else { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_11, 1); -lean_inc(x_15); -lean_dec(x_11); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_1); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_object* x_16; +lean_free_object(x_11); +lean_dec(x_1); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +x_1 = x_16; +x_10 = x_14; +goto _start; } } else { -lean_object* x_17; lean_object* x_18; -lean_dec(x_1); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = lean_ctor_get(x_12, 0); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_11, 0); +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); lean_inc(x_18); -lean_dec(x_12); -x_1 = x_18; -x_10 = x_17; +lean_dec(x_11); +x_20 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_18, x_1); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_1); +lean_ctor_set(x_21, 1, x_19); +return x_21; +} +else +{ +lean_object* x_22; +lean_dec(x_1); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +lean_dec(x_20); +x_1 = x_22; +x_10 = x_19; goto _start; } } } +} LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -348,7 +365,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntryAtAux___at___private_ _start: { lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_1, 1); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); x_8 = lean_array_get_size(x_2); x_9 = lean_nat_dec_lt(x_5, x_8); @@ -429,7 +446,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_6 = lean_ctor_get(x_2, 0); -x_7 = lean_ctor_get(x_1, 1); +x_7 = lean_ctor_get(x_1, 2); lean_inc(x_7); x_8 = 5; x_9 = l_Lean_PersistentHashMap_findEntryAux___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__5___closed__2; @@ -531,7 +548,7 @@ lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; size_t x_32; lea x_28 = lean_ctor_get(x_2, 0); lean_inc(x_28); lean_dec(x_2); -x_29 = lean_ctor_get(x_1, 1); +x_29 = lean_ctor_get(x_1, 2); lean_inc(x_29); x_30 = 5; x_31 = l_Lean_PersistentHashMap_findEntryAux___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__5___closed__2; @@ -628,7 +645,7 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findEntry_x3f___at___private_L _start: { lean_object* x_4; uint64_t x_5; size_t x_6; lean_object* x_7; -x_4 = lean_ctor_get(x_1, 1); +x_4 = lean_ctor_get(x_1, 2); lean_inc(x_4); lean_inc(x_3); x_5 = l_Lean_Meta_Grind_congrHash(x_4, x_3); @@ -685,7 +702,7 @@ static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(40u); +x_3 = lean_unsigned_to_nat(41u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -695,161 +712,145 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_14; uint8_t x_15; +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_inc(x_3); x_14 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__2(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_16, x_1); -lean_dec(x_16); -if (x_18 == 0) +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_15, x_1); +lean_dec(x_15); +if (x_17 == 0) { -lean_object* x_19; lean_object* x_20; -lean_free_object(x_14); +lean_object* x_18; lean_object* x_19; lean_dec(x_3); lean_dec(x_2); -x_19 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__6; -x_20 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__3(x_19, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -return x_20; +x_18 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__6; +x_19 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__3(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); +return x_19; } else { -lean_object* x_21; -x_21 = l_Lean_Meta_Grind_getNext(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_20; uint8_t x_21; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); +x_20 = lean_st_ref_get(x_5, x_16); lean_dec(x_5); -if (lean_obj_tag(x_21) == 0) +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = l_Lean_Meta_Grind_Goal_getNext(x_22, x_3, x_11, x_12, x_23); +lean_dec(x_12); +lean_dec(x_11); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_23; uint8_t x_24; -x_23 = lean_ctor_get(x_21, 0); -x_24 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_23); -if (x_24 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_24); +if (x_25 == 0) { -lean_object* x_25; -lean_ctor_set(x_14, 1, x_2); -lean_ctor_set(x_14, 0, x_23); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_14); -lean_ctor_set(x_21, 0, x_25); -return x_21; +lean_object* x_26; uint8_t x_27; +x_26 = lean_ctor_get(x_24, 0); +x_27 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_26); +if (x_27 == 0) +{ +lean_object* x_28; +lean_ctor_set(x_20, 1, x_2); +lean_ctor_set(x_20, 0, x_26); +x_28 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_28, 0, x_20); +lean_ctor_set(x_24, 0, x_28); +return x_24; } else { -lean_object* x_26; -lean_ctor_set(x_14, 1, x_2); -lean_ctor_set(x_14, 0, x_23); -x_26 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_26, 0, x_14); -lean_ctor_set(x_21, 0, x_26); -return x_21; +lean_object* x_29; +lean_ctor_set(x_20, 1, x_2); +lean_ctor_set(x_20, 0, x_26); +x_29 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_29, 0, x_20); +lean_ctor_set(x_24, 0, x_29); +return x_24; } } else { -lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_27 = lean_ctor_get(x_21, 0); -x_28 = lean_ctor_get(x_21, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_21); -x_29 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_27); -if (x_29 == 0) +lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_30 = lean_ctor_get(x_24, 0); +x_31 = lean_ctor_get(x_24, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_24); +x_32 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_30); +if (x_32 == 0) { -lean_object* x_30; lean_object* x_31; -lean_ctor_set(x_14, 1, x_2); -lean_ctor_set(x_14, 0, x_27); -x_30 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_30, 0, x_14); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_28); -return x_31; +lean_object* x_33; lean_object* x_34; +lean_ctor_set(x_20, 1, x_2); +lean_ctor_set(x_20, 0, x_30); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_20); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_31); +return x_34; } else { -lean_object* x_32; lean_object* x_33; -lean_ctor_set(x_14, 1, x_2); -lean_ctor_set(x_14, 0, x_27); -x_32 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_32, 0, x_14); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_28); -return x_33; +lean_object* x_35; lean_object* x_36; +lean_ctor_set(x_20, 1, x_2); +lean_ctor_set(x_20, 0, x_30); +x_35 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_35, 0, x_20); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_31); +return x_36; } } } else { -uint8_t x_34; -lean_free_object(x_14); +uint8_t x_37; +lean_free_object(x_20); lean_dec(x_2); -x_34 = !lean_is_exclusive(x_21); -if (x_34 == 0) -{ -return x_21; -} -else +x_37 = !lean_is_exclusive(x_24); +if (x_37 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_21, 0); -x_36 = lean_ctor_get(x_21, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_21); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} -} +return x_24; } else { -lean_object* x_38; lean_object* x_39; uint8_t x_40; -x_38 = lean_ctor_get(x_14, 0); -x_39 = lean_ctor_get(x_14, 1); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_24, 0); +x_39 = lean_ctor_get(x_24, 1); lean_inc(x_39); lean_inc(x_38); -lean_dec(x_14); -x_40 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_38, x_1); -lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; lean_object* x_42; -lean_dec(x_3); -lean_dec(x_2); -x_41 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__6; -x_42 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__3(x_41, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); -return x_42; +lean_dec(x_24); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} } else { -lean_object* x_43; -x_43 = l_Lean_Meta_Grind_getNext(x_3, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_39); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_20, 0); +x_42 = lean_ctor_get(x_20, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_20); +x_43 = l_Lean_Meta_Grind_Goal_getNext(x_41, x_3, x_11, x_12, x_42); lean_dec(x_12); lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); if (lean_obj_tag(x_43) == 0) { lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; @@ -954,7 +955,7 @@ static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(32u); +x_3 = lean_unsigned_to_nat(33u); x_4 = lean_unsigned_to_nat(6u); x_5 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -965,7 +966,7 @@ LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_ _start: { uint8_t x_15; -x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 4); +x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*11 + 4); if (x_15 == 0) { lean_object* x_16; @@ -1076,7 +1077,7 @@ static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(22u); +x_3 = lean_unsigned_to_nat(23u); x_4 = lean_unsigned_to_nat(4u); x_5 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1107,7 +1108,7 @@ static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(29u); +x_3 = lean_unsigned_to_nat(30u); x_4 = lean_unsigned_to_nat(8u); x_5 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__5; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1138,7 +1139,7 @@ static lean_object* _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(27u); +x_3 = lean_unsigned_to_nat(28u); x_4 = lean_unsigned_to_nat(10u); x_5 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__8; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1148,7 +1149,7 @@ return x_6; LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_object* x_13; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; x_29 = lean_ctor_get(x_3, 0); lean_inc(x_29); x_30 = lean_ctor_get(x_3, 1); @@ -1157,24 +1158,30 @@ lean_dec(x_3); x_31 = lean_unsigned_to_nat(1u); x_32 = lean_nat_add(x_30, x_31); lean_dec(x_30); -lean_inc(x_29); -x_33 = l_Lean_Meta_Grind_getRoot(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_33 = lean_st_ref_get(x_4, x_12); x_34 = lean_ctor_get(x_33, 0); lean_inc(x_34); x_35 = lean_ctor_get(x_33, 1); lean_inc(x_35); lean_dec(x_33); -x_36 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_34, x_2); -lean_dec(x_34); -if (x_36 == 0) +lean_inc(x_29); +x_36 = l_Lean_Meta_Grind_Goal_getRoot(x_34, x_29, x_10, x_11, x_35); +if (lean_obj_tag(x_36) == 0) { -lean_object* x_37; lean_object* x_38; +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +x_39 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_37, x_2); +lean_dec(x_37); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; lean_dec(x_32); lean_dec(x_29); -x_37 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__3; +x_40 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__3; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1183,18 +1190,18 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_38 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_37, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_35); -x_13 = x_38; +x_41 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_40, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); +x_13 = x_41; goto block_28; } else { -uint8_t x_39; -x_39 = l_Lean_Expr_isApp(x_29); -if (x_39 == 0) +uint8_t x_42; +x_42 = l_Lean_Expr_isApp(x_29); +if (x_42 == 0) { -lean_object* x_40; lean_object* x_41; -x_40 = lean_box(0); +lean_object* x_43; lean_object* x_44; +x_43 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1204,44 +1211,44 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_41 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_40, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_35); -x_13 = x_41; +x_44 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_43, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_38); +x_13 = x_44; goto block_28; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_42 = lean_st_ref_get(x_4, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -x_45 = lean_ctor_get(x_43, 3); -lean_inc(x_45); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_45 = lean_st_ref_get(x_4, x_38); +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = lean_ctor_get(x_46, 4); +lean_inc(x_48); lean_inc(x_29); -x_46 = l_Lean_PersistentHashMap_findEntry_x3f___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__4(x_43, x_45, x_29); -if (lean_obj_tag(x_46) == 0) +x_49 = l_Lean_PersistentHashMap_findEntry_x3f___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__4(x_46, x_48, x_29); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_47; +lean_object* x_50; lean_inc(x_29); -x_47 = l_Lean_Meta_Grind_isCongrRoot(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_44); -if (lean_obj_tag(x_47) == 0) +x_50 = l_Lean_Meta_Grind_isCongrRoot(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_48; uint8_t x_49; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_unbox(x_48); -lean_dec(x_48); -if (x_49 == 0) +lean_object* x_51; uint8_t x_52; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +x_52 = lean_unbox(x_51); +lean_dec(x_51); +if (x_52 == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_dec(x_32); lean_dec(x_29); -x_50 = lean_ctor_get(x_47, 1); -lean_inc(x_50); -lean_dec(x_47); -x_51 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__6; +x_53 = lean_ctor_get(x_50, 1); +lean_inc(x_53); +lean_dec(x_50); +x_54 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__6; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1250,17 +1257,17 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_52 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_51, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_50); -x_13 = x_52; +x_55 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_54, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_53); +x_13 = x_55; goto block_28; } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_47, 1); -lean_inc(x_53); -lean_dec(x_47); -x_54 = lean_box(0); +lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_56 = lean_ctor_get(x_50, 1); +lean_inc(x_56); +lean_dec(x_50); +x_57 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1270,69 +1277,69 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_55 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_54, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_53); -x_13 = x_55; +x_58 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_57, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_56); +x_13 = x_58; goto block_28; } } else { -uint8_t x_56; +uint8_t x_59; lean_dec(x_32); lean_dec(x_29); -x_56 = !lean_is_exclusive(x_47); -if (x_56 == 0) +x_59 = !lean_is_exclusive(x_50); +if (x_59 == 0) { -x_13 = x_47; +x_13 = x_50; goto block_28; } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_47, 0); -x_58 = lean_ctor_get(x_47, 1); -lean_inc(x_58); -lean_inc(x_57); -lean_dec(x_47); -x_59 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_59, 0, x_57); -lean_ctor_set(x_59, 1, x_58); -x_13 = x_59; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_50, 0); +x_61 = lean_ctor_get(x_50, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_50); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +x_13 = x_62; goto block_28; } } } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_60 = lean_ctor_get(x_46, 0); -lean_inc(x_60); -lean_dec(x_46); -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -lean_dec(x_60); -x_62 = l_Lean_Expr_getAppFn(x_61); -x_63 = l_Lean_Expr_getAppFn(x_29); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_63 = lean_ctor_get(x_49, 0); +lean_inc(x_63); +lean_dec(x_49); +x_64 = lean_ctor_get(x_63, 0); +lean_inc(x_64); +lean_dec(x_63); +x_65 = l_Lean_Expr_getAppFn(x_64); +x_66 = l_Lean_Expr_getAppFn(x_29); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_64 = l_Lean_Meta_Grind_hasSameType(x_62, x_63, x_8, x_9, x_10, x_11, x_44); -if (lean_obj_tag(x_64) == 0) +x_67 = l_Lean_Meta_Grind_hasSameType(x_65, x_66, x_8, x_9, x_10, x_11, x_47); +if (lean_obj_tag(x_67) == 0) { -lean_object* x_65; uint8_t x_66; -x_65 = lean_ctor_get(x_64, 0); -lean_inc(x_65); -x_66 = lean_unbox(x_65); -lean_dec(x_65); -if (x_66 == 0) +lean_object* x_68; uint8_t x_69; +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_unbox(x_68); +lean_dec(x_68); +if (x_69 == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -lean_dec(x_61); -x_67 = lean_ctor_get(x_64, 1); -lean_inc(x_67); +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_dec(x_64); -x_68 = lean_box(0); +x_70 = lean_ctor_get(x_67, 1); +lean_inc(x_70); +lean_dec(x_67); +x_71 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1342,35 +1349,35 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_69 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_68, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_67); -x_13 = x_69; +x_72 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_71, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_13 = x_72; goto block_28; } else { -lean_object* x_70; lean_object* x_71; -x_70 = lean_ctor_get(x_64, 1); -lean_inc(x_70); -lean_dec(x_64); +lean_object* x_73; lean_object* x_74; +x_73 = lean_ctor_get(x_67, 1); +lean_inc(x_73); +lean_dec(x_67); lean_inc(x_29); -x_71 = l_Lean_Meta_Grind_getCongrRoot(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_70); -if (lean_obj_tag(x_71) == 0) +x_74 = l_Lean_Meta_Grind_getCongrRoot(x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_73); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_72; lean_object* x_73; uint8_t x_74; -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -lean_dec(x_71); -x_74 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_61, x_72); -lean_dec(x_72); -lean_dec(x_61); -if (x_74 == 0) +lean_object* x_75; lean_object* x_76; uint8_t x_77; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_64, x_75); +lean_dec(x_75); +lean_dec(x_64); +if (x_77 == 0) { -lean_object* x_75; lean_object* x_76; +lean_object* x_78; lean_object* x_79; lean_dec(x_32); lean_dec(x_29); -x_75 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9; +x_78 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9; lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1379,14 +1386,14 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_76 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_75, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_73); -x_13 = x_76; +x_79 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1(x_78, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_76); +x_13 = x_79; goto block_28; } else { -lean_object* x_77; lean_object* x_78; -x_77 = lean_box(0); +lean_object* x_80; lean_object* x_81; +x_80 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -1396,35 +1403,35 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_78 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_77, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_73); -x_13 = x_78; +x_81 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__2(x_2, x_32, x_1, x_29, x_80, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_76); +x_13 = x_81; goto block_28; } } else { -uint8_t x_79; -lean_dec(x_61); +uint8_t x_82; +lean_dec(x_64); lean_dec(x_32); lean_dec(x_29); -x_79 = !lean_is_exclusive(x_71); -if (x_79 == 0) +x_82 = !lean_is_exclusive(x_74); +if (x_82 == 0) { -x_13 = x_71; +x_13 = x_74; goto block_28; } else { -lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_80 = lean_ctor_get(x_71, 0); -x_81 = lean_ctor_get(x_71, 1); -lean_inc(x_81); -lean_inc(x_80); -lean_dec(x_71); -x_82 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_82, 0, x_80); -lean_ctor_set(x_82, 1, x_81); -x_13 = x_82; +lean_object* x_83; lean_object* x_84; lean_object* x_85; +x_83 = lean_ctor_get(x_74, 0); +x_84 = lean_ctor_get(x_74, 1); +lean_inc(x_84); +lean_inc(x_83); +lean_dec(x_74); +x_85 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_85, 0, x_83); +lean_ctor_set(x_85, 1, x_84); +x_13 = x_85; goto block_28; } } @@ -1432,28 +1439,28 @@ goto block_28; } else { -uint8_t x_83; -lean_dec(x_61); +uint8_t x_86; +lean_dec(x_64); lean_dec(x_32); lean_dec(x_29); -x_83 = !lean_is_exclusive(x_64); -if (x_83 == 0) +x_86 = !lean_is_exclusive(x_67); +if (x_86 == 0) { -x_13 = x_64; +x_13 = x_67; goto block_28; } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_64, 0); -x_85 = lean_ctor_get(x_64, 1); -lean_inc(x_85); -lean_inc(x_84); -lean_dec(x_64); -x_86 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_86, 0, x_84); -lean_ctor_set(x_86, 1, x_85); -x_13 = x_86; +lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_67, 0); +x_88 = lean_ctor_get(x_67, 1); +lean_inc(x_88); +lean_inc(x_87); +lean_dec(x_67); +x_89 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_89, 0, x_87); +lean_ctor_set(x_89, 1, x_88); +x_13 = x_89; goto block_28; } } @@ -1463,27 +1470,27 @@ goto block_28; } else { -uint8_t x_87; +uint8_t x_90; lean_dec(x_32); lean_dec(x_29); -x_87 = !lean_is_exclusive(x_33); -if (x_87 == 0) +x_90 = !lean_is_exclusive(x_36); +if (x_90 == 0) { -x_13 = x_33; +x_13 = x_36; goto block_28; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; -x_88 = lean_ctor_get(x_33, 0); -x_89 = lean_ctor_get(x_33, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_33); -x_90 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_90, 0, x_88); -lean_ctor_set(x_90, 1, x_89); -x_13 = x_90; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_36, 0); +x_92 = lean_ctor_get(x_36, 1); +lean_inc(x_92); +lean_inc(x_91); +lean_dec(x_36); +x_93 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_93, 0, x_91); +lean_ctor_set(x_93, 1, x_92); +x_13 = x_93; goto block_28; } } @@ -1581,26 +1588,6 @@ return x_27; } } } -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__4; -x_2 = l_instInhabitedPUnit; -x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1; -x_12 = lean_panic_fn(x_11, x_1); -x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; -} -} static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__1() { _start: { @@ -1625,7 +1612,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Gr lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__5; -x_3 = lean_unsigned_to_nat(46u); +x_3 = lean_unsigned_to_nat(47u); x_4 = lean_unsigned_to_nat(2u); x_5 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -1675,7 +1662,7 @@ if (x_20 == 0) lean_object* x_21; lean_object* x_22; lean_free_object(x_15); x_21 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__3; -x_22 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +x_22 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); return x_22; } else @@ -1712,7 +1699,7 @@ if (x_27 == 0) { lean_object* x_28; lean_object* x_29; x_28 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__3; -x_29 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8(x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +x_29 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_28, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); return x_29; } else @@ -1848,87 +1835,100 @@ return x_19; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; +lean_object* x_20; lean_object* x_21; uint8_t x_22; x_20 = lean_array_uget(x_4, x_6); -x_21 = l_Lean_Meta_Grind_getRoot_x3f(x_20, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_21 = lean_st_ref_get(x_8, x_16); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_21, 0); +x_24 = lean_ctor_get(x_21, 1); +x_25 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_23, x_20); lean_dec(x_20); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) +if (lean_obj_tag(x_25) == 0) { -lean_object* x_23; size_t x_24; size_t x_25; -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = 1; -x_25 = lean_usize_add(x_6, x_24); -x_6 = x_25; -x_16 = x_23; +size_t x_26; size_t x_27; +lean_free_object(x_21); +x_26 = 1; +x_27 = lean_usize_add(x_6, x_26); +x_6 = x_27; +x_16 = x_24; goto _start; } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_28 = lean_ctor_get(x_21, 1); -x_29 = lean_ctor_get(x_21, 0); +lean_object* x_29; uint8_t x_30; +x_29 = lean_ctor_get(x_25, 0); +lean_inc(x_29); +lean_dec(x_25); +x_30 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_29, x_1); lean_dec(x_29); -x_30 = lean_ctor_get(x_22, 0); -lean_inc(x_30); -lean_dec(x_22); -x_31 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_30, x_1); -lean_dec(x_30); -if (x_31 == 0) +if (x_30 == 0) { -size_t x_32; size_t x_33; +size_t x_31; size_t x_32; lean_free_object(x_21); -x_32 = 1; -x_33 = lean_usize_add(x_6, x_32); -x_6 = x_33; -x_16 = x_28; +x_31 = 1; +x_32 = lean_usize_add(x_6, x_31); +x_6 = x_32; +x_16 = x_24; goto _start; } else { -uint8_t x_35; lean_object* x_36; -x_35 = 1; -x_36 = lean_box(x_35); -lean_ctor_set(x_21, 0, x_36); +uint8_t x_34; lean_object* x_35; +x_34 = 1; +x_35 = lean_box(x_34); +lean_ctor_set(x_21, 0, x_35); return x_21; } } +} else { -lean_object* x_37; lean_object* x_38; uint8_t x_39; +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_21, 0); x_37 = lean_ctor_get(x_21, 1); lean_inc(x_37); +lean_inc(x_36); lean_dec(x_21); -x_38 = lean_ctor_get(x_22, 0); -lean_inc(x_38); -lean_dec(x_22); -x_39 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_38, x_1); +x_38 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_36, x_20); +lean_dec(x_20); +if (lean_obj_tag(x_38) == 0) +{ +size_t x_39; size_t x_40; +x_39 = 1; +x_40 = lean_usize_add(x_6, x_39); +x_6 = x_40; +x_16 = x_37; +goto _start; +} +else +{ +lean_object* x_42; uint8_t x_43; +x_42 = lean_ctor_get(x_38, 0); +lean_inc(x_42); lean_dec(x_38); -if (x_39 == 0) +x_43 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_42, x_1); +lean_dec(x_42); +if (x_43 == 0) { -size_t x_40; size_t x_41; -x_40 = 1; -x_41 = lean_usize_add(x_6, x_40); -x_6 = x_41; +size_t x_44; size_t x_45; +x_44 = 1; +x_45 = lean_usize_add(x_6, x_44); +x_6 = x_45; x_16 = x_37; goto _start; } else { -uint8_t x_43; lean_object* x_44; lean_object* x_45; -x_43 = 1; -x_44 = lean_box(x_43); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_37); -return x_45; +uint8_t x_47; lean_object* x_48; lean_object* x_49; +x_47 = 1; +x_48 = lean_box(x_47); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_37); +return x_49; } } } @@ -1969,7 +1969,7 @@ static lean_object* _init_l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tac _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("( __do_lift._@.Lean.Meta.Tactic.Grind.Inv._hyg.782.0 )\n ", 57, 57); +x_1 = lean_mk_string_unchecked("( __do_lift._@.Lean.Meta.Tactic.Grind.Inv._hyg.787.0 )\n ", 57, 57); return x_1; } } @@ -1997,7 +1997,7 @@ static lean_object* _init_l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tac lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__3; -x_3 = lean_unsigned_to_nat(65u); +x_3 = lean_unsigned_to_nat(69u); x_4 = lean_unsigned_to_nat(8u); x_5 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2019,48 +2019,44 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tact { if (x_3 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_14; lean_object* x_15; uint8_t x_16; x_14 = l_Lean_Expr_getAppFn(x_1); -x_15 = l_Lean_Meta_Grind_getRoot_x3f(x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -lean_dec(x_14); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -if (lean_obj_tag(x_16) == 0) +x_15 = lean_st_ref_get(x_5, x_13); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; -x_19 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_17); -return x_19; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_17, x_14); +lean_dec(x_14); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_free_object(x_15); +x_20 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; +x_21 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +return x_21; } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_21 = lean_ctor_get(x_15, 1); -x_22 = lean_ctor_get(x_15, 0); +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_19, 0); +lean_inc(x_22); +lean_dec(x_19); +x_23 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_22, x_2); lean_dec(x_22); -x_23 = lean_ctor_get(x_16, 0); -lean_inc(x_23); -lean_dec(x_16); -x_24 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_23, x_2); -lean_dec(x_23); -if (x_24 == 0) +if (x_23 == 0) { -lean_object* x_25; lean_object* x_26; +lean_object* x_24; lean_object* x_25; lean_free_object(x_15); -x_25 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; -x_26 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_25, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_21); -return x_26; +x_24 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; +x_25 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_24, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +return x_25; } else { -lean_object* x_27; +lean_object* x_26; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -2069,32 +2065,47 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_27 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; -lean_ctor_set(x_15, 0, x_27); +x_26 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; +lean_ctor_set(x_15, 0, x_26); return x_15; } } +} else { -lean_object* x_28; lean_object* x_29; uint8_t x_30; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_15, 0); x_28 = lean_ctor_get(x_15, 1); lean_inc(x_28); +lean_inc(x_27); lean_dec(x_15); -x_29 = lean_ctor_get(x_16, 0); -lean_inc(x_29); -lean_dec(x_16); -x_30 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_29, x_2); +x_29 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_27, x_14); +lean_dec(x_14); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; +x_31 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_30, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); +return x_31; +} +else +{ +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_29, 0); +lean_inc(x_32); lean_dec(x_29); -if (x_30 == 0) +x_33 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_32, x_2); +lean_dec(x_32); +if (x_33 == 0) { -lean_object* x_31; lean_object* x_32; -x_31 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; -x_32 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_31, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); -return x_32; +lean_object* x_34; lean_object* x_35; +x_34 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__4; +x_35 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__2(x_34, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_28); +return x_35; } else { -lean_object* x_33; lean_object* x_34; +lean_object* x_36; lean_object* x_37; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -2103,18 +2114,18 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_33 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_28); -return x_34; +x_36 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_36); +lean_ctor_set(x_37, 1, x_28); +return x_37; } } } } else { -lean_object* x_35; lean_object* x_36; +lean_object* x_38; lean_object* x_39; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -2123,11 +2134,71 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_35 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_13); -return x_36; +x_38 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__5; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_13); +return x_39; +} +} +} +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +uint8_t x_15; +x_15 = l_Lean_Expr_hasLooseBVars(x_1); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_st_ref_get(x_6, x_14); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_17, x_1); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_box(0); +x_21 = lean_box(x_4); +x_22 = lean_apply_11(x_2, x_21, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +return x_22; +} +else +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_19, 0); +lean_inc(x_23); +lean_dec(x_19); +x_24 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_23, x_3); +lean_dec(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_box(0); +x_26 = lean_box(x_4); +x_27 = lean_apply_11(x_2, x_26, x_25, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +return x_27; +} +else +{ +uint8_t x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_28 = 1; +x_29 = lean_box(0); +x_30 = lean_box(x_28); +x_31 = lean_apply_11(x_2, x_30, x_29, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); +return x_31; +} +} +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_box(0); +x_33 = lean_box(x_4); +x_34 = lean_apply_11(x_2, x_33, x_32, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +return x_34; } } } @@ -2154,6 +2225,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_1); x_13 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_13, 0, x_3); x_14 = lean_alloc_ctor(0, 2, 0); @@ -2179,6 +2251,7 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); +lean_inc(x_1); x_18 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3(x_1, x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_18) == 0) { @@ -2198,6 +2271,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_1); x_20 = !lean_is_exclusive(x_18); if (x_20 == 0) { @@ -2243,7 +2317,7 @@ x_50 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0_ lean_dec(x_45); if (lean_obj_tag(x_16) == 7) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; lean_object* x_57; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); x_52 = lean_ctor_get(x_50, 1); @@ -2251,48 +2325,45 @@ lean_inc(x_52); lean_dec(x_50); x_53 = lean_ctor_get(x_16, 1); lean_inc(x_53); -x_54 = l_Lean_Meta_Grind_getRoot_x3f(x_53, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_52); +x_54 = lean_ctor_get(x_16, 2); +lean_inc(x_54); +lean_inc(x_1); +x_55 = lean_alloc_closure((void*)(l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___boxed), 13, 2); +lean_closure_set(x_55, 0, x_16); +lean_closure_set(x_55, 1, x_1); +x_65 = lean_st_ref_get(x_4, x_52); +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_66, x_53); lean_dec(x_53); -x_55 = lean_ctor_get(x_54, 0); -lean_inc(x_55); -if (lean_obj_tag(x_55) == 0) +if (lean_obj_tag(x_68) == 0) { -lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; -x_56 = lean_ctor_get(x_54, 1); -lean_inc(x_56); -lean_dec(x_54); -x_57 = lean_box(0); -x_58 = lean_unbox(x_51); -lean_dec(x_51); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -x_59 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1(x_16, x_1, x_58, x_57, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_56); -lean_dec(x_16); -x_25 = x_59; -goto block_38; +x_56 = x_49; +x_57 = x_67; +goto block_64; } else { -lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_60 = lean_ctor_get(x_54, 1); -lean_inc(x_60); -lean_dec(x_54); -x_61 = lean_ctor_get(x_55, 0); -lean_inc(x_61); -lean_dec(x_55); -x_62 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_61, x_1); -lean_dec(x_61); -if (x_62 == 0) +lean_object* x_69; uint8_t x_70; +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +lean_dec(x_68); +x_70 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_69, x_1); +lean_dec(x_69); +x_56 = x_70; +x_57 = x_67; +goto block_64; +} +block_64: { -lean_object* x_63; uint8_t x_64; lean_object* x_65; -x_63 = lean_box(0); -x_64 = lean_unbox(x_51); +if (x_56 == 0) +{ +lean_object* x_58; uint8_t x_59; lean_object* x_60; +x_58 = lean_box(0); +x_59 = lean_unbox(x_51); lean_dec(x_51); lean_inc(x_11); lean_inc(x_10); @@ -2302,17 +2373,17 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_65 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1(x_16, x_1, x_64, x_63, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_60); -lean_dec(x_16); -x_25 = x_65; +x_60 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2(x_54, x_55, x_1, x_59, x_58, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_57); +lean_dec(x_54); +x_25 = x_60; goto block_38; } else { -uint8_t x_66; lean_object* x_67; lean_object* x_68; +uint8_t x_61; lean_object* x_62; lean_object* x_63; lean_dec(x_51); -x_66 = 1; -x_67 = lean_box(0); +x_61 = 1; +x_62 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -2321,24 +2392,24 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_68 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1(x_16, x_1, x_66, x_67, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_60); -lean_dec(x_16); -x_25 = x_68; +x_63 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2(x_54, x_55, x_1, x_61, x_62, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_57); +lean_dec(x_54); +x_25 = x_63; goto block_38; } } } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; lean_object* x_73; -x_69 = lean_ctor_get(x_50, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_50, 1); -lean_inc(x_70); +lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; lean_object* x_75; +x_71 = lean_ctor_get(x_50, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_50, 1); +lean_inc(x_72); lean_dec(x_50); -x_71 = lean_box(0); -x_72 = lean_unbox(x_69); -lean_dec(x_69); +x_73 = lean_box(0); +x_74 = lean_unbox(x_71); +lean_dec(x_71); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -2347,9 +2418,9 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -x_73 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1(x_16, x_1, x_72, x_71, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_70); +x_75 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1(x_16, x_1, x_74, x_73, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_72); lean_dec(x_16); -x_25 = x_73; +x_25 = x_75; goto block_38; } block_38: @@ -2371,6 +2442,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_1); x_27 = !lean_is_exclusive(x_25); if (x_27 == 0) { @@ -2418,6 +2490,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_1); x_34 = !lean_is_exclusive(x_25); if (x_34 == 0) { @@ -2442,7 +2515,7 @@ return x_37; } else { -uint8_t x_74; +uint8_t x_76; lean_dec(x_17); lean_dec(x_16); lean_dec(x_11); @@ -2453,23 +2526,24 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -x_74 = !lean_is_exclusive(x_18); -if (x_74 == 0) +lean_dec(x_1); +x_76 = !lean_is_exclusive(x_18); +if (x_76 == 0) { return x_18; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_18, 0); -x_76 = lean_ctor_get(x_18, 1); -lean_inc(x_76); -lean_inc(x_75); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_18, 0); +x_78 = lean_ctor_get(x_18, 1); +lean_inc(x_78); +lean_inc(x_77); lean_dec(x_18); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } @@ -2479,7 +2553,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Gr _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("( __do_lift._@.Lean.Meta.Tactic.Grind.Inv._hyg.805.0 ).isEmpty\n\n", 64, 64); +x_1 = lean_mk_string_unchecked("( __do_lift._@.Lean.Meta.Tactic.Grind.Inv._hyg.817.0 ).isEmpty\n\n", 64, 64); return x_1; } } @@ -2499,7 +2573,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Gr lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__1___closed__3; -x_3 = lean_unsigned_to_nat(68u); +x_3 = lean_unsigned_to_nat(72u); x_4 = lean_unsigned_to_nat(4u); x_5 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2522,6 +2596,7 @@ x_14 = lean_ctor_get(x_11, 1); lean_inc(x_14); lean_dec(x_11); x_15 = l_Lean_Meta_Grind_getParents(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +lean_dec(x_1); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); if (lean_obj_tag(x_16) == 0) @@ -2566,7 +2641,7 @@ x_23 = lean_ctor_get(x_15, 1); lean_inc(x_23); lean_dec(x_15); x_24 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___closed__3; -x_25 = l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8(x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +x_25 = l_panic___at___private_Lean_Meta_Tactic_Grind_Arith_Offset_0__Lean_Meta_Grind_Arith_Offset_setUnsat___spec__1(x_24, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); return x_25; } } @@ -2672,22 +2747,17 @@ lean_dec(x_1); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_13; -x_13 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -return x_13; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_15; lean_object* x_16; +x_15 = lean_unbox(x_4); +lean_dec(x_4); +x_16 = l_Lean_RBNode_forIn_visit___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents___spec__3___lambda__2(x_1, x_2, x_3, x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_1); -return x_11; +return x_16; } } LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -2732,7 +2802,7 @@ static lean_object* _init_l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Ta lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__3; -x_3 = lean_unsigned_to_nat(79u); +x_3 = lean_unsigned_to_nat(83u); x_4 = lean_unsigned_to_nat(6u); x_5 = l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__2; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -2763,7 +2833,7 @@ static lean_object* _init_l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Ta lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___lambda__1___closed__4; x_2 = l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__3; -x_3 = lean_unsigned_to_nat(77u); +x_3 = lean_unsigned_to_nat(81u); x_4 = lean_unsigned_to_nat(6u); x_5 = l_Std_Range_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq___spec__2___closed__6; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); @@ -4678,96 +4748,63 @@ return x_27; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_getEqcs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_10 = lean_st_ref_get(x_1, x_9); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = lean_box(0); +x_13 = l_Lean_Meta_Grind_Goal_getEqcs(x_11); x_14 = lean_box(0); -lean_inc(x_11); -x_15 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__3(x_11, x_13, x_11, x_11, x_14, lean_box(0), x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -lean_dec(x_11); -if (lean_obj_tag(x_15) == 0) +x_15 = lean_box(0); +lean_inc(x_13); +x_16 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkProofs___spec__3(x_13, x_14, x_13, x_13, x_15, lean_box(0), x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); +lean_dec(x_13); +if (lean_obj_tag(x_16) == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -lean_object* x_17; -x_17 = lean_ctor_get(x_15, 0); -lean_dec(x_17); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_18; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +lean_ctor_set(x_16, 0, x_15); +return x_16; } else { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_14); -lean_ctor_set(x_19, 1, x_18); -return x_19; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_dec(x_16); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_15); +lean_ctor_set(x_20, 1, x_19); +return x_20; } } else { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_15); -if (x_20 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) { -return x_15; +return x_16; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_15, 0); -x_22 = lean_ctor_get(x_15, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); lean_inc(x_22); -lean_inc(x_21); -lean_dec(x_15); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; -} -} -} -else -{ -uint8_t x_24; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_24 = !lean_is_exclusive(x_10); -if (x_24 == 0) -{ -return x_10; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_10, 0); -x_26 = lean_ctor_get(x_10, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_10); -x_27 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_dec(x_16); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } @@ -5762,6 +5799,7 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); +lean_inc(x_13); x_14 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkParents(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); if (lean_obj_tag(x_14) == 0) { @@ -5966,6 +6004,63 @@ return x_49; } } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_12 = l_Lean_Meta_Grind_Arith_Offset_checkInvariants(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_apply_10(x_1, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +return x_15; +} +else +{ +uint8_t x_16; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_16 = !lean_is_exclusive(x_12); +if (x_16 == 0) +{ +return x_12; +} +else +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_17 = lean_ctor_get(x_12, 0); +x_18 = lean_ctor_get(x_12, 1); +lean_inc(x_18); +lean_inc(x_17); +lean_dec(x_12); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +return x_19; +} +} +} +} static lean_object* _init_l_Lean_Meta_Grind_checkInvariants___closed__1() { _start: { @@ -5985,33 +6080,37 @@ return x_1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; uint8_t x_13; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; x_11 = lean_ctor_get(x_8, 2); lean_inc(x_11); -x_12 = l_Lean_Meta_Grind_checkInvariants___closed__1; -x_13 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_12); +x_12 = lean_box(x_1); +x_13 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_checkInvariants___lambda__1___boxed), 11, 1); +lean_closure_set(x_13, 0, x_12); +x_14 = l_Lean_Meta_Grind_checkInvariants___closed__1; +x_15 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_14); lean_dec(x_11); -if (x_13 == 0) +if (x_15 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_box(0); -x_15 = l_Lean_Meta_Grind_checkInvariants___lambda__1(x_1, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_15; +lean_object* x_16; lean_object* x_17; +lean_dec(x_13); +x_16 = lean_box(0); +x_17 = l_Lean_Meta_Grind_checkInvariants___lambda__1(x_1, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_17; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_16 = lean_st_ref_get(x_2, x_10); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_ctor_get(x_17, 1); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_18 = lean_st_ref_get(x_2, x_10); +x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -lean_dec(x_17); -x_20 = lean_box(0); -x_21 = l_Lean_Meta_Grind_checkInvariants___closed__2; +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_19, 2); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_box(0); +x_23 = l_Lean_Meta_Grind_checkInvariants___closed__2; lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -6020,24 +6119,24 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_22 = l_Lean_PersistentHashMap_forIn___at_Lean_Meta_Grind_checkInvariants___spec__1(x_19, x_20, x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); -if (lean_obj_tag(x_22) == 0) +x_24 = l_Lean_PersistentHashMap_forIn___at_Lean_Meta_Grind_checkInvariants___spec__1(x_21, x_22, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); +if (lean_obj_tag(x_24) == 0) { if (x_1 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_22, 1); -lean_inc(x_23); -lean_dec(x_22); -x_24 = l_Lean_Meta_Grind_checkInvariants___lambda__1(x_1, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); -return x_24; +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_24, 1); +lean_inc(x_25); +lean_dec(x_24); +x_26 = l_Lean_Meta_Grind_checkInvariants___lambda__3(x_13, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); +return x_26; } else { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_24, 1); +lean_inc(x_27); +lean_dec(x_24); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); @@ -6046,22 +6145,23 @@ lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); -x_26 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -if (lean_obj_tag(x_26) == 0) +x_28 = l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkPtrEqImpliesStructEq(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_26, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l_Lean_Meta_Grind_checkInvariants___lambda__1(x_1, x_27, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_28); -lean_dec(x_27); -return x_29; +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l_Lean_Meta_Grind_checkInvariants___lambda__3(x_13, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); +lean_dec(x_29); +return x_31; } else { -uint8_t x_30; +uint8_t x_32; +lean_dec(x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6070,30 +6170,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_30 = !lean_is_exclusive(x_26); -if (x_30 == 0) +x_32 = !lean_is_exclusive(x_28); +if (x_32 == 0) { -return x_26; +return x_28; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_26, 0); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_26); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_28, 0); +x_34 = lean_ctor_get(x_28, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_28); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } } else { -uint8_t x_34; +uint8_t x_36; +lean_dec(x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -6102,23 +6203,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_34 = !lean_is_exclusive(x_22); -if (x_34 == 0) +x_36 = !lean_is_exclusive(x_24); +if (x_36 == 0) { -return x_22; +return x_24; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_22, 0); -x_36 = lean_ctor_get(x_22, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_22); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_24, 0); +x_38 = lean_ctor_get(x_24, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_24); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } @@ -6167,6 +6268,15 @@ lean_dec(x_2); return x_12; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Meta_Grind_checkInvariants___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkInvariants___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -6461,6 +6571,7 @@ return x_12; } lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Proof(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Inv(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Inv(uint8_t builtin, lean_object* w) { lean_object * res; @@ -6472,6 +6583,9 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Proof(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Inv(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__1 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__1(); lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__1); l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__2 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__1___closed__2(); @@ -6524,8 +6638,6 @@ l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Gr lean_mark_persistent(l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__8); l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9 = _init_l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9(); lean_mark_persistent(l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__7___closed__9); -l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1(); -lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___spec__8___closed__1); l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__1); l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Inv_0__Lean_Meta_Grind_checkEqc___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Main.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Main.c index 8077766a5a90..1895a06bed36 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Main.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Main.c @@ -19,12 +19,12 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkMethods___lambda__2(lean_object*, l LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkMethods(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__14; -lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkNatLit(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); lean_object* l_Lean_Meta_Grind_ematchStar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static double l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1; lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_main___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__1; static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; @@ -38,11 +38,13 @@ size_t lean_uint64_to_usize(uint64_t); lean_object* l_Lean_Meta_Grind_getSimprocs___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Meta_Grind_mkMethods___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_main___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkMethods___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3; lean_object* l_Lean_stringToMessageData(lean_object*); @@ -57,8 +59,10 @@ lean_object* l_Lean_Meta_Grind_getFalseExpr___rarg(lean_object*, lean_object*, l size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GrindM_run(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; lean_object* l_Lean_Meta_Grind_Goal_checkInvariants(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_take(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__2___closed__2; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -68,39 +72,39 @@ static lean_object* l_Lean_Meta_Grind_main___lambda__2___closed__3; static lean_object* l_Lean_Meta_Grind_main___lambda__2___closed__1; LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_propagateProjEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_MessageData_ofFormat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getTrueExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; lean_object* lean_st_ref_get(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__13; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Lean_Meta_appendTagSuffix(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_forM___at___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_mkMethods___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__3___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__1___closed__2; static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__15; lean_object* l_ShareCommon_mkStateImpl(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5; uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GrindM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Grind_builtinPropagatorsRef; lean_object* l_Lean_Meta_Grind_GrindTactic_iterate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_main___lambda__2___closed__5; lean_object* l_Lean_MVarId_clearAuxDecls(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__7; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__12; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_GrindTactic_andThen(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_main___lambda__2___closed__4; @@ -108,21 +112,25 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main(lean_object*, lean_object*, lean static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__6; LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_ensureNoMVar(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkMethods___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_empty___at___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___spec__1; extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__3; LEAN_EXPORT lean_object* l_List_filterMapM_loop___at_Lean_Meta_Grind_main___spec__2___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l_Lean_Name_hash___override(lean_object*); +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Meta_Grind_mkMethods___spec__1(lean_object*, lean_object*); lean_object* l_Lean_MVarId_transformTarget(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__2___closed__1; -lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__17; lean_object* l_Lean_Meta_Grind_mkENodeCore(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); @@ -136,12 +144,15 @@ lean_object* lean_array_mk(lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__4; LEAN_EXPORT lean_object* l_List_foldlM___at_Lean_Meta_Grind_all___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_ensureProp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_isTracingEnabledForCore(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__8; static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__1___closed__1; lean_object* lean_array_uget(lean_object*, size_t); +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_unfoldReducible(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__9; lean_object* l_Lean_Meta_Grind_propagateForallPropUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4; lean_object* lean_array_get_size(lean_object*); extern lean_object* l_Lean_ShareCommon_objectFactory; lean_object* lean_state_sharecommon(lean_object*, lean_object*, lean_object*); @@ -150,7 +161,7 @@ static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__16; static lean_object* l_Lean_Meta_Grind_GrindM_run___rarg___closed__2; lean_object* l_Lean_Meta_Grind_applyToAll(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_main___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_ppGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_ppGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_betaReduce___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; size_t lean_usize_land(size_t, size_t); @@ -953,19 +964,18 @@ return x_3; static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__9() { _start: { -lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = l_Lean_mkNatLit(x_1); +return x_2; } } static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__10() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__9; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; } } static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__11() { @@ -973,10 +983,8 @@ static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__11() { { lean_object* x_1; lean_object* x_2; x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; -x_2 = lean_alloc_ctor(0, 3, 0); +x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); return x_2; } } @@ -984,7 +992,7 @@ static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; +x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -1032,7 +1040,7 @@ static lean_object* _init_l_Lean_Meta_Grind_GrindM_run___rarg___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; +x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; x_2 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__15; x_3 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_3, 0, x_1); @@ -1057,7 +1065,7 @@ return x_3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GrindM_run___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; x_10 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__5; x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); @@ -1071,113 +1079,120 @@ lean_inc(x_16); x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); lean_dec(x_15); -x_18 = l_Lean_Meta_Grind_getSimprocs___rarg(x_7, x_8, x_9); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); +x_18 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__9; +x_19 = lean_state_sharecommon(x_13, x_17, x_18); +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Meta_Grind_getSimpContext(x_5, x_6, x_7, x_8, x_20); -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = l_Lean_Meta_Grind_getSimprocs___rarg(x_7, x_8, x_9); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_23 = lean_ctor_get(x_22, 0); lean_inc(x_23); -lean_dec(x_21); -x_24 = l_Lean_Meta_Grind_mkMethods(x_4, x_7, x_8, x_23); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); +x_24 = lean_ctor_get(x_22, 1); +lean_inc(x_24); +lean_dec(x_22); +x_25 = l_Lean_Meta_Grind_getSimpContext(x_5, x_6, x_7, x_8, x_24); +x_26 = lean_ctor_get(x_25, 0); lean_inc(x_26); -lean_dec(x_24); -x_27 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_27, 0, x_22); -lean_ctor_set(x_27, 1, x_19); -lean_ctor_set(x_27, 2, x_2); -lean_ctor_set(x_27, 3, x_3); -x_28 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; -x_29 = lean_unsigned_to_nat(1u); -x_30 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; -x_31 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__17; -x_32 = lean_box(0); -x_33 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_33, 0, x_28); -lean_ctor_set(x_33, 1, x_17); -lean_ctor_set(x_33, 2, x_29); -lean_ctor_set(x_33, 3, x_30); -lean_ctor_set(x_33, 4, x_31); -lean_ctor_set(x_33, 5, x_16); -lean_ctor_set(x_33, 6, x_11); -lean_ctor_set(x_33, 7, x_32); -x_34 = lean_st_mk_ref(x_33, x_26); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -lean_inc(x_35); -x_37 = lean_apply_8(x_1, x_25, x_27, x_35, x_5, x_6, x_7, x_8, x_36); -if (lean_obj_tag(x_37) == 0) -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_Meta_Grind_mkMethods(x_4, x_7, x_8, x_27); +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_31, 0, x_26); +lean_ctor_set(x_31, 1, x_23); +lean_ctor_set(x_31, 2, x_2); +lean_ctor_set(x_31, 3, x_3); +x_32 = lean_unsigned_to_nat(1u); +x_33 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; +x_34 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__17; +x_35 = lean_box(0); +x_36 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_36, 0, x_21); +lean_ctor_set(x_36, 1, x_32); +lean_ctor_set(x_36, 2, x_33); +lean_ctor_set(x_36, 3, x_34); +lean_ctor_set(x_36, 4, x_16); +lean_ctor_set(x_36, 5, x_11); +lean_ctor_set(x_36, 6, x_20); +lean_ctor_set(x_36, 7, x_35); +x_37 = lean_st_mk_ref(x_36, x_30); x_38 = lean_ctor_get(x_37, 0); lean_inc(x_38); x_39 = lean_ctor_get(x_37, 1); lean_inc(x_39); lean_dec(x_37); -x_40 = lean_st_ref_get(x_35, x_39); -lean_dec(x_35); -x_41 = !lean_is_exclusive(x_40); -if (x_41 == 0) +lean_inc(x_38); +x_40 = lean_apply_8(x_1, x_29, x_31, x_38, x_5, x_6, x_7, x_8, x_39); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_42; -x_42 = lean_ctor_get(x_40, 0); -lean_dec(x_42); -lean_ctor_set(x_40, 0, x_38); -return x_40; +lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_st_ref_get(x_38, x_42); +lean_dec(x_38); +x_44 = !lean_is_exclusive(x_43); +if (x_44 == 0) +{ +lean_object* x_45; +x_45 = lean_ctor_get(x_43, 0); +lean_dec(x_45); +lean_ctor_set(x_43, 0, x_41); +return x_43; } else { -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_40, 1); -lean_inc(x_43); -lean_dec(x_40); -x_44 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_44, 0, x_38); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_46; lean_object* x_47; +x_46 = lean_ctor_get(x_43, 1); +lean_inc(x_46); +lean_dec(x_43); +x_47 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_47, 0, x_41); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } else { -uint8_t x_45; -lean_dec(x_35); -x_45 = !lean_is_exclusive(x_37); -if (x_45 == 0) +uint8_t x_48; +lean_dec(x_38); +x_48 = !lean_is_exclusive(x_40); +if (x_48 == 0) { -return x_37; +return x_40; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_37, 0); -x_47 = lean_ctor_get(x_37, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_37); -x_48 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -return x_48; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_40, 0); +x_50 = lean_ctor_get(x_40, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_40); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } } } else { -uint8_t x_49; -lean_dec(x_17); +uint8_t x_52; +lean_dec(x_21); +lean_dec(x_20); lean_dec(x_16); lean_dec(x_11); lean_dec(x_8); @@ -1188,23 +1203,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_49 = !lean_is_exclusive(x_18); -if (x_49 == 0) +x_52 = !lean_is_exclusive(x_22); +if (x_52 == 0) { -return x_18; +return x_22; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_18, 0); -x_51 = lean_ctor_get(x_18, 1); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_18); -x_52 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_52, 0, x_50); -lean_ctor_set(x_52, 1, x_51); -return x_52; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_22, 0); +x_54 = lean_ctor_get(x_22, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_22); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } @@ -1221,7 +1236,7 @@ static lean_object* _init_l_Lean_PersistentHashMap_empty___at___private_Lean_Met _start: { lean_object* x_1; -x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; +x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; return x_1; } } @@ -1250,84 +1265,88 @@ return x_14; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_12 = 1; -x_13 = 0; -x_14 = lean_unsigned_to_nat(0u); -x_15 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_12, x_13, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_16 = lean_ctor_get(x_15, 1); -lean_inc(x_16); -lean_dec(x_15); -x_17 = l_Lean_Meta_Grind_mkENodeCore(x_2, x_12, x_13, x_14, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); -x_18 = lean_ctor_get(x_17, 1); -lean_inc(x_18); -lean_dec(x_17); -x_19 = lean_st_ref_get(x_3, x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) -{ -lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_21 = lean_ctor_get(x_19, 1); -x_22 = lean_st_ref_get(x_3, x_21); +uint8_t x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_13 = 1; +x_14 = 0; +x_15 = lean_unsigned_to_nat(0u); +x_16 = l_Lean_Meta_Grind_mkENodeCore(x_1, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_17 = lean_ctor_get(x_16, 1); +lean_inc(x_17); +lean_dec(x_16); +x_18 = l_Lean_Meta_Grind_mkENodeCore(x_2, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +x_19 = lean_ctor_get(x_18, 1); +lean_inc(x_19); +lean_dec(x_18); +x_20 = l_Lean_Meta_Grind_mkENodeCore(x_3, x_13, x_14, x_15, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); +x_21 = lean_ctor_get(x_20, 1); +lean_inc(x_21); +lean_dec(x_20); +x_22 = lean_st_ref_get(x_4, x_21); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_22, 0); -lean_ctor_set(x_19, 1, x_24); -lean_ctor_set(x_22, 0, x_19); -return x_22; +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_22, 1); +x_25 = lean_st_ref_get(x_4, x_24); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) +{ +lean_object* x_27; +x_27 = lean_ctor_get(x_25, 0); +lean_ctor_set(x_22, 1, x_27); +lean_ctor_set(x_25, 0, x_22); +return x_25; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_22, 0); -x_26 = lean_ctor_get(x_22, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_22); -lean_ctor_set(x_19, 1, x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_19); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_25, 0); +x_29 = lean_ctor_get(x_25, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_25); +lean_ctor_set(x_22, 1, x_28); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_22); +lean_ctor_set(x_30, 1, x_29); +return x_30; } } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_28 = lean_ctor_get(x_19, 0); -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_19); -x_30 = lean_st_ref_get(x_3, x_29); -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_31 = lean_ctor_get(x_22, 0); +x_32 = lean_ctor_get(x_22, 1); lean_inc(x_32); -if (lean_is_exclusive(x_30)) { - lean_ctor_release(x_30, 0); - lean_ctor_release(x_30, 1); - x_33 = x_30; +lean_inc(x_31); +lean_dec(x_22); +x_33 = lean_st_ref_get(x_4, x_32); +x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_33, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_33)) { + lean_ctor_release(x_33, 0); + lean_ctor_release(x_33, 1); + x_36 = x_33; } else { - lean_dec_ref(x_30); - x_33 = lean_box(0); -} -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_28); -lean_ctor_set(x_34, 1, x_31); -if (lean_is_scalar(x_33)) { - x_35 = lean_alloc_ctor(0, 2, 0); + lean_dec_ref(x_33); + x_36 = lean_box(0); +} +x_37 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_37, 0, x_31); +lean_ctor_set(x_37, 1, x_34); +if (lean_is_scalar(x_36)) { + x_38 = lean_alloc_ctor(0, 2, 0); } else { - x_35 = x_33; + x_38 = x_36; } -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_32); -return x_35; +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_35); +return x_38; } } } @@ -1361,12 +1380,41 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_G _start: { lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; +x_2 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; x_1 = lean_box(0); x_2 = lean_array_mk(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__15; +x_2 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; +x_3 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 2, x_2); +lean_ctor_set(x_3, 3, x_2); +lean_ctor_set(x_3, 4, x_1); +lean_ctor_set(x_3, 5, x_1); +lean_ctor_set(x_3, 6, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4() { _start: { lean_object* x_1; @@ -1374,7 +1422,7 @@ x_1 = l_Std_Queue_empty(lean_box(0)); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5() { _start: { lean_object* x_1; @@ -1385,7 +1433,7 @@ return x_1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; x_10 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); x_11 = lean_ctor_get(x_10, 0); lean_inc(x_11); @@ -1398,60 +1446,72 @@ lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = l_Lean_Meta_Grind_getEMatchTheorems___rarg(x_8, x_15); +x_16 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_15); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = lean_box(0); -x_20 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__10; -x_21 = l_Lean_PersistentHashMap_empty___at___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___spec__1; -x_22 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__1; -x_23 = 0; -x_24 = lean_unsigned_to_nat(0u); -x_25 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__15; -x_26 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2; -x_27 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; -x_28 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; -x_29 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__3; +x_19 = l_Lean_Meta_Grind_getEMatchTheorems___rarg(x_8, x_18); +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_box(0); +x_23 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__1; +x_24 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__11; +x_25 = l_Lean_PersistentHashMap_empty___at___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___spec__1; +x_26 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; +x_27 = 0; +x_28 = lean_unsigned_to_nat(0u); +x_29 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3; +x_30 = l_Lean_Meta_Grind_GrindM_run___rarg___closed__15; +x_31 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2; +x_32 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4; +x_33 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Match_instInhabitedMatchEqnsExtState___spec__1; +x_34 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__3; lean_inc(x_1); -x_30 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_30, 0, x_1); -lean_ctor_set(x_30, 1, x_20); -lean_ctor_set(x_30, 2, x_20); -lean_ctor_set(x_30, 3, x_21); -lean_ctor_set(x_30, 4, x_20); -lean_ctor_set(x_30, 5, x_22); -lean_ctor_set(x_30, 6, x_24); -lean_ctor_set(x_30, 7, x_24); -lean_ctor_set(x_30, 8, x_25); -lean_ctor_set(x_30, 9, x_25); -lean_ctor_set(x_30, 10, x_17); -lean_ctor_set(x_30, 11, x_24); -lean_ctor_set(x_30, 12, x_24); -lean_ctor_set(x_30, 13, x_26); -lean_ctor_set(x_30, 14, x_27); -lean_ctor_set(x_30, 15, x_28); -lean_ctor_set(x_30, 16, x_19); -lean_ctor_set(x_30, 17, x_24); -lean_ctor_set(x_30, 18, x_29); -lean_ctor_set(x_30, 19, x_24); -lean_ctor_set_uint8(x_30, sizeof(void*)*20, x_23); -x_31 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__1___boxed), 9, 1); -lean_closure_set(x_31, 0, x_30); -x_32 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed), 11, 2); -lean_closure_set(x_32, 0, x_14); -lean_closure_set(x_32, 1, x_11); -x_33 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_33, 0, x_31); -lean_closure_set(x_33, 1, x_32); -x_34 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3; -x_35 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_35, 0, x_33); -lean_closure_set(x_35, 1, x_34); -x_36 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -return x_36; +x_35 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_35, 0, x_1); +lean_ctor_set(x_35, 1, x_23); +lean_ctor_set(x_35, 2, x_24); +lean_ctor_set(x_35, 3, x_24); +lean_ctor_set(x_35, 4, x_25); +lean_ctor_set(x_35, 5, x_24); +lean_ctor_set(x_35, 6, x_26); +lean_ctor_set(x_35, 7, x_28); +lean_ctor_set(x_35, 8, x_28); +lean_ctor_set(x_35, 9, x_29); +lean_ctor_set(x_35, 10, x_30); +lean_ctor_set(x_35, 11, x_30); +lean_ctor_set(x_35, 12, x_20); +lean_ctor_set(x_35, 13, x_28); +lean_ctor_set(x_35, 14, x_28); +lean_ctor_set(x_35, 15, x_31); +lean_ctor_set(x_35, 16, x_32); +lean_ctor_set(x_35, 17, x_33); +lean_ctor_set(x_35, 18, x_22); +lean_ctor_set(x_35, 19, x_28); +lean_ctor_set(x_35, 20, x_34); +lean_ctor_set(x_35, 21, x_28); +lean_ctor_set(x_35, 22, x_30); +lean_ctor_set_uint8(x_35, sizeof(void*)*23, x_27); +x_36 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__1___boxed), 9, 1); +lean_closure_set(x_36, 0, x_35); +x_37 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed), 12, 3); +lean_closure_set(x_37, 0, x_14); +lean_closure_set(x_37, 1, x_11); +lean_closure_set(x_37, 2, x_17); +x_38 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_38, 0, x_36); +lean_closure_set(x_38, 1, x_37); +x_39 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5; +x_40 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); +lean_closure_set(x_40, 0, x_38); +lean_closure_set(x_40, 1, x_39); +x_41 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_1, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_21); +return x_41; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -1469,11 +1529,12 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -1481,8 +1542,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); -return x_12; +return x_13; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -1593,7 +1653,7 @@ else lean_object* x_4; uint8_t x_5; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); -x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*20); +x_5 = lean_ctor_get_uint8(x_4, sizeof(void*)*23); if (x_5 == 0) { uint8_t x_6; @@ -2549,7 +2609,7 @@ lean_closure_set(x_14, 0, x_2); x_15 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); lean_closure_set(x_15, 0, x_13); lean_closure_set(x_15, 1, x_14); -x_16 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3; +x_16 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5; x_17 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); lean_closure_set(x_17, 0, x_15); lean_closure_set(x_17, 1, x_16); @@ -2566,7 +2626,7 @@ if (lean_obj_tag(x_18) == 0) lean_object* x_19; uint8_t x_20; x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); -x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*20); +x_20 = lean_ctor_get_uint8(x_19, sizeof(void*)*23); if (x_20 == 0) { lean_object* x_21; lean_object* x_22; lean_object* x_23; @@ -2675,7 +2735,7 @@ else lean_object* x_14; uint8_t x_15; x_14 = lean_ctor_get(x_2, 0); lean_inc(x_14); -x_15 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); +x_15 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); if (x_15 == 0) { uint8_t x_16; @@ -2866,67 +2926,376 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_main___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -if (lean_obj_tag(x_1) == 0) +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_7, 2); +x_11 = l_Lean_isTracingEnabledForCore(x_1, x_10, x_9); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -lean_object* x_3; -x_3 = l_List_reverse___rarg(x_2); +return x_11; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_11); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +static double _init_l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); return x_3; } +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_11 = lean_ctor_get(x_8, 5); +x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_st_ref_take(x_9, x_14); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_16, 3); +lean_inc(x_17); +x_18 = !lean_is_exclusive(x_15); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_15, 1); +x_20 = lean_ctor_get(x_15, 0); +lean_dec(x_20); +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_16, 3); +lean_dec(x_22); +x_23 = !lean_is_exclusive(x_17); +if (x_23 == 0) +{ +lean_object* x_24; double x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_24 = lean_ctor_get(x_17, 0); +x_25 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1; +x_26 = 0; +x_27 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; +x_28 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_28, 0, x_1); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set_float(x_28, sizeof(void*)*2, x_25); +lean_ctor_set_float(x_28, sizeof(void*)*2 + 8, x_25); +lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 16, x_26); +x_29 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; +x_30 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_13); +lean_ctor_set(x_30, 2, x_29); +lean_inc(x_11); +lean_ctor_set(x_15, 1, x_30); +lean_ctor_set(x_15, 0, x_11); +x_31 = l_Lean_PersistentArray_push___rarg(x_24, x_15); +lean_ctor_set(x_17, 0, x_31); +x_32 = lean_st_ref_set(x_9, x_16, x_19); +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_32, 0); +lean_dec(x_34); +x_35 = lean_box(0); +lean_ctor_set(x_32, 0, x_35); +return x_32; +} else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_1); -if (x_4 == 0) +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_32, 1); +lean_inc(x_36); +lean_dec(x_32); +x_37 = lean_box(0); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +return x_38; +} +} +else { -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = lean_ctor_get(x_1, 0); -x_6 = lean_ctor_get(x_1, 1); -x_7 = lean_ctor_get(x_5, 0); -lean_inc(x_7); -lean_dec(x_5); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_7); +uint64_t x_39; lean_object* x_40; double x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_39 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); +x_40 = lean_ctor_get(x_17, 0); +lean_inc(x_40); +lean_dec(x_17); +x_41 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1; +x_42 = 0; +x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; +x_44 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_44, 0, x_1); +lean_ctor_set(x_44, 1, x_43); +lean_ctor_set_float(x_44, sizeof(void*)*2, x_41); +lean_ctor_set_float(x_44, sizeof(void*)*2 + 8, x_41); +lean_ctor_set_uint8(x_44, sizeof(void*)*2 + 16, x_42); +x_45 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; +x_46 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_13); +lean_ctor_set(x_46, 2, x_45); +lean_inc(x_11); +lean_ctor_set(x_15, 1, x_46); +lean_ctor_set(x_15, 0, x_11); +x_47 = l_Lean_PersistentArray_push___rarg(x_40, x_15); +x_48 = lean_alloc_ctor(0, 1, 8); +lean_ctor_set(x_48, 0, x_47); +lean_ctor_set_uint64(x_48, sizeof(void*)*1, x_39); +lean_ctor_set(x_16, 3, x_48); +x_49 = lean_st_ref_set(x_9, x_16, x_19); +x_50 = lean_ctor_get(x_49, 1); +lean_inc(x_50); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_51 = x_49; +} else { + lean_dec_ref(x_49); + x_51 = lean_box(0); +} +x_52 = lean_box(0); +if (lean_is_scalar(x_51)) { + x_53 = lean_alloc_ctor(0, 2, 0); +} else { + x_53 = x_51; +} +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_50); +return x_53; +} +} +else { -lean_object* _tmp_0 = x_6; -lean_object* _tmp_1 = x_1; -x_1 = _tmp_0; -x_2 = _tmp_1; +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; lean_object* x_62; lean_object* x_63; double x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_54 = lean_ctor_get(x_16, 0); +x_55 = lean_ctor_get(x_16, 1); +x_56 = lean_ctor_get(x_16, 2); +x_57 = lean_ctor_get(x_16, 4); +x_58 = lean_ctor_get(x_16, 5); +x_59 = lean_ctor_get(x_16, 6); +x_60 = lean_ctor_get(x_16, 7); +lean_inc(x_60); +lean_inc(x_59); +lean_inc(x_58); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_dec(x_16); +x_61 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); +x_62 = lean_ctor_get(x_17, 0); +lean_inc(x_62); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_63 = x_17; +} else { + lean_dec_ref(x_17); + x_63 = lean_box(0); +} +x_64 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1; +x_65 = 0; +x_66 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; +x_67 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_67, 0, x_1); +lean_ctor_set(x_67, 1, x_66); +lean_ctor_set_float(x_67, sizeof(void*)*2, x_64); +lean_ctor_set_float(x_67, sizeof(void*)*2 + 8, x_64); +lean_ctor_set_uint8(x_67, sizeof(void*)*2 + 16, x_65); +x_68 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; +x_69 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_13); +lean_ctor_set(x_69, 2, x_68); +lean_inc(x_11); +lean_ctor_set(x_15, 1, x_69); +lean_ctor_set(x_15, 0, x_11); +x_70 = l_Lean_PersistentArray_push___rarg(x_62, x_15); +if (lean_is_scalar(x_63)) { + x_71 = lean_alloc_ctor(0, 1, 8); +} else { + x_71 = x_63; +} +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set_uint64(x_71, sizeof(void*)*1, x_61); +x_72 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_72, 0, x_54); +lean_ctor_set(x_72, 1, x_55); +lean_ctor_set(x_72, 2, x_56); +lean_ctor_set(x_72, 3, x_71); +lean_ctor_set(x_72, 4, x_57); +lean_ctor_set(x_72, 5, x_58); +lean_ctor_set(x_72, 6, x_59); +lean_ctor_set(x_72, 7, x_60); +x_73 = lean_st_ref_set(x_9, x_72, x_19); +x_74 = lean_ctor_get(x_73, 1); +lean_inc(x_74); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_75 = x_73; +} else { + lean_dec_ref(x_73); + x_75 = lean_box(0); +} +x_76 = lean_box(0); +if (lean_is_scalar(x_75)) { + x_77 = lean_alloc_ctor(0, 2, 0); +} else { + x_77 = x_75; +} +lean_ctor_set(x_77, 0, x_76); +lean_ctor_set(x_77, 1, x_74); +return x_77; } -goto _start; } else { -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_9 = lean_ctor_get(x_1, 0); -x_10 = lean_ctor_get(x_1, 1); -lean_inc(x_10); -lean_inc(x_9); -lean_dec(x_1); -x_11 = lean_ctor_get(x_9, 0); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint64_t x_87; lean_object* x_88; lean_object* x_89; double x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_78 = lean_ctor_get(x_15, 1); +lean_inc(x_78); +lean_dec(x_15); +x_79 = lean_ctor_get(x_16, 0); +lean_inc(x_79); +x_80 = lean_ctor_get(x_16, 1); +lean_inc(x_80); +x_81 = lean_ctor_get(x_16, 2); +lean_inc(x_81); +x_82 = lean_ctor_get(x_16, 4); +lean_inc(x_82); +x_83 = lean_ctor_get(x_16, 5); +lean_inc(x_83); +x_84 = lean_ctor_get(x_16, 6); +lean_inc(x_84); +x_85 = lean_ctor_get(x_16, 7); +lean_inc(x_85); +if (lean_is_exclusive(x_16)) { + lean_ctor_release(x_16, 0); + lean_ctor_release(x_16, 1); + lean_ctor_release(x_16, 2); + lean_ctor_release(x_16, 3); + lean_ctor_release(x_16, 4); + lean_ctor_release(x_16, 5); + lean_ctor_release(x_16, 6); + lean_ctor_release(x_16, 7); + x_86 = x_16; +} else { + lean_dec_ref(x_16); + x_86 = lean_box(0); +} +x_87 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); +x_88 = lean_ctor_get(x_17, 0); +lean_inc(x_88); +if (lean_is_exclusive(x_17)) { + lean_ctor_release(x_17, 0); + x_89 = x_17; +} else { + lean_dec_ref(x_17); + x_89 = lean_box(0); +} +x_90 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1; +x_91 = 0; +x_92 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; +x_93 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_93, 0, x_1); +lean_ctor_set(x_93, 1, x_92); +lean_ctor_set_float(x_93, sizeof(void*)*2, x_90); +lean_ctor_set_float(x_93, sizeof(void*)*2 + 8, x_90); +lean_ctor_set_uint8(x_93, sizeof(void*)*2 + 16, x_91); +x_94 = l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2; +x_95 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_95, 0, x_93); +lean_ctor_set(x_95, 1, x_13); +lean_ctor_set(x_95, 2, x_94); lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_12, 0, x_11); -lean_ctor_set(x_12, 1, x_2); -x_1 = x_10; -x_2 = x_12; -goto _start; +x_96 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_11); +lean_ctor_set(x_96, 1, x_95); +x_97 = l_Lean_PersistentArray_push___rarg(x_88, x_96); +if (lean_is_scalar(x_89)) { + x_98 = lean_alloc_ctor(0, 1, 8); +} else { + x_98 = x_89; } +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set_uint64(x_98, sizeof(void*)*1, x_87); +if (lean_is_scalar(x_86)) { + x_99 = lean_alloc_ctor(0, 8, 0); +} else { + x_99 = x_86; +} +lean_ctor_set(x_99, 0, x_79); +lean_ctor_set(x_99, 1, x_80); +lean_ctor_set(x_99, 2, x_81); +lean_ctor_set(x_99, 3, x_98); +lean_ctor_set(x_99, 4, x_82); +lean_ctor_set(x_99, 5, x_83); +lean_ctor_set(x_99, 6, x_84); +lean_ctor_set(x_99, 7, x_85); +x_100 = lean_st_ref_set(x_9, x_99, x_78); +x_101 = lean_ctor_get(x_100, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + x_102 = x_100; +} else { + lean_dec_ref(x_100); + x_102 = lean_box(0); +} +x_103 = lean_box(0); +if (lean_is_scalar(x_102)) { + x_104 = lean_alloc_ctor(0, 2, 0); +} else { + x_104 = x_102; } +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_101); +return x_104; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; lean_object* x_13; -x_12 = l_List_mapTR_loop___at_Lean_Meta_Grind_main___spec__3(x_1, x_2); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_object* x_11; +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_1); +lean_ctor_set(x_11, 1, x_10); +return x_11; } } static lean_object* _init_l_Lean_Meta_Grind_main___lambda__2___closed__1() { @@ -2959,16 +3328,8 @@ return x_4; static lean_object* _init_l_Lean_Meta_Grind_main___lambda__2___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_Grind_main___lambda__2___closed__5() { -_start: -{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_main___lambda__2___closed__4; +x_1 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } @@ -3012,19 +3373,14 @@ x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); x_19 = l_Lean_Meta_Grind_main___lambda__2___closed__3; -x_20 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); +x_20 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3(x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_18); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); x_22 = lean_unbox(x_21); lean_dec(x_21); if (x_22 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_20, 1); -lean_inc(x_23); -lean_dec(x_20); -x_24 = lean_box(0); -x_25 = l_Lean_Meta_Grind_main___lambda__1(x_17, x_15, x_24, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +uint8_t x_23; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3032,50 +3388,55 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -return x_25; +x_23 = !lean_is_exclusive(x_20); +if (x_23 == 0) +{ +lean_object* x_24; +x_24 = lean_ctor_get(x_20, 0); +lean_dec(x_24); +lean_ctor_set(x_20, 0, x_17); +return x_20; } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_20); -if (x_26 == 0) +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_20, 1); +lean_inc(x_25); +lean_dec(x_20); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_17); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_object* x_27; lean_object* x_28; x_27 = lean_ctor_get(x_20, 1); -x_28 = lean_ctor_get(x_20, 0); -lean_dec(x_28); +lean_inc(x_27); +lean_dec(x_20); lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); lean_inc(x_17); -x_29 = l_Lean_Meta_Grind_ppGoals(x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); -if (lean_obj_tag(x_29) == 0) +x_28 = l_Lean_Meta_Grind_ppGoals(x_17, x_6, x_7, x_8, x_9, x_27); +if (lean_obj_tag(x_28) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_30 = lean_ctor_get(x_29, 0); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = l_Lean_MessageData_ofFormat(x_30); -x_33 = l_Lean_Meta_Grind_main___lambda__2___closed__5; -lean_ctor_set_tag(x_20, 7); -lean_ctor_set(x_20, 1, x_32); -lean_ctor_set(x_20, 0, x_33); -x_34 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_34, 0, x_20); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_19, x_34, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_31); -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = l_Lean_Meta_Grind_main___lambda__1(x_17, x_15, x_36, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_37); +lean_dec(x_28); +x_31 = l_Lean_Meta_Grind_main___lambda__2___closed__4; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_29); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +x_34 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4(x_19, x_33, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_30); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3083,13 +3444,30 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +x_35 = !lean_is_exclusive(x_34); +if (x_35 == 0) +{ +lean_object* x_36; +x_36 = lean_ctor_get(x_34, 0); lean_dec(x_36); +lean_ctor_set(x_34, 0, x_17); +return x_34; +} +else +{ +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 1); +lean_inc(x_37); +lean_dec(x_34); +x_38 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_38, 0, x_17); +lean_ctor_set(x_38, 1, x_37); return x_38; } +} else { uint8_t x_39; -lean_free_object(x_20); lean_dec(x_17); lean_dec(x_9); lean_dec(x_8); @@ -3098,19 +3476,19 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_39 = !lean_is_exclusive(x_29); +x_39 = !lean_is_exclusive(x_28); if (x_39 == 0) { -return x_29; +return x_28; } else { lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_29, 0); -x_41 = lean_ctor_get(x_29, 1); +x_40 = lean_ctor_get(x_28, 0); +x_41 = lean_ctor_get(x_28, 1); lean_inc(x_41); lean_inc(x_40); -lean_dec(x_29); +lean_dec(x_28); x_42 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_42, 0, x_40); lean_ctor_set(x_42, 1, x_41); @@ -3118,92 +3496,10 @@ return x_42; } } } -else -{ -lean_object* x_43; lean_object* x_44; -x_43 = lean_ctor_get(x_20, 1); -lean_inc(x_43); -lean_dec(x_20); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_17); -x_44 = l_Lean_Meta_Grind_ppGoals(x_17, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_43); -if (lean_obj_tag(x_44) == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_45 = lean_ctor_get(x_44, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_44, 1); -lean_inc(x_46); -lean_dec(x_44); -x_47 = l_Lean_MessageData_ofFormat(x_45); -x_48 = l_Lean_Meta_Grind_main___lambda__2___closed__5; -x_49 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_47); -x_50 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -x_51 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_19, x_50, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_46); -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); -lean_inc(x_53); -lean_dec(x_51); -x_54 = l_Lean_Meta_Grind_main___lambda__1(x_17, x_15, x_52, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_53); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_52); -return x_54; -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_17); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_55 = lean_ctor_get(x_44, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_44, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_44)) { - lean_ctor_release(x_44, 0); - lean_ctor_release(x_44, 1); - x_57 = x_44; -} else { - lean_dec_ref(x_44); - x_57 = lean_box(0); -} -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); -} else { - x_58 = x_57; -} -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; -} -} -} } else { -uint8_t x_59; +uint8_t x_43; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3211,29 +3507,29 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -x_59 = !lean_is_exclusive(x_16); -if (x_59 == 0) +x_43 = !lean_is_exclusive(x_16); +if (x_43 == 0) { return x_16; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_16, 0); -x_61 = lean_ctor_get(x_16, 1); -lean_inc(x_61); -lean_inc(x_60); +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_16, 0); +x_45 = lean_ctor_get(x_16, 1); +lean_inc(x_45); +lean_inc(x_44); lean_dec(x_16); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; } } } else { -uint8_t x_63; +uint8_t x_47; lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3242,23 +3538,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_12); -if (x_63 == 0) +x_47 = !lean_is_exclusive(x_12); +if (x_47 == 0) { return x_12; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_12, 0); -x_65 = lean_ctor_get(x_12, 1); -lean_inc(x_65); -lean_inc(x_64); +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_12, 0); +x_49 = lean_ctor_get(x_12, 1); +lean_inc(x_49); +lean_inc(x_48); lean_dec(x_12); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } } } @@ -3336,12 +3632,26 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_12; -x_12 = l_Lean_Meta_Grind_main___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); +lean_object* x_10; +x_10 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_main___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3349,7 +3659,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -return x_12; +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_main___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_main___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; } } lean_object* initialize_Init_Grind_Lemmas(uint8_t builtin, lean_object*); @@ -3449,6 +3775,10 @@ l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2 = lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__2); l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__3); +l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__4); +l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_mkGoal___closed__5); l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__1); l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_initCore___closed__2(); @@ -3473,6 +3803,9 @@ l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__3___ lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___lambda__3___closed__1); l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Main_0__Lean_Meta_Grind_simple___closed__1); +l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__1(); +l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2(); +lean_mark_persistent(l_Lean_addTrace___at_Lean_Meta_Grind_main___spec__4___closed__2); l_Lean_Meta_Grind_main___lambda__2___closed__1 = _init_l_Lean_Meta_Grind_main___lambda__2___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_main___lambda__2___closed__1); l_Lean_Meta_Grind_main___lambda__2___closed__2 = _init_l_Lean_Meta_Grind_main___lambda__2___closed__2(); @@ -3481,8 +3814,6 @@ l_Lean_Meta_Grind_main___lambda__2___closed__3 = _init_l_Lean_Meta_Grind_main___ lean_mark_persistent(l_Lean_Meta_Grind_main___lambda__2___closed__3); l_Lean_Meta_Grind_main___lambda__2___closed__4 = _init_l_Lean_Meta_Grind_main___lambda__2___closed__4(); lean_mark_persistent(l_Lean_Meta_Grind_main___lambda__2___closed__4); -l_Lean_Meta_Grind_main___lambda__2___closed__5 = _init_l_Lean_Meta_Grind_main___lambda__2___closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_main___lambda__2___closed__5); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/PP.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/PP.c index 0e511d3997ea..568ffc2fba86 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/PP.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/PP.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind.PP -// Imports: Init.Grind.Util Lean.Meta.Tactic.Grind.Types +// Imports: Init.Grind.Util Init.Grind.PP Lean.Meta.Tactic.Grind.Types Lean.Meta.Tactic.Grind.Arith.Model #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,102 +13,210 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__3; -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1; lean_object* l_Lean_Meta_ppExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1; -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___closed__4; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalsToMessageData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_mkNatLit(lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4; -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___closed__3; -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2; +lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_Goal_ppState___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5; +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_joinSep(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4; +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7; uint8_t l_Lean_Expr_isApp(lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalToMessageData___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6; +lean_object* l_Lean_MessageData_ofList(lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2; lean_object* lean_mk_array(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getEqcs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2; -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__2; -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__6; +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2; +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2; +lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getENodes(lean_object*); +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7; +lean_object* l_List_find_x3f___rarg(lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5; +lean_object* l_Lean_stringToMessageData(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2; +LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3; +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6; extern lean_object* l_Lean_Meta_Grind_grind_debug; -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1; -lean_object* l_Lean_Meta_Grind_getTarget_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1; -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__1; -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__5; -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDeclValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3; +lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_goalToMessageData___closed__3; +LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2; +static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1; +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3; +lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1; +static double l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1; +lean_object* l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofFormat(lean_object*); +lean_object* l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3; +lean_object* l_Lean_Meta_getLevel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_goalToMessageData___closed__2; lean_object* lean_st_ref_get(lean_object*, lean_object*); -lean_object* lean_st_mk_ref(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12; +uint8_t l_List_isEmpty___rarg(lean_object*); +lean_object* lean_array_to_list(lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppState___closed__1; +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8; extern lean_object* l_Lean_levelZero; -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppState(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1; +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_goalsToMessageData___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +lean_object* l_Lean_Expr_isFalse___boxed(lean_object*); lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2; -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___closed__2; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7; uint8_t l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_getENodes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDeclValue___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8; +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalToMessageData(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Array_append___rarg(lean_object*, lean_object*); +lean_object* l_Lean_MessageData_ofExpr(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Arith_Offset_mkModel(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8; +lean_object* l_Lean_Meta_Grind_Origin_pp___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_ppState(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1; +static lean_object* l_Lean_Meta_Grind_goalToMessageData___closed__1; +uint8_t l_Lean_Expr_isFalse(lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2; +lean_object* l_Lean_Expr_isTrue___boxed(lean_object*); +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3; +lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getEqcs(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4; -static lean_object* l_Lean_Meta_Grind_ppState___closed__2; -static lean_object* l_Lean_Meta_Grind_ppENodeDeclValue___closed__1; -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Std_Format_joinSep___at_Prod_repr___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1(size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4; lean_object* lean_nat_sub(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5; -lean_object* l_Lean_Meta_Grind_getENode_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3; -lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3; +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +lean_object* l_Lean_Meta_Grind_Goal_getENode_x3f(lean_object*, lean_object*); +lean_object* lean_array_mk(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(lean_object*, lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isTrue(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeRef___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +static lean_object* l_Lean_Meta_Grind_Goal_ppState___closed__2; +uint8_t l_Lean_PersistentArray_isEmpty___rarg(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1; +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5; +static lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3; +static lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3; +static lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Meta_Grind_ppENodeRef___closed__4; -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2; uint8_t l_Lean_Expr_isConst(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_ppState___closed__1; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppGoals(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); lean_object* l_Lean_Meta_isLitValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__1() { +static lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1; +lean_object* l_Lean_Meta_isProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2; +uint8_t l_Array_isEmpty___rarg(lean_object*); +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1() { _start: { lean_object* x_1; @@ -116,35 +224,61 @@ x_1 = lean_mk_string_unchecked("_", 1, 1); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeRef___closed__1; +x_1 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("#", 1, 1); +x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeRef___closed__3; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Grind", 5, 5); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("node_def", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4; +x_2 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5; +x_3 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8() { _start: { lean_object* x_1; @@ -152,164 +286,203 @@ x_1 = lean_mk_string_unchecked("", 0, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeRef___closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeRef___closed__5; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_ppENodeRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { +lean_object* x_8; +x_8 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_1, x_2); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_9 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3; +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_7); +return x_10; +} +else +{ lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Meta_Grind_getENode_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); +x_11 = lean_ctor_get(x_8, 0); +lean_inc(x_11); +lean_dec(x_8); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_12 = lean_infer_type(x_2, x_3, x_4, x_5, x_6, x_7); if (lean_obj_tag(x_12) == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +lean_inc(x_13); +x_15 = l_Lean_Meta_getLevel(x_13, x_3, x_4, x_5, x_6, x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = l_Lean_Meta_Grind_ppENodeRef___closed__2; -lean_ctor_set(x_11, 0, x_15); -return x_11; +uint8_t x_16; +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_box(0); +x_19 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_19, 0, x_17); +lean_ctor_set(x_19, 1, x_18); +x_20 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7; +x_21 = l_Lean_Expr_const___override(x_20, x_19); +x_22 = lean_ctor_get(x_11, 7); +lean_inc(x_22); +lean_dec(x_11); +x_23 = l_Lean_mkNatLit(x_22); +x_24 = l_Lean_mkApp3(x_21, x_23, x_13, x_2); +x_25 = l_Lean_MessageData_ofExpr(x_24); +x_26 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +lean_ctor_set(x_15, 0, x_28); +return x_15; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_29 = lean_ctor_get(x_15, 0); +x_30 = lean_ctor_get(x_15, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_15); +x_31 = lean_box(0); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_29); +lean_ctor_set(x_32, 1, x_31); +x_33 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7; +x_34 = l_Lean_Expr_const___override(x_33, x_32); +x_35 = lean_ctor_get(x_11, 7); +lean_inc(x_35); lean_dec(x_11); -x_17 = l_Lean_Meta_Grind_ppENodeRef___closed__2; -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +x_36 = l_Lean_mkNatLit(x_35); +x_37 = l_Lean_mkApp3(x_34, x_36, x_13, x_2); +x_38 = l_Lean_MessageData_ofExpr(x_37); +x_39 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_38); +x_41 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_39); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_30); +return x_42; } } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) -{ -lean_object* x_20; uint8_t x_21; -x_20 = lean_ctor_get(x_11, 0); -lean_dec(x_20); -x_21 = !lean_is_exclusive(x_12); -if (x_21 == 0) +uint8_t x_43; +lean_dec(x_13); +lean_dec(x_11); +lean_dec(x_2); +x_43 = !lean_is_exclusive(x_15); +if (x_43 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_22 = lean_ctor_get(x_12, 0); -x_23 = lean_ctor_get(x_22, 7); -lean_inc(x_23); -lean_dec(x_22); -x_24 = l___private_Init_Data_Repr_0__Nat_reprFast(x_23); -lean_ctor_set_tag(x_12, 3); -lean_ctor_set(x_12, 0, x_24); -x_25 = l_Lean_Meta_Grind_ppENodeRef___closed__4; -x_26 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_12); -x_27 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -x_28 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set(x_11, 0, x_28); -return x_11; +return x_15; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_29 = lean_ctor_get(x_12, 0); -lean_inc(x_29); -lean_dec(x_12); -x_30 = lean_ctor_get(x_29, 7); -lean_inc(x_30); -lean_dec(x_29); -x_31 = l___private_Init_Data_Repr_0__Nat_reprFast(x_30); -x_32 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = l_Lean_Meta_Grind_ppENodeRef___closed__4; -x_34 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_32); -x_35 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -x_36 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -lean_ctor_set(x_11, 0, x_36); -return x_11; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_15, 0); +x_45 = lean_ctor_get(x_15, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_15); +x_46 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_46, 0, x_44); +lean_ctor_set(x_46, 1, x_45); +return x_46; +} } } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_37 = lean_ctor_get(x_11, 1); -lean_inc(x_37); +uint8_t x_47; lean_dec(x_11); -x_38 = lean_ctor_get(x_12, 0); -lean_inc(x_38); -if (lean_is_exclusive(x_12)) { - lean_ctor_release(x_12, 0); - x_39 = x_12; -} else { - lean_dec_ref(x_12); - x_39 = lean_box(0); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_47 = !lean_is_exclusive(x_12); +if (x_47 == 0) +{ +return x_12; +} +else +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_12, 0); +x_49 = lean_ctor_get(x_12, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_12); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } -x_40 = lean_ctor_get(x_38, 7); -lean_inc(x_40); -lean_dec(x_38); -x_41 = l___private_Init_Data_Repr_0__Nat_reprFast(x_40); -if (lean_is_scalar(x_39)) { - x_42 = lean_alloc_ctor(3, 1, 0); -} else { - x_42 = x_39; - lean_ctor_set_tag(x_42, 3); } -lean_ctor_set(x_42, 0, x_41); -x_43 = l_Lean_Meta_Grind_ppENodeRef___closed__4; -x_44 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_42); -x_45 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -x_46 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_46); -lean_ctor_set(x_47, 1, x_37); -return x_47; } } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeRef(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_12, x_1, x_6, x_7, x_8, x_9, x_13); +return x_14; +} } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeRef___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; x_11 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); return x_11; } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1() { _start: { lean_object* x_1; @@ -317,164 +490,254 @@ x_1 = lean_mk_string_unchecked(" ", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1; +x_1 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3() { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_5, x_4); -if (x_16 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_17; -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_6); -lean_ctor_set(x_17, 1, x_15); -return x_17; +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_6, x_5); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_7); +lean_ctor_set(x_14, 1, x_12); +return x_14; } else { -lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_18 = lean_array_uget(x_3, x_5); -x_19 = l_Lean_Meta_Grind_ppENodeRef(x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_18); -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +lean_object* x_15; lean_object* x_16; +x_15 = lean_array_uget(x_4, x_6); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_1); +x_16 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_15, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; size_t x_25; size_t x_26; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_ctor_get(x_19, 1); -x_23 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2; -lean_ctor_set_tag(x_19, 5); -lean_ctor_set(x_19, 1, x_23); -lean_ctor_set(x_19, 0, x_6); -x_24 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_24, 0, x_19); -lean_ctor_set(x_24, 1, x_21); -x_25 = 1; -x_26 = lean_usize_add(x_5, x_25); -x_5 = x_26; -x_6 = x_24; -x_15 = x_22; +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; size_t x_22; size_t x_23; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3; +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_7); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_17); +x_22 = 1; +x_23 = lean_usize_add(x_6, x_22); +x_6 = x_23; +x_7 = x_21; +x_12 = x_18; goto _start; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; size_t x_33; size_t x_34; -x_28 = lean_ctor_get(x_19, 0); -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_19); -x_30 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2; -x_31 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_31, 0, x_6); -lean_ctor_set(x_31, 1, x_30); -x_32 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_28); -x_33 = 1; -x_34 = lean_usize_add(x_5, x_33); -x_5 = x_34; -x_6 = x_32; -x_15 = x_29; -goto _start; +uint8_t x_25; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_1); +x_25 = !lean_is_exclusive(x_16); +if (x_25 == 0) +{ +return x_16; +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_16, 0); +x_27 = lean_ctor_get(x_16, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_16); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; +} } } } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_12; size_t x_13; size_t x_14; lean_object* x_15; uint8_t x_16; -x_12 = lean_box(0); -x_13 = lean_array_size(x_1); -x_14 = 0; -x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1(x_1, x_12, x_1, x_13, x_14, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_object* x_9; size_t x_10; size_t x_11; lean_object* x_12; +x_9 = lean_box(0); +x_10 = lean_array_size(x_1); +x_11 = 0; +x_12 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1(x_2, x_1, x_9, x_1, x_10, x_11, x_3, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_12) == 0) { -return x_15; +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +return x_12; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_15); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -return x_19; -} +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_12); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: +else { -if (lean_obj_tag(x_1) == 5) +uint8_t x_17; +x_17 = !lean_is_exclusive(x_12); +if (x_17 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_1, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_1, 1); -lean_inc(x_14); -lean_dec(x_1); -x_15 = lean_array_set(x_2, x_3, x_14); -x_16 = lean_unsigned_to_nat(1u); -x_17 = lean_nat_sub(x_3, x_16); -lean_dec(x_3); -x_1 = x_13; -x_2 = x_15; -x_3 = x_17; -goto _start; +return x_12; } else { -uint8_t x_19; -lean_dec(x_3); -x_19 = l_Lean_Expr_isConst(x_1); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_20 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_1); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1(x_2, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_12, 0); +x_19 = lean_ctor_get(x_12, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_12); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (lean_obj_tag(x_2) == 5) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = lean_ctor_get(x_2, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_2, 1); +lean_inc(x_11); lean_dec(x_2); -return x_23; +x_12 = lean_array_set(x_3, x_4, x_11); +x_13 = lean_unsigned_to_nat(1u); +x_14 = lean_nat_sub(x_4, x_13); +lean_dec(x_4); +x_2 = x_10; +x_3 = x_12; +x_4 = x_14; +goto _start; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = l_Lean_Meta_ppExpr(x_1, x_8, x_9, x_10, x_11, x_12); -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1(x_2, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); -lean_dec(x_2); -return x_27; +uint8_t x_16; +lean_dec(x_4); +x_16 = l_Lean_Expr_isConst(x_2); +if (x_16 == 0) +{ +lean_object* x_17; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_1); +x_17 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_2, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1(x_3, x_1, x_18, x_5, x_6, x_7, x_8, x_19); +lean_dec(x_3); +return x_20; +} +else +{ +uint8_t x_21; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_1); +x_21 = !lean_is_exclusive(x_17); +if (x_21 == 0) +{ +return x_17; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_17); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = l_Lean_MessageData_ofExpr(x_2); +x_26 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +x_29 = l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1(x_3, x_1, x_28, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_3); +return x_29; } } } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDeclValue___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -483,187 +746,186 @@ x_2 = l_Lean_Expr_sort___override(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDeclValue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_11; -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); +lean_object* x_8; lean_inc(x_6); -lean_inc(x_1); -x_11 = l_Lean_Meta_isLitValue(x_1, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_8 = l_Lean_Meta_isLitValue(x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = l_Lean_Expr_isApp(x_1); -if (x_14 == 0) +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Lean_Expr_isApp(x_2); +if (x_11 == 0) { -lean_object* x_15; -lean_dec(x_12); -x_15 = l_Lean_Meta_ppExpr(x_1, x_6, x_7, x_8, x_9, x_13); +lean_object* x_12; uint8_t x_13; lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_1); +x_12 = l_Lean_Meta_ppExpr(x_2, x_3, x_4, x_5, x_6, x_10); lean_dec(x_6); -return x_15; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_MessageData_ofFormat(x_14); +lean_ctor_set(x_12, 0, x_15); +return x_12; } else { -uint8_t x_16; -x_16 = lean_unbox(x_12); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_12, 0); +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_inc(x_16); lean_dec(x_12); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_unsigned_to_nat(0u); -x_18 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_17); -x_19 = l_Lean_Meta_Grind_ppENodeDeclValue___closed__1; -lean_inc(x_18); -x_20 = lean_mk_array(x_18, x_19); -x_21 = lean_unsigned_to_nat(1u); -x_22 = lean_nat_sub(x_18, x_21); -lean_dec(x_18); -x_23 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2(x_1, x_20, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_23; +x_18 = l_Lean_MessageData_ofFormat(x_16); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; +} } else { -lean_object* x_24; -x_24 = l_Lean_Meta_ppExpr(x_1, x_6, x_7, x_8, x_9, x_13); +uint8_t x_20; +x_20 = lean_unbox(x_9); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -return x_24; -} -} +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_21 = lean_unsigned_to_nat(0u); +x_22 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_2, x_21); +x_23 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1; +lean_inc(x_22); +x_24 = lean_mk_array(x_22, x_23); +x_25 = lean_unsigned_to_nat(1u); +x_26 = lean_nat_sub(x_22, x_25); +lean_dec(x_22); +x_27 = l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2(x_1, x_2, x_24, x_26, x_3, x_4, x_5, x_6, x_10); +return x_27; } else { -uint8_t x_25; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +lean_object* x_28; uint8_t x_29; lean_dec(x_1); -x_25 = !lean_is_exclusive(x_11); -if (x_25 == 0) +x_28 = l_Lean_Meta_ppExpr(x_2, x_3, x_4, x_5, x_6, x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_29 = !lean_is_exclusive(x_28); +if (x_29 == 0) { -return x_11; +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_28, 0); +x_31 = l_Lean_MessageData_ofFormat(x_30); +lean_ctor_set(x_28, 0, x_31); +return x_28; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_11, 0); -x_27 = lean_ctor_get(x_11, 1); -lean_inc(x_27); -lean_inc(x_26); -lean_dec(x_11); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_27); -return x_28; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_32 = lean_ctor_get(x_28, 0); +x_33 = lean_ctor_get(x_28, 1); +lean_inc(x_33); +lean_inc(x_32); +lean_dec(x_28); +x_34 = l_Lean_MessageData_ofFormat(x_32); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_33); +return x_35; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: +else { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_17 = lean_unbox_usize(x_5); +uint8_t x_36; +lean_dec(x_6); lean_dec(x_5); -x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1(x_1, x_2, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_18; -} +x_36 = !lean_is_exclusive(x_8); +if (x_36 == 0) +{ +return x_8; } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_8, 0); +x_38 = lean_ctor_get(x_8, 1); +lean_inc(x_38); +lean_inc(x_37); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -return x_12; +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } -LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; -x_13 = l_Lean_Expr_withAppAux___at_Lean_Meta_Grind_ppENodeDeclValue___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_13; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDeclValue___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_ppENodeDeclValue(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_5); lean_dec(x_5); +x_14 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_15 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_11; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_12; -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_11); -return x_12; +lean_object* x_9; +x_9 = l_Lean_Expr_withAppAux___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__2___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_1); +return x_9; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +return x_8; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_ppENodeDecl___lambda__1___boxed), 11, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1___boxed), 7, 0); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2() { _start: { lean_object* x_1; @@ -671,7 +933,7 @@ x_1 = l_Lean_Meta_Grind_grind_debug; return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3() { _start: { lean_object* x_1; @@ -679,156 +941,114 @@ x_1 = lean_mk_string_unchecked(" ↝ ", 5, 3); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_14 = lean_ctor_get(x_11, 2); -lean_inc(x_14); -x_15 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1; -x_16 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2; -x_17 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_14, x_16); -lean_dec(x_14); -if (x_17 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_ctor_get(x_8, 2); +lean_inc(x_11); +x_12 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1; +x_13 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2; +x_14 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_11, x_13); +lean_dec(x_11); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +lean_dec(x_3); +lean_dec(x_1); +x_15 = lean_box(0); +x_16 = lean_apply_7(x_12, x_4, x_15, x_6, x_7, x_8, x_9, x_10); +return x_16; +} +else +{ +lean_object* x_17; +lean_inc(x_1); +x_17 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_1, x_2); +if (lean_obj_tag(x_17) == 0) { lean_object* x_18; lean_object* x_19; -lean_dec(x_2); +lean_dec(x_3); +lean_dec(x_1); x_18 = lean_box(0); -x_19 = lean_apply_11(x_15, x_3, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +x_19 = lean_apply_7(x_12, x_4, x_18, x_6, x_7, x_8, x_9, x_10); return x_19; } else { lean_object* x_20; lean_object* x_21; -x_20 = l_Lean_Meta_Grind_getTarget_x3f(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_2); -x_22 = lean_ctor_get(x_20, 1); +x_20 = lean_ctor_get(x_17, 0); +lean_inc(x_20); +lean_dec(x_17); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_21 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_20, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -lean_dec(x_20); -x_23 = lean_box(0); -x_24 = lean_apply_11(x_15, x_3, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); -return x_24; +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4; +x_25 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_22); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_3); +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_4); +lean_ctor_set(x_27, 1, x_26); +x_28 = lean_box(0); +x_29 = lean_apply_7(x_12, x_27, x_28, x_6, x_7, x_8, x_9, x_23); +return x_29; } else { -uint8_t x_25; -x_25 = !lean_is_exclusive(x_20); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_26 = lean_ctor_get(x_20, 1); -x_27 = lean_ctor_get(x_20, 0); -lean_dec(x_27); -x_28 = lean_ctor_get(x_21, 0); -lean_inc(x_28); -lean_dec(x_21); -x_29 = l_Lean_Meta_Grind_ppENodeRef(x_28, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_26); -lean_dec(x_28); -x_30 = !lean_is_exclusive(x_29); +uint8_t x_30; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_4); +lean_dec(x_3); +x_30 = !lean_is_exclusive(x_21); if (x_30 == 0) { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_31 = lean_ctor_get(x_29, 0); -x_32 = lean_ctor_get(x_29, 1); -x_33 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4; -lean_ctor_set_tag(x_29, 5); -lean_ctor_set(x_29, 1, x_31); -lean_ctor_set(x_29, 0, x_33); -lean_ctor_set_tag(x_20, 5); -lean_ctor_set(x_20, 1, x_2); -lean_ctor_set(x_20, 0, x_29); -x_34 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_34, 0, x_3); -lean_ctor_set(x_34, 1, x_20); -x_35 = lean_box(0); -x_36 = lean_apply_11(x_15, x_34, x_35, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_32); -return x_36; -} -else -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_37 = lean_ctor_get(x_29, 0); -x_38 = lean_ctor_get(x_29, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_29); -x_39 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4; -x_40 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_37); -lean_ctor_set_tag(x_20, 5); -lean_ctor_set(x_20, 1, x_2); -lean_ctor_set(x_20, 0, x_40); -x_41 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_41, 0, x_3); -lean_ctor_set(x_41, 1, x_20); -x_42 = lean_box(0); -x_43 = lean_apply_11(x_15, x_41, x_42, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_38); -return x_43; -} +return x_21; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_44 = lean_ctor_get(x_20, 1); -lean_inc(x_44); -lean_dec(x_20); -x_45 = lean_ctor_get(x_21, 0); -lean_inc(x_45); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_21, 0); +x_32 = lean_ctor_get(x_21, 1); +lean_inc(x_32); +lean_inc(x_31); lean_dec(x_21); -x_46 = l_Lean_Meta_Grind_ppENodeRef(x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_44); -lean_dec(x_45); -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_49 = x_46; -} else { - lean_dec_ref(x_46); - x_49 = lean_box(0); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } -x_50 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4; -if (lean_is_scalar(x_49)) { - x_51 = lean_alloc_ctor(5, 2, 0); -} else { - x_51 = x_49; - lean_ctor_set_tag(x_51, 5); -} -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_47); -x_52 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_2); -x_53 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_53, 0, x_3); -lean_ctor_set(x_53, 1, x_52); -x_54 = lean_box(0); -x_55 = lean_apply_11(x_15, x_53, x_54, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_48); -return x_55; } } } } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -836,42 +1056,51 @@ x_1 = lean_mk_string_unchecked(", [ctor]", 8, 8); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3() { _start: { -uint8_t x_15; -x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 2); -if (x_15 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_16; lean_object* x_17; -x_16 = lean_box(0); -x_17 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2(x_1, x_2, x_4, x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_17; +uint8_t x_12; +x_12 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 2); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2(x_1, x_2, x_3, x_5, x_13, x_7, x_8, x_9, x_10, x_11); +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2; -x_19 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_19, 0, x_4); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_box(0); -x_21 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2(x_1, x_2, x_19, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_21; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_15); +x_17 = lean_box(0); +x_18 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2(x_1, x_2, x_3, x_16, x_17, x_7, x_8, x_9, x_10, x_11); +return x_18; } } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1() { _start: { lean_object* x_1; @@ -879,42 +1108,51 @@ x_1 = lean_mk_string_unchecked(", [val]", 7, 7); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -uint8_t x_15; -x_15 = lean_ctor_get_uint8(x_3, sizeof(void*)*10 + 1); -if (x_15 == 0) +uint8_t x_12; +x_12 = lean_ctor_get_uint8(x_4, sizeof(void*)*11 + 1); +if (x_12 == 0) { -lean_object* x_16; lean_object* x_17; -x_16 = lean_box(0); -x_17 = l_Lean_Meta_Grind_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_4, x_16, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_17; +lean_object* x_13; lean_object* x_14; +x_13 = lean_box(0); +x_14 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_13, x_7, x_8, x_9, x_10, x_11); +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2; -x_19 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_19, 0, x_4); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_box(0); -x_21 = l_Lean_Meta_Grind_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_19, x_20, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -return x_21; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_5); +lean_ctor_set(x_16, 1, x_15); +x_17 = lean_box(0); +x_18 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_4, x_16, x_17, x_7, x_8, x_9, x_10, x_11); +return x_18; } } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1() { _start: { lean_object* x_1; @@ -922,17 +1160,16 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeDecl___closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3() { _start: { lean_object* x_1; @@ -940,418 +1177,288 @@ x_1 = lean_mk_string_unchecked(" ↦ ", 5, 3); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppENodeDecl___closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppENodeDecl___closed__3; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = l_Lean_Meta_Grind_ppENodeRef(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_8 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_8, 0); lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); lean_inc(x_1); -x_15 = l_Lean_Meta_Grind_ppENodeDeclValue(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -if (lean_obj_tag(x_15) == 0) +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue(x_1, x_2, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -lean_ctor_set_tag(x_11, 5); -lean_ctor_set(x_11, 1, x_13); -lean_ctor_set(x_11, 0, x_18); -x_19 = l_Lean_Meta_Grind_ppENodeDecl___closed__2; -x_20 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_20, 0, x_11); -lean_ctor_set(x_20, 1, x_19); -x_21 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_16); -x_22 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_18); +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_9); +x_16 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2; +x_17 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_12); +x_19 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_14); +lean_inc(x_2); lean_inc(x_1); -x_23 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); -if (lean_obj_tag(x_23) == 0) +x_20 = l_Lean_Meta_Grind_Goal_getENode(x_1, x_2, x_5, x_6, x_13); +if (lean_obj_tag(x_20) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_ctor_get(x_24, 2); -lean_inc(x_26); -x_27 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_26); -if (x_27 == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = lean_ctor_get(x_21, 2); +lean_inc(x_23); +x_24 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_2, x_23); +if (x_24 == 0) { -lean_object* x_28; uint8_t x_29; -x_28 = l_Lean_Meta_Grind_ppENodeRef(x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -lean_dec(x_26); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +lean_object* x_25; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_25 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_23, x_3, x_4, x_5, x_6, x_22); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_30 = lean_ctor_get(x_28, 0); -x_31 = lean_ctor_get(x_28, 1); -x_32 = l_Lean_Meta_Grind_ppENodeDecl___closed__4; -lean_ctor_set_tag(x_28, 5); -lean_ctor_set(x_28, 1, x_30); -lean_ctor_set(x_28, 0, x_32); -x_33 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_33, 0, x_28); -lean_ctor_set(x_33, 1, x_18); -x_34 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_34, 0, x_22); -lean_ctor_set(x_34, 1, x_33); -x_35 = lean_box(0); -x_36 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_18, x_24, x_34, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_31); -lean_dec(x_24); -lean_dec(x_1); -return x_36; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4; +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_26); +x_30 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_14); +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_19); +lean_ctor_set(x_31, 1, x_30); +x_32 = lean_box(0); +x_33 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4(x_1, x_2, x_14, x_21, x_31, x_32, x_3, x_4, x_5, x_6, x_27); +lean_dec(x_21); +lean_dec(x_2); +return x_33; } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_37 = lean_ctor_get(x_28, 0); -x_38 = lean_ctor_get(x_28, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_28); -x_39 = l_Lean_Meta_Grind_ppENodeDecl___closed__4; -x_40 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_37); -x_41 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_18); -x_42 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_42, 0, x_22); -lean_ctor_set(x_42, 1, x_41); -x_43 = lean_box(0); -x_44 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_18, x_24, x_42, x_43, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_38); -lean_dec(x_24); +uint8_t x_34; +lean_dec(x_21); +lean_dec(x_19); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -return x_44; +x_34 = !lean_is_exclusive(x_25); +if (x_34 == 0) +{ +return x_25; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_25, 0); +x_36 = lean_ctor_get(x_25, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_25); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} } } else { -lean_object* x_45; lean_object* x_46; -lean_dec(x_26); -x_45 = lean_box(0); -x_46 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_18, x_24, x_22, x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -lean_dec(x_24); -lean_dec(x_1); -return x_46; +lean_object* x_38; lean_object* x_39; +lean_dec(x_23); +x_38 = lean_box(0); +x_39 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4(x_1, x_2, x_14, x_21, x_19, x_38, x_3, x_4, x_5, x_6, x_22); +lean_dec(x_21); +lean_dec(x_2); +return x_39; } } else { -uint8_t x_47; -lean_dec(x_22); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +uint8_t x_40; +lean_dec(x_19); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_47 = !lean_is_exclusive(x_23); -if (x_47 == 0) +x_40 = !lean_is_exclusive(x_20); +if (x_40 == 0) { -return x_23; +return x_20; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_23, 0); -x_49 = lean_ctor_get(x_23, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_23); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_20, 0); +x_42 = lean_ctor_get(x_20, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_20); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -uint8_t x_51; -lean_free_object(x_11); -lean_dec(x_13); +uint8_t x_44; lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_51 = !lean_is_exclusive(x_15); -if (x_51 == 0) +x_44 = !lean_is_exclusive(x_11); +if (x_44 == 0) { -return x_15; -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_15, 0); -x_53 = lean_ctor_get(x_15, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_15); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; -} -} +return x_11; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_11, 0); -x_56 = lean_ctor_get(x_11, 1); -lean_inc(x_56); -lean_inc(x_55); +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_11, 0); +x_46 = lean_ctor_get(x_11, 1); +lean_inc(x_46); +lean_inc(x_45); lean_dec(x_11); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_1); -x_57 = l_Lean_Meta_Grind_ppENodeDeclValue(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_56); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -x_60 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -x_61 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_55); -x_62 = l_Lean_Meta_Grind_ppENodeDecl___closed__2; -x_63 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_63, 0, x_61); -lean_ctor_set(x_63, 1, x_62); -x_64 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_64, 0, x_63); -lean_ctor_set(x_64, 1, x_58); -x_65 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_60); -lean_inc(x_1); -x_66 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_59); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_ctor_get(x_67, 2); -lean_inc(x_69); -x_70 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_69); -if (x_70 == 0) -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_71 = l_Lean_Meta_Grind_ppENodeRef(x_69, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_68); -lean_dec(x_69); -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_74 = x_71; -} else { - lean_dec_ref(x_71); - x_74 = lean_box(0); -} -x_75 = l_Lean_Meta_Grind_ppENodeDecl___closed__4; -if (lean_is_scalar(x_74)) { - x_76 = lean_alloc_ctor(5, 2, 0); -} else { - x_76 = x_74; - lean_ctor_set_tag(x_76, 5); -} -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_72); -x_77 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_60); -x_78 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_78, 0, x_65); -lean_ctor_set(x_78, 1, x_77); -x_79 = lean_box(0); -x_80 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_60, x_67, x_78, x_79, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_73); -lean_dec(x_67); -lean_dec(x_1); -return x_80; +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } -else -{ -lean_object* x_81; lean_object* x_82; -lean_dec(x_69); -x_81 = lean_box(0); -x_82 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_60, x_67, x_65, x_81, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_68); -lean_dec(x_67); -lean_dec(x_1); -return x_82; } } else { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -lean_dec(x_65); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +uint8_t x_48; lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_83 = lean_ctor_get(x_66, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_66, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_85 = x_66; -} else { - lean_dec_ref(x_66); - x_85 = lean_box(0); +x_48 = !lean_is_exclusive(x_8); +if (x_48 == 0) +{ +return x_8; } -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(1, 2, 0); -} else { - x_86 = x_85; +else +{ +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_8, 0); +x_50 = lean_ctor_get(x_8, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_8); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; } -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_84); -return x_86; } } -else +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; -lean_dec(x_55); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_8; +x_8 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_87 = lean_ctor_get(x_57, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_57, 1); -lean_inc(x_88); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_89 = x_57; -} else { - lean_dec_ref(x_57); - x_89 = lean_box(0); -} -if (lean_is_scalar(x_89)) { - x_90 = lean_alloc_ctor(1, 2, 0); -} else { - x_90 = x_89; -} -lean_ctor_set(x_90, 0, x_87); -lean_ctor_set(x_90, 1, x_88); -return x_90; +return x_8; } } +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_2); +return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l_Lean_Meta_Grind_ppENodeDecl___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +x_12 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_14; -x_14 = l_Lean_Meta_Grind_ppENodeDecl___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); lean_dec(x_4); -lean_dec(x_1); -return x_14; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -x_15 = l_Lean_Meta_Grind_ppENodeDecl___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_1); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppENodeDecl___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -x_15 = l_Lean_Meta_Grind_ppENodeDecl___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_1); -return x_15; +lean_dec(x_2); +return x_12; } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1() { _start: { lean_object* x_1; @@ -1359,176 +1466,258 @@ x_1 = lean_mk_string_unchecked("\n", 1, 1); return x_1; } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1; +x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3() { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_5, x_4); -if (x_16 == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_17; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_6, x_5); +if (x_13 == 0) +{ +lean_object* x_14; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -lean_dec(x_7); -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_6); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_7); +lean_ctor_set(x_14, 1, x_12); +return x_14; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_array_uget(x_3, x_5); -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -lean_dec(x_18); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_array_uget(x_4, x_6); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_20 = l_Lean_Meta_Grind_ppENodeDecl(x_19, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_20) == 0) +lean_inc(x_1); +x_17 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl(x_1, x_16, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_17) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; size_t x_26; size_t x_27; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -x_23 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2; -x_24 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_24, 0, x_6); -lean_ctor_set(x_24, 1, x_23); -x_25 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_21); -x_26 = 1; -x_27 = lean_usize_add(x_5, x_26); -x_5 = x_27; -x_6 = x_25; -x_15 = x_22; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; size_t x_23; size_t x_24; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3; +x_21 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_21, 0, x_7); +lean_ctor_set(x_21, 1, x_20); +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_18); +x_23 = 1; +x_24 = lean_usize_add(x_6, x_23); +x_6 = x_24; +x_7 = x_22; +x_12 = x_19; goto _start; } else { -uint8_t x_29; -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); +uint8_t x_26; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -x_29 = !lean_is_exclusive(x_20); -if (x_29 == 0) +lean_dec(x_1); +x_26 = !lean_is_exclusive(x_17); +if (x_26 == 0) { -return x_20; +return x_17; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_20, 0); -x_31 = lean_ctor_get(x_20, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_20); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_17, 0); +x_28 = lean_ctor_get(x_17, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_17); +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_Goal_ppState___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -if (lean_obj_tag(x_1) == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_12; lean_object* x_13; -x_12 = l_List_reverse___rarg(x_2); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -return x_13; +lean_object* x_9; lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_1); +x_9 = l_List_reverse___rarg(x_3); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_8); +return x_10; } else { -uint8_t x_14; -x_14 = !lean_is_exclusive(x_1); -if (x_14 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_1, 0); -x_16 = lean_ctor_get(x_1, 1); -x_17 = l_Lean_Meta_Grind_ppENodeRef(x_15, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_15); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -lean_ctor_set(x_1, 1, x_2); -lean_ctor_set(x_1, 0, x_18); +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_ctor_get(x_2, 1); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_14 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_12, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) { -lean_object* _tmp_0 = x_16; -lean_object* _tmp_1 = x_1; -lean_object* _tmp_10 = x_19; -x_1 = _tmp_0; +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +lean_ctor_set(x_2, 1, x_3); +lean_ctor_set(x_2, 0, x_15); +{ +lean_object* _tmp_1 = x_13; +lean_object* _tmp_2 = x_2; +lean_object* _tmp_7 = x_16; x_2 = _tmp_1; -x_11 = _tmp_10; +x_3 = _tmp_2; +x_8 = _tmp_7; } goto _start; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_21 = lean_ctor_get(x_1, 0); -x_22 = lean_ctor_get(x_1, 1); -lean_inc(x_22); -lean_inc(x_21); +uint8_t x_18; +lean_free_object(x_2); +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); lean_dec(x_1); -x_23 = l_Lean_Meta_Grind_ppENodeRef(x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_21); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) +{ +return x_14; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_14, 0); +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_14); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_2, 0); +x_23 = lean_ctor_get(x_2, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_2); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_1); +x_24 = l_Lean_Meta_Grind_Goal_ppENodeRef(x_1, x_22, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_2); -x_1 = x_22; -x_2 = x_26; -x_11 = x_25; +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_3); +x_2 = x_23; +x_3 = x_27; +x_8 = x_26; goto _start; } +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +lean_dec(x_23); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_29 = lean_ctor_get(x_24, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_24)) { + lean_ctor_release(x_24, 0); + lean_ctor_release(x_24, 1); + x_31 = x_24; +} else { + lean_dec_ref(x_24); + x_31 = lean_box(0); +} +if (lean_is_scalar(x_31)) { + x_32 = lean_alloc_ctor(1, 2, 0); +} else { + x_32 = x_31; +} +lean_ctor_set(x_32, 0, x_29); +lean_ctor_set(x_32, 1, x_30); +return x_32; } } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1() { +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1() { _start: { lean_object* x_1; @@ -1536,17 +1725,26 @@ x_1 = lean_mk_string_unchecked("{", 1, 1); return x_1; } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2() { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3() { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4() { _start: { lean_object* x_1; @@ -1554,17 +1752,26 @@ x_1 = lean_mk_string_unchecked(", ", 2, 2); return x_1; } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4() { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5() { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7() { _start: { lean_object* x_1; @@ -1572,186 +1779,234 @@ x_1 = lean_mk_string_unchecked("}", 1, 1); return x_1; } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6() { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9() { _start: { -if (lean_obj_tag(x_4) == 0) +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_16; -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_5); -lean_ctor_set(x_16, 1, x_15); -return x_16; +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_13; +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_6); +lean_ctor_set(x_13, 1, x_12); +return x_13; } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_4); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_18 = lean_ctor_get(x_4, 0); -x_19 = lean_ctor_get(x_4, 1); -x_20 = lean_unsigned_to_nat(0u); -x_21 = l_List_lengthTRAux___rarg(x_18, x_20); -x_22 = lean_unsigned_to_nat(1u); -x_23 = lean_nat_dec_lt(x_22, x_21); -lean_dec(x_21); -if (x_23 == 0) +uint8_t x_14; +x_14 = !lean_is_exclusive(x_5); +if (x_14 == 0) { -lean_free_object(x_4); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_15 = lean_ctor_get(x_5, 0); +x_16 = lean_ctor_get(x_5, 1); +x_17 = lean_unsigned_to_nat(0u); +x_18 = l_List_lengthTRAux___rarg(x_15, x_17); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_dec_lt(x_19, x_18); lean_dec(x_18); -x_4 = x_19; -x_6 = lean_box(0); +if (x_20 == 0) +{ +lean_free_object(x_5); +lean_dec(x_15); +x_5 = x_16; +x_7 = lean_box(0); goto _start; } else { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_25 = lean_box(0); -x_26 = l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2(x_18, x_25, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -x_27 = !lean_is_exclusive(x_26); -if (x_27 == 0) -{ -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_28 = lean_ctor_get(x_26, 0); -x_29 = lean_ctor_get(x_26, 1); -x_30 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2; -lean_ctor_set_tag(x_26, 5); -lean_ctor_set(x_26, 1, x_30); -lean_ctor_set(x_26, 0, x_5); -x_31 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2; -lean_ctor_set_tag(x_4, 5); -lean_ctor_set(x_4, 1, x_31); -lean_ctor_set(x_4, 0, x_26); -x_32 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4; -x_33 = l_Std_Format_joinSep___at_Prod_repr___spec__1(x_28, x_32); -x_34 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_34, 0, x_4); -lean_ctor_set(x_34, 1, x_33); -x_35 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6; -x_36 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -x_4 = x_19; -x_5 = x_36; -x_6 = lean_box(0); -x_15 = x_29; +lean_object* x_22; lean_object* x_23; +x_22 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_1); +x_23 = l_List_mapM_loop___at_Lean_Meta_Grind_Goal_ppState___spec__2(x_1, x_15, x_22, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3; +lean_ctor_set_tag(x_5, 7); +lean_ctor_set(x_5, 1, x_26); +lean_ctor_set(x_5, 0, x_6); +x_27 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_5); +lean_ctor_set(x_28, 1, x_27); +x_29 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6; +x_30 = l_Lean_MessageData_joinSep(x_24, x_29); +x_31 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_31, 0, x_28); +lean_ctor_set(x_31, 1, x_30); +x_32 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +x_5 = x_16; +x_6 = x_33; +x_7 = lean_box(0); +x_12 = x_25; goto _start; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_38 = lean_ctor_get(x_26, 0); -x_39 = lean_ctor_get(x_26, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_26); -x_40 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2; -x_41 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_41, 0, x_5); -lean_ctor_set(x_41, 1, x_40); -x_42 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2; -lean_ctor_set_tag(x_4, 5); -lean_ctor_set(x_4, 1, x_42); -lean_ctor_set(x_4, 0, x_41); -x_43 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4; -x_44 = l_Std_Format_joinSep___at_Prod_repr___spec__1(x_38, x_43); -x_45 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_45, 0, x_4); -lean_ctor_set(x_45, 1, x_44); -x_46 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6; -x_47 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -x_4 = x_19; -x_5 = x_47; -x_6 = lean_box(0); -x_15 = x_39; -goto _start; +uint8_t x_35; +lean_free_object(x_5); +lean_dec(x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_35 = !lean_is_exclusive(x_23); +if (x_35 == 0) +{ +return x_23; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_23, 0); +x_37 = lean_ctor_get(x_23, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_23); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } } else { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_49 = lean_ctor_get(x_4, 0); -x_50 = lean_ctor_get(x_4, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_4); -x_51 = lean_unsigned_to_nat(0u); -x_52 = l_List_lengthTRAux___rarg(x_49, x_51); -x_53 = lean_unsigned_to_nat(1u); -x_54 = lean_nat_dec_lt(x_53, x_52); -lean_dec(x_52); -if (x_54 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_39 = lean_ctor_get(x_5, 0); +x_40 = lean_ctor_get(x_5, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_5); +x_41 = lean_unsigned_to_nat(0u); +x_42 = l_List_lengthTRAux___rarg(x_39, x_41); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_dec_lt(x_43, x_42); +lean_dec(x_42); +if (x_44 == 0) +{ +lean_dec(x_39); +x_5 = x_40; +x_7 = lean_box(0); +goto _start; +} +else { -lean_dec(x_49); -x_4 = x_50; -x_6 = lean_box(0); +lean_object* x_46; lean_object* x_47; +x_46 = lean_box(0); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_1); +x_47 = l_List_mapM_loop___at_Lean_Meta_Grind_Goal_ppState___spec__2(x_1, x_39, x_46, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_47) == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_47, 1); +lean_inc(x_49); +lean_dec(x_47); +x_50 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3; +x_51 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_51, 0, x_6); +lean_ctor_set(x_51, 1, x_50); +x_52 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +x_53 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +x_54 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6; +x_55 = l_Lean_MessageData_joinSep(x_48, x_54); +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_53); +lean_ctor_set(x_56, 1, x_55); +x_57 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +x_58 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_58, 0, x_56); +lean_ctor_set(x_58, 1, x_57); +x_5 = x_40; +x_6 = x_58; +x_7 = lean_box(0); +x_12 = x_49; goto _start; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_56 = lean_box(0); -x_57 = l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2(x_49, x_56, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_60 = x_57; +lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; +lean_dec(x_40); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_6); +lean_dec(x_1); +x_60 = lean_ctor_get(x_47, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_47, 1); +lean_inc(x_61); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + lean_ctor_release(x_47, 1); + x_62 = x_47; } else { - lean_dec_ref(x_57); - x_60 = lean_box(0); + lean_dec_ref(x_47); + x_62 = lean_box(0); } -x_61 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2; -if (lean_is_scalar(x_60)) { - x_62 = lean_alloc_ctor(5, 2, 0); +if (lean_is_scalar(x_62)) { + x_63 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_60; - lean_ctor_set_tag(x_62, 5); -} -lean_ctor_set(x_62, 0, x_5); -lean_ctor_set(x_62, 1, x_61); -x_63 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2; -x_64 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -x_65 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4; -x_66 = l_Std_Format_joinSep___at_Prod_repr___spec__1(x_58, x_65); -x_67 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_67, 0, x_64); -lean_ctor_set(x_67, 1, x_66); -x_68 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6; -x_69 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -x_4 = x_50; -x_5 = x_69; -x_6 = lean_box(0); -x_15 = x_59; -goto _start; + x_63 = x_62; +} +lean_ctor_set(x_63, 0, x_60); +lean_ctor_set(x_63, 1, x_61); +return x_63; +} } } } } } -static lean_object* _init_l_Lean_Meta_Grind_ppState___closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppState___closed__1() { _start: { lean_object* x_1; @@ -1759,619 +2014,3460 @@ x_1 = lean_mk_string_unchecked("Goal:", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_ppState___closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_Goal_ppState___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_ppState___closed__1; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); +x_1 = l_Lean_Meta_Grind_Goal_ppState___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppState(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_ppState(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; size_t x_14; size_t x_15; lean_object* x_16; lean_object* x_17; -x_10 = l_Lean_Meta_Grind_getENodes(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_box(0); -x_14 = lean_array_size(x_11); -x_15 = 0; -x_16 = l_Lean_Meta_Grind_ppState___closed__2; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); +lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; +x_7 = l_Lean_Meta_Grind_Goal_getENodes(x_1); +x_8 = lean_box(0); +x_9 = lean_array_size(x_7); +x_10 = 0; +x_11 = l_Lean_Meta_Grind_Goal_ppState___closed__2; lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); lean_inc(x_2); lean_inc(x_1); -x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1(x_11, x_13, x_11, x_14, x_15, x_16, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_12); -lean_dec(x_11); -if (lean_obj_tag(x_17) == 0) +x_12 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1(x_1, x_7, x_8, x_7, x_9, x_10, x_11, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_7); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_ctor_get(x_17, 1); -lean_inc(x_19); -lean_dec(x_17); -x_20 = l_Lean_Meta_Grind_getEqcs(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_19); -if (lean_obj_tag(x_20) == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +lean_inc(x_1); +x_15 = l_Lean_Meta_Grind_Goal_getEqcs(x_1); +lean_inc(x_15); +x_16 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3(x_1, x_15, x_8, x_15, x_15, x_13, lean_box(0), x_2, x_3, x_4, x_5, x_14); +lean_dec(x_15); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); -lean_inc(x_22); -lean_dec(x_20); -lean_inc(x_21); -x_23 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3(x_21, x_13, x_21, x_21, x_18, lean_box(0), x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_22); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -lean_dec(x_21); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +uint8_t x_17; +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) { -return x_23; +return x_16; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_23); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_25); -lean_ctor_set(x_27, 1, x_26); -return x_27; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_16, 0); +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_16); +x_20 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; } } else { -uint8_t x_28; -lean_dec(x_18); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_28 = !lean_is_exclusive(x_20); -if (x_28 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_16); +if (x_21 == 0) { -return x_20; +return x_16; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_20, 0); -x_30 = lean_ctor_get(x_20, 1); -lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_20); -x_31 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_31, 0, x_29); -lean_ctor_set(x_31, 1, x_30); -return x_31; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_16, 0); +x_23 = lean_ctor_get(x_16, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_16); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } else { -uint8_t x_32; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +uint8_t x_25; lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_32 = !lean_is_exclusive(x_17); -if (x_32 == 0) +x_25 = !lean_is_exclusive(x_12); +if (x_25 == 0) { -return x_17; +return x_12; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_17, 0); -x_34 = lean_ctor_get(x_17, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_17); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_12, 0); +x_27 = lean_ctor_get(x_12, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_12); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_17 = lean_unbox_usize(x_5); +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_5); lean_dec(x_5); -x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1(x_1, x_2, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); +x_14 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -return x_18; +return x_15; } } -LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_12; -x_12 = l_List_mapM_loop___at_Lean_Meta_Grind_ppState___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_object* x_13; +x_13 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_4); lean_dec(x_3); -return x_12; +lean_dec(x_2); +return x_13; } } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1() { _start: { -lean_object* x_16; -x_16 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(1); +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +if (lean_obj_tag(x_4) == 0) +{ +lean_object* x_12; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_16; -} +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_5); +lean_ctor_set(x_12, 1, x_11); +return x_12; } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_mk_ref(x_1, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +uint8_t x_13; +x_13 = !lean_is_exclusive(x_4); +if (x_13 == 0) { -return x_10; +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_4, 0); +x_15 = lean_ctor_get(x_4, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_16 = l_Lean_Meta_Grind_Goal_ppState(x_14, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; +lean_ctor_set_tag(x_4, 7); +lean_ctor_set(x_4, 1, x_19); +lean_ctor_set(x_4, 0, x_5); +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_4); +lean_ctor_set(x_20, 1, x_17); +x_4 = x_15; +x_5 = x_20; +x_6 = lean_box(0); +x_11 = x_18; +goto _start; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_inc(x_12); +uint8_t x_22; +lean_free_object(x_4); +lean_dec(x_15); lean_dec(x_10); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) +{ +return x_16; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_16, 0); +x_24 = lean_ctor_get(x_16, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_16); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; +} +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_4, 0); +x_27 = lean_ctor_get(x_4, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_4); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_28 = l_Lean_Meta_Grind_Goal_ppState(x_26, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; +x_32 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_32, 0, x_5); +lean_ctor_set(x_32, 1, x_31); +x_33 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_29); +x_4 = x_27; +x_5 = x_33; +x_6 = lean_box(0); +x_11 = x_30; +goto _start; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_dec(x_27); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +x_35 = lean_ctor_get(x_28, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_28, 1); +lean_inc(x_36); +if (lean_is_exclusive(x_28)) { + lean_ctor_release(x_28, 0); + lean_ctor_release(x_28, 1); + x_37 = x_28; +} else { + lean_dec_ref(x_28); + x_37 = lean_box(0); +} +if (lean_is_scalar(x_37)) { + x_38 = lean_alloc_ctor(1, 2, 0); +} else { + x_38 = x_37; +} +lean_ctor_set(x_38, 0, x_35); +lean_ctor_set(x_38, 1, x_36); +return x_38; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppGoals(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_box(0); +x_8 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +lean_inc(x_1); +x_9 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(x_1, x_7, x_1, x_1, x_8, lean_box(0), x_2, x_3, x_4, x_5, x_6); +lean_dec(x_1); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +return x_9; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_ctor_get(x_9, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_9); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_12); +return x_13; +} +} +else +{ +uint8_t x_14; +x_14 = !lean_is_exclusive(x_9); +if (x_14 == 0) +{ +return x_9; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_9, 0); +x_16 = lean_ctor_get(x_9, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_9); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_12; +} +} +static double _init_l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +_start: +{ +uint8_t x_5; +x_5 = lean_usize_dec_lt(x_3, x_2); +if (x_5 == 0) +{ +lean_dec(x_1); +return x_4; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; double x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; size_t x_19; size_t x_20; lean_object* x_21; +x_6 = lean_array_uget(x_4, x_3); +x_7 = lean_unsigned_to_nat(0u); +x_8 = lean_array_uset(x_4, x_3, x_7); +x_9 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_10 = 1; +x_11 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +lean_inc(x_1); +x_12 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); +lean_ctor_set_float(x_12, sizeof(void*)*2, x_9); +lean_ctor_set_float(x_12, sizeof(void*)*2 + 8, x_9); +lean_ctor_set_uint8(x_12, sizeof(void*)*2 + 16, x_10); +x_13 = l_Lean_MessageData_ofExpr(x_6); +x_14 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_15 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_18 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_18, 0, x_12); +lean_ctor_set(x_18, 1, x_16); +lean_ctor_set(x_18, 2, x_17); +x_19 = 1; +x_20 = lean_usize_add(x_3, x_19); +x_21 = lean_array_uset(x_8, x_3, x_18); +x_3 = x_20; +x_4 = x_21; +goto _start; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; double x_8; uint8_t x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_5 = lean_array_size(x_3); +x_6 = 0; +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1(x_4, x_5, x_6, x_3); +x_8 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_9 = 1; +x_10 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_11 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_11, 0, x_1); +lean_ctor_set(x_11, 1, x_10); +lean_ctor_set_float(x_11, sizeof(void*)*2, x_8); +lean_ctor_set_float(x_11, sizeof(void*)*2 + 8, x_8); +lean_ctor_set_uint8(x_11, sizeof(void*)*2 + 16, x_9); +x_12 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_12, 0, x_2); +x_13 = l_Lean_MessageData_ofFormat(x_12); +x_14 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_14, 0, x_11); lean_ctor_set(x_14, 1, x_13); +lean_ctor_set(x_14, 2, x_7); return x_14; } } +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +size_t x_5; size_t x_6; lean_object* x_7; +x_5 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_6 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1(x_1, x_5, x_6, x_4); +return x_7; +} } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_10; -lean_inc(x_1); -x_10 = l_Lean_Meta_Grind_ppState(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_10) == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = lean_ctor_get(x_10, 0); +lean_object* x_3; +x_3 = l_List_reverse___rarg(x_2); +return x_3; +} +else +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +x_7 = l_Lean_Expr_isFalse(x_5); +if (x_7 == 0) +{ +lean_ctor_set(x_1, 1, x_2); +{ +lean_object* _tmp_0 = x_6; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; +} +goto _start; +} +else +{ +lean_free_object(x_1); +lean_dec(x_5); +x_1 = x_6; +goto _start; +} +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_ctor_get(x_1, 1); lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = lean_st_ref_get(x_1, x_12); +lean_inc(x_10); lean_dec(x_1); -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) +lean_inc(x_10); +x_12 = l_Lean_Expr_isFalse(x_10); +if (x_12 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_11); -lean_ctor_set(x_16, 1, x_15); -lean_ctor_set(x_13, 0, x_16); -return x_13; +lean_object* x_13; +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_10); +lean_ctor_set(x_13, 1, x_2); +x_1 = x_11; +x_2 = x_13; +goto _start; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_13, 0); -x_18 = lean_ctor_get(x_13, 1); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_13); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_11); -lean_ctor_set(x_19, 1, x_17); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_18); -return x_20; +lean_dec(x_10); +x_1 = x_11; +goto _start; } } +} +} +} +LEAN_EXPORT lean_object* l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_object* x_3; +x_3 = l_List_reverse___rarg(x_2); +return x_3; +} else { -uint8_t x_21; +uint8_t x_4; +x_4 = !lean_is_exclusive(x_1); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_ctor_get(x_1, 0); +x_6 = lean_ctor_get(x_1, 1); +lean_inc(x_5); +x_7 = l_Lean_Expr_isTrue(x_5); +if (x_7 == 0) +{ +lean_ctor_set(x_1, 1, x_2); +{ +lean_object* _tmp_0 = x_6; +lean_object* _tmp_1 = x_1; +x_1 = _tmp_0; +x_2 = _tmp_1; +} +goto _start; +} +else +{ +lean_free_object(x_1); +lean_dec(x_5); +x_1 = x_6; +goto _start; +} +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_1, 0); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_1); +lean_inc(x_10); +x_12 = l_Lean_Expr_isTrue(x_10); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_10); +lean_ctor_set(x_13, 1, x_2); +x_1 = x_11; +x_2 = x_13; +goto _start; +} +else +{ +lean_dec(x_10); +x_1 = x_11; +goto _start; +} +} +} +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Expr_isTrue___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Expr_isFalse___boxed), 1, 0); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("eqc", 3, 3); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5() { +_start: +{ +lean_object* x_1; double x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_3 = 1; +x_4 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_5 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +lean_ctor_set_float(x_5, sizeof(void*)*2, x_2); +lean_ctor_set_float(x_5, sizeof(void*)*2 + 8, x_2); +lean_ctor_set_uint8(x_5, sizeof(void*)*2 + 16, x_3); +return x_5; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(",", 1, 1); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8; +x_2 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; +x_3 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("prop", 4, 4); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("False propositions", 18, 18); +return x_1; +} +} +static lean_object* _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("True propositions", 17, 17); +return x_1; +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_14; +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_7); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_22; +x_15 = lean_ctor_get(x_6, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_6, 1); +lean_inc(x_16); +lean_dec(x_6); +x_22 = !lean_is_exclusive(x_7); +if (x_22 == 0) +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_ctor_get(x_7, 1); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_7, 0); +x_26 = lean_ctor_get(x_23, 0); +x_27 = lean_ctor_get(x_23, 1); +x_28 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1; +lean_inc(x_15); +x_29 = l_List_find_x3f___rarg(x_28, x_15); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2; +lean_inc(x_15); +x_31 = l_List_find_x3f___rarg(x_30, x_15); +if (lean_obj_tag(x_31) == 0) +{ +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_32; +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_7); +x_17 = x_32; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_33; +x_33 = lean_ctor_get(x_15, 1); +lean_inc(x_33); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; +lean_dec(x_15); +x_34 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_34, 0, x_7); +x_17 = x_34; +x_18 = x_13; +goto block_21; +} +else +{ +uint8_t x_35; +x_35 = !lean_is_exclusive(x_33); +if (x_35 == 0) +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_33, 1); +lean_dec(x_36); +x_37 = lean_ctor_get(x_33, 0); +lean_dec(x_37); +x_38 = lean_ctor_get(x_15, 0); +lean_inc(x_38); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_39 = l_Lean_Meta_isProof(x_38, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_39) == 0) +{ +lean_object* x_40; uint8_t x_41; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_unbox(x_40); +lean_dec(x_40); +if (x_41 == 0) +{ +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = lean_ctor_get(x_39, 1); +lean_inc(x_42); +lean_dec(x_39); +lean_inc(x_1); +lean_inc(x_15); +x_43 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_15, x_1); +x_44 = !lean_is_exclusive(x_15); +if (x_44 == 0) +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_45 = lean_ctor_get(x_15, 1); +lean_dec(x_45); +x_46 = lean_ctor_get(x_15, 0); +lean_dec(x_46); +x_47 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +x_48 = l_Lean_MessageData_joinSep(x_43, x_47); +x_49 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +lean_ctor_set_tag(x_33, 7); +lean_ctor_set(x_33, 1, x_48); +lean_ctor_set(x_33, 0, x_49); +x_50 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_50); +lean_ctor_set(x_15, 0, x_33); +x_51 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_51, 0, x_15); +x_52 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +lean_inc(x_2); +x_53 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +lean_ctor_set(x_53, 2, x_2); +x_54 = lean_array_push(x_26, x_53); +lean_ctor_set(x_23, 0, x_54); +x_55 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_55, 0, x_7); +x_17 = x_55; +x_18 = x_42; +goto block_21; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_15); +x_56 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +x_57 = l_Lean_MessageData_joinSep(x_43, x_56); +x_58 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +lean_ctor_set_tag(x_33, 7); +lean_ctor_set(x_33, 1, x_57); +lean_ctor_set(x_33, 0, x_58); +x_59 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +x_60 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_60, 0, x_33); +lean_ctor_set(x_60, 1, x_59); +x_61 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_61, 0, x_60); +x_62 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +lean_inc(x_2); +x_63 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_63, 0, x_62); +lean_ctor_set(x_63, 1, x_61); +lean_ctor_set(x_63, 2, x_2); +x_64 = lean_array_push(x_26, x_63); +lean_ctor_set(x_23, 0, x_64); +x_65 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_65, 0, x_7); +x_17 = x_65; +x_18 = x_42; +goto block_21; +} +} +else +{ +lean_object* x_66; lean_object* x_67; +lean_free_object(x_33); +lean_dec(x_15); +x_66 = lean_ctor_get(x_39, 1); +lean_inc(x_66); +lean_dec(x_39); +x_67 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_67, 0, x_7); +x_17 = x_67; +x_18 = x_66; +goto block_21; +} +} +else +{ +uint8_t x_68; +lean_free_object(x_33); +lean_free_object(x_23); +lean_dec(x_27); +lean_dec(x_26); +lean_free_object(x_7); +lean_dec(x_25); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_68 = !lean_is_exclusive(x_39); +if (x_68 == 0) +{ +return x_39; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_39, 0); +x_70 = lean_ctor_get(x_39, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_39); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; +} +} +} +else +{ +lean_object* x_72; lean_object* x_73; +lean_dec(x_33); +x_72 = lean_ctor_get(x_15, 0); +lean_inc(x_72); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_73 = l_Lean_Meta_isProof(x_72, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_73) == 0) +{ +lean_object* x_74; uint8_t x_75; +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_unbox(x_74); +lean_dec(x_74); +if (x_75 == 0) +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; +x_76 = lean_ctor_get(x_73, 1); +lean_inc(x_76); +lean_dec(x_73); +lean_inc(x_1); +lean_inc(x_15); +x_77 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_15, x_1); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + x_78 = x_15; +} else { + lean_dec_ref(x_15); + x_78 = lean_box(0); +} +x_79 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +x_80 = l_Lean_MessageData_joinSep(x_77, x_79); +x_81 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +x_82 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_82, 0, x_81); +lean_ctor_set(x_82, 1, x_80); +x_83 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +if (lean_is_scalar(x_78)) { + x_84 = lean_alloc_ctor(7, 2, 0); +} else { + x_84 = x_78; + lean_ctor_set_tag(x_84, 7); +} +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +x_85 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_85, 0, x_84); +x_86 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +lean_inc(x_2); +x_87 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_85); +lean_ctor_set(x_87, 2, x_2); +x_88 = lean_array_push(x_26, x_87); +lean_ctor_set(x_23, 0, x_88); +x_89 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_89, 0, x_7); +x_17 = x_89; +x_18 = x_76; +goto block_21; +} +else +{ +lean_object* x_90; lean_object* x_91; +lean_dec(x_15); +x_90 = lean_ctor_get(x_73, 1); +lean_inc(x_90); +lean_dec(x_73); +x_91 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_91, 0, x_7); +x_17 = x_91; +x_18 = x_90; +goto block_21; +} +} +else +{ +lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; +lean_free_object(x_23); +lean_dec(x_27); +lean_dec(x_26); +lean_free_object(x_7); +lean_dec(x_25); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_92 = lean_ctor_get(x_73, 0); +lean_inc(x_92); +x_93 = lean_ctor_get(x_73, 1); +lean_inc(x_93); +if (lean_is_exclusive(x_73)) { + lean_ctor_release(x_73, 0); + lean_ctor_release(x_73, 1); + x_94 = x_73; +} else { + lean_dec_ref(x_73); + x_94 = lean_box(0); +} +if (lean_is_scalar(x_94)) { + x_95 = lean_alloc_ctor(1, 2, 0); +} else { + x_95 = x_94; +} +lean_ctor_set(x_95, 0, x_92); +lean_ctor_set(x_95, 1, x_93); +return x_95; +} +} +} +} +} +else +{ +uint8_t x_96; +x_96 = !lean_is_exclusive(x_31); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; lean_object* x_99; uint8_t x_100; +x_97 = lean_ctor_get(x_31, 0); +lean_dec(x_97); +x_98 = lean_box(0); +x_99 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(x_15, x_98); +x_100 = l_List_isEmpty___rarg(x_99); +if (x_100 == 0) +{ +lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +lean_dec(x_25); +x_101 = lean_array_mk(x_99); +x_102 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_103 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12; +x_104 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_105 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_102, x_103, x_101, x_104); +lean_ctor_set(x_31, 0, x_105); +lean_ctor_set(x_7, 0, x_31); +x_106 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_106, 0, x_7); +x_17 = x_106; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_107; +lean_dec(x_99); +lean_free_object(x_31); +x_107 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_107, 0, x_7); +x_17 = x_107; +x_18 = x_13; +goto block_21; +} +} +else +{ +lean_object* x_108; lean_object* x_109; uint8_t x_110; +lean_dec(x_31); +x_108 = lean_box(0); +x_109 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(x_15, x_108); +x_110 = l_List_isEmpty___rarg(x_109); +if (x_110 == 0) +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +lean_dec(x_25); +x_111 = lean_array_mk(x_109); +x_112 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_113 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12; +x_114 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_115 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_112, x_113, x_111, x_114); +x_116 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_7, 0, x_116); +x_117 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_117, 0, x_7); +x_17 = x_117; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_118; +lean_dec(x_109); +x_118 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_118, 0, x_7); +x_17 = x_118; +x_18 = x_13; +goto block_21; +} +} +} +} +else +{ +uint8_t x_119; +x_119 = !lean_is_exclusive(x_29); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; +x_120 = lean_ctor_get(x_29, 0); +lean_dec(x_120); +x_121 = lean_box(0); +x_122 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(x_15, x_121); +x_123 = l_List_isEmpty___rarg(x_122); +if (x_123 == 0) +{ +lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; +lean_dec(x_27); +x_124 = lean_array_mk(x_122); +x_125 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_126 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13; +x_127 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_128 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_125, x_126, x_124, x_127); +lean_ctor_set(x_29, 0, x_128); +lean_ctor_set(x_23, 1, x_29); +x_129 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_129, 0, x_7); +x_17 = x_129; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_130; +lean_dec(x_122); +lean_free_object(x_29); +x_130 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_130, 0, x_7); +x_17 = x_130; +x_18 = x_13; +goto block_21; +} +} +else +{ +lean_object* x_131; lean_object* x_132; uint8_t x_133; +lean_dec(x_29); +x_131 = lean_box(0); +x_132 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(x_15, x_131); +x_133 = l_List_isEmpty___rarg(x_132); +if (x_133 == 0) +{ +lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; +lean_dec(x_27); +x_134 = lean_array_mk(x_132); +x_135 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_136 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13; +x_137 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_138 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_135, x_136, x_134, x_137); +x_139 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_139, 0, x_138); +lean_ctor_set(x_23, 1, x_139); +x_140 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_140, 0, x_7); +x_17 = x_140; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_141; +lean_dec(x_132); +x_141 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_141, 0, x_7); +x_17 = x_141; +x_18 = x_13; +goto block_21; +} +} +} +} +else +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_142 = lean_ctor_get(x_7, 0); +x_143 = lean_ctor_get(x_23, 0); +x_144 = lean_ctor_get(x_23, 1); +lean_inc(x_144); +lean_inc(x_143); +lean_dec(x_23); +x_145 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1; +lean_inc(x_15); +x_146 = l_List_find_x3f___rarg(x_145, x_15); +if (lean_obj_tag(x_146) == 0) +{ +lean_object* x_147; lean_object* x_148; +x_147 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2; +lean_inc(x_15); +x_148 = l_List_find_x3f___rarg(x_147, x_15); +if (lean_obj_tag(x_148) == 0) +{ +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_149; lean_object* x_150; +x_149 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_149, 0, x_143); +lean_ctor_set(x_149, 1, x_144); +lean_ctor_set(x_7, 1, x_149); +x_150 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_150, 0, x_7); +x_17 = x_150; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_151; +x_151 = lean_ctor_get(x_15, 1); +lean_inc(x_151); +if (lean_obj_tag(x_151) == 0) +{ +lean_object* x_152; lean_object* x_153; +lean_dec(x_15); +x_152 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_152, 0, x_143); +lean_ctor_set(x_152, 1, x_144); +lean_ctor_set(x_7, 1, x_152); +x_153 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_153, 0, x_7); +x_17 = x_153; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_154; lean_object* x_155; lean_object* x_156; +if (lean_is_exclusive(x_151)) { + lean_ctor_release(x_151, 0); + lean_ctor_release(x_151, 1); + x_154 = x_151; +} else { + lean_dec_ref(x_151); + x_154 = lean_box(0); +} +x_155 = lean_ctor_get(x_15, 0); +lean_inc(x_155); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_156 = l_Lean_Meta_isProof(x_155, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_156) == 0) +{ +lean_object* x_157; uint8_t x_158; +x_157 = lean_ctor_get(x_156, 0); +lean_inc(x_157); +x_158 = lean_unbox(x_157); +lean_dec(x_157); +if (x_158 == 0) +{ +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; +x_159 = lean_ctor_get(x_156, 1); +lean_inc(x_159); +lean_dec(x_156); +lean_inc(x_1); +lean_inc(x_15); +x_160 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_15, x_1); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + x_161 = x_15; +} else { + lean_dec_ref(x_15); + x_161 = lean_box(0); +} +x_162 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +x_163 = l_Lean_MessageData_joinSep(x_160, x_162); +x_164 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +if (lean_is_scalar(x_154)) { + x_165 = lean_alloc_ctor(7, 2, 0); +} else { + x_165 = x_154; + lean_ctor_set_tag(x_165, 7); +} +lean_ctor_set(x_165, 0, x_164); +lean_ctor_set(x_165, 1, x_163); +x_166 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +if (lean_is_scalar(x_161)) { + x_167 = lean_alloc_ctor(7, 2, 0); +} else { + x_167 = x_161; + lean_ctor_set_tag(x_167, 7); +} +lean_ctor_set(x_167, 0, x_165); +lean_ctor_set(x_167, 1, x_166); +x_168 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_168, 0, x_167); +x_169 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +lean_inc(x_2); +x_170 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_170, 0, x_169); +lean_ctor_set(x_170, 1, x_168); +lean_ctor_set(x_170, 2, x_2); +x_171 = lean_array_push(x_143, x_170); +x_172 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_172, 0, x_171); +lean_ctor_set(x_172, 1, x_144); +lean_ctor_set(x_7, 1, x_172); +x_173 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_173, 0, x_7); +x_17 = x_173; +x_18 = x_159; +goto block_21; +} +else +{ +lean_object* x_174; lean_object* x_175; lean_object* x_176; +lean_dec(x_154); +lean_dec(x_15); +x_174 = lean_ctor_get(x_156, 1); +lean_inc(x_174); +lean_dec(x_156); +x_175 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_175, 0, x_143); +lean_ctor_set(x_175, 1, x_144); +lean_ctor_set(x_7, 1, x_175); +x_176 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_176, 0, x_7); +x_17 = x_176; +x_18 = x_174; +goto block_21; +} +} +else +{ +lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; +lean_dec(x_154); +lean_dec(x_144); +lean_dec(x_143); +lean_free_object(x_7); +lean_dec(x_142); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_177 = lean_ctor_get(x_156, 0); +lean_inc(x_177); +x_178 = lean_ctor_get(x_156, 1); +lean_inc(x_178); +if (lean_is_exclusive(x_156)) { + lean_ctor_release(x_156, 0); + lean_ctor_release(x_156, 1); + x_179 = x_156; +} else { + lean_dec_ref(x_156); + x_179 = lean_box(0); +} +if (lean_is_scalar(x_179)) { + x_180 = lean_alloc_ctor(1, 2, 0); +} else { + x_180 = x_179; +} +lean_ctor_set(x_180, 0, x_177); +lean_ctor_set(x_180, 1, x_178); +return x_180; +} +} +} +} +else +{ +lean_object* x_181; lean_object* x_182; lean_object* x_183; uint8_t x_184; +if (lean_is_exclusive(x_148)) { + lean_ctor_release(x_148, 0); + x_181 = x_148; +} else { + lean_dec_ref(x_148); + x_181 = lean_box(0); +} +x_182 = lean_box(0); +x_183 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(x_15, x_182); +x_184 = l_List_isEmpty___rarg(x_183); +if (x_184 == 0) +{ +lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_dec(x_142); +x_185 = lean_array_mk(x_183); +x_186 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_187 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12; +x_188 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_189 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_186, x_187, x_185, x_188); +if (lean_is_scalar(x_181)) { + x_190 = lean_alloc_ctor(1, 1, 0); +} else { + x_190 = x_181; +} +lean_ctor_set(x_190, 0, x_189); +x_191 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_191, 0, x_143); +lean_ctor_set(x_191, 1, x_144); +lean_ctor_set(x_7, 1, x_191); +lean_ctor_set(x_7, 0, x_190); +x_192 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_192, 0, x_7); +x_17 = x_192; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_193; lean_object* x_194; +lean_dec(x_183); +lean_dec(x_181); +x_193 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_193, 0, x_143); +lean_ctor_set(x_193, 1, x_144); +lean_ctor_set(x_7, 1, x_193); +x_194 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_194, 0, x_7); +x_17 = x_194; +x_18 = x_13; +goto block_21; +} +} +} +else +{ +lean_object* x_195; lean_object* x_196; lean_object* x_197; uint8_t x_198; +if (lean_is_exclusive(x_146)) { + lean_ctor_release(x_146, 0); + x_195 = x_146; +} else { + lean_dec_ref(x_146); + x_195 = lean_box(0); +} +x_196 = lean_box(0); +x_197 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(x_15, x_196); +x_198 = l_List_isEmpty___rarg(x_197); +if (x_198 == 0) +{ +lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; +lean_dec(x_144); +x_199 = lean_array_mk(x_197); +x_200 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_201 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13; +x_202 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_203 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_200, x_201, x_199, x_202); +if (lean_is_scalar(x_195)) { + x_204 = lean_alloc_ctor(1, 1, 0); +} else { + x_204 = x_195; +} +lean_ctor_set(x_204, 0, x_203); +x_205 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_205, 0, x_143); +lean_ctor_set(x_205, 1, x_204); +lean_ctor_set(x_7, 1, x_205); +x_206 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_206, 0, x_7); +x_17 = x_206; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_207; lean_object* x_208; +lean_dec(x_197); +lean_dec(x_195); +x_207 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_207, 0, x_143); +lean_ctor_set(x_207, 1, x_144); +lean_ctor_set(x_7, 1, x_207); +x_208 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_208, 0, x_7); +x_17 = x_208; +x_18 = x_13; +goto block_21; +} +} +} +} +else +{ +lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; +x_209 = lean_ctor_get(x_7, 1); +x_210 = lean_ctor_get(x_7, 0); +lean_inc(x_209); +lean_inc(x_210); +lean_dec(x_7); +x_211 = lean_ctor_get(x_209, 0); +lean_inc(x_211); +x_212 = lean_ctor_get(x_209, 1); +lean_inc(x_212); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_213 = x_209; +} else { + lean_dec_ref(x_209); + x_213 = lean_box(0); +} +x_214 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1; +lean_inc(x_15); +x_215 = l_List_find_x3f___rarg(x_214, x_15); +if (lean_obj_tag(x_215) == 0) +{ +lean_object* x_216; lean_object* x_217; +x_216 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2; +lean_inc(x_15); +x_217 = l_List_find_x3f___rarg(x_216, x_15); +if (lean_obj_tag(x_217) == 0) +{ +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_218; lean_object* x_219; lean_object* x_220; +if (lean_is_scalar(x_213)) { + x_218 = lean_alloc_ctor(0, 2, 0); +} else { + x_218 = x_213; +} +lean_ctor_set(x_218, 0, x_211); +lean_ctor_set(x_218, 1, x_212); +x_219 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_219, 0, x_210); +lean_ctor_set(x_219, 1, x_218); +x_220 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_220, 0, x_219); +x_17 = x_220; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_221; +x_221 = lean_ctor_get(x_15, 1); +lean_inc(x_221); +if (lean_obj_tag(x_221) == 0) +{ +lean_object* x_222; lean_object* x_223; lean_object* x_224; +lean_dec(x_15); +if (lean_is_scalar(x_213)) { + x_222 = lean_alloc_ctor(0, 2, 0); +} else { + x_222 = x_213; +} +lean_ctor_set(x_222, 0, x_211); +lean_ctor_set(x_222, 1, x_212); +x_223 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_223, 0, x_210); +lean_ctor_set(x_223, 1, x_222); +x_224 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_224, 0, x_223); +x_17 = x_224; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_225; lean_object* x_226; lean_object* x_227; +if (lean_is_exclusive(x_221)) { + lean_ctor_release(x_221, 0); + lean_ctor_release(x_221, 1); + x_225 = x_221; +} else { + lean_dec_ref(x_221); + x_225 = lean_box(0); +} +x_226 = lean_ctor_get(x_15, 0); +lean_inc(x_226); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +x_227 = l_Lean_Meta_isProof(x_226, x_9, x_10, x_11, x_12, x_13); +if (lean_obj_tag(x_227) == 0) +{ +lean_object* x_228; uint8_t x_229; +x_228 = lean_ctor_get(x_227, 0); +lean_inc(x_228); +x_229 = lean_unbox(x_228); +lean_dec(x_228); +if (x_229 == 0) +{ +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +x_230 = lean_ctor_get(x_227, 1); +lean_inc(x_230); +lean_dec(x_227); +lean_inc(x_1); +lean_inc(x_15); +x_231 = l_List_mapTR_loop___at_Lean_MessageData_instCoeListExpr___spec__1(x_15, x_1); +if (lean_is_exclusive(x_15)) { + lean_ctor_release(x_15, 0); + lean_ctor_release(x_15, 1); + x_232 = x_15; +} else { + lean_dec_ref(x_15); + x_232 = lean_box(0); +} +x_233 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9; +x_234 = l_Lean_MessageData_joinSep(x_231, x_233); +x_235 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3; +if (lean_is_scalar(x_225)) { + x_236 = lean_alloc_ctor(7, 2, 0); +} else { + x_236 = x_225; + lean_ctor_set_tag(x_236, 7); +} +lean_ctor_set(x_236, 0, x_235); +lean_ctor_set(x_236, 1, x_234); +x_237 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9; +if (lean_is_scalar(x_232)) { + x_238 = lean_alloc_ctor(7, 2, 0); +} else { + x_238 = x_232; + lean_ctor_set_tag(x_238, 7); +} +lean_ctor_set(x_238, 0, x_236); +lean_ctor_set(x_238, 1, x_237); +x_239 = lean_alloc_ctor(6, 1, 0); +lean_ctor_set(x_239, 0, x_238); +x_240 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +lean_inc(x_2); +x_241 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_241, 0, x_240); +lean_ctor_set(x_241, 1, x_239); +lean_ctor_set(x_241, 2, x_2); +x_242 = lean_array_push(x_211, x_241); +if (lean_is_scalar(x_213)) { + x_243 = lean_alloc_ctor(0, 2, 0); +} else { + x_243 = x_213; +} +lean_ctor_set(x_243, 0, x_242); +lean_ctor_set(x_243, 1, x_212); +x_244 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_244, 0, x_210); +lean_ctor_set(x_244, 1, x_243); +x_245 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_245, 0, x_244); +x_17 = x_245; +x_18 = x_230; +goto block_21; +} +else +{ +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_225); +lean_dec(x_15); +x_246 = lean_ctor_get(x_227, 1); +lean_inc(x_246); +lean_dec(x_227); +if (lean_is_scalar(x_213)) { + x_247 = lean_alloc_ctor(0, 2, 0); +} else { + x_247 = x_213; +} +lean_ctor_set(x_247, 0, x_211); +lean_ctor_set(x_247, 1, x_212); +x_248 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_248, 0, x_210); +lean_ctor_set(x_248, 1, x_247); +x_249 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_249, 0, x_248); +x_17 = x_249; +x_18 = x_246; +goto block_21; +} +} +else +{ +lean_object* x_250; lean_object* x_251; lean_object* x_252; lean_object* x_253; +lean_dec(x_225); +lean_dec(x_213); +lean_dec(x_212); +lean_dec(x_211); +lean_dec(x_210); +lean_dec(x_16); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_2); +lean_dec(x_1); +x_250 = lean_ctor_get(x_227, 0); +lean_inc(x_250); +x_251 = lean_ctor_get(x_227, 1); +lean_inc(x_251); +if (lean_is_exclusive(x_227)) { + lean_ctor_release(x_227, 0); + lean_ctor_release(x_227, 1); + x_252 = x_227; +} else { + lean_dec_ref(x_227); + x_252 = lean_box(0); +} +if (lean_is_scalar(x_252)) { + x_253 = lean_alloc_ctor(1, 2, 0); +} else { + x_253 = x_252; +} +lean_ctor_set(x_253, 0, x_250); +lean_ctor_set(x_253, 1, x_251); +return x_253; +} +} +} +} +else +{ +lean_object* x_254; lean_object* x_255; lean_object* x_256; uint8_t x_257; +if (lean_is_exclusive(x_217)) { + lean_ctor_release(x_217, 0); + x_254 = x_217; +} else { + lean_dec_ref(x_217); + x_254 = lean_box(0); +} +x_255 = lean_box(0); +x_256 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__1(x_15, x_255); +x_257 = l_List_isEmpty___rarg(x_256); +if (x_257 == 0) +{ +lean_object* x_258; lean_object* x_259; lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; +lean_dec(x_210); +x_258 = lean_array_mk(x_256); +x_259 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_260 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12; +x_261 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_262 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_259, x_260, x_258, x_261); +if (lean_is_scalar(x_254)) { + x_263 = lean_alloc_ctor(1, 1, 0); +} else { + x_263 = x_254; +} +lean_ctor_set(x_263, 0, x_262); +if (lean_is_scalar(x_213)) { + x_264 = lean_alloc_ctor(0, 2, 0); +} else { + x_264 = x_213; +} +lean_ctor_set(x_264, 0, x_211); +lean_ctor_set(x_264, 1, x_212); +x_265 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_265, 0, x_263); +lean_ctor_set(x_265, 1, x_264); +x_266 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_266, 0, x_265); +x_17 = x_266; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_267; lean_object* x_268; lean_object* x_269; +lean_dec(x_256); +lean_dec(x_254); +if (lean_is_scalar(x_213)) { + x_267 = lean_alloc_ctor(0, 2, 0); +} else { + x_267 = x_213; +} +lean_ctor_set(x_267, 0, x_211); +lean_ctor_set(x_267, 1, x_212); +x_268 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_268, 0, x_210); +lean_ctor_set(x_268, 1, x_267); +x_269 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_269, 0, x_268); +x_17 = x_269; +x_18 = x_13; +goto block_21; +} +} +} +else +{ +lean_object* x_270; lean_object* x_271; lean_object* x_272; uint8_t x_273; +if (lean_is_exclusive(x_215)) { + lean_ctor_release(x_215, 0); + x_270 = x_215; +} else { + lean_dec_ref(x_215); + x_270 = lean_box(0); +} +x_271 = lean_box(0); +x_272 = l_List_filterTR_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__2(x_15, x_271); +x_273 = l_List_isEmpty___rarg(x_272); +if (x_273 == 0) +{ +lean_object* x_274; lean_object* x_275; lean_object* x_276; lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; lean_object* x_281; lean_object* x_282; +lean_dec(x_212); +x_274 = lean_array_mk(x_272); +x_275 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4; +x_276 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13; +x_277 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_278 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_275, x_276, x_274, x_277); +if (lean_is_scalar(x_270)) { + x_279 = lean_alloc_ctor(1, 1, 0); +} else { + x_279 = x_270; +} +lean_ctor_set(x_279, 0, x_278); +if (lean_is_scalar(x_213)) { + x_280 = lean_alloc_ctor(0, 2, 0); +} else { + x_280 = x_213; +} +lean_ctor_set(x_280, 0, x_211); +lean_ctor_set(x_280, 1, x_279); +x_281 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_281, 0, x_210); +lean_ctor_set(x_281, 1, x_280); +x_282 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_282, 0, x_281); +x_17 = x_282; +x_18 = x_13; +goto block_21; +} +else +{ +lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_272); +lean_dec(x_270); +if (lean_is_scalar(x_213)) { + x_283 = lean_alloc_ctor(0, 2, 0); +} else { + x_283 = x_213; +} +lean_ctor_set(x_283, 0, x_211); +lean_ctor_set(x_283, 1, x_212); +x_284 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_284, 0, x_210); +lean_ctor_set(x_284, 1, x_283); +x_285 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_285, 0, x_284); +x_17 = x_285; +x_18 = x_13; +goto block_21; +} +} +} +block_21: +{ +lean_object* x_19; +x_19 = lean_ctor_get(x_17, 0); +lean_inc(x_19); +lean_dec(x_17); +x_6 = x_16; +x_7 = x_19; +x_8 = lean_box(0); +x_13 = x_18; +goto _start; +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Equivalence classes", 19, 19); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; +x_9 = l_Array_isEmpty___rarg(x_1); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5; +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3; +x_12 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_12, 0, x_10); +lean_ctor_set(x_12, 1, x_11); +lean_ctor_set(x_12, 2, x_1); +x_13 = lean_array_push(x_2, x_12); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_8); +return x_14; +} +else +{ +lean_object* x_15; +lean_dec(x_1); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_8); +return x_15; +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1(x_1, x_3, x_10, x_5, x_6, x_7, x_8, x_9); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_12 = lean_ctor_get(x_2, 0); +lean_inc(x_12); +lean_dec(x_2); +x_13 = lean_array_push(x_3, x_12); +x_14 = lean_box(0); +x_15 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1(x_1, x_13, x_14, x_5, x_6, x_7, x_8, x_9); +return x_15; +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_2); +lean_ctor_set(x_3, 1, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1; +x_3 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_7 = lean_box(0); +x_8 = l_Lean_Meta_Grind_Goal_getEqcs(x_1); +x_9 = lean_box(0); +x_10 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2; +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_8); +x_12 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3(x_7, x_10, x_8, x_9, x_8, x_8, x_11, lean_box(0), x_2, x_3, x_4, x_5, x_6); +lean_dec(x_8); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 1); +lean_inc(x_14); +x_15 = lean_ctor_get(x_14, 1); +lean_inc(x_15); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_16 = lean_ctor_get(x_12, 1); +lean_inc(x_16); +lean_dec(x_12); +x_17 = lean_ctor_get(x_13, 0); +lean_inc(x_17); +lean_dec(x_13); +x_18 = lean_ctor_get(x_14, 0); +lean_inc(x_18); +lean_dec(x_14); +x_19 = lean_box(0); +x_20 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2(x_18, x_17, x_10, x_19, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_20; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_21 = lean_ctor_get(x_12, 1); +lean_inc(x_21); +lean_dec(x_12); +x_22 = lean_ctor_get(x_13, 0); +lean_inc(x_22); +lean_dec(x_13); +x_23 = lean_ctor_get(x_14, 0); +lean_inc(x_23); +lean_dec(x_14); +x_24 = lean_ctor_get(x_15, 0); +lean_inc(x_24); +lean_dec(x_15); +x_25 = lean_array_push(x_10, x_24); +x_26 = lean_box(0); +x_27 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2(x_23, x_22, x_25, x_26, x_2, x_3, x_4, x_5, x_21); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_27; +} +} +else +{ +uint8_t x_28; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_28 = !lean_is_exclusive(x_12); +if (x_28 == 0) +{ +return x_12; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_12, 0); +x_30 = lean_ctor_get(x_12, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_12); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +} +} +LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_14; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; +x_9 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_9; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_10; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("\npatterns: ", 11, 11); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("thm", 3, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6() { +_start: +{ +lean_object* x_1; double x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_3 = 1; +x_4 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_5 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +lean_ctor_set_float(x_5, sizeof(void*)*2, x_2); +lean_ctor_set_float(x_5, sizeof(void*)*2 + 8, x_2); +lean_ctor_set_uint8(x_5, sizeof(void*)*2 + 16, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_1, 5); +lean_inc(x_7); +x_8 = l_Lean_Meta_Grind_Origin_pp___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__3(x_7, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_ctor_get(x_1, 1); +lean_inc(x_11); +x_12 = lean_infer_type(x_11, x_2, x_3, x_4, x_5, x_10); +if (lean_obj_tag(x_12) == 0) +{ +uint8_t x_13; +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_14 = lean_ctor_get(x_12, 0); +x_15 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_16 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_9); +x_17 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1; +x_18 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_18, 0, x_16); +lean_ctor_set(x_18, 1, x_17); +x_19 = l_Lean_MessageData_ofExpr(x_14); +x_20 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_21 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = lean_ctor_get(x_1, 3); +lean_inc(x_23); +lean_dec(x_1); +x_24 = lean_box(0); +x_25 = l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__1(x_23, x_24); +x_26 = l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__2(x_25, x_24); +x_27 = l_Lean_MessageData_ofList(x_26); +x_28 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_27); +x_29 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_15); +x_30 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6; +x_31 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_32 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_29); +lean_ctor_set(x_32, 2, x_31); +lean_ctor_set(x_12, 0, x_32); +return x_12; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_33 = lean_ctor_get(x_12, 0); +x_34 = lean_ctor_get(x_12, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_12); +x_35 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_36 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_9); +x_37 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +x_39 = l_Lean_MessageData_ofExpr(x_33); +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3; +x_42 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +x_43 = lean_ctor_get(x_1, 3); +lean_inc(x_43); +lean_dec(x_1); +x_44 = lean_box(0); +x_45 = l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__1(x_43, x_44); +x_46 = l_List_mapTR_loop___at_Lean_Meta_Grind_mkEMatchTheoremCore___spec__2(x_45, x_44); +x_47 = l_Lean_MessageData_ofList(x_46); +x_48 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_48, 0, x_42); +lean_ctor_set(x_48, 1, x_47); +x_49 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_35); +x_50 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6; +x_51 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_52 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_49); +lean_ctor_set(x_52, 2, x_51); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_34); +return x_53; +} +} +else +{ +uint8_t x_54; +lean_dec(x_9); +lean_dec(x_1); +x_54 = !lean_is_exclusive(x_12); +if (x_54 == 0) +{ +return x_12; +} +else +{ +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_12, 0); +x_56 = lean_ctor_get(x_12, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_12); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; +} +} +} +else +{ +uint8_t x_58; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_58 = !lean_is_exclusive(x_8); +if (x_58 == 0) +{ +return x_8; +} +else +{ +lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_59 = lean_ctor_get(x_8, 0); +x_60 = lean_ctor_get(x_8, 1); +lean_inc(x_60); +lean_inc(x_59); +lean_dec(x_8); +x_61 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_61, 0, x_59); +lean_ctor_set(x_61, 1, x_60); +return x_61; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1(size_t x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +uint8_t x_9; +x_9 = lean_usize_dec_lt(x_2, x_1); +if (x_9 == 0) +{ +lean_object* x_10; +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_3); +lean_ctor_set(x_10, 1, x_8); +return x_10; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_array_uget(x_3, x_2); +x_12 = lean_unsigned_to_nat(0u); +x_13 = lean_array_uset(x_3, x_2, x_12); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +x_14 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem(x_11, x_4, x_5, x_6, x_7, x_8); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; size_t x_17; size_t x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = 1; +x_18 = lean_usize_add(x_2, x_17); +x_19 = lean_array_uset(x_13, x_2, x_15); +x_2 = x_18; +x_3 = x_19; +x_8 = x_16; +goto _start; +} +else +{ +uint8_t x_21; +lean_dec(x_13); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +x_21 = !lean_is_exclusive(x_14); +if (x_21 == 0) +{ +return x_14; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_14, 0); +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_14); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; +} +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ematch", 6, 6); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3() { +_start: +{ +lean_object* x_1; double x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_3 = 1; +x_4 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_5 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +lean_ctor_set_float(x_5, sizeof(void*)*2, x_2); +lean_ctor_set_float(x_5, sizeof(void*)*2 + 8, x_2); +lean_ctor_set_uint8(x_5, sizeof(void*)*2 + 16, x_3); +return x_5; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("E-matching", 10, 10); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_7 = lean_ctor_get(x_1, 10); +x_8 = l_Lean_PersistentArray_toArray___rarg(x_7); +x_9 = lean_array_size(x_8); +x_10 = 0; +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1(x_9, x_10, x_8, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; size_t x_16; lean_object* x_17; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_ctor_get(x_1, 11); +x_15 = l_Lean_PersistentArray_toArray___rarg(x_14); +x_16 = lean_array_size(x_15); +x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1(x_16, x_10, x_15, x_2, x_3, x_4, x_5, x_13); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_ctor_get(x_17, 0); +x_20 = l_Array_append___rarg(x_12, x_19); +lean_dec(x_19); +x_21 = l_Array_isEmpty___rarg(x_20); +if (x_21 == 0) +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3; +x_23 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6; +x_24 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +lean_ctor_set(x_24, 2, x_20); +lean_ctor_set(x_17, 0, x_24); +return x_17; +} +else +{ +lean_object* x_25; +lean_dec(x_20); +x_25 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8; +lean_ctor_set(x_17, 0, x_25); +return x_17; +} +} +else +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_26 = lean_ctor_get(x_17, 0); +x_27 = lean_ctor_get(x_17, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_17); +x_28 = l_Array_append___rarg(x_12, x_26); +lean_dec(x_26); +x_29 = l_Array_isEmpty___rarg(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3; +x_31 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6; +x_32 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_28); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_27); +return x_33; +} +else +{ +lean_object* x_34; lean_object* x_35; +lean_dec(x_28); +x_34 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8; +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_27); +return x_35; +} +} +} +else +{ +uint8_t x_36; +lean_dec(x_12); +x_36 = !lean_is_exclusive(x_17); +if (x_36 == 0) +{ +return x_17; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_17, 0); +x_38 = lean_ctor_get(x_17, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_17); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; +} +} +} +else +{ +uint8_t x_40; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_40 = !lean_is_exclusive(x_11); +if (x_40 == 0) +{ +return x_11; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_11, 0); +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_11); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +size_t x_9; size_t x_10; lean_object* x_11; +x_9 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_10 = lean_unbox_usize(x_2); +lean_dec(x_2); +x_11 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___spec__1(x_9, x_10, x_3, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_1); +return x_7; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("assign", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3() { +_start: +{ +lean_object* x_1; double x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_3 = 1; +x_4 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_5 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +lean_ctor_set_float(x_5, sizeof(void*)*2, x_2); +lean_ctor_set_float(x_5, sizeof(void*)*2 + 8, x_2); +lean_ctor_set_uint8(x_5, sizeof(void*)*2 + 16, x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; +x_13 = lean_usize_dec_lt(x_6, x_5); +if (x_13 == 0) +{ +lean_object* x_14; +lean_dec(x_2); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_7); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +else +{ +lean_object* x_15; uint8_t x_16; +x_15 = lean_array_uget(x_4, x_6); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; size_t x_31; size_t x_32; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = l_Lean_MessageData_ofExpr(x_17); +x_20 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_19); +lean_ctor_set(x_15, 0, x_20); +x_21 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2; +x_22 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_22, 0, x_15); +lean_ctor_set(x_22, 1, x_21); +x_23 = l___private_Init_Data_Repr_0__Nat_reprFast(x_18); +x_24 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_24, 0, x_23); +x_25 = l_Lean_MessageData_ofFormat(x_24); +x_26 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_26, 0, x_22); +lean_ctor_set(x_26, 1, x_25); +x_27 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_20); +x_28 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3; +lean_inc(x_2); +x_29 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +lean_ctor_set(x_29, 2, x_2); +x_30 = lean_array_push(x_7, x_29); +x_31 = 1; +x_32 = lean_usize_add(x_6, x_31); +x_6 = x_32; +x_7 = x_30; +goto _start; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; size_t x_49; size_t x_50; +x_34 = lean_ctor_get(x_15, 0); +x_35 = lean_ctor_get(x_15, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_15); +x_36 = l_Lean_MessageData_ofExpr(x_34); +x_37 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9; +x_38 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 1, x_36); +x_39 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2; +x_40 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +x_41 = l___private_Init_Data_Repr_0__Nat_reprFast(x_35); +x_42 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_42, 0, x_41); +x_43 = l_Lean_MessageData_ofFormat(x_42); +x_44 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_44, 0, x_40); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_37); +x_46 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3; +lean_inc(x_2); +x_47 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_47, 0, x_46); +lean_ctor_set(x_47, 1, x_45); +lean_ctor_set(x_47, 2, x_2); +x_48 = lean_array_push(x_7, x_47); +x_49 = 1; +x_50 = lean_usize_add(x_6, x_49); +x_6 = x_50; +x_7 = x_48; +goto _start; +} +} +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("offset", 6, 6); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; double x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2; +x_2 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1; +x_3 = 1; +x_4 = l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8; +x_5 = lean_alloc_ctor(0, 2, 17); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_4); +lean_ctor_set_float(x_5, sizeof(void*)*2, x_2); +lean_ctor_set_float(x_5, sizeof(void*)*2 + 8, x_2); +lean_ctor_set_uint8(x_5, sizeof(void*)*2 + 16, x_3); +return x_5; +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Assignment satisfying offset contraints", 39, 39); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5; +x_2 = l_Lean_MessageData_ofFormat(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_8 = l_Lean_Meta_Grind_Arith_Offset_mkModel(x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = lean_box(0); +x_12 = lean_array_size(x_9); +x_13 = 0; +x_14 = l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2; +x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1(x_9, x_14, x_11, x_9, x_12, x_13, x_14, x_3, x_4, x_5, x_6, x_10); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_9); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_15, 0); +x_18 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3; +x_19 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6; +x_20 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +lean_ctor_set(x_20, 2, x_17); +lean_ctor_set(x_15, 0, x_20); +return x_15; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_21 = lean_ctor_get(x_15, 0); +x_22 = lean_ctor_get(x_15, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_15); +x_23 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3; +x_24 = l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6; +x_25 = lean_alloc_ctor(9, 3, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +lean_ctor_set(x_25, 2, x_21); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_22); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_27 = !lean_is_exclusive(x_8); +if (x_27 == 0) +{ +return x_8; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_8, 0); +x_29 = lean_ctor_get(x_8, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_8); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; uint8_t x_9; +x_7 = lean_ctor_get(x_1, 9); +lean_inc(x_7); +x_8 = lean_ctor_get(x_7, 0); +lean_inc(x_8); +lean_dec(x_7); +x_9 = l_Lean_PersistentArray_isEmpty___rarg(x_8); +lean_dec(x_8); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_box(0); +x_11 = l_Lean_Meta_Grind_ppOffset___lambda__1(x_1, x_10, x_2, x_3, x_4, x_5, x_6); +return x_11; +} +else +{ +lean_object* x_12; lean_object* x_13; +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_12 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8; +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_6); +return x_13; +} +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +size_t x_13; size_t x_14; lean_object* x_15; +x_13 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_14 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_15 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_15; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppOffset___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +x_8 = l_Lean_Meta_Grind_ppOffset___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7); +lean_dec(x_2); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalToMessageData___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +lean_object* x_8; +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_1); +x_8 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs(x_1, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +x_10 = lean_ctor_get(x_8, 1); +lean_inc(x_10); +lean_dec(x_8); +x_11 = l_Array_append___rarg(x_2, x_9); +lean_dec(x_9); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_12 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems(x_1, x_3, x_4, x_5, x_6, x_10); +if (lean_obj_tag(x_12) == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_12, 1); +lean_inc(x_14); +lean_dec(x_12); +x_15 = lean_array_push(x_11, x_13); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_16 = l_Lean_Meta_Grind_ppOffset(x_1, x_3, x_4, x_5, x_6, x_14); +if (lean_obj_tag(x_16) == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_array_push(x_15, x_17); +x_20 = lean_array_to_list(x_19); +x_21 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8; +x_22 = l_Lean_MessageData_joinSep(x_20, x_21); +x_23 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_22, x_3, x_4, x_5, x_6, x_18); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_23; +} +else +{ +uint8_t x_24; +lean_dec(x_15); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_24 = !lean_is_exclusive(x_16); +if (x_24 == 0) +{ +return x_16; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_16, 0); +x_26 = lean_ctor_get(x_16, 1); +lean_inc(x_26); +lean_inc(x_25); +lean_dec(x_16); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; +} +} +} +else +{ +uint8_t x_28; +lean_dec(x_11); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_28 = !lean_is_exclusive(x_12); +if (x_28 == 0) +{ +return x_12; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_12, 0); +x_30 = lean_ctor_get(x_12, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_12); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +} +} +else +{ +uint8_t x_32; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); lean_dec(x_1); -x_21 = !lean_is_exclusive(x_10); -if (x_21 == 0) +x_32 = !lean_is_exclusive(x_8); +if (x_32 == 0) { -return x_10; +return x_8; } else { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_10, 0); -x_23 = lean_ctor_get(x_10, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_10); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_8, 0); +x_34 = lean_ctor_get(x_8, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_8); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } } -static lean_object* _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_goalToMessageData___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__2), 9, 0); +x_1 = lean_mk_string_unchecked("facts", 5, 5); return x_1; } } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +static lean_object* _init_l_Lean_Meta_Grind_goalToMessageData___closed__2() { _start: { -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_15; -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_5); -lean_ctor_set(x_15, 1, x_14); -return x_15; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_goalToMessageData___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l_Lean_Meta_Grind_goalToMessageData___closed__3() { +_start: { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_4); -if (x_16 == 0) +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Asserted facts", 14, 14); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalToMessageData(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_17 = lean_ctor_get(x_4, 0); -x_18 = lean_ctor_get(x_4, 1); -x_19 = lean_ctor_get(x_17, 0); -lean_inc(x_19); -x_20 = lean_alloc_closure((void*)(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1___boxed), 9, 1); -lean_closure_set(x_20, 0, x_17); -x_21 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; -x_22 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_22, 0, x_20); -lean_closure_set(x_22, 1, x_21); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_7 = lean_ctor_get(x_1, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_1, 22); lean_inc(x_8); lean_inc(x_7); -x_23 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_19, x_22, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_23) == 0) +x_9 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_9, 0, x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +x_12 = lean_array_mk(x_11); +x_13 = l_Lean_PersistentArray_toArray___rarg(x_8); +lean_dec(x_8); +x_14 = l_Lean_Meta_Grind_goalToMessageData___closed__2; +x_15 = l_Lean_Meta_Grind_goalToMessageData___closed__3; +x_16 = l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11; +x_17 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray(x_14, x_15, x_13, x_16); +x_18 = lean_array_push(x_12, x_17); +x_19 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_goalToMessageData___lambda__1), 7, 2); +lean_closure_set(x_19, 0, x_1); +lean_closure_set(x_19, 1, x_18); +x_20 = l_Lean_MVarId_withContext___at___private_Lean_Meta_SynthInstance_0__Lean_Meta_synthPendingImp___spec__2___rarg(x_7, x_19, x_2, x_3, x_4, x_5, x_6); +return x_20; +} +} +LEAN_EXPORT lean_object* l_List_mapM_loop___at_Lean_Meta_Grind_goalsToMessageData___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: { -lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +if (lean_obj_tag(x_1) == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_24, 0); -x_28 = lean_ctor_get(x_24, 1); -lean_dec(x_28); -x_29 = lean_box(1); -lean_ctor_set_tag(x_24, 5); -lean_ctor_set(x_24, 1, x_29); -lean_ctor_set(x_24, 0, x_5); -lean_ctor_set_tag(x_4, 5); -lean_ctor_set(x_4, 1, x_27); -lean_ctor_set(x_4, 0, x_24); -{ -lean_object* _tmp_3 = x_18; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_5 = lean_box(0); -lean_object* _tmp_13 = x_25; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_6 = _tmp_5; -x_14 = _tmp_13; -} -goto _start; +lean_object* x_8; lean_object* x_9; +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_8 = l_List_reverse___rarg(x_2); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_8); +lean_ctor_set(x_9, 1, x_7); +return x_9; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_24, 0); -lean_inc(x_31); -lean_dec(x_24); -x_32 = lean_box(1); -x_33 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_33, 0, x_5); -lean_ctor_set(x_33, 1, x_32); -lean_ctor_set_tag(x_4, 5); -lean_ctor_set(x_4, 1, x_31); -lean_ctor_set(x_4, 0, x_33); -{ -lean_object* _tmp_3 = x_18; -lean_object* _tmp_4 = x_4; -lean_object* _tmp_5 = lean_box(0); -lean_object* _tmp_13 = x_25; -x_4 = _tmp_3; -x_5 = _tmp_4; -x_6 = _tmp_5; -x_14 = _tmp_13; +uint8_t x_10; +x_10 = !lean_is_exclusive(x_1); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_1, 0); +x_12 = lean_ctor_get(x_1, 1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_13 = l_Lean_Meta_Grind_goalToMessageData(x_11, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; lean_object* x_15; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +lean_ctor_set(x_1, 1, x_2); +lean_ctor_set(x_1, 0, x_14); +{ +lean_object* _tmp_0 = x_12; +lean_object* _tmp_1 = x_1; +lean_object* _tmp_6 = x_15; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_7 = _tmp_6; } goto _start; } -} else { -uint8_t x_35; -lean_free_object(x_4); -lean_dec(x_18); -lean_dec(x_13); +uint8_t x_17; +lean_free_object(x_1); lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -x_35 = !lean_is_exclusive(x_23); -if (x_35 == 0) +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_17 = !lean_is_exclusive(x_13); +if (x_17 == 0) { -return x_23; +return x_13; } else { -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_23, 0); -x_37 = lean_ctor_get(x_23, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_23); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_18 = lean_ctor_get(x_13, 0); +x_19 = lean_ctor_get(x_13, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_13); +x_20 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +return x_20; } } } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_39 = lean_ctor_get(x_4, 0); -x_40 = lean_ctor_get(x_4, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_4); -x_41 = lean_ctor_get(x_39, 0); -lean_inc(x_41); -x_42 = lean_alloc_closure((void*)(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1___boxed), 9, 1); -lean_closure_set(x_42, 0, x_39); -x_43 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1; -x_44 = lean_alloc_closure((void*)(l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg), 10, 2); -lean_closure_set(x_44, 0, x_42); -lean_closure_set(x_44, 1, x_43); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_45 = l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(x_41, x_44, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_45) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_1, 0); +x_22 = lean_ctor_get(x_1, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_1); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +x_23 = l_Lean_Meta_Grind_goalToMessageData(x_21, x_3, x_4, x_5, x_6, x_7); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = lean_ctor_get(x_46, 0); -lean_inc(x_48); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_49 = x_46; -} else { - lean_dec_ref(x_46); - x_49 = lean_box(0); -} -x_50 = lean_box(1); -if (lean_is_scalar(x_49)) { - x_51 = lean_alloc_ctor(5, 2, 0); -} else { - x_51 = x_49; - lean_ctor_set_tag(x_51, 5); -} -lean_ctor_set(x_51, 0, x_5); -lean_ctor_set(x_51, 1, x_50); -x_52 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_48); -x_4 = x_40; -x_5 = x_52; -x_6 = lean_box(0); -x_14 = x_47; +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_2); +x_1 = x_22; +x_2 = x_26; +x_7 = x_25; goto _start; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -lean_dec(x_40); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_22); +lean_dec(x_6); lean_dec(x_5); -x_54 = lean_ctor_get(x_45, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_45, 1); -lean_inc(x_55); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_56 = x_45; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_28 = lean_ctor_get(x_23, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_23, 1); +lean_inc(x_29); +if (lean_is_exclusive(x_23)) { + lean_ctor_release(x_23, 0); + lean_ctor_release(x_23, 1); + x_30 = x_23; } else { - lean_dec_ref(x_45); - x_56 = lean_box(0); + lean_dec_ref(x_23); + x_30 = lean_box(0); } -if (lean_is_scalar(x_56)) { - x_57 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_30)) { + x_31 = lean_alloc_ctor(1, 2, 0); } else { - x_57 = x_56; + x_31 = x_30; } -lean_ctor_set(x_57, 0, x_54); -lean_ctor_set(x_57, 1, x_55); -return x_57; +lean_ctor_set(x_31, 0, x_28); +lean_ctor_set(x_31, 1, x_29); +return x_31; } } } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ppGoals(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_goalsToMessageData(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_10 = lean_box(0); -x_11 = l_Lean_Meta_Grind_ppENodeRef___closed__6; -lean_inc(x_1); -x_12 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(x_1, x_10, x_1, x_1, x_11, lean_box(0), x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_1); -if (lean_obj_tag(x_12) == 0) +lean_object* x_7; lean_object* x_8; +x_7 = lean_box(0); +x_8 = l_List_mapM_loop___at_Lean_Meta_Grind_goalsToMessageData___spec__1(x_1, x_7, x_2, x_3, x_4, x_5, x_6); +if (lean_obj_tag(x_8) == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +uint8_t x_9; +x_9 = !lean_is_exclusive(x_8); +if (x_9 == 0) { -return x_12; +lean_object* x_10; lean_object* x_11; lean_object* x_12; +x_10 = lean_ctor_get(x_8, 0); +x_11 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1; +x_12 = l_Lean_MessageData_joinSep(x_10, x_11); +lean_ctor_set(x_8, 0, x_12); +return x_8; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_8, 0); +x_14 = lean_ctor_get(x_8, 1); lean_inc(x_14); -lean_dec(x_12); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; +lean_inc(x_13); +lean_dec(x_8); +x_15 = l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1; +x_16 = l_Lean_MessageData_joinSep(x_13, x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_14); +return x_17; } } else { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_12); -if (x_17 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_8); +if (x_18 == 0) { -return x_12; +return x_8; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_18 = lean_ctor_get(x_12, 0); -x_19 = lean_ctor_get(x_12, 1); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_8, 0); +x_20 = lean_ctor_get(x_8, 1); +lean_inc(x_20); lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_12); -x_20 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_20, 0, x_18); -lean_ctor_set(x_20, 1, x_19); -return x_20; -} -} -} -} -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } -LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { -_start: -{ -lean_object* x_15; -x_15 = l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_15; } } lean_object* initialize_Init_Grind_Util(uint8_t builtin, lean_object*); +lean_object* initialize_Init_Grind_PP(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Model(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_PP(uint8_t builtin, lean_object* w) { lean_object * res; @@ -2380,73 +5476,190 @@ _G_initialized = true; res = initialize_Init_Grind_Util(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Init_Grind_PP(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Types(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_Grind_ppENodeRef___closed__1 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__1); -l_Lean_Meta_Grind_ppENodeRef___closed__2 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__2); -l_Lean_Meta_Grind_ppENodeRef___closed__3 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__3); -l_Lean_Meta_Grind_ppENodeRef___closed__4 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__4); -l_Lean_Meta_Grind_ppENodeRef___closed__5 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__5); -l_Lean_Meta_Grind_ppENodeRef___closed__6 = _init_l_Lean_Meta_Grind_ppENodeRef___closed__6(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeRef___closed__6); -l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__1); -l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppENodeDeclValue___spec__1___closed__2); -l_Lean_Meta_Grind_ppENodeDeclValue___closed__1 = _init_l_Lean_Meta_Grind_ppENodeDeclValue___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDeclValue___closed__1); -l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__1); -l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__2); -l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__3); -l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__2___closed__4); -l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__1); -l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__3___closed__2); -l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__1); -l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2 = _init_l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___lambda__4___closed__2); -l_Lean_Meta_Grind_ppENodeDecl___closed__1 = _init_l_Lean_Meta_Grind_ppENodeDecl___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___closed__1); -l_Lean_Meta_Grind_ppENodeDecl___closed__2 = _init_l_Lean_Meta_Grind_ppENodeDecl___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___closed__2); -l_Lean_Meta_Grind_ppENodeDecl___closed__3 = _init_l_Lean_Meta_Grind_ppENodeDecl___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___closed__3); -l_Lean_Meta_Grind_ppENodeDecl___closed__4 = _init_l_Lean_Meta_Grind_ppENodeDecl___closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_ppENodeDecl___closed__4); -l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__1); -l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppState___spec__1___closed__2); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__1); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__2); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__3); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__4); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__5); -l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6(); -lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppState___spec__3___closed__6); -l_Lean_Meta_Grind_ppState___closed__1 = _init_l_Lean_Meta_Grind_ppState___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_ppState___closed__1); -l_Lean_Meta_Grind_ppState___closed__2 = _init_l_Lean_Meta_Grind_ppState___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_ppState___closed__2); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Model(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__1); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__2); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__3); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__4); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__5); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__6); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__7); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__8); +l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9 = _init_l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppENodeRef___closed__9); +l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__1); +l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__2); +l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3 = _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___spec__1___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDeclValue___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__2___closed__4); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__3___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___lambda__4___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_Goal_ppENodeDecl___closed__4); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__2); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_ppState___spec__1___closed__3); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__1); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__2); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__3); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__4); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__5); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__6); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__7); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__8); +l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9(); +lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_Goal_ppState___spec__3___closed__9); +l_Lean_Meta_Grind_Goal_ppState___closed__1 = _init_l_Lean_Meta_Grind_Goal_ppState___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppState___closed__1); +l_Lean_Meta_Grind_Goal_ppState___closed__2 = _init_l_Lean_Meta_Grind_Goal_ppState___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_Goal_ppState___closed__2); l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1 = _init_l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1(); lean_mark_persistent(l_List_forIn_x27_loop___at_Lean_Meta_Grind_ppGoals___spec__1___closed__1); +l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__1(); +l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2 = _init_l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppExprArray___spec__1___closed__2); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__1); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__2); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__3); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__4); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__5); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__6); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__7); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__8); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__9); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__10); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__11); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__12); +l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13 = _init_l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13(); +lean_mark_persistent(l_List_forIn_x27_loop___at___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___spec__3___closed__13); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___lambda__1___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEqcs___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__4); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__5); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppEMatchTheorem___closed__6); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__1); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__2); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__3); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__4); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__5); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__6); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__7); +l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_PP_0__Lean_Meta_Grind_ppActiveTheorems___closed__8); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__2); +l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_ppOffset___spec__1___closed__3); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__1); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__2); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__3); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__4); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__5); +l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6 = _init_l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_ppOffset___lambda__1___closed__6); +l_Lean_Meta_Grind_goalToMessageData___closed__1 = _init_l_Lean_Meta_Grind_goalToMessageData___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_goalToMessageData___closed__1); +l_Lean_Meta_Grind_goalToMessageData___closed__2 = _init_l_Lean_Meta_Grind_goalToMessageData___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_goalToMessageData___closed__2); +l_Lean_Meta_Grind_goalToMessageData___closed__3 = _init_l_Lean_Meta_Grind_goalToMessageData___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_goalToMessageData___closed__3); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Proj.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Proj.c index 5cfa35c8a3b9..009d0d887eed 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Proj.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Proj.c @@ -20,6 +20,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__4(lean_obje LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_Goal_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); @@ -28,7 +29,6 @@ lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object*, lean_object*, lean_obje lean_object* l_Lean_Expr_appArg_x21(lean_object*); static lean_object* l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_Grind_propagateProjEq___spec__1___closed__1; extern lean_object* l_Lean_projectionFnInfoExt; -lean_object* l_Lean_Meta_Grind_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -62,7 +62,7 @@ lean_object* l_Lean_Expr_getAppFn(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__3___closed__2; lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* _init_l_Lean_getProjectionFnInfo_x3f___at_Lean_Meta_Grind_propagateProjEq___spec__1___closed__1() { _start: @@ -436,12 +436,13 @@ lean_dec(x_18); x_21 = l_Lean_Meta_Grind_getGeneration(x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_20); if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); x_23 = lean_ctor_get(x_21, 1); lean_inc(x_23); lean_dec(x_21); +x_24 = lean_box(0); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -451,24 +452,24 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_19); -x_24 = l_Lean_Meta_Grind_internalize(x_19, x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_23); -if (lean_obj_tag(x_24) == 0) +x_25 = l_Lean_Meta_Grind_internalize(x_19, x_22, x_24, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_23); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_25; lean_object* x_26; -x_25 = lean_ctor_get(x_24, 1); -lean_inc(x_25); -lean_dec(x_24); -x_26 = l_Lean_Meta_Grind_propagateProjEq___lambda__3(x_1, x_2, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_25, 1); +lean_inc(x_26); +lean_dec(x_25); +x_27 = l_Lean_Meta_Grind_propagateProjEq___lambda__3(x_1, x_2, x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_26); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_2); -return x_26; +return x_27; } else { -uint8_t x_27; +uint8_t x_28; lean_dec(x_19); lean_dec(x_13); lean_dec(x_12); @@ -479,29 +480,29 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_2); -x_27 = !lean_is_exclusive(x_24); -if (x_27 == 0) +x_28 = !lean_is_exclusive(x_25); +if (x_28 == 0) { -return x_24; +return x_25; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_24, 0); -x_29 = lean_ctor_get(x_24, 1); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_25, 0); +x_30 = lean_ctor_get(x_25, 1); +lean_inc(x_30); lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_24); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_dec(x_25); +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } } else { -uint8_t x_31; +uint8_t x_32; lean_dec(x_19); lean_dec(x_13); lean_dec(x_12); @@ -512,61 +513,67 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_2); -x_31 = !lean_is_exclusive(x_21); -if (x_31 == 0) +x_32 = !lean_is_exclusive(x_21); +if (x_32 == 0) { return x_21; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_21, 0); -x_33 = lean_ctor_get(x_21, 1); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_21, 0); +x_34 = lean_ctor_get(x_21, 1); +lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); lean_dec(x_21); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } else { -lean_object* x_35; -x_35 = l_Lean_Meta_Grind_propagateProjEq___lambda__3(x_1, x_2, x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_object* x_36; +x_36 = l_Lean_Meta_Grind_propagateProjEq___lambda__3(x_1, x_2, x_4, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_2); -return x_35; +return x_36; } } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateProjEq___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_13; lean_object* x_14; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_13 = l_Lean_Expr_appArg_x21(x_1); +x_14 = lean_st_ref_get(x_4, x_12); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); lean_inc(x_13); -x_14 = l_Lean_Meta_Grind_getRoot(x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_14) == 0) +x_17 = l_Lean_Meta_Grind_Goal_getRoot(x_15, x_13, x_10, x_11, x_16); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_2, 0); -x_19 = l_Lean_Expr_isAppOf(x_16, x_18); -if (x_19 == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_ctor_get(x_2, 0); +x_22 = l_Lean_Expr_isAppOf(x_19, x_21); +if (x_22 == 0) { -lean_object* x_20; -lean_dec(x_16); +lean_object* x_23; +lean_dec(x_19); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); @@ -577,34 +584,34 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_20 = lean_box(0); -lean_ctor_set(x_14, 0, x_20); -return x_14; +x_23 = lean_box(0); +lean_ctor_set(x_17, 0, x_23); +return x_17; } else { -lean_object* x_21; lean_object* x_22; -lean_free_object(x_14); -x_21 = lean_box(0); -x_22 = l_Lean_Meta_Grind_propagateProjEq___lambda__4(x_2, x_16, x_13, x_1, x_21, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_17); +lean_object* x_24; lean_object* x_25; +lean_free_object(x_17); +x_24 = lean_box(0); +x_25 = l_Lean_Meta_Grind_propagateProjEq___lambda__4(x_2, x_19, x_13, x_1, x_24, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_20); lean_dec(x_13); -return x_22; +return x_25; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_23 = lean_ctor_get(x_14, 0); -x_24 = lean_ctor_get(x_14, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_14); -x_25 = lean_ctor_get(x_2, 0); -x_26 = l_Lean_Expr_isAppOf(x_23, x_25); -if (x_26 == 0) +lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_26 = lean_ctor_get(x_17, 0); +x_27 = lean_ctor_get(x_17, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_17); +x_28 = lean_ctor_get(x_2, 0); +x_29 = l_Lean_Expr_isAppOf(x_26, x_28); +if (x_29 == 0) { -lean_object* x_27; lean_object* x_28; -lean_dec(x_23); +lean_object* x_30; lean_object* x_31; +lean_dec(x_26); lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); @@ -615,25 +622,25 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_27 = lean_box(0); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_24); -return x_28; +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_27); +return x_31; } else { -lean_object* x_29; lean_object* x_30; -x_29 = lean_box(0); -x_30 = l_Lean_Meta_Grind_propagateProjEq___lambda__4(x_2, x_23, x_13, x_1, x_29, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_24); +lean_object* x_32; lean_object* x_33; +x_32 = lean_box(0); +x_33 = l_Lean_Meta_Grind_propagateProjEq___lambda__4(x_2, x_26, x_13, x_1, x_32, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_27); lean_dec(x_13); -return x_30; +return x_33; } } } else { -uint8_t x_31; +uint8_t x_34; lean_dec(x_13); lean_dec(x_11); lean_dec(x_10); @@ -644,23 +651,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_31 = !lean_is_exclusive(x_14); -if (x_31 == 0) +x_34 = !lean_is_exclusive(x_17); +if (x_34 == 0) { -return x_14; +return x_17; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_14, 0); -x_33 = lean_ctor_get(x_14, 1); -lean_inc(x_33); -lean_inc(x_32); -lean_dec(x_14); -x_34 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); -return x_34; +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_17, 0); +x_36 = lean_ctor_get(x_17, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_17); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; } } } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Proof.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Proof.c index 8a674a81ce00..84d0d31b49d0 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Proof.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Proof.c @@ -72,6 +72,7 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqCongrProof___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedPUnit; +lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_isCongrDefaultProofTarget_loop___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); @@ -186,7 +187,6 @@ static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_ lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqOfHEqIfNeeded___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkCongrDefaultProof___closed__1; -lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkHCongrProof___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqCongrProof___lambda__1___closed__7; static lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqCongrProof___lambda__1___closed__3; @@ -3067,202 +3067,214 @@ uint8_t x_12; x_12 = !lean_is_exclusive(x_2); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; x_13 = lean_ctor_get(x_2, 0); x_14 = lean_ctor_get(x_2, 1); +x_15 = lean_st_ref_get(x_3, x_11); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); lean_inc(x_13); -x_15 = l_Lean_Meta_Grind_getENode(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_15) == 0) +x_18 = l_Lean_Meta_Grind_Goal_getENode(x_16, x_13, x_9, x_10, x_17); +if (lean_obj_tag(x_18) == 0) { -uint8_t x_16; -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -x_19 = lean_ctor_get(x_17, 7); -lean_inc(x_19); -x_20 = lean_ctor_get(x_17, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_17, 4); -lean_inc(x_21); -lean_dec(x_17); -x_22 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_14, x_19, x_20); -if (lean_obj_tag(x_21) == 0) +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +x_22 = lean_ctor_get(x_20, 7); +lean_inc(x_22); +x_23 = lean_ctor_get(x_20, 0); +lean_inc(x_23); +x_24 = lean_ctor_get(x_20, 4); +lean_inc(x_24); +lean_dec(x_20); +x_25 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_14, x_22, x_23); +if (lean_obj_tag(x_24) == 0) { -lean_ctor_set(x_2, 1, x_22); -lean_ctor_set(x_15, 0, x_2); -return x_15; +lean_ctor_set(x_2, 1, x_25); +lean_ctor_set(x_18, 0, x_2); +return x_18; } else { -lean_object* x_23; -lean_free_object(x_15); +lean_object* x_26; +lean_free_object(x_18); lean_dec(x_13); -x_23 = lean_ctor_get(x_21, 0); -lean_inc(x_23); -lean_dec(x_21); -lean_ctor_set(x_2, 1, x_22); -lean_ctor_set(x_2, 0, x_23); -x_11 = x_18; +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +lean_dec(x_24); +lean_ctor_set(x_2, 1, x_25); +lean_ctor_set(x_2, 0, x_26); +x_11 = x_21; goto _start; } } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_25 = lean_ctor_get(x_15, 0); -x_26 = lean_ctor_get(x_15, 1); -lean_inc(x_26); -lean_inc(x_25); -lean_dec(x_15); -x_27 = lean_ctor_get(x_25, 7); -lean_inc(x_27); -x_28 = lean_ctor_get(x_25, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_25, 4); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_18, 0); +x_29 = lean_ctor_get(x_18, 1); lean_inc(x_29); -lean_dec(x_25); -x_30 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_14, x_27, x_28); -if (lean_obj_tag(x_29) == 0) +lean_inc(x_28); +lean_dec(x_18); +x_30 = lean_ctor_get(x_28, 7); +lean_inc(x_30); +x_31 = lean_ctor_get(x_28, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_28, 4); +lean_inc(x_32); +lean_dec(x_28); +x_33 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_14, x_30, x_31); +if (lean_obj_tag(x_32) == 0) { -lean_object* x_31; -lean_ctor_set(x_2, 1, x_30); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_2); -lean_ctor_set(x_31, 1, x_26); -return x_31; +lean_object* x_34; +lean_ctor_set(x_2, 1, x_33); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_2); +lean_ctor_set(x_34, 1, x_29); +return x_34; } else { -lean_object* x_32; +lean_object* x_35; lean_dec(x_13); -x_32 = lean_ctor_get(x_29, 0); -lean_inc(x_32); -lean_dec(x_29); -lean_ctor_set(x_2, 1, x_30); -lean_ctor_set(x_2, 0, x_32); -x_11 = x_26; +x_35 = lean_ctor_get(x_32, 0); +lean_inc(x_35); +lean_dec(x_32); +lean_ctor_set(x_2, 1, x_33); +lean_ctor_set(x_2, 0, x_35); +x_11 = x_29; goto _start; } } } else { -uint8_t x_34; +uint8_t x_37; lean_free_object(x_2); lean_dec(x_14); lean_dec(x_13); -x_34 = !lean_is_exclusive(x_15); -if (x_34 == 0) +x_37 = !lean_is_exclusive(x_18); +if (x_37 == 0) { -return x_15; +return x_18; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_15, 0); -x_36 = lean_ctor_get(x_15, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_15); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_18, 0); +x_39 = lean_ctor_get(x_18, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_18); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_2, 0); -x_39 = lean_ctor_get(x_2, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_2); -lean_inc(x_38); -x_40 = l_Lean_Meta_Grind_getENode(x_38, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_40) == 0) -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -x_42 = lean_ctor_get(x_40, 1); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_41 = lean_ctor_get(x_2, 0); +x_42 = lean_ctor_get(x_2, 1); lean_inc(x_42); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_43 = x_40; -} else { - lean_dec_ref(x_40); - x_43 = lean_box(0); -} -x_44 = lean_ctor_get(x_41, 7); +lean_inc(x_41); +lean_dec(x_2); +x_43 = lean_st_ref_get(x_3, x_11); +x_44 = lean_ctor_get(x_43, 0); lean_inc(x_44); -x_45 = lean_ctor_get(x_41, 0); +x_45 = lean_ctor_get(x_43, 1); lean_inc(x_45); -x_46 = lean_ctor_get(x_41, 4); -lean_inc(x_46); -lean_dec(x_41); -x_47 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_39, x_44, x_45); +lean_dec(x_43); +lean_inc(x_41); +x_46 = l_Lean_Meta_Grind_Goal_getENode(x_44, x_41, x_9, x_10, x_45); if (lean_obj_tag(x_46) == 0) { -lean_object* x_48; lean_object* x_49; -x_48 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_48, 0, x_38); -lean_ctor_set(x_48, 1, x_47); -if (lean_is_scalar(x_43)) { - x_49 = lean_alloc_ctor(0, 2, 0); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_47 = lean_ctor_get(x_46, 0); +lean_inc(x_47); +x_48 = lean_ctor_get(x_46, 1); +lean_inc(x_48); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_49 = x_46; } else { - x_49 = x_43; + lean_dec_ref(x_46); + x_49 = lean_box(0); } -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_42); -return x_49; +x_50 = lean_ctor_get(x_47, 7); +lean_inc(x_50); +x_51 = lean_ctor_get(x_47, 0); +lean_inc(x_51); +x_52 = lean_ctor_get(x_47, 4); +lean_inc(x_52); +lean_dec(x_47); +x_53 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_42, x_50, x_51); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_54; lean_object* x_55; +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_41); +lean_ctor_set(x_54, 1, x_53); +if (lean_is_scalar(x_49)) { + x_55 = lean_alloc_ctor(0, 2, 0); +} else { + x_55 = x_49; +} +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_48); +return x_55; } else { -lean_object* x_50; lean_object* x_51; -lean_dec(x_43); -lean_dec(x_38); -x_50 = lean_ctor_get(x_46, 0); -lean_inc(x_50); -lean_dec(x_46); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_47); -x_2 = x_51; -x_11 = x_42; +lean_object* x_56; lean_object* x_57; +lean_dec(x_49); +lean_dec(x_41); +x_56 = lean_ctor_get(x_52, 0); +lean_inc(x_56); +lean_dec(x_52); +x_57 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_53); +x_2 = x_57; +x_11 = x_48; goto _start; } } else { -lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -lean_dec(x_39); -lean_dec(x_38); -x_53 = lean_ctor_get(x_40, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_40, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_40)) { - lean_ctor_release(x_40, 0); - lean_ctor_release(x_40, 1); - x_55 = x_40; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; +lean_dec(x_42); +lean_dec(x_41); +x_59 = lean_ctor_get(x_46, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_46, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_46)) { + lean_ctor_release(x_46, 0); + lean_ctor_release(x_46, 1); + x_61 = x_46; } else { - lean_dec_ref(x_40); - x_55 = lean_box(0); + lean_dec_ref(x_46); + x_61 = lean_box(0); } -if (lean_is_scalar(x_55)) { - x_56 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(1, 2, 0); } else { - x_56 = x_55; + x_62 = x_61; } -lean_ctor_set(x_56, 0, x_53); -lean_ctor_set(x_56, 1, x_54); -return x_56; +lean_ctor_set(x_62, 0, x_59); +lean_ctor_set(x_62, 1, x_60); +return x_62; } } } @@ -3274,202 +3286,214 @@ uint8_t x_11; x_11 = !lean_is_exclusive(x_1); if (x_11 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_12 = lean_ctor_get(x_1, 0); x_13 = lean_ctor_get(x_1, 1); +x_14 = lean_st_ref_get(x_2, x_10); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); lean_inc(x_12); -x_14 = l_Lean_Meta_Grind_getENode(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_14) == 0) +x_17 = l_Lean_Meta_Grind_Goal_getENode(x_15, x_12, x_8, x_9, x_16); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_14, 1); -x_18 = lean_ctor_get(x_16, 7); -lean_inc(x_18); -x_19 = lean_ctor_get(x_16, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_16, 4); -lean_inc(x_20); -lean_dec(x_16); -x_21 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_13, x_18, x_19); -if (lean_obj_tag(x_20) == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_17, 1); +x_21 = lean_ctor_get(x_19, 7); +lean_inc(x_21); +x_22 = lean_ctor_get(x_19, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_19, 4); +lean_inc(x_23); +lean_dec(x_19); +x_24 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_13, x_21, x_22); +if (lean_obj_tag(x_23) == 0) { -lean_ctor_set(x_1, 1, x_21); -lean_ctor_set(x_14, 0, x_1); -return x_14; +lean_ctor_set(x_1, 1, x_24); +lean_ctor_set(x_17, 0, x_1); +return x_17; } else { -lean_object* x_22; -lean_free_object(x_14); +lean_object* x_25; +lean_free_object(x_17); lean_dec(x_12); -x_22 = lean_ctor_get(x_20, 0); -lean_inc(x_22); -lean_dec(x_20); -lean_ctor_set(x_1, 1, x_21); -lean_ctor_set(x_1, 0, x_22); -x_10 = x_17; +x_25 = lean_ctor_get(x_23, 0); +lean_inc(x_25); +lean_dec(x_23); +lean_ctor_set(x_1, 1, x_24); +lean_ctor_set(x_1, 0, x_25); +x_10 = x_20; goto _start; } } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_24 = lean_ctor_get(x_14, 0); -x_25 = lean_ctor_get(x_14, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_14); -x_26 = lean_ctor_get(x_24, 7); -lean_inc(x_26); -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_24, 4); +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_27 = lean_ctor_get(x_17, 0); +x_28 = lean_ctor_get(x_17, 1); lean_inc(x_28); -lean_dec(x_24); -x_29 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_13, x_26, x_27); -if (lean_obj_tag(x_28) == 0) +lean_inc(x_27); +lean_dec(x_17); +x_29 = lean_ctor_get(x_27, 7); +lean_inc(x_29); +x_30 = lean_ctor_get(x_27, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_27, 4); +lean_inc(x_31); +lean_dec(x_27); +x_32 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_13, x_29, x_30); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_30; -lean_ctor_set(x_1, 1, x_29); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_1); -lean_ctor_set(x_30, 1, x_25); -return x_30; +lean_object* x_33; +lean_ctor_set(x_1, 1, x_32); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_1); +lean_ctor_set(x_33, 1, x_28); +return x_33; } else { -lean_object* x_31; +lean_object* x_34; lean_dec(x_12); -x_31 = lean_ctor_get(x_28, 0); -lean_inc(x_31); -lean_dec(x_28); -lean_ctor_set(x_1, 1, x_29); -lean_ctor_set(x_1, 0, x_31); -x_10 = x_25; +x_34 = lean_ctor_get(x_31, 0); +lean_inc(x_34); +lean_dec(x_31); +lean_ctor_set(x_1, 1, x_32); +lean_ctor_set(x_1, 0, x_34); +x_10 = x_28; goto _start; } } } else { -uint8_t x_33; +uint8_t x_36; lean_free_object(x_1); lean_dec(x_13); lean_dec(x_12); -x_33 = !lean_is_exclusive(x_14); -if (x_33 == 0) +x_36 = !lean_is_exclusive(x_17); +if (x_36 == 0) { -return x_14; +return x_17; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_14, 0); -x_35 = lean_ctor_get(x_14, 1); -lean_inc(x_35); -lean_inc(x_34); -lean_dec(x_14); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_17, 0); +x_38 = lean_ctor_get(x_17, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_17); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_1, 0); -x_38 = lean_ctor_get(x_1, 1); -lean_inc(x_38); -lean_inc(x_37); -lean_dec(x_1); -lean_inc(x_37); -x_39 = l_Lean_Meta_Grind_getENode(x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); +lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_40 = lean_ctor_get(x_1, 0); +x_41 = lean_ctor_get(x_1, 1); lean_inc(x_41); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_42 = x_39; -} else { - lean_dec_ref(x_39); - x_42 = lean_box(0); -} -x_43 = lean_ctor_get(x_40, 7); +lean_inc(x_40); +lean_dec(x_1); +x_42 = lean_st_ref_get(x_2, x_10); +x_43 = lean_ctor_get(x_42, 0); lean_inc(x_43); -x_44 = lean_ctor_get(x_40, 0); +x_44 = lean_ctor_get(x_42, 1); lean_inc(x_44); -x_45 = lean_ctor_get(x_40, 4); -lean_inc(x_45); -lean_dec(x_40); -x_46 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_38, x_43, x_44); +lean_dec(x_42); +lean_inc(x_40); +x_45 = l_Lean_Meta_Grind_Goal_getENode(x_43, x_40, x_8, x_9, x_44); if (lean_obj_tag(x_45) == 0) { -lean_object* x_47; lean_object* x_48; -x_47 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_47, 0, x_37); -lean_ctor_set(x_47, 1, x_46); -if (lean_is_scalar(x_42)) { - x_48 = lean_alloc_ctor(0, 2, 0); +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_48 = x_45; } else { - x_48 = x_42; + lean_dec_ref(x_45); + x_48 = lean_box(0); } -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_41); -return x_48; +x_49 = lean_ctor_get(x_46, 7); +lean_inc(x_49); +x_50 = lean_ctor_get(x_46, 0); +lean_inc(x_50); +x_51 = lean_ctor_get(x_46, 4); +lean_inc(x_51); +lean_dec(x_46); +x_52 = l_Lean_RBNode_insert___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__1(x_41, x_49, x_50); +if (lean_obj_tag(x_51) == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_40); +lean_ctor_set(x_53, 1, x_52); +if (lean_is_scalar(x_48)) { + x_54 = lean_alloc_ctor(0, 2, 0); +} else { + x_54 = x_48; +} +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_47); +return x_54; } else { -lean_object* x_49; lean_object* x_50; -lean_dec(x_42); -lean_dec(x_37); -x_49 = lean_ctor_get(x_45, 0); -lean_inc(x_49); -lean_dec(x_45); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_46); -x_1 = x_50; -x_10 = x_41; +lean_object* x_55; lean_object* x_56; +lean_dec(x_48); +lean_dec(x_40); +x_55 = lean_ctor_get(x_51, 0); +lean_inc(x_55); +lean_dec(x_51); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_52); +x_1 = x_56; +x_10 = x_47; goto _start; } } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -lean_dec(x_38); -lean_dec(x_37); -x_52 = lean_ctor_get(x_39, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_39, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_54 = x_39; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_41); +lean_dec(x_40); +x_58 = lean_ctor_get(x_45, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_45, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_60 = x_45; } else { - lean_dec_ref(x_39); - x_54 = lean_box(0); + lean_dec_ref(x_45); + x_60 = lean_box(0); } -if (lean_is_scalar(x_54)) { - x_55 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); } else { - x_55 = x_54; + x_61 = x_60; } -lean_ctor_set(x_55, 0, x_52); -lean_ctor_set(x_55, 1, x_53); -return x_55; +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; } } } @@ -3733,31 +3757,37 @@ uint8_t x_14; x_14 = !lean_is_exclusive(x_4); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; x_15 = lean_ctor_get(x_4, 1); x_16 = lean_ctor_get(x_4, 0); lean_dec(x_16); +x_17 = lean_st_ref_get(x_5, x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); lean_inc(x_15); -x_17 = l_Lean_Meta_Grind_getENode(x_15, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_17) == 0) +x_20 = l_Lean_Meta_Grind_Goal_getENode(x_18, x_15, x_11, x_12, x_19); +if (lean_obj_tag(x_20) == 0) { -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_20); +if (x_21 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -x_21 = lean_ctor_get(x_19, 7); -lean_inc(x_21); -x_22 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_21); -lean_dec(x_21); -if (lean_obj_tag(x_22) == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_22 = lean_ctor_get(x_20, 0); +x_23 = lean_ctor_get(x_20, 1); +x_24 = lean_ctor_get(x_22, 7); +lean_inc(x_24); +x_25 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_24); +lean_dec(x_24); +if (lean_obj_tag(x_25) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_17); +lean_object* x_26; lean_object* x_27; +lean_free_object(x_20); lean_free_object(x_4); -x_23 = lean_box(0); +x_26 = lean_box(0); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -3767,15 +3797,15 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_24 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_19, x_3, x_15, x_23, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); -if (lean_obj_tag(x_24) == 0) +x_27 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_22, x_3, x_15, x_26, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_25; -x_25 = lean_ctor_get(x_24, 0); -lean_inc(x_25); -if (lean_obj_tag(x_25) == 0) +lean_object* x_28; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +if (lean_obj_tag(x_28) == 0) { -uint8_t x_26; +uint8_t x_29; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3785,50 +3815,50 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) +x_29 = !lean_is_exclusive(x_27); +if (x_29 == 0) { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -x_28 = lean_ctor_get(x_25, 0); -lean_inc(x_28); -lean_dec(x_25); -lean_ctor_set(x_24, 0, x_28); -return x_24; +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 0); +lean_dec(x_30); +x_31 = lean_ctor_get(x_28, 0); +lean_inc(x_31); +lean_dec(x_28); +lean_ctor_set(x_27, 0, x_31); +return x_27; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_24, 1); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_ctor_get(x_25, 0); -lean_inc(x_30); -lean_dec(x_25); -x_31 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_29); -return x_31; +lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_27, 1); +lean_inc(x_32); +lean_dec(x_27); +x_33 = lean_ctor_get(x_28, 0); +lean_inc(x_33); +lean_dec(x_28); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_32); +return x_34; } } else { -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_24, 1); -lean_inc(x_32); -lean_dec(x_24); -x_33 = lean_ctor_get(x_25, 0); -lean_inc(x_33); -lean_dec(x_25); -x_4 = x_33; -x_13 = x_32; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_27, 1); +lean_inc(x_35); +lean_dec(x_27); +x_36 = lean_ctor_get(x_28, 0); +lean_inc(x_36); +lean_dec(x_28); +x_4 = x_36; +x_13 = x_35; goto _start; } } else { -uint8_t x_35; +uint8_t x_38; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3837,31 +3867,31 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_3); -x_35 = !lean_is_exclusive(x_24); -if (x_35 == 0) -{ -return x_24; -} -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_24, 0); -x_37 = lean_ctor_get(x_24, 1); -lean_inc(x_37); -lean_inc(x_36); -lean_dec(x_24); -x_38 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_dec(x_3); +x_38 = !lean_is_exclusive(x_27); +if (x_38 == 0) +{ +return x_27; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_27, 0); +x_40 = lean_ctor_get(x_27, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_27); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } } else { -uint8_t x_39; -lean_dec(x_19); +uint8_t x_42; +lean_dec(x_22); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3871,44 +3901,44 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_39 = !lean_is_exclusive(x_22); -if (x_39 == 0) +x_42 = !lean_is_exclusive(x_25); +if (x_42 == 0) { -lean_ctor_set(x_4, 0, x_22); -lean_ctor_set(x_17, 0, x_4); -return x_17; +lean_ctor_set(x_4, 0, x_25); +lean_ctor_set(x_20, 0, x_4); +return x_20; } else { -lean_object* x_40; lean_object* x_41; -x_40 = lean_ctor_get(x_22, 0); -lean_inc(x_40); -lean_dec(x_22); -x_41 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_4, 0, x_41); -lean_ctor_set(x_17, 0, x_4); -return x_17; +lean_object* x_43; lean_object* x_44; +x_43 = lean_ctor_get(x_25, 0); +lean_inc(x_43); +lean_dec(x_25); +x_44 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_4, 0, x_44); +lean_ctor_set(x_20, 0, x_4); +return x_20; } } } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_42 = lean_ctor_get(x_17, 0); -x_43 = lean_ctor_get(x_17, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_17); -x_44 = lean_ctor_get(x_42, 7); -lean_inc(x_44); -x_45 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_44); -lean_dec(x_44); -if (lean_obj_tag(x_45) == 0) +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_45 = lean_ctor_get(x_20, 0); +x_46 = lean_ctor_get(x_20, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_20); +x_47 = lean_ctor_get(x_45, 7); +lean_inc(x_47); +x_48 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_47); +lean_dec(x_47); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_46; lean_object* x_47; +lean_object* x_49; lean_object* x_50; lean_free_object(x_4); -x_46 = lean_box(0); +x_49 = lean_box(0); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -3918,15 +3948,15 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_47 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_42, x_3, x_15, x_46, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_43); -if (lean_obj_tag(x_47) == 0) +x_50 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_45, x_3, x_15, x_49, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_46); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_48; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -if (lean_obj_tag(x_48) == 0) +lean_object* x_51; +x_51 = lean_ctor_get(x_50, 0); +lean_inc(x_51); +if (lean_obj_tag(x_51) == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3936,45 +3966,45 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_50 = x_47; +x_52 = lean_ctor_get(x_50, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_53 = x_50; } else { - lean_dec_ref(x_47); - x_50 = lean_box(0); + lean_dec_ref(x_50); + x_53 = lean_box(0); } -x_51 = lean_ctor_get(x_48, 0); -lean_inc(x_51); -lean_dec(x_48); -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); +x_54 = lean_ctor_get(x_51, 0); +lean_inc(x_54); +lean_dec(x_51); +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); } else { - x_52 = x_50; + x_55 = x_53; } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } else { -lean_object* x_53; lean_object* x_54; -x_53 = lean_ctor_get(x_47, 1); -lean_inc(x_53); -lean_dec(x_47); -x_54 = lean_ctor_get(x_48, 0); -lean_inc(x_54); -lean_dec(x_48); -x_4 = x_54; -x_13 = x_53; +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_50, 1); +lean_inc(x_56); +lean_dec(x_50); +x_57 = lean_ctor_get(x_51, 0); +lean_inc(x_57); +lean_dec(x_51); +x_4 = x_57; +x_13 = x_56; goto _start; } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -3984,32 +4014,32 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_56 = lean_ctor_get(x_47, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_47, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_58 = x_47; +x_59 = lean_ctor_get(x_50, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_50, 1); +lean_inc(x_60); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_61 = x_50; } else { - lean_dec_ref(x_47); - x_58 = lean_box(0); + lean_dec_ref(x_50); + x_61 = lean_box(0); } -if (lean_is_scalar(x_58)) { - x_59 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_61)) { + x_62 = lean_alloc_ctor(1, 2, 0); } else { - x_59 = x_58; + x_62 = x_61; } -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_57); -return x_59; +lean_ctor_set(x_62, 0, x_59); +lean_ctor_set(x_62, 1, x_60); +return x_62; } } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; -lean_dec(x_42); +lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +lean_dec(x_45); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4019,32 +4049,32 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_60 = lean_ctor_get(x_45, 0); -lean_inc(x_60); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - x_61 = x_45; +x_63 = lean_ctor_get(x_48, 0); +lean_inc(x_63); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + x_64 = x_48; } else { - lean_dec_ref(x_45); - x_61 = lean_box(0); + lean_dec_ref(x_48); + x_64 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(1, 1, 0); } else { - x_62 = x_61; + x_65 = x_64; } -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_4, 0, x_62); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_4); -lean_ctor_set(x_63, 1, x_43); -return x_63; +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_4, 0, x_65); +x_66 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_66, 0, x_4); +lean_ctor_set(x_66, 1, x_46); +return x_66; } } } else { -uint8_t x_64; +uint8_t x_67; lean_free_object(x_4); lean_dec(x_15); lean_dec(x_12); @@ -4056,58 +4086,64 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_64 = !lean_is_exclusive(x_17); -if (x_64 == 0) +x_67 = !lean_is_exclusive(x_20); +if (x_67 == 0) { -return x_17; +return x_20; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_17, 0); -x_66 = lean_ctor_get(x_17, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_17); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_20, 0); +x_69 = lean_ctor_get(x_20, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_20); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } } else { -lean_object* x_68; lean_object* x_69; -x_68 = lean_ctor_get(x_4, 1); -lean_inc(x_68); +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_71 = lean_ctor_get(x_4, 1); +lean_inc(x_71); lean_dec(x_4); -lean_inc(x_68); -x_69 = l_Lean_Meta_Grind_getENode(x_68, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); -if (lean_obj_tag(x_69) == 0) -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_70 = lean_ctor_get(x_69, 0); -lean_inc(x_70); -x_71 = lean_ctor_get(x_69, 1); +x_72 = lean_st_ref_get(x_5, x_13); +x_73 = lean_ctor_get(x_72, 0); +lean_inc(x_73); +x_74 = lean_ctor_get(x_72, 1); +lean_inc(x_74); +lean_dec(x_72); lean_inc(x_71); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_72 = x_69; +x_75 = l_Lean_Meta_Grind_Goal_getENode(x_73, x_71, x_11, x_12, x_74); +if (lean_obj_tag(x_75) == 0) +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_76 = lean_ctor_get(x_75, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_75, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_78 = x_75; } else { - lean_dec_ref(x_69); - x_72 = lean_box(0); + lean_dec_ref(x_75); + x_78 = lean_box(0); } -x_73 = lean_ctor_get(x_70, 7); -lean_inc(x_73); -x_74 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_73); -lean_dec(x_73); -if (lean_obj_tag(x_74) == 0) +x_79 = lean_ctor_get(x_76, 7); +lean_inc(x_79); +x_80 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_2, x_79); +lean_dec(x_79); +if (lean_obj_tag(x_80) == 0) { -lean_object* x_75; lean_object* x_76; -lean_dec(x_72); -x_75 = lean_box(0); +lean_object* x_81; lean_object* x_82; +lean_dec(x_78); +x_81 = lean_box(0); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -4117,15 +4153,15 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_3); -x_76 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_70, x_3, x_68, x_75, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_71); -if (lean_obj_tag(x_76) == 0) +x_82 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_76, x_3, x_71, x_81, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_77); +if (lean_obj_tag(x_82) == 0) { -lean_object* x_77; -x_77 = lean_ctor_get(x_76, 0); -lean_inc(x_77); -if (lean_obj_tag(x_77) == 0) +lean_object* x_83; +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +if (lean_obj_tag(x_83) == 0) { -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4135,45 +4171,45 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_78 = lean_ctor_get(x_76, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_79 = x_76; +x_84 = lean_ctor_get(x_82, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + x_85 = x_82; } else { - lean_dec_ref(x_76); - x_79 = lean_box(0); + lean_dec_ref(x_82); + x_85 = lean_box(0); } -x_80 = lean_ctor_get(x_77, 0); -lean_inc(x_80); -lean_dec(x_77); -if (lean_is_scalar(x_79)) { - x_81 = lean_alloc_ctor(0, 2, 0); +x_86 = lean_ctor_get(x_83, 0); +lean_inc(x_86); +lean_dec(x_83); +if (lean_is_scalar(x_85)) { + x_87 = lean_alloc_ctor(0, 2, 0); } else { - x_81 = x_79; + x_87 = x_85; } -lean_ctor_set(x_81, 0, x_80); -lean_ctor_set(x_81, 1, x_78); -return x_81; +lean_ctor_set(x_87, 0, x_86); +lean_ctor_set(x_87, 1, x_84); +return x_87; } else { -lean_object* x_82; lean_object* x_83; -x_82 = lean_ctor_get(x_76, 1); -lean_inc(x_82); -lean_dec(x_76); -x_83 = lean_ctor_get(x_77, 0); -lean_inc(x_83); -lean_dec(x_77); -x_4 = x_83; -x_13 = x_82; +lean_object* x_88; lean_object* x_89; +x_88 = lean_ctor_get(x_82, 1); +lean_inc(x_88); +lean_dec(x_82); +x_89 = lean_ctor_get(x_83, 0); +lean_inc(x_89); +lean_dec(x_83); +x_4 = x_89; +x_13 = x_88; goto _start; } } else { -lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4183,32 +4219,32 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_85 = lean_ctor_get(x_76, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_76, 1); -lean_inc(x_86); -if (lean_is_exclusive(x_76)) { - lean_ctor_release(x_76, 0); - lean_ctor_release(x_76, 1); - x_87 = x_76; +x_91 = lean_ctor_get(x_82, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_82, 1); +lean_inc(x_92); +if (lean_is_exclusive(x_82)) { + lean_ctor_release(x_82, 0); + lean_ctor_release(x_82, 1); + x_93 = x_82; } else { - lean_dec_ref(x_76); - x_87 = lean_box(0); + lean_dec_ref(x_82); + x_93 = lean_box(0); } -if (lean_is_scalar(x_87)) { - x_88 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_93)) { + x_94 = lean_alloc_ctor(1, 2, 0); } else { - x_88 = x_87; + x_94 = x_93; } -lean_ctor_set(x_88, 0, x_85); -lean_ctor_set(x_88, 1, x_86); -return x_88; +lean_ctor_set(x_94, 0, x_91); +lean_ctor_set(x_94, 1, x_92); +return x_94; } } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; -lean_dec(x_70); +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; +lean_dec(x_76); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4218,38 +4254,38 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_89 = lean_ctor_get(x_74, 0); -lean_inc(x_89); -if (lean_is_exclusive(x_74)) { - lean_ctor_release(x_74, 0); - x_90 = x_74; +x_95 = lean_ctor_get(x_80, 0); +lean_inc(x_95); +if (lean_is_exclusive(x_80)) { + lean_ctor_release(x_80, 0); + x_96 = x_80; } else { - lean_dec_ref(x_74); - x_90 = lean_box(0); + lean_dec_ref(x_80); + x_96 = lean_box(0); } -if (lean_is_scalar(x_90)) { - x_91 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_96)) { + x_97 = lean_alloc_ctor(1, 1, 0); } else { - x_91 = x_90; + x_97 = x_96; } -lean_ctor_set(x_91, 0, x_89); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_68); -if (lean_is_scalar(x_72)) { - x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_95); +x_98 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_71); +if (lean_is_scalar(x_78)) { + x_99 = lean_alloc_ctor(0, 2, 0); } else { - x_93 = x_72; + x_99 = x_78; } -lean_ctor_set(x_93, 0, x_92); -lean_ctor_set(x_93, 1, x_71); -return x_93; +lean_ctor_set(x_99, 0, x_98); +lean_ctor_set(x_99, 1, x_77); +return x_99; } } else { -lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -lean_dec(x_68); +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; +lean_dec(x_71); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4259,26 +4295,26 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); -x_94 = lean_ctor_get(x_69, 0); -lean_inc(x_94); -x_95 = lean_ctor_get(x_69, 1); -lean_inc(x_95); -if (lean_is_exclusive(x_69)) { - lean_ctor_release(x_69, 0); - lean_ctor_release(x_69, 1); - x_96 = x_69; +x_100 = lean_ctor_get(x_75, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_75, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_75)) { + lean_ctor_release(x_75, 0); + lean_ctor_release(x_75, 1); + x_102 = x_75; } else { - lean_dec_ref(x_69); - x_96 = lean_box(0); + lean_dec_ref(x_75); + x_102 = lean_box(0); } -if (lean_is_scalar(x_96)) { - x_97 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_102)) { + x_103 = lean_alloc_ctor(1, 2, 0); } else { - x_97 = x_96; + x_103 = x_102; } -lean_ctor_set(x_97, 0, x_94); -lean_ctor_set(x_97, 1, x_95); -return x_97; +lean_ctor_set(x_103, 0, x_100); +lean_ctor_set(x_103, 1, x_101); +return x_103; } } } @@ -4290,31 +4326,37 @@ uint8_t x_13; x_13 = !lean_is_exclusive(x_3); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; x_14 = lean_ctor_get(x_3, 1); x_15 = lean_ctor_get(x_3, 0); lean_dec(x_15); +x_16 = lean_st_ref_get(x_4, x_12); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); lean_inc(x_14); -x_16 = l_Lean_Meta_Grind_getENode(x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_16) == 0) +x_19 = l_Lean_Meta_Grind_Goal_getENode(x_17, x_14, x_10, x_11, x_18); +if (lean_obj_tag(x_19) == 0) { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_20; +x_20 = !lean_is_exclusive(x_19); +if (x_20 == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -x_20 = lean_ctor_get(x_18, 7); -lean_inc(x_20); -x_21 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_20); -lean_dec(x_20); -if (lean_obj_tag(x_21) == 0) +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_19, 0); +x_22 = lean_ctor_get(x_19, 1); +x_23 = lean_ctor_get(x_21, 7); +lean_inc(x_23); +x_24 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_23); +lean_dec(x_23); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_22; lean_object* x_23; -lean_free_object(x_16); +lean_object* x_25; lean_object* x_26; +lean_free_object(x_19); lean_free_object(x_3); -x_22 = lean_box(0); +x_25 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -4324,15 +4366,15 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_23 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_18, x_2, x_14, x_22, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_19); -if (lean_obj_tag(x_23) == 0) +x_26 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_21, x_2, x_14, x_25, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_24; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -if (lean_obj_tag(x_24) == 0) +lean_object* x_27; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +if (lean_obj_tag(x_27) == 0) { -uint8_t x_25; +uint8_t x_28; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4342,50 +4384,50 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_25 = !lean_is_exclusive(x_23); -if (x_25 == 0) +x_28 = !lean_is_exclusive(x_26); +if (x_28 == 0) { -lean_object* x_26; lean_object* x_27; -x_26 = lean_ctor_get(x_23, 0); -lean_dec(x_26); -x_27 = lean_ctor_get(x_24, 0); -lean_inc(x_27); -lean_dec(x_24); -lean_ctor_set(x_23, 0, x_27); -return x_23; +lean_object* x_29; lean_object* x_30; +x_29 = lean_ctor_get(x_26, 0); +lean_dec(x_29); +x_30 = lean_ctor_get(x_27, 0); +lean_inc(x_30); +lean_dec(x_27); +lean_ctor_set(x_26, 0, x_30); +return x_26; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_23, 1); -lean_inc(x_28); -lean_dec(x_23); -x_29 = lean_ctor_get(x_24, 0); -lean_inc(x_29); -lean_dec(x_24); -x_30 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -return x_30; +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_26, 1); +lean_inc(x_31); +lean_dec(x_26); +x_32 = lean_ctor_get(x_27, 0); +lean_inc(x_32); +lean_dec(x_27); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +return x_33; } } else { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_23, 1); -lean_inc(x_31); -lean_dec(x_23); -x_32 = lean_ctor_get(x_24, 0); -lean_inc(x_32); -lean_dec(x_24); -x_3 = x_32; -x_12 = x_31; +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_26, 1); +lean_inc(x_34); +lean_dec(x_26); +x_35 = lean_ctor_get(x_27, 0); +lean_inc(x_35); +lean_dec(x_27); +x_3 = x_35; +x_12 = x_34; goto _start; } } else { -uint8_t x_34; +uint8_t x_37; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4395,30 +4437,30 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_34 = !lean_is_exclusive(x_23); -if (x_34 == 0) +x_37 = !lean_is_exclusive(x_26); +if (x_37 == 0) { -return x_23; +return x_26; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_23, 0); -x_36 = lean_ctor_get(x_23, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_23); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_26, 0); +x_39 = lean_ctor_get(x_26, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_26); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } } else { -uint8_t x_38; -lean_dec(x_18); +uint8_t x_41; +lean_dec(x_21); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4428,44 +4470,44 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_38 = !lean_is_exclusive(x_21); -if (x_38 == 0) +x_41 = !lean_is_exclusive(x_24); +if (x_41 == 0) { -lean_ctor_set(x_3, 0, x_21); -lean_ctor_set(x_16, 0, x_3); -return x_16; +lean_ctor_set(x_3, 0, x_24); +lean_ctor_set(x_19, 0, x_3); +return x_19; } else { -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_21, 0); -lean_inc(x_39); -lean_dec(x_21); -x_40 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_3, 0, x_40); -lean_ctor_set(x_16, 0, x_3); -return x_16; +lean_object* x_42; lean_object* x_43; +x_42 = lean_ctor_get(x_24, 0); +lean_inc(x_42); +lean_dec(x_24); +x_43 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_3, 0, x_43); +lean_ctor_set(x_19, 0, x_3); +return x_19; } } } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_41 = lean_ctor_get(x_16, 0); -x_42 = lean_ctor_get(x_16, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_16); -x_43 = lean_ctor_get(x_41, 7); -lean_inc(x_43); -x_44 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_43); -lean_dec(x_43); -if (lean_obj_tag(x_44) == 0) +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_44 = lean_ctor_get(x_19, 0); +x_45 = lean_ctor_get(x_19, 1); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_19); +x_46 = lean_ctor_get(x_44, 7); +lean_inc(x_46); +x_47 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_46); +lean_dec(x_46); +if (lean_obj_tag(x_47) == 0) { -lean_object* x_45; lean_object* x_46; +lean_object* x_48; lean_object* x_49; lean_free_object(x_3); -x_45 = lean_box(0); +x_48 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -4475,15 +4517,15 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_46 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_41, x_2, x_14, x_45, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_42); -if (lean_obj_tag(x_46) == 0) +x_49 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_44, x_2, x_14, x_48, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_45); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_47; -x_47 = lean_ctor_get(x_46, 0); -lean_inc(x_47); -if (lean_obj_tag(x_47) == 0) +lean_object* x_50; +x_50 = lean_ctor_get(x_49, 0); +lean_inc(x_50); +if (lean_obj_tag(x_50) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4493,45 +4535,45 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_49 = x_46; +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_52 = x_49; } else { - lean_dec_ref(x_46); - x_49 = lean_box(0); + lean_dec_ref(x_49); + x_52 = lean_box(0); } -x_50 = lean_ctor_get(x_47, 0); -lean_inc(x_50); -lean_dec(x_47); -if (lean_is_scalar(x_49)) { - x_51 = lean_alloc_ctor(0, 2, 0); +x_53 = lean_ctor_get(x_50, 0); +lean_inc(x_53); +lean_dec(x_50); +if (lean_is_scalar(x_52)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_49; + x_54 = x_52; } -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_48); -return x_51; +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_51); +return x_54; } else { -lean_object* x_52; lean_object* x_53; -x_52 = lean_ctor_get(x_46, 1); -lean_inc(x_52); -lean_dec(x_46); -x_53 = lean_ctor_get(x_47, 0); -lean_inc(x_53); -lean_dec(x_47); -x_3 = x_53; -x_12 = x_52; +lean_object* x_55; lean_object* x_56; +x_55 = lean_ctor_get(x_49, 1); +lean_inc(x_55); +lean_dec(x_49); +x_56 = lean_ctor_get(x_50, 0); +lean_inc(x_56); +lean_dec(x_50); +x_3 = x_56; +x_12 = x_55; goto _start; } } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4541,32 +4583,32 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_55 = lean_ctor_get(x_46, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_46, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_46)) { - lean_ctor_release(x_46, 0); - lean_ctor_release(x_46, 1); - x_57 = x_46; +x_58 = lean_ctor_get(x_49, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_49, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_49)) { + lean_ctor_release(x_49, 0); + lean_ctor_release(x_49, 1); + x_60 = x_49; } else { - lean_dec_ref(x_46); - x_57 = lean_box(0); + lean_dec_ref(x_49); + x_60 = lean_box(0); } -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); } else { - x_58 = x_57; + x_61 = x_60; } -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; } } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -lean_dec(x_41); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_44); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4576,32 +4618,32 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_59 = lean_ctor_get(x_44, 0); -lean_inc(x_59); -if (lean_is_exclusive(x_44)) { - lean_ctor_release(x_44, 0); - x_60 = x_44; +x_62 = lean_ctor_get(x_47, 0); +lean_inc(x_62); +if (lean_is_exclusive(x_47)) { + lean_ctor_release(x_47, 0); + x_63 = x_47; } else { - lean_dec_ref(x_44); - x_60 = lean_box(0); + lean_dec_ref(x_47); + x_63 = lean_box(0); } -if (lean_is_scalar(x_60)) { - x_61 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_63)) { + x_64 = lean_alloc_ctor(1, 1, 0); } else { - x_61 = x_60; + x_64 = x_63; } -lean_ctor_set(x_61, 0, x_59); -lean_ctor_set(x_3, 0, x_61); -x_62 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_62, 0, x_3); -lean_ctor_set(x_62, 1, x_42); -return x_62; +lean_ctor_set(x_64, 0, x_62); +lean_ctor_set(x_3, 0, x_64); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_3); +lean_ctor_set(x_65, 1, x_45); +return x_65; } } } else { -uint8_t x_63; +uint8_t x_66; lean_free_object(x_3); lean_dec(x_14); lean_dec(x_11); @@ -4613,58 +4655,64 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_63 = !lean_is_exclusive(x_16); -if (x_63 == 0) +x_66 = !lean_is_exclusive(x_19); +if (x_66 == 0) { -return x_16; +return x_19; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_16, 0); -x_65 = lean_ctor_get(x_16, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_16); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_19, 0); +x_68 = lean_ctor_get(x_19, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_19); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; } } } else { -lean_object* x_67; lean_object* x_68; -x_67 = lean_ctor_get(x_3, 1); -lean_inc(x_67); +lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_70 = lean_ctor_get(x_3, 1); +lean_inc(x_70); lean_dec(x_3); -lean_inc(x_67); -x_68 = l_Lean_Meta_Grind_getENode(x_67, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_68) == 0) -{ -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_69 = lean_ctor_get(x_68, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_68, 1); +x_71 = lean_st_ref_get(x_4, x_12); +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); lean_inc(x_70); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_71 = x_68; +x_74 = l_Lean_Meta_Grind_Goal_getENode(x_72, x_70, x_10, x_11, x_73); +if (lean_obj_tag(x_74) == 0) +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_77 = x_74; } else { - lean_dec_ref(x_68); - x_71 = lean_box(0); + lean_dec_ref(x_74); + x_77 = lean_box(0); } -x_72 = lean_ctor_get(x_69, 7); -lean_inc(x_72); -x_73 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_72); -lean_dec(x_72); -if (lean_obj_tag(x_73) == 0) +x_78 = lean_ctor_get(x_75, 7); +lean_inc(x_78); +x_79 = l_Lean_RBNode_find___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__6(x_1, x_78); +lean_dec(x_78); +if (lean_obj_tag(x_79) == 0) { -lean_object* x_74; lean_object* x_75; -lean_dec(x_71); -x_74 = lean_box(0); +lean_object* x_80; lean_object* x_81; +lean_dec(x_77); +x_80 = lean_box(0); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -4674,15 +4722,15 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_75 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_69, x_2, x_67, x_74, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_70); -if (lean_obj_tag(x_75) == 0) +x_81 = l_Lean_Loop_forIn_loop___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__7___lambda__1(x_75, x_2, x_70, x_80, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_76); +if (lean_obj_tag(x_81) == 0) { -lean_object* x_76; -x_76 = lean_ctor_get(x_75, 0); -lean_inc(x_76); -if (lean_obj_tag(x_76) == 0) +lean_object* x_82; +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +if (lean_obj_tag(x_82) == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4692,45 +4740,45 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_77 = lean_ctor_get(x_75, 1); -lean_inc(x_77); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_78 = x_75; +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_84 = x_81; } else { - lean_dec_ref(x_75); - x_78 = lean_box(0); + lean_dec_ref(x_81); + x_84 = lean_box(0); } -x_79 = lean_ctor_get(x_76, 0); -lean_inc(x_79); -lean_dec(x_76); -if (lean_is_scalar(x_78)) { - x_80 = lean_alloc_ctor(0, 2, 0); +x_85 = lean_ctor_get(x_82, 0); +lean_inc(x_85); +lean_dec(x_82); +if (lean_is_scalar(x_84)) { + x_86 = lean_alloc_ctor(0, 2, 0); } else { - x_80 = x_78; + x_86 = x_84; } -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_77); -return x_80; +lean_ctor_set(x_86, 0, x_85); +lean_ctor_set(x_86, 1, x_83); +return x_86; } else { -lean_object* x_81; lean_object* x_82; -x_81 = lean_ctor_get(x_75, 1); -lean_inc(x_81); -lean_dec(x_75); -x_82 = lean_ctor_get(x_76, 0); -lean_inc(x_82); -lean_dec(x_76); -x_3 = x_82; -x_12 = x_81; +lean_object* x_87; lean_object* x_88; +x_87 = lean_ctor_get(x_81, 1); +lean_inc(x_87); +lean_dec(x_81); +x_88 = lean_ctor_get(x_82, 0); +lean_inc(x_88); +lean_dec(x_82); +x_3 = x_88; +x_12 = x_87; goto _start; } } else { -lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4740,32 +4788,32 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_84 = lean_ctor_get(x_75, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_75, 1); -lean_inc(x_85); -if (lean_is_exclusive(x_75)) { - lean_ctor_release(x_75, 0); - lean_ctor_release(x_75, 1); - x_86 = x_75; +x_90 = lean_ctor_get(x_81, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_81, 1); +lean_inc(x_91); +if (lean_is_exclusive(x_81)) { + lean_ctor_release(x_81, 0); + lean_ctor_release(x_81, 1); + x_92 = x_81; } else { - lean_dec_ref(x_75); - x_86 = lean_box(0); + lean_dec_ref(x_81); + x_92 = lean_box(0); } -if (lean_is_scalar(x_86)) { - x_87 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_92)) { + x_93 = lean_alloc_ctor(1, 2, 0); } else { - x_87 = x_86; + x_93 = x_92; } -lean_ctor_set(x_87, 0, x_84); -lean_ctor_set(x_87, 1, x_85); -return x_87; +lean_ctor_set(x_93, 0, x_90); +lean_ctor_set(x_93, 1, x_91); +return x_93; } } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -lean_dec(x_69); +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; +lean_dec(x_75); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4775,38 +4823,38 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_88 = lean_ctor_get(x_73, 0); -lean_inc(x_88); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - x_89 = x_73; +x_94 = lean_ctor_get(x_79, 0); +lean_inc(x_94); +if (lean_is_exclusive(x_79)) { + lean_ctor_release(x_79, 0); + x_95 = x_79; } else { - lean_dec_ref(x_73); - x_89 = lean_box(0); + lean_dec_ref(x_79); + x_95 = lean_box(0); } -if (lean_is_scalar(x_89)) { - x_90 = lean_alloc_ctor(1, 1, 0); +if (lean_is_scalar(x_95)) { + x_96 = lean_alloc_ctor(1, 1, 0); } else { - x_90 = x_89; + x_96 = x_95; } -lean_ctor_set(x_90, 0, x_88); -x_91 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_91, 0, x_90); -lean_ctor_set(x_91, 1, x_67); -if (lean_is_scalar(x_71)) { - x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_96, 0, x_94); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_70); +if (lean_is_scalar(x_77)) { + x_98 = lean_alloc_ctor(0, 2, 0); } else { - x_92 = x_71; + x_98 = x_77; } -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_70); -return x_92; +lean_ctor_set(x_98, 0, x_97); +lean_ctor_set(x_98, 1, x_76); +return x_98; } } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_67); +lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; +lean_dec(x_70); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4816,26 +4864,26 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); -x_93 = lean_ctor_get(x_68, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_68, 1); -lean_inc(x_94); -if (lean_is_exclusive(x_68)) { - lean_ctor_release(x_68, 0); - lean_ctor_release(x_68, 1); - x_95 = x_68; +x_99 = lean_ctor_get(x_74, 0); +lean_inc(x_99); +x_100 = lean_ctor_get(x_74, 1); +lean_inc(x_100); +if (lean_is_exclusive(x_74)) { + lean_ctor_release(x_74, 0); + lean_ctor_release(x_74, 1); + x_101 = x_74; } else { - lean_dec_ref(x_68); - x_95 = lean_box(0); + lean_dec_ref(x_74); + x_101 = lean_box(0); } -if (lean_is_scalar(x_95)) { - x_96 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_101)) { + x_102 = lean_alloc_ctor(1, 2, 0); } else { - x_96 = x_95; + x_102 = x_101; } -lean_ctor_set(x_96, 0, x_93); -lean_ctor_set(x_96, 1, x_94); -return x_96; +lean_ctor_set(x_102, 0, x_99); +lean_ctor_set(x_102, 1, x_100); +return x_102; } } } @@ -5754,55 +5802,67 @@ lean_inc(x_1); x_14 = l_Lean_Meta_Grind_getRootENode(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); if (lean_obj_tag(x_14) == 0) { -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; x_15 = lean_ctor_get(x_14, 0); lean_inc(x_15); x_16 = lean_ctor_get(x_14, 1); lean_inc(x_16); lean_dec(x_14); -x_17 = lean_ctor_get_uint8(x_15, sizeof(void*)*10 + 4); +x_17 = lean_ctor_get_uint8(x_15, sizeof(void*)*11 + 4); lean_dec(x_15); -lean_inc(x_1); -x_18 = l_Lean_Meta_Grind_getENode(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_16); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_st_ref_get(x_5, x_16); x_19 = lean_ctor_get(x_18, 0); lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); lean_inc(x_20); lean_dec(x_18); -lean_inc(x_2); -x_21 = l_Lean_Meta_Grind_getENode(x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_20); +lean_inc(x_1); +x_21 = l_Lean_Meta_Grind_Goal_getENode(x_19, x_1, x_11, x_12, x_20); if (lean_obj_tag(x_21) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); x_23 = lean_ctor_get(x_21, 1); lean_inc(x_23); lean_dec(x_21); -x_24 = lean_ctor_get(x_19, 2); -lean_inc(x_24); -lean_dec(x_19); -x_25 = lean_ctor_get(x_22, 2); +x_24 = lean_st_ref_get(x_5, x_23); +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_22); -x_26 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_24, x_25); -lean_dec(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); lean_dec(x_24); -if (x_26 == 0) +lean_inc(x_2); +x_27 = l_Lean_Meta_Grind_Goal_getENode(x_25, x_2, x_11, x_12, x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_27; lean_object* x_28; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_30 = lean_ctor_get(x_22, 2); +lean_inc(x_30); +lean_dec(x_22); +x_31 = lean_ctor_get(x_28, 2); +lean_inc(x_31); +lean_dec(x_28); +x_32 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_30, x_31); +lean_dec(x_31); +lean_dec(x_30); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_dec(x_2); lean_dec(x_1); -x_27 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqProofCore___lambda__1___closed__5; -x_28 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__9(x_27, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); -return x_28; +x_33 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqProofCore___lambda__1___closed__5; +x_34 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__9(x_33, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_29); +return x_34; } else { -lean_object* x_29; +lean_object* x_35; lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -5813,16 +5873,16 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_2); lean_inc(x_1); -x_29 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_23); -if (lean_obj_tag(x_29) == 0) +x_35 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon(x_1, x_2, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_29); +if (lean_obj_tag(x_35) == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_ctor_get(x_29, 1); -lean_inc(x_31); -lean_dec(x_29); -x_32 = lean_box(0); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_box(0); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -5831,15 +5891,15 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_33 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_1, x_30, x_32, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_31); -if (lean_obj_tag(x_33) == 0) +x_39 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_1, x_36, x_38, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_37); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); @@ -5848,117 +5908,117 @@ lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); -x_36 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_2, x_30, x_34, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_35); -lean_dec(x_30); -if (lean_obj_tag(x_36) == 0) +x_42 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_2, x_36, x_40, x_17, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_41); +lean_dec(x_36); +if (lean_obj_tag(x_42) == 0) { -lean_object* x_37; -x_37 = lean_ctor_get(x_36, 0); -lean_inc(x_37); -if (lean_obj_tag(x_37) == 0) +lean_object* x_43; +x_43 = lean_ctor_get(x_42, 0); +lean_inc(x_43); +if (lean_obj_tag(x_43) == 0) { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_36, 1); -lean_inc(x_38); -lean_dec(x_36); -x_39 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqProofCore___lambda__1___closed__6; -x_40 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__9(x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_38); -return x_40; +lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_44 = lean_ctor_get(x_42, 1); +lean_inc(x_44); +lean_dec(x_42); +x_45 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkEqProofCore___lambda__1___closed__6; +x_46 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_findCommon___spec__9(x_45, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_44); +return x_46; } else { -lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_41 = lean_ctor_get(x_36, 1); -lean_inc(x_41); -if (lean_is_exclusive(x_36)) { - lean_ctor_release(x_36, 0); - lean_ctor_release(x_36, 1); - x_42 = x_36; +x_47 = lean_ctor_get(x_42, 1); +lean_inc(x_47); +if (lean_is_exclusive(x_42)) { + lean_ctor_release(x_42, 0); + lean_ctor_release(x_42, 1); + x_48 = x_42; } else { - lean_dec_ref(x_36); - x_42 = lean_box(0); + lean_dec_ref(x_42); + x_48 = lean_box(0); } -x_43 = lean_ctor_get(x_37, 0); -lean_inc(x_43); -lean_dec(x_37); +x_49 = lean_ctor_get(x_43, 0); +lean_inc(x_49); +lean_dec(x_43); if (x_3 == 0) { if (x_17 == 0) { -uint8_t x_49; -x_49 = 1; -x_44 = x_49; -goto block_48; +uint8_t x_55; +x_55 = 1; +x_50 = x_55; +goto block_54; } else { -uint8_t x_50; -x_50 = 0; -x_44 = x_50; -goto block_48; +uint8_t x_56; +x_56 = 0; +x_50 = x_56; +goto block_54; } } else { if (x_17 == 0) { -uint8_t x_51; -x_51 = 0; -x_44 = x_51; -goto block_48; +uint8_t x_57; +x_57 = 0; +x_50 = x_57; +goto block_54; } else { -uint8_t x_52; -x_52 = 1; -x_44 = x_52; -goto block_48; +uint8_t x_58; +x_58 = 1; +x_50 = x_58; +goto block_54; } } -block_48: +block_54: { -if (x_44 == 0) +if (x_50 == 0) { -lean_dec(x_42); +lean_dec(x_48); if (x_3 == 0) { -lean_object* x_45; -x_45 = l_Lean_Meta_mkEqOfHEq(x_43, x_9, x_10, x_11, x_12, x_41); -return x_45; +lean_object* x_51; +x_51 = l_Lean_Meta_mkEqOfHEq(x_49, x_9, x_10, x_11, x_12, x_47); +return x_51; } else { -lean_object* x_46; -x_46 = l_Lean_Meta_mkHEqOfEq(x_43, x_9, x_10, x_11, x_12, x_41); -return x_46; +lean_object* x_52; +x_52 = l_Lean_Meta_mkHEqOfEq(x_49, x_9, x_10, x_11, x_12, x_47); +return x_52; } } else { -lean_object* x_47; +lean_object* x_53; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); -if (lean_is_scalar(x_42)) { - x_47 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_48)) { + x_53 = lean_alloc_ctor(0, 2, 0); } else { - x_47 = x_42; + x_53 = x_48; } -lean_ctor_set(x_47, 0, x_43); -lean_ctor_set(x_47, 1, x_41); -return x_47; +lean_ctor_set(x_53, 0, x_49); +lean_ctor_set(x_53, 1, x_47); +return x_53; } } } } else { -uint8_t x_53; +uint8_t x_59; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -5967,30 +6027,30 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -x_53 = !lean_is_exclusive(x_36); -if (x_53 == 0) +x_59 = !lean_is_exclusive(x_42); +if (x_59 == 0) { -return x_36; +return x_42; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_36, 0); -x_55 = lean_ctor_get(x_36, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_36); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_42, 0); +x_61 = lean_ctor_get(x_42, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_42); +x_62 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_62, 0, x_60); +lean_ctor_set(x_62, 1, x_61); +return x_62; } } } else { -uint8_t x_57; -lean_dec(x_30); +uint8_t x_63; +lean_dec(x_36); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -6000,29 +6060,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); -x_57 = !lean_is_exclusive(x_33); -if (x_57 == 0) +x_63 = !lean_is_exclusive(x_39); +if (x_63 == 0) { -return x_33; +return x_39; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_33, 0); -x_59 = lean_ctor_get(x_33, 1); -lean_inc(x_59); -lean_inc(x_58); -lean_dec(x_33); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +lean_object* x_64; lean_object* x_65; lean_object* x_66; +x_64 = lean_ctor_get(x_39, 0); +x_65 = lean_ctor_get(x_39, 1); +lean_inc(x_65); +lean_inc(x_64); +lean_dec(x_39); +x_66 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_66, 0, x_64); +lean_ctor_set(x_66, 1, x_65); +return x_66; } } } else { -uint8_t x_61; +uint8_t x_67; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -6033,31 +6093,31 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_61 = !lean_is_exclusive(x_29); -if (x_61 == 0) +x_67 = !lean_is_exclusive(x_35); +if (x_67 == 0) { -return x_29; +return x_35; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_62 = lean_ctor_get(x_29, 0); -x_63 = lean_ctor_get(x_29, 1); -lean_inc(x_63); -lean_inc(x_62); -lean_dec(x_29); -x_64 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_64, 0, x_62); -lean_ctor_set(x_64, 1, x_63); -return x_64; +lean_object* x_68; lean_object* x_69; lean_object* x_70; +x_68 = lean_ctor_get(x_35, 0); +x_69 = lean_ctor_get(x_35, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_35); +x_70 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +return x_70; } } } } else { -uint8_t x_65; -lean_dec(x_19); +uint8_t x_71; +lean_dec(x_22); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -6068,29 +6128,29 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_21); -if (x_65 == 0) +x_71 = !lean_is_exclusive(x_27); +if (x_71 == 0) { -return x_21; +return x_27; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_21, 0); -x_67 = lean_ctor_get(x_21, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_21); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_27, 0); +x_73 = lean_ctor_get(x_27, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_27); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; } } } else { -uint8_t x_69; +uint8_t x_75; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -6101,29 +6161,29 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_75 = !lean_is_exclusive(x_21); +if (x_75 == 0) { -return x_18; +return x_21; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_21, 0); +x_77 = lean_ctor_get(x_21, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_21); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; } } } else { -uint8_t x_73; +uint8_t x_79; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -6134,23 +6194,23 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); -x_73 = !lean_is_exclusive(x_14); -if (x_73 == 0) +x_79 = !lean_is_exclusive(x_14); +if (x_79 == 0) { return x_14; } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_14, 0); -x_75 = lean_ctor_get(x_14, 1); -lean_inc(x_75); -lean_inc(x_74); +lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_80 = lean_ctor_get(x_14, 0); +x_81 = lean_ctor_get(x_14, 1); +lean_inc(x_81); +lean_inc(x_80); lean_dec(x_14); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; +x_82 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_82, 0, x_80); +lean_ctor_set(x_82, 1, x_81); +return x_82; } } } @@ -6280,68 +6340,74 @@ return x_6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_15; -lean_inc(x_1); -x_15 = l_Lean_Meta_Grind_getENode(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_st_ref_get(x_6, x_14); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 4); +x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); -if (lean_obj_tag(x_17) == 0) +lean_dec(x_15); +lean_inc(x_1); +x_18 = l_Lean_Meta_Grind_Goal_getENode(x_16, x_1, x_12, x_13, x_17); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_16); +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_19, 4); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_19); lean_dec(x_4); lean_dec(x_1); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1___closed__2; -x_20 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); -return x_20; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1___closed__2; +x_23 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_21); +return x_23; } else { -lean_object* x_21; -x_21 = lean_ctor_get(x_16, 5); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +lean_object* x_24; +x_24 = lean_ctor_get(x_19, 5); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_17); -lean_dec(x_16); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_20); +lean_dec(x_19); lean_dec(x_4); lean_dec(x_1); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_dec(x_15); -x_23 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1___closed__3; -x_24 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); -return x_24; +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_dec(x_18); +x_26 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___lambda__1___closed__3; +x_27 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +return x_27; } else { -uint8_t x_25; -x_25 = lean_ctor_get_uint8(x_16, sizeof(void*)*10); -lean_dec(x_16); -if (x_25 == 0) -{ -lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = lean_ctor_get(x_15, 1); -lean_inc(x_26); -lean_dec(x_15); -x_27 = lean_ctor_get(x_17, 0); -lean_inc(x_27); -lean_dec(x_17); -x_28 = !lean_is_exclusive(x_21); +uint8_t x_28; +x_28 = lean_ctor_get_uint8(x_19, sizeof(void*)*11); +lean_dec(x_19); if (x_28 == 0) { -lean_object* x_29; uint8_t x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_21, 0); -x_30 = 1; +lean_object* x_29; lean_object* x_30; uint8_t x_31; +x_29 = lean_ctor_get(x_18, 1); +lean_inc(x_29); +lean_dec(x_18); +x_30 = lean_ctor_get(x_20, 0); +lean_inc(x_30); +lean_dec(x_20); +x_31 = !lean_is_exclusive(x_24); +if (x_31 == 0) +{ +lean_object* x_32; uint8_t x_33; lean_object* x_34; +x_32 = lean_ctor_get(x_24, 0); +x_33 = 1; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6350,21 +6416,8 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_27); -x_31 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_27, x_1, x_29, x_30, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_26); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; -x_32 = lean_ctor_get(x_31, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_31, 1); -lean_inc(x_33); -lean_dec(x_31); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_34 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_27, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_33); +lean_inc(x_30); +x_34 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_30, x_1, x_32, x_33, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_29); if (lean_obj_tag(x_34) == 0) { lean_object* x_35; lean_object* x_36; lean_object* x_37; @@ -6373,92 +6426,105 @@ lean_inc(x_35); x_36 = lean_ctor_get(x_34, 1); lean_inc(x_36); lean_dec(x_34); -x_37 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_35, x_32, x_2, x_10, x_11, x_12, x_13, x_36); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_37 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_30, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_36); if (lean_obj_tag(x_37) == 0) { -uint8_t x_38; -x_38 = !lean_is_exclusive(x_37); -if (x_38 == 0) +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_37, 1); +lean_inc(x_39); +lean_dec(x_37); +x_40 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_38, x_35, x_2, x_10, x_11, x_12, x_13, x_39); +if (lean_obj_tag(x_40) == 0) { -lean_object* x_39; -x_39 = lean_ctor_get(x_37, 0); -lean_ctor_set(x_21, 0, x_39); -lean_ctor_set(x_37, 0, x_21); -return x_37; +uint8_t x_41; +x_41 = !lean_is_exclusive(x_40); +if (x_41 == 0) +{ +lean_object* x_42; +x_42 = lean_ctor_get(x_40, 0); +lean_ctor_set(x_24, 0, x_42); +lean_ctor_set(x_40, 0, x_24); +return x_40; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; -x_40 = lean_ctor_get(x_37, 0); -x_41 = lean_ctor_get(x_37, 1); -lean_inc(x_41); -lean_inc(x_40); -lean_dec(x_37); -lean_ctor_set(x_21, 0, x_40); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_21); -lean_ctor_set(x_42, 1, x_41); -return x_42; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_40, 0); +x_44 = lean_ctor_get(x_40, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_40); +lean_ctor_set(x_24, 0, x_43); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_24); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } else { -uint8_t x_43; -lean_free_object(x_21); -x_43 = !lean_is_exclusive(x_37); -if (x_43 == 0) +uint8_t x_46; +lean_free_object(x_24); +x_46 = !lean_is_exclusive(x_40); +if (x_46 == 0) { -return x_37; +return x_40; } else { -lean_object* x_44; lean_object* x_45; lean_object* x_46; -x_44 = lean_ctor_get(x_37, 0); -x_45 = lean_ctor_get(x_37, 1); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_37); -x_46 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_45); -return x_46; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_40, 0); +x_48 = lean_ctor_get(x_40, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_40); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } } else { -uint8_t x_47; -lean_dec(x_32); -lean_free_object(x_21); +uint8_t x_50; +lean_dec(x_35); +lean_free_object(x_24); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_47 = !lean_is_exclusive(x_34); -if (x_47 == 0) +x_50 = !lean_is_exclusive(x_37); +if (x_50 == 0) { -return x_34; +return x_37; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_34, 0); -x_49 = lean_ctor_get(x_34, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_34); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_51; lean_object* x_52; lean_object* x_53; +x_51 = lean_ctor_get(x_37, 0); +x_52 = lean_ctor_get(x_37, 1); +lean_inc(x_52); +lean_inc(x_51); +lean_dec(x_37); +x_53 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_53, 0, x_51); +lean_ctor_set(x_53, 1, x_52); +return x_53; } } } else { -uint8_t x_51; -lean_free_object(x_21); -lean_dec(x_27); +uint8_t x_54; +lean_free_object(x_24); +lean_dec(x_30); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6468,33 +6534,33 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_51 = !lean_is_exclusive(x_31); -if (x_51 == 0) +x_54 = !lean_is_exclusive(x_34); +if (x_54 == 0) { -return x_31; +return x_34; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; -x_52 = lean_ctor_get(x_31, 0); -x_53 = lean_ctor_get(x_31, 1); -lean_inc(x_53); -lean_inc(x_52); -lean_dec(x_31); -x_54 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -return x_54; +lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_34, 0); +x_56 = lean_ctor_get(x_34, 1); +lean_inc(x_56); +lean_inc(x_55); +lean_dec(x_34); +x_57 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_57, 0, x_55); +lean_ctor_set(x_57, 1, x_56); +return x_57; } } } else { -lean_object* x_55; uint8_t x_56; lean_object* x_57; -x_55 = lean_ctor_get(x_21, 0); -lean_inc(x_55); -lean_dec(x_21); -x_56 = 1; +lean_object* x_58; uint8_t x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_24, 0); +lean_inc(x_58); +lean_dec(x_24); +x_59 = 1; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6503,21 +6569,8 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_27); -x_57 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_27, x_1, x_55, x_56, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_26); -if (lean_obj_tag(x_57) == 0) -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_60 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_27, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_59); +lean_inc(x_30); +x_60 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_30, x_1, x_58, x_59, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_29); if (lean_obj_tag(x_60) == 0) { lean_object* x_61; lean_object* x_62; lean_object* x_63; @@ -6526,92 +6579,105 @@ lean_inc(x_61); x_62 = lean_ctor_get(x_60, 1); lean_inc(x_62); lean_dec(x_60); -x_63 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_61, x_58, x_2, x_10, x_11, x_12, x_13, x_62); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_63 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_30, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_62); if (lean_obj_tag(x_63) == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +lean_object* x_64; lean_object* x_65; lean_object* x_66; x_64 = lean_ctor_get(x_63, 0); lean_inc(x_64); x_65 = lean_ctor_get(x_63, 1); lean_inc(x_65); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_66 = x_63; +lean_dec(x_63); +x_66 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_64, x_61, x_2, x_10, x_11, x_12, x_13, x_65); +if (lean_obj_tag(x_66) == 0) +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_69 = x_66; } else { - lean_dec_ref(x_63); - x_66 = lean_box(0); + lean_dec_ref(x_66); + x_69 = lean_box(0); } -x_67 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_67, 0, x_64); -if (lean_is_scalar(x_66)) { - x_68 = lean_alloc_ctor(0, 2, 0); +x_70 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_70, 0, x_67); +if (lean_is_scalar(x_69)) { + x_71 = lean_alloc_ctor(0, 2, 0); } else { - x_68 = x_66; + x_71 = x_69; } -lean_ctor_set(x_68, 0, x_67); -lean_ctor_set(x_68, 1, x_65); -return x_68; +lean_ctor_set(x_71, 0, x_70); +lean_ctor_set(x_71, 1, x_68); +return x_71; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_69 = lean_ctor_get(x_63, 0); -lean_inc(x_69); -x_70 = lean_ctor_get(x_63, 1); -lean_inc(x_70); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_71 = x_63; +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_72 = lean_ctor_get(x_66, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_66, 1); +lean_inc(x_73); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_74 = x_66; } else { - lean_dec_ref(x_63); - x_71 = lean_box(0); + lean_dec_ref(x_66); + x_74 = lean_box(0); } -if (lean_is_scalar(x_71)) { - x_72 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_74)) { + x_75 = lean_alloc_ctor(1, 2, 0); } else { - x_72 = x_71; + x_75 = x_74; } -lean_ctor_set(x_72, 0, x_69); -lean_ctor_set(x_72, 1, x_70); -return x_72; +lean_ctor_set(x_75, 0, x_72); +lean_ctor_set(x_75, 1, x_73); +return x_75; } } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -lean_dec(x_58); +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_61); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_73 = lean_ctor_get(x_60, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_60, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_60)) { - lean_ctor_release(x_60, 0); - lean_ctor_release(x_60, 1); - x_75 = x_60; +x_76 = lean_ctor_get(x_63, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_63, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_63)) { + lean_ctor_release(x_63, 0); + lean_ctor_release(x_63, 1); + x_78 = x_63; } else { - lean_dec_ref(x_60); - x_75 = lean_box(0); + lean_dec_ref(x_63); + x_78 = lean_box(0); } -if (lean_is_scalar(x_75)) { - x_76 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_78)) { + x_79 = lean_alloc_ctor(1, 2, 0); } else { - x_76 = x_75; + x_79 = x_78; } -lean_ctor_set(x_76, 0, x_73); -lean_ctor_set(x_76, 1, x_74); -return x_76; +lean_ctor_set(x_79, 0, x_76); +lean_ctor_set(x_79, 1, x_77); +return x_79; } } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_27); +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_30); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6621,44 +6687,44 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_77 = lean_ctor_get(x_57, 0); -lean_inc(x_77); -x_78 = lean_ctor_get(x_57, 1); -lean_inc(x_78); -if (lean_is_exclusive(x_57)) { - lean_ctor_release(x_57, 0); - lean_ctor_release(x_57, 1); - x_79 = x_57; +x_80 = lean_ctor_get(x_60, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_60, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_60)) { + lean_ctor_release(x_60, 0); + lean_ctor_release(x_60, 1); + x_82 = x_60; } else { - lean_dec_ref(x_57); - x_79 = lean_box(0); + lean_dec_ref(x_60); + x_82 = lean_box(0); } -if (lean_is_scalar(x_79)) { - x_80 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); } else { - x_80 = x_79; + x_83 = x_82; } -lean_ctor_set(x_80, 0, x_77); -lean_ctor_set(x_80, 1, x_78); -return x_80; +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; } } } else { -lean_object* x_81; lean_object* x_82; uint8_t x_83; -x_81 = lean_ctor_get(x_15, 1); -lean_inc(x_81); -lean_dec(x_15); -x_82 = lean_ctor_get(x_17, 0); -lean_inc(x_82); -lean_dec(x_17); -x_83 = !lean_is_exclusive(x_21); -if (x_83 == 0) +lean_object* x_84; lean_object* x_85; uint8_t x_86; +x_84 = lean_ctor_get(x_18, 1); +lean_inc(x_84); +lean_dec(x_18); +x_85 = lean_ctor_get(x_20, 0); +lean_inc(x_85); +lean_dec(x_20); +x_86 = !lean_is_exclusive(x_24); +if (x_86 == 0) { -lean_object* x_84; uint8_t x_85; lean_object* x_86; -x_84 = lean_ctor_get(x_21, 0); -x_85 = 0; +lean_object* x_87; uint8_t x_88; lean_object* x_89; +x_87 = lean_ctor_get(x_24, 0); +x_88 = 0; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6667,21 +6733,8 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_82); -x_86 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_82, x_1, x_84, x_85, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_81); -if (lean_obj_tag(x_86) == 0) -{ -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_89 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_82, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_88); +lean_inc(x_85); +x_89 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_85, x_1, x_87, x_88, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_84); if (lean_obj_tag(x_89) == 0) { lean_object* x_90; lean_object* x_91; lean_object* x_92; @@ -6690,92 +6743,105 @@ lean_inc(x_90); x_91 = lean_ctor_get(x_89, 1); lean_inc(x_91); lean_dec(x_89); -x_92 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_90, x_87, x_2, x_10, x_11, x_12, x_13, x_91); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_92 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_85, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_91); if (lean_obj_tag(x_92) == 0) { -uint8_t x_93; -x_93 = !lean_is_exclusive(x_92); -if (x_93 == 0) +lean_object* x_93; lean_object* x_94; lean_object* x_95; +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_ctor_get(x_92, 1); +lean_inc(x_94); +lean_dec(x_92); +x_95 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_93, x_90, x_2, x_10, x_11, x_12, x_13, x_94); +if (lean_obj_tag(x_95) == 0) { -lean_object* x_94; -x_94 = lean_ctor_get(x_92, 0); -lean_ctor_set(x_21, 0, x_94); -lean_ctor_set(x_92, 0, x_21); -return x_92; +uint8_t x_96; +x_96 = !lean_is_exclusive(x_95); +if (x_96 == 0) +{ +lean_object* x_97; +x_97 = lean_ctor_get(x_95, 0); +lean_ctor_set(x_24, 0, x_97); +lean_ctor_set(x_95, 0, x_24); +return x_95; } else { -lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_95 = lean_ctor_get(x_92, 0); -x_96 = lean_ctor_get(x_92, 1); -lean_inc(x_96); -lean_inc(x_95); -lean_dec(x_92); -lean_ctor_set(x_21, 0, x_95); -x_97 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_97, 0, x_21); -lean_ctor_set(x_97, 1, x_96); -return x_97; +lean_object* x_98; lean_object* x_99; lean_object* x_100; +x_98 = lean_ctor_get(x_95, 0); +x_99 = lean_ctor_get(x_95, 1); +lean_inc(x_99); +lean_inc(x_98); +lean_dec(x_95); +lean_ctor_set(x_24, 0, x_98); +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_24); +lean_ctor_set(x_100, 1, x_99); +return x_100; } } else { -uint8_t x_98; -lean_free_object(x_21); -x_98 = !lean_is_exclusive(x_92); -if (x_98 == 0) +uint8_t x_101; +lean_free_object(x_24); +x_101 = !lean_is_exclusive(x_95); +if (x_101 == 0) { -return x_92; +return x_95; } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_92, 0); -x_100 = lean_ctor_get(x_92, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_92); -x_101 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_101, 0, x_99); -lean_ctor_set(x_101, 1, x_100); -return x_101; +lean_object* x_102; lean_object* x_103; lean_object* x_104; +x_102 = lean_ctor_get(x_95, 0); +x_103 = lean_ctor_get(x_95, 1); +lean_inc(x_103); +lean_inc(x_102); +lean_dec(x_95); +x_104 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +return x_104; } } } else { -uint8_t x_102; -lean_dec(x_87); -lean_free_object(x_21); +uint8_t x_105; +lean_dec(x_90); +lean_free_object(x_24); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_102 = !lean_is_exclusive(x_89); -if (x_102 == 0) +x_105 = !lean_is_exclusive(x_92); +if (x_105 == 0) { -return x_89; +return x_92; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; -x_103 = lean_ctor_get(x_89, 0); -x_104 = lean_ctor_get(x_89, 1); -lean_inc(x_104); -lean_inc(x_103); -lean_dec(x_89); -x_105 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_105, 0, x_103); -lean_ctor_set(x_105, 1, x_104); -return x_105; +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_92, 0); +x_107 = lean_ctor_get(x_92, 1); +lean_inc(x_107); +lean_inc(x_106); +lean_dec(x_92); +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 1, x_107); +return x_108; } } } else { -uint8_t x_106; -lean_free_object(x_21); -lean_dec(x_82); +uint8_t x_109; +lean_free_object(x_24); +lean_dec(x_85); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6785,33 +6851,33 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_106 = !lean_is_exclusive(x_86); -if (x_106 == 0) +x_109 = !lean_is_exclusive(x_89); +if (x_109 == 0) { -return x_86; +return x_89; } else { -lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_107 = lean_ctor_get(x_86, 0); -x_108 = lean_ctor_get(x_86, 1); -lean_inc(x_108); -lean_inc(x_107); -lean_dec(x_86); -x_109 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_109, 0, x_107); -lean_ctor_set(x_109, 1, x_108); -return x_109; +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_89, 0); +x_111 = lean_ctor_get(x_89, 1); +lean_inc(x_111); +lean_inc(x_110); +lean_dec(x_89); +x_112 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +return x_112; } } } else { -lean_object* x_110; uint8_t x_111; lean_object* x_112; -x_110 = lean_ctor_get(x_21, 0); -lean_inc(x_110); -lean_dec(x_21); -x_111 = 0; +lean_object* x_113; uint8_t x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_24, 0); +lean_inc(x_113); +lean_dec(x_24); +x_114 = 0; lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -6820,21 +6886,8 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_82); -x_112 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_82, x_1, x_110, x_111, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_81); -if (lean_obj_tag(x_112) == 0) -{ -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_112, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_112, 1); -lean_inc(x_114); -lean_dec(x_112); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_115 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_82, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_114); +lean_inc(x_85); +x_115 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_85, x_1, x_113, x_114, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_84); if (lean_obj_tag(x_115) == 0) { lean_object* x_116; lean_object* x_117; lean_object* x_118; @@ -6843,92 +6896,105 @@ lean_inc(x_116); x_117 = lean_ctor_get(x_115, 1); lean_inc(x_117); lean_dec(x_115); -x_118 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_116, x_113, x_2, x_10, x_11, x_12, x_13, x_117); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_118 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom(x_85, x_3, x_4, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_117); if (lean_obj_tag(x_118) == 0) { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; +lean_object* x_119; lean_object* x_120; lean_object* x_121; x_119 = lean_ctor_get(x_118, 0); lean_inc(x_119); x_120 = lean_ctor_get(x_118, 1); lean_inc(x_120); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_121 = x_118; +lean_dec(x_118); +x_121 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_119, x_116, x_2, x_10, x_11, x_12, x_13, x_120); +if (lean_obj_tag(x_121) == 0) +{ +lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_122 = lean_ctor_get(x_121, 0); +lean_inc(x_122); +x_123 = lean_ctor_get(x_121, 1); +lean_inc(x_123); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + x_124 = x_121; } else { - lean_dec_ref(x_118); - x_121 = lean_box(0); + lean_dec_ref(x_121); + x_124 = lean_box(0); } -x_122 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_122, 0, x_119); -if (lean_is_scalar(x_121)) { - x_123 = lean_alloc_ctor(0, 2, 0); +x_125 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_125, 0, x_122); +if (lean_is_scalar(x_124)) { + x_126 = lean_alloc_ctor(0, 2, 0); } else { - x_123 = x_121; + x_126 = x_124; } -lean_ctor_set(x_123, 0, x_122); -lean_ctor_set(x_123, 1, x_120); -return x_123; +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_123); +return x_126; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_124 = lean_ctor_get(x_118, 0); -lean_inc(x_124); -x_125 = lean_ctor_get(x_118, 1); -lean_inc(x_125); -if (lean_is_exclusive(x_118)) { - lean_ctor_release(x_118, 0); - lean_ctor_release(x_118, 1); - x_126 = x_118; +lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_127 = lean_ctor_get(x_121, 0); +lean_inc(x_127); +x_128 = lean_ctor_get(x_121, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_121)) { + lean_ctor_release(x_121, 0); + lean_ctor_release(x_121, 1); + x_129 = x_121; } else { - lean_dec_ref(x_118); - x_126 = lean_box(0); + lean_dec_ref(x_121); + x_129 = lean_box(0); } -if (lean_is_scalar(x_126)) { - x_127 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(1, 2, 0); } else { - x_127 = x_126; + x_130 = x_129; } -lean_ctor_set(x_127, 0, x_124); -lean_ctor_set(x_127, 1, x_125); -return x_127; +lean_ctor_set(x_130, 0, x_127); +lean_ctor_set(x_130, 1, x_128); +return x_130; } } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; -lean_dec(x_113); +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +lean_dec(x_116); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); -x_128 = lean_ctor_get(x_115, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_115, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_115)) { - lean_ctor_release(x_115, 0); - lean_ctor_release(x_115, 1); - x_130 = x_115; +x_131 = lean_ctor_get(x_118, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_118, 1); +lean_inc(x_132); +if (lean_is_exclusive(x_118)) { + lean_ctor_release(x_118, 0); + lean_ctor_release(x_118, 1); + x_133 = x_118; } else { - lean_dec_ref(x_115); - x_130 = lean_box(0); + lean_dec_ref(x_118); + x_133 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_134 = x_133; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -lean_dec(x_82); +lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; +lean_dec(x_85); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6938,26 +7004,26 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); -x_132 = lean_ctor_get(x_112, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_112, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_112)) { - lean_ctor_release(x_112, 0); - lean_ctor_release(x_112, 1); - x_134 = x_112; +x_135 = lean_ctor_get(x_115, 0); +lean_inc(x_135); +x_136 = lean_ctor_get(x_115, 1); +lean_inc(x_136); +if (lean_is_exclusive(x_115)) { + lean_ctor_release(x_115, 0); + lean_ctor_release(x_115, 1); + x_137 = x_115; } else { - lean_dec_ref(x_112); - x_134 = lean_box(0); + lean_dec_ref(x_115); + x_137 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_137)) { + x_138 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_138 = x_137; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_138, 0, x_135); +lean_ctor_set(x_138, 1, x_136); +return x_138; } } } @@ -6966,7 +7032,7 @@ return x_135; } else { -uint8_t x_136; +uint8_t x_139; lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -6977,23 +7043,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_1); -x_136 = !lean_is_exclusive(x_15); -if (x_136 == 0) +x_139 = !lean_is_exclusive(x_18); +if (x_139 == 0) { -return x_15; +return x_18; } else { -lean_object* x_137; lean_object* x_138; lean_object* x_139; -x_137 = lean_ctor_get(x_15, 0); -x_138 = lean_ctor_get(x_15, 1); -lean_inc(x_138); -lean_inc(x_137); -lean_dec(x_15); -x_139 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_139, 0, x_137); -lean_ctor_set(x_139, 1, x_138); -return x_139; +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_18, 0); +x_141 = lean_ctor_get(x_18, 1); +lean_inc(x_141); +lean_inc(x_140); +lean_dec(x_18); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } @@ -9000,7 +9066,7 @@ lean_inc(x_21); x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); lean_dec(x_20); -x_23 = lean_ctor_get(x_21, 1); +x_23 = lean_ctor_get(x_21, 2); lean_inc(x_23); lean_dec(x_21); x_24 = l_Lean_Expr_constLevels_x21(x_1); @@ -9709,64 +9775,70 @@ return x_6; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo___lambda__1(lean_object* x_1, uint8_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_15; -lean_inc(x_1); -x_15 = l_Lean_Meta_Grind_getENode(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); -if (lean_obj_tag(x_15) == 0) -{ -lean_object* x_16; lean_object* x_17; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_st_ref_get(x_6, x_14); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 4); +x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); -if (lean_obj_tag(x_17) == 0) +lean_dec(x_15); +lean_inc(x_1); +x_18 = l_Lean_Meta_Grind_Goal_getENode(x_16, x_1, x_12, x_13, x_17); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_16); +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_19, 4); +lean_inc(x_20); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_19); lean_dec(x_3); lean_dec(x_1); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -lean_dec(x_15); -x_19 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo___lambda__1___closed__2; -x_20 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_19, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_18); -return x_20; +x_21 = lean_ctor_get(x_18, 1); +lean_inc(x_21); +lean_dec(x_18); +x_22 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo___lambda__1___closed__2; +x_23 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_22, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_21); +return x_23; } else { -lean_object* x_21; -x_21 = lean_ctor_get(x_16, 5); -lean_inc(x_21); -if (lean_obj_tag(x_21) == 0) +lean_object* x_24; +x_24 = lean_ctor_get(x_19, 5); +lean_inc(x_24); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -lean_dec(x_17); -lean_dec(x_16); +lean_object* x_25; lean_object* x_26; lean_object* x_27; +lean_dec(x_20); +lean_dec(x_19); lean_dec(x_3); lean_dec(x_1); -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); -lean_dec(x_15); -x_23 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo___lambda__1___closed__3; -x_24 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_22); -return x_24; +x_25 = lean_ctor_get(x_18, 1); +lean_inc(x_25); +lean_dec(x_18); +x_26 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo___lambda__1___closed__3; +x_27 = l_panic___at___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofFrom___spec__1(x_26, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); +return x_27; } else { -lean_object* x_25; lean_object* x_26; uint8_t x_27; -x_25 = lean_ctor_get(x_15, 1); -lean_inc(x_25); -lean_dec(x_15); -x_26 = lean_ctor_get(x_17, 0); -lean_inc(x_26); -lean_dec(x_17); -x_27 = !lean_is_exclusive(x_21); -if (x_27 == 0) +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_ctor_get(x_18, 1); +lean_inc(x_28); +lean_dec(x_18); +x_29 = lean_ctor_get(x_20, 0); +lean_inc(x_29); +lean_dec(x_20); +x_30 = !lean_is_exclusive(x_24); +if (x_30 == 0) { -lean_object* x_28; uint8_t x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_21, 0); -x_29 = lean_ctor_get_uint8(x_16, sizeof(void*)*10); -lean_dec(x_16); +lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_24, 0); +x_32 = lean_ctor_get_uint8(x_19, sizeof(void*)*11); +lean_dec(x_19); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9775,21 +9847,8 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_26); -x_30 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_1, x_26, x_28, x_29, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_30, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_30, 1); -lean_inc(x_32); -lean_dec(x_30); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_33 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_3, x_31, x_2, x_10, x_11, x_12, x_13, x_32); +lean_inc(x_29); +x_33 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_1, x_29, x_31, x_32, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_28); if (lean_obj_tag(x_33) == 0) { lean_object* x_34; lean_object* x_35; lean_object* x_36; @@ -9798,15 +9857,28 @@ lean_inc(x_34); x_35 = lean_ctor_get(x_33, 1); lean_inc(x_35); lean_dec(x_33); -lean_ctor_set(x_21, 0, x_34); -x_36 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_26, x_4, x_21, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_35); -return x_36; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_36 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_3, x_34, x_2, x_10, x_11, x_12, x_13, x_35); +if (lean_obj_tag(x_36) == 0) +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_36, 0); +lean_inc(x_37); +x_38 = lean_ctor_get(x_36, 1); +lean_inc(x_38); +lean_dec(x_36); +lean_ctor_set(x_24, 0, x_37); +x_39 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_29, x_4, x_24, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_38); +return x_39; } else { -uint8_t x_37; -lean_free_object(x_21); -lean_dec(x_26); +uint8_t x_40; +lean_free_object(x_24); +lean_dec(x_29); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9815,31 +9887,31 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_37 = !lean_is_exclusive(x_33); -if (x_37 == 0) +x_40 = !lean_is_exclusive(x_36); +if (x_40 == 0) { -return x_33; +return x_36; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_33, 0); -x_39 = lean_ctor_get(x_33, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_33); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_36, 0); +x_42 = lean_ctor_get(x_36, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_36); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -uint8_t x_41; -lean_free_object(x_21); -lean_dec(x_26); +uint8_t x_44; +lean_free_object(x_24); +lean_dec(x_29); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9849,34 +9921,34 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); -x_41 = !lean_is_exclusive(x_30); -if (x_41 == 0) +x_44 = !lean_is_exclusive(x_33); +if (x_44 == 0) { -return x_30; +return x_33; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_30, 0); -x_43 = lean_ctor_get(x_30, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_30); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_33, 0); +x_46 = lean_ctor_get(x_33, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_33); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } else { -lean_object* x_45; uint8_t x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_21, 0); -lean_inc(x_45); -lean_dec(x_21); -x_46 = lean_ctor_get_uint8(x_16, sizeof(void*)*10); -lean_dec(x_16); +lean_object* x_48; uint8_t x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_24, 0); +lean_inc(x_48); +lean_dec(x_24); +x_49 = lean_ctor_get_uint8(x_19, sizeof(void*)*11); +lean_dec(x_19); lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); @@ -9885,38 +9957,38 @@ lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_26); -x_47 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_1, x_26, x_45, x_46, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_25); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_47, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_47, 1); -lean_inc(x_49); -lean_dec(x_47); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -x_50 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_3, x_48, x_2, x_10, x_11, x_12, x_13, x_49); +lean_inc(x_29); +x_50 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_realizeEqProof(x_1, x_29, x_48, x_49, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_28); if (lean_obj_tag(x_50) == 0) { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +lean_object* x_51; lean_object* x_52; lean_object* x_53; x_51 = lean_ctor_get(x_50, 0); lean_inc(x_51); x_52 = lean_ctor_get(x_50, 1); lean_inc(x_52); lean_dec(x_50); -x_53 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_53, 0, x_51); -x_54 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_26, x_4, x_53, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_52); -return x_54; +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +x_53 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkTrans_x27(x_3, x_51, x_2, x_10, x_11, x_12, x_13, x_52); +if (lean_obj_tag(x_53) == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +x_54 = lean_ctor_get(x_53, 0); +lean_inc(x_54); +x_55 = lean_ctor_get(x_53, 1); +lean_inc(x_55); +lean_dec(x_53); +x_56 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_56, 0, x_54); +x_57 = l___private_Lean_Meta_Tactic_Grind_Proof_0__Lean_Meta_Grind_mkProofTo(x_29, x_4, x_56, x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_55); +return x_57; } else { -lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; -lean_dec(x_26); +lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +lean_dec(x_29); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9925,32 +9997,32 @@ lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -x_55 = lean_ctor_get(x_50, 0); -lean_inc(x_55); -x_56 = lean_ctor_get(x_50, 1); -lean_inc(x_56); -if (lean_is_exclusive(x_50)) { - lean_ctor_release(x_50, 0); - lean_ctor_release(x_50, 1); - x_57 = x_50; +x_58 = lean_ctor_get(x_53, 0); +lean_inc(x_58); +x_59 = lean_ctor_get(x_53, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_53)) { + lean_ctor_release(x_53, 0); + lean_ctor_release(x_53, 1); + x_60 = x_53; } else { - lean_dec_ref(x_50); - x_57 = lean_box(0); + lean_dec_ref(x_53); + x_60 = lean_box(0); } -if (lean_is_scalar(x_57)) { - x_58 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(1, 2, 0); } else { - x_58 = x_57; + x_61 = x_60; } -lean_ctor_set(x_58, 0, x_55); -lean_ctor_set(x_58, 1, x_56); -return x_58; +lean_ctor_set(x_61, 0, x_58); +lean_ctor_set(x_61, 1, x_59); +return x_61; } } else { -lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -lean_dec(x_26); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_dec(x_29); lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9960,26 +10032,26 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); -x_59 = lean_ctor_get(x_47, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_47, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_47)) { - lean_ctor_release(x_47, 0); - lean_ctor_release(x_47, 1); - x_61 = x_47; +x_62 = lean_ctor_get(x_50, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_50, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_50)) { + lean_ctor_release(x_50, 0); + lean_ctor_release(x_50, 1); + x_64 = x_50; } else { - lean_dec_ref(x_47); - x_61 = lean_box(0); + lean_dec_ref(x_50); + x_64 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_64)) { + x_65 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_65 = x_64; } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; +lean_ctor_set(x_65, 0, x_62); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } } @@ -9987,7 +10059,7 @@ return x_62; } else { -uint8_t x_63; +uint8_t x_66; lean_dec(x_13); lean_dec(x_12); lean_dec(x_11); @@ -9998,23 +10070,23 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_3); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_15); -if (x_63 == 0) +x_66 = !lean_is_exclusive(x_18); +if (x_66 == 0) { -return x_15; +return x_18; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_15, 0); -x_65 = lean_ctor_get(x_15, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_15); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_18, 0); +x_68 = lean_ctor_get(x_18, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_18); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; } } } diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Propagate.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Propagate.c index 7f380dd9a3ac..d1fdfd81281c 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Propagate.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Propagate.c @@ -18,11 +18,11 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateEqMatchDown___closed__2; static lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1___closed__2; lean_object* l_Lean_Meta_Simp_Result_getProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1; static lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1___closed__3; static lean_object* l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__4; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateAndUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_383____closed__1; static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__11; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateOrDown___lambda__1___closed__4; static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -33,15 +33,16 @@ static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__10; static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateNotUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1486_(lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2; static lean_object* l_Lean_Meta_Grind_propagateIte___closed__1; static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__5; static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__2; static lean_object* l_Lean_Meta_Grind_propagateNotUp___closed__2; +lean_object* l_Lean_Meta_mkEqTrueCore(lean_object*, lean_object*); lean_object* l_Lean_mkApp8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1___closed__6; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1; uint8_t l_Lean_Expr_isApp(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -50,17 +51,17 @@ static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__8; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateOrUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_985____closed__1; static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__3; static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__6; -static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1; +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1; static lean_object* l_Lean_Meta_Grind_propagateHEqDown___closed__1; lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__1; static lean_object* l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__7; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateAndDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_604____closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateAndUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__1; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__6; @@ -73,14 +74,13 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateNotDown(lean_object*, lean_o static lean_object* l_Lean_Meta_Grind_propagateEqMatchDown___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateDIte(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateHEqDown___closed__2; -lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__4; static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__7; static lean_object* l_Lean_Meta_Grind_propagateOrDown___lambda__1___closed__2; lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7; static lean_object* l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__3; static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__12; static lean_object* l_Lean_Meta_Grind_propagateAndUp___closed__1; @@ -90,21 +90,19 @@ lean_object* l_Lean_Meta_Grind_closeGoal(lean_object*, lean_object*, lean_object LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__4; static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__8; +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1; +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateHEqUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__9; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqDown___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__6; static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__2; -static lean_object* l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateOrDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1206_(lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__1; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateOrDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1206____closed__1; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1; static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__11; static lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1___closed__4; lean_object* l_Lean_Meta_Grind_pushEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -118,14 +116,13 @@ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getGeneration(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__2; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateIte___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__7; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__3; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__10; static lean_object* l_Lean_Meta_Grind_propagateNotDown___lambda__1___closed__5; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148_(lean_object*); +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617_(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateIte___lambda__1___closed__1; static lean_object* l_Lean_Meta_Grind_propagateDIte___closed__2; static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__9; @@ -138,14 +135,13 @@ LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateAndDown_declare static lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateOrDown___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__4; -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530_(lean_object*); lean_object* lean_grind_mk_eq_proof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateEqUp___closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054_(lean_object*); lean_object* lean_grind_mk_heq_proof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_constLevels_x21(lean_object*); static lean_object* l_Lean_Meta_Grind_propagateDIte___closed__1; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateNotUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1486____closed__1; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1; static lean_object* l_Lean_Meta_Grind_propagateIte___lambda__1___closed__4; lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -161,12 +157,11 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateAndDown(lean_object*, lean_o static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__2; uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_isEqv(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1; lean_object* l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(lean_object*, uint8_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347_(lean_object*); lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_mkOfEqTrueCore(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1; -static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateIte(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndDown___lambda__1___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqMatchDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -177,11 +172,13 @@ lean_object* l_Lean_Meta_Grind_pushEqFalse(lean_object*, lean_object*, lean_obje static lean_object* l_Lean_Meta_Grind_propagateOrDown___lambda__1___closed__5; static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateNotDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1766____closed__1; static lean_object* l_Lean_Meta_Grind_propagateIte___lambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1; +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339_(lean_object*); lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__12; static lean_object* l_Lean_Meta_Grind_propagateNotUp___lambda__1___closed__3; +static lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1; static lean_object* l_Lean_Meta_Grind_propagateOrUp___closed__2; -static lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9; static lean_object* l_Lean_Meta_Grind_propagateNotUp___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateOrUp___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateHEqDown___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -190,9 +187,8 @@ static lean_object* l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__6; static lean_object* l_Lean_Meta_Grind_propagateEqUp___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateHEqUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateHEqDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_internalize(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateNotDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_1766_(lean_object*); -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078_(lean_object*); static lean_object* _init_l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__1() { _start: { @@ -3685,18 +3681,19 @@ static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_true", 7, 7); +x_1 = lean_mk_string_unchecked("eq_eq_of_eq_true_right", 22, 22); return x_1; } } static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__2() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__1; +x_2 = l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__2; +x_3 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__1; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; } } static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__3() { @@ -3713,7 +3710,7 @@ static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_eq_of_eq_true_right", 22, 22); +x_1 = lean_mk_string_unchecked("eq_eq_of_eq_true_left", 21, 21); return x_1; } } @@ -3738,35 +3735,6 @@ x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("eq_eq_of_eq_true_left", 21, 21); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__1; -x_2 = l_Lean_Meta_Grind_propagateAndUp___lambda__1___closed__2; -x_3 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7; -x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); -return x_4; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqUp___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { @@ -3865,16 +3833,15 @@ lean_inc(x_4); x_31 = lean_grind_mk_eq_proof(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); if (lean_obj_tag(x_31) == 0) { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); x_33 = lean_ctor_get(x_31, 1); lean_inc(x_33); lean_dec(x_31); -x_34 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__3; lean_inc(x_1); -x_35 = l_Lean_mkAppB(x_34, x_1, x_32); -x_36 = l_Lean_Meta_Grind_pushEqTrue(x_1, x_35, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +x_34 = l_Lean_Meta_mkEqTrueCore(x_1, x_32); +x_35 = l_Lean_Meta_Grind_pushEqTrue(x_1, x_34, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3883,11 +3850,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_36; +return x_35; } else { -uint8_t x_37; +uint8_t x_36; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3897,30 +3864,30 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_37 = !lean_is_exclusive(x_31); -if (x_37 == 0) +x_36 = !lean_is_exclusive(x_31); +if (x_36 == 0) { return x_31; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_31, 0); -x_39 = lean_ctor_get(x_31, 1); -lean_inc(x_39); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_31, 0); +x_38 = lean_ctor_get(x_31, 1); lean_inc(x_38); +lean_inc(x_37); lean_dec(x_31); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } } else { -uint8_t x_41; +uint8_t x_40; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3932,31 +3899,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_41 = !lean_is_exclusive(x_21); -if (x_41 == 0) +x_40 = !lean_is_exclusive(x_21); +if (x_40 == 0) { return x_21; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_21, 0); -x_43 = lean_ctor_get(x_21, 1); -lean_inc(x_43); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_21, 0); +x_42 = lean_ctor_get(x_21, 1); lean_inc(x_42); +lean_inc(x_41); lean_dec(x_21); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_42); -lean_ctor_set(x_44, 1, x_43); -return x_44; +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -lean_object* x_45; lean_object* x_46; -x_45 = lean_ctor_get(x_17, 1); -lean_inc(x_45); +lean_object* x_44; lean_object* x_45; +x_44 = lean_ctor_get(x_17, 1); +lean_inc(x_44); lean_dec(x_17); lean_inc(x_11); lean_inc(x_10); @@ -3967,20 +3934,20 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_3); -x_46 = l_Lean_Meta_Grind_mkEqTrueProof(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_45); -if (lean_obj_tag(x_46) == 0) +x_45 = l_Lean_Meta_Grind_mkEqTrueProof(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_44); +if (lean_obj_tag(x_45) == 0) { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_object* x_52; -x_47 = lean_ctor_get(x_46, 0); +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); lean_inc(x_47); -x_48 = lean_ctor_get(x_46, 1); -lean_inc(x_48); -lean_dec(x_46); -x_49 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__6; +lean_dec(x_45); +x_48 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__3; lean_inc(x_2); -x_50 = l_Lean_mkApp3(x_49, x_2, x_3, x_47); -x_51 = 0; -x_52 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_50, x_51, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_48); +x_49 = l_Lean_mkApp3(x_48, x_2, x_3, x_46); +x_50 = 0; +x_51 = l_Lean_Meta_Grind_pushEqCore(x_1, x_2, x_49, x_50, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_47); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -3989,11 +3956,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_52; +return x_51; } else { -uint8_t x_53; +uint8_t x_52; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4005,30 +3972,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_53 = !lean_is_exclusive(x_46); -if (x_53 == 0) +x_52 = !lean_is_exclusive(x_45); +if (x_52 == 0) { -return x_46; +return x_45; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_46, 0); -x_55 = lean_ctor_get(x_46, 1); -lean_inc(x_55); +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_45, 0); +x_54 = lean_ctor_get(x_45, 1); lean_inc(x_54); -lean_dec(x_46); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_inc(x_53); +lean_dec(x_45); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } } else { -uint8_t x_57; +uint8_t x_56; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4040,31 +4007,31 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_57 = !lean_is_exclusive(x_17); -if (x_57 == 0) +x_56 = !lean_is_exclusive(x_17); +if (x_56 == 0) { return x_17; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_58 = lean_ctor_get(x_17, 0); -x_59 = lean_ctor_get(x_17, 1); -lean_inc(x_59); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_17, 0); +x_58 = lean_ctor_get(x_17, 1); lean_inc(x_58); +lean_inc(x_57); lean_dec(x_17); -x_60 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_60, 0, x_58); -lean_ctor_set(x_60, 1, x_59); -return x_60; +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } else { -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_13, 1); -lean_inc(x_61); +lean_object* x_60; lean_object* x_61; +x_60 = lean_ctor_get(x_13, 1); +lean_inc(x_60); lean_dec(x_13); lean_inc(x_11); lean_inc(x_10); @@ -4075,20 +4042,20 @@ lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); lean_inc(x_2); -x_62 = l_Lean_Meta_Grind_mkEqTrueProof(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_61); -if (lean_obj_tag(x_62) == 0) +x_61 = l_Lean_Meta_Grind_mkEqTrueProof(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_60); +if (lean_obj_tag(x_61) == 0) { -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; uint8_t x_67; lean_object* x_68; -x_63 = lean_ctor_get(x_62, 0); +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; lean_object* x_67; +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_61, 1); lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); -lean_dec(x_62); -x_65 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9; +lean_dec(x_61); +x_64 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__6; lean_inc(x_3); -x_66 = l_Lean_mkApp3(x_65, x_2, x_3, x_63); -x_67 = 0; -x_68 = l_Lean_Meta_Grind_pushEqCore(x_1, x_3, x_66, x_67, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_64); +x_65 = l_Lean_mkApp3(x_64, x_2, x_3, x_62); +x_66 = 0; +x_67 = l_Lean_Meta_Grind_pushEqCore(x_1, x_3, x_65, x_66, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_63); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4097,11 +4064,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_68; +return x_67; } else { -uint8_t x_69; +uint8_t x_68; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4113,30 +4080,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_62); -if (x_69 == 0) +x_68 = !lean_is_exclusive(x_61); +if (x_68 == 0) { -return x_62; +return x_61; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_62, 0); -x_71 = lean_ctor_get(x_62, 1); -lean_inc(x_71); +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_61, 0); +x_70 = lean_ctor_get(x_61, 1); lean_inc(x_70); -lean_dec(x_62); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +lean_inc(x_69); +lean_dec(x_61); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; } } } } else { -uint8_t x_73; +uint8_t x_72; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4148,23 +4115,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_73 = !lean_is_exclusive(x_13); -if (x_73 == 0) +x_72 = !lean_is_exclusive(x_13); +if (x_72 == 0) { return x_13; } else { -lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_74 = lean_ctor_get(x_13, 0); -x_75 = lean_ctor_get(x_13, 1); -lean_inc(x_75); +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_13, 0); +x_74 = lean_ctor_get(x_13, 1); lean_inc(x_74); +lean_inc(x_73); lean_dec(x_13); -x_76 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_76, 0, x_74); -lean_ctor_set(x_76, 1, x_75); -return x_76; +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; } } } @@ -4304,7 +4271,7 @@ return x_30; } } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1() { _start: { lean_object* x_1; @@ -4312,45 +4279,17 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateEqUp), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateEqUp___closed__2; x_3 = 1; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("of_eq_true", 10, 10); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateEqDown___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { @@ -4367,16 +4306,15 @@ lean_inc(x_1); x_13 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3; -x_17 = l_Lean_mkAppB(x_16, x_1, x_14); -x_18 = 0; -x_19 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_16 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_14); +x_17 = 0; +x_18 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_16, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4385,11 +4323,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_19; +return x_18; } else { -uint8_t x_20; +uint8_t x_19; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -4401,23 +4339,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_13); -if (x_20 == 0) +x_19 = !lean_is_exclusive(x_13); +if (x_19 == 0) { return x_13; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_13, 0); -x_22 = lean_ctor_get(x_13, 1); -lean_inc(x_22); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_13, 0); +x_21 = lean_ctor_get(x_13, 1); lean_inc(x_21); +lean_inc(x_20); lean_dec(x_13); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } @@ -4738,7 +4676,7 @@ return x_63; } } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1() { _start: { lean_object* x_1; @@ -4746,13 +4684,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateEqDown), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateEqUp___closed__2; x_3 = 0; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -4780,16 +4718,15 @@ lean_inc(x_1); x_16 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_15); if (lean_obj_tag(x_16) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3; -x_20 = l_Lean_mkAppB(x_19, x_1, x_17); -x_21 = 0; -x_22 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_20, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); +x_19 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_17); +x_20 = 0; +x_21 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_19, x_20, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_18); lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4798,11 +4735,11 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -return x_22; +return x_21; } else { -uint8_t x_23; +uint8_t x_22; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4814,29 +4751,29 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_23 = !lean_is_exclusive(x_16); -if (x_23 == 0) +x_22 = !lean_is_exclusive(x_16); +if (x_22 == 0) { return x_16; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_16, 0); -x_25 = lean_ctor_get(x_16, 1); -lean_inc(x_25); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_16, 0); +x_24 = lean_ctor_get(x_16, 1); lean_inc(x_24); +lean_inc(x_23); lean_dec(x_16); -x_26 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_26, 0, x_24); -lean_ctor_set(x_26, 1, x_25); -return x_26; +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } else { -uint8_t x_27; +uint8_t x_26; lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); @@ -4848,23 +4785,23 @@ lean_dec(x_5); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_27 = !lean_is_exclusive(x_14); -if (x_27 == 0) +x_26 = !lean_is_exclusive(x_14); +if (x_26 == 0) { return x_14; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_14, 0); -x_29 = lean_ctor_get(x_14, 1); -lean_inc(x_29); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_14, 0); +x_28 = lean_ctor_get(x_14, 1); lean_inc(x_28); +lean_inc(x_27); lean_dec(x_14); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +x_29 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_29, 0, x_27); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } } @@ -5262,7 +5199,7 @@ return x_72; } } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1() { _start: { lean_object* x_1; @@ -5270,13 +5207,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateEqMatchDown), 10, 0) return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateEqMatchDown___closed__2; x_3 = 0; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -5297,16 +5234,15 @@ lean_inc(x_1); x_13 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); if (lean_obj_tag(x_13) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3; -x_17 = l_Lean_mkAppB(x_16, x_1, x_14); -x_18 = 1; -x_19 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); +x_16 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_14); +x_17 = 1; +x_18 = l_Lean_Meta_Grind_pushEqCore(x_2, x_3, x_16, x_17, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_15); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5315,11 +5251,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_19; +return x_18; } else { -uint8_t x_20; +uint8_t x_19; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5331,23 +5267,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_20 = !lean_is_exclusive(x_13); -if (x_20 == 0) +x_19 = !lean_is_exclusive(x_13); +if (x_19 == 0) { return x_13; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_13, 0); -x_22 = lean_ctor_get(x_13, 1); -lean_inc(x_22); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_13, 0); +x_21 = lean_ctor_get(x_13, 1); lean_inc(x_21); +lean_inc(x_20); lean_dec(x_13); -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -return x_23; +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } @@ -5736,7 +5672,7 @@ return x_70; } } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1() { _start: { lean_object* x_1; @@ -5744,13 +5680,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateHEqDown), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateHEqDown___closed__2; x_3 = 0; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -5823,16 +5759,15 @@ lean_inc(x_4); x_23 = lean_grind_mk_heq_proof(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_22); if (lean_obj_tag(x_23) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); x_25 = lean_ctor_get(x_23, 1); lean_inc(x_25); lean_dec(x_23); -x_26 = l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__3; lean_inc(x_1); -x_27 = l_Lean_mkAppB(x_26, x_1, x_24); -x_28 = l_Lean_Meta_Grind_pushEqTrue(x_1, x_27, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); +x_26 = l_Lean_Meta_mkEqTrueCore(x_1, x_24); +x_27 = l_Lean_Meta_Grind_pushEqTrue(x_1, x_26, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_25); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5841,11 +5776,11 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_28; +return x_27; } else { -uint8_t x_29; +uint8_t x_28; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5855,30 +5790,30 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); -x_29 = !lean_is_exclusive(x_23); -if (x_29 == 0) +x_28 = !lean_is_exclusive(x_23); +if (x_28 == 0) { return x_23; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_23, 0); -x_31 = lean_ctor_get(x_23, 1); -lean_inc(x_31); +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_23, 0); +x_30 = lean_ctor_get(x_23, 1); lean_inc(x_30); +lean_inc(x_29); lean_dec(x_23); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +x_31 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_31, 0, x_29); +lean_ctor_set(x_31, 1, x_30); +return x_31; } } } } else { -uint8_t x_33; +uint8_t x_32; lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -5890,23 +5825,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_33 = !lean_is_exclusive(x_13); -if (x_33 == 0) +x_32 = !lean_is_exclusive(x_13); +if (x_32 == 0) { return x_13; } else { -lean_object* x_34; lean_object* x_35; lean_object* x_36; -x_34 = lean_ctor_get(x_13, 0); -x_35 = lean_ctor_get(x_13, 1); -lean_inc(x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_13, 0); +x_34 = lean_ctor_get(x_13, 1); lean_inc(x_34); +lean_inc(x_33); lean_dec(x_13); -x_36 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_36, 0, x_34); -lean_ctor_set(x_36, 1, x_35); -return x_36; +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } @@ -6054,7 +5989,7 @@ return x_34; } } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1() { _start: { lean_object* x_1; @@ -6062,13 +5997,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateHEqUp), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateHEqDown___closed__2; x_3 = 1; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -6618,7 +6553,7 @@ lean_dec(x_2); return x_17; } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1() { _start: { lean_object* x_1; @@ -6626,13 +6561,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateIte), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateIte___closed__2; x_3 = 1; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -6806,7 +6741,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_10); -x_37 = l_Lean_Meta_Grind_simp(x_36, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_33); +x_37 = l_Lean_Meta_Grind_simp(x_36, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_33); if (lean_obj_tag(x_37) == 0) { lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; @@ -6834,12 +6769,13 @@ lean_inc(x_1); x_44 = l_Lean_Meta_Grind_getGeneration(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_43); if (lean_obj_tag(x_44) == 0) { -lean_object* x_45; lean_object* x_46; lean_object* x_47; +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); x_46 = lean_ctor_get(x_44, 1); lean_inc(x_46); lean_dec(x_44); +x_47 = lean_box(0); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -6849,20 +6785,20 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_40); -x_47 = l_Lean_Meta_Grind_internalize(x_40, x_45, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); -if (lean_obj_tag(x_47) == 0) +x_48 = l_Lean_Meta_Grind_internalize(x_40, x_45, x_47, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_46); +if (lean_obj_tag(x_48) == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -x_49 = l_Lean_Expr_constLevels_x21(x_2); -x_50 = l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__5; -x_51 = l_Lean_Expr_const___override(x_50, x_49); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +lean_dec(x_48); +x_50 = l_Lean_Expr_constLevels_x21(x_2); +x_51 = l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__5; +x_52 = l_Lean_Expr_const___override(x_51, x_50); lean_inc(x_40); -x_52 = l_Lean_mkApp8(x_51, x_3, x_4, x_5, x_6, x_7, x_40, x_32, x_42); -x_53 = 0; -x_54 = l_Lean_Meta_Grind_pushEqCore(x_1, x_40, x_52, x_53, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_48); +x_53 = l_Lean_mkApp8(x_52, x_3, x_4, x_5, x_6, x_7, x_40, x_32, x_42); +x_54 = 0; +x_55 = l_Lean_Meta_Grind_pushEqCore(x_1, x_40, x_53, x_54, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_49); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -6871,11 +6807,11 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_54; +return x_55; } else { -uint8_t x_55; +uint8_t x_56; lean_dec(x_42); lean_dec(x_40); lean_dec(x_32); @@ -6893,29 +6829,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_55 = !lean_is_exclusive(x_47); -if (x_55 == 0) +x_56 = !lean_is_exclusive(x_48); +if (x_56 == 0) { -return x_47; +return x_48; } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; -x_56 = lean_ctor_get(x_47, 0); -x_57 = lean_ctor_get(x_47, 1); +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_48, 0); +x_58 = lean_ctor_get(x_48, 1); +lean_inc(x_58); lean_inc(x_57); -lean_inc(x_56); -lean_dec(x_47); -x_58 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_58, 0, x_56); -lean_ctor_set(x_58, 1, x_57); -return x_58; +lean_dec(x_48); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } else { -uint8_t x_59; +uint8_t x_60; lean_dec(x_42); lean_dec(x_40); lean_dec(x_32); @@ -6933,29 +6869,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_59 = !lean_is_exclusive(x_44); -if (x_59 == 0) +x_60 = !lean_is_exclusive(x_44); +if (x_60 == 0) { return x_44; } else { -lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_60 = lean_ctor_get(x_44, 0); -x_61 = lean_ctor_get(x_44, 1); +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_44, 0); +x_62 = lean_ctor_get(x_44, 1); +lean_inc(x_62); lean_inc(x_61); -lean_inc(x_60); lean_dec(x_44); -x_62 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_62, 0, x_60); -lean_ctor_set(x_62, 1, x_61); -return x_62; +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; } } } else { -uint8_t x_63; +uint8_t x_64; lean_dec(x_40); lean_dec(x_32); lean_dec(x_15); @@ -6972,29 +6908,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_41); -if (x_63 == 0) +x_64 = !lean_is_exclusive(x_41); +if (x_64 == 0) { return x_41; } else { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_41, 0); -x_65 = lean_ctor_get(x_41, 1); +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_41, 0); +x_66 = lean_ctor_get(x_41, 1); +lean_inc(x_66); lean_inc(x_65); -lean_inc(x_64); lean_dec(x_41); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } } } else { -uint8_t x_67; +uint8_t x_68; lean_dec(x_32); lean_dec(x_15); lean_dec(x_14); @@ -7010,29 +6946,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_67 = !lean_is_exclusive(x_37); -if (x_67 == 0) +x_68 = !lean_is_exclusive(x_37); +if (x_68 == 0) { return x_37; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_37, 0); -x_69 = lean_ctor_get(x_37, 1); +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_37, 0); +x_70 = lean_ctor_get(x_37, 1); +lean_inc(x_70); lean_inc(x_69); -lean_inc(x_68); lean_dec(x_37); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -return x_70; +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; } } } else { -uint8_t x_71; +uint8_t x_72; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7047,30 +6983,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_71 = !lean_is_exclusive(x_31); -if (x_71 == 0) +x_72 = !lean_is_exclusive(x_31); +if (x_72 == 0) { return x_31; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_72 = lean_ctor_get(x_31, 0); -x_73 = lean_ctor_get(x_31, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; +x_73 = lean_ctor_get(x_31, 0); +x_74 = lean_ctor_get(x_31, 1); +lean_inc(x_74); lean_inc(x_73); -lean_inc(x_72); lean_dec(x_31); -x_74 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_74, 0, x_72); -lean_ctor_set(x_74, 1, x_73); -return x_74; +x_75 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_75, 0, x_73); +lean_ctor_set(x_75, 1, x_74); +return x_75; } } } } else { -uint8_t x_75; +uint8_t x_76; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7085,31 +7021,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_75 = !lean_is_exclusive(x_21); -if (x_75 == 0) +x_76 = !lean_is_exclusive(x_21); +if (x_76 == 0) { return x_21; } else { -lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_76 = lean_ctor_get(x_21, 0); -x_77 = lean_ctor_get(x_21, 1); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_21, 0); +x_78 = lean_ctor_get(x_21, 1); +lean_inc(x_78); lean_inc(x_77); -lean_inc(x_76); lean_dec(x_21); -x_78 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -return x_78; +x_79 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_79, 0, x_77); +lean_ctor_set(x_79, 1, x_78); +return x_79; } } } else { -lean_object* x_79; lean_object* x_80; -x_79 = lean_ctor_get(x_17, 1); -lean_inc(x_79); +lean_object* x_80; lean_object* x_81; +x_80 = lean_ctor_get(x_17, 1); +lean_inc(x_80); lean_dec(x_17); lean_inc(x_15); lean_inc(x_14); @@ -7120,19 +7056,18 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_4); -x_80 = l_Lean_Meta_Grind_mkEqTrueProof(x_4, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_79); -if (lean_obj_tag(x_80) == 0) +x_81 = l_Lean_Meta_Grind_mkEqTrueProof(x_4, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_80); +if (lean_obj_tag(x_81) == 0) { -lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +x_82 = lean_ctor_get(x_81, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_81, 1); +lean_inc(x_83); +lean_dec(x_81); lean_inc(x_82); -lean_dec(x_80); -x_83 = l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3; -lean_inc(x_81); lean_inc(x_4); -x_84 = l_Lean_mkAppB(x_83, x_4, x_81); +x_84 = l_Lean_Meta_mkOfEqTrueCore(x_4, x_82); lean_inc(x_6); x_85 = l_Lean_Expr_app___override(x_6, x_84); lean_inc(x_15); @@ -7140,7 +7075,7 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_inc(x_10); -x_86 = l_Lean_Meta_Grind_simp(x_85, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_82); +x_86 = l_Lean_Meta_Grind_simp(x_85, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_83); if (lean_obj_tag(x_86) == 0) { lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; @@ -7168,12 +7103,13 @@ lean_inc(x_1); x_93 = l_Lean_Meta_Grind_getGeneration(x_1, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_92); if (lean_obj_tag(x_93) == 0) { -lean_object* x_94; lean_object* x_95; lean_object* x_96; +lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; x_94 = lean_ctor_get(x_93, 0); lean_inc(x_94); x_95 = lean_ctor_get(x_93, 1); lean_inc(x_95); lean_dec(x_93); +x_96 = lean_box(0); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); @@ -7183,20 +7119,20 @@ lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); lean_inc(x_89); -x_96 = l_Lean_Meta_Grind_internalize(x_89, x_94, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_95); -if (lean_obj_tag(x_96) == 0) -{ -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; lean_object* x_103; -x_97 = lean_ctor_get(x_96, 1); -lean_inc(x_97); -lean_dec(x_96); -x_98 = l_Lean_Expr_constLevels_x21(x_2); -x_99 = l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__7; -x_100 = l_Lean_Expr_const___override(x_99, x_98); +x_97 = l_Lean_Meta_Grind_internalize(x_89, x_94, x_96, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_95); +if (lean_obj_tag(x_97) == 0) +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; +x_98 = lean_ctor_get(x_97, 1); +lean_inc(x_98); +lean_dec(x_97); +x_99 = l_Lean_Expr_constLevels_x21(x_2); +x_100 = l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__7; +x_101 = l_Lean_Expr_const___override(x_100, x_99); lean_inc(x_89); -x_101 = l_Lean_mkApp8(x_100, x_3, x_4, x_5, x_6, x_7, x_89, x_81, x_91); -x_102 = 0; -x_103 = l_Lean_Meta_Grind_pushEqCore(x_1, x_89, x_101, x_102, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_97); +x_102 = l_Lean_mkApp8(x_101, x_3, x_4, x_5, x_6, x_7, x_89, x_82, x_91); +x_103 = 0; +x_104 = l_Lean_Meta_Grind_pushEqCore(x_1, x_89, x_102, x_103, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_98); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7205,14 +7141,14 @@ lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); -return x_103; +return x_104; } else { -uint8_t x_104; +uint8_t x_105; lean_dec(x_91); lean_dec(x_89); -lean_dec(x_81); +lean_dec(x_82); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7227,32 +7163,32 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_104 = !lean_is_exclusive(x_96); -if (x_104 == 0) +x_105 = !lean_is_exclusive(x_97); +if (x_105 == 0) { -return x_96; +return x_97; } else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; -x_105 = lean_ctor_get(x_96, 0); -x_106 = lean_ctor_get(x_96, 1); +lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_106 = lean_ctor_get(x_97, 0); +x_107 = lean_ctor_get(x_97, 1); +lean_inc(x_107); lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_96); -x_107 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -return x_107; +lean_dec(x_97); +x_108 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 1, x_107); +return x_108; } } } else { -uint8_t x_108; +uint8_t x_109; lean_dec(x_91); lean_dec(x_89); -lean_dec(x_81); +lean_dec(x_82); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7267,31 +7203,31 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_108 = !lean_is_exclusive(x_93); -if (x_108 == 0) +x_109 = !lean_is_exclusive(x_93); +if (x_109 == 0) { return x_93; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_93, 0); -x_110 = lean_ctor_get(x_93, 1); +lean_object* x_110; lean_object* x_111; lean_object* x_112; +x_110 = lean_ctor_get(x_93, 0); +x_111 = lean_ctor_get(x_93, 1); +lean_inc(x_111); lean_inc(x_110); -lean_inc(x_109); lean_dec(x_93); -x_111 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_111, 0, x_109); -lean_ctor_set(x_111, 1, x_110); -return x_111; +x_112 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +return x_112; } } } else { -uint8_t x_112; +uint8_t x_113; lean_dec(x_89); -lean_dec(x_81); +lean_dec(x_82); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7306,30 +7242,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_112 = !lean_is_exclusive(x_90); -if (x_112 == 0) +x_113 = !lean_is_exclusive(x_90); +if (x_113 == 0) { return x_90; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; -x_113 = lean_ctor_get(x_90, 0); -x_114 = lean_ctor_get(x_90, 1); +lean_object* x_114; lean_object* x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_90, 0); +x_115 = lean_ctor_get(x_90, 1); +lean_inc(x_115); lean_inc(x_114); -lean_inc(x_113); lean_dec(x_90); -x_115 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_115, 0, x_113); -lean_ctor_set(x_115, 1, x_114); -return x_115; +x_116 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_116, 0, x_114); +lean_ctor_set(x_116, 1, x_115); +return x_116; } } } else { -uint8_t x_116; -lean_dec(x_81); +uint8_t x_117; +lean_dec(x_82); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7344,29 +7280,29 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_116 = !lean_is_exclusive(x_86); -if (x_116 == 0) +x_117 = !lean_is_exclusive(x_86); +if (x_117 == 0) { return x_86; } else { -lean_object* x_117; lean_object* x_118; lean_object* x_119; -x_117 = lean_ctor_get(x_86, 0); -x_118 = lean_ctor_get(x_86, 1); +lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_118 = lean_ctor_get(x_86, 0); +x_119 = lean_ctor_get(x_86, 1); +lean_inc(x_119); lean_inc(x_118); -lean_inc(x_117); lean_dec(x_86); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_117); -lean_ctor_set(x_119, 1, x_118); -return x_119; +x_120 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_120, 0, x_118); +lean_ctor_set(x_120, 1, x_119); +return x_120; } } } else { -uint8_t x_120; +uint8_t x_121; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7381,30 +7317,30 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_120 = !lean_is_exclusive(x_80); -if (x_120 == 0) +x_121 = !lean_is_exclusive(x_81); +if (x_121 == 0) { -return x_80; +return x_81; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; -x_121 = lean_ctor_get(x_80, 0); -x_122 = lean_ctor_get(x_80, 1); +lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_122 = lean_ctor_get(x_81, 0); +x_123 = lean_ctor_get(x_81, 1); +lean_inc(x_123); lean_inc(x_122); -lean_inc(x_121); -lean_dec(x_80); -x_123 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_123, 0, x_121); -lean_ctor_set(x_123, 1, x_122); -return x_123; +lean_dec(x_81); +x_124 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 1, x_123); +return x_124; } } } } else { -uint8_t x_124; +uint8_t x_125; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -7419,23 +7355,23 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_124 = !lean_is_exclusive(x_17); -if (x_124 == 0) +x_125 = !lean_is_exclusive(x_17); +if (x_125 == 0) { return x_17; } else { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_17, 0); -x_126 = lean_ctor_get(x_17, 1); +lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_126 = lean_ctor_get(x_17, 0); +x_127 = lean_ctor_get(x_17, 1); +lean_inc(x_127); lean_inc(x_126); -lean_inc(x_125); lean_dec(x_17); -x_127 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_127, 0, x_125); -lean_ctor_set(x_127, 1, x_126); -return x_127; +x_128 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); +return x_128; } } } @@ -7648,7 +7584,7 @@ lean_dec(x_2); return x_17; } } -static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1() { +static lean_object* _init_l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1() { _start: { lean_object* x_1; @@ -7656,13 +7592,13 @@ x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_propagateDIte), 10, 0); return x_1; } } -LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078_(lean_object* x_1) { +LEAN_EXPORT lean_object* l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054_(lean_object* x_1) { _start: { lean_object* x_2; uint8_t x_3; lean_object* x_4; lean_object* x_5; x_2 = l_Lean_Meta_Grind_propagateDIte___closed__2; x_3 = 1; -x_4 = l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1; +x_4 = l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1; x_5 = l___private_Lean_Meta_Tactic_Grind_PropagatorAttr_0__Lean_Meta_Grind_registerBuiltinPropagatorCore(x_2, x_3, x_4, x_1); return x_5; } @@ -7854,53 +7790,41 @@ l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__5 = _init_l_Lean_Meta_Grin lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__5); l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__6 = _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__6(); lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__6); -l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7 = _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__7); -l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8 = _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__8); -l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9 = _init_l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___lambda__1___closed__9); l_Lean_Meta_Grind_propagateEqUp___closed__1 = _init_l_Lean_Meta_Grind_propagateEqUp___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___closed__1); l_Lean_Meta_Grind_propagateEqUp___closed__2 = _init_l_Lean_Meta_Grind_propagateEqUp___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateEqUp___closed__2); -l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2118_(lean_io_mk_world()); +l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2114_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__1); -l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2 = _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__2); -l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3 = _init_l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_propagateEqDown___lambda__1___closed__3); -l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2347_(lean_io_mk_world()); +}l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2339_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Meta_Grind_propagateEqMatchDown___closed__1 = _init_l_Lean_Meta_Grind_propagateEqMatchDown___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_propagateEqMatchDown___closed__1); l_Lean_Meta_Grind_propagateEqMatchDown___closed__2 = _init_l_Lean_Meta_Grind_propagateEqMatchDown___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateEqMatchDown___closed__2); -l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2629_(lean_io_mk_world()); +l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateEqMatchDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2617_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Meta_Grind_propagateHEqDown___closed__1 = _init_l_Lean_Meta_Grind_propagateHEqDown___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_propagateHEqDown___closed__1); l_Lean_Meta_Grind_propagateHEqDown___closed__2 = _init_l_Lean_Meta_Grind_propagateHEqDown___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateHEqDown___closed__2); -l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2888_(lean_io_mk_world()); +l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateHEqDown_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_2872_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -}l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3148_(lean_io_mk_world()); +}l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateHEqUp_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3128_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Meta_Grind_propagateIte___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_propagateIte___lambda__1___closed__1(); @@ -7915,9 +7839,9 @@ l_Lean_Meta_Grind_propagateIte___closed__1 = _init_l_Lean_Meta_Grind_propagateIt lean_mark_persistent(l_Lean_Meta_Grind_propagateIte___closed__1); l_Lean_Meta_Grind_propagateIte___closed__2 = _init_l_Lean_Meta_Grind_propagateIte___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateIte___closed__2); -l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3530_(lean_io_mk_world()); +l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_3510_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__1 = _init_l_Lean_Meta_Grind_propagateDIte___lambda__1___closed__1(); @@ -7938,9 +7862,9 @@ l_Lean_Meta_Grind_propagateDIte___closed__1 = _init_l_Lean_Meta_Grind_propagateD lean_mark_persistent(l_Lean_Meta_Grind_propagateDIte___closed__1); l_Lean_Meta_Grind_propagateDIte___closed__2 = _init_l_Lean_Meta_Grind_propagateDIte___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_propagateDIte___closed__2); -l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1(); -lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078____closed__1); -if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4078_(lean_io_mk_world()); +l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1 = _init_l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1(); +lean_mark_persistent(l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054____closed__1); +if (builtin) {res = l___regBuiltin_Lean_Meta_Grind_propagateDIte_declare__1____x40_Lean_Meta_Tactic_Grind_Propagate___hyg_4054_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); }return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/PropagatorAttr.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/PropagatorAttr.c index 2beff5c9839d..848af7f89890 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/PropagatorAttr.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/PropagatorAttr.c @@ -3000,8 +3000,6 @@ x_34 = lean_ctor_get(x_32, 1); lean_inc(x_34); lean_dec(x_32); x_35 = l_Lean_declareBuiltin(x_33, x_29, x_3, x_4, x_34); -lean_dec(x_4); -lean_dec(x_3); if (lean_obj_tag(x_35) == 0) { lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Simp.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Simp.c index ba110f27abd9..7b057f2a3bc6 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Simp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Simp.c @@ -14,64 +14,55 @@ extern "C" { #endif static lean_object* l_Lean_Meta_Grind_simp___closed__7; -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_abstractNestedProofs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3; lean_object* l_Lean_Meta_Grind_eraseIrrelevantMData___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_unfoldReducible___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_foldProjs___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_normalizeLevels___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__12; lean_object* l_Lean_stringToMessageData(lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__1; static lean_object* l_Lean_Meta_Grind_simp___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_hasMVar(lean_object*); -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; static lean_object* l_Lean_Meta_Grind_simp___closed__4; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_eraseIrrelevantMData___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__9; lean_object* l_Lean_Meta_simp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_markNestedProofsImpl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__14; lean_object* l_Lean_Meta_Grind_foldProjs___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_eraseDoNotSimp___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__5; -double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); +lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_shareCommon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__3; +lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__15; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simpCore(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simpCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__11; -lean_object* lean_array_mk(lean_object*); lean_object* l_Lean_instantiateMVarsCore(lean_object*, lean_object*); -lean_object* l_Lean_isTracingEnabledForCore(lean_object*, lean_object*, lean_object*); -static double l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1; static lean_object* l_Lean_Meta_Grind_simp___closed__8; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_simp___closed__10; static lean_object* l_Lean_Meta_Grind_simp___closed__6; static lean_object* l_Lean_Meta_Grind_simp___closed__13; -lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_eraseDoNotSimp___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_simp___closed__16; lean_object* l_Lean_Meta_Grind_unfoldReducible___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simpCore(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: @@ -83,7 +74,7 @@ lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 4); +x_13 = lean_ctor_get(x_11, 3); lean_inc(x_13); lean_dec(x_11); x_14 = lean_ctor_get(x_3, 0); @@ -116,9 +107,9 @@ x_25 = !lean_is_exclusive(x_23); if (x_25 == 0) { lean_object* x_26; lean_object* x_27; uint8_t x_28; -x_26 = lean_ctor_get(x_23, 4); +x_26 = lean_ctor_get(x_23, 3); lean_dec(x_26); -lean_ctor_set(x_23, 4, x_21); +lean_ctor_set(x_23, 3, x_21); x_27 = lean_st_ref_set(x_4, x_23, x_24); x_28 = !lean_is_exclusive(x_27); if (x_28 == 0) @@ -147,7 +138,7 @@ lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean x_32 = lean_ctor_get(x_23, 0); x_33 = lean_ctor_get(x_23, 1); x_34 = lean_ctor_get(x_23, 2); -x_35 = lean_ctor_get(x_23, 3); +x_35 = lean_ctor_get(x_23, 4); x_36 = lean_ctor_get(x_23, 5); x_37 = lean_ctor_get(x_23, 6); x_38 = lean_ctor_get(x_23, 7); @@ -163,8 +154,8 @@ x_39 = lean_alloc_ctor(0, 8, 0); lean_ctor_set(x_39, 0, x_32); lean_ctor_set(x_39, 1, x_33); lean_ctor_set(x_39, 2, x_34); -lean_ctor_set(x_39, 3, x_35); -lean_ctor_set(x_39, 4, x_21); +lean_ctor_set(x_39, 3, x_21); +lean_ctor_set(x_39, 4, x_35); lean_ctor_set(x_39, 5, x_36); lean_ctor_set(x_39, 6, x_37); lean_ctor_set(x_39, 7, x_38); @@ -223,496 +214,125 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_10; -x_10 = l_Lean_Expr_hasMVar(x_1); -if (x_10 == 0) +uint8_t x_11; +x_11 = l_Lean_Expr_hasMVar(x_1); +if (x_11 == 0) { -lean_object* x_11; -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_1); -lean_ctor_set(x_11, 1, x_9); -return x_11; +lean_object* x_12; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_10); +return x_12; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_12 = lean_st_ref_get(x_6, x_9); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; +x_13 = lean_st_ref_get(x_7, x_10); +x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_ctor_get(x_13, 0); +x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = l_Lean_instantiateMVarsCore(x_15, x_1); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_16, 1); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_instantiateMVarsCore(x_16, x_1); +x_18 = lean_ctor_get(x_17, 0); lean_inc(x_18); -lean_dec(x_16); -x_19 = lean_st_ref_take(x_6, x_14); -x_20 = lean_ctor_get(x_19, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_19, 1); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = lean_st_ref_take(x_7, x_15); +x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); -lean_dec(x_19); -x_22 = !lean_is_exclusive(x_20); -if (x_22 == 0) +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +x_23 = !lean_is_exclusive(x_21); +if (x_23 == 0) { -lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_23 = lean_ctor_get(x_20, 0); -lean_dec(x_23); -lean_ctor_set(x_20, 0, x_18); -x_24 = lean_st_ref_set(x_6, x_20, x_21); -x_25 = !lean_is_exclusive(x_24); -if (x_25 == 0) +lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_24 = lean_ctor_get(x_21, 0); +lean_dec(x_24); +lean_ctor_set(x_21, 0, x_19); +x_25 = lean_st_ref_set(x_7, x_21, x_22); +x_26 = !lean_is_exclusive(x_25); +if (x_26 == 0) { -lean_object* x_26; -x_26 = lean_ctor_get(x_24, 0); -lean_dec(x_26); -lean_ctor_set(x_24, 0, x_17); -return x_24; +lean_object* x_27; +x_27 = lean_ctor_get(x_25, 0); +lean_dec(x_27); +lean_ctor_set(x_25, 0, x_18); +return x_25; } else { -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_24, 1); -lean_inc(x_27); -lean_dec(x_24); -x_28 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_28, 0, x_17); -lean_ctor_set(x_28, 1, x_27); -return x_28; +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_25, 1); +lean_inc(x_28); +lean_dec(x_25); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_18); +lean_ctor_set(x_29, 1, x_28); +return x_29; } } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_29 = lean_ctor_get(x_20, 1); -x_30 = lean_ctor_get(x_20, 2); -x_31 = lean_ctor_get(x_20, 3); -x_32 = lean_ctor_get(x_20, 4); +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_30 = lean_ctor_get(x_21, 1); +x_31 = lean_ctor_get(x_21, 2); +x_32 = lean_ctor_get(x_21, 3); +x_33 = lean_ctor_get(x_21, 4); +lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); -lean_inc(x_29); -lean_dec(x_20); -x_33 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_33, 0, x_18); -lean_ctor_set(x_33, 1, x_29); -lean_ctor_set(x_33, 2, x_30); -lean_ctor_set(x_33, 3, x_31); -lean_ctor_set(x_33, 4, x_32); -x_34 = lean_st_ref_set(x_6, x_33, x_21); -x_35 = lean_ctor_get(x_34, 1); -lean_inc(x_35); -if (lean_is_exclusive(x_34)) { - lean_ctor_release(x_34, 0); - lean_ctor_release(x_34, 1); - x_36 = x_34; +lean_dec(x_21); +x_34 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_34, 0, x_19); +lean_ctor_set(x_34, 1, x_30); +lean_ctor_set(x_34, 2, x_31); +lean_ctor_set(x_34, 3, x_32); +lean_ctor_set(x_34, 4, x_33); +x_35 = lean_st_ref_set(x_7, x_34, x_22); +x_36 = lean_ctor_get(x_35, 1); +lean_inc(x_36); +if (lean_is_exclusive(x_35)) { + lean_ctor_release(x_35, 0); + lean_ctor_release(x_35, 1); + x_37 = x_35; } else { - lean_dec_ref(x_34); - x_36 = lean_box(0); + lean_dec_ref(x_35); + x_37 = lean_box(0); } -if (lean_is_scalar(x_36)) { - x_37 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_37)) { + x_38 = lean_alloc_ctor(0, 2, 0); } else { - x_37 = x_36; -} -lean_ctor_set(x_37, 0, x_17); -lean_ctor_set(x_37, 1, x_35); -return x_37; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_ctor_get(x_7, 2); -x_11 = l_Lean_isTracingEnabledForCore(x_1, x_10, x_9); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -return x_11; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -lean_inc(x_14); -lean_inc(x_13); -lean_dec(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set(x_15, 1, x_14); -return x_15; -} -} -} -static double _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1() { -_start: -{ -lean_object* x_1; uint8_t x_2; double x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = 0; -x_3 = l_Float_ofScientific(x_1, x_2, x_1); -return x_3; -} -} -static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; -} -} -static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_11 = lean_ctor_get(x_8, 5); -x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_6, x_7, x_8, x_9, x_10); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_12, 1); -lean_inc(x_14); -lean_dec(x_12); -x_15 = lean_st_ref_take(x_9, x_14); -x_16 = lean_ctor_get(x_15, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_16, 3); -lean_inc(x_17); -x_18 = !lean_is_exclusive(x_15); -if (x_18 == 0) -{ -lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_19 = lean_ctor_get(x_15, 1); -x_20 = lean_ctor_get(x_15, 0); -lean_dec(x_20); -x_21 = !lean_is_exclusive(x_16); -if (x_21 == 0) -{ -lean_object* x_22; uint8_t x_23; -x_22 = lean_ctor_get(x_16, 3); -lean_dec(x_22); -x_23 = !lean_is_exclusive(x_17); -if (x_23 == 0) -{ -lean_object* x_24; double x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_24 = lean_ctor_get(x_17, 0); -x_25 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1; -x_26 = 0; -x_27 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; -x_28 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_28, 0, x_1); -lean_ctor_set(x_28, 1, x_27); -lean_ctor_set_float(x_28, sizeof(void*)*2, x_25); -lean_ctor_set_float(x_28, sizeof(void*)*2 + 8, x_25); -lean_ctor_set_uint8(x_28, sizeof(void*)*2 + 16, x_26); -x_29 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3; -x_30 = lean_alloc_ctor(9, 3, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_13); -lean_ctor_set(x_30, 2, x_29); -lean_inc(x_11); -lean_ctor_set(x_15, 1, x_30); -lean_ctor_set(x_15, 0, x_11); -x_31 = l_Lean_PersistentArray_push___rarg(x_24, x_15); -lean_ctor_set(x_17, 0, x_31); -x_32 = lean_st_ref_set(x_9, x_16, x_19); -x_33 = !lean_is_exclusive(x_32); -if (x_33 == 0) -{ -lean_object* x_34; lean_object* x_35; -x_34 = lean_ctor_get(x_32, 0); -lean_dec(x_34); -x_35 = lean_box(0); -lean_ctor_set(x_32, 0, x_35); -return x_32; + x_38 = x_37; } -else -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_36 = lean_ctor_get(x_32, 1); -lean_inc(x_36); -lean_dec(x_32); -x_37 = lean_box(0); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_37); +lean_ctor_set(x_38, 0, x_18); lean_ctor_set(x_38, 1, x_36); return x_38; } } -else -{ -uint64_t x_39; lean_object* x_40; double x_41; uint8_t x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_39 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); -x_40 = lean_ctor_get(x_17, 0); -lean_inc(x_40); -lean_dec(x_17); -x_41 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1; -x_42 = 0; -x_43 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; -x_44 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_44, 0, x_1); -lean_ctor_set(x_44, 1, x_43); -lean_ctor_set_float(x_44, sizeof(void*)*2, x_41); -lean_ctor_set_float(x_44, sizeof(void*)*2 + 8, x_41); -lean_ctor_set_uint8(x_44, sizeof(void*)*2 + 16, x_42); -x_45 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3; -x_46 = lean_alloc_ctor(9, 3, 0); -lean_ctor_set(x_46, 0, x_44); -lean_ctor_set(x_46, 1, x_13); -lean_ctor_set(x_46, 2, x_45); -lean_inc(x_11); -lean_ctor_set(x_15, 1, x_46); -lean_ctor_set(x_15, 0, x_11); -x_47 = l_Lean_PersistentArray_push___rarg(x_40, x_15); -x_48 = lean_alloc_ctor(0, 1, 8); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set_uint64(x_48, sizeof(void*)*1, x_39); -lean_ctor_set(x_16, 3, x_48); -x_49 = lean_st_ref_set(x_9, x_16, x_19); -x_50 = lean_ctor_get(x_49, 1); -lean_inc(x_50); -if (lean_is_exclusive(x_49)) { - lean_ctor_release(x_49, 0); - lean_ctor_release(x_49, 1); - x_51 = x_49; -} else { - lean_dec_ref(x_49); - x_51 = lean_box(0); -} -x_52 = lean_box(0); -if (lean_is_scalar(x_51)) { - x_53 = lean_alloc_ctor(0, 2, 0); -} else { - x_53 = x_51; -} -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_50); -return x_53; -} -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; lean_object* x_62; lean_object* x_63; double x_64; uint8_t x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_54 = lean_ctor_get(x_16, 0); -x_55 = lean_ctor_get(x_16, 1); -x_56 = lean_ctor_get(x_16, 2); -x_57 = lean_ctor_get(x_16, 4); -x_58 = lean_ctor_get(x_16, 5); -x_59 = lean_ctor_get(x_16, 6); -x_60 = lean_ctor_get(x_16, 7); -lean_inc(x_60); -lean_inc(x_59); -lean_inc(x_58); -lean_inc(x_57); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_16); -x_61 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); -x_62 = lean_ctor_get(x_17, 0); -lean_inc(x_62); -if (lean_is_exclusive(x_17)) { - lean_ctor_release(x_17, 0); - x_63 = x_17; -} else { - lean_dec_ref(x_17); - x_63 = lean_box(0); -} -x_64 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1; -x_65 = 0; -x_66 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; -x_67 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_67, 0, x_1); -lean_ctor_set(x_67, 1, x_66); -lean_ctor_set_float(x_67, sizeof(void*)*2, x_64); -lean_ctor_set_float(x_67, sizeof(void*)*2 + 8, x_64); -lean_ctor_set_uint8(x_67, sizeof(void*)*2 + 16, x_65); -x_68 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3; -x_69 = lean_alloc_ctor(9, 3, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_13); -lean_ctor_set(x_69, 2, x_68); -lean_inc(x_11); -lean_ctor_set(x_15, 1, x_69); -lean_ctor_set(x_15, 0, x_11); -x_70 = l_Lean_PersistentArray_push___rarg(x_62, x_15); -if (lean_is_scalar(x_63)) { - x_71 = lean_alloc_ctor(0, 1, 8); -} else { - x_71 = x_63; -} -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set_uint64(x_71, sizeof(void*)*1, x_61); -x_72 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_72, 0, x_54); -lean_ctor_set(x_72, 1, x_55); -lean_ctor_set(x_72, 2, x_56); -lean_ctor_set(x_72, 3, x_71); -lean_ctor_set(x_72, 4, x_57); -lean_ctor_set(x_72, 5, x_58); -lean_ctor_set(x_72, 6, x_59); -lean_ctor_set(x_72, 7, x_60); -x_73 = lean_st_ref_set(x_9, x_72, x_19); -x_74 = lean_ctor_get(x_73, 1); -lean_inc(x_74); -if (lean_is_exclusive(x_73)) { - lean_ctor_release(x_73, 0); - lean_ctor_release(x_73, 1); - x_75 = x_73; -} else { - lean_dec_ref(x_73); - x_75 = lean_box(0); -} -x_76 = lean_box(0); -if (lean_is_scalar(x_75)) { - x_77 = lean_alloc_ctor(0, 2, 0); -} else { - x_77 = x_75; -} -lean_ctor_set(x_77, 0, x_76); -lean_ctor_set(x_77, 1, x_74); -return x_77; -} -} -else -{ -lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; uint64_t x_87; lean_object* x_88; lean_object* x_89; double x_90; uint8_t x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -x_78 = lean_ctor_get(x_15, 1); -lean_inc(x_78); -lean_dec(x_15); -x_79 = lean_ctor_get(x_16, 0); -lean_inc(x_79); -x_80 = lean_ctor_get(x_16, 1); -lean_inc(x_80); -x_81 = lean_ctor_get(x_16, 2); -lean_inc(x_81); -x_82 = lean_ctor_get(x_16, 4); -lean_inc(x_82); -x_83 = lean_ctor_get(x_16, 5); -lean_inc(x_83); -x_84 = lean_ctor_get(x_16, 6); -lean_inc(x_84); -x_85 = lean_ctor_get(x_16, 7); -lean_inc(x_85); -if (lean_is_exclusive(x_16)) { - lean_ctor_release(x_16, 0); - lean_ctor_release(x_16, 1); - lean_ctor_release(x_16, 2); - lean_ctor_release(x_16, 3); - lean_ctor_release(x_16, 4); - lean_ctor_release(x_16, 5); - lean_ctor_release(x_16, 6); - lean_ctor_release(x_16, 7); - x_86 = x_16; -} else { - lean_dec_ref(x_16); - x_86 = lean_box(0); -} -x_87 = lean_ctor_get_uint64(x_17, sizeof(void*)*1); -x_88 = lean_ctor_get(x_17, 0); -lean_inc(x_88); -if (lean_is_exclusive(x_17)) { - lean_ctor_release(x_17, 0); - x_89 = x_17; -} else { - lean_dec_ref(x_17); - x_89 = lean_box(0); -} -x_90 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1; -x_91 = 0; -x_92 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; -x_93 = lean_alloc_ctor(0, 2, 17); -lean_ctor_set(x_93, 0, x_1); -lean_ctor_set(x_93, 1, x_92); -lean_ctor_set_float(x_93, sizeof(void*)*2, x_90); -lean_ctor_set_float(x_93, sizeof(void*)*2 + 8, x_90); -lean_ctor_set_uint8(x_93, sizeof(void*)*2 + 16, x_91); -x_94 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3; -x_95 = lean_alloc_ctor(9, 3, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_13); -lean_ctor_set(x_95, 2, x_94); -lean_inc(x_11); -x_96 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_96, 0, x_11); -lean_ctor_set(x_96, 1, x_95); -x_97 = l_Lean_PersistentArray_push___rarg(x_88, x_96); -if (lean_is_scalar(x_89)) { - x_98 = lean_alloc_ctor(0, 1, 8); -} else { - x_98 = x_89; -} -lean_ctor_set(x_98, 0, x_97); -lean_ctor_set_uint64(x_98, sizeof(void*)*1, x_87); -if (lean_is_scalar(x_86)) { - x_99 = lean_alloc_ctor(0, 8, 0); -} else { - x_99 = x_86; -} -lean_ctor_set(x_99, 0, x_79); -lean_ctor_set(x_99, 1, x_80); -lean_ctor_set(x_99, 2, x_81); -lean_ctor_set(x_99, 3, x_98); -lean_ctor_set(x_99, 4, x_82); -lean_ctor_set(x_99, 5, x_83); -lean_ctor_set(x_99, 6, x_84); -lean_ctor_set(x_99, 7, x_85); -x_100 = lean_st_ref_set(x_9, x_99, x_78); -x_101 = lean_ctor_get(x_100, 1); -lean_inc(x_101); -if (lean_is_exclusive(x_100)) { - lean_ctor_release(x_100, 0); - lean_ctor_release(x_100, 1); - x_102 = x_100; -} else { - lean_dec_ref(x_100); - x_102 = lean_box(0); -} -x_103 = lean_box(0); -if (lean_is_scalar(x_102)) { - x_104 = lean_alloc_ctor(0, 2, 0); -} else { - x_104 = x_102; } -lean_ctor_set(x_104, 0, x_103); -lean_ctor_set(x_104, 1, x_101); -return x_104; } -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1(lean_object* x_1, lean_object* x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_13; lean_object* x_14; -x_13 = lean_alloc_ctor(0, 2, 1); -lean_ctor_set(x_13, 0, x_1); -lean_ctor_set(x_13, 1, x_2); -lean_ctor_set_uint8(x_13, sizeof(void*)*2, x_3); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_13); -lean_ctor_set(x_14, 1, x_12); -return x_14; +lean_object* x_14; lean_object* x_15; +x_14 = lean_alloc_ctor(0, 2, 1); +lean_ctor_set(x_14, 0, x_1); +lean_ctor_set(x_14, 1, x_2); +lean_ctor_set_uint8(x_14, sizeof(void*)*2, x_3); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_13); +return x_15; } } static lean_object* _init_l_Lean_Meta_Grind_simp___closed__1() { @@ -816,13 +436,21 @@ return x_3; static lean_object* _init_l_Lean_Meta_Grind_simp___closed__13() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_simp___closed__14() { +_start: +{ lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2; +x_1 = l_Lean_Meta_Grind_simp___closed__13; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_simp___closed__14() { +static lean_object* _init_l_Lean_Meta_Grind_simp___closed__15() { _start: { lean_object* x_1; @@ -830,1182 +458,1152 @@ x_1 = lean_mk_string_unchecked("\n===>\n", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_simp___closed__15() { +static lean_object* _init_l_Lean_Meta_Grind_simp___closed__16() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_simp___closed__14; +x_1 = l_Lean_Meta_Grind_simp___closed__15; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +lean_object* x_11; uint8_t x_12; +x_11 = l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_12); -x_14 = l_Lean_Meta_Grind_simpCore(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -if (lean_obj_tag(x_14) == 0) +lean_inc(x_4); +lean_inc(x_13); +x_15 = l_Lean_Meta_Grind_simpCore(x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +if (lean_obj_tag(x_15) == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; +x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = lean_ctor_get(x_15, 0); +x_17 = lean_ctor_get(x_15, 1); lean_inc(x_17); -x_18 = lean_ctor_get(x_15, 1); -lean_inc(x_18); -x_19 = lean_ctor_get_uint8(x_15, sizeof(void*)*2); lean_dec(x_15); +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_16, 1); +lean_inc(x_19); +x_20 = lean_ctor_get_uint8(x_16, sizeof(void*)*2); +lean_dec(x_16); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_20 = l_Lean_Meta_Grind_abstractNestedProofs(x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_16); -if (lean_obj_tag(x_20) == 0) +x_21 = l_Lean_Meta_Grind_abstractNestedProofs(x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +if (lean_obj_tag(x_21) == 0) { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_20, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_20, 1); +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_21, 0); lean_inc(x_22); -lean_dec(x_20); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_23 = l_Lean_Meta_Grind_markNestedProofsImpl(x_21, x_5, x_6, x_7, x_8, x_22); -if (lean_obj_tag(x_23) == 0) +x_24 = l_Lean_Meta_Grind_markNestedProofsImpl(x_22, x_6, x_7, x_8, x_9, x_23); +if (lean_obj_tag(x_24) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_24, 0); lean_inc(x_25); -lean_dec(x_23); -x_26 = l_Lean_Meta_Grind_simp___closed__1; -x_27 = l_Lean_Meta_Grind_simp___closed__2; +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_Meta_Grind_simp___closed__1; +x_28 = l_Lean_Meta_Grind_simp___closed__2; +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_28 = l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(x_24, x_26, x_27, x_5, x_6, x_7, x_8, x_25); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); +x_29 = l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(x_25, x_27, x_28, x_6, x_7, x_8, x_9, x_26); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; +x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_Meta_Grind_simp___closed__3; -x_32 = l_Lean_Meta_Grind_simp___closed__4; +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = l_Lean_Meta_Grind_simp___closed__3; +x_33 = l_Lean_Meta_Grind_simp___closed__4; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_33 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_29, x_31, x_32, x_7, x_8, x_30); -if (lean_obj_tag(x_33) == 0) +x_34 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_30, x_32, x_33, x_8, x_9, x_31); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); +lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; +x_35 = lean_ctor_get(x_34, 0); lean_inc(x_35); -lean_dec(x_33); -x_36 = l_Lean_Meta_Grind_simp___closed__5; -x_37 = l_Lean_Meta_Grind_simp___closed__6; -x_38 = 0; +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = l_Lean_Meta_Grind_simp___closed__5; +x_38 = l_Lean_Meta_Grind_simp___closed__6; +x_39 = 0; +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_39 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_34, x_36, x_37, x_38, x_38, x_5, x_6, x_7, x_8, x_35); -if (lean_obj_tag(x_39) == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_39, 0); -lean_inc(x_40); -x_41 = lean_ctor_get(x_39, 1); +x_40 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_35, x_37, x_38, x_39, x_39, x_6, x_7, x_8, x_9, x_36); +if (lean_obj_tag(x_40) == 0) +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_41 = lean_ctor_get(x_40, 0); lean_inc(x_41); -lean_dec(x_39); -x_42 = l_Lean_Meta_Grind_simp___closed__7; +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = l_Lean_Meta_Grind_simp___closed__7; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_43 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_40, x_42, x_32, x_7, x_8, x_41); -if (lean_obj_tag(x_43) == 0) +x_44 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_41, x_43, x_33, x_8, x_9, x_42); +if (lean_obj_tag(x_44) == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_44 = lean_ctor_get(x_43, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_43, 1); +lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_45 = lean_ctor_get(x_44, 0); lean_inc(x_45); -lean_dec(x_43); -x_46 = l_Lean_Meta_Grind_simp___closed__8; -x_47 = l_Lean_Meta_Grind_simp___closed__9; +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = l_Lean_Meta_Grind_simp___closed__8; +x_48 = l_Lean_Meta_Grind_simp___closed__9; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_48 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_44, x_46, x_47, x_7, x_8, x_45); -if (lean_obj_tag(x_48) == 0) +x_49 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_45, x_47, x_48, x_8, x_9, x_46); +if (lean_obj_tag(x_49) == 0) { -lean_object* x_49; lean_object* x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_48, 0); -lean_inc(x_49); -x_50 = lean_ctor_get(x_48, 1); +lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_50 = lean_ctor_get(x_49, 0); lean_inc(x_50); -lean_dec(x_48); +x_51 = lean_ctor_get(x_49, 1); +lean_inc(x_51); +lean_dec(x_49); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_51 = l_Lean_Meta_Grind_canon(x_49, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_50); -if (lean_obj_tag(x_51) == 0) -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_52 = lean_ctor_get(x_51, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_51, 1); +x_52 = l_Lean_Meta_Grind_canon(x_50, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_51); +if (lean_obj_tag(x_52) == 0) +{ +lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_53 = lean_ctor_get(x_52, 0); lean_inc(x_53); -lean_dec(x_51); -x_54 = l_Lean_Meta_Grind_shareCommon(x_52, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_53); -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_56 = lean_ctor_get(x_54, 0); -x_57 = lean_ctor_get(x_54, 1); -x_58 = l_Lean_Meta_Grind_simp___closed__12; -x_59 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(x_58, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_57); -x_60 = lean_ctor_get(x_59, 0); -lean_inc(x_60); -x_61 = lean_unbox(x_60); +x_54 = lean_ctor_get(x_52, 1); +lean_inc(x_54); +lean_dec(x_52); +x_55 = l_Lean_Meta_Grind_shareCommon(x_53, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_54); +x_56 = !lean_is_exclusive(x_55); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; +x_57 = lean_ctor_get(x_55, 0); +x_58 = lean_ctor_get(x_55, 1); +x_59 = l_Lean_Meta_Grind_simp___closed__12; +x_60 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_59, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_58); +x_61 = lean_ctor_get(x_60, 0); +lean_inc(x_61); +x_62 = lean_unbox(x_61); +lean_dec(x_61); +if (x_62 == 0) +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_free_object(x_55); +lean_free_object(x_11); +lean_dec(x_13); +x_63 = lean_ctor_get(x_60, 1); +lean_inc(x_63); lean_dec(x_60); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; -lean_free_object(x_54); -lean_free_object(x_10); -lean_dec(x_12); -x_62 = lean_ctor_get(x_59, 1); -lean_inc(x_62); -lean_dec(x_59); -x_63 = lean_box(0); -x_64 = l_Lean_Meta_Grind_simp___lambda__1(x_56, x_18, x_19, x_63, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_62); +x_64 = lean_box(0); +x_65 = l_Lean_Meta_Grind_simp___lambda__1(x_57, x_19, x_20, x_64, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_63); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_64; +lean_dec(x_4); +return x_65; } else { -uint8_t x_65; -x_65 = !lean_is_exclusive(x_59); -if (x_65 == 0) -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_66 = lean_ctor_get(x_59, 1); -x_67 = lean_ctor_get(x_59, 0); -lean_dec(x_67); -x_68 = l_Lean_MessageData_ofExpr(x_12); -x_69 = l_Lean_Meta_Grind_simp___closed__13; -lean_ctor_set_tag(x_59, 7); -lean_ctor_set(x_59, 1, x_68); -lean_ctor_set(x_59, 0, x_69); -x_70 = l_Lean_Meta_Grind_simp___closed__15; -lean_ctor_set_tag(x_54, 7); -lean_ctor_set(x_54, 1, x_70); -lean_ctor_set(x_54, 0, x_59); -lean_inc(x_56); -x_71 = l_Lean_MessageData_ofExpr(x_56); -lean_ctor_set_tag(x_10, 7); -lean_ctor_set(x_10, 1, x_71); -lean_ctor_set(x_10, 0, x_54); -x_72 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_72, 0, x_10); -lean_ctor_set(x_72, 1, x_69); -x_73 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_58, x_72, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_66); -x_74 = lean_ctor_get(x_73, 0); -lean_inc(x_74); -x_75 = lean_ctor_get(x_73, 1); +uint8_t x_66; +x_66 = !lean_is_exclusive(x_60); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; +x_67 = lean_ctor_get(x_60, 1); +x_68 = lean_ctor_get(x_60, 0); +lean_dec(x_68); +x_69 = l_Lean_MessageData_ofExpr(x_13); +x_70 = l_Lean_Meta_Grind_simp___closed__14; +lean_ctor_set_tag(x_60, 7); +lean_ctor_set(x_60, 1, x_69); +lean_ctor_set(x_60, 0, x_70); +x_71 = l_Lean_Meta_Grind_simp___closed__16; +lean_ctor_set_tag(x_55, 7); +lean_ctor_set(x_55, 1, x_71); +lean_ctor_set(x_55, 0, x_60); +lean_inc(x_57); +x_72 = l_Lean_MessageData_ofExpr(x_57); +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_72); +lean_ctor_set(x_11, 0, x_55); +x_73 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_73, 0, x_11); +lean_ctor_set(x_73, 1, x_70); +x_74 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_59, x_73, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_67); +x_75 = lean_ctor_get(x_74, 0); lean_inc(x_75); -lean_dec(x_73); -x_76 = l_Lean_Meta_Grind_simp___lambda__1(x_56, x_18, x_19, x_74, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_77 = l_Lean_Meta_Grind_simp___lambda__1(x_57, x_19, x_20, x_75, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_76); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_74); -return x_76; +lean_dec(x_4); +lean_dec(x_75); +return x_77; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_77 = lean_ctor_get(x_59, 1); -lean_inc(x_77); -lean_dec(x_59); -x_78 = l_Lean_MessageData_ofExpr(x_12); -x_79 = l_Lean_Meta_Grind_simp___closed__13; -x_80 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_80, 0, x_79); -lean_ctor_set(x_80, 1, x_78); -x_81 = l_Lean_Meta_Grind_simp___closed__15; -lean_ctor_set_tag(x_54, 7); -lean_ctor_set(x_54, 1, x_81); -lean_ctor_set(x_54, 0, x_80); -lean_inc(x_56); -x_82 = l_Lean_MessageData_ofExpr(x_56); -lean_ctor_set_tag(x_10, 7); -lean_ctor_set(x_10, 1, x_82); -lean_ctor_set(x_10, 0, x_54); -x_83 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_83, 0, x_10); -lean_ctor_set(x_83, 1, x_79); -x_84 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_58, x_83, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_77); -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -x_86 = lean_ctor_get(x_84, 1); +lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_78 = lean_ctor_get(x_60, 1); +lean_inc(x_78); +lean_dec(x_60); +x_79 = l_Lean_MessageData_ofExpr(x_13); +x_80 = l_Lean_Meta_Grind_simp___closed__14; +x_81 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_79); +x_82 = l_Lean_Meta_Grind_simp___closed__16; +lean_ctor_set_tag(x_55, 7); +lean_ctor_set(x_55, 1, x_82); +lean_ctor_set(x_55, 0, x_81); +lean_inc(x_57); +x_83 = l_Lean_MessageData_ofExpr(x_57); +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_83); +lean_ctor_set(x_11, 0, x_55); +x_84 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_84, 0, x_11); +lean_ctor_set(x_84, 1, x_80); +x_85 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_59, x_84, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_78); +x_86 = lean_ctor_get(x_85, 0); lean_inc(x_86); -lean_dec(x_84); -x_87 = l_Lean_Meta_Grind_simp___lambda__1(x_56, x_18, x_19, x_85, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_86); +x_87 = lean_ctor_get(x_85, 1); +lean_inc(x_87); +lean_dec(x_85); +x_88 = l_Lean_Meta_Grind_simp___lambda__1(x_57, x_19, x_20, x_86, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_87); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_85); -return x_87; +lean_dec(x_4); +lean_dec(x_86); +return x_88; } } } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; -x_88 = lean_ctor_get(x_54, 0); -x_89 = lean_ctor_get(x_54, 1); +lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; +x_89 = lean_ctor_get(x_55, 0); +x_90 = lean_ctor_get(x_55, 1); +lean_inc(x_90); lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_54); -x_90 = l_Lean_Meta_Grind_simp___closed__12; -x_91 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(x_90, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_89); -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_unbox(x_92); +lean_dec(x_55); +x_91 = l_Lean_Meta_Grind_simp___closed__12; +x_92 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_91, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_90); +x_93 = lean_ctor_get(x_92, 0); +lean_inc(x_93); +x_94 = lean_unbox(x_93); +lean_dec(x_93); +if (x_94 == 0) +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; +lean_free_object(x_11); +lean_dec(x_13); +x_95 = lean_ctor_get(x_92, 1); +lean_inc(x_95); lean_dec(x_92); -if (x_93 == 0) -{ -lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_free_object(x_10); -lean_dec(x_12); -x_94 = lean_ctor_get(x_91, 1); -lean_inc(x_94); -lean_dec(x_91); -x_95 = lean_box(0); -x_96 = l_Lean_Meta_Grind_simp___lambda__1(x_88, x_18, x_19, x_95, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_94); +x_96 = lean_box(0); +x_97 = l_Lean_Meta_Grind_simp___lambda__1(x_89, x_19, x_20, x_96, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_95); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_96; +lean_dec(x_4); +return x_97; } else { -lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_97 = lean_ctor_get(x_91, 1); -lean_inc(x_97); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_98 = x_91; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +x_98 = lean_ctor_get(x_92, 1); +lean_inc(x_98); +if (lean_is_exclusive(x_92)) { + lean_ctor_release(x_92, 0); + lean_ctor_release(x_92, 1); + x_99 = x_92; } else { - lean_dec_ref(x_91); - x_98 = lean_box(0); + lean_dec_ref(x_92); + x_99 = lean_box(0); } -x_99 = l_Lean_MessageData_ofExpr(x_12); -x_100 = l_Lean_Meta_Grind_simp___closed__13; -if (lean_is_scalar(x_98)) { - x_101 = lean_alloc_ctor(7, 2, 0); +x_100 = l_Lean_MessageData_ofExpr(x_13); +x_101 = l_Lean_Meta_Grind_simp___closed__14; +if (lean_is_scalar(x_99)) { + x_102 = lean_alloc_ctor(7, 2, 0); } else { - x_101 = x_98; - lean_ctor_set_tag(x_101, 7); -} -lean_ctor_set(x_101, 0, x_100); -lean_ctor_set(x_101, 1, x_99); -x_102 = l_Lean_Meta_Grind_simp___closed__15; -x_103 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_103, 0, x_101); -lean_ctor_set(x_103, 1, x_102); -lean_inc(x_88); -x_104 = l_Lean_MessageData_ofExpr(x_88); -lean_ctor_set_tag(x_10, 7); -lean_ctor_set(x_10, 1, x_104); -lean_ctor_set(x_10, 0, x_103); -x_105 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_105, 0, x_10); -lean_ctor_set(x_105, 1, x_100); -x_106 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_90, x_105, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_97); -x_107 = lean_ctor_get(x_106, 0); -lean_inc(x_107); -x_108 = lean_ctor_get(x_106, 1); + x_102 = x_99; + lean_ctor_set_tag(x_102, 7); +} +lean_ctor_set(x_102, 0, x_101); +lean_ctor_set(x_102, 1, x_100); +x_103 = l_Lean_Meta_Grind_simp___closed__16; +x_104 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_104, 0, x_102); +lean_ctor_set(x_104, 1, x_103); +lean_inc(x_89); +x_105 = l_Lean_MessageData_ofExpr(x_89); +lean_ctor_set_tag(x_11, 7); +lean_ctor_set(x_11, 1, x_105); +lean_ctor_set(x_11, 0, x_104); +x_106 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_106, 0, x_11); +lean_ctor_set(x_106, 1, x_101); +x_107 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_91, x_106, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_98); +x_108 = lean_ctor_get(x_107, 0); lean_inc(x_108); -lean_dec(x_106); -x_109 = l_Lean_Meta_Grind_simp___lambda__1(x_88, x_18, x_19, x_107, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_108); +x_109 = lean_ctor_get(x_107, 1); +lean_inc(x_109); +lean_dec(x_107); +x_110 = l_Lean_Meta_Grind_simp___lambda__1(x_89, x_19, x_20, x_108, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_109); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_107); -return x_109; +lean_dec(x_4); +lean_dec(x_108); +return x_110; } } } else { -uint8_t x_110; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_111; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_110 = !lean_is_exclusive(x_51); -if (x_110 == 0) +lean_dec(x_4); +x_111 = !lean_is_exclusive(x_52); +if (x_111 == 0) { -return x_51; +return x_52; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; -x_111 = lean_ctor_get(x_51, 0); -x_112 = lean_ctor_get(x_51, 1); +lean_object* x_112; lean_object* x_113; lean_object* x_114; +x_112 = lean_ctor_get(x_52, 0); +x_113 = lean_ctor_get(x_52, 1); +lean_inc(x_113); lean_inc(x_112); -lean_inc(x_111); -lean_dec(x_51); -x_113 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_113, 0, x_111); -lean_ctor_set(x_113, 1, x_112); -return x_113; +lean_dec(x_52); +x_114 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_114, 0, x_112); +lean_ctor_set(x_114, 1, x_113); +return x_114; } } } else { -uint8_t x_114; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_115; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_114 = !lean_is_exclusive(x_48); -if (x_114 == 0) +lean_dec(x_4); +x_115 = !lean_is_exclusive(x_49); +if (x_115 == 0) { -return x_48; +return x_49; } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; -x_115 = lean_ctor_get(x_48, 0); -x_116 = lean_ctor_get(x_48, 1); +lean_object* x_116; lean_object* x_117; lean_object* x_118; +x_116 = lean_ctor_get(x_49, 0); +x_117 = lean_ctor_get(x_49, 1); +lean_inc(x_117); lean_inc(x_116); -lean_inc(x_115); -lean_dec(x_48); -x_117 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_117, 0, x_115); -lean_ctor_set(x_117, 1, x_116); -return x_117; +lean_dec(x_49); +x_118 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +return x_118; } } } else { -uint8_t x_118; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_119; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_118 = !lean_is_exclusive(x_43); -if (x_118 == 0) +lean_dec(x_4); +x_119 = !lean_is_exclusive(x_44); +if (x_119 == 0) { -return x_43; +return x_44; } else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; -x_119 = lean_ctor_get(x_43, 0); -x_120 = lean_ctor_get(x_43, 1); +lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_120 = lean_ctor_get(x_44, 0); +x_121 = lean_ctor_get(x_44, 1); +lean_inc(x_121); lean_inc(x_120); -lean_inc(x_119); -lean_dec(x_43); -x_121 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_121, 0, x_119); -lean_ctor_set(x_121, 1, x_120); -return x_121; +lean_dec(x_44); +x_122 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_122, 0, x_120); +lean_ctor_set(x_122, 1, x_121); +return x_122; } } } else { -uint8_t x_122; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_123; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_122 = !lean_is_exclusive(x_39); -if (x_122 == 0) +lean_dec(x_4); +x_123 = !lean_is_exclusive(x_40); +if (x_123 == 0) { -return x_39; +return x_40; } else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_123 = lean_ctor_get(x_39, 0); -x_124 = lean_ctor_get(x_39, 1); +lean_object* x_124; lean_object* x_125; lean_object* x_126; +x_124 = lean_ctor_get(x_40, 0); +x_125 = lean_ctor_get(x_40, 1); +lean_inc(x_125); lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_39); -x_125 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_125, 0, x_123); -lean_ctor_set(x_125, 1, x_124); -return x_125; +lean_dec(x_40); +x_126 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_126, 0, x_124); +lean_ctor_set(x_126, 1, x_125); +return x_126; } } } else { -uint8_t x_126; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_127; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_126 = !lean_is_exclusive(x_33); -if (x_126 == 0) +lean_dec(x_4); +x_127 = !lean_is_exclusive(x_34); +if (x_127 == 0) { -return x_33; +return x_34; } else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_127 = lean_ctor_get(x_33, 0); -x_128 = lean_ctor_get(x_33, 1); +lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_128 = lean_ctor_get(x_34, 0); +x_129 = lean_ctor_get(x_34, 1); +lean_inc(x_129); lean_inc(x_128); -lean_inc(x_127); -lean_dec(x_33); -x_129 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_129, 0, x_127); -lean_ctor_set(x_129, 1, x_128); -return x_129; +lean_dec(x_34); +x_130 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_130, 0, x_128); +lean_ctor_set(x_130, 1, x_129); +return x_130; } } } else { -uint8_t x_130; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_131; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_130 = !lean_is_exclusive(x_28); -if (x_130 == 0) +lean_dec(x_4); +x_131 = !lean_is_exclusive(x_29); +if (x_131 == 0) { -return x_28; +return x_29; } else { -lean_object* x_131; lean_object* x_132; lean_object* x_133; -x_131 = lean_ctor_get(x_28, 0); -x_132 = lean_ctor_get(x_28, 1); +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_29, 0); +x_133 = lean_ctor_get(x_29, 1); +lean_inc(x_133); lean_inc(x_132); -lean_inc(x_131); -lean_dec(x_28); -x_133 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_133, 0, x_131); -lean_ctor_set(x_133, 1, x_132); -return x_133; +lean_dec(x_29); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; } } } else { -uint8_t x_134; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_135; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_134 = !lean_is_exclusive(x_23); -if (x_134 == 0) +lean_dec(x_4); +x_135 = !lean_is_exclusive(x_24); +if (x_135 == 0) { -return x_23; +return x_24; } else { -lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_135 = lean_ctor_get(x_23, 0); -x_136 = lean_ctor_get(x_23, 1); +lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_136 = lean_ctor_get(x_24, 0); +x_137 = lean_ctor_get(x_24, 1); +lean_inc(x_137); lean_inc(x_136); -lean_inc(x_135); -lean_dec(x_23); -x_137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_137, 0, x_135); -lean_ctor_set(x_137, 1, x_136); -return x_137; +lean_dec(x_24); +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +return x_138; } } } else { -uint8_t x_138; -lean_dec(x_18); -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_139; +lean_dec(x_19); +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_138 = !lean_is_exclusive(x_20); -if (x_138 == 0) +lean_dec(x_4); +x_139 = !lean_is_exclusive(x_21); +if (x_139 == 0) { -return x_20; +return x_21; } else { -lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_139 = lean_ctor_get(x_20, 0); -x_140 = lean_ctor_get(x_20, 1); +lean_object* x_140; lean_object* x_141; lean_object* x_142; +x_140 = lean_ctor_get(x_21, 0); +x_141 = lean_ctor_get(x_21, 1); +lean_inc(x_141); lean_inc(x_140); -lean_inc(x_139); -lean_dec(x_20); -x_141 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_141, 0, x_139); -lean_ctor_set(x_141, 1, x_140); -return x_141; +lean_dec(x_21); +x_142 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 1, x_141); +return x_142; } } } else { -uint8_t x_142; -lean_free_object(x_10); -lean_dec(x_12); +uint8_t x_143; +lean_free_object(x_11); +lean_dec(x_13); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_142 = !lean_is_exclusive(x_14); -if (x_142 == 0) +lean_dec(x_4); +x_143 = !lean_is_exclusive(x_15); +if (x_143 == 0) { -return x_14; +return x_15; } else { -lean_object* x_143; lean_object* x_144; lean_object* x_145; -x_143 = lean_ctor_get(x_14, 0); -x_144 = lean_ctor_get(x_14, 1); +lean_object* x_144; lean_object* x_145; lean_object* x_146; +x_144 = lean_ctor_get(x_15, 0); +x_145 = lean_ctor_get(x_15, 1); +lean_inc(x_145); lean_inc(x_144); -lean_inc(x_143); -lean_dec(x_14); -x_145 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_145, 0, x_143); -lean_ctor_set(x_145, 1, x_144); -return x_145; +lean_dec(x_15); +x_146 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +return x_146; } } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_146 = lean_ctor_get(x_10, 0); -x_147 = lean_ctor_get(x_10, 1); +lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_147 = lean_ctor_get(x_11, 0); +x_148 = lean_ctor_get(x_11, 1); +lean_inc(x_148); lean_inc(x_147); -lean_inc(x_146); -lean_dec(x_10); +lean_dec(x_11); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_3); -lean_inc(x_146); -x_148 = l_Lean_Meta_Grind_simpCore(x_146, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_147); -if (lean_obj_tag(x_148) == 0) -{ -lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; uint8_t x_153; lean_object* x_154; -x_149 = lean_ctor_get(x_148, 0); -lean_inc(x_149); -x_150 = lean_ctor_get(x_148, 1); +lean_inc(x_4); +lean_inc(x_147); +x_149 = l_Lean_Meta_Grind_simpCore(x_147, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_148); +if (lean_obj_tag(x_149) == 0) +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; lean_object* x_155; +x_150 = lean_ctor_get(x_149, 0); lean_inc(x_150); -lean_dec(x_148); -x_151 = lean_ctor_get(x_149, 0); +x_151 = lean_ctor_get(x_149, 1); lean_inc(x_151); -x_152 = lean_ctor_get(x_149, 1); -lean_inc(x_152); -x_153 = lean_ctor_get_uint8(x_149, sizeof(void*)*2); lean_dec(x_149); +x_152 = lean_ctor_get(x_150, 0); +lean_inc(x_152); +x_153 = lean_ctor_get(x_150, 1); +lean_inc(x_153); +x_154 = lean_ctor_get_uint8(x_150, sizeof(void*)*2); +lean_dec(x_150); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_154 = l_Lean_Meta_Grind_abstractNestedProofs(x_151, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_150); -if (lean_obj_tag(x_154) == 0) -{ -lean_object* x_155; lean_object* x_156; lean_object* x_157; -x_155 = lean_ctor_get(x_154, 0); -lean_inc(x_155); -x_156 = lean_ctor_get(x_154, 1); +x_155 = l_Lean_Meta_Grind_abstractNestedProofs(x_152, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_151); +if (lean_obj_tag(x_155) == 0) +{ +lean_object* x_156; lean_object* x_157; lean_object* x_158; +x_156 = lean_ctor_get(x_155, 0); lean_inc(x_156); -lean_dec(x_154); +x_157 = lean_ctor_get(x_155, 1); +lean_inc(x_157); +lean_dec(x_155); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_157 = l_Lean_Meta_Grind_markNestedProofsImpl(x_155, x_5, x_6, x_7, x_8, x_156); -if (lean_obj_tag(x_157) == 0) -{ -lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; -x_158 = lean_ctor_get(x_157, 0); -lean_inc(x_158); -x_159 = lean_ctor_get(x_157, 1); +x_158 = l_Lean_Meta_Grind_markNestedProofsImpl(x_156, x_6, x_7, x_8, x_9, x_157); +if (lean_obj_tag(x_158) == 0) +{ +lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_159 = lean_ctor_get(x_158, 0); lean_inc(x_159); -lean_dec(x_157); -x_160 = l_Lean_Meta_Grind_simp___closed__1; -x_161 = l_Lean_Meta_Grind_simp___closed__2; +x_160 = lean_ctor_get(x_158, 1); +lean_inc(x_160); +lean_dec(x_158); +x_161 = l_Lean_Meta_Grind_simp___closed__1; +x_162 = l_Lean_Meta_Grind_simp___closed__2; +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_162 = l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(x_158, x_160, x_161, x_5, x_6, x_7, x_8, x_159); -if (lean_obj_tag(x_162) == 0) -{ -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; -x_163 = lean_ctor_get(x_162, 0); -lean_inc(x_163); -x_164 = lean_ctor_get(x_162, 1); +x_163 = l_Lean_Core_transform___at_Lean_Meta_Grind_unfoldReducible___spec__1(x_159, x_161, x_162, x_6, x_7, x_8, x_9, x_160); +if (lean_obj_tag(x_163) == 0) +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; +x_164 = lean_ctor_get(x_163, 0); lean_inc(x_164); -lean_dec(x_162); -x_165 = l_Lean_Meta_Grind_simp___closed__3; -x_166 = l_Lean_Meta_Grind_simp___closed__4; +x_165 = lean_ctor_get(x_163, 1); +lean_inc(x_165); +lean_dec(x_163); +x_166 = l_Lean_Meta_Grind_simp___closed__3; +x_167 = l_Lean_Meta_Grind_simp___closed__4; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_167 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_163, x_165, x_166, x_7, x_8, x_164); -if (lean_obj_tag(x_167) == 0) +x_168 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_164, x_166, x_167, x_8, x_9, x_165); +if (lean_obj_tag(x_168) == 0) { -lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; uint8_t x_172; lean_object* x_173; -x_168 = lean_ctor_get(x_167, 0); -lean_inc(x_168); -x_169 = lean_ctor_get(x_167, 1); +lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; uint8_t x_173; lean_object* x_174; +x_169 = lean_ctor_get(x_168, 0); lean_inc(x_169); -lean_dec(x_167); -x_170 = l_Lean_Meta_Grind_simp___closed__5; -x_171 = l_Lean_Meta_Grind_simp___closed__6; -x_172 = 0; +x_170 = lean_ctor_get(x_168, 1); +lean_inc(x_170); +lean_dec(x_168); +x_171 = l_Lean_Meta_Grind_simp___closed__5; +x_172 = l_Lean_Meta_Grind_simp___closed__6; +x_173 = 0; +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_173 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_168, x_170, x_171, x_172, x_172, x_5, x_6, x_7, x_8, x_169); -if (lean_obj_tag(x_173) == 0) -{ -lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; -x_174 = lean_ctor_get(x_173, 0); -lean_inc(x_174); -x_175 = lean_ctor_get(x_173, 1); +x_174 = l_Lean_Meta_transform___at_Lean_Meta_zetaReduce___spec__1(x_169, x_171, x_172, x_173, x_173, x_6, x_7, x_8, x_9, x_170); +if (lean_obj_tag(x_174) == 0) +{ +lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; +x_175 = lean_ctor_get(x_174, 0); lean_inc(x_175); -lean_dec(x_173); -x_176 = l_Lean_Meta_Grind_simp___closed__7; +x_176 = lean_ctor_get(x_174, 1); +lean_inc(x_176); +lean_dec(x_174); +x_177 = l_Lean_Meta_Grind_simp___closed__7; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_177 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_174, x_176, x_166, x_7, x_8, x_175); -if (lean_obj_tag(x_177) == 0) +x_178 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_175, x_177, x_167, x_8, x_9, x_176); +if (lean_obj_tag(x_178) == 0) { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; -x_178 = lean_ctor_get(x_177, 0); -lean_inc(x_178); -x_179 = lean_ctor_get(x_177, 1); +lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +x_179 = lean_ctor_get(x_178, 0); lean_inc(x_179); -lean_dec(x_177); -x_180 = l_Lean_Meta_Grind_simp___closed__8; -x_181 = l_Lean_Meta_Grind_simp___closed__9; +x_180 = lean_ctor_get(x_178, 1); +lean_inc(x_180); +lean_dec(x_178); +x_181 = l_Lean_Meta_Grind_simp___closed__8; +x_182 = l_Lean_Meta_Grind_simp___closed__9; +lean_inc(x_9); lean_inc(x_8); -lean_inc(x_7); -x_182 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_178, x_180, x_181, x_7, x_8, x_179); -if (lean_obj_tag(x_182) == 0) +x_183 = l_Lean_Core_transform___at_Lean_Core_betaReduce___spec__1(x_179, x_181, x_182, x_8, x_9, x_180); +if (lean_obj_tag(x_183) == 0) { -lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_183 = lean_ctor_get(x_182, 0); -lean_inc(x_183); -x_184 = lean_ctor_get(x_182, 1); +lean_object* x_184; lean_object* x_185; lean_object* x_186; +x_184 = lean_ctor_get(x_183, 0); lean_inc(x_184); -lean_dec(x_182); +x_185 = lean_ctor_get(x_183, 1); +lean_inc(x_185); +lean_dec(x_183); +lean_inc(x_9); lean_inc(x_8); lean_inc(x_7); lean_inc(x_6); -lean_inc(x_5); -x_185 = l_Lean_Meta_Grind_canon(x_183, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_184); -if (lean_obj_tag(x_185) == 0) -{ -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; uint8_t x_195; -x_186 = lean_ctor_get(x_185, 0); -lean_inc(x_186); -x_187 = lean_ctor_get(x_185, 1); +x_186 = l_Lean_Meta_Grind_canon(x_184, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_185); +if (lean_obj_tag(x_186) == 0) +{ +lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; uint8_t x_196; +x_187 = lean_ctor_get(x_186, 0); lean_inc(x_187); -lean_dec(x_185); -x_188 = l_Lean_Meta_Grind_shareCommon(x_186, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_187); -x_189 = lean_ctor_get(x_188, 0); -lean_inc(x_189); -x_190 = lean_ctor_get(x_188, 1); +x_188 = lean_ctor_get(x_186, 1); +lean_inc(x_188); +lean_dec(x_186); +x_189 = l_Lean_Meta_Grind_shareCommon(x_187, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_188); +x_190 = lean_ctor_get(x_189, 0); lean_inc(x_190); -if (lean_is_exclusive(x_188)) { - lean_ctor_release(x_188, 0); - lean_ctor_release(x_188, 1); - x_191 = x_188; +x_191 = lean_ctor_get(x_189, 1); +lean_inc(x_191); +if (lean_is_exclusive(x_189)) { + lean_ctor_release(x_189, 0); + lean_ctor_release(x_189, 1); + x_192 = x_189; } else { - lean_dec_ref(x_188); - x_191 = lean_box(0); -} -x_192 = l_Lean_Meta_Grind_simp___closed__12; -x_193 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(x_192, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_190); -x_194 = lean_ctor_get(x_193, 0); -lean_inc(x_194); -x_195 = lean_unbox(x_194); + lean_dec_ref(x_189); + x_192 = lean_box(0); +} +x_193 = l_Lean_Meta_Grind_simp___closed__12; +x_194 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_193, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_191); +x_195 = lean_ctor_get(x_194, 0); +lean_inc(x_195); +x_196 = lean_unbox(x_195); +lean_dec(x_195); +if (x_196 == 0) +{ +lean_object* x_197; lean_object* x_198; lean_object* x_199; +lean_dec(x_192); +lean_dec(x_147); +x_197 = lean_ctor_get(x_194, 1); +lean_inc(x_197); lean_dec(x_194); -if (x_195 == 0) -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; -lean_dec(x_191); -lean_dec(x_146); -x_196 = lean_ctor_get(x_193, 1); -lean_inc(x_196); -lean_dec(x_193); -x_197 = lean_box(0); -x_198 = l_Lean_Meta_Grind_simp___lambda__1(x_189, x_152, x_153, x_197, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_196); +x_198 = lean_box(0); +x_199 = l_Lean_Meta_Grind_simp___lambda__1(x_190, x_153, x_154, x_198, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_197); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -return x_198; +lean_dec(x_4); +return x_199; } else { -lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; -x_199 = lean_ctor_get(x_193, 1); -lean_inc(x_199); -if (lean_is_exclusive(x_193)) { - lean_ctor_release(x_193, 0); - lean_ctor_release(x_193, 1); - x_200 = x_193; +lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; +x_200 = lean_ctor_get(x_194, 1); +lean_inc(x_200); +if (lean_is_exclusive(x_194)) { + lean_ctor_release(x_194, 0); + lean_ctor_release(x_194, 1); + x_201 = x_194; } else { - lean_dec_ref(x_193); - x_200 = lean_box(0); + lean_dec_ref(x_194); + x_201 = lean_box(0); } -x_201 = l_Lean_MessageData_ofExpr(x_146); -x_202 = l_Lean_Meta_Grind_simp___closed__13; -if (lean_is_scalar(x_200)) { - x_203 = lean_alloc_ctor(7, 2, 0); +x_202 = l_Lean_MessageData_ofExpr(x_147); +x_203 = l_Lean_Meta_Grind_simp___closed__14; +if (lean_is_scalar(x_201)) { + x_204 = lean_alloc_ctor(7, 2, 0); } else { - x_203 = x_200; - lean_ctor_set_tag(x_203, 7); -} -lean_ctor_set(x_203, 0, x_202); -lean_ctor_set(x_203, 1, x_201); -x_204 = l_Lean_Meta_Grind_simp___closed__15; -if (lean_is_scalar(x_191)) { - x_205 = lean_alloc_ctor(7, 2, 0); + x_204 = x_201; + lean_ctor_set_tag(x_204, 7); +} +lean_ctor_set(x_204, 0, x_203); +lean_ctor_set(x_204, 1, x_202); +x_205 = l_Lean_Meta_Grind_simp___closed__16; +if (lean_is_scalar(x_192)) { + x_206 = lean_alloc_ctor(7, 2, 0); } else { - x_205 = x_191; - lean_ctor_set_tag(x_205, 7); -} -lean_ctor_set(x_205, 0, x_203); -lean_ctor_set(x_205, 1, x_204); -lean_inc(x_189); -x_206 = l_Lean_MessageData_ofExpr(x_189); -x_207 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_207, 0, x_205); -lean_ctor_set(x_207, 1, x_206); + x_206 = x_192; + lean_ctor_set_tag(x_206, 7); +} +lean_ctor_set(x_206, 0, x_204); +lean_ctor_set(x_206, 1, x_205); +lean_inc(x_190); +x_207 = l_Lean_MessageData_ofExpr(x_190); x_208 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_208, 0, x_207); -lean_ctor_set(x_208, 1, x_202); -x_209 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_192, x_208, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_199); -x_210 = lean_ctor_get(x_209, 0); -lean_inc(x_210); -x_211 = lean_ctor_get(x_209, 1); +lean_ctor_set(x_208, 0, x_206); +lean_ctor_set(x_208, 1, x_207); +x_209 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_209, 0, x_208); +lean_ctor_set(x_209, 1, x_203); +x_210 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_193, x_209, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_200); +x_211 = lean_ctor_get(x_210, 0); lean_inc(x_211); -lean_dec(x_209); -x_212 = l_Lean_Meta_Grind_simp___lambda__1(x_189, x_152, x_153, x_210, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_211); +x_212 = lean_ctor_get(x_210, 1); +lean_inc(x_212); +lean_dec(x_210); +x_213 = l_Lean_Meta_Grind_simp___lambda__1(x_190, x_153, x_154, x_211, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_212); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_210); -return x_212; +lean_dec(x_4); +lean_dec(x_211); +return x_213; } } else { -lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_213 = lean_ctor_get(x_185, 0); -lean_inc(x_213); -x_214 = lean_ctor_get(x_185, 1); +lean_dec(x_4); +x_214 = lean_ctor_get(x_186, 0); lean_inc(x_214); -if (lean_is_exclusive(x_185)) { - lean_ctor_release(x_185, 0); - lean_ctor_release(x_185, 1); - x_215 = x_185; +x_215 = lean_ctor_get(x_186, 1); +lean_inc(x_215); +if (lean_is_exclusive(x_186)) { + lean_ctor_release(x_186, 0); + lean_ctor_release(x_186, 1); + x_216 = x_186; } else { - lean_dec_ref(x_185); - x_215 = lean_box(0); + lean_dec_ref(x_186); + x_216 = lean_box(0); } -if (lean_is_scalar(x_215)) { - x_216 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_216)) { + x_217 = lean_alloc_ctor(1, 2, 0); } else { - x_216 = x_215; + x_217 = x_216; } -lean_ctor_set(x_216, 0, x_213); -lean_ctor_set(x_216, 1, x_214); -return x_216; +lean_ctor_set(x_217, 0, x_214); +lean_ctor_set(x_217, 1, x_215); +return x_217; } } else { -lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_217 = lean_ctor_get(x_182, 0); -lean_inc(x_217); -x_218 = lean_ctor_get(x_182, 1); +lean_dec(x_4); +x_218 = lean_ctor_get(x_183, 0); lean_inc(x_218); -if (lean_is_exclusive(x_182)) { - lean_ctor_release(x_182, 0); - lean_ctor_release(x_182, 1); - x_219 = x_182; +x_219 = lean_ctor_get(x_183, 1); +lean_inc(x_219); +if (lean_is_exclusive(x_183)) { + lean_ctor_release(x_183, 0); + lean_ctor_release(x_183, 1); + x_220 = x_183; } else { - lean_dec_ref(x_182); - x_219 = lean_box(0); + lean_dec_ref(x_183); + x_220 = lean_box(0); } -if (lean_is_scalar(x_219)) { - x_220 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_220)) { + x_221 = lean_alloc_ctor(1, 2, 0); } else { - x_220 = x_219; + x_221 = x_220; } -lean_ctor_set(x_220, 0, x_217); -lean_ctor_set(x_220, 1, x_218); -return x_220; +lean_ctor_set(x_221, 0, x_218); +lean_ctor_set(x_221, 1, x_219); +return x_221; } } else { -lean_object* x_221; lean_object* x_222; lean_object* x_223; lean_object* x_224; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_221 = lean_ctor_get(x_177, 0); -lean_inc(x_221); -x_222 = lean_ctor_get(x_177, 1); +lean_dec(x_4); +x_222 = lean_ctor_get(x_178, 0); lean_inc(x_222); -if (lean_is_exclusive(x_177)) { - lean_ctor_release(x_177, 0); - lean_ctor_release(x_177, 1); - x_223 = x_177; +x_223 = lean_ctor_get(x_178, 1); +lean_inc(x_223); +if (lean_is_exclusive(x_178)) { + lean_ctor_release(x_178, 0); + lean_ctor_release(x_178, 1); + x_224 = x_178; } else { - lean_dec_ref(x_177); - x_223 = lean_box(0); + lean_dec_ref(x_178); + x_224 = lean_box(0); } -if (lean_is_scalar(x_223)) { - x_224 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_224)) { + x_225 = lean_alloc_ctor(1, 2, 0); } else { - x_224 = x_223; + x_225 = x_224; } -lean_ctor_set(x_224, 0, x_221); -lean_ctor_set(x_224, 1, x_222); -return x_224; +lean_ctor_set(x_225, 0, x_222); +lean_ctor_set(x_225, 1, x_223); +return x_225; } } else { -lean_object* x_225; lean_object* x_226; lean_object* x_227; lean_object* x_228; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_226; lean_object* x_227; lean_object* x_228; lean_object* x_229; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_225 = lean_ctor_get(x_173, 0); -lean_inc(x_225); -x_226 = lean_ctor_get(x_173, 1); +lean_dec(x_4); +x_226 = lean_ctor_get(x_174, 0); lean_inc(x_226); -if (lean_is_exclusive(x_173)) { - lean_ctor_release(x_173, 0); - lean_ctor_release(x_173, 1); - x_227 = x_173; +x_227 = lean_ctor_get(x_174, 1); +lean_inc(x_227); +if (lean_is_exclusive(x_174)) { + lean_ctor_release(x_174, 0); + lean_ctor_release(x_174, 1); + x_228 = x_174; } else { - lean_dec_ref(x_173); - x_227 = lean_box(0); + lean_dec_ref(x_174); + x_228 = lean_box(0); } -if (lean_is_scalar(x_227)) { - x_228 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_228)) { + x_229 = lean_alloc_ctor(1, 2, 0); } else { - x_228 = x_227; + x_229 = x_228; } -lean_ctor_set(x_228, 0, x_225); -lean_ctor_set(x_228, 1, x_226); -return x_228; +lean_ctor_set(x_229, 0, x_226); +lean_ctor_set(x_229, 1, x_227); +return x_229; } } else { -lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_229 = lean_ctor_get(x_167, 0); -lean_inc(x_229); -x_230 = lean_ctor_get(x_167, 1); +lean_dec(x_4); +x_230 = lean_ctor_get(x_168, 0); lean_inc(x_230); -if (lean_is_exclusive(x_167)) { - lean_ctor_release(x_167, 0); - lean_ctor_release(x_167, 1); - x_231 = x_167; +x_231 = lean_ctor_get(x_168, 1); +lean_inc(x_231); +if (lean_is_exclusive(x_168)) { + lean_ctor_release(x_168, 0); + lean_ctor_release(x_168, 1); + x_232 = x_168; } else { - lean_dec_ref(x_167); - x_231 = lean_box(0); + lean_dec_ref(x_168); + x_232 = lean_box(0); } -if (lean_is_scalar(x_231)) { - x_232 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_232)) { + x_233 = lean_alloc_ctor(1, 2, 0); } else { - x_232 = x_231; + x_233 = x_232; } -lean_ctor_set(x_232, 0, x_229); -lean_ctor_set(x_232, 1, x_230); -return x_232; +lean_ctor_set(x_233, 0, x_230); +lean_ctor_set(x_233, 1, x_231); +return x_233; } } else { -lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_233 = lean_ctor_get(x_162, 0); -lean_inc(x_233); -x_234 = lean_ctor_get(x_162, 1); +lean_dec(x_4); +x_234 = lean_ctor_get(x_163, 0); lean_inc(x_234); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_235 = x_162; +x_235 = lean_ctor_get(x_163, 1); +lean_inc(x_235); +if (lean_is_exclusive(x_163)) { + lean_ctor_release(x_163, 0); + lean_ctor_release(x_163, 1); + x_236 = x_163; } else { - lean_dec_ref(x_162); - x_235 = lean_box(0); + lean_dec_ref(x_163); + x_236 = lean_box(0); } -if (lean_is_scalar(x_235)) { - x_236 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_236)) { + x_237 = lean_alloc_ctor(1, 2, 0); } else { - x_236 = x_235; + x_237 = x_236; } -lean_ctor_set(x_236, 0, x_233); -lean_ctor_set(x_236, 1, x_234); -return x_236; +lean_ctor_set(x_237, 0, x_234); +lean_ctor_set(x_237, 1, x_235); +return x_237; } } else { -lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_237 = lean_ctor_get(x_157, 0); -lean_inc(x_237); -x_238 = lean_ctor_get(x_157, 1); +lean_dec(x_4); +x_238 = lean_ctor_get(x_158, 0); lean_inc(x_238); -if (lean_is_exclusive(x_157)) { - lean_ctor_release(x_157, 0); - lean_ctor_release(x_157, 1); - x_239 = x_157; +x_239 = lean_ctor_get(x_158, 1); +lean_inc(x_239); +if (lean_is_exclusive(x_158)) { + lean_ctor_release(x_158, 0); + lean_ctor_release(x_158, 1); + x_240 = x_158; } else { - lean_dec_ref(x_157); - x_239 = lean_box(0); + lean_dec_ref(x_158); + x_240 = lean_box(0); } -if (lean_is_scalar(x_239)) { - x_240 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_240)) { + x_241 = lean_alloc_ctor(1, 2, 0); } else { - x_240 = x_239; + x_241 = x_240; } -lean_ctor_set(x_240, 0, x_237); -lean_ctor_set(x_240, 1, x_238); -return x_240; +lean_ctor_set(x_241, 0, x_238); +lean_ctor_set(x_241, 1, x_239); +return x_241; } } else { -lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; -lean_dec(x_152); -lean_dec(x_146); +lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; +lean_dec(x_153); +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_241 = lean_ctor_get(x_154, 0); -lean_inc(x_241); -x_242 = lean_ctor_get(x_154, 1); +lean_dec(x_4); +x_242 = lean_ctor_get(x_155, 0); lean_inc(x_242); -if (lean_is_exclusive(x_154)) { - lean_ctor_release(x_154, 0); - lean_ctor_release(x_154, 1); - x_243 = x_154; +x_243 = lean_ctor_get(x_155, 1); +lean_inc(x_243); +if (lean_is_exclusive(x_155)) { + lean_ctor_release(x_155, 0); + lean_ctor_release(x_155, 1); + x_244 = x_155; } else { - lean_dec_ref(x_154); - x_243 = lean_box(0); + lean_dec_ref(x_155); + x_244 = lean_box(0); } -if (lean_is_scalar(x_243)) { - x_244 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_244)) { + x_245 = lean_alloc_ctor(1, 2, 0); } else { - x_244 = x_243; + x_245 = x_244; } -lean_ctor_set(x_244, 0, x_241); -lean_ctor_set(x_244, 1, x_242); -return x_244; +lean_ctor_set(x_245, 0, x_242); +lean_ctor_set(x_245, 1, x_243); +return x_245; } } else { -lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; -lean_dec(x_146); +lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; +lean_dec(x_147); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_3); -x_245 = lean_ctor_get(x_148, 0); -lean_inc(x_245); -x_246 = lean_ctor_get(x_148, 1); +lean_dec(x_4); +x_246 = lean_ctor_get(x_149, 0); lean_inc(x_246); -if (lean_is_exclusive(x_148)) { - lean_ctor_release(x_148, 0); - lean_ctor_release(x_148, 1); - x_247 = x_148; +x_247 = lean_ctor_get(x_149, 1); +lean_inc(x_247); +if (lean_is_exclusive(x_149)) { + lean_ctor_release(x_149, 0); + lean_ctor_release(x_149, 1); + x_248 = x_149; } else { - lean_dec_ref(x_148); - x_247 = lean_box(0); + lean_dec_ref(x_149); + x_248 = lean_box(0); } -if (lean_is_scalar(x_247)) { - x_248 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_248)) { + x_249 = lean_alloc_ctor(1, 2, 0); } else { - x_248 = x_247; + x_249 = x_248; } -lean_ctor_set(x_248, 0, x_245); -lean_ctor_set(x_248, 1, x_246); -return x_248; +lean_ctor_set(x_249, 0, x_246); +lean_ctor_set(x_249, 1, x_247); +return x_249; } } } } -LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_simp___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l_Lean_instantiateMVars___at_Lean_Meta_Grind_simp___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -2013,16 +1611,18 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); +lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -uint8_t x_13; lean_object* x_14; -x_13 = lean_unbox(x_3); +uint8_t x_14; lean_object* x_15; +x_14 = lean_unbox(x_3); lean_dec(x_3); -x_14 = l_Lean_Meta_Grind_simp___lambda__1(x_1, x_2, x_13, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_Meta_Grind_simp___lambda__1(x_1, x_2, x_14, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2031,17 +1631,18 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -return x_14; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_simp___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_simp(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_simp(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_3); lean_dec(x_2); -return x_10; +return x_11; } } lean_object* initialize_Init_Grind_Lemmas(uint8_t builtin, lean_object*); @@ -2077,11 +1678,6 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_MarkNestedProofs(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__1(); -l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__2); -l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3 = _init_l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3(); -lean_mark_persistent(l_Lean_addTrace___at_Lean_Meta_Grind_simp___spec__3___closed__3); l_Lean_Meta_Grind_simp___closed__1 = _init_l_Lean_Meta_Grind_simp___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_simp___closed__1); l_Lean_Meta_Grind_simp___closed__2 = _init_l_Lean_Meta_Grind_simp___closed__2(); @@ -2112,6 +1708,8 @@ l_Lean_Meta_Grind_simp___closed__14 = _init_l_Lean_Meta_Grind_simp___closed__14( lean_mark_persistent(l_Lean_Meta_Grind_simp___closed__14); l_Lean_Meta_Grind_simp___closed__15 = _init_l_Lean_Meta_Grind_simp___closed__15(); lean_mark_persistent(l_Lean_Meta_Grind_simp___closed__15); +l_Lean_Meta_Grind_simp___closed__16 = _init_l_Lean_Meta_Grind_simp___closed__16(); +lean_mark_persistent(l_Lean_Meta_Grind_simp___closed__16); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Split.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Split.c index cec2dde45cfe..d859544b5252 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Split.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Split.c @@ -13,104 +13,112 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2; lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_introNewHyp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isApp(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__7; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_splitNext___lambda__4___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqCaseSplitStatus; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_splitNext___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1; lean_object* l_Lean_stringToMessageData(lean_object*); -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18_(uint8_t, uint8_t); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_List_appendTR___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_take(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx(uint8_t); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18____boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofFormat(lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__2; +lean_object* l_Lean_Meta_Match_MatcherInfo_numAlts(lean_object*); LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Meta_Grind_splitNext___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_checkMaxCaseSplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Meta_isInductivePredicate(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_casesMatch(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx___boxed(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34____boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6; +lean_object* l_List_lengthTRAux___rarg(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__4; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_getGeneration(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__5; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1; +lean_object* l_Lean_Meta_isMatcherAppCore_x3f(lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_updateLastTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_instMonadMetaM; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instInhabitedCaseSplitStatus; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedCaseSplitStatus; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10; lean_object* l_Lean_MessageData_ofExpr(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_isResolvedCaseSplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__8; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4; lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg(uint8_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5; lean_object* l_Lean_Meta_Grind_intros(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* lean_panic_fn(lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2; @@ -118,175 +126,157 @@ lean_object* l_Lean_Expr_getAppFn(lean_object*); lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; +lean_object* l_Lean_Meta_mkOfEqTrueCore(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1; lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8; lean_object* l_List_reverse___rarg(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkEM(lean_object*); lean_object* l_Lean_Meta_Grind_isEqFalse(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instInhabitedOfMonad___rarg(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34_(lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion(lean_object*); lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Meta_isInductivePredicate_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_splitNext___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_cases(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__1; static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_splitNext___lambda__4___closed__2; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__6; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_splitNext___closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1___boxed(lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); -static lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5; lean_object* l_ReaderT_instMonad___rarg(lean_object*); static lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__3; lean_object* l_Lean_Meta_isMatcherApp___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx(uint8_t x_1) { +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedCaseSplitStatus() { _start: { -switch (x_1) { +lean_object* x_1; +x_1 = lean_box(0); +return x_1; +} +} +LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34_(lean_object* x_1, lean_object* x_2) { +_start: +{ +switch (lean_obj_tag(x_1)) { case 0: { -lean_object* x_2; -x_2 = lean_unsigned_to_nat(0u); -return x_2; -} -case 1: +if (lean_obj_tag(x_2) == 0) { -lean_object* x_3; -x_3 = lean_unsigned_to_nat(1u); +uint8_t x_3; +x_3 = 1; return x_3; } -default: +else { -lean_object* x_4; -x_4 = lean_unsigned_to_nat(2u); +uint8_t x_4; +x_4 = 0; return x_4; } } -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx___boxed(lean_object* x_1) { -_start: +case 1: { -uint8_t x_2; lean_object* x_3; -x_2 = lean_unbox(x_1); -lean_dec(x_1); -x_3 = l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1(lean_object* x_1) { -_start: +if (lean_obj_tag(x_2) == 1) { -lean_inc(x_1); -return x_1; -} +uint8_t x_5; +x_5 = 1; +return x_5; } -static lean_object* _init_l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1___boxed), 1, 0); -return x_1; +uint8_t x_6; +x_6 = 0; +return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg(uint8_t x_1, uint8_t x_2, lean_object* x_3) { -_start: +default: { -lean_object* x_4; -x_4 = l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1; -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion(lean_object* x_1) { -_start: +if (lean_obj_tag(x_2) == 2) { -lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___boxed), 3, 0); -return x_2; +lean_object* x_7; uint8_t x_8; lean_object* x_9; uint8_t x_10; uint8_t x_11; +x_7 = lean_ctor_get(x_1, 0); +x_8 = lean_ctor_get_uint8(x_1, sizeof(void*)*1); +x_9 = lean_ctor_get(x_2, 0); +x_10 = lean_ctor_get_uint8(x_2, sizeof(void*)*1); +x_11 = lean_nat_dec_eq(x_7, x_9); +if (x_11 == 0) +{ +uint8_t x_12; +x_12 = 0; +return x_12; } +else +{ +if (x_8 == 0) +{ +if (x_10 == 0) +{ +uint8_t x_13; +x_13 = 1; +return x_13; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1___boxed(lean_object* x_1) { -_start: +else { -lean_object* x_2; -x_2 = l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___lambda__1(x_1); -lean_dec(x_1); -return x_2; +uint8_t x_14; +x_14 = 0; +return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -uint8_t x_4; uint8_t x_5; lean_object* x_6; -x_4 = lean_unbox(x_1); -lean_dec(x_1); -x_5 = lean_unbox(x_2); -lean_dec(x_2); -x_6 = l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg(x_4, x_5, x_3); -return x_6; +return x_10; } } -static uint8_t _init_l_Lean_Meta_Grind_instInhabitedCaseSplitStatus() { -_start: +} +else { -uint8_t x_1; -x_1 = 0; -return x_1; +uint8_t x_15; +x_15 = 0; +return x_15; +} } } -LEAN_EXPORT uint8_t l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18_(uint8_t x_1, uint8_t x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx(x_1); -x_4 = l_Lean_Meta_Grind_CaseSplitStatus_toCtorIdx(x_2); -x_5 = lean_nat_dec_eq(x_3, x_4); -lean_dec(x_4); -lean_dec(x_3); -return x_5; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34____boxed(lean_object* x_1, lean_object* x_2) { _start: { -uint8_t x_3; uint8_t x_4; uint8_t x_5; lean_object* x_6; -x_3 = lean_unbox(x_1); -lean_dec(x_1); -x_4 = lean_unbox(x_2); +uint8_t x_3; lean_object* x_4; +x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34_(x_1, x_2); lean_dec(x_2); -x_5 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18_(x_3, x_4); -x_6 = lean_box(x_5); -return x_6; +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } } static lean_object* _init_l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_18____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_beqCaseSplitStatus____x40_Lean_Meta_Tactic_Grind_Split___hyg_34____boxed), 2, 0); return x_1; } } @@ -298,64 +288,19 @@ x_1 = l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1; return x_1; } } -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_instMonadMetaM; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__3; -x_2 = l_ReaderT_instMonad___rarg(x_1); -return x_2; -} -} -static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5() { -_start: -{ -lean_object* x_1; uint8_t x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4; -x_2 = l_Lean_Meta_Grind_instInhabitedCaseSplitStatus; -x_3 = lean_box(x_2); -x_4 = l_instInhabitedOfMonad___rarg(x_1, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1() { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_11 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5; -x_12 = lean_panic_fn(x_11, x_1); -x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -return x_13; +lean_object* x_1; uint8_t x_2; lean_object* x_3; +x_1 = lean_unsigned_to_nat(2u); +x_2 = 0; +x_3 = lean_alloc_ctor(2, 1, 1); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set_uint8(x_3, sizeof(void*)*1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; @@ -388,136 +333,146 @@ uint8_t x_18; x_18 = !lean_is_exclusive(x_15); if (x_18 == 0) { -lean_object* x_19; uint8_t x_20; lean_object* x_21; +lean_object* x_19; lean_object* x_20; x_19 = lean_ctor_get(x_15, 0); lean_dec(x_19); -x_20 = 2; -x_21 = lean_box(x_20); -lean_ctor_set(x_15, 0, x_21); +x_20 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +lean_ctor_set(x_15, 0, x_20); return x_15; } else { -lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_15, 1); -lean_inc(x_22); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_15, 1); +lean_inc(x_21); lean_dec(x_15); -x_23 = 2; -x_24 = lean_box(x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_22); -return x_25; +x_22 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; } } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_15); -if (x_26 == 0) +uint8_t x_24; +x_24 = !lean_is_exclusive(x_15); +if (x_24 == 0) { -lean_object* x_27; uint8_t x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_15, 0); -lean_dec(x_27); -x_28 = 0; -x_29 = lean_box(x_28); -lean_ctor_set(x_15, 0, x_29); +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_15, 0); +lean_dec(x_25); +x_26 = lean_box(0); +lean_ctor_set(x_15, 0, x_26); return x_15; } else { -lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_15, 1); -lean_inc(x_30); +lean_object* x_27; lean_object* x_28; lean_object* x_29; +x_27 = lean_ctor_get(x_15, 1); +lean_inc(x_27); lean_dec(x_15); -x_31 = 0; -x_32 = lean_box(x_31); -x_33 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_33, 0, x_32); -lean_ctor_set(x_33, 1, x_30); -return x_33; +x_28 = lean_box(0); +x_29 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_29, 0, x_28); +lean_ctor_set(x_29, 1, x_27); +return x_29; } } } else { -uint8_t x_34; -x_34 = !lean_is_exclusive(x_15); -if (x_34 == 0) +uint8_t x_30; +x_30 = !lean_is_exclusive(x_15); +if (x_30 == 0) { return x_15; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_15, 0); -x_36 = lean_ctor_get(x_15, 1); -lean_inc(x_36); -lean_inc(x_35); +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_15, 0); +x_32 = lean_ctor_get(x_15, 1); +lean_inc(x_32); +lean_inc(x_31); lean_dec(x_15); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } } else { -uint8_t x_38; +uint8_t x_34; lean_dec(x_1); -x_38 = !lean_is_exclusive(x_11); -if (x_38 == 0) +x_34 = !lean_is_exclusive(x_11); +if (x_34 == 0) { -lean_object* x_39; uint8_t x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_11, 0); -lean_dec(x_39); -x_40 = 0; -x_41 = lean_box(x_40); -lean_ctor_set(x_11, 0, x_41); +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_11, 0); +lean_dec(x_35); +x_36 = lean_box(0); +lean_ctor_set(x_11, 0, x_36); return x_11; } else { -lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; -x_42 = lean_ctor_get(x_11, 1); -lean_inc(x_42); +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_11, 1); +lean_inc(x_37); lean_dec(x_11); -x_43 = 0; -x_44 = lean_box(x_43); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_42); -return x_45; +x_38 = lean_box(0); +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); +return x_39; } } } else { -uint8_t x_46; +uint8_t x_40; lean_dec(x_1); -x_46 = !lean_is_exclusive(x_11); -if (x_46 == 0) +x_40 = !lean_is_exclusive(x_11); +if (x_40 == 0) { return x_11; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_47 = lean_ctor_get(x_11, 0); -x_48 = lean_ctor_get(x_11, 1); -lean_inc(x_48); -lean_inc(x_47); +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_11, 0); +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_inc(x_41); lean_dec(x_11); -x_49 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_49, 0, x_47); -lean_ctor_set(x_49, 1, x_48); -return x_49; +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -533,6 +488,8 @@ lean_dec(x_14); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; +lean_dec(x_3); +lean_dec(x_2); x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); @@ -547,137 +504,157 @@ lean_dec(x_18); if (x_19 == 0) { uint8_t x_20; -lean_dec(x_3); -lean_dec(x_2); x_20 = !lean_is_exclusive(x_17); if (x_20 == 0) { -lean_object* x_21; uint8_t x_22; lean_object* x_23; +lean_object* x_21; lean_object* x_22; x_21 = lean_ctor_get(x_17, 0); lean_dec(x_21); -x_22 = 1; -x_23 = lean_box(x_22); -lean_ctor_set(x_17, 0, x_23); +x_22 = lean_box(1); +lean_ctor_set(x_17, 0, x_22); return x_17; } else { -lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); lean_dec(x_17); -x_25 = 1; -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; +x_24 = lean_box(1); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; } } else { -lean_object* x_28; lean_object* x_29; -x_28 = lean_ctor_get(x_17, 1); -lean_inc(x_28); -lean_dec(x_17); -x_29 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_28); -if (lean_obj_tag(x_29) == 0) -{ -lean_object* x_30; uint8_t x_31; -x_30 = lean_ctor_get(x_29, 0); -lean_inc(x_30); -x_31 = lean_unbox(x_30); -lean_dec(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; -x_32 = lean_ctor_get(x_29, 1); -lean_inc(x_32); -lean_dec(x_29); -x_33 = l_Lean_Meta_Grind_isEqFalse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_32); -if (lean_obj_tag(x_33) == 0) -{ -lean_object* x_34; uint8_t x_35; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_unbox(x_34); -lean_dec(x_34); -if (x_35 == 0) -{ -uint8_t x_36; -x_36 = !lean_is_exclusive(x_33); -if (x_36 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_17); +if (x_26 == 0) { -lean_object* x_37; uint8_t x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_33, 0); -lean_dec(x_37); -x_38 = 2; -x_39 = lean_box(x_38); -lean_ctor_set(x_33, 0, x_39); -return x_33; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_17, 0); +lean_dec(x_27); +x_28 = lean_box(0); +lean_ctor_set(x_17, 0, x_28); +return x_17; } else { -lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_33, 1); -lean_inc(x_40); -lean_dec(x_33); -x_41 = 2; -x_42 = lean_box(x_41); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_40); -return x_43; -} -} +lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_29 = lean_ctor_get(x_17, 1); +lean_inc(x_29); +lean_dec(x_17); +x_30 = lean_box(0); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_29); +return x_31; +} +} +} +else +{ +uint8_t x_32; +x_32 = !lean_is_exclusive(x_17); +if (x_32 == 0) +{ +return x_17; +} +else +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; +x_33 = lean_ctor_get(x_17, 0); +x_34 = lean_ctor_get(x_17, 1); +lean_inc(x_34); +lean_inc(x_33); +lean_dec(x_17); +x_35 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +return x_35; +} +} +} else { +lean_object* x_36; lean_object* x_37; +lean_dec(x_1); +x_36 = lean_ctor_get(x_13, 1); +lean_inc(x_36); +lean_dec(x_13); +x_37 = l_Lean_Meta_Grind_isEqTrue(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_36); +if (lean_obj_tag(x_37) == 0) +{ +lean_object* x_38; uint8_t x_39; +x_38 = lean_ctor_get(x_37, 0); +lean_inc(x_38); +x_39 = lean_unbox(x_38); +lean_dec(x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_37, 1); +lean_inc(x_40); +lean_dec(x_37); +x_41 = l_Lean_Meta_Grind_isEqTrue(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_40); +if (lean_obj_tag(x_41) == 0) +{ +lean_object* x_42; uint8_t x_43; +x_42 = lean_ctor_get(x_41, 0); +lean_inc(x_42); +x_43 = lean_unbox(x_42); +lean_dec(x_42); +if (x_43 == 0) +{ uint8_t x_44; -x_44 = !lean_is_exclusive(x_33); +x_44 = !lean_is_exclusive(x_41); if (x_44 == 0) { -lean_object* x_45; uint8_t x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_33, 0); +lean_object* x_45; lean_object* x_46; +x_45 = lean_ctor_get(x_41, 0); lean_dec(x_45); -x_46 = 0; -x_47 = lean_box(x_46); -lean_ctor_set(x_33, 0, x_47); -return x_33; +x_46 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +lean_ctor_set(x_41, 0, x_46); +return x_41; } else { -lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; -x_48 = lean_ctor_get(x_33, 1); -lean_inc(x_48); -lean_dec(x_33); -x_49 = 0; -x_50 = lean_box(x_49); -x_51 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_51, 0, x_50); -lean_ctor_set(x_51, 1, x_48); -return x_51; -} +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_41, 1); +lean_inc(x_47); +lean_dec(x_41); +x_48 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_47); +return x_49; } } else { -uint8_t x_52; -x_52 = !lean_is_exclusive(x_33); -if (x_52 == 0) +uint8_t x_50; +x_50 = !lean_is_exclusive(x_41); +if (x_50 == 0) { -return x_33; +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_41, 0); +lean_dec(x_51); +x_52 = lean_box(0); +lean_ctor_set(x_41, 0, x_52); +return x_41; } else { lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_53 = lean_ctor_get(x_33, 0); -x_54 = lean_ctor_get(x_33, 1); -lean_inc(x_54); +x_53 = lean_ctor_get(x_41, 1); lean_inc(x_53); -lean_dec(x_33); -x_55 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_55, 0, x_53); -lean_ctor_set(x_55, 1, x_54); +lean_dec(x_41); +x_54 = lean_box(0); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_53); return x_55; } } @@ -685,143 +662,123 @@ return x_55; else { uint8_t x_56; -lean_dec(x_3); -x_56 = !lean_is_exclusive(x_29); +x_56 = !lean_is_exclusive(x_41); if (x_56 == 0) { -lean_object* x_57; uint8_t x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_29, 0); -lean_dec(x_57); -x_58 = 0; -x_59 = lean_box(x_58); -lean_ctor_set(x_29, 0, x_59); -return x_29; +return x_41; } else { -lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; -x_60 = lean_ctor_get(x_29, 1); -lean_inc(x_60); -lean_dec(x_29); -x_61 = 0; -x_62 = lean_box(x_61); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_60); -return x_63; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_41, 0); +x_58 = lean_ctor_get(x_41, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_41); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; } } } else { -uint8_t x_64; +uint8_t x_60; lean_dec(x_3); -x_64 = !lean_is_exclusive(x_29); -if (x_64 == 0) +x_60 = !lean_is_exclusive(x_37); +if (x_60 == 0) { -return x_29; +lean_object* x_61; lean_object* x_62; +x_61 = lean_ctor_get(x_37, 0); +lean_dec(x_61); +x_62 = lean_box(0); +lean_ctor_set(x_37, 0, x_62); +return x_37; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_29, 0); -x_66 = lean_ctor_get(x_29, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_29); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; -} +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_37, 1); +lean_inc(x_63); +lean_dec(x_37); +x_64 = lean_box(0); +x_65 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_63); +return x_65; } } } else { -uint8_t x_68; +uint8_t x_66; lean_dec(x_3); -lean_dec(x_2); -x_68 = !lean_is_exclusive(x_17); -if (x_68 == 0) +x_66 = !lean_is_exclusive(x_37); +if (x_66 == 0) { -return x_17; +return x_37; } else { -lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_17, 0); -x_70 = lean_ctor_get(x_17, 1); -lean_inc(x_70); -lean_inc(x_69); -lean_dec(x_17); -x_71 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_71, 0, x_69); -lean_ctor_set(x_71, 1, x_70); -return x_71; +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_37, 0); +x_68 = lean_ctor_get(x_37, 1); +lean_inc(x_68); +lean_inc(x_67); +lean_dec(x_37); +x_69 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_69, 0, x_67); +lean_ctor_set(x_69, 1, x_68); +return x_69; +} } } } else { -uint8_t x_72; +uint8_t x_70; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_72 = !lean_is_exclusive(x_13); -if (x_72 == 0) +x_70 = !lean_is_exclusive(x_13); +if (x_70 == 0) { -lean_object* x_73; uint8_t x_74; lean_object* x_75; -x_73 = lean_ctor_get(x_13, 0); -lean_dec(x_73); -x_74 = 0; -x_75 = lean_box(x_74); -lean_ctor_set(x_13, 0, x_75); return x_13; } else { -lean_object* x_76; uint8_t x_77; lean_object* x_78; lean_object* x_79; -x_76 = lean_ctor_get(x_13, 1); -lean_inc(x_76); +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_13, 0); +x_72 = lean_ctor_get(x_13, 1); +lean_inc(x_72); +lean_inc(x_71); lean_dec(x_13); -x_77 = 0; -x_78 = lean_box(x_77); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_78); -lean_ctor_set(x_79, 1, x_76); -return x_79; +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; } } } -else -{ -uint8_t x_80; -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_80 = !lean_is_exclusive(x_13); -if (x_80 == 0) -{ -return x_13; } -else +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_13, 0); -x_82 = lean_ctor_get(x_13, 1); -lean_inc(x_82); -lean_inc(x_81); -lean_dec(x_13); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; -} -} +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -837,8 +794,6 @@ lean_dec(x_14); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; -lean_dec(x_3); -lean_dec(x_2); x_16 = lean_ctor_get(x_13, 1); lean_inc(x_16); lean_dec(x_13); @@ -853,485 +808,1257 @@ lean_dec(x_18); if (x_19 == 0) { uint8_t x_20; +lean_dec(x_3); +lean_dec(x_2); x_20 = !lean_is_exclusive(x_17); if (x_20 == 0) { -lean_object* x_21; uint8_t x_22; lean_object* x_23; +lean_object* x_21; lean_object* x_22; x_21 = lean_ctor_get(x_17, 0); lean_dec(x_21); -x_22 = 1; -x_23 = lean_box(x_22); -lean_ctor_set(x_17, 0, x_23); +x_22 = lean_box(1); +lean_ctor_set(x_17, 0, x_22); return x_17; } else { -lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); lean_dec(x_17); -x_25 = 1; -x_26 = lean_box(x_25); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_24); -return x_27; +x_24 = lean_box(1); +x_25 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_25, 0, x_24); +lean_ctor_set(x_25, 1, x_23); +return x_25; } } else { -uint8_t x_28; -x_28 = !lean_is_exclusive(x_17); -if (x_28 == 0) +lean_object* x_26; lean_object* x_27; +x_26 = lean_ctor_get(x_17, 1); +lean_inc(x_26); +lean_dec(x_17); +x_27 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_26); +if (lean_obj_tag(x_27) == 0) { -lean_object* x_29; uint8_t x_30; lean_object* x_31; -x_29 = lean_ctor_get(x_17, 0); -lean_dec(x_29); -x_30 = 0; -x_31 = lean_box(x_30); -lean_ctor_set(x_17, 0, x_31); -return x_17; -} -else +lean_object* x_28; uint8_t x_29; +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_unbox(x_28); +lean_dec(x_28); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_ctor_get(x_27, 1); +lean_inc(x_30); +lean_dec(x_27); +x_31 = l_Lean_Meta_Grind_isEqFalse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_30); +if (lean_obj_tag(x_31) == 0) { -lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; -x_32 = lean_ctor_get(x_17, 1); +lean_object* x_32; uint8_t x_33; +x_32 = lean_ctor_get(x_31, 0); lean_inc(x_32); -lean_dec(x_17); -x_33 = 0; -x_34 = lean_box(x_33); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_32); -return x_35; -} -} -} -else +x_33 = lean_unbox(x_32); +lean_dec(x_32); +if (x_33 == 0) { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_17); -if (x_36 == 0) +uint8_t x_34; +x_34 = !lean_is_exclusive(x_31); +if (x_34 == 0) { -return x_17; +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_31, 0); +lean_dec(x_35); +x_36 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +lean_ctor_set(x_31, 0, x_36); +return x_31; } else { lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_17, 0); -x_38 = lean_ctor_get(x_17, 1); -lean_inc(x_38); +x_37 = lean_ctor_get(x_31, 1); lean_inc(x_37); -lean_dec(x_17); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_37); -lean_ctor_set(x_39, 1, x_38); +lean_dec(x_31); +x_38 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +x_39 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set(x_39, 1, x_37); return x_39; } } -} else { -lean_object* x_40; lean_object* x_41; -lean_dec(x_1); -x_40 = lean_ctor_get(x_13, 1); -lean_inc(x_40); -lean_dec(x_13); -x_41 = l_Lean_Meta_Grind_isEqTrue(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_40); -if (lean_obj_tag(x_41) == 0) -{ -lean_object* x_42; uint8_t x_43; -x_42 = lean_ctor_get(x_41, 0); -lean_inc(x_42); -x_43 = lean_unbox(x_42); -lean_dec(x_42); -if (x_43 == 0) +uint8_t x_40; +x_40 = !lean_is_exclusive(x_31); +if (x_40 == 0) { -lean_object* x_44; lean_object* x_45; -x_44 = lean_ctor_get(x_41, 1); -lean_inc(x_44); +lean_object* x_41; lean_object* x_42; +x_41 = lean_ctor_get(x_31, 0); lean_dec(x_41); -x_45 = l_Lean_Meta_Grind_isEqTrue(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_44); -if (lean_obj_tag(x_45) == 0) -{ -lean_object* x_46; uint8_t x_47; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_unbox(x_46); -lean_dec(x_46); -if (x_47 == 0) -{ -uint8_t x_48; -x_48 = !lean_is_exclusive(x_45); -if (x_48 == 0) -{ -lean_object* x_49; uint8_t x_50; lean_object* x_51; -x_49 = lean_ctor_get(x_45, 0); -lean_dec(x_49); -x_50 = 2; -x_51 = lean_box(x_50); -lean_ctor_set(x_45, 0, x_51); -return x_45; +x_42 = lean_box(0); +lean_ctor_set(x_31, 0, x_42); +return x_31; } else { -lean_object* x_52; uint8_t x_53; lean_object* x_54; lean_object* x_55; -x_52 = lean_ctor_get(x_45, 1); -lean_inc(x_52); -lean_dec(x_45); -x_53 = 2; -x_54 = lean_box(x_53); -x_55 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_31, 1); +lean_inc(x_43); +lean_dec(x_31); +x_44 = lean_box(0); +x_45 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_43); +return x_45; +} } } else { -uint8_t x_56; -x_56 = !lean_is_exclusive(x_45); -if (x_56 == 0) +uint8_t x_46; +x_46 = !lean_is_exclusive(x_31); +if (x_46 == 0) { -lean_object* x_57; uint8_t x_58; lean_object* x_59; -x_57 = lean_ctor_get(x_45, 0); -lean_dec(x_57); -x_58 = 0; -x_59 = lean_box(x_58); -lean_ctor_set(x_45, 0, x_59); -return x_45; +return x_31; } else { -lean_object* x_60; uint8_t x_61; lean_object* x_62; lean_object* x_63; -x_60 = lean_ctor_get(x_45, 1); -lean_inc(x_60); -lean_dec(x_45); -x_61 = 0; -x_62 = lean_box(x_61); -x_63 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_60); -return x_63; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_31, 0); +x_48 = lean_ctor_get(x_31, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_31); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } } else { -uint8_t x_64; -x_64 = !lean_is_exclusive(x_45); -if (x_64 == 0) -{ -return x_45; +uint8_t x_50; +lean_dec(x_3); +x_50 = !lean_is_exclusive(x_27); +if (x_50 == 0) +{ +lean_object* x_51; lean_object* x_52; +x_51 = lean_ctor_get(x_27, 0); +lean_dec(x_51); +x_52 = lean_box(0); +lean_ctor_set(x_27, 0, x_52); +return x_27; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_65 = lean_ctor_get(x_45, 0); -x_66 = lean_ctor_get(x_45, 1); -lean_inc(x_66); -lean_inc(x_65); -lean_dec(x_45); -x_67 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_67, 0, x_65); -lean_ctor_set(x_67, 1, x_66); -return x_67; +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_27, 1); +lean_inc(x_53); +lean_dec(x_27); +x_54 = lean_box(0); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_53); +return x_55; } } } else { -uint8_t x_68; +uint8_t x_56; lean_dec(x_3); -x_68 = !lean_is_exclusive(x_41); -if (x_68 == 0) +x_56 = !lean_is_exclusive(x_27); +if (x_56 == 0) { -lean_object* x_69; uint8_t x_70; lean_object* x_71; -x_69 = lean_ctor_get(x_41, 0); -lean_dec(x_69); -x_70 = 0; -x_71 = lean_box(x_70); -lean_ctor_set(x_41, 0, x_71); -return x_41; +return x_27; } else { -lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; -x_72 = lean_ctor_get(x_41, 1); -lean_inc(x_72); -lean_dec(x_41); -x_73 = 0; -x_74 = lean_box(x_73); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_74); -lean_ctor_set(x_75, 1, x_72); -return x_75; +lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_57 = lean_ctor_get(x_27, 0); +x_58 = lean_ctor_get(x_27, 1); +lean_inc(x_58); +lean_inc(x_57); +lean_dec(x_27); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_57); +lean_ctor_set(x_59, 1, x_58); +return x_59; +} } } } else { -uint8_t x_76; +uint8_t x_60; lean_dec(x_3); -x_76 = !lean_is_exclusive(x_41); -if (x_76 == 0) +lean_dec(x_2); +x_60 = !lean_is_exclusive(x_17); +if (x_60 == 0) { -return x_41; +return x_17; } else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; -x_77 = lean_ctor_get(x_41, 0); -x_78 = lean_ctor_get(x_41, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_41); -x_79 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_79, 0, x_77); -lean_ctor_set(x_79, 1, x_78); -return x_79; -} +lean_object* x_61; lean_object* x_62; lean_object* x_63; +x_61 = lean_ctor_get(x_17, 0); +x_62 = lean_ctor_get(x_17, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_17); +x_63 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_63, 0, x_61); +lean_ctor_set(x_63, 1, x_62); +return x_63; } } } else { -uint8_t x_80; +uint8_t x_64; lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_80 = !lean_is_exclusive(x_13); -if (x_80 == 0) +x_64 = !lean_is_exclusive(x_13); +if (x_64 == 0) { +lean_object* x_65; lean_object* x_66; +x_65 = lean_ctor_get(x_13, 0); +lean_dec(x_65); +x_66 = lean_box(0); +lean_ctor_set(x_13, 0, x_66); return x_13; } else { -lean_object* x_81; lean_object* x_82; lean_object* x_83; -x_81 = lean_ctor_get(x_13, 0); -x_82 = lean_ctor_get(x_13, 1); -lean_inc(x_82); -lean_inc(x_81); +lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_67 = lean_ctor_get(x_13, 1); +lean_inc(x_67); lean_dec(x_13); -x_83 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_83, 0, x_81); -lean_ctor_set(x_83, 1, x_82); -return x_83; -} +x_68 = lean_box(0); +x_69 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_69, 0, x_68); +lean_ctor_set(x_69, 1, x_67); +return x_69; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else +{ +uint8_t x_70; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_70 = !lean_is_exclusive(x_13); +if (x_70 == 0) { -uint8_t x_11; lean_object* x_12; lean_object* x_13; -x_11 = 1; -x_12 = lean_box(x_11); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_10); return x_13; } -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.Grind.Split", 28, 28); -return x_1; +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_ctor_get(x_13, 0); +x_72 = lean_ctor_get(x_13, 1); +lean_inc(x_72); +lean_inc(x_71); +lean_dec(x_13); +x_73 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +return x_73; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("_private.Lean.Meta.Tactic.Grind.Split.0.Lean.Meta.Grind.checkCaseSplitStatus", 76, 76); -return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); -return x_1; +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4() { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2; -x_3 = lean_unsigned_to_nat(58u); -x_4 = lean_unsigned_to_nat(43u); -x_5 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3; -x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); -return x_6; -} +uint8_t x_13; lean_object* x_14; lean_object* x_20; +lean_inc(x_1); +x_20 = l_Lean_Meta_Grind_isEqTrue(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; uint8_t x_22; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_unbox(x_21); +lean_dec(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = l_Lean_Meta_Grind_isEqFalse(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_23); +if (lean_obj_tag(x_24) == 0) +{ +lean_object* x_25; uint8_t x_26; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +uint8_t x_27; +lean_dec(x_3); +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_24); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_ctor_get(x_24, 0); +lean_dec(x_28); +x_29 = lean_box(1); +lean_ctor_set(x_24, 0, x_29); +return x_24; } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4___boxed), 10, 0); -return x_1; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_24, 1); +lean_inc(x_30); +lean_dec(x_24); +x_31 = lean_box(1); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_31); +lean_ctor_set(x_32, 1, x_30); +return x_32; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l_Lean_Expr_getAppFn(x_1); -if (lean_obj_tag(x_12) == 4) +lean_object* x_33; lean_object* x_34; +x_33 = lean_ctor_get(x_24, 1); +lean_inc(x_33); +lean_dec(x_24); +lean_inc(x_2); +x_34 = l_Lean_Meta_Grind_isEqTrue(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_33); +if (lean_obj_tag(x_34) == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -lean_dec(x_12); -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -x_14 = l_Lean_Meta_isInductivePredicate(x_13, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_14) == 0) +lean_object* x_35; uint8_t x_36; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_unbox(x_35); +lean_dec(x_35); +if (x_36 == 0) { -lean_object* x_15; uint8_t x_16; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_unbox(x_15); -lean_dec(x_15); -if (x_16 == 0) +lean_object* x_37; lean_object* x_38; +x_37 = lean_ctor_get(x_34, 1); +lean_inc(x_37); +lean_dec(x_34); +x_38 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_37); +if (lean_obj_tag(x_38) == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -lean_dec(x_1); -x_17 = lean_ctor_get(x_14, 1); -lean_inc(x_17); -lean_dec(x_14); -x_18 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; -x_19 = lean_box(0); -x_20 = lean_apply_10(x_18, x_19, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -return x_20; +lean_object* x_39; uint8_t x_40; +x_39 = lean_ctor_get(x_38, 0); +lean_inc(x_39); +x_40 = lean_unbox(x_39); +if (x_40 == 0) +{ +lean_object* x_41; uint8_t x_42; +lean_dec(x_3); +x_41 = lean_ctor_get(x_38, 1); +lean_inc(x_41); +lean_dec(x_38); +x_42 = lean_unbox(x_39); +lean_dec(x_39); +x_13 = x_42; +x_14 = x_41; +goto block_19; } else { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_dec(x_14); -x_22 = l_Lean_Meta_Grind_isEqTrue(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_21); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; uint8_t x_24; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_unbox(x_23); -lean_dec(x_23); -if (x_24 == 0) +lean_object* x_43; lean_object* x_44; +lean_dec(x_39); +x_43 = lean_ctor_get(x_38, 1); +lean_inc(x_43); +lean_dec(x_38); +x_44 = l_Lean_Meta_Grind_isEqTrue(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_43); +if (lean_obj_tag(x_44) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_22, 1); -lean_inc(x_25); -lean_dec(x_22); -x_26 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; -x_27 = lean_box(0); -x_28 = lean_apply_10(x_26, x_27, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); -return x_28; +lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_45 = lean_ctor_get(x_44, 0); +lean_inc(x_45); +x_46 = lean_ctor_get(x_44, 1); +lean_inc(x_46); +lean_dec(x_44); +x_47 = lean_unbox(x_45); +lean_dec(x_45); +x_13 = x_47; +x_14 = x_46; +goto block_19; } else { -uint8_t x_29; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_29 = !lean_is_exclusive(x_22); -if (x_29 == 0) +uint8_t x_48; +x_48 = !lean_is_exclusive(x_44); +if (x_48 == 0) { -lean_object* x_30; uint8_t x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_22, 0); -lean_dec(x_30); -x_31 = 2; -x_32 = lean_box(x_31); -lean_ctor_set(x_22, 0, x_32); -return x_22; +return x_44; } else { -lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; -x_33 = lean_ctor_get(x_22, 1); -lean_inc(x_33); -lean_dec(x_22); -x_34 = 2; -x_35 = lean_box(x_34); -x_36 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_36, 0, x_35); -lean_ctor_set(x_36, 1, x_33); -return x_36; +lean_object* x_49; lean_object* x_50; lean_object* x_51; +x_49 = lean_ctor_get(x_44, 0); +x_50 = lean_ctor_get(x_44, 1); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_44); +x_51 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_51, 0, x_49); +lean_ctor_set(x_51, 1, x_50); +return x_51; +} } } } else { -uint8_t x_37; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +uint8_t x_52; lean_dec(x_3); -x_37 = !lean_is_exclusive(x_22); -if (x_37 == 0) +x_52 = !lean_is_exclusive(x_38); +if (x_52 == 0) { -return x_22; +return x_38; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; -x_38 = lean_ctor_get(x_22, 0); -x_39 = lean_ctor_get(x_22, 1); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_22); -x_40 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_40, 0, x_38); -lean_ctor_set(x_40, 1, x_39); -return x_40; -} +lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_53 = lean_ctor_get(x_38, 0); +x_54 = lean_ctor_get(x_38, 1); +lean_inc(x_54); +lean_inc(x_53); +lean_dec(x_38); +x_55 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +return x_55; } } } else { -uint8_t x_41; -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_1); -x_41 = !lean_is_exclusive(x_14); -if (x_41 == 0) +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_34, 1); +lean_inc(x_56); +lean_dec(x_34); +lean_inc(x_3); +x_57 = l_Lean_Meta_Grind_isEqFalse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_56); +if (lean_obj_tag(x_57) == 0) { -return x_14; -} -else +lean_object* x_58; uint8_t x_59; +x_58 = lean_ctor_get(x_57, 0); +lean_inc(x_58); +x_59 = lean_unbox(x_58); +if (x_59 == 0) +{ +lean_object* x_60; lean_object* x_61; +lean_dec(x_58); +x_60 = lean_ctor_get(x_57, 1); +lean_inc(x_60); +lean_dec(x_57); +x_61 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_60); +if (lean_obj_tag(x_61) == 0) +{ +lean_object* x_62; uint8_t x_63; +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_unbox(x_62); +if (x_63 == 0) +{ +lean_object* x_64; uint8_t x_65; +lean_dec(x_3); +x_64 = lean_ctor_get(x_61, 1); +lean_inc(x_64); +lean_dec(x_61); +x_65 = lean_unbox(x_62); +lean_dec(x_62); +x_13 = x_65; +x_14 = x_64; +goto block_19; +} +else +{ +lean_object* x_66; lean_object* x_67; +lean_dec(x_62); +x_66 = lean_ctor_get(x_61, 1); +lean_inc(x_66); +lean_dec(x_61); +x_67 = l_Lean_Meta_Grind_isEqTrue(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_66); +if (lean_obj_tag(x_67) == 0) +{ +lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_68 = lean_ctor_get(x_67, 0); +lean_inc(x_68); +x_69 = lean_ctor_get(x_67, 1); +lean_inc(x_69); +lean_dec(x_67); +x_70 = lean_unbox(x_68); +lean_dec(x_68); +x_13 = x_70; +x_14 = x_69; +goto block_19; +} +else +{ +uint8_t x_71; +x_71 = !lean_is_exclusive(x_67); +if (x_71 == 0) +{ +return x_67; +} +else +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_72 = lean_ctor_get(x_67, 0); +x_73 = lean_ctor_get(x_67, 1); +lean_inc(x_73); +lean_inc(x_72); +lean_dec(x_67); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_72); +lean_ctor_set(x_74, 1, x_73); +return x_74; +} +} +} +} +else +{ +uint8_t x_75; +lean_dec(x_3); +x_75 = !lean_is_exclusive(x_61); +if (x_75 == 0) +{ +return x_61; +} +else +{ +lean_object* x_76; lean_object* x_77; lean_object* x_78; +x_76 = lean_ctor_get(x_61, 0); +x_77 = lean_ctor_get(x_61, 1); +lean_inc(x_77); +lean_inc(x_76); +lean_dec(x_61); +x_78 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +return x_78; +} +} +} +else +{ +lean_object* x_79; uint8_t x_80; +lean_dec(x_3); +lean_dec(x_2); +x_79 = lean_ctor_get(x_57, 1); +lean_inc(x_79); +lean_dec(x_57); +x_80 = lean_unbox(x_58); +lean_dec(x_58); +x_13 = x_80; +x_14 = x_79; +goto block_19; +} +} +else +{ +uint8_t x_81; +lean_dec(x_3); +lean_dec(x_2); +x_81 = !lean_is_exclusive(x_57); +if (x_81 == 0) +{ +return x_57; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; +x_82 = lean_ctor_get(x_57, 0); +x_83 = lean_ctor_get(x_57, 1); +lean_inc(x_83); +lean_inc(x_82); +lean_dec(x_57); +x_84 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_84, 0, x_82); +lean_ctor_set(x_84, 1, x_83); +return x_84; +} +} +} +} +else +{ +uint8_t x_85; +lean_dec(x_3); +lean_dec(x_2); +x_85 = !lean_is_exclusive(x_34); +if (x_85 == 0) +{ +return x_34; +} +else +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_34, 0); +x_87 = lean_ctor_get(x_34, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_34); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; +} +} +} +} +else +{ +uint8_t x_89; +lean_dec(x_3); +lean_dec(x_2); +x_89 = !lean_is_exclusive(x_24); +if (x_89 == 0) +{ +return x_24; +} +else +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_24, 0); +x_91 = lean_ctor_get(x_24, 1); +lean_inc(x_91); +lean_inc(x_90); +lean_dec(x_24); +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; +} +} +} +else +{ +lean_object* x_93; lean_object* x_94; +lean_dec(x_1); +x_93 = lean_ctor_get(x_20, 1); +lean_inc(x_93); +lean_dec(x_20); +lean_inc(x_2); +x_94 = l_Lean_Meta_Grind_isEqTrue(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_93); +if (lean_obj_tag(x_94) == 0) +{ +lean_object* x_95; uint8_t x_96; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_unbox(x_95); +lean_dec(x_95); +if (x_96 == 0) +{ +lean_object* x_97; lean_object* x_98; +x_97 = lean_ctor_get(x_94, 1); +lean_inc(x_97); +lean_dec(x_94); +x_98 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_97); +if (lean_obj_tag(x_98) == 0) +{ +lean_object* x_99; uint8_t x_100; +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +x_100 = lean_unbox(x_99); +if (x_100 == 0) +{ +lean_object* x_101; uint8_t x_102; +lean_dec(x_3); +x_101 = lean_ctor_get(x_98, 1); +lean_inc(x_101); +lean_dec(x_98); +x_102 = lean_unbox(x_99); +lean_dec(x_99); +x_13 = x_102; +x_14 = x_101; +goto block_19; +} +else +{ +lean_object* x_103; lean_object* x_104; +lean_dec(x_99); +x_103 = lean_ctor_get(x_98, 1); +lean_inc(x_103); +lean_dec(x_98); +x_104 = l_Lean_Meta_Grind_isEqFalse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_103); +if (lean_obj_tag(x_104) == 0) +{ +lean_object* x_105; lean_object* x_106; uint8_t x_107; +x_105 = lean_ctor_get(x_104, 0); +lean_inc(x_105); +x_106 = lean_ctor_get(x_104, 1); +lean_inc(x_106); +lean_dec(x_104); +x_107 = lean_unbox(x_105); +lean_dec(x_105); +x_13 = x_107; +x_14 = x_106; +goto block_19; +} +else +{ +uint8_t x_108; +x_108 = !lean_is_exclusive(x_104); +if (x_108 == 0) +{ +return x_104; +} +else +{ +lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_109 = lean_ctor_get(x_104, 0); +x_110 = lean_ctor_get(x_104, 1); +lean_inc(x_110); +lean_inc(x_109); +lean_dec(x_104); +x_111 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_111, 0, x_109); +lean_ctor_set(x_111, 1, x_110); +return x_111; +} +} +} +} +else +{ +uint8_t x_112; +lean_dec(x_3); +x_112 = !lean_is_exclusive(x_98); +if (x_112 == 0) +{ +return x_98; +} +else +{ +lean_object* x_113; lean_object* x_114; lean_object* x_115; +x_113 = lean_ctor_get(x_98, 0); +x_114 = lean_ctor_get(x_98, 1); +lean_inc(x_114); +lean_inc(x_113); +lean_dec(x_98); +x_115 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_115, 0, x_113); +lean_ctor_set(x_115, 1, x_114); +return x_115; +} +} +} +else +{ +lean_object* x_116; lean_object* x_117; +x_116 = lean_ctor_get(x_94, 1); +lean_inc(x_116); +lean_dec(x_94); +lean_inc(x_3); +x_117 = l_Lean_Meta_Grind_isEqTrue(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_116); +if (lean_obj_tag(x_117) == 0) +{ +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_117, 0); +lean_inc(x_118); +x_119 = lean_unbox(x_118); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; +lean_dec(x_118); +x_120 = lean_ctor_get(x_117, 1); +lean_inc(x_120); +lean_dec(x_117); +x_121 = l_Lean_Meta_Grind_isEqFalse(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_120); +if (lean_obj_tag(x_121) == 0) +{ +lean_object* x_122; uint8_t x_123; +x_122 = lean_ctor_get(x_121, 0); +lean_inc(x_122); +x_123 = lean_unbox(x_122); +if (x_123 == 0) +{ +lean_object* x_124; uint8_t x_125; +lean_dec(x_3); +x_124 = lean_ctor_get(x_121, 1); +lean_inc(x_124); +lean_dec(x_121); +x_125 = lean_unbox(x_122); +lean_dec(x_122); +x_13 = x_125; +x_14 = x_124; +goto block_19; +} +else +{ +lean_object* x_126; lean_object* x_127; +lean_dec(x_122); +x_126 = lean_ctor_get(x_121, 1); +lean_inc(x_126); +lean_dec(x_121); +x_127 = l_Lean_Meta_Grind_isEqFalse(x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_126); +if (lean_obj_tag(x_127) == 0) +{ +lean_object* x_128; lean_object* x_129; uint8_t x_130; +x_128 = lean_ctor_get(x_127, 0); +lean_inc(x_128); +x_129 = lean_ctor_get(x_127, 1); +lean_inc(x_129); +lean_dec(x_127); +x_130 = lean_unbox(x_128); +lean_dec(x_128); +x_13 = x_130; +x_14 = x_129; +goto block_19; +} +else +{ +uint8_t x_131; +x_131 = !lean_is_exclusive(x_127); +if (x_131 == 0) +{ +return x_127; +} +else +{ +lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_132 = lean_ctor_get(x_127, 0); +x_133 = lean_ctor_get(x_127, 1); +lean_inc(x_133); +lean_inc(x_132); +lean_dec(x_127); +x_134 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_134, 0, x_132); +lean_ctor_set(x_134, 1, x_133); +return x_134; +} +} +} +} +else +{ +uint8_t x_135; +lean_dec(x_3); +x_135 = !lean_is_exclusive(x_121); +if (x_135 == 0) +{ +return x_121; +} +else +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; +x_136 = lean_ctor_get(x_121, 0); +x_137 = lean_ctor_get(x_121, 1); +lean_inc(x_137); +lean_inc(x_136); +lean_dec(x_121); +x_138 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_138, 0, x_136); +lean_ctor_set(x_138, 1, x_137); +return x_138; +} +} +} +else +{ +lean_object* x_139; uint8_t x_140; +lean_dec(x_3); +lean_dec(x_2); +x_139 = lean_ctor_get(x_117, 1); +lean_inc(x_139); +lean_dec(x_117); +x_140 = lean_unbox(x_118); +lean_dec(x_118); +x_13 = x_140; +x_14 = x_139; +goto block_19; +} +} +else +{ +uint8_t x_141; +lean_dec(x_3); +lean_dec(x_2); +x_141 = !lean_is_exclusive(x_117); +if (x_141 == 0) +{ +return x_117; +} +else +{ +lean_object* x_142; lean_object* x_143; lean_object* x_144; +x_142 = lean_ctor_get(x_117, 0); +x_143 = lean_ctor_get(x_117, 1); +lean_inc(x_143); +lean_inc(x_142); +lean_dec(x_117); +x_144 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_144, 0, x_142); +lean_ctor_set(x_144, 1, x_143); +return x_144; +} +} +} +} +else +{ +uint8_t x_145; +lean_dec(x_3); +lean_dec(x_2); +x_145 = !lean_is_exclusive(x_94); +if (x_145 == 0) +{ +return x_94; +} +else +{ +lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_146 = lean_ctor_get(x_94, 0); +x_147 = lean_ctor_get(x_94, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_94); +x_148 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_148, 0, x_146); +lean_ctor_set(x_148, 1, x_147); +return x_148; +} +} +} +} +else +{ +uint8_t x_149; +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_149 = !lean_is_exclusive(x_20); +if (x_149 == 0) +{ +return x_20; +} +else +{ +lean_object* x_150; lean_object* x_151; lean_object* x_152; +x_150 = lean_ctor_get(x_20, 0); +x_151 = lean_ctor_get(x_20, 1); +lean_inc(x_151); +lean_inc(x_150); +lean_dec(x_20); +x_152 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 1, x_151); +return x_152; +} +} +block_19: +{ +if (x_13 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1; +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_15); +lean_ctor_set(x_16, 1, x_14); +return x_16; +} +else +{ +lean_object* x_17; lean_object* x_18; +x_17 = lean_box(0); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_14); +return x_18; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_13; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_instMonadMetaM; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__3; +x_2 = l_ReaderT_instMonad___rarg(x_1); +return x_2; +} +} +static lean_object* _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4; +x_2 = l_Lean_Meta_Grind_instInhabitedCaseSplitStatus; +x_3 = l_instInhabitedOfMonad___rarg(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5; +x_12 = lean_panic_fn(x_11, x_1); +x_13 = lean_apply_9(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +return x_13; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(1); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +return x_12; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean.Meta.Tactic.Grind.Split", 28, 28); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("_private.Lean.Meta.Tactic.Grind.Split.0.Lean.Meta.Grind.checkCaseSplitStatus", 76, 76); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("unreachable code has been reached", 33, 33); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2; +x_3 = lean_unsigned_to_nat(90u); +x_4 = lean_unsigned_to_nat(43u); +x_5 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3; +x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); +return x_6; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1___boxed), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Expr_getAppFn(x_1); +if (lean_obj_tag(x_12) == 4) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +lean_dec(x_12); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +x_14 = l_Lean_Meta_isInductivePredicate_x3f(x_13, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5; +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_dec(x_1); +x_18 = lean_box(0); +x_19 = lean_apply_10(x_17, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +return x_19; +} +else +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_15, 0); +lean_inc(x_20); +lean_dec(x_15); +x_21 = l_Lean_Meta_Grind_isEqTrue(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_16); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; uint8_t x_23; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_unbox(x_22); +lean_dec(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_20); +x_24 = lean_ctor_get(x_21, 1); +lean_inc(x_24); +lean_dec(x_21); +x_25 = lean_box(0); +x_26 = lean_apply_10(x_17, x_25, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_24); +return x_26; +} +else +{ +uint8_t x_27; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_27 = !lean_is_exclusive(x_21); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; +x_28 = lean_ctor_get(x_21, 0); +lean_dec(x_28); +x_29 = lean_ctor_get(x_20, 4); +lean_inc(x_29); +x_30 = lean_unsigned_to_nat(0u); +x_31 = l_List_lengthTRAux___rarg(x_29, x_30); +lean_dec(x_29); +x_32 = lean_ctor_get_uint8(x_20, sizeof(void*)*6); +lean_dec(x_20); +x_33 = lean_alloc_ctor(2, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +lean_ctor_set(x_21, 0, x_33); +return x_21; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; +x_34 = lean_ctor_get(x_21, 1); +lean_inc(x_34); +lean_dec(x_21); +x_35 = lean_ctor_get(x_20, 4); +lean_inc(x_35); +x_36 = lean_unsigned_to_nat(0u); +x_37 = l_List_lengthTRAux___rarg(x_35, x_36); +lean_dec(x_35); +x_38 = lean_ctor_get_uint8(x_20, sizeof(void*)*6); +lean_dec(x_20); +x_39 = lean_alloc_ctor(2, 1, 1); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set_uint8(x_39, sizeof(void*)*1, x_38); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_39); +lean_ctor_set(x_40, 1, x_34); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_20); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +x_41 = !lean_is_exclusive(x_21); +if (x_41 == 0) +{ +return x_21; +} +else { lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_42 = lean_ctor_get(x_14, 0); -x_43 = lean_ctor_get(x_14, 1); +x_42 = lean_ctor_get(x_21, 0); +x_43 = lean_ctor_get(x_21, 1); lean_inc(x_43); lean_inc(x_42); -lean_dec(x_14); +lean_dec(x_21); x_44 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_44, 0, x_42); lean_ctor_set(x_44, 1, x_43); @@ -1339,39 +2066,77 @@ return x_44; } } } +} else { -lean_object* x_45; lean_object* x_46; +uint8_t x_45; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_45 = !lean_is_exclusive(x_14); +if (x_45 == 0) +{ +return x_14; +} +else +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_14, 0); +x_47 = lean_ctor_get(x_14, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_14); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; +} +} +} +else +{ +lean_object* x_49; lean_object* x_50; lean_dec(x_12); lean_dec(x_1); -x_45 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4; -x_46 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1(x_45, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_46; +x_49 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4; +x_50 = l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1(x_49, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_50; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = l_Lean_Meta_isMatcherApp___at___private_Lean_Meta_Tactic_Grind_Internalize_0__Lean_Meta_Grind_checkAndAddSplitCandidate___spec__1(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -x_14 = lean_unbox(x_13); -lean_dec(x_13); -if (x_14 == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_st_ref_get(x_10, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) { -lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_12, 0); x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = lean_box(0); -x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -return x_17; +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Meta_isMatcherAppCore_x3f(x_16, x_1); +lean_dec(x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_object* x_18; lean_object* x_19; +lean_free_object(x_12); +x_18 = lean_box(0); +x_19 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(x_1, x_18, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +return x_19; } else { -uint8_t x_18; +lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -1381,46 +2146,80 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); -x_18 = !lean_is_exclusive(x_12); -if (x_18 == 0) -{ -lean_object* x_19; uint8_t x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_12, 0); -lean_dec(x_19); -x_20 = 2; -x_21 = lean_box(x_20); -lean_ctor_set(x_12, 0, x_21); +x_20 = lean_ctor_get(x_17, 0); +lean_inc(x_20); +lean_dec(x_17); +x_21 = l_Lean_Meta_Match_MatcherInfo_numAlts(x_20); +lean_dec(x_20); +x_22 = 0; +x_23 = lean_alloc_ctor(2, 1, 1); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set_uint8(x_23, sizeof(void*)*1, x_22); +lean_ctor_set(x_12, 0, x_23); return x_12; } +} else { -lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_22 = lean_ctor_get(x_12, 1); -lean_inc(x_22); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_24 = lean_ctor_get(x_12, 0); +x_25 = lean_ctor_get(x_12, 1); +lean_inc(x_25); +lean_inc(x_24); lean_dec(x_12); -x_23 = 2; -x_24 = lean_box(x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_22); -return x_25; +x_26 = lean_ctor_get(x_24, 0); +lean_inc(x_26); +lean_dec(x_24); +x_27 = l_Lean_Meta_isMatcherAppCore_x3f(x_26, x_1); +lean_dec(x_26); +if (lean_obj_tag(x_27) == 0) +{ +lean_object* x_28; lean_object* x_29; +x_28 = lean_box(0); +x_29 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(x_1, x_28, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_25); +return x_29; +} +else +{ +lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_30 = lean_ctor_get(x_27, 0); +lean_inc(x_30); +lean_dec(x_27); +x_31 = l_Lean_Meta_Match_MatcherInfo_numAlts(x_30); +lean_dec(x_30); +x_32 = 0; +x_33 = lean_alloc_ctor(2, 1, 1); +lean_ctor_set(x_33, 0, x_31); +lean_ctor_set_uint8(x_33, sizeof(void*)*1, x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_25); +return x_34; } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_11; lean_object* x_12; lean_object* x_13; -x_11 = 0; -x_12 = lean_box(x_11); -x_13 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_10); -return x_13; +lean_object* x_11; lean_object* x_12; +x_11 = lean_box(0); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_11); +lean_ctor_set(x_12, 1, x_10); +return x_12; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1() { _start: { lean_object* x_1; @@ -1428,7 +2227,7 @@ x_1 = lean_mk_string_unchecked("grind", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2() { _start: { lean_object* x_1; @@ -1436,7 +2235,7 @@ x_1 = lean_mk_string_unchecked("debug", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3() { _start: { lean_object* x_1; @@ -1444,26 +2243,26 @@ x_1 = lean_mk_string_unchecked("split", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2; -x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7___boxed), 10, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4___boxed), 10, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6() { _start: { lean_object* x_1; @@ -1471,16 +2270,16 @@ x_1 = lean_mk_string_unchecked("split resolved: ", 16, 16); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8() { _start: { lean_object* x_1; @@ -1488,16 +2287,16 @@ x_1 = lean_mk_string_unchecked("", 0, 0); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; lean_object* x_13; uint8_t x_14; @@ -1513,7 +2312,7 @@ x_15 = lean_ctor_get(x_12, 1); lean_inc(x_15); lean_dec(x_12); x_16 = lean_box(0); -x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6(x_1, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(x_1, x_16, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); return x_17; } else @@ -1526,7 +2325,7 @@ lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint x_19 = lean_ctor_get(x_12, 1); x_20 = lean_ctor_get(x_12, 0); lean_dec(x_20); -x_21 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4; +x_21 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4; x_22 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_21, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_19); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) @@ -1534,7 +2333,7 @@ if (x_23 == 0) lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; x_24 = lean_ctor_get(x_22, 0); x_25 = lean_ctor_get(x_22, 1); -x_26 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5; +x_26 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; x_27 = lean_unbox(x_24); lean_dec(x_24); if (x_27 == 0) @@ -1551,11 +2350,11 @@ else { lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; x_30 = l_Lean_MessageData_ofExpr(x_1); -x_31 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7; +x_31 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7; lean_ctor_set_tag(x_22, 7); lean_ctor_set(x_22, 1, x_30); lean_ctor_set(x_22, 0, x_31); -x_32 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; +x_32 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_32); lean_ctor_set(x_12, 0, x_22); @@ -1577,7 +2376,7 @@ x_38 = lean_ctor_get(x_22, 1); lean_inc(x_38); lean_inc(x_37); lean_dec(x_22); -x_39 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5; +x_39 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; x_40 = lean_unbox(x_37); lean_dec(x_37); if (x_40 == 0) @@ -1593,11 +2392,11 @@ else { lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; x_43 = l_Lean_MessageData_ofExpr(x_1); -x_44 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7; +x_44 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7; x_45 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_45, 0, x_44); lean_ctor_set(x_45, 1, x_43); -x_46 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; +x_46 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9; lean_ctor_set_tag(x_12, 7); lean_ctor_set(x_12, 1, x_46); lean_ctor_set(x_12, 0, x_45); @@ -1618,7 +2417,7 @@ lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean x_51 = lean_ctor_get(x_12, 1); lean_inc(x_51); lean_dec(x_12); -x_52 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4; +x_52 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4; x_53 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_52, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_51); x_54 = lean_ctor_get(x_53, 0); lean_inc(x_54); @@ -1632,7 +2431,7 @@ if (lean_is_exclusive(x_53)) { lean_dec_ref(x_53); x_56 = lean_box(0); } -x_57 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5; +x_57 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5; x_58 = lean_unbox(x_54); lean_dec(x_54); if (x_58 == 0) @@ -1648,7 +2447,7 @@ else { lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; x_61 = l_Lean_MessageData_ofExpr(x_1); -x_62 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7; +x_62 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7; if (lean_is_scalar(x_56)) { x_63 = lean_alloc_ctor(7, 2, 0); } else { @@ -1657,7 +2456,7 @@ if (lean_is_scalar(x_56)) { } lean_ctor_set(x_63, 0, x_62); lean_ctor_set(x_63, 1, x_61); -x_64 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; +x_64 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9; x_65 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_65, 0, x_63); lean_ctor_set(x_65, 1, x_64); @@ -1678,7 +2477,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__1___boxed), 10, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___boxed), 10, 0); return x_1; } } @@ -1722,7 +2521,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("dite", 4, 4); +x_1 = lean_mk_string_unchecked("Eq", 2, 2); return x_1; } } @@ -1740,7 +2539,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_ _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ite", 3, 3); +x_1 = lean_mk_string_unchecked("dite", 4, 4); return x_1; } } @@ -1754,6 +2553,24 @@ x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ite", 3, 3); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -1773,7 +2590,7 @@ if (x_16 == 0) lean_object* x_17; lean_object* x_18; lean_dec(x_15); x_17 = lean_box(0); -x_18 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_18 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_18; } else @@ -1788,7 +2605,7 @@ lean_object* x_22; lean_object* x_23; lean_dec(x_20); lean_dec(x_19); x_22 = lean_box(0); -x_23 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_23 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_23; } else @@ -1806,90 +2623,113 @@ x_29 = l_Lean_Expr_isConstOf(x_25, x_28); if (x_29 == 0) { uint8_t x_30; -lean_dec(x_24); -lean_dec(x_19); x_30 = l_Lean_Expr_isApp(x_25); if (x_30 == 0) { lean_object* x_31; lean_object* x_32; lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_19); x_31 = lean_box(0); -x_32 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_32 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_31, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_32; } else { -lean_object* x_33; uint8_t x_34; +lean_object* x_33; lean_object* x_34; uint8_t x_35; x_33 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); -x_34 = l_Lean_Expr_isApp(x_33); -if (x_34 == 0) +x_34 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__7; +x_35 = l_Lean_Expr_isConstOf(x_33, x_34); +if (x_35 == 0) { -lean_object* x_35; lean_object* x_36; +uint8_t x_36; +lean_dec(x_24); +lean_dec(x_19); +x_36 = l_Lean_Expr_isApp(x_33); +if (x_36 == 0) +{ +lean_object* x_37; lean_object* x_38; lean_dec(x_33); -x_35 = lean_box(0); -x_36 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_36; +x_37 = lean_box(0); +x_38 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_38; } else { -lean_object* x_37; lean_object* x_38; uint8_t x_39; -x_37 = l_Lean_Expr_appArg(x_33, lean_box(0)); -x_38 = l_Lean_Expr_appFnCleanup(x_33, lean_box(0)); -x_39 = l_Lean_Expr_isApp(x_38); -if (x_39 == 0) +lean_object* x_39; lean_object* x_40; uint8_t x_41; +x_39 = l_Lean_Expr_appArg(x_33, lean_box(0)); +x_40 = l_Lean_Expr_appFnCleanup(x_33, lean_box(0)); +x_41 = l_Lean_Expr_isApp(x_40); +if (x_41 == 0) { -lean_object* x_40; lean_object* x_41; -lean_dec(x_38); -lean_dec(x_37); -x_40 = lean_box(0); -x_41 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_41; +lean_object* x_42; lean_object* x_43; +lean_dec(x_40); +lean_dec(x_39); +x_42 = lean_box(0); +x_43 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_42, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_43; } else { -lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_42 = l_Lean_Expr_appFnCleanup(x_38, lean_box(0)); -x_43 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__7; -x_44 = l_Lean_Expr_isConstOf(x_42, x_43); -if (x_44 == 0) -{ -lean_object* x_45; uint8_t x_46; +lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_44 = l_Lean_Expr_appFnCleanup(x_40, lean_box(0)); x_45 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9; -x_46 = l_Lean_Expr_isConstOf(x_42, x_45); -lean_dec(x_42); +x_46 = l_Lean_Expr_isConstOf(x_44, x_45); if (x_46 == 0) { -lean_object* x_47; lean_object* x_48; -lean_dec(x_37); -x_47 = lean_box(0); -x_48 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_48; +lean_object* x_47; uint8_t x_48; +x_47 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11; +x_48 = l_Lean_Expr_isConstOf(x_44, x_47); +lean_dec(x_44); +if (x_48 == 0) +{ +lean_object* x_49; lean_object* x_50; +lean_dec(x_39); +x_49 = lean_box(0); +x_50 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5(x_1, x_49, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_50; } else { -lean_object* x_49; +lean_object* x_51; lean_dec(x_1); -x_49 = lean_apply_10(x_14, x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_49; +x_51 = lean_apply_10(x_14, x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_51; } } else { -lean_object* x_50; -lean_dec(x_42); +lean_object* x_52; +lean_dec(x_44); lean_dec(x_1); -x_50 = lean_apply_10(x_14, x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_50; +x_52 = lean_apply_10(x_14, x_39, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_52; +} +} } } +else +{ +lean_object* x_53; +lean_dec(x_33); +x_53 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIffStatus(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_53; } } } else { -lean_object* x_51; +lean_object* x_54; lean_dec(x_25); -x_51 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_54 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkDisjunctStatus(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -1898,14 +2738,14 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_51; +return x_54; } } else { -lean_object* x_52; +lean_object* x_55; lean_dec(x_25); -x_52 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_55 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkConjunctStatus(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -1914,7 +2754,7 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_52; +return x_55; } } } @@ -1933,39 +2773,26 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); +lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_13; -x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_13; +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_13; -x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_13; +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_2); +return x_12; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -1994,49 +2821,148 @@ lean_dec(x_2); return x_12; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_2); -return x_12; +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_1); +lean_ctor_set(x_12, 1, x_11); +return x_12; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +uint8_t x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_nat_dec_lt(x_1, x_2); +x_14 = lean_box(x_13); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_12); +return x_15; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { +_start: +{ +lean_object* x_15; +x_15 = l_Lean_Meta_Grind_getGeneration(x_1, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +if (lean_obj_tag(x_15) == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +x_17 = lean_ctor_get(x_15, 1); +lean_inc(x_17); +lean_dec(x_15); +x_18 = l_Lean_Meta_Grind_getGeneration(x_2, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_17); +if (lean_obj_tag(x_18) == 0) +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_18, 0); +x_21 = lean_ctor_get(x_18, 1); +x_22 = lean_nat_dec_lt(x_16, x_20); +lean_dec(x_20); +lean_dec(x_16); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +lean_free_object(x_18); +x_23 = lean_box(0); +x_24 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2(x_3, x_4, x_23, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_21); +return x_24; +} +else +{ +uint8_t x_25; lean_object* x_26; +x_25 = 1; +x_26 = lean_box(x_25); +lean_ctor_set(x_18, 0, x_26); +return x_18; +} +} +else +{ +lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_27 = lean_ctor_get(x_18, 0); +x_28 = lean_ctor_get(x_18, 1); +lean_inc(x_28); +lean_inc(x_27); +lean_dec(x_18); +x_29 = lean_nat_dec_lt(x_16, x_27); +lean_dec(x_27); +lean_dec(x_16); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = lean_box(0); +x_31 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2(x_3, x_4, x_30, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_28); +return x_31; +} +else +{ +uint8_t x_32; lean_object* x_33; lean_object* x_34; +x_32 = 1; +x_33 = lean_box(x_32); +x_34 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_34, 0, x_33); +lean_ctor_set(x_34, 1, x_28); +return x_34; +} +} +} +else +{ +uint8_t x_35; +lean_dec(x_16); +x_35 = !lean_is_exclusive(x_18); +if (x_35 == 0) +{ +return x_18; +} +else +{ +lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_36 = lean_ctor_get(x_18, 0); +x_37 = lean_ctor_get(x_18, 1); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_18); +x_38 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_38, 0, x_36); +lean_ctor_set(x_38, 1, x_37); +return x_38; +} } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +uint8_t x_39; lean_dec(x_2); -lean_dec(x_1); -return x_11; -} +x_39 = !lean_is_exclusive(x_15); +if (x_39 == 0) +{ +return x_15; } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_2); -return x_12; +lean_object* x_40; lean_object* x_41; lean_object* x_42; +x_40 = lean_ctor_get(x_15, 0); +x_41 = lean_ctor_get(x_15, 1); +lean_inc(x_41); +lean_inc(x_40); +lean_dec(x_15); +x_42 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_42, 0, x_40); +lean_ctor_set(x_42, 1, x_41); +return x_42; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: -{ -lean_object* x_12; -x_12 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_11); -return x_12; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { @@ -2062,10 +2988,10 @@ x_16 = !lean_is_exclusive(x_14); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_14, 16); +x_17 = lean_ctor_get(x_14, 18); lean_dec(x_17); x_18 = l_List_reverse___rarg(x_3); -lean_ctor_set(x_14, 16, x_18); +lean_ctor_set(x_14, 18, x_18); x_19 = lean_st_ref_set(x_4, x_14, x_15); if (lean_obj_tag(x_2) == 0) { @@ -2094,75 +3020,139 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; x_24 = lean_ctor_get(x_19, 1); lean_inc(x_24); lean_dec(x_19); -x_25 = lean_st_ref_take(x_4, x_24); -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); +x_25 = lean_ctor_get(x_2, 1); +lean_inc(x_25); +x_26 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); +x_27 = lean_st_ref_get(x_4, x_24); +x_28 = lean_ctor_get(x_27, 0); +lean_inc(x_28); +x_29 = lean_ctor_get(x_27, 1); +lean_inc(x_29); +lean_dec(x_27); +x_71 = lean_ctor_get(x_28, 19); +lean_inc(x_71); +lean_dec(x_28); +x_72 = lean_unsigned_to_nat(1u); +x_73 = lean_nat_dec_lt(x_72, x_25); lean_dec(x_25); -x_28 = !lean_is_exclusive(x_26); -if (x_28 == 0) +x_74 = lean_st_ref_take(x_4, x_29); +if (x_73 == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_29 = lean_ctor_get(x_26, 17); -x_30 = lean_ctor_get(x_26, 12); -lean_dec(x_30); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_nat_add(x_29, x_31); -lean_dec(x_29); -x_33 = lean_unsigned_to_nat(0u); -lean_ctor_set(x_26, 17, x_32); -lean_ctor_set(x_26, 12, x_33); -x_34 = lean_st_ref_set(x_4, x_26, x_27); -lean_dec(x_4); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +if (x_26 == 0) { -lean_object* x_36; -x_36 = lean_ctor_get(x_34, 0); -lean_dec(x_36); -lean_ctor_set(x_34, 0, x_2); -return x_34; +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_74, 1); +lean_inc(x_76); +lean_dec(x_74); +x_30 = x_71; +x_31 = x_75; +x_32 = x_76; +goto block_70; } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_74, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_74, 1); +lean_inc(x_78); +lean_dec(x_74); +x_79 = lean_nat_add(x_71, x_72); +lean_dec(x_71); +x_30 = x_79; +x_31 = x_77; +x_32 = x_78; +goto block_70; +} +} +else +{ +lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +lean_dec(x_74); +x_82 = lean_nat_add(x_71, x_72); +lean_dec(x_71); +x_30 = x_82; +x_31 = x_80; +x_32 = x_81; +goto block_70; +} +block_70: +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_31); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_34 = lean_ctor_get(x_31, 19); lean_dec(x_34); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_2); -lean_ctor_set(x_38, 1, x_37); -return x_38; +x_35 = lean_ctor_get(x_31, 14); +lean_dec(x_35); +x_36 = lean_unsigned_to_nat(0u); +lean_ctor_set(x_31, 19, x_30); +lean_ctor_set(x_31, 14, x_36); +x_37 = lean_st_ref_set(x_4, x_31, x_32); +lean_dec(x_4); +x_38 = !lean_is_exclusive(x_37); +if (x_38 == 0) +{ +lean_object* x_39; +x_39 = lean_ctor_get(x_37, 0); +lean_dec(x_39); +lean_ctor_set(x_37, 0, x_2); +return x_37; +} +else +{ +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_37, 1); +lean_inc(x_40); +lean_dec(x_37); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_2); +lean_ctor_set(x_41, 1, x_40); +return x_41; } } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_39 = lean_ctor_get(x_26, 0); -x_40 = lean_ctor_get(x_26, 1); -x_41 = lean_ctor_get(x_26, 2); -x_42 = lean_ctor_get(x_26, 3); -x_43 = lean_ctor_get(x_26, 4); -x_44 = lean_ctor_get(x_26, 5); -x_45 = lean_ctor_get_uint8(x_26, sizeof(void*)*20); -x_46 = lean_ctor_get(x_26, 6); -x_47 = lean_ctor_get(x_26, 7); -x_48 = lean_ctor_get(x_26, 8); -x_49 = lean_ctor_get(x_26, 9); -x_50 = lean_ctor_get(x_26, 10); -x_51 = lean_ctor_get(x_26, 11); -x_52 = lean_ctor_get(x_26, 13); -x_53 = lean_ctor_get(x_26, 14); -x_54 = lean_ctor_get(x_26, 15); -x_55 = lean_ctor_get(x_26, 16); -x_56 = lean_ctor_get(x_26, 17); -x_57 = lean_ctor_get(x_26, 18); -x_58 = lean_ctor_get(x_26, 19); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +x_42 = lean_ctor_get(x_31, 0); +x_43 = lean_ctor_get(x_31, 1); +x_44 = lean_ctor_get(x_31, 2); +x_45 = lean_ctor_get(x_31, 3); +x_46 = lean_ctor_get(x_31, 4); +x_47 = lean_ctor_get(x_31, 5); +x_48 = lean_ctor_get(x_31, 6); +x_49 = lean_ctor_get_uint8(x_31, sizeof(void*)*23); +x_50 = lean_ctor_get(x_31, 7); +x_51 = lean_ctor_get(x_31, 8); +x_52 = lean_ctor_get(x_31, 9); +x_53 = lean_ctor_get(x_31, 10); +x_54 = lean_ctor_get(x_31, 11); +x_55 = lean_ctor_get(x_31, 12); +x_56 = lean_ctor_get(x_31, 13); +x_57 = lean_ctor_get(x_31, 15); +x_58 = lean_ctor_get(x_31, 16); +x_59 = lean_ctor_get(x_31, 17); +x_60 = lean_ctor_get(x_31, 18); +x_61 = lean_ctor_get(x_31, 20); +x_62 = lean_ctor_get(x_31, 21); +x_63 = lean_ctor_get(x_31, 22); +lean_inc(x_63); +lean_inc(x_62); +lean_inc(x_61); +lean_inc(x_60); +lean_inc(x_59); lean_inc(x_58); lean_inc(x_57); lean_inc(x_56); @@ -2172,295 +3162,369 @@ lean_inc(x_53); lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); -lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); +lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_26); -x_59 = lean_unsigned_to_nat(1u); -x_60 = lean_nat_add(x_56, x_59); -lean_dec(x_56); -x_61 = lean_unsigned_to_nat(0u); -x_62 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_62, 0, x_39); -lean_ctor_set(x_62, 1, x_40); -lean_ctor_set(x_62, 2, x_41); -lean_ctor_set(x_62, 3, x_42); -lean_ctor_set(x_62, 4, x_43); -lean_ctor_set(x_62, 5, x_44); -lean_ctor_set(x_62, 6, x_46); -lean_ctor_set(x_62, 7, x_47); -lean_ctor_set(x_62, 8, x_48); -lean_ctor_set(x_62, 9, x_49); -lean_ctor_set(x_62, 10, x_50); -lean_ctor_set(x_62, 11, x_51); -lean_ctor_set(x_62, 12, x_61); -lean_ctor_set(x_62, 13, x_52); -lean_ctor_set(x_62, 14, x_53); -lean_ctor_set(x_62, 15, x_54); -lean_ctor_set(x_62, 16, x_55); -lean_ctor_set(x_62, 17, x_60); -lean_ctor_set(x_62, 18, x_57); -lean_ctor_set(x_62, 19, x_58); -lean_ctor_set_uint8(x_62, sizeof(void*)*20, x_45); -x_63 = lean_st_ref_set(x_4, x_62, x_27); +lean_dec(x_31); +x_64 = lean_unsigned_to_nat(0u); +x_65 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_65, 0, x_42); +lean_ctor_set(x_65, 1, x_43); +lean_ctor_set(x_65, 2, x_44); +lean_ctor_set(x_65, 3, x_45); +lean_ctor_set(x_65, 4, x_46); +lean_ctor_set(x_65, 5, x_47); +lean_ctor_set(x_65, 6, x_48); +lean_ctor_set(x_65, 7, x_50); +lean_ctor_set(x_65, 8, x_51); +lean_ctor_set(x_65, 9, x_52); +lean_ctor_set(x_65, 10, x_53); +lean_ctor_set(x_65, 11, x_54); +lean_ctor_set(x_65, 12, x_55); +lean_ctor_set(x_65, 13, x_56); +lean_ctor_set(x_65, 14, x_64); +lean_ctor_set(x_65, 15, x_57); +lean_ctor_set(x_65, 16, x_58); +lean_ctor_set(x_65, 17, x_59); +lean_ctor_set(x_65, 18, x_60); +lean_ctor_set(x_65, 19, x_30); +lean_ctor_set(x_65, 20, x_61); +lean_ctor_set(x_65, 21, x_62); +lean_ctor_set(x_65, 22, x_63); +lean_ctor_set_uint8(x_65, sizeof(void*)*23, x_49); +x_66 = lean_st_ref_set(x_4, x_65, x_32); lean_dec(x_4); -x_64 = lean_ctor_get(x_63, 1); -lean_inc(x_64); -if (lean_is_exclusive(x_63)) { - lean_ctor_release(x_63, 0); - lean_ctor_release(x_63, 1); - x_65 = x_63; +x_67 = lean_ctor_get(x_66, 1); +lean_inc(x_67); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_68 = x_66; } else { - lean_dec_ref(x_63); - x_65 = lean_box(0); + lean_dec_ref(x_66); + x_68 = lean_box(0); } -if (lean_is_scalar(x_65)) { - x_66 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_68)) { + x_69 = lean_alloc_ctor(0, 2, 0); } else { - x_66 = x_65; -} -lean_ctor_set(x_66, 0, x_2); -lean_ctor_set(x_66, 1, x_64); -return x_66; -} -} -} -else -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_67 = lean_ctor_get(x_14, 0); -x_68 = lean_ctor_get(x_14, 1); -x_69 = lean_ctor_get(x_14, 2); -x_70 = lean_ctor_get(x_14, 3); -x_71 = lean_ctor_get(x_14, 4); -x_72 = lean_ctor_get(x_14, 5); -x_73 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); -x_74 = lean_ctor_get(x_14, 6); -x_75 = lean_ctor_get(x_14, 7); -x_76 = lean_ctor_get(x_14, 8); -x_77 = lean_ctor_get(x_14, 9); -x_78 = lean_ctor_get(x_14, 10); -x_79 = lean_ctor_get(x_14, 11); -x_80 = lean_ctor_get(x_14, 12); -x_81 = lean_ctor_get(x_14, 13); -x_82 = lean_ctor_get(x_14, 14); -x_83 = lean_ctor_get(x_14, 15); -x_84 = lean_ctor_get(x_14, 17); -x_85 = lean_ctor_get(x_14, 18); -x_86 = lean_ctor_get(x_14, 19); + x_69 = x_68; +} +lean_ctor_set(x_69, 0, x_2); +lean_ctor_set(x_69, 1, x_67); +return x_69; +} +} +} +} +else +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; +x_83 = lean_ctor_get(x_14, 0); +x_84 = lean_ctor_get(x_14, 1); +x_85 = lean_ctor_get(x_14, 2); +x_86 = lean_ctor_get(x_14, 3); +x_87 = lean_ctor_get(x_14, 4); +x_88 = lean_ctor_get(x_14, 5); +x_89 = lean_ctor_get(x_14, 6); +x_90 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); +x_91 = lean_ctor_get(x_14, 7); +x_92 = lean_ctor_get(x_14, 8); +x_93 = lean_ctor_get(x_14, 9); +x_94 = lean_ctor_get(x_14, 10); +x_95 = lean_ctor_get(x_14, 11); +x_96 = lean_ctor_get(x_14, 12); +x_97 = lean_ctor_get(x_14, 13); +x_98 = lean_ctor_get(x_14, 14); +x_99 = lean_ctor_get(x_14, 15); +x_100 = lean_ctor_get(x_14, 16); +x_101 = lean_ctor_get(x_14, 17); +x_102 = lean_ctor_get(x_14, 19); +x_103 = lean_ctor_get(x_14, 20); +x_104 = lean_ctor_get(x_14, 21); +x_105 = lean_ctor_get(x_14, 22); +lean_inc(x_105); +lean_inc(x_104); +lean_inc(x_103); +lean_inc(x_102); +lean_inc(x_101); +lean_inc(x_100); +lean_inc(x_99); +lean_inc(x_98); +lean_inc(x_97); +lean_inc(x_96); +lean_inc(x_95); +lean_inc(x_94); +lean_inc(x_93); +lean_inc(x_92); +lean_inc(x_91); +lean_inc(x_89); +lean_inc(x_88); +lean_inc(x_87); lean_inc(x_86); lean_inc(x_85); lean_inc(x_84); lean_inc(x_83); -lean_inc(x_82); -lean_inc(x_81); -lean_inc(x_80); -lean_inc(x_79); -lean_inc(x_78); -lean_inc(x_77); -lean_inc(x_76); -lean_inc(x_75); -lean_inc(x_74); -lean_inc(x_72); -lean_inc(x_71); -lean_inc(x_70); -lean_inc(x_69); -lean_inc(x_68); -lean_inc(x_67); lean_dec(x_14); -x_87 = l_List_reverse___rarg(x_3); -x_88 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_88, 0, x_67); -lean_ctor_set(x_88, 1, x_68); -lean_ctor_set(x_88, 2, x_69); -lean_ctor_set(x_88, 3, x_70); -lean_ctor_set(x_88, 4, x_71); -lean_ctor_set(x_88, 5, x_72); -lean_ctor_set(x_88, 6, x_74); -lean_ctor_set(x_88, 7, x_75); -lean_ctor_set(x_88, 8, x_76); -lean_ctor_set(x_88, 9, x_77); -lean_ctor_set(x_88, 10, x_78); -lean_ctor_set(x_88, 11, x_79); -lean_ctor_set(x_88, 12, x_80); -lean_ctor_set(x_88, 13, x_81); -lean_ctor_set(x_88, 14, x_82); -lean_ctor_set(x_88, 15, x_83); -lean_ctor_set(x_88, 16, x_87); -lean_ctor_set(x_88, 17, x_84); -lean_ctor_set(x_88, 18, x_85); -lean_ctor_set(x_88, 19, x_86); -lean_ctor_set_uint8(x_88, sizeof(void*)*20, x_73); -x_89 = lean_st_ref_set(x_4, x_88, x_15); +x_106 = l_List_reverse___rarg(x_3); +x_107 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_107, 0, x_83); +lean_ctor_set(x_107, 1, x_84); +lean_ctor_set(x_107, 2, x_85); +lean_ctor_set(x_107, 3, x_86); +lean_ctor_set(x_107, 4, x_87); +lean_ctor_set(x_107, 5, x_88); +lean_ctor_set(x_107, 6, x_89); +lean_ctor_set(x_107, 7, x_91); +lean_ctor_set(x_107, 8, x_92); +lean_ctor_set(x_107, 9, x_93); +lean_ctor_set(x_107, 10, x_94); +lean_ctor_set(x_107, 11, x_95); +lean_ctor_set(x_107, 12, x_96); +lean_ctor_set(x_107, 13, x_97); +lean_ctor_set(x_107, 14, x_98); +lean_ctor_set(x_107, 15, x_99); +lean_ctor_set(x_107, 16, x_100); +lean_ctor_set(x_107, 17, x_101); +lean_ctor_set(x_107, 18, x_106); +lean_ctor_set(x_107, 19, x_102); +lean_ctor_set(x_107, 20, x_103); +lean_ctor_set(x_107, 21, x_104); +lean_ctor_set(x_107, 22, x_105); +lean_ctor_set_uint8(x_107, sizeof(void*)*23, x_90); +x_108 = lean_st_ref_set(x_4, x_107, x_15); if (lean_obj_tag(x_2) == 0) { -lean_object* x_90; lean_object* x_91; lean_object* x_92; +lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_dec(x_4); -x_90 = lean_ctor_get(x_89, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_89)) { - lean_ctor_release(x_89, 0); - lean_ctor_release(x_89, 1); - x_91 = x_89; +x_109 = lean_ctor_get(x_108, 1); +lean_inc(x_109); +if (lean_is_exclusive(x_108)) { + lean_ctor_release(x_108, 0); + lean_ctor_release(x_108, 1); + x_110 = x_108; } else { - lean_dec_ref(x_89); - x_91 = lean_box(0); + lean_dec_ref(x_108); + x_110 = lean_box(0); } -if (lean_is_scalar(x_91)) { - x_92 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_110)) { + x_111 = lean_alloc_ctor(0, 2, 0); } else { - x_92 = x_91; + x_111 = x_110; } -lean_ctor_set(x_92, 0, x_2); -lean_ctor_set(x_92, 1, x_90); -return x_92; +lean_ctor_set(x_111, 0, x_2); +lean_ctor_set(x_111, 1, x_109); +return x_111; } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; uint8_t x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_93 = lean_ctor_get(x_89, 1); -lean_inc(x_93); -lean_dec(x_89); -x_94 = lean_st_ref_take(x_4, x_93); -x_95 = lean_ctor_get(x_94, 0); -lean_inc(x_95); -x_96 = lean_ctor_get(x_94, 1); -lean_inc(x_96); -lean_dec(x_94); -x_97 = lean_ctor_get(x_95, 0); -lean_inc(x_97); -x_98 = lean_ctor_get(x_95, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_95, 2); -lean_inc(x_99); -x_100 = lean_ctor_get(x_95, 3); -lean_inc(x_100); -x_101 = lean_ctor_get(x_95, 4); -lean_inc(x_101); -x_102 = lean_ctor_get(x_95, 5); -lean_inc(x_102); -x_103 = lean_ctor_get_uint8(x_95, sizeof(void*)*20); -x_104 = lean_ctor_get(x_95, 6); -lean_inc(x_104); -x_105 = lean_ctor_get(x_95, 7); -lean_inc(x_105); -x_106 = lean_ctor_get(x_95, 8); -lean_inc(x_106); -x_107 = lean_ctor_get(x_95, 9); -lean_inc(x_107); -x_108 = lean_ctor_get(x_95, 10); -lean_inc(x_108); -x_109 = lean_ctor_get(x_95, 11); -lean_inc(x_109); -x_110 = lean_ctor_get(x_95, 13); -lean_inc(x_110); -x_111 = lean_ctor_get(x_95, 14); -lean_inc(x_111); -x_112 = lean_ctor_get(x_95, 15); +lean_object* x_112; lean_object* x_113; uint8_t x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_151; lean_object* x_152; uint8_t x_153; lean_object* x_154; +x_112 = lean_ctor_get(x_108, 1); lean_inc(x_112); -x_113 = lean_ctor_get(x_95, 16); +lean_dec(x_108); +x_113 = lean_ctor_get(x_2, 1); lean_inc(x_113); -x_114 = lean_ctor_get(x_95, 17); -lean_inc(x_114); -x_115 = lean_ctor_get(x_95, 18); -lean_inc(x_115); -x_116 = lean_ctor_get(x_95, 19); +x_114 = lean_ctor_get_uint8(x_2, sizeof(void*)*2); +x_115 = lean_st_ref_get(x_4, x_112); +x_116 = lean_ctor_get(x_115, 0); lean_inc(x_116); -if (lean_is_exclusive(x_95)) { - lean_ctor_release(x_95, 0); - lean_ctor_release(x_95, 1); - lean_ctor_release(x_95, 2); - lean_ctor_release(x_95, 3); - lean_ctor_release(x_95, 4); - lean_ctor_release(x_95, 5); - lean_ctor_release(x_95, 6); - lean_ctor_release(x_95, 7); - lean_ctor_release(x_95, 8); - lean_ctor_release(x_95, 9); - lean_ctor_release(x_95, 10); - lean_ctor_release(x_95, 11); - lean_ctor_release(x_95, 12); - lean_ctor_release(x_95, 13); - lean_ctor_release(x_95, 14); - lean_ctor_release(x_95, 15); - lean_ctor_release(x_95, 16); - lean_ctor_release(x_95, 17); - lean_ctor_release(x_95, 18); - lean_ctor_release(x_95, 19); - x_117 = x_95; +x_117 = lean_ctor_get(x_115, 1); +lean_inc(x_117); +lean_dec(x_115); +x_151 = lean_ctor_get(x_116, 19); +lean_inc(x_151); +lean_dec(x_116); +x_152 = lean_unsigned_to_nat(1u); +x_153 = lean_nat_dec_lt(x_152, x_113); +lean_dec(x_113); +x_154 = lean_st_ref_take(x_4, x_117); +if (x_153 == 0) +{ +if (x_114 == 0) +{ +lean_object* x_155; lean_object* x_156; +x_155 = lean_ctor_get(x_154, 0); +lean_inc(x_155); +x_156 = lean_ctor_get(x_154, 1); +lean_inc(x_156); +lean_dec(x_154); +x_118 = x_151; +x_119 = x_155; +x_120 = x_156; +goto block_150; +} +else +{ +lean_object* x_157; lean_object* x_158; lean_object* x_159; +x_157 = lean_ctor_get(x_154, 0); +lean_inc(x_157); +x_158 = lean_ctor_get(x_154, 1); +lean_inc(x_158); +lean_dec(x_154); +x_159 = lean_nat_add(x_151, x_152); +lean_dec(x_151); +x_118 = x_159; +x_119 = x_157; +x_120 = x_158; +goto block_150; +} +} +else +{ +lean_object* x_160; lean_object* x_161; lean_object* x_162; +x_160 = lean_ctor_get(x_154, 0); +lean_inc(x_160); +x_161 = lean_ctor_get(x_154, 1); +lean_inc(x_161); +lean_dec(x_154); +x_162 = lean_nat_add(x_151, x_152); +lean_dec(x_151); +x_118 = x_162; +x_119 = x_160; +x_120 = x_161; +goto block_150; +} +block_150: +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; uint8_t x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; +x_121 = lean_ctor_get(x_119, 0); +lean_inc(x_121); +x_122 = lean_ctor_get(x_119, 1); +lean_inc(x_122); +x_123 = lean_ctor_get(x_119, 2); +lean_inc(x_123); +x_124 = lean_ctor_get(x_119, 3); +lean_inc(x_124); +x_125 = lean_ctor_get(x_119, 4); +lean_inc(x_125); +x_126 = lean_ctor_get(x_119, 5); +lean_inc(x_126); +x_127 = lean_ctor_get(x_119, 6); +lean_inc(x_127); +x_128 = lean_ctor_get_uint8(x_119, sizeof(void*)*23); +x_129 = lean_ctor_get(x_119, 7); +lean_inc(x_129); +x_130 = lean_ctor_get(x_119, 8); +lean_inc(x_130); +x_131 = lean_ctor_get(x_119, 9); +lean_inc(x_131); +x_132 = lean_ctor_get(x_119, 10); +lean_inc(x_132); +x_133 = lean_ctor_get(x_119, 11); +lean_inc(x_133); +x_134 = lean_ctor_get(x_119, 12); +lean_inc(x_134); +x_135 = lean_ctor_get(x_119, 13); +lean_inc(x_135); +x_136 = lean_ctor_get(x_119, 15); +lean_inc(x_136); +x_137 = lean_ctor_get(x_119, 16); +lean_inc(x_137); +x_138 = lean_ctor_get(x_119, 17); +lean_inc(x_138); +x_139 = lean_ctor_get(x_119, 18); +lean_inc(x_139); +x_140 = lean_ctor_get(x_119, 20); +lean_inc(x_140); +x_141 = lean_ctor_get(x_119, 21); +lean_inc(x_141); +x_142 = lean_ctor_get(x_119, 22); +lean_inc(x_142); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + lean_ctor_release(x_119, 1); + lean_ctor_release(x_119, 2); + lean_ctor_release(x_119, 3); + lean_ctor_release(x_119, 4); + lean_ctor_release(x_119, 5); + lean_ctor_release(x_119, 6); + lean_ctor_release(x_119, 7); + lean_ctor_release(x_119, 8); + lean_ctor_release(x_119, 9); + lean_ctor_release(x_119, 10); + lean_ctor_release(x_119, 11); + lean_ctor_release(x_119, 12); + lean_ctor_release(x_119, 13); + lean_ctor_release(x_119, 14); + lean_ctor_release(x_119, 15); + lean_ctor_release(x_119, 16); + lean_ctor_release(x_119, 17); + lean_ctor_release(x_119, 18); + lean_ctor_release(x_119, 19); + lean_ctor_release(x_119, 20); + lean_ctor_release(x_119, 21); + lean_ctor_release(x_119, 22); + x_143 = x_119; } else { - lean_dec_ref(x_95); - x_117 = lean_box(0); -} -x_118 = lean_unsigned_to_nat(1u); -x_119 = lean_nat_add(x_114, x_118); -lean_dec(x_114); -x_120 = lean_unsigned_to_nat(0u); -if (lean_is_scalar(x_117)) { - x_121 = lean_alloc_ctor(0, 20, 1); + lean_dec_ref(x_119); + x_143 = lean_box(0); +} +x_144 = lean_unsigned_to_nat(0u); +if (lean_is_scalar(x_143)) { + x_145 = lean_alloc_ctor(0, 23, 1); } else { - x_121 = x_117; -} -lean_ctor_set(x_121, 0, x_97); -lean_ctor_set(x_121, 1, x_98); -lean_ctor_set(x_121, 2, x_99); -lean_ctor_set(x_121, 3, x_100); -lean_ctor_set(x_121, 4, x_101); -lean_ctor_set(x_121, 5, x_102); -lean_ctor_set(x_121, 6, x_104); -lean_ctor_set(x_121, 7, x_105); -lean_ctor_set(x_121, 8, x_106); -lean_ctor_set(x_121, 9, x_107); -lean_ctor_set(x_121, 10, x_108); -lean_ctor_set(x_121, 11, x_109); -lean_ctor_set(x_121, 12, x_120); -lean_ctor_set(x_121, 13, x_110); -lean_ctor_set(x_121, 14, x_111); -lean_ctor_set(x_121, 15, x_112); -lean_ctor_set(x_121, 16, x_113); -lean_ctor_set(x_121, 17, x_119); -lean_ctor_set(x_121, 18, x_115); -lean_ctor_set(x_121, 19, x_116); -lean_ctor_set_uint8(x_121, sizeof(void*)*20, x_103); -x_122 = lean_st_ref_set(x_4, x_121, x_96); + x_145 = x_143; +} +lean_ctor_set(x_145, 0, x_121); +lean_ctor_set(x_145, 1, x_122); +lean_ctor_set(x_145, 2, x_123); +lean_ctor_set(x_145, 3, x_124); +lean_ctor_set(x_145, 4, x_125); +lean_ctor_set(x_145, 5, x_126); +lean_ctor_set(x_145, 6, x_127); +lean_ctor_set(x_145, 7, x_129); +lean_ctor_set(x_145, 8, x_130); +lean_ctor_set(x_145, 9, x_131); +lean_ctor_set(x_145, 10, x_132); +lean_ctor_set(x_145, 11, x_133); +lean_ctor_set(x_145, 12, x_134); +lean_ctor_set(x_145, 13, x_135); +lean_ctor_set(x_145, 14, x_144); +lean_ctor_set(x_145, 15, x_136); +lean_ctor_set(x_145, 16, x_137); +lean_ctor_set(x_145, 17, x_138); +lean_ctor_set(x_145, 18, x_139); +lean_ctor_set(x_145, 19, x_118); +lean_ctor_set(x_145, 20, x_140); +lean_ctor_set(x_145, 21, x_141); +lean_ctor_set(x_145, 22, x_142); +lean_ctor_set_uint8(x_145, sizeof(void*)*23, x_128); +x_146 = lean_st_ref_set(x_4, x_145, x_120); lean_dec(x_4); -x_123 = lean_ctor_get(x_122, 1); -lean_inc(x_123); -if (lean_is_exclusive(x_122)) { - lean_ctor_release(x_122, 0); - lean_ctor_release(x_122, 1); - x_124 = x_122; +x_147 = lean_ctor_get(x_146, 1); +lean_inc(x_147); +if (lean_is_exclusive(x_146)) { + lean_ctor_release(x_146, 0); + lean_ctor_release(x_146, 1); + x_148 = x_146; } else { - lean_dec_ref(x_122); - x_124 = lean_box(0); + lean_dec_ref(x_146); + x_148 = lean_box(0); } -if (lean_is_scalar(x_124)) { - x_125 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_148)) { + x_149 = lean_alloc_ctor(0, 2, 0); } else { - x_125 = x_124; + x_149 = x_148; +} +lean_ctor_set(x_149, 0, x_2); +lean_ctor_set(x_149, 1, x_147); +return x_149; } -lean_ctor_set(x_125, 0, x_2); -lean_ctor_set(x_125, 1, x_123); -return x_125; } } } else { -uint8_t x_126; -x_126 = !lean_is_exclusive(x_1); -if (x_126 == 0) +uint8_t x_163; +x_163 = !lean_is_exclusive(x_1); +if (x_163 == 0) { -lean_object* x_127; lean_object* x_128; lean_object* x_129; -x_127 = lean_ctor_get(x_1, 0); -x_128 = lean_ctor_get(x_1, 1); +lean_object* x_164; lean_object* x_165; lean_object* x_166; +x_164 = lean_ctor_get(x_1, 0); +x_165 = lean_ctor_get(x_1, 1); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); @@ -2469,100 +3533,243 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_127); -x_129 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(x_127, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_129) == 0) +lean_inc(x_164); +x_166 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(x_164, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_166) == 0) { -lean_object* x_130; uint8_t x_131; -x_130 = lean_ctor_get(x_129, 0); -lean_inc(x_130); -x_131 = lean_unbox(x_130); -lean_dec(x_130); -switch (x_131) { +lean_object* x_167; +x_167 = lean_ctor_get(x_166, 0); +lean_inc(x_167); +switch (lean_obj_tag(x_167)) { case 0: { -lean_object* x_132; +lean_object* x_168; lean_free_object(x_1); -lean_dec(x_127); -x_132 = lean_ctor_get(x_129, 1); -lean_inc(x_132); -lean_dec(x_129); -x_1 = x_128; -x_12 = x_132; +lean_dec(x_164); +x_168 = lean_ctor_get(x_166, 1); +lean_inc(x_168); +lean_dec(x_166); +x_1 = x_165; +x_12 = x_168; +goto _start; +} +case 1: +{ +lean_object* x_170; +x_170 = lean_ctor_get(x_166, 1); +lean_inc(x_170); +lean_dec(x_166); +lean_ctor_set(x_1, 1, x_3); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_170; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +default: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_172; lean_object* x_173; uint8_t x_174; lean_object* x_175; +lean_free_object(x_1); +x_172 = lean_ctor_get(x_166, 1); +lean_inc(x_172); +lean_dec(x_166); +x_173 = lean_ctor_get(x_167, 0); +lean_inc(x_173); +x_174 = lean_ctor_get_uint8(x_167, sizeof(void*)*1); +lean_dec(x_167); +x_175 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_175, 0, x_164); +lean_ctor_set(x_175, 1, x_173); +lean_ctor_set_uint8(x_175, sizeof(void*)*2, x_174); +x_1 = x_165; +x_2 = x_175; +x_12 = x_172; +goto _start; +} +else +{ +lean_object* x_177; lean_object* x_178; uint8_t x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_177 = lean_ctor_get(x_166, 1); +lean_inc(x_177); +lean_dec(x_166); +x_178 = lean_ctor_get(x_167, 0); +lean_inc(x_178); +x_179 = lean_ctor_get_uint8(x_167, sizeof(void*)*1); +lean_dec(x_167); +x_180 = lean_ctor_get(x_2, 0); +lean_inc(x_180); +x_181 = lean_ctor_get(x_2, 1); +lean_inc(x_181); +x_182 = lean_unsigned_to_nat(1u); +x_183 = lean_nat_dec_eq(x_178, x_182); +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; +x_184 = lean_box(0); +lean_inc(x_180); +lean_inc(x_164); +x_185 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_164, x_180, x_178, x_181, x_184, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_177); +lean_dec(x_181); +if (lean_obj_tag(x_185) == 0) +{ +lean_object* x_186; uint8_t x_187; +x_186 = lean_ctor_get(x_185, 0); +lean_inc(x_186); +x_187 = lean_unbox(x_186); +lean_dec(x_186); +if (x_187 == 0) +{ +lean_object* x_188; +lean_dec(x_180); +lean_dec(x_178); +x_188 = lean_ctor_get(x_185, 1); +lean_inc(x_188); +lean_dec(x_185); +lean_ctor_set(x_1, 1, x_3); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_188; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +else +{ +uint8_t x_190; +x_190 = !lean_is_exclusive(x_2); +if (x_190 == 0) +{ +lean_object* x_191; lean_object* x_192; lean_object* x_193; +x_191 = lean_ctor_get(x_2, 1); +lean_dec(x_191); +x_192 = lean_ctor_get(x_2, 0); +lean_dec(x_192); +x_193 = lean_ctor_get(x_185, 1); +lean_inc(x_193); +lean_dec(x_185); +lean_ctor_set(x_2, 1, x_178); +lean_ctor_set(x_2, 0, x_164); +lean_ctor_set_uint8(x_2, sizeof(void*)*2, x_179); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_193; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} goto _start; } -case 1: +else { -lean_object* x_134; -x_134 = lean_ctor_get(x_129, 1); -lean_inc(x_134); -lean_dec(x_129); +lean_object* x_195; lean_object* x_196; +lean_dec(x_2); +x_195 = lean_ctor_get(x_185, 1); +lean_inc(x_195); +lean_dec(x_185); +x_196 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_196, 0, x_164); +lean_ctor_set(x_196, 1, x_178); +lean_ctor_set_uint8(x_196, sizeof(void*)*2, x_179); lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); { -lean_object* _tmp_0 = x_128; +lean_object* _tmp_0 = x_165; +lean_object* _tmp_1 = x_196; lean_object* _tmp_2 = x_1; -lean_object* _tmp_11 = x_134; +lean_object* _tmp_11 = x_195; x_1 = _tmp_0; +x_2 = _tmp_1; x_3 = _tmp_2; x_12 = _tmp_11; } goto _start; } -default: -{ -if (lean_obj_tag(x_2) == 0) +} +} +else { -lean_object* x_136; lean_object* x_137; +uint8_t x_198; +lean_dec(x_180); +lean_dec(x_178); lean_free_object(x_1); -x_136 = lean_ctor_get(x_129, 1); -lean_inc(x_136); -lean_dec(x_129); -x_137 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_137, 0, x_127); -x_1 = x_128; -x_2 = x_137; -x_12 = x_136; -goto _start; +lean_dec(x_165); +lean_dec(x_164); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_198 = !lean_is_exclusive(x_185); +if (x_198 == 0) +{ +return x_185; } else { -lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_139 = lean_ctor_get(x_129, 1); -lean_inc(x_139); -lean_dec(x_129); -x_140 = lean_ctor_get(x_2, 0); -lean_inc(x_140); -lean_inc(x_127); -x_141 = l_Lean_Meta_Grind_getGeneration(x_127, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_139); -if (lean_obj_tag(x_141) == 0) +lean_object* x_199; lean_object* x_200; lean_object* x_201; +x_199 = lean_ctor_get(x_185, 0); +x_200 = lean_ctor_get(x_185, 1); +lean_inc(x_200); +lean_inc(x_199); +lean_dec(x_185); +x_201 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_201, 0, x_199); +lean_ctor_set(x_201, 1, x_200); +return x_201; +} +} +} +else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_142 = lean_ctor_get(x_141, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_141, 1); -lean_inc(x_143); -lean_dec(x_141); -lean_inc(x_140); -x_144 = l_Lean_Meta_Grind_getGeneration(x_140, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_143); -if (lean_obj_tag(x_144) == 0) +if (x_179 == 0) { -lean_object* x_145; lean_object* x_146; uint8_t x_147; -x_145 = lean_ctor_get(x_144, 0); -lean_inc(x_145); -x_146 = lean_ctor_get(x_144, 1); -lean_inc(x_146); -lean_dec(x_144); -x_147 = lean_nat_dec_lt(x_142, x_145); -lean_dec(x_145); -lean_dec(x_142); -if (x_147 == 0) +uint8_t x_202; +x_202 = lean_nat_dec_lt(x_182, x_181); +if (x_202 == 0) +{ +lean_object* x_203; lean_object* x_204; +x_203 = lean_box(0); +lean_inc(x_180); +lean_inc(x_164); +x_204 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_164, x_180, x_178, x_181, x_203, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_177); +lean_dec(x_181); +if (lean_obj_tag(x_204) == 0) { -lean_dec(x_140); +lean_object* x_205; uint8_t x_206; +x_205 = lean_ctor_get(x_204, 0); +lean_inc(x_205); +x_206 = lean_unbox(x_205); +lean_dec(x_205); +if (x_206 == 0) +{ +lean_object* x_207; +lean_dec(x_180); +lean_dec(x_178); +x_207 = lean_ctor_get(x_204, 1); +lean_inc(x_207); +lean_dec(x_204); lean_ctor_set(x_1, 1, x_3); { -lean_object* _tmp_0 = x_128; +lean_object* _tmp_0 = x_165; lean_object* _tmp_2 = x_1; -lean_object* _tmp_11 = x_146; +lean_object* _tmp_11 = x_207; x_1 = _tmp_0; x_3 = _tmp_2; x_12 = _tmp_11; @@ -2571,20 +3778,27 @@ goto _start; } else { -uint8_t x_149; -x_149 = !lean_is_exclusive(x_2); -if (x_149 == 0) +uint8_t x_209; +x_209 = !lean_is_exclusive(x_2); +if (x_209 == 0) { -lean_object* x_150; -x_150 = lean_ctor_get(x_2, 0); -lean_dec(x_150); -lean_ctor_set(x_2, 0, x_127); +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_2, 1); +lean_dec(x_210); +x_211 = lean_ctor_get(x_2, 0); +lean_dec(x_211); +x_212 = lean_ctor_get(x_204, 1); +lean_inc(x_212); +lean_dec(x_204); +lean_ctor_set(x_2, 1, x_178); +lean_ctor_set(x_2, 0, x_164); +lean_ctor_set_uint8(x_2, sizeof(void*)*2, x_179); lean_ctor_set(x_1, 1, x_3); -lean_ctor_set(x_1, 0, x_140); +lean_ctor_set(x_1, 0, x_180); { -lean_object* _tmp_0 = x_128; +lean_object* _tmp_0 = x_165; lean_object* _tmp_2 = x_1; -lean_object* _tmp_11 = x_146; +lean_object* _tmp_11 = x_212; x_1 = _tmp_0; x_3 = _tmp_2; x_12 = _tmp_11; @@ -2593,17 +3807,22 @@ goto _start; } else { -lean_object* x_152; +lean_object* x_214; lean_object* x_215; lean_dec(x_2); -x_152 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_152, 0, x_127); +x_214 = lean_ctor_get(x_204, 1); +lean_inc(x_214); +lean_dec(x_204); +x_215 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_215, 0, x_164); +lean_ctor_set(x_215, 1, x_178); +lean_ctor_set_uint8(x_215, sizeof(void*)*2, x_179); lean_ctor_set(x_1, 1, x_3); -lean_ctor_set(x_1, 0, x_140); +lean_ctor_set(x_1, 0, x_180); { -lean_object* _tmp_0 = x_128; -lean_object* _tmp_1 = x_152; +lean_object* _tmp_0 = x_165; +lean_object* _tmp_1 = x_215; lean_object* _tmp_2 = x_1; -lean_object* _tmp_11 = x_146; +lean_object* _tmp_11 = x_214; x_1 = _tmp_0; x_2 = _tmp_1; x_3 = _tmp_2; @@ -2615,12 +3834,12 @@ goto _start; } else { -uint8_t x_154; -lean_dec(x_142); -lean_dec(x_140); +uint8_t x_217; +lean_dec(x_180); +lean_dec(x_178); lean_free_object(x_1); -lean_dec(x_128); -lean_dec(x_127); +lean_dec(x_165); +lean_dec(x_164); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2631,33 +3850,175 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_154 = !lean_is_exclusive(x_144); -if (x_154 == 0) +x_217 = !lean_is_exclusive(x_204); +if (x_217 == 0) { -return x_144; +return x_204; } else { -lean_object* x_155; lean_object* x_156; lean_object* x_157; -x_155 = lean_ctor_get(x_144, 0); -x_156 = lean_ctor_get(x_144, 1); -lean_inc(x_156); -lean_inc(x_155); -lean_dec(x_144); -x_157 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_157, 0, x_155); -lean_ctor_set(x_157, 1, x_156); -return x_157; +lean_object* x_218; lean_object* x_219; lean_object* x_220; +x_218 = lean_ctor_get(x_204, 0); +x_219 = lean_ctor_get(x_204, 1); +lean_inc(x_219); +lean_inc(x_218); +lean_dec(x_204); +x_220 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_220, 0, x_218); +lean_ctor_set(x_220, 1, x_219); +return x_220; +} +} +} +else +{ +uint8_t x_221; +lean_dec(x_181); +x_221 = !lean_is_exclusive(x_2); +if (x_221 == 0) +{ +lean_object* x_222; lean_object* x_223; +x_222 = lean_ctor_get(x_2, 1); +lean_dec(x_222); +x_223 = lean_ctor_get(x_2, 0); +lean_dec(x_223); +lean_ctor_set(x_2, 1, x_178); +lean_ctor_set(x_2, 0, x_164); +lean_ctor_set_uint8(x_2, sizeof(void*)*2, x_179); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_177; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +else +{ +lean_object* x_225; +lean_dec(x_2); +x_225 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_225, 0, x_164); +lean_ctor_set(x_225, 1, x_178); +lean_ctor_set_uint8(x_225, sizeof(void*)*2, x_179); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_1 = x_225; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_177; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +} +} +else +{ +lean_object* x_227; lean_object* x_228; +x_227 = lean_box(0); +lean_inc(x_180); +lean_inc(x_164); +x_228 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_164, x_180, x_178, x_181, x_227, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_177); +lean_dec(x_181); +if (lean_obj_tag(x_228) == 0) +{ +lean_object* x_229; uint8_t x_230; +x_229 = lean_ctor_get(x_228, 0); +lean_inc(x_229); +x_230 = lean_unbox(x_229); +lean_dec(x_229); +if (x_230 == 0) +{ +lean_object* x_231; +lean_dec(x_180); +lean_dec(x_178); +x_231 = lean_ctor_get(x_228, 1); +lean_inc(x_231); +lean_dec(x_228); +lean_ctor_set(x_1, 1, x_3); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_231; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +else +{ +uint8_t x_233; +x_233 = !lean_is_exclusive(x_2); +if (x_233 == 0) +{ +lean_object* x_234; lean_object* x_235; lean_object* x_236; +x_234 = lean_ctor_get(x_2, 1); +lean_dec(x_234); +x_235 = lean_ctor_get(x_2, 0); +lean_dec(x_235); +x_236 = lean_ctor_get(x_228, 1); +lean_inc(x_236); +lean_dec(x_228); +lean_ctor_set(x_2, 1, x_178); +lean_ctor_set(x_2, 0, x_164); +lean_ctor_set_uint8(x_2, sizeof(void*)*2, x_179); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_236; +x_1 = _tmp_0; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; +} +else +{ +lean_object* x_238; lean_object* x_239; +lean_dec(x_2); +x_238 = lean_ctor_get(x_228, 1); +lean_inc(x_238); +lean_dec(x_228); +x_239 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_239, 0, x_164); +lean_ctor_set(x_239, 1, x_178); +lean_ctor_set_uint8(x_239, sizeof(void*)*2, x_179); +lean_ctor_set(x_1, 1, x_3); +lean_ctor_set(x_1, 0, x_180); +{ +lean_object* _tmp_0 = x_165; +lean_object* _tmp_1 = x_239; +lean_object* _tmp_2 = x_1; +lean_object* _tmp_11 = x_238; +x_1 = _tmp_0; +x_2 = _tmp_1; +x_3 = _tmp_2; +x_12 = _tmp_11; +} +goto _start; } } } else { -uint8_t x_158; -lean_dec(x_140); +uint8_t x_241; +lean_dec(x_180); +lean_dec(x_178); lean_free_object(x_1); -lean_dec(x_128); -lean_dec(x_127); +lean_dec(x_165); +lean_dec(x_164); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2668,23 +4029,25 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_158 = !lean_is_exclusive(x_141); -if (x_158 == 0) +x_241 = !lean_is_exclusive(x_228); +if (x_241 == 0) { -return x_141; +return x_228; } else { -lean_object* x_159; lean_object* x_160; lean_object* x_161; -x_159 = lean_ctor_get(x_141, 0); -x_160 = lean_ctor_get(x_141, 1); -lean_inc(x_160); -lean_inc(x_159); -lean_dec(x_141); -x_161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_161, 0, x_159); -lean_ctor_set(x_161, 1, x_160); -return x_161; +lean_object* x_242; lean_object* x_243; lean_object* x_244; +x_242 = lean_ctor_get(x_228, 0); +x_243 = lean_ctor_get(x_228, 1); +lean_inc(x_243); +lean_inc(x_242); +lean_dec(x_228); +x_244 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_244, 0, x_242); +lean_ctor_set(x_244, 1, x_243); +return x_244; +} +} } } } @@ -2693,10 +4056,10 @@ return x_161; } else { -uint8_t x_162; +uint8_t x_245; lean_free_object(x_1); -lean_dec(x_128); -lean_dec(x_127); +lean_dec(x_165); +lean_dec(x_164); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2707,33 +4070,33 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_162 = !lean_is_exclusive(x_129); -if (x_162 == 0) +x_245 = !lean_is_exclusive(x_166); +if (x_245 == 0) { -return x_129; +return x_166; } else { -lean_object* x_163; lean_object* x_164; lean_object* x_165; -x_163 = lean_ctor_get(x_129, 0); -x_164 = lean_ctor_get(x_129, 1); -lean_inc(x_164); -lean_inc(x_163); -lean_dec(x_129); -x_165 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_165, 0, x_163); -lean_ctor_set(x_165, 1, x_164); -return x_165; +lean_object* x_246; lean_object* x_247; lean_object* x_248; +x_246 = lean_ctor_get(x_166, 0); +x_247 = lean_ctor_get(x_166, 1); +lean_inc(x_247); +lean_inc(x_246); +lean_dec(x_166); +x_248 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_248, 0, x_246); +lean_ctor_set(x_248, 1, x_247); +return x_248; } } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; -x_166 = lean_ctor_get(x_1, 0); -x_167 = lean_ctor_get(x_1, 1); -lean_inc(x_167); -lean_inc(x_166); +lean_object* x_249; lean_object* x_250; lean_object* x_251; +x_249 = lean_ctor_get(x_1, 0); +x_250 = lean_ctor_get(x_1, 1); +lean_inc(x_250); +lean_inc(x_249); lean_dec(x_1); lean_inc(x_11); lean_inc(x_10); @@ -2743,132 +4106,254 @@ lean_inc(x_7); lean_inc(x_6); lean_inc(x_5); lean_inc(x_4); -lean_inc(x_166); -x_168 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(x_166, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_168) == 0) -{ -lean_object* x_169; uint8_t x_170; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -x_170 = lean_unbox(x_169); -lean_dec(x_169); -switch (x_170) { +lean_inc(x_249); +x_251 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus(x_249, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_251) == 0) +{ +lean_object* x_252; +x_252 = lean_ctor_get(x_251, 0); +lean_inc(x_252); +switch (lean_obj_tag(x_252)) { case 0: { -lean_object* x_171; -lean_dec(x_166); -x_171 = lean_ctor_get(x_168, 1); -lean_inc(x_171); -lean_dec(x_168); -x_1 = x_167; -x_12 = x_171; +lean_object* x_253; +lean_dec(x_249); +x_253 = lean_ctor_get(x_251, 1); +lean_inc(x_253); +lean_dec(x_251); +x_1 = x_250; +x_12 = x_253; goto _start; } case 1: { -lean_object* x_173; lean_object* x_174; -x_173 = lean_ctor_get(x_168, 1); -lean_inc(x_173); -lean_dec(x_168); -x_174 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_174, 0, x_166); -lean_ctor_set(x_174, 1, x_3); -x_1 = x_167; -x_3 = x_174; -x_12 = x_173; +lean_object* x_255; lean_object* x_256; +x_255 = lean_ctor_get(x_251, 1); +lean_inc(x_255); +lean_dec(x_251); +x_256 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_256, 0, x_249); +lean_ctor_set(x_256, 1, x_3); +x_1 = x_250; +x_3 = x_256; +x_12 = x_255; goto _start; } default: { if (lean_obj_tag(x_2) == 0) { -lean_object* x_176; lean_object* x_177; -x_176 = lean_ctor_get(x_168, 1); -lean_inc(x_176); -lean_dec(x_168); -x_177 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_177, 0, x_166); -x_1 = x_167; -x_2 = x_177; -x_12 = x_176; +lean_object* x_258; lean_object* x_259; uint8_t x_260; lean_object* x_261; +x_258 = lean_ctor_get(x_251, 1); +lean_inc(x_258); +lean_dec(x_251); +x_259 = lean_ctor_get(x_252, 0); +lean_inc(x_259); +x_260 = lean_ctor_get_uint8(x_252, sizeof(void*)*1); +lean_dec(x_252); +x_261 = lean_alloc_ctor(1, 2, 1); +lean_ctor_set(x_261, 0, x_249); +lean_ctor_set(x_261, 1, x_259); +lean_ctor_set_uint8(x_261, sizeof(void*)*2, x_260); +x_1 = x_250; +x_2 = x_261; +x_12 = x_258; goto _start; } else { -lean_object* x_179; lean_object* x_180; lean_object* x_181; -x_179 = lean_ctor_get(x_168, 1); -lean_inc(x_179); -lean_dec(x_168); -x_180 = lean_ctor_get(x_2, 0); -lean_inc(x_180); -lean_inc(x_166); -x_181 = l_Lean_Meta_Grind_getGeneration(x_166, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_179); -if (lean_obj_tag(x_181) == 0) -{ -lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_182 = lean_ctor_get(x_181, 0); -lean_inc(x_182); -x_183 = lean_ctor_get(x_181, 1); -lean_inc(x_183); -lean_dec(x_181); -lean_inc(x_180); -x_184 = l_Lean_Meta_Grind_getGeneration(x_180, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_183); -if (lean_obj_tag(x_184) == 0) +lean_object* x_263; lean_object* x_264; uint8_t x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; uint8_t x_269; +x_263 = lean_ctor_get(x_251, 1); +lean_inc(x_263); +lean_dec(x_251); +x_264 = lean_ctor_get(x_252, 0); +lean_inc(x_264); +x_265 = lean_ctor_get_uint8(x_252, sizeof(void*)*1); +lean_dec(x_252); +x_266 = lean_ctor_get(x_2, 0); +lean_inc(x_266); +x_267 = lean_ctor_get(x_2, 1); +lean_inc(x_267); +x_268 = lean_unsigned_to_nat(1u); +x_269 = lean_nat_dec_eq(x_264, x_268); +if (x_269 == 0) +{ +lean_object* x_270; lean_object* x_271; +x_270 = lean_box(0); +lean_inc(x_266); +lean_inc(x_249); +x_271 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_249, x_266, x_264, x_267, x_270, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_263); +lean_dec(x_267); +if (lean_obj_tag(x_271) == 0) +{ +lean_object* x_272; uint8_t x_273; +x_272 = lean_ctor_get(x_271, 0); +lean_inc(x_272); +x_273 = lean_unbox(x_272); +lean_dec(x_272); +if (x_273 == 0) +{ +lean_object* x_274; lean_object* x_275; +lean_dec(x_266); +lean_dec(x_264); +x_274 = lean_ctor_get(x_271, 1); +lean_inc(x_274); +lean_dec(x_271); +x_275 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_275, 0, x_249); +lean_ctor_set(x_275, 1, x_3); +x_1 = x_250; +x_3 = x_275; +x_12 = x_274; +goto _start; +} +else { -lean_object* x_185; lean_object* x_186; uint8_t x_187; -x_185 = lean_ctor_get(x_184, 0); -lean_inc(x_185); -x_186 = lean_ctor_get(x_184, 1); -lean_inc(x_186); -lean_dec(x_184); -x_187 = lean_nat_dec_lt(x_182, x_185); -lean_dec(x_185); -lean_dec(x_182); -if (x_187 == 0) +lean_object* x_277; lean_object* x_278; lean_object* x_279; lean_object* x_280; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + lean_ctor_release(x_2, 1); + x_277 = x_2; +} else { + lean_dec_ref(x_2); + x_277 = lean_box(0); +} +x_278 = lean_ctor_get(x_271, 1); +lean_inc(x_278); +lean_dec(x_271); +if (lean_is_scalar(x_277)) { + x_279 = lean_alloc_ctor(1, 2, 1); +} else { + x_279 = x_277; +} +lean_ctor_set(x_279, 0, x_249); +lean_ctor_set(x_279, 1, x_264); +lean_ctor_set_uint8(x_279, sizeof(void*)*2, x_265); +x_280 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_280, 0, x_266); +lean_ctor_set(x_280, 1, x_3); +x_1 = x_250; +x_2 = x_279; +x_3 = x_280; +x_12 = x_278; +goto _start; +} +} +else { -lean_object* x_188; -lean_dec(x_180); -x_188 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_188, 0, x_166); -lean_ctor_set(x_188, 1, x_3); -x_1 = x_167; -x_3 = x_188; -x_12 = x_186; +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_266); +lean_dec(x_264); +lean_dec(x_250); +lean_dec(x_249); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_282 = lean_ctor_get(x_271, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_271, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_271)) { + lean_ctor_release(x_271, 0); + lean_ctor_release(x_271, 1); + x_284 = x_271; +} else { + lean_dec_ref(x_271); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +if (x_265 == 0) +{ +uint8_t x_286; +x_286 = lean_nat_dec_lt(x_268, x_267); +if (x_286 == 0) +{ +lean_object* x_287; lean_object* x_288; +x_287 = lean_box(0); +lean_inc(x_266); +lean_inc(x_249); +x_288 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_249, x_266, x_264, x_267, x_287, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_263); +lean_dec(x_267); +if (lean_obj_tag(x_288) == 0) +{ +lean_object* x_289; uint8_t x_290; +x_289 = lean_ctor_get(x_288, 0); +lean_inc(x_289); +x_290 = lean_unbox(x_289); +lean_dec(x_289); +if (x_290 == 0) +{ +lean_object* x_291; lean_object* x_292; +lean_dec(x_266); +lean_dec(x_264); +x_291 = lean_ctor_get(x_288, 1); +lean_inc(x_291); +lean_dec(x_288); +x_292 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_292, 0, x_249); +lean_ctor_set(x_292, 1, x_3); +x_1 = x_250; +x_3 = x_292; +x_12 = x_291; goto _start; } else { -lean_object* x_190; lean_object* x_191; lean_object* x_192; +lean_object* x_294; lean_object* x_295; lean_object* x_296; lean_object* x_297; if (lean_is_exclusive(x_2)) { lean_ctor_release(x_2, 0); - x_190 = x_2; + lean_ctor_release(x_2, 1); + x_294 = x_2; } else { lean_dec_ref(x_2); - x_190 = lean_box(0); + x_294 = lean_box(0); } -if (lean_is_scalar(x_190)) { - x_191 = lean_alloc_ctor(1, 1, 0); +x_295 = lean_ctor_get(x_288, 1); +lean_inc(x_295); +lean_dec(x_288); +if (lean_is_scalar(x_294)) { + x_296 = lean_alloc_ctor(1, 2, 1); } else { - x_191 = x_190; -} -lean_ctor_set(x_191, 0, x_166); -x_192 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_192, 0, x_180); -lean_ctor_set(x_192, 1, x_3); -x_1 = x_167; -x_2 = x_191; -x_3 = x_192; -x_12 = x_186; + x_296 = x_294; +} +lean_ctor_set(x_296, 0, x_249); +lean_ctor_set(x_296, 1, x_264); +lean_ctor_set_uint8(x_296, sizeof(void*)*2, x_265); +x_297 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_297, 0, x_266); +lean_ctor_set(x_297, 1, x_3); +x_1 = x_250; +x_2 = x_296; +x_3 = x_297; +x_12 = x_295; goto _start; } } else { -lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; -lean_dec(x_182); -lean_dec(x_180); -lean_dec(x_167); -lean_dec(x_166); +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_266); +lean_dec(x_264); +lean_dec(x_250); +lean_dec(x_249); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2879,34 +4364,128 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_194 = lean_ctor_get(x_184, 0); -lean_inc(x_194); -x_195 = lean_ctor_get(x_184, 1); -lean_inc(x_195); -if (lean_is_exclusive(x_184)) { - lean_ctor_release(x_184, 0); - lean_ctor_release(x_184, 1); - x_196 = x_184; +x_299 = lean_ctor_get(x_288, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_288, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_288)) { + lean_ctor_release(x_288, 0); + lean_ctor_release(x_288, 1); + x_301 = x_288; } else { - lean_dec_ref(x_184); - x_196 = lean_box(0); + lean_dec_ref(x_288); + x_301 = lean_box(0); } -if (lean_is_scalar(x_196)) { - x_197 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); } else { - x_197 = x_196; + x_302 = x_301; } -lean_ctor_set(x_197, 0, x_194); -lean_ctor_set(x_197, 1, x_195); -return x_197; +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; } } else { -lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; -lean_dec(x_180); -lean_dec(x_167); -lean_dec(x_166); +lean_object* x_303; lean_object* x_304; lean_object* x_305; +lean_dec(x_267); +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + lean_ctor_release(x_2, 1); + x_303 = x_2; +} else { + lean_dec_ref(x_2); + x_303 = lean_box(0); +} +if (lean_is_scalar(x_303)) { + x_304 = lean_alloc_ctor(1, 2, 1); +} else { + x_304 = x_303; +} +lean_ctor_set(x_304, 0, x_249); +lean_ctor_set(x_304, 1, x_264); +lean_ctor_set_uint8(x_304, sizeof(void*)*2, x_265); +x_305 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_305, 0, x_266); +lean_ctor_set(x_305, 1, x_3); +x_1 = x_250; +x_2 = x_304; +x_3 = x_305; +x_12 = x_263; +goto _start; +} +} +else +{ +lean_object* x_307; lean_object* x_308; +x_307 = lean_box(0); +lean_inc(x_266); +lean_inc(x_249); +x_308 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_249, x_266, x_264, x_267, x_307, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_263); +lean_dec(x_267); +if (lean_obj_tag(x_308) == 0) +{ +lean_object* x_309; uint8_t x_310; +x_309 = lean_ctor_get(x_308, 0); +lean_inc(x_309); +x_310 = lean_unbox(x_309); +lean_dec(x_309); +if (x_310 == 0) +{ +lean_object* x_311; lean_object* x_312; +lean_dec(x_266); +lean_dec(x_264); +x_311 = lean_ctor_get(x_308, 1); +lean_inc(x_311); +lean_dec(x_308); +x_312 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_312, 0, x_249); +lean_ctor_set(x_312, 1, x_3); +x_1 = x_250; +x_3 = x_312; +x_12 = x_311; +goto _start; +} +else +{ +lean_object* x_314; lean_object* x_315; lean_object* x_316; lean_object* x_317; +if (lean_is_exclusive(x_2)) { + lean_ctor_release(x_2, 0); + lean_ctor_release(x_2, 1); + x_314 = x_2; +} else { + lean_dec_ref(x_2); + x_314 = lean_box(0); +} +x_315 = lean_ctor_get(x_308, 1); +lean_inc(x_315); +lean_dec(x_308); +if (lean_is_scalar(x_314)) { + x_316 = lean_alloc_ctor(1, 2, 1); +} else { + x_316 = x_314; +} +lean_ctor_set(x_316, 0, x_249); +lean_ctor_set(x_316, 1, x_264); +lean_ctor_set_uint8(x_316, sizeof(void*)*2, x_265); +x_317 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_317, 0, x_266); +lean_ctor_set(x_317, 1, x_3); +x_1 = x_250; +x_2 = x_316; +x_3 = x_317; +x_12 = x_315; +goto _start; +} +} +else +{ +lean_object* x_319; lean_object* x_320; lean_object* x_321; lean_object* x_322; +lean_dec(x_266); +lean_dec(x_264); +lean_dec(x_250); +lean_dec(x_249); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2917,26 +4496,28 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_198 = lean_ctor_get(x_181, 0); -lean_inc(x_198); -x_199 = lean_ctor_get(x_181, 1); -lean_inc(x_199); -if (lean_is_exclusive(x_181)) { - lean_ctor_release(x_181, 0); - lean_ctor_release(x_181, 1); - x_200 = x_181; +x_319 = lean_ctor_get(x_308, 0); +lean_inc(x_319); +x_320 = lean_ctor_get(x_308, 1); +lean_inc(x_320); +if (lean_is_exclusive(x_308)) { + lean_ctor_release(x_308, 0); + lean_ctor_release(x_308, 1); + x_321 = x_308; } else { - lean_dec_ref(x_181); - x_200 = lean_box(0); + lean_dec_ref(x_308); + x_321 = lean_box(0); } -if (lean_is_scalar(x_200)) { - x_201 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_321)) { + x_322 = lean_alloc_ctor(1, 2, 0); } else { - x_201 = x_200; + x_322 = x_321; +} +lean_ctor_set(x_322, 0, x_319); +lean_ctor_set(x_322, 1, x_320); +return x_322; +} } -lean_ctor_set(x_201, 0, x_198); -lean_ctor_set(x_201, 1, x_199); -return x_201; } } } @@ -2944,9 +4525,66 @@ return x_201; } else { -lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; -lean_dec(x_167); -lean_dec(x_166); +lean_object* x_323; lean_object* x_324; lean_object* x_325; lean_object* x_326; +lean_dec(x_250); +lean_dec(x_249); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_323 = lean_ctor_get(x_251, 0); +lean_inc(x_323); +x_324 = lean_ctor_get(x_251, 1); +lean_inc(x_324); +if (lean_is_exclusive(x_251)) { + lean_ctor_release(x_251, 0); + lean_ctor_release(x_251, 1); + x_325 = x_251; +} else { + lean_dec_ref(x_251); + x_325 = lean_box(0); +} +if (lean_is_scalar(x_325)) { + x_326 = lean_alloc_ctor(1, 2, 0); +} else { + x_326 = x_325; +} +lean_ctor_set(x_326, 0, x_323); +lean_ctor_set(x_326, 1, x_324); +return x_326; +} +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_12; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +x_13 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); @@ -2957,36 +4595,18 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -x_202 = lean_ctor_get(x_168, 0); -lean_inc(x_202); -x_203 = lean_ctor_get(x_168, 1); -lean_inc(x_203); -if (lean_is_exclusive(x_168)) { - lean_ctor_release(x_168, 0); - lean_ctor_release(x_168, 1); - x_204 = x_168; -} else { - lean_dec_ref(x_168); - x_204 = lean_box(0); -} -if (lean_is_scalar(x_204)) { - x_205 = lean_alloc_ctor(1, 2, 0); -} else { - x_205 = x_204; -} -lean_ctor_set(x_205, 0, x_202); -lean_ctor_set(x_205, 1, x_203); -return x_205; -} -} -} +lean_dec(x_1); +return x_13; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14) { _start: { -lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_object* x_15; +x_15 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); @@ -2995,8 +4615,7 @@ lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_12; +return x_15; } } LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -3009,12 +4628,12 @@ lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = lean_ctor_get(x_12, 16); +x_14 = lean_ctor_get(x_12, 18); lean_inc(x_14); lean_dec(x_12); x_15 = lean_box(0); x_16 = lean_box(0); -x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go(x_14, x_15, x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f_go(x_14, x_16, x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_17; } } @@ -3048,71 +4667,338 @@ return x_17; } else { -uint8_t x_18; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); +uint8_t x_18; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_18 = !lean_is_exclusive(x_11); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_11, 0); +lean_dec(x_19); +x_20 = lean_box(0); +lean_ctor_set(x_11, 0, x_20); +return x_11; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_11, 1); +lean_inc(x_21); +lean_dec(x_11); +x_22 = lean_box(0); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_21); +return x_23; +} +} +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___boxed), 10, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1; +x_15 = lean_box(0); +x_16 = lean_apply_10(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); +return x_16; +} +else +{ +uint8_t x_17; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_17 = !lean_is_exclusive(x_10); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_10, 0); +lean_dec(x_18); +x_19 = lean_box(0); +lean_ctor_set(x_10, 0, x_19); +return x_10; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_10, 1); +lean_inc(x_20); +lean_dec(x_10); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_1); +return x_11; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Grind", 5, 5); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_eq_eq_false", 14, 14); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("of_eq_eq_true", 13, 13); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6; +x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); +return x_4; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7; +x_3 = l_Lean_Expr_const___override(x_2, x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; +lean_inc(x_1); +x_13 = l_Lean_Meta_Grind_isEqTrue(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +if (lean_obj_tag(x_13) == 0) +{ +lean_object* x_14; uint8_t x_15; +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_unbox(x_14); +lean_dec(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_dec(x_13); +x_17 = l_Lean_Meta_Grind_mkEqFalseProof(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_16); +if (lean_obj_tag(x_17) == 0) +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_17, 0); +x_20 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5; +x_21 = l_Lean_mkApp3(x_20, x_2, x_3, x_19); +lean_ctor_set(x_17, 0, x_21); +return x_17; +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_22 = lean_ctor_get(x_17, 0); +x_23 = lean_ctor_get(x_17, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_17); +x_24 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5; +x_25 = l_Lean_mkApp3(x_24, x_2, x_3, x_22); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_23); +return x_26; +} +} +else +{ +uint8_t x_27; +lean_dec(x_3); +lean_dec(x_2); +x_27 = !lean_is_exclusive(x_17); +if (x_27 == 0) +{ +return x_17; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_17, 0); +x_29 = lean_ctor_get(x_17, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_17); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +else +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_13, 1); +lean_inc(x_31); +lean_dec(x_13); +x_32 = l_Lean_Meta_Grind_mkEqTrueProof(x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_31); +if (lean_obj_tag(x_32) == 0) +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_32); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_32, 0); +x_35 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8; +x_36 = l_Lean_mkApp3(x_35, x_2, x_3, x_34); +lean_ctor_set(x_32, 0, x_36); +return x_32; +} +else +{ +lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_37 = lean_ctor_get(x_32, 0); +x_38 = lean_ctor_get(x_32, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_32); +x_39 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8; +x_40 = l_Lean_mkApp3(x_39, x_2, x_3, x_37); +x_41 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_41, 0, x_40); +lean_ctor_set(x_41, 1, x_38); +return x_41; +} +} +else +{ +uint8_t x_42; lean_dec(x_3); lean_dec(x_2); -x_18 = !lean_is_exclusive(x_11); -if (x_18 == 0) +x_42 = !lean_is_exclusive(x_32); +if (x_42 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_11, 0); -lean_dec(x_19); -x_20 = lean_box(0); -lean_ctor_set(x_11, 0, x_20); -return x_11; +return x_32; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_11, 1); -lean_inc(x_21); -lean_dec(x_11); -x_22 = lean_box(0); -x_23 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; -} -} +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_32, 0); +x_44 = lean_ctor_get(x_32, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_32); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___boxed), 10, 0); -return x_1; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_unbox(x_11); +uint8_t x_46; lean_dec(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); lean_dec(x_10); -x_14 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1; -x_15 = lean_box(0); -x_16 = lean_apply_10(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -return x_16; -} -else -{ -uint8_t x_17; +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -3121,50 +5007,28 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_17 = !lean_is_exclusive(x_10); -if (x_17 == 0) +x_46 = !lean_is_exclusive(x_13); +if (x_46 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_10, 0); -lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_10, 0, x_19); -return x_10; +return x_13; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_10, 1); -lean_inc(x_20); -lean_dec(x_10); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; -} -} -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_ctor_get(x_13, 0); +x_48 = lean_ctor_get(x_13, 1); +lean_inc(x_48); +lean_inc(x_47); +lean_dec(x_13); +x_49 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_49, 0, x_47); +lean_ctor_set(x_49, 1, x_48); +return x_49; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; @@ -3175,23 +5039,7 @@ lean_ctor_set(x_12, 1, x_10); return x_12; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Lean", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("Grind", 5, 5); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1() { _start: { lean_object* x_1; @@ -3199,28 +5047,28 @@ x_1 = lean_mk_string_unchecked("or_of_and_eq_false", 18, 18); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2; -x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2; +x_3 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2; x_3 = l_Lean_Expr_const___override(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; @@ -3233,7 +5081,7 @@ if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; x_15 = lean_ctor_get(x_13, 0); -x_16 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5; +x_16 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3; x_17 = l_Lean_mkApp3(x_16, x_2, x_3, x_15); lean_ctor_set(x_13, 0, x_17); return x_13; @@ -3246,7 +5094,7 @@ x_19 = lean_ctor_get(x_13, 1); lean_inc(x_19); lean_inc(x_18); lean_dec(x_13); -x_20 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5; +x_20 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3; x_21 = l_Lean_mkApp3(x_20, x_2, x_3, x_18); x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_21); @@ -3280,35 +5128,7 @@ return x_26; } } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("of_eq_true", 10, 10); -return x_1; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2; -x_3 = l_Lean_Expr_const___override(x_2, x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; @@ -3320,50 +5140,48 @@ uint8_t x_13; x_13 = !lean_is_exclusive(x_12); if (x_13 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_14; lean_object* x_15; x_14 = lean_ctor_get(x_12, 0); -x_15 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3; -x_16 = l_Lean_mkAppB(x_15, x_1, x_14); -lean_ctor_set(x_12, 0, x_16); +x_15 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_14); +lean_ctor_set(x_12, 0, x_15); return x_12; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_17 = lean_ctor_get(x_12, 0); -x_18 = lean_ctor_get(x_12, 1); -lean_inc(x_18); +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_16 = lean_ctor_get(x_12, 0); +x_17 = lean_ctor_get(x_12, 1); lean_inc(x_17); +lean_inc(x_16); lean_dec(x_12); -x_19 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__3; -x_20 = l_Lean_mkAppB(x_19, x_1, x_17); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_18); -return x_21; +x_18 = l_Lean_Meta_mkOfEqTrueCore(x_1, x_16); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_17); +return x_19; } } else { -uint8_t x_22; +uint8_t x_20; lean_dec(x_1); -x_22 = !lean_is_exclusive(x_12); -if (x_22 == 0) +x_20 = !lean_is_exclusive(x_12); +if (x_20 == 0) { return x_12; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_12, 0); -x_24 = lean_ctor_get(x_12, 1); -lean_inc(x_24); -lean_inc(x_23); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_12, 0); +x_22 = lean_ctor_get(x_12, 1); +lean_inc(x_22); +lean_inc(x_21); lean_dec(x_12); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; +x_23 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_23, 0, x_21); +lean_ctor_set(x_23, 1, x_22); +return x_23; } } } @@ -3372,7 +5190,7 @@ static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_ _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___boxed), 10, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___boxed), 10, 0); return x_1; } } @@ -3395,7 +5213,7 @@ if (x_16 == 0) lean_object* x_17; lean_object* x_18; lean_dec(x_15); x_17 = lean_box(0); -x_18 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_18 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_18; } else @@ -3410,7 +5228,7 @@ lean_object* x_22; lean_object* x_23; lean_dec(x_20); lean_dec(x_19); x_22 = lean_box(0); -x_23 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_23 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_22, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_23; } else @@ -3423,101 +5241,116 @@ x_27 = l_Lean_Expr_isConstOf(x_25, x_26); if (x_27 == 0) { uint8_t x_28; -lean_dec(x_24); -lean_dec(x_19); x_28 = l_Lean_Expr_isApp(x_25); if (x_28 == 0) { lean_object* x_29; lean_object* x_30; lean_dec(x_25); +lean_dec(x_24); +lean_dec(x_19); x_29 = lean_box(0); -x_30 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_30 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_29, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); return x_30; } else { -lean_object* x_31; uint8_t x_32; +lean_object* x_31; lean_object* x_32; uint8_t x_33; x_31 = l_Lean_Expr_appFnCleanup(x_25, lean_box(0)); -x_32 = l_Lean_Expr_isApp(x_31); -if (x_32 == 0) +x_32 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__7; +x_33 = l_Lean_Expr_isConstOf(x_31, x_32); +if (x_33 == 0) { -lean_object* x_33; lean_object* x_34; +uint8_t x_34; +lean_dec(x_24); +lean_dec(x_19); +x_34 = l_Lean_Expr_isApp(x_31); +if (x_34 == 0) +{ +lean_object* x_35; lean_object* x_36; lean_dec(x_31); -x_33 = lean_box(0); -x_34 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_33, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_34; +x_35 = lean_box(0); +x_36 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_36; } else { -lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_35 = l_Lean_Expr_appArg(x_31, lean_box(0)); -x_36 = l_Lean_Expr_appFnCleanup(x_31, lean_box(0)); -x_37 = l_Lean_Expr_isApp(x_36); -if (x_37 == 0) +lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_37 = l_Lean_Expr_appArg(x_31, lean_box(0)); +x_38 = l_Lean_Expr_appFnCleanup(x_31, lean_box(0)); +x_39 = l_Lean_Expr_isApp(x_38); +if (x_39 == 0) { -lean_object* x_38; lean_object* x_39; -lean_dec(x_36); -lean_dec(x_35); -x_38 = lean_box(0); -x_39 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_38, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_39; +lean_object* x_40; lean_object* x_41; +lean_dec(x_38); +lean_dec(x_37); +x_40 = lean_box(0); +x_41 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_40, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_41; } else { -lean_object* x_40; lean_object* x_41; uint8_t x_42; -x_40 = l_Lean_Expr_appFnCleanup(x_36, lean_box(0)); -x_41 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__7; -x_42 = l_Lean_Expr_isConstOf(x_40, x_41); -if (x_42 == 0) -{ -lean_object* x_43; uint8_t x_44; +lean_object* x_42; lean_object* x_43; uint8_t x_44; +x_42 = l_Lean_Expr_appFnCleanup(x_38, lean_box(0)); x_43 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9; -x_44 = l_Lean_Expr_isConstOf(x_40, x_43); -lean_dec(x_40); +x_44 = l_Lean_Expr_isConstOf(x_42, x_43); if (x_44 == 0) { -lean_object* x_45; lean_object* x_46; -lean_dec(x_35); -x_45 = lean_box(0); -x_46 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_45, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_46; +lean_object* x_45; uint8_t x_46; +x_45 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11; +x_46 = l_Lean_Expr_isConstOf(x_42, x_45); +lean_dec(x_42); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; +lean_dec(x_37); +x_47 = lean_box(0); +x_48 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_47, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_48; } else { -lean_object* x_47; +lean_object* x_49; lean_dec(x_1); -x_47 = lean_apply_10(x_14, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_47; +x_49 = lean_apply_10(x_14, x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_49; } } else { -lean_object* x_48; -lean_dec(x_40); +lean_object* x_50; +lean_dec(x_42); lean_dec(x_1); -x_48 = lean_apply_10(x_14, x_35, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_48; +x_50 = lean_apply_10(x_14, x_37, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_50; +} } } } +else +{ +lean_object* x_51; +lean_dec(x_31); +x_51 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_51; +} } } else { -lean_object* x_49; +lean_object* x_52; lean_dec(x_25); -x_49 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_49; +x_52 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_24, x_19, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_52; } } } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +x_11 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -3529,11 +5362,11 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { lean_object* x_12; -x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +x_12 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_2); return x_12; } @@ -3639,7 +5472,7 @@ uint8_t x_5; x_5 = !lean_is_exclusive(x_2); if (x_5 == 0) { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; x_6 = lean_ctor_get(x_2, 0); x_7 = lean_ctor_get(x_2, 1); x_8 = lean_ctor_get(x_1, 1); @@ -3647,8 +5480,8 @@ x_9 = lean_ctor_get(x_1, 2); x_10 = lean_ctor_get(x_1, 3); x_11 = lean_ctor_get(x_1, 4); x_12 = lean_ctor_get(x_1, 5); -x_13 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_14 = lean_ctor_get(x_1, 6); +x_13 = lean_ctor_get(x_1, 6); +x_14 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); x_15 = lean_ctor_get(x_1, 7); x_16 = lean_ctor_get(x_1, 8); x_17 = lean_ctor_get(x_1, 9); @@ -3662,6 +5495,12 @@ x_24 = lean_ctor_get(x_1, 16); x_25 = lean_ctor_get(x_1, 17); x_26 = lean_ctor_get(x_1, 18); x_27 = lean_ctor_get(x_1, 19); +x_28 = lean_ctor_get(x_1, 20); +x_29 = lean_ctor_get(x_1, 21); +x_30 = lean_ctor_get(x_1, 22); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); @@ -3675,36 +5514,39 @@ lean_inc(x_18); lean_inc(x_17); lean_inc(x_16); lean_inc(x_15); -lean_inc(x_14); +lean_inc(x_13); lean_inc(x_12); lean_inc(x_11); lean_inc(x_10); lean_inc(x_9); lean_inc(x_8); -x_28 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_8); -lean_ctor_set(x_28, 2, x_9); -lean_ctor_set(x_28, 3, x_10); -lean_ctor_set(x_28, 4, x_11); -lean_ctor_set(x_28, 5, x_12); -lean_ctor_set(x_28, 6, x_14); -lean_ctor_set(x_28, 7, x_15); -lean_ctor_set(x_28, 8, x_16); -lean_ctor_set(x_28, 9, x_17); -lean_ctor_set(x_28, 10, x_18); -lean_ctor_set(x_28, 11, x_19); -lean_ctor_set(x_28, 12, x_20); -lean_ctor_set(x_28, 13, x_21); -lean_ctor_set(x_28, 14, x_22); -lean_ctor_set(x_28, 15, x_23); -lean_ctor_set(x_28, 16, x_24); -lean_ctor_set(x_28, 17, x_25); -lean_ctor_set(x_28, 18, x_26); -lean_ctor_set(x_28, 19, x_27); -lean_ctor_set_uint8(x_28, sizeof(void*)*20, x_13); +x_31 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_31, 0, x_6); +lean_ctor_set(x_31, 1, x_8); +lean_ctor_set(x_31, 2, x_9); +lean_ctor_set(x_31, 3, x_10); +lean_ctor_set(x_31, 4, x_11); +lean_ctor_set(x_31, 5, x_12); +lean_ctor_set(x_31, 6, x_13); +lean_ctor_set(x_31, 7, x_15); +lean_ctor_set(x_31, 8, x_16); +lean_ctor_set(x_31, 9, x_17); +lean_ctor_set(x_31, 10, x_18); +lean_ctor_set(x_31, 11, x_19); +lean_ctor_set(x_31, 12, x_20); +lean_ctor_set(x_31, 13, x_21); +lean_ctor_set(x_31, 14, x_22); +lean_ctor_set(x_31, 15, x_23); +lean_ctor_set(x_31, 16, x_24); +lean_ctor_set(x_31, 17, x_25); +lean_ctor_set(x_31, 18, x_26); +lean_ctor_set(x_31, 19, x_27); +lean_ctor_set(x_31, 20, x_28); +lean_ctor_set(x_31, 21, x_29); +lean_ctor_set(x_31, 22, x_30); +lean_ctor_set_uint8(x_31, sizeof(void*)*23, x_14); lean_ctor_set(x_2, 1, x_3); -lean_ctor_set(x_2, 0, x_28); +lean_ctor_set(x_2, 0, x_31); { lean_object* _tmp_1 = x_7; lean_object* _tmp_2 = x_2; @@ -3715,32 +5557,41 @@ goto _start; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -x_30 = lean_ctor_get(x_2, 0); -x_31 = lean_ctor_get(x_2, 1); -lean_inc(x_31); -lean_inc(x_30); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_33 = lean_ctor_get(x_2, 0); +x_34 = lean_ctor_get(x_2, 1); +lean_inc(x_34); +lean_inc(x_33); lean_dec(x_2); -x_32 = lean_ctor_get(x_1, 1); -x_33 = lean_ctor_get(x_1, 2); -x_34 = lean_ctor_get(x_1, 3); -x_35 = lean_ctor_get(x_1, 4); -x_36 = lean_ctor_get(x_1, 5); -x_37 = lean_ctor_get_uint8(x_1, sizeof(void*)*20); -x_38 = lean_ctor_get(x_1, 6); -x_39 = lean_ctor_get(x_1, 7); -x_40 = lean_ctor_get(x_1, 8); -x_41 = lean_ctor_get(x_1, 9); -x_42 = lean_ctor_get(x_1, 10); -x_43 = lean_ctor_get(x_1, 11); -x_44 = lean_ctor_get(x_1, 12); -x_45 = lean_ctor_get(x_1, 13); -x_46 = lean_ctor_get(x_1, 14); -x_47 = lean_ctor_get(x_1, 15); -x_48 = lean_ctor_get(x_1, 16); -x_49 = lean_ctor_get(x_1, 17); -x_50 = lean_ctor_get(x_1, 18); -x_51 = lean_ctor_get(x_1, 19); +x_35 = lean_ctor_get(x_1, 1); +x_36 = lean_ctor_get(x_1, 2); +x_37 = lean_ctor_get(x_1, 3); +x_38 = lean_ctor_get(x_1, 4); +x_39 = lean_ctor_get(x_1, 5); +x_40 = lean_ctor_get(x_1, 6); +x_41 = lean_ctor_get_uint8(x_1, sizeof(void*)*23); +x_42 = lean_ctor_get(x_1, 7); +x_43 = lean_ctor_get(x_1, 8); +x_44 = lean_ctor_get(x_1, 9); +x_45 = lean_ctor_get(x_1, 10); +x_46 = lean_ctor_get(x_1, 11); +x_47 = lean_ctor_get(x_1, 12); +x_48 = lean_ctor_get(x_1, 13); +x_49 = lean_ctor_get(x_1, 14); +x_50 = lean_ctor_get(x_1, 15); +x_51 = lean_ctor_get(x_1, 16); +x_52 = lean_ctor_get(x_1, 17); +x_53 = lean_ctor_get(x_1, 18); +x_54 = lean_ctor_get(x_1, 19); +x_55 = lean_ctor_get(x_1, 20); +x_56 = lean_ctor_get(x_1, 21); +x_57 = lean_ctor_get(x_1, 22); +lean_inc(x_57); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); @@ -3751,42 +5602,42 @@ lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); -lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); +lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -x_52 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_52, 0, x_30); -lean_ctor_set(x_52, 1, x_32); -lean_ctor_set(x_52, 2, x_33); -lean_ctor_set(x_52, 3, x_34); -lean_ctor_set(x_52, 4, x_35); -lean_ctor_set(x_52, 5, x_36); -lean_ctor_set(x_52, 6, x_38); -lean_ctor_set(x_52, 7, x_39); -lean_ctor_set(x_52, 8, x_40); -lean_ctor_set(x_52, 9, x_41); -lean_ctor_set(x_52, 10, x_42); -lean_ctor_set(x_52, 11, x_43); -lean_ctor_set(x_52, 12, x_44); -lean_ctor_set(x_52, 13, x_45); -lean_ctor_set(x_52, 14, x_46); -lean_ctor_set(x_52, 15, x_47); -lean_ctor_set(x_52, 16, x_48); -lean_ctor_set(x_52, 17, x_49); -lean_ctor_set(x_52, 18, x_50); -lean_ctor_set(x_52, 19, x_51); -lean_ctor_set_uint8(x_52, sizeof(void*)*20, x_37); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_52); -lean_ctor_set(x_53, 1, x_3); -x_2 = x_31; -x_3 = x_53; +x_58 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_58, 0, x_33); +lean_ctor_set(x_58, 1, x_35); +lean_ctor_set(x_58, 2, x_36); +lean_ctor_set(x_58, 3, x_37); +lean_ctor_set(x_58, 4, x_38); +lean_ctor_set(x_58, 5, x_39); +lean_ctor_set(x_58, 6, x_40); +lean_ctor_set(x_58, 7, x_42); +lean_ctor_set(x_58, 8, x_43); +lean_ctor_set(x_58, 9, x_44); +lean_ctor_set(x_58, 10, x_45); +lean_ctor_set(x_58, 11, x_46); +lean_ctor_set(x_58, 12, x_47); +lean_ctor_set(x_58, 13, x_48); +lean_ctor_set(x_58, 14, x_49); +lean_ctor_set(x_58, 15, x_50); +lean_ctor_set(x_58, 16, x_51); +lean_ctor_set(x_58, 17, x_52); +lean_ctor_set(x_58, 18, x_53); +lean_ctor_set(x_58, 19, x_54); +lean_ctor_set(x_58, 20, x_55); +lean_ctor_set(x_58, 21, x_56); +lean_ctor_set(x_58, 22, x_57); +lean_ctor_set_uint8(x_58, sizeof(void*)*23, x_41); +x_59 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_3); +x_2 = x_34; +x_3 = x_59; goto _start; } } @@ -3820,7 +5671,7 @@ return x_14; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_12 = lean_st_ref_get(x_3, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); @@ -3830,58 +5681,56 @@ lean_dec(x_12); x_15 = lean_box(0); x_16 = l_List_mapTR_loop___at_Lean_Meta_Grind_splitNext___spec__1(x_13, x_2, x_15); lean_dec(x_13); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_add(x_1, x_17); -x_19 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_introNewHyp(x_16, x_15, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -if (lean_obj_tag(x_19) == 0) +x_17 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_introNewHyp(x_16, x_15, x_1, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +if (lean_obj_tag(x_17) == 0) { -uint8_t x_20; -x_20 = !lean_is_exclusive(x_19); -if (x_20 == 0) +uint8_t x_18; +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_21; lean_object* x_22; -x_21 = lean_ctor_get(x_19, 0); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_19, 0, x_22); -return x_19; +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_17, 0, x_20); +return x_17; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_19, 0); -x_24 = lean_ctor_get(x_19, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_19); -x_25 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_25, 0, x_23); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_24); -return x_26; +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_17, 0); +x_22 = lean_ctor_get(x_17, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_17); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_21); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; } } else { -uint8_t x_27; -x_27 = !lean_is_exclusive(x_19); -if (x_27 == 0) +uint8_t x_25; +x_25 = !lean_is_exclusive(x_17); +if (x_25 == 0) { -return x_19; +return x_17; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; -x_28 = lean_ctor_get(x_19, 0); -x_29 = lean_ctor_get(x_19, 1); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_19); -x_30 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_30, 0, x_28); -lean_ctor_set(x_30, 1, x_29); -return x_30; +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_17, 0); +x_27 = lean_ctor_get(x_17, 1); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_17); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_26); +lean_ctor_set(x_28, 1, x_27); +return x_28; } } } @@ -3955,6 +5804,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_2); x_28 = !lean_is_exclusive(x_24); if (x_28 == 0) { @@ -3986,6 +5836,7 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_2); x_32 = !lean_is_exclusive(x_17); if (x_32 == 0) { @@ -4049,372 +5900,77 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +lean_dec(x_2); x_45 = !lean_is_exclusive(x_41); if (x_45 == 0) { -return x_41; -} -else -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_41, 0); -x_47 = lean_ctor_get(x_41, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_41); -x_48 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -return x_48; -} -} -} -} -} -static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1; -x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", generation: ", 14, 14); -return x_1; -} -} -static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__3() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; lean_object* x_11; lean_object* x_21; -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -lean_inc(x_1); -x_21 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -if (lean_obj_tag(x_21) == 0) -{ -lean_object* x_22; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -if (lean_obj_tag(x_22) == 0) -{ -lean_object* x_23; lean_object* x_24; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -x_24 = lean_box(0); -x_10 = x_24; -x_11 = x_23; -goto block_20; -} -else -{ -lean_object* x_25; uint8_t x_26; -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_25); -lean_dec(x_21); -x_26 = !lean_is_exclusive(x_22); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; -x_27 = lean_ctor_get(x_22, 0); -lean_inc(x_27); -x_28 = l_Lean_Meta_Grind_getGeneration(x_27, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_25); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); -lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__1; -x_32 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_31, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_30); -x_33 = lean_ctor_get(x_32, 0); -lean_inc(x_33); -x_34 = lean_unbox(x_33); -lean_dec(x_33); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -lean_free_object(x_22); -x_35 = lean_ctor_get(x_32, 1); -lean_inc(x_35); -lean_dec(x_32); -x_36 = lean_box(0); -lean_inc(x_1); -x_37 = l_Lean_Meta_Grind_splitNext___lambda__3(x_27, x_29, x_36, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_35); -lean_dec(x_29); -if (lean_obj_tag(x_37) == 0) -{ -lean_object* x_38; lean_object* x_39; -x_38 = lean_ctor_get(x_37, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_37, 1); -lean_inc(x_39); -lean_dec(x_37); -x_10 = x_38; -x_11 = x_39; -goto block_20; -} -else -{ -uint8_t x_40; -lean_dec(x_1); -x_40 = !lean_is_exclusive(x_37); -if (x_40 == 0) -{ -return x_37; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_37, 0); -x_42 = lean_ctor_get(x_37, 1); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_37); -x_43 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); -return x_43; -} -} -} -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_32); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_32, 1); -x_46 = lean_ctor_get(x_32, 0); -lean_dec(x_46); -x_47 = l_Lean_Meta_Grind_updateLastTag(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_45); -if (lean_obj_tag(x_47) == 0) -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_48 = lean_ctor_get(x_47, 1); -lean_inc(x_48); -lean_dec(x_47); -lean_inc(x_27); -x_49 = l_Lean_MessageData_ofExpr(x_27); -x_50 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; -lean_ctor_set_tag(x_32, 7); -lean_ctor_set(x_32, 1, x_49); -lean_ctor_set(x_32, 0, x_50); -x_51 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__3; -x_52 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_52, 0, x_32); -lean_ctor_set(x_52, 1, x_51); -lean_inc(x_29); -x_53 = l___private_Init_Data_Repr_0__Nat_reprFast(x_29); -lean_ctor_set_tag(x_22, 3); -lean_ctor_set(x_22, 0, x_53); -x_54 = l_Lean_MessageData_ofFormat(x_22); -x_55 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_55, 0, x_52); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_50); -x_57 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_31, x_56, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_48); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_57, 1); -lean_inc(x_59); -lean_dec(x_57); -lean_inc(x_1); -x_60 = l_Lean_Meta_Grind_splitNext___lambda__3(x_27, x_29, x_58, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_59); -lean_dec(x_58); -lean_dec(x_29); -if (lean_obj_tag(x_60) == 0) -{ -lean_object* x_61; lean_object* x_62; -x_61 = lean_ctor_get(x_60, 0); -lean_inc(x_61); -x_62 = lean_ctor_get(x_60, 1); -lean_inc(x_62); -lean_dec(x_60); -x_10 = x_61; -x_11 = x_62; -goto block_20; -} -else -{ -uint8_t x_63; -lean_dec(x_1); -x_63 = !lean_is_exclusive(x_60); -if (x_63 == 0) -{ -return x_60; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_60, 0); -x_65 = lean_ctor_get(x_60, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_60); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; -} -} -} -else -{ -uint8_t x_67; -lean_free_object(x_32); -lean_dec(x_29); -lean_free_object(x_22); -lean_dec(x_27); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_67 = !lean_is_exclusive(x_47); -if (x_67 == 0) -{ -return x_47; +return x_41; } else { -lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_68 = lean_ctor_get(x_47, 0); -x_69 = lean_ctor_get(x_47, 1); -lean_inc(x_69); -lean_inc(x_68); -lean_dec(x_47); -x_70 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_70, 0, x_68); -lean_ctor_set(x_70, 1, x_69); -return x_70; +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_41, 0); +x_47 = lean_ctor_get(x_41, 1); +lean_inc(x_47); +lean_inc(x_46); +lean_dec(x_41); +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } } -else -{ -lean_object* x_71; lean_object* x_72; -x_71 = lean_ctor_get(x_32, 1); -lean_inc(x_71); -lean_dec(x_32); -x_72 = l_Lean_Meta_Grind_updateLastTag(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_71); -if (lean_obj_tag(x_72) == 0) -{ -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -x_73 = lean_ctor_get(x_72, 1); -lean_inc(x_73); -lean_dec(x_72); -lean_inc(x_27); -x_74 = l_Lean_MessageData_ofExpr(x_27); -x_75 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; -x_76 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_74); -x_77 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__3; -x_78 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -lean_inc(x_29); -x_79 = l___private_Init_Data_Repr_0__Nat_reprFast(x_29); -lean_ctor_set_tag(x_22, 3); -lean_ctor_set(x_22, 0, x_79); -x_80 = l_Lean_MessageData_ofFormat(x_22); -x_81 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_81, 0, x_78); -lean_ctor_set(x_81, 1, x_80); -x_82 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_82, 0, x_81); -lean_ctor_set(x_82, 1, x_75); -x_83 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_31, x_82, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_73); -x_84 = lean_ctor_get(x_83, 0); -lean_inc(x_84); -x_85 = lean_ctor_get(x_83, 1); -lean_inc(x_85); -lean_dec(x_83); -lean_inc(x_1); -x_86 = l_Lean_Meta_Grind_splitNext___lambda__3(x_27, x_29, x_84, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_85); -lean_dec(x_84); -lean_dec(x_29); -if (lean_obj_tag(x_86) == 0) +} +} +static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__1() { +_start: { -lean_object* x_87; lean_object* x_88; -x_87 = lean_ctor_get(x_86, 0); -lean_inc(x_87); -x_88 = lean_ctor_get(x_86, 1); -lean_inc(x_88); -lean_dec(x_86); -x_10 = x_87; -x_11 = x_88; -goto block_20; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1; +x_2 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } -else +} +static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__2() { +_start: { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; -lean_dec(x_1); -x_89 = lean_ctor_get(x_86, 0); -lean_inc(x_89); -x_90 = lean_ctor_get(x_86, 1); -lean_inc(x_90); -if (lean_is_exclusive(x_86)) { - lean_ctor_release(x_86, 0); - lean_ctor_release(x_86, 1); - x_91 = x_86; -} else { - lean_dec_ref(x_86); - x_91 = lean_box(0); +lean_object* x_1; +x_1 = lean_mk_string_unchecked(", generation: ", 14, 14); +return x_1; } -if (lean_is_scalar(x_91)) { - x_92 = lean_alloc_ctor(1, 2, 0); -} else { - x_92 = x_91; } -lean_ctor_set(x_92, 0, x_89); -lean_ctor_set(x_92, 1, x_90); -return x_92; +static lean_object* _init_l_Lean_Meta_Grind_splitNext___lambda__4___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; -lean_dec(x_29); -lean_free_object(x_22); -lean_dec(x_27); +lean_object* x_10; lean_object* x_11; lean_object* x_21; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +lean_inc(x_1); +x_21 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +if (lean_obj_tag(x_22) == 0) +{ +lean_object* x_23; lean_object* x_24; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4422,234 +5978,218 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_93 = lean_ctor_get(x_72, 0); -lean_inc(x_93); -x_94 = lean_ctor_get(x_72, 1); -lean_inc(x_94); -if (lean_is_exclusive(x_72)) { - lean_ctor_release(x_72, 0); - lean_ctor_release(x_72, 1); - x_95 = x_72; -} else { - lean_dec_ref(x_72); - x_95 = lean_box(0); -} -if (lean_is_scalar(x_95)) { - x_96 = lean_alloc_ctor(1, 2, 0); -} else { - x_96 = x_95; -} -lean_ctor_set(x_96, 0, x_93); -lean_ctor_set(x_96, 1, x_94); -return x_96; -} -} -} +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +x_24 = lean_box(0); +x_10 = x_24; +x_11 = x_23; +goto block_20; } else { -uint8_t x_97; -lean_free_object(x_22); +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; lean_object* x_29; +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_dec(x_21); +x_26 = lean_ctor_get(x_22, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_22, 1); +lean_inc(x_27); +x_28 = lean_ctor_get_uint8(x_22, sizeof(void*)*2); +lean_dec(x_22); +lean_inc(x_26); +x_29 = l_Lean_Meta_Grind_getGeneration(x_26, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_25); +if (lean_obj_tag(x_29) == 0) +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_73; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_unsigned_to_nat(1u); +x_33 = lean_nat_dec_lt(x_32, x_27); lean_dec(x_27); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_97 = !lean_is_exclusive(x_28); -if (x_97 == 0) +x_34 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__1; +x_73 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_34, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_31); +if (x_33 == 0) { -return x_28; +if (x_28 == 0) +{ +lean_object* x_74; lean_object* x_75; uint8_t x_76; +x_74 = lean_ctor_get(x_73, 0); +lean_inc(x_74); +x_75 = lean_ctor_get(x_73, 1); +lean_inc(x_75); +lean_dec(x_73); +x_76 = lean_unbox(x_74); +lean_dec(x_74); +lean_inc(x_30); +x_35 = x_30; +x_36 = x_76; +x_37 = x_75; +goto block_72; } else { -lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_98 = lean_ctor_get(x_28, 0); -x_99 = lean_ctor_get(x_28, 1); -lean_inc(x_99); -lean_inc(x_98); -lean_dec(x_28); -x_100 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_100, 0, x_98); -lean_ctor_set(x_100, 1, x_99); -return x_100; -} +lean_object* x_77; lean_object* x_78; lean_object* x_79; uint8_t x_80; +x_77 = lean_ctor_get(x_73, 0); +lean_inc(x_77); +x_78 = lean_ctor_get(x_73, 1); +lean_inc(x_78); +lean_dec(x_73); +x_79 = lean_nat_add(x_30, x_32); +x_80 = lean_unbox(x_77); +lean_dec(x_77); +x_35 = x_79; +x_36 = x_80; +x_37 = x_78; +goto block_72; } } else { -lean_object* x_101; lean_object* x_102; -x_101 = lean_ctor_get(x_22, 0); -lean_inc(x_101); -lean_dec(x_22); -lean_inc(x_101); -x_102 = l_Lean_Meta_Grind_getGeneration(x_101, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_25); -if (lean_obj_tag(x_102) == 0) +lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_81 = lean_ctor_get(x_73, 0); +lean_inc(x_81); +x_82 = lean_ctor_get(x_73, 1); +lean_inc(x_82); +lean_dec(x_73); +x_83 = lean_nat_add(x_30, x_32); +x_84 = lean_unbox(x_81); +lean_dec(x_81); +x_35 = x_83; +x_36 = x_84; +x_37 = x_82; +goto block_72; +} +block_72: { -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; -x_103 = lean_ctor_get(x_102, 0); -lean_inc(x_103); -x_104 = lean_ctor_get(x_102, 1); -lean_inc(x_104); -lean_dec(x_102); -x_105 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__1; -x_106 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_105, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_104); -x_107 = lean_ctor_get(x_106, 0); -lean_inc(x_107); -x_108 = lean_unbox(x_107); -lean_dec(x_107); -if (x_108 == 0) +if (x_36 == 0) { -lean_object* x_109; lean_object* x_110; lean_object* x_111; -x_109 = lean_ctor_get(x_106, 1); -lean_inc(x_109); -lean_dec(x_106); -x_110 = lean_box(0); +lean_object* x_38; lean_object* x_39; +lean_dec(x_30); +x_38 = lean_box(0); lean_inc(x_1); -x_111 = l_Lean_Meta_Grind_splitNext___lambda__3(x_101, x_103, x_110, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_109); -lean_dec(x_103); -if (lean_obj_tag(x_111) == 0) +x_39 = l_Lean_Meta_Grind_splitNext___lambda__3(x_26, x_35, x_38, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_37); +if (lean_obj_tag(x_39) == 0) { -lean_object* x_112; lean_object* x_113; -x_112 = lean_ctor_get(x_111, 0); -lean_inc(x_112); -x_113 = lean_ctor_get(x_111, 1); -lean_inc(x_113); -lean_dec(x_111); -x_10 = x_112; -x_11 = x_113; +lean_object* x_40; lean_object* x_41; +x_40 = lean_ctor_get(x_39, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_39, 1); +lean_inc(x_41); +lean_dec(x_39); +x_10 = x_40; +x_11 = x_41; goto block_20; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; +uint8_t x_42; lean_dec(x_1); -x_114 = lean_ctor_get(x_111, 0); -lean_inc(x_114); -x_115 = lean_ctor_get(x_111, 1); -lean_inc(x_115); -if (lean_is_exclusive(x_111)) { - lean_ctor_release(x_111, 0); - lean_ctor_release(x_111, 1); - x_116 = x_111; -} else { - lean_dec_ref(x_111); - x_116 = lean_box(0); +x_42 = !lean_is_exclusive(x_39); +if (x_42 == 0) +{ +return x_39; } -if (lean_is_scalar(x_116)) { - x_117 = lean_alloc_ctor(1, 2, 0); -} else { - x_117 = x_116; +else +{ +lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_43 = lean_ctor_get(x_39, 0); +x_44 = lean_ctor_get(x_39, 1); +lean_inc(x_44); +lean_inc(x_43); +lean_dec(x_39); +x_45 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_45, 0, x_43); +lean_ctor_set(x_45, 1, x_44); +return x_45; } -lean_ctor_set(x_117, 0, x_114); -lean_ctor_set(x_117, 1, x_115); -return x_117; } } else { -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_106, 1); -lean_inc(x_118); -if (lean_is_exclusive(x_106)) { - lean_ctor_release(x_106, 0); - lean_ctor_release(x_106, 1); - x_119 = x_106; -} else { - lean_dec_ref(x_106); - x_119 = lean_box(0); -} -x_120 = l_Lean_Meta_Grind_updateLastTag(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_118); -if (lean_obj_tag(x_120) == 0) +lean_object* x_46; +x_46 = l_Lean_Meta_Grind_updateLastTag(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_37); +if (lean_obj_tag(x_46) == 0) { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_121 = lean_ctor_get(x_120, 1); -lean_inc(x_121); -lean_dec(x_120); -lean_inc(x_101); -x_122 = l_Lean_MessageData_ofExpr(x_101); -x_123 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9; -if (lean_is_scalar(x_119)) { - x_124 = lean_alloc_ctor(7, 2, 0); -} else { - x_124 = x_119; - lean_ctor_set_tag(x_124, 7); -} -lean_ctor_set(x_124, 0, x_123); -lean_ctor_set(x_124, 1, x_122); -x_125 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__3; -x_126 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_126, 0, x_124); -lean_ctor_set(x_126, 1, x_125); -lean_inc(x_103); -x_127 = l___private_Init_Data_Repr_0__Nat_reprFast(x_103); -x_128 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_128, 0, x_127); -x_129 = l_Lean_MessageData_ofFormat(x_128); -x_130 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_130, 0, x_126); -lean_ctor_set(x_130, 1, x_129); -x_131 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_131, 0, x_130); -lean_ctor_set(x_131, 1, x_123); -x_132 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_105, x_131, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_121); -x_133 = lean_ctor_get(x_132, 0); -lean_inc(x_133); -x_134 = lean_ctor_get(x_132, 1); -lean_inc(x_134); -lean_dec(x_132); +lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_47 = lean_ctor_get(x_46, 1); +lean_inc(x_47); +lean_dec(x_46); +lean_inc(x_26); +x_48 = l_Lean_MessageData_ofExpr(x_26); +x_49 = l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_48); +x_51 = l_Lean_Meta_Grind_splitNext___lambda__4___closed__3; +x_52 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_52, 0, x_50); +lean_ctor_set(x_52, 1, x_51); +x_53 = l___private_Init_Data_Repr_0__Nat_reprFast(x_30); +x_54 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_54, 0, x_53); +x_55 = l_Lean_MessageData_ofFormat(x_54); +x_56 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_56, 0, x_52); +lean_ctor_set(x_56, 1, x_55); +x_57 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_57, 0, x_56); +lean_ctor_set(x_57, 1, x_49); +x_58 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_34, x_57, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_47); +x_59 = lean_ctor_get(x_58, 0); +lean_inc(x_59); +x_60 = lean_ctor_get(x_58, 1); +lean_inc(x_60); +lean_dec(x_58); lean_inc(x_1); -x_135 = l_Lean_Meta_Grind_splitNext___lambda__3(x_101, x_103, x_133, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_134); -lean_dec(x_133); -lean_dec(x_103); -if (lean_obj_tag(x_135) == 0) +x_61 = l_Lean_Meta_Grind_splitNext___lambda__3(x_26, x_35, x_59, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_60); +lean_dec(x_59); +if (lean_obj_tag(x_61) == 0) { -lean_object* x_136; lean_object* x_137; -x_136 = lean_ctor_get(x_135, 0); -lean_inc(x_136); -x_137 = lean_ctor_get(x_135, 1); -lean_inc(x_137); -lean_dec(x_135); -x_10 = x_136; -x_11 = x_137; +lean_object* x_62; lean_object* x_63; +x_62 = lean_ctor_get(x_61, 0); +lean_inc(x_62); +x_63 = lean_ctor_get(x_61, 1); +lean_inc(x_63); +lean_dec(x_61); +x_10 = x_62; +x_11 = x_63; goto block_20; } else { -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; +uint8_t x_64; lean_dec(x_1); -x_138 = lean_ctor_get(x_135, 0); -lean_inc(x_138); -x_139 = lean_ctor_get(x_135, 1); -lean_inc(x_139); -if (lean_is_exclusive(x_135)) { - lean_ctor_release(x_135, 0); - lean_ctor_release(x_135, 1); - x_140 = x_135; -} else { - lean_dec_ref(x_135); - x_140 = lean_box(0); +x_64 = !lean_is_exclusive(x_61); +if (x_64 == 0) +{ +return x_61; } -if (lean_is_scalar(x_140)) { - x_141 = lean_alloc_ctor(1, 2, 0); -} else { - x_141 = x_140; +else +{ +lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_65 = lean_ctor_get(x_61, 0); +x_66 = lean_ctor_get(x_61, 1); +lean_inc(x_66); +lean_inc(x_65); +lean_dec(x_61); +x_67 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_67, 0, x_65); +lean_ctor_set(x_67, 1, x_66); +return x_67; } -lean_ctor_set(x_141, 0, x_138); -lean_ctor_set(x_141, 1, x_139); -return x_141; } } else { -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; -lean_dec(x_119); -lean_dec(x_103); -lean_dec(x_101); +uint8_t x_68; +lean_dec(x_35); +lean_dec(x_30); +lean_dec(x_26); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4658,33 +6198,33 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_142 = lean_ctor_get(x_120, 0); -lean_inc(x_142); -x_143 = lean_ctor_get(x_120, 1); -lean_inc(x_143); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_144 = x_120; -} else { - lean_dec_ref(x_120); - x_144 = lean_box(0); +x_68 = !lean_is_exclusive(x_46); +if (x_68 == 0) +{ +return x_46; +} +else +{ +lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_46, 0); +x_70 = lean_ctor_get(x_46, 1); +lean_inc(x_70); +lean_inc(x_69); +lean_dec(x_46); +x_71 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_71, 0, x_69); +lean_ctor_set(x_71, 1, x_70); +return x_71; } -if (lean_is_scalar(x_144)) { - x_145 = lean_alloc_ctor(1, 2, 0); -} else { - x_145 = x_144; } -lean_ctor_set(x_145, 0, x_142); -lean_ctor_set(x_145, 1, x_143); -return x_145; } } } else { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; -lean_dec(x_101); +uint8_t x_85; +lean_dec(x_27); +lean_dec(x_26); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4693,33 +6233,30 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_146 = lean_ctor_get(x_102, 0); -lean_inc(x_146); -x_147 = lean_ctor_get(x_102, 1); -lean_inc(x_147); -if (lean_is_exclusive(x_102)) { - lean_ctor_release(x_102, 0); - lean_ctor_release(x_102, 1); - x_148 = x_102; -} else { - lean_dec_ref(x_102); - x_148 = lean_box(0); -} -if (lean_is_scalar(x_148)) { - x_149 = lean_alloc_ctor(1, 2, 0); -} else { - x_149 = x_148; +x_85 = !lean_is_exclusive(x_29); +if (x_85 == 0) +{ +return x_29; } -lean_ctor_set(x_149, 0, x_146); -lean_ctor_set(x_149, 1, x_147); -return x_149; +else +{ +lean_object* x_86; lean_object* x_87; lean_object* x_88; +x_86 = lean_ctor_get(x_29, 0); +x_87 = lean_ctor_get(x_29, 1); +lean_inc(x_87); +lean_inc(x_86); +lean_dec(x_29); +x_88 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_88, 0, x_86); +lean_ctor_set(x_88, 1, x_87); +return x_88; } } } } else { -uint8_t x_150; +uint8_t x_89; lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -4728,23 +6265,23 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_150 = !lean_is_exclusive(x_21); -if (x_150 == 0) +x_89 = !lean_is_exclusive(x_21); +if (x_89 == 0) { return x_21; } else { -lean_object* x_151; lean_object* x_152; lean_object* x_153; -x_151 = lean_ctor_get(x_21, 0); -x_152 = lean_ctor_get(x_21, 1); -lean_inc(x_152); -lean_inc(x_151); +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_21, 0); +x_91 = lean_ctor_get(x_21, 1); +lean_inc(x_91); +lean_inc(x_90); lean_dec(x_21); -x_153 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_153, 0, x_151); -lean_ctor_set(x_153, 1, x_152); -return x_153; +x_92 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_92, 0, x_90); +lean_ctor_set(x_92, 1, x_91); +return x_92; } } block_20: @@ -4888,7 +6425,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__2___boxed(lean_ob lean_object* x_12; x_12 = l_Lean_Meta_Grind_splitNext___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); lean_dec(x_3); -lean_dec(x_1); return x_12; } } @@ -4898,7 +6434,6 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_splitNext___lambda__3___boxed(lean_ob lean_object* x_13; x_13 = l_Lean_Meta_Grind_splitNext___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_3); -lean_dec(x_2); return x_13; } } @@ -4923,13 +6458,14 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_CasesMatch(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1 = _init_l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_CaseSplitStatus_noConfusion___rarg___closed__1); l_Lean_Meta_Grind_instInhabitedCaseSplitStatus = _init_l_Lean_Meta_Grind_instInhabitedCaseSplitStatus(); +lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedCaseSplitStatus); l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1 = _init_l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_instBEqCaseSplitStatus___closed__1); l_Lean_Meta_Grind_instBEqCaseSplitStatus = _init_l_Lean_Meta_Grind_instBEqCaseSplitStatus(); lean_mark_persistent(l_Lean_Meta_Grind_instBEqCaseSplitStatus); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkIteCondStatus___closed__1); l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1(); lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__1); l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__2(); @@ -4940,6 +6476,16 @@ l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCase lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__4); l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5 = _init_l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5(); lean_mark_persistent(l_panic___at___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___spec__1___closed__5); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__1); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__2); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__3); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__4); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__2___closed__5); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__1); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__2(); @@ -4950,24 +6496,14 @@ l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__4); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__5); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__1); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__2); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__3); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__4); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__5); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__6); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__7); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__8); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__8___closed__9); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__6); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__7); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__8); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___lambda__5___closed__9); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__1); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__2(); @@ -4986,20 +6522,30 @@ l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__8); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__9); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__10); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_checkCaseSplitStatus___closed__11); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___lambda__2___closed__1); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_selectNextSplit_x3f___closed__1); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__1); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__2); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__3); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__4); -l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__2___closed__5); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__1); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__2); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__3); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__4); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__5); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__6); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__7); +l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__1___closed__8); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1(); lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__1); l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Split_0__Lean_Meta_Grind_mkCasesMajor___lambda__3___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Grind/Types.c b/stage0/stdlib/Lean/Meta/Tactic/Grind/Types.c index cd9abe19d6cb..7ff34964af35 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Grind/Types.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Grind/Types.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Lean.Meta.Tactic.Grind.Types -// Imports: Init.Grind.Tactics Init.Data.Queue Lean.Util.ShareCommon Lean.HeadIndex Lean.Meta.Basic Lean.Meta.CongrTheorems Lean.Meta.AbstractNestedProofs Lean.Meta.Tactic.Simp.Types Lean.Meta.Tactic.Util Lean.Meta.Tactic.Grind.Canon Lean.Meta.Tactic.Grind.Attr Lean.Meta.Tactic.Grind.EMatchTheorem +// Imports: Init.Grind.Tactics Init.Data.Queue Lean.Util.ShareCommon Lean.HeadIndex Lean.Meta.Basic Lean.Meta.CongrTheorems Lean.Meta.AbstractNestedProofs Lean.Meta.Tactic.Simp.Types Lean.Meta.Tactic.Util Lean.Meta.Tactic.Grind.ENodeKey Lean.Meta.Tactic.Grind.Canon Lean.Meta.Tactic.Grind.Attr Lean.Meta.Tactic.Grind.Arith.Types Lean.Meta.Tactic.Grind.EMatchTheorem #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,50 +13,57 @@ #ifdef __cplusplus extern "C" { #endif -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__52; static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_instBEqPreInstance___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21; lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__60; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__43; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedMethods; LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Meta_Grind_registerParent___spec__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instInhabitedENode___closed__1; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__4; static lean_object* l_Lean_Meta_Grind_updateLastTag___closed__1; lean_object* l_Lean_Syntax_mkNameLit(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashablePreInstance_unsafe__1___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_setENode___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instReprENode; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__21; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachENode___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_markTheoremInstance___spec__4(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqv___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__23; lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addNewFact___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_right(size_t, size_t); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41; +static lean_object* l_Lean_Meta_Grind_isNatNum___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqHEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__16; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_ENode_isCongrRoot___boxed(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20; static lean_object* l_Lean_Meta_Grind_markAsInconsistent___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_abstractNestedProofs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__14; LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTrueExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__1; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4; -static size_t l_Lean_Meta_Grind_instInhabitedGoal___closed__3; +static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__3; LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Meta_Grind_instInhabitedMethods___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_congrHash_goEq___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTarget_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_updateLastTag___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -71,35 +78,31 @@ uint8_t lean_usize_dec_le(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMethodsRef(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_getParentsAndReset___spec__1(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqENodeKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_instHashablePreInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_filterENodes___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__2___closed__1; uint64_t lean_uint64_of_nat(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run(lean_object*); lean_object* l_Lean_Meta_isExprDefEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_setENode_unsafe__1___rarg(lean_object*); size_t lean_uint64_to_usize(uint64_t); uint64_t lean_uint64_lor(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__5; -static lean_object* l_Lean_Meta_Grind_getENode___closed__2; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__22; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMainDeclName___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run_x27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__53; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__24; uint8_t l_Lean_Expr_isApp(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118_(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isCongruent(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_getId(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53; uint8_t l_Lean_RBNode_isRed___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInterpreted(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentArray_push___rarg(lean_object*, lean_object*); @@ -108,49 +111,63 @@ static lean_object* l_Lean_Meta_Grind_markAsInconsistent___closed__1; lean_object* l_Array_toSubarray___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__20; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__7; +static lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1; size_t lean_usize_mul(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_alreadyInternalized___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56; lean_object* lean_mk_array(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHCongrWithArity___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_uint64_dec_lt(uint64_t, uint64_t); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__5; -uint8_t lean_usize_dec_eq(size_t, size_t); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__12; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr_unsafe__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isNatNum___lambda__1(lean_object*); LEAN_EXPORT uint64_t l_Lean_Meta_Grind_congrHash(lean_object*, lean_object*); lean_object* l_Lean_Expr_bvar___override(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMaxGeneration___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getFalseExpr___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_grind_debug_proofs; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr(lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Meta_Grind_instInhabitedMethods___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_registerParent___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__24; lean_object* l_Lean_MVarId_getTag(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqCore(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc_go(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_forEachENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__10; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateDown(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENodes(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__2(lean_object*, size_t, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_forEachEqc(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_alreadyInternalized___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqcs(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_Queue_enqueue___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_hasSameRoot(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableCongrTheoremCacheKey(lean_object*); +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_registerParent___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -160,6 +177,7 @@ lean_object* l_Lean_Name_mkStr5(lean_object*, lean_object*, lean_object*, lean_o size_t lean_usize_of_nat(lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMethods___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15; lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__51; lean_object* l_Lean_stringToMessageData(lean_object*); @@ -168,13 +186,16 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMainDeclName___rarg(lean_object*, static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__13; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_mkHCongrWithArity___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHCongrWithArity___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__36; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getFalseExpr(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_Goal_getENodes___spec__2(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedMethods___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_processNewOffsetEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__41; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28; +static lean_object* l_Lean_Meta_Grind_isNatNum___closed__4; LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_registerParent___spec__6(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_registerParent___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -187,6 +208,7 @@ static uint64_t l_Lean_Meta_Grind_hasSameType___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqCongrKey___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqCongrTheoremCacheKey___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Methods_toMethodsRef___boxed(lean_object*); @@ -196,25 +218,26 @@ static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types___ LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_alreadyInternalized___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_setENode___spec__4(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_grind_debug; LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_MethodsRef_toMethods(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25; lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_AbstractNestedProofs_visit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_propagateUp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isResolvedCaseSplit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqTrue___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum___lambda__1___boxed(lean_object*); LEAN_EXPORT uint64_t l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_instHashablePreInstance___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_markTheoremInstance___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashablePreInstance___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_registerParent___spec__5(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMaxGeneration___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -224,14 +247,17 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_ma LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxEmatchExceeded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isLambda(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__3___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_updateLastTag___closed__5; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3; size_t lean_ptr_addr(lean_object*); lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqCore___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getFalseExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Methods_toMethodsRef_unsafe__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTarget_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -239,10 +265,9 @@ lean_object* l_Lean_PersistentHashMap_isUnaryNode___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_registerParent___spec__8(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxEmatchExceeded___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__48; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_Goal_getENodes___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__14; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_setENode_unsafe__1___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27; static lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__3; LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqPreInstance___lambda__1(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -250,65 +275,67 @@ static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__ static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markTheoremInstance___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRootENode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34; lean_object* lean_st_ref_take(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_hasSameRoot___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqFalse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getParentsAndReset___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode_x3f___boxed(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_isNatNum___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_filterENodes___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__2___closed__2; static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__3; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__30; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__6; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashablePreInstance_unsafe__2___boxed(lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getGeneration___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SourceInfo_fromRef(lean_object*, uint8_t); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10; lean_object* l_Lean_RBNode_setBlack___rarg(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addTheoremInstance___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_usize_to_uint64(size_t); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25; lean_object* lean_nat_to_int(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24; lean_object* l_Lean_Syntax_node6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_registerParent___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqHEqProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_getType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f(lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39; static lean_object* l_Lean_Meta_Grind_abstractNestedProofs___closed__1; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqHEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36; +static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxInstancesExceeded(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_closeGoal(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MVarId_admit(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode_x3f___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getConfig___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHCongrWithArity___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxInstancesExceeded___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_isNatNum___closed__1; lean_object* l_Lean_Meta_mkHCongrWithArityForConst_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_setENode___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17; static lean_object* l_Lean_Meta_Grind_updateLastTag___closed__4; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__31; lean_object* l_Lean_Syntax_getKind(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markTheoremInstance___spec__3___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78_(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxCaseSplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_markTheoremInstance___spec__11___lambda__2(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__5(lean_object*, lean_object*, lean_object*, size_t, size_t, uint64_t); @@ -316,9 +343,9 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode___boxed(lean_object*, lean_o LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTrueExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_quoteNameMk(lean_object*); LEAN_EXPORT uint64_t l_Lean_Meta_Grind_congrHash_goEq(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__49; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkENode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_markTheoremInstance___spec__13___lambda__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__58; lean_object* lean_st_ref_get(lean_object*, lean_object*); @@ -333,31 +360,36 @@ lean_object* lean_st_mk_ref(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markTheoremInstance___spec__7(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__46; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__19; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23; lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongruent___boxed(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_Basic_0__Lean_Meta_withMVarContextImp___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext_x3f___boxed(lean_object*, lean_object*); +lean_object* l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMainDeclName(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35; -static lean_object* l_Lean_Meta_Grind_canon___closed__3; lean_object* l_Lean_Syntax_node3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445_(lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashablePreInstance(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__16; +static lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongruent_goEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3(size_t, size_t, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__33; -LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey(lean_object*); LEAN_EXPORT uint64_t l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_mkHCongrWithArity___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot_x3f___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_MethodsRef_toMethods_unsafe__1(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr___boxed(lean_object*, lean_object*); static size_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__2; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__39; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMethodsRef___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_congrHash___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsOffsetTerm(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqCongrTheoremCacheKey(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_markTheoremInstance___spec__9(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__11; @@ -368,25 +400,28 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqcs___boxed(lean_object*, lean_ob static lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__3; lean_object* l_Lean_addMacroScope(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__50; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_canon___closed__1; +static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__8; static lean_object* l_Lean_Meta_Grind_congrHash___closed__1; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4; uint8_t lean_name_eq(lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getGeneration(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqENodeKey___boxed(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkHCongrWithArity(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5; +uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_alreadyInternalized(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Syntax_node2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_alreadyInternalized___spec__2(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongruent_go___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNext___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_registerParent___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3___boxed(lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMethods(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMainDeclName___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -396,14 +431,16 @@ LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_G static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__8; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getParents(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_markTheoremInstance___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__5; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_processNewOffsetEqLit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInterpreted___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_process_new_offset_eq_lit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markTheoremInstance___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_getENodes___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__1; lean_object* l_Lean_Expr_appFn_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_applyFallback(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -412,28 +449,30 @@ static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__ static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__3; LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_markTheoremInstance___spec__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Meta_Grind_GoalM_run___spec__1(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19; lean_object* l_Array_eraseIdx___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_hasSameType(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHEqProof___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableCongrKey___boxed(lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashablePreInstance_unsafe__1(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_traverseEqc(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__10; LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__2(lean_object*, size_t, lean_object*); uint8_t l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(lean_object*, lean_object*); lean_object* l_Lean_Meta_mkFalseElim(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109_(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8; static lean_object* l_Lean_Meta_Grind_instInhabitedENode___closed__2; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48; lean_object* lean_usize_to_nat(size_t); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isCongruent_go(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__18; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getParents___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_updateLastTag___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_alreadyInternalized___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_getENode___closed__3; LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableCongrKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Grind_Canon_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); @@ -442,26 +481,22 @@ lean_object* l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoB static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__26; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__4; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3; static lean_object* l_Lean_Meta_Grind_instReprENode___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_shareCommon___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__10(lean_object*, lean_object*, lean_object*, size_t, size_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isResolvedCaseSplit(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENodes___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_registerParent___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560_(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markTheoremInstance___spec__7___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_GoalM_run_x27___closed__1; static lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__2; @@ -481,46 +516,55 @@ lean_object* lean_grind_mk_heq_proof(lean_object*, lean_object*, lean_object*, l LEAN_EXPORT uint64_t l_Lean_Meta_Grind_congrHash_go(lean_object*, lean_object*, uint64_t); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedMethods___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_process_new_offset_eq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__1___boxed(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__34; LEAN_EXPORT lean_object* l_Lean_MVarId_withContext___at_Lean_Meta_Grind_GoalM_run___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addNewFact(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_instBEqPreInstance___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_markTheoremInstance___spec__11___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_congrPlaceholderProof___closed__3; LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Meta_Grind_instInhabitedMethods___spec__1(lean_object*); lean_object* l___private_Init_Meta_0__Lean_getEscapedNameParts_x3f(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markTheoremInstance___spec__7___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_alreadyInternalized___spec__1___boxed(lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4; static lean_object* l_Lean_Meta_Grind_congrHash___closed__3; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_abstractNestedProofs___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqcs(lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_shareCommon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markTheoremInstance___spec__7___lambda__2___boxed(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_mkHCongrWithArity___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_addTheoremInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_MethodsRef_toMethods___boxed(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__42; uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9; LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_markTheoremInstance___spec__13___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__32; +static lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__22; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run_x27___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_setENode___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45; lean_object* l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_instInhabitedMethods___closed__1; LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -529,15 +573,15 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___boxed(lean_object*, le lean_object* l_Lean_Meta_isConstructorAppCore_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__9; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__1; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc_go(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markTheoremInstance___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_registerParent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__7; -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr(lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5; static lean_object* l_Lean_Meta_Grind_markAsInconsistent___closed__3; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34; static lean_object* l_Lean_Meta_Grind_congrPlaceholderProof___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__59; +static lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; lean_object* l_Lean_indentExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMaxGeneration___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -552,30 +596,31 @@ static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__2; lean_object* l_Lean_Syntax_node1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__18; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__7; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markTheoremInstance(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__21; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHCongrWithArity___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum(lean_object*); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqCongrKey(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___boxed(lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_insertAtCollisionNodeAux___at_Lean_Meta_Grind_markTheoremInstance___spec__7___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_markTheoremInstance___spec__9___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1(lean_object*); lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24; +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_eraseAux___at_Lean_Meta_Grind_getParentsAndReset___spec__2(lean_object*, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__2; static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqv(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqFalse___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___boxed(lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3036_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot_x3f(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Methods_toMethodsRef(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -583,7 +628,7 @@ LEAN_EXPORT lean_object* l_Array_indexOfAux___at_Lean_Meta_Grind_getParentsAndRe LEAN_EXPORT lean_object* l_Array_indexOfAux___at_Lean_Meta_Grind_getParentsAndReset___spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isRoot___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_setENode___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_copyParentsTo___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_left(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Methods_toMethodsRef_unsafe__1(lean_object*); @@ -596,32 +641,33 @@ static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types___ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTrueExpr(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__15; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkENodeCore(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__44; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run_x27___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachENode___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_erase_macro_scopes(lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__40; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__17; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52; static lean_object* l_Lean_Meta_Grind_congrHash___closed__4; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__9; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___boxed(lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__47; -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode_x3f(lean_object*, lean_object*); lean_object* l_String_intercalate(lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__20; -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1___boxed(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getParentsAndReset(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -635,37 +681,35 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_congrHash_go___boxed(lean_object*, le static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markTheoremInstance___spec__3___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_isTracingEnabledForCore(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object*); +uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object*); size_t lean_usize_add(size_t, size_t); extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__8; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_getParentsAndReset___spec__1___boxed(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__55; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableCongrTheoremCacheKey___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedNewFact; -static lean_object* l_Lean_Meta_Grind_getENode___closed__1; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMaxGeneration(lean_object*); +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____boxed(lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isCongruent_goEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Grind_instInhabitedGoal___closed__4; +static size_t l_Lean_Meta_Grind_instInhabitedGoal___closed__4; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__19; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushHEq___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__1; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31; +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_getENodes___spec__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__6(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkENode___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_shift_left(size_t, size_t); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_MethodsRef_toMethods_unsafe__1___boxed(lean_object*); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1; -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___lambda__1(lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12; LEAN_EXPORT uint64_t l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1(lean_object*); static lean_object* l_Lean_Meta_Grind_congrHash___closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHCongrWithArity___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -674,36 +718,30 @@ static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types___ extern lean_object* l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__37; LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_markTheoremInstance___spec__3___lambda__1(lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_pushEqTrue___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqPreInstance___lambda__3(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47; -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13; static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__11; extern lean_object* l_Lean_ShareCommon_objectFactory; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRootENode(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_state_sharecommon(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(lean_object*, lean_object*, lean_object*); lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32; uint8_t lean_usize_dec_lt(size_t, size_t); -static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40; -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markTheoremInstance___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29; uint64_t l_Lean_Meta_TransparencyMode_toUInt64(uint8_t); lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__38; @@ -713,12 +751,14 @@ lean_object* l_Lean_PersistentHashMap_getCollisionNodeSize___rarg(lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_markTheoremInstance___spec__11(lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentHashMap_containsAtAux___at_Lean_Meta_Grind_alreadyInternalized___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__25; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49; +static lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9; static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__35; +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_MethodsRefPointed; -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d____; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__10; -static lean_object* l_Lean_Meta_Grind_canon___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_instBEqPreInstance___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__57; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run_x27___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -729,76 +769,40 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_GoalM_run___rarg___lambda__2(lean_obj LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getFalseExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey___boxed(lean_object*); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT size_t l_Lean_Meta_Grind_instHashableCongrTheoremCacheKey_unsafe__1(lean_object*); lean_object* lean_array_get(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26; lean_object* l_Lean_Meta_isLitValue(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_forEachEqcRoot(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1; +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Grind_updateLastTag___closed__3; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInterpreted___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Grind_updateLastTag___closed__2; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__6___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_containsAux___at_Lean_Meta_Grind_markTheoremInstance___spec__11___lambda__2___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_checkMaxCaseSplit___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instInhabitedGoal; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableCongrTheoremCacheKey_unsafe__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkENode___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_setENode___spec__2(lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_updateLastTag___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); -static lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9; LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getConfig___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_setENode___spec__3(size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_46____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_mkHCongrWithArity___spec__5___boxed(lean_object*, lean_object*); LEAN_EXPORT uint64_t l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_markTheoremInstance___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, uint64_t); static lean_object* l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__9; -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr_unsafe__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -size_t x_3; size_t x_4; uint8_t x_5; -x_3 = lean_ptr_addr(x_1); -x_4 = lean_ptr_addr(x_2); -x_5 = lean_usize_dec_eq(x_3, x_4); -return x_5; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr_unsafe__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} -} -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isSameExpr(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; -x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isSameExpr___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Meta_Grind_isSameExpr(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} -} static lean_object* _init_l_Lean_Meta_Grind_congrPlaceholderProof___closed__1() { _start: { @@ -902,7 +906,7 @@ lean_dec(x_2); return x_8; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1() { _start: { lean_object* x_1; @@ -910,7 +914,7 @@ x_1 = lean_mk_string_unchecked("grind", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2() { _start: { lean_object* x_1; @@ -918,17 +922,17 @@ x_1 = lean_mk_string_unchecked("debug", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4() { _start: { lean_object* x_1; @@ -936,13 +940,13 @@ x_1 = lean_mk_string_unchecked("check invariants after updates", 30, 30); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -951,7 +955,7 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6() { _start: { lean_object* x_1; @@ -959,7 +963,7 @@ x_1 = lean_mk_string_unchecked("Lean", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7() { _start: { lean_object* x_1; @@ -967,7 +971,7 @@ x_1 = lean_mk_string_unchecked("Meta", 4, 4); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8() { _start: { lean_object* x_1; @@ -975,31 +979,31 @@ x_1 = lean_mk_string_unchecked("Grind", 5, 5); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; -x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; +x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; x_6 = l_Lean_Name_mkStr5(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9; x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1() { _start: { lean_object* x_1; @@ -1007,18 +1011,18 @@ x_1 = lean_mk_string_unchecked("proofs", 6, 6); return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3() { _start: { lean_object* x_1; @@ -1026,13 +1030,13 @@ x_1 = lean_mk_string_unchecked("check proofs between the elements of all equival return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4() { _start: { uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 0; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3; x_4 = lean_box(x_1); x_5 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_5, 0, x_4); @@ -1041,27 +1045,27 @@ lean_ctor_set(x_5, 2, x_3); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; -x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2; -x_6 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; +x_5 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2; +x_6 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1; x_7 = l_Lean_Name_mkStr6(x_1, x_2, x_3, x_4, x_5, x_6); return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118_(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109_(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4; -x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4; +x_4 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5; x_5 = l_Lean_Option_register___at_Lean_Elab_initFn____x40_Lean_Elab_AutoBound___hyg_6____spec__1(x_2, x_3, x_4, x_1); return x_5; } @@ -1200,7 +1204,7 @@ if (x_8 == 0) { lean_object* x_9; lean_object* x_10; x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_9, 5); +x_10 = lean_ctor_get(x_9, 4); lean_inc(x_10); lean_dec(x_9); lean_ctor_set(x_7, 0, x_10); @@ -1214,7 +1218,7 @@ x_12 = lean_ctor_get(x_7, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_7); -x_13 = lean_ctor_get(x_11, 5); +x_13 = lean_ctor_get(x_11, 4); lean_inc(x_13); lean_dec(x_11); x_14 = lean_alloc_ctor(0, 2, 0); @@ -1265,7 +1269,7 @@ if (x_8 == 0) { lean_object* x_9; lean_object* x_10; x_9 = lean_ctor_get(x_7, 0); -x_10 = lean_ctor_get(x_9, 6); +x_10 = lean_ctor_get(x_9, 5); lean_inc(x_10); lean_dec(x_9); lean_ctor_set(x_7, 0, x_10); @@ -1279,7 +1283,7 @@ x_12 = lean_ctor_get(x_7, 1); lean_inc(x_12); lean_inc(x_11); lean_dec(x_7); -x_13 = lean_ctor_get(x_11, 6); +x_13 = lean_ctor_get(x_11, 5); lean_inc(x_13); lean_dec(x_11); x_14 = lean_alloc_ctor(0, 2, 0); @@ -1320,6 +1324,71 @@ lean_dec(x_1); return x_3; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; uint8_t x_8; +x_7 = lean_st_ref_get(x_1, x_6); +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_9, 6); +lean_inc(x_10); +lean_dec(x_9); +lean_ctor_set(x_7, 0, x_10); +return x_7; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_ctor_get(x_7, 0); +x_12 = lean_ctor_get(x_7, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_7); +x_13 = lean_ctor_get(x_11, 6); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +return x_14; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_getNatZeroExpr___rarg___boxed), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; +x_7 = l_Lean_Meta_Grind_getNatZeroExpr___rarg(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNatZeroExpr___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_getNatZeroExpr(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getMainDeclName___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { @@ -1494,7 +1563,7 @@ lean_inc(x_11); x_12 = lean_ctor_get(x_10, 1); lean_inc(x_12); lean_dec(x_10); -x_13 = lean_ctor_get(x_11, 2); +x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); x_14 = l_Lean_Meta_Grind_getMainDeclName___rarg(x_3, x_4, x_5, x_6, x_7, x_8, x_12); @@ -1549,9 +1618,9 @@ x_35 = !lean_is_exclusive(x_33); if (x_35 == 0) { lean_object* x_36; lean_object* x_37; uint8_t x_38; -x_36 = lean_ctor_get(x_33, 2); +x_36 = lean_ctor_get(x_33, 1); lean_dec(x_36); -lean_ctor_set(x_33, 2, x_30); +lean_ctor_set(x_33, 1, x_30); x_37 = lean_st_ref_set(x_4, x_33, x_34); x_38 = !lean_is_exclusive(x_37); if (x_38 == 0) @@ -1578,7 +1647,7 @@ else { lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; x_42 = lean_ctor_get(x_33, 0); -x_43 = lean_ctor_get(x_33, 1); +x_43 = lean_ctor_get(x_33, 2); x_44 = lean_ctor_get(x_33, 3); x_45 = lean_ctor_get(x_33, 4); x_46 = lean_ctor_get(x_33, 5); @@ -1594,8 +1663,8 @@ lean_inc(x_42); lean_dec(x_33); x_49 = lean_alloc_ctor(0, 8, 0); lean_ctor_set(x_49, 0, x_42); -lean_ctor_set(x_49, 1, x_43); -lean_ctor_set(x_49, 2, x_30); +lean_ctor_set(x_49, 1, x_30); +lean_ctor_set(x_49, 2, x_43); lean_ctor_set(x_49, 3, x_44); lean_ctor_set(x_49, 4, x_45); lean_ctor_set(x_49, 5, x_46); @@ -1673,7 +1742,7 @@ x_13 = !lean_is_exclusive(x_11); if (x_13 == 0) { lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_14 = lean_ctor_get(x_11, 1); +x_14 = lean_ctor_get(x_11, 0); x_15 = l_Lean_ShareCommon_objectFactory; x_16 = lean_state_sharecommon(x_15, x_14, x_1); x_17 = lean_ctor_get(x_16, 0); @@ -1681,7 +1750,7 @@ lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -lean_ctor_set(x_11, 1, x_18); +lean_ctor_set(x_11, 0, x_18); x_19 = lean_st_ref_set(x_4, x_11, x_12); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) @@ -1725,15 +1794,15 @@ lean_inc(x_25); lean_inc(x_24); lean_dec(x_11); x_32 = l_Lean_ShareCommon_objectFactory; -x_33 = lean_state_sharecommon(x_32, x_25, x_1); +x_33 = lean_state_sharecommon(x_32, x_24, x_1); x_34 = lean_ctor_get(x_33, 0); lean_inc(x_34); x_35 = lean_ctor_get(x_33, 1); lean_inc(x_35); lean_dec(x_33); x_36 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_36, 0, x_24); -lean_ctor_set(x_36, 1, x_35); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_25); lean_ctor_set(x_36, 2, x_26); lean_ctor_set(x_36, 3, x_27); lean_ctor_set(x_36, 4, x_28); @@ -1777,428 +1846,104 @@ lean_dec(x_2); return x_10; } } -static lean_object* _init_l_Lean_Meta_Grind_canon___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; -} +lean_object* x_10; uint8_t x_11; +x_10 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_12); +lean_dec(x_12); +x_14 = lean_box(x_13); +lean_ctor_set(x_10, 0, x_14); +return x_10; } -static lean_object* _init_l_Lean_Meta_Grind_canon___closed__2() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_canon___closed__1; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); +lean_dec(x_15); +x_18 = lean_box(x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_16); +return x_19; +} } } -static lean_object* _init_l_Lean_Meta_Grind_canon___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_canon___closed__2; -x_2 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); -return x_2; +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_isTrueExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_st_ref_take(x_4, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_10, 1); -lean_inc(x_12); -lean_dec(x_10); -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_14 = lean_ctor_get(x_11, 0); -x_15 = l_Lean_Meta_Grind_canon___closed__3; -lean_ctor_set(x_11, 0, x_15); -x_16 = lean_st_ref_set(x_4, x_11, x_12); -x_17 = lean_ctor_get(x_16, 1); -lean_inc(x_17); -lean_dec(x_16); -x_18 = l_Lean_Meta_Grind_Canon_canon(x_1, x_14, x_5, x_6, x_7, x_8, x_17); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_19, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_19, 1); -lean_inc(x_22); -lean_dec(x_19); -x_23 = lean_st_ref_take(x_4, x_20); -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = !lean_is_exclusive(x_24); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_27 = lean_ctor_get(x_24, 0); -lean_dec(x_27); -lean_ctor_set(x_24, 0, x_22); -x_28 = lean_st_ref_set(x_4, x_24, x_25); -x_29 = !lean_is_exclusive(x_28); -if (x_29 == 0) +lean_object* x_10; uint8_t x_11; +x_10 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_30; -x_30 = lean_ctor_get(x_28, 0); -lean_dec(x_30); -lean_ctor_set(x_28, 0, x_21); -return x_28; +lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_12); +lean_dec(x_12); +x_14 = lean_box(x_13); +lean_ctor_set(x_10, 0, x_14); +return x_10; } else { -lean_object* x_31; lean_object* x_32; -x_31 = lean_ctor_get(x_28, 1); -lean_inc(x_31); -lean_dec(x_28); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_21); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); +lean_dec(x_15); +x_18 = lean_box(x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_16); +return x_19; } } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_33 = lean_ctor_get(x_24, 1); -x_34 = lean_ctor_get(x_24, 2); -x_35 = lean_ctor_get(x_24, 3); -x_36 = lean_ctor_get(x_24, 4); -x_37 = lean_ctor_get(x_24, 5); -x_38 = lean_ctor_get(x_24, 6); -x_39 = lean_ctor_get(x_24, 7); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_24); -x_40 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_40, 0, x_22); -lean_ctor_set(x_40, 1, x_33); -lean_ctor_set(x_40, 2, x_34); -lean_ctor_set(x_40, 3, x_35); -lean_ctor_set(x_40, 4, x_36); -lean_ctor_set(x_40, 5, x_37); -lean_ctor_set(x_40, 6, x_38); -lean_ctor_set(x_40, 7, x_39); -x_41 = lean_st_ref_set(x_4, x_40, x_25); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -if (lean_is_exclusive(x_41)) { - lean_ctor_release(x_41, 0); - lean_ctor_release(x_41, 1); - x_43 = x_41; -} else { - lean_dec_ref(x_41); - x_43 = lean_box(0); -} -if (lean_is_scalar(x_43)) { - x_44 = lean_alloc_ctor(0, 2, 0); -} else { - x_44 = x_43; -} -lean_ctor_set(x_44, 0, x_21); -lean_ctor_set(x_44, 1, x_42); -return x_44; -} -} -else -{ -uint8_t x_45; -x_45 = !lean_is_exclusive(x_18); -if (x_45 == 0) -{ -return x_18; -} -else -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_46 = lean_ctor_get(x_18, 0); -x_47 = lean_ctor_get(x_18, 1); -lean_inc(x_47); -lean_inc(x_46); -lean_dec(x_18); -x_48 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_48, 0, x_46); -lean_ctor_set(x_48, 1, x_47); -return x_48; -} -} -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; -x_49 = lean_ctor_get(x_11, 0); -x_50 = lean_ctor_get(x_11, 1); -x_51 = lean_ctor_get(x_11, 2); -x_52 = lean_ctor_get(x_11, 3); -x_53 = lean_ctor_get(x_11, 4); -x_54 = lean_ctor_get(x_11, 5); -x_55 = lean_ctor_get(x_11, 6); -x_56 = lean_ctor_get(x_11, 7); -lean_inc(x_56); -lean_inc(x_55); -lean_inc(x_54); -lean_inc(x_53); -lean_inc(x_52); -lean_inc(x_51); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_11); -x_57 = l_Lean_Meta_Grind_canon___closed__3; -x_58 = lean_alloc_ctor(0, 8, 0); -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_50); -lean_ctor_set(x_58, 2, x_51); -lean_ctor_set(x_58, 3, x_52); -lean_ctor_set(x_58, 4, x_53); -lean_ctor_set(x_58, 5, x_54); -lean_ctor_set(x_58, 6, x_55); -lean_ctor_set(x_58, 7, x_56); -x_59 = lean_st_ref_set(x_4, x_58, x_12); -x_60 = lean_ctor_get(x_59, 1); -lean_inc(x_60); -lean_dec(x_59); -x_61 = l_Lean_Meta_Grind_Canon_canon(x_1, x_49, x_5, x_6, x_7, x_8, x_60); -if (lean_obj_tag(x_61) == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_62 = lean_ctor_get(x_61, 0); -lean_inc(x_62); -x_63 = lean_ctor_get(x_61, 1); -lean_inc(x_63); -lean_dec(x_61); -x_64 = lean_ctor_get(x_62, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_62, 1); -lean_inc(x_65); -lean_dec(x_62); -x_66 = lean_st_ref_take(x_4, x_63); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = lean_ctor_get(x_67, 1); -lean_inc(x_69); -x_70 = lean_ctor_get(x_67, 2); -lean_inc(x_70); -x_71 = lean_ctor_get(x_67, 3); -lean_inc(x_71); -x_72 = lean_ctor_get(x_67, 4); -lean_inc(x_72); -x_73 = lean_ctor_get(x_67, 5); -lean_inc(x_73); -x_74 = lean_ctor_get(x_67, 6); -lean_inc(x_74); -x_75 = lean_ctor_get(x_67, 7); -lean_inc(x_75); -if (lean_is_exclusive(x_67)) { - lean_ctor_release(x_67, 0); - lean_ctor_release(x_67, 1); - lean_ctor_release(x_67, 2); - lean_ctor_release(x_67, 3); - lean_ctor_release(x_67, 4); - lean_ctor_release(x_67, 5); - lean_ctor_release(x_67, 6); - lean_ctor_release(x_67, 7); - x_76 = x_67; -} else { - lean_dec_ref(x_67); - x_76 = lean_box(0); -} -if (lean_is_scalar(x_76)) { - x_77 = lean_alloc_ctor(0, 8, 0); -} else { - x_77 = x_76; -} -lean_ctor_set(x_77, 0, x_65); -lean_ctor_set(x_77, 1, x_69); -lean_ctor_set(x_77, 2, x_70); -lean_ctor_set(x_77, 3, x_71); -lean_ctor_set(x_77, 4, x_72); -lean_ctor_set(x_77, 5, x_73); -lean_ctor_set(x_77, 6, x_74); -lean_ctor_set(x_77, 7, x_75); -x_78 = lean_st_ref_set(x_4, x_77, x_68); -x_79 = lean_ctor_get(x_78, 1); -lean_inc(x_79); -if (lean_is_exclusive(x_78)) { - lean_ctor_release(x_78, 0); - lean_ctor_release(x_78, 1); - x_80 = x_78; -} else { - lean_dec_ref(x_78); - x_80 = lean_box(0); -} -if (lean_is_scalar(x_80)) { - x_81 = lean_alloc_ctor(0, 2, 0); -} else { - x_81 = x_80; -} -lean_ctor_set(x_81, 0, x_64); -lean_ctor_set(x_81, 1, x_79); -return x_81; -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_82 = lean_ctor_get(x_61, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_61, 1); -lean_inc(x_83); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_84 = x_61; -} else { - lean_dec_ref(x_61); - x_84 = lean_box(0); -} -if (lean_is_scalar(x_84)) { - x_85 = lean_alloc_ctor(1, 2, 0); -} else { - x_85 = x_84; -} -lean_ctor_set(x_85, 0, x_82); -lean_ctor_set(x_85, 1, x_83); -return x_85; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_canon(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; uint8_t x_11; -x_10 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_12); -lean_dec(x_12); -x_14 = lean_box(x_13); -lean_ctor_set(x_10, 0, x_14); -return x_10; -} -else -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_10); -x_17 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); -lean_dec(x_15); -x_18 = lean_box(x_17); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_16); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isTrueExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_isTrueExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_10; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; uint8_t x_11; -x_10 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_4, x_5, x_6, x_7, x_8, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_12); -lean_dec(x_12); -x_14 = lean_box(x_13); -lean_ctor_set(x_10, 0, x_14); -return x_10; -} -else -{ -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_10); -x_17 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); -lean_dec(x_15); -x_18 = lean_box(x_17); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_16); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isFalseExpr___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: -{ -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_isFalseExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_10; +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_isFalseExpr(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } } LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_mkHCongrWithArity___spec__3(size_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -3147,10 +2892,10 @@ x_19 = !lean_is_exclusive(x_17); if (x_19 == 0) { lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_ctor_get(x_17, 3); +x_20 = lean_ctor_get(x_17, 2); lean_inc(x_14); x_21 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(x_20, x_3, x_14); -lean_ctor_set(x_17, 3, x_21); +lean_ctor_set(x_17, 2, x_21); x_22 = lean_st_ref_set(x_7, x_17, x_18); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) @@ -3194,12 +2939,12 @@ lean_inc(x_28); lean_inc(x_27); lean_dec(x_17); lean_inc(x_14); -x_35 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(x_30, x_3, x_14); +x_35 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(x_29, x_3, x_14); x_36 = lean_alloc_ctor(0, 8, 0); lean_ctor_set(x_36, 0, x_27); lean_ctor_set(x_36, 1, x_28); -lean_ctor_set(x_36, 2, x_29); -lean_ctor_set(x_36, 3, x_35); +lean_ctor_set(x_36, 2, x_35); +lean_ctor_set(x_36, 3, x_30); lean_ctor_set(x_36, 4, x_31); lean_ctor_set(x_36, 5, x_32); lean_ctor_set(x_36, 6, x_33); @@ -3308,10 +3053,10 @@ x_26 = lean_ctor_get(x_23, 1); lean_inc(x_26); x_27 = lean_ctor_get(x_23, 2); lean_inc(x_27); -x_28 = lean_ctor_get(x_23, 3); -lean_inc(x_28); lean_inc(x_21); -x_29 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(x_28, x_3, x_21); +x_28 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_mkHCongrWithArity___spec__1(x_27, x_3, x_21); +x_29 = lean_ctor_get(x_23, 3); +lean_inc(x_29); x_30 = lean_ctor_get(x_23, 4); lean_inc(x_30); x_31 = lean_ctor_get(x_23, 5); @@ -3324,7 +3069,7 @@ lean_dec(x_23); x_34 = lean_alloc_ctor(0, 8, 0); lean_ctor_set(x_34, 0, x_25); lean_ctor_set(x_34, 1, x_26); -lean_ctor_set(x_34, 2, x_27); +lean_ctor_set(x_34, 2, x_28); lean_ctor_set(x_34, 3, x_29); lean_ctor_set(x_34, 4, x_30); lean_ctor_set(x_34, 5, x_31); @@ -3408,7 +3153,7 @@ if (x_13 == 0) lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; x_14 = lean_ctor_get(x_12, 0); x_15 = lean_ctor_get(x_12, 1); -x_16 = lean_ctor_get(x_14, 3); +x_16 = lean_ctor_get(x_14, 2); lean_inc(x_16); lean_dec(x_14); x_17 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_mkHCongrWithArity___spec__5(x_16, x_11); @@ -3445,7 +3190,7 @@ x_22 = lean_ctor_get(x_12, 1); lean_inc(x_22); lean_inc(x_21); lean_dec(x_12); -x_23 = lean_ctor_get(x_21, 3); +x_23 = lean_ctor_get(x_21, 2); lean_inc(x_23); lean_dec(x_21); x_24 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_mkHCongrWithArity___spec__5(x_23, x_11); @@ -3584,7 +3329,7 @@ x_1 = lean_box(0); x_2 = l_Lean_Meta_Grind_instInhabitedENode___closed__1; x_3 = 0; x_4 = lean_unsigned_to_nat(0u); -x_5 = lean_alloc_ctor(0, 10, 5); +x_5 = lean_alloc_ctor(0, 11, 5); lean_ctor_set(x_5, 0, x_2); lean_ctor_set(x_5, 1, x_2); lean_ctor_set(x_5, 2, x_2); @@ -3595,11 +3340,12 @@ lean_ctor_set(x_5, 6, x_4); lean_ctor_set(x_5, 7, x_4); lean_ctor_set(x_5, 8, x_4); lean_ctor_set(x_5, 9, x_4); -lean_ctor_set_uint8(x_5, sizeof(void*)*10, x_3); -lean_ctor_set_uint8(x_5, sizeof(void*)*10 + 1, x_3); -lean_ctor_set_uint8(x_5, sizeof(void*)*10 + 2, x_3); -lean_ctor_set_uint8(x_5, sizeof(void*)*10 + 3, x_3); -lean_ctor_set_uint8(x_5, sizeof(void*)*10 + 4, x_3); +lean_ctor_set(x_5, 10, x_1); +lean_ctor_set_uint8(x_5, sizeof(void*)*11, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*11 + 1, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*11 + 2, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*11 + 3, x_3); +lean_ctor_set_uint8(x_5, sizeof(void*)*11 + 4, x_3); return x_5; } } @@ -3611,7 +3357,7 @@ x_1 = l_Lean_Meta_Grind_instInhabitedENode___closed__2; return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1() { _start: { lean_object* x_1; @@ -3619,29 +3365,29 @@ x_1 = lean_mk_string_unchecked("self", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2; +x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4() { _start: { lean_object* x_1; @@ -3649,29 +3395,29 @@ x_1 = lean_mk_string_unchecked(" := ", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3; -x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3; +x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5; x_3 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7() { _start: { lean_object* x_1; lean_object* x_2; @@ -3680,7 +3426,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8() { _start: { lean_object* x_1; @@ -3688,17 +3434,17 @@ x_1 = lean_mk_string_unchecked(",", 1, 1); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10() { _start: { lean_object* x_1; @@ -3706,17 +3452,17 @@ x_1 = lean_mk_string_unchecked("next", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12() { _start: { lean_object* x_1; @@ -3724,17 +3470,17 @@ x_1 = lean_mk_string_unchecked("root", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14() { _start: { lean_object* x_1; @@ -3742,17 +3488,17 @@ x_1 = lean_mk_string_unchecked("congr", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16() { _start: { lean_object* x_1; lean_object* x_2; @@ -3761,7 +3507,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17() { _start: { lean_object* x_1; @@ -3769,17 +3515,17 @@ x_1 = lean_mk_string_unchecked("target\?", 7, 7); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19() { _start: { lean_object* x_1; lean_object* x_2; @@ -3788,7 +3534,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20() { _start: { lean_object* x_1; @@ -3796,17 +3542,17 @@ x_1 = lean_mk_string_unchecked("proof\?", 6, 6); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22() { _start: { lean_object* x_1; lean_object* x_2; @@ -3815,7 +3561,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23() { _start: { lean_object* x_1; @@ -3823,17 +3569,17 @@ x_1 = lean_mk_string_unchecked("flipped", 7, 7); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25() { _start: { lean_object* x_1; @@ -3841,17 +3587,17 @@ x_1 = lean_mk_string_unchecked("size", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27() { _start: { lean_object* x_1; @@ -3859,17 +3605,17 @@ x_1 = lean_mk_string_unchecked("interpreted", 11, 11); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29() { _start: { lean_object* x_1; lean_object* x_2; @@ -3878,7 +3624,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30() { _start: { lean_object* x_1; @@ -3886,17 +3632,17 @@ x_1 = lean_mk_string_unchecked("ctor", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32() { _start: { lean_object* x_1; @@ -3904,17 +3650,17 @@ x_1 = lean_mk_string_unchecked("hasLambdas", 10, 10); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34() { _start: { lean_object* x_1; lean_object* x_2; @@ -3923,7 +3669,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35() { _start: { lean_object* x_1; @@ -3931,17 +3677,17 @@ x_1 = lean_mk_string_unchecked("heqProofs", 9, 9); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37() { _start: { lean_object* x_1; lean_object* x_2; @@ -3950,7 +3696,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38() { _start: { lean_object* x_1; @@ -3958,17 +3704,17 @@ x_1 = lean_mk_string_unchecked("idx", 3, 3); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40() { _start: { lean_object* x_1; lean_object* x_2; @@ -3977,7 +3723,7 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41() { _start: { lean_object* x_1; @@ -3985,17 +3731,17 @@ x_1 = lean_mk_string_unchecked("generation", 10, 10); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43() { _start: { lean_object* x_1; @@ -4003,17 +3749,17 @@ x_1 = lean_mk_string_unchecked("mt", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45() { _start: { lean_object* x_1; lean_object* x_2; @@ -4022,7 +3768,25 @@ x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("offset\?", 7, 7); +return x_1; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48() { _start: { lean_object* x_1; @@ -4030,35 +3794,35 @@ x_1 = lean_mk_string_unchecked("{ ", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48; x_2 = lean_string_length(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49; x_2 = lean_nat_to_int(x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52() { _start: { lean_object* x_1; @@ -4066,17 +3830,17 @@ x_1 = lean_mk_string_unchecked(" }", 2, 2); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54() { _start: { lean_object* x_1; @@ -4084,17 +3848,17 @@ x_1 = lean_mk_string_unchecked("false", 5, 5); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56() { _start: { lean_object* x_1; @@ -4102,25 +3866,25 @@ x_1 = lean_mk_string_unchecked("true", 4, 4); return x_1; } } -static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55() { +static lean_object* _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54; +x_1 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56; x_2 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560_(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445_(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; uint8_t x_80; uint8_t x_81; uint8_t x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; x_3 = lean_ctor_get(x_1, 0); lean_inc(x_3); x_4 = lean_unsigned_to_nat(0u); x_5 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3036_(x_3, x_4); -x_6 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7; +x_6 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); @@ -4128,11 +3892,11 @@ x_8 = 0; x_9 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_9, 0, x_7); lean_ctor_set_uint8(x_9, sizeof(void*)*1, x_8); -x_10 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6; +x_10 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6; x_11 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_11, 0, x_10); lean_ctor_set(x_11, 1, x_9); -x_12 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9; +x_12 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9; x_13 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_13, 0, x_11); lean_ctor_set(x_13, 1, x_12); @@ -4140,11 +3904,11 @@ x_14 = lean_box(1); x_15 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_15, 0, x_13); lean_ctor_set(x_15, 1, x_14); -x_16 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11; +x_16 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11; x_17 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); -x_18 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5; +x_18 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5; x_19 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); @@ -4166,7 +3930,7 @@ lean_ctor_set(x_25, 1, x_12); x_26 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_26, 0, x_25); lean_ctor_set(x_26, 1, x_14); -x_27 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13; +x_27 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13; x_28 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_28, 0, x_26); lean_ctor_set(x_28, 1, x_27); @@ -4191,7 +3955,7 @@ lean_ctor_set(x_35, 1, x_12); x_36 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_36, 0, x_35); lean_ctor_set(x_36, 1, x_14); -x_37 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15; +x_37 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15; x_38 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_38, 0, x_36); lean_ctor_set(x_38, 1, x_37); @@ -4201,7 +3965,7 @@ lean_ctor_set(x_39, 1, x_18); x_40 = lean_ctor_get(x_1, 3); lean_inc(x_40); x_41 = l___private_Lean_Expr_0__Lean_reprExpr____x40_Lean_Expr___hyg_3036_(x_40, x_4); -x_42 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16; +x_42 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16; x_43 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_41); @@ -4217,7 +3981,7 @@ lean_ctor_set(x_46, 1, x_12); x_47 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_47, 0, x_46); lean_ctor_set(x_47, 1, x_14); -x_48 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18; +x_48 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18; x_49 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_49, 0, x_47); lean_ctor_set(x_49, 1, x_48); @@ -4227,7 +3991,7 @@ lean_ctor_set(x_50, 1, x_18); x_51 = lean_ctor_get(x_1, 4); lean_inc(x_51); x_52 = l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_46____spec__1(x_51, x_4); -x_53 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19; +x_53 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19; x_54 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_54, 0, x_53); lean_ctor_set(x_54, 1, x_52); @@ -4243,7 +4007,7 @@ lean_ctor_set(x_57, 1, x_12); x_58 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_58, 0, x_57); lean_ctor_set(x_58, 1, x_14); -x_59 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21; +x_59 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21; x_60 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_60, 0, x_58); lean_ctor_set(x_60, 1, x_59); @@ -4253,7 +4017,7 @@ lean_ctor_set(x_61, 1, x_18); x_62 = lean_ctor_get(x_1, 5); lean_inc(x_62); x_63 = l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_46____spec__1(x_62, x_4); -x_64 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22; +x_64 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22; x_65 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_65, 0, x_64); lean_ctor_set(x_65, 1, x_63); @@ -4269,14 +4033,14 @@ lean_ctor_set(x_68, 1, x_12); x_69 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_69, 0, x_68); lean_ctor_set(x_69, 1, x_14); -x_70 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24; +x_70 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24; x_71 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_71, 0, x_69); lean_ctor_set(x_71, 1, x_70); x_72 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_72, 0, x_71); lean_ctor_set(x_72, 1, x_18); -x_73 = lean_ctor_get_uint8(x_1, sizeof(void*)*10); +x_73 = lean_ctor_get_uint8(x_1, sizeof(void*)*11); x_74 = lean_ctor_get(x_1, 6); lean_inc(x_74); x_75 = l___private_Init_Data_Repr_0__Nat_reprFast(x_74); @@ -4288,16 +4052,16 @@ lean_ctor_set(x_77, 1, x_76); x_78 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_78, 0, x_77); lean_ctor_set_uint8(x_78, sizeof(void*)*1, x_8); -x_79 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 1); -x_80 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 2); -x_81 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 3); -x_82 = lean_ctor_get_uint8(x_1, sizeof(void*)*10 + 4); +x_79 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 1); +x_80 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 2); +x_81 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 3); +x_82 = lean_ctor_get_uint8(x_1, sizeof(void*)*11 + 4); x_83 = lean_ctor_get(x_1, 7); lean_inc(x_83); x_84 = l___private_Init_Data_Repr_0__Nat_reprFast(x_83); x_85 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_85, 0, x_84); -x_86 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40; +x_86 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40; x_87 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_87, 0, x_86); lean_ctor_set(x_87, 1, x_85); @@ -4309,7 +4073,7 @@ lean_inc(x_89); x_90 = l___private_Init_Data_Repr_0__Nat_reprFast(x_89); x_91 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_91, 0, x_90); -x_92 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34; +x_92 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34; x_93 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_93, 0, x_92); lean_ctor_set(x_93, 1, x_91); @@ -4318,281 +4082,306 @@ lean_ctor_set(x_94, 0, x_93); lean_ctor_set_uint8(x_94, sizeof(void*)*1, x_8); x_95 = lean_ctor_get(x_1, 9); lean_inc(x_95); -lean_dec(x_1); x_96 = l___private_Init_Data_Repr_0__Nat_reprFast(x_95); x_97 = lean_alloc_ctor(3, 1, 0); lean_ctor_set(x_97, 0, x_96); -x_98 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45; +x_98 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45; x_99 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_99, 0, x_98); lean_ctor_set(x_99, 1, x_97); x_100 = lean_alloc_ctor(6, 1, 1); lean_ctor_set(x_100, 0, x_99); lean_ctor_set_uint8(x_100, sizeof(void*)*1, x_8); +x_101 = lean_ctor_get(x_1, 10); +lean_inc(x_101); +lean_dec(x_1); +x_102 = l_Option_repr___at___private_Lean_Meta_Transform_0__Lean_reprTransformStep____x40_Lean_Meta_Transform___hyg_46____spec__1(x_101, x_4); +x_103 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_103, 0, x_53); +lean_ctor_set(x_103, 1, x_102); +x_104 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set_uint8(x_104, sizeof(void*)*1, x_8); if (x_73 == 0) { -lean_object* x_187; -x_187 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -x_101 = x_187; -goto block_186; +lean_object* x_197; +x_197 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; +x_105 = x_197; +goto block_196; } else { -lean_object* x_188; -x_188 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; -x_101 = x_188; -goto block_186; +lean_object* x_198; +x_198 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; +x_105 = x_198; +goto block_196; } -block_186: +block_196: { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_102 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_102, 0, x_53); -lean_ctor_set(x_102, 1, x_101); -x_103 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_103, 0, x_102); -lean_ctor_set_uint8(x_103, sizeof(void*)*1, x_8); -x_104 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_104, 0, x_72); -lean_ctor_set(x_104, 1, x_103); -x_105 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_105, 0, x_104); -lean_ctor_set(x_105, 1, x_12); -x_106 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_106, 0, x_105); -lean_ctor_set(x_106, 1, x_14); -x_107 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26; +lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; +x_106 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_106, 0, x_53); +lean_ctor_set(x_106, 1, x_105); +x_107 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_107, 0, x_106); +lean_ctor_set_uint8(x_107, sizeof(void*)*1, x_8); x_108 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_108, 0, x_106); +lean_ctor_set(x_108, 0, x_72); lean_ctor_set(x_108, 1, x_107); x_109 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_18); +lean_ctor_set(x_109, 1, x_12); x_110 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_78); -x_111 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_111, 0, x_110); -lean_ctor_set(x_111, 1, x_12); +lean_ctor_set(x_110, 1, x_14); +x_111 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26; x_112 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_112, 0, x_111); -lean_ctor_set(x_112, 1, x_14); -x_113 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28; +lean_ctor_set(x_112, 0, x_110); +lean_ctor_set(x_112, 1, x_111); +x_113 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_113, 0, x_112); +lean_ctor_set(x_113, 1, x_18); x_114 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_114, 0, x_112); -lean_ctor_set(x_114, 1, x_113); +lean_ctor_set(x_114, 0, x_113); +lean_ctor_set(x_114, 1, x_78); x_115 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_115, 0, x_114); -lean_ctor_set(x_115, 1, x_18); +lean_ctor_set(x_115, 1, x_12); +x_116 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_116, 0, x_115); +lean_ctor_set(x_116, 1, x_14); +x_117 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28; +x_118 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_118, 0, x_116); +lean_ctor_set(x_118, 1, x_117); +x_119 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_119, 0, x_118); +lean_ctor_set(x_119, 1, x_18); if (x_79 == 0) { -lean_object* x_184; -x_184 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -x_116 = x_184; -goto block_183; +lean_object* x_194; +x_194 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; +x_120 = x_194; +goto block_193; } else { -lean_object* x_185; -x_185 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; -x_116 = x_185; -goto block_183; -} -block_183: -{ -lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -x_117 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29; -x_118 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_118, 0, x_117); -lean_ctor_set(x_118, 1, x_116); -x_119 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set_uint8(x_119, sizeof(void*)*1, x_8); -x_120 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_120, 0, x_115); -lean_ctor_set(x_120, 1, x_119); -x_121 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_121, 0, x_120); -lean_ctor_set(x_121, 1, x_12); -x_122 = lean_alloc_ctor(5, 2, 0); +lean_object* x_195; +x_195 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; +x_120 = x_195; +goto block_193; +} +block_193: +{ +lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_121 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29; +x_122 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_122, 0, x_121); -lean_ctor_set(x_122, 1, x_14); -x_123 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31; +lean_ctor_set(x_122, 1, x_120); +x_123 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_123, 0, x_122); +lean_ctor_set_uint8(x_123, sizeof(void*)*1, x_8); x_124 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_124, 0, x_122); +lean_ctor_set(x_124, 0, x_119); lean_ctor_set(x_124, 1, x_123); x_125 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_125, 0, x_124); -lean_ctor_set(x_125, 1, x_18); +lean_ctor_set(x_125, 1, x_12); +x_126 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_126, 0, x_125); +lean_ctor_set(x_126, 1, x_14); +x_127 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31; +x_128 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_128, 0, x_126); +lean_ctor_set(x_128, 1, x_127); +x_129 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_129, 0, x_128); +lean_ctor_set(x_129, 1, x_18); if (x_80 == 0) { -lean_object* x_181; -x_181 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -x_126 = x_181; -goto block_180; +lean_object* x_191; +x_191 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; +x_130 = x_191; +goto block_190; } else { -lean_object* x_182; -x_182 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; -x_126 = x_182; -goto block_180; +lean_object* x_192; +x_192 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; +x_130 = x_192; +goto block_190; } -block_180: +block_190: { -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_127 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_127, 0, x_6); -lean_ctor_set(x_127, 1, x_126); -x_128 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_128, 0, x_127); -lean_ctor_set_uint8(x_128, sizeof(void*)*1, x_8); -x_129 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_129, 0, x_125); -lean_ctor_set(x_129, 1, x_128); -x_130 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_130, 0, x_129); -lean_ctor_set(x_130, 1, x_12); -x_131 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_131, 0, x_130); -lean_ctor_set(x_131, 1, x_14); -x_132 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33; +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; +x_131 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_131, 0, x_6); +lean_ctor_set(x_131, 1, x_130); +x_132 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_132, 0, x_131); +lean_ctor_set_uint8(x_132, sizeof(void*)*1, x_8); x_133 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_133, 0, x_131); +lean_ctor_set(x_133, 0, x_129); lean_ctor_set(x_133, 1, x_132); x_134 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_134, 0, x_133); -lean_ctor_set(x_134, 1, x_18); +lean_ctor_set(x_134, 1, x_12); +x_135 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_135, 0, x_134); +lean_ctor_set(x_135, 1, x_14); +x_136 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33; +x_137 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_137, 0, x_135); +lean_ctor_set(x_137, 1, x_136); +x_138 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_138, 0, x_137); +lean_ctor_set(x_138, 1, x_18); if (x_81 == 0) { -lean_object* x_178; -x_178 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -x_135 = x_178; -goto block_177; +lean_object* x_188; +x_188 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; +x_139 = x_188; +goto block_187; } else { -lean_object* x_179; -x_179 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; -x_135 = x_179; -goto block_177; +lean_object* x_189; +x_189 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; +x_139 = x_189; +goto block_187; } -block_177: +block_187: { -lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; -x_136 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_136, 0, x_92); -lean_ctor_set(x_136, 1, x_135); -x_137 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set_uint8(x_137, sizeof(void*)*1, x_8); -x_138 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_138, 0, x_134); -lean_ctor_set(x_138, 1, x_137); -x_139 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_139, 0, x_138); -lean_ctor_set(x_139, 1, x_12); -x_140 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_140, 0, x_139); -lean_ctor_set(x_140, 1, x_14); -x_141 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36; +lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; +x_140 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_140, 0, x_92); +lean_ctor_set(x_140, 1, x_139); +x_141 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_141, 0, x_140); +lean_ctor_set_uint8(x_141, sizeof(void*)*1, x_8); x_142 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_142, 0, x_140); +lean_ctor_set(x_142, 0, x_138); lean_ctor_set(x_142, 1, x_141); x_143 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_143, 0, x_142); -lean_ctor_set(x_143, 1, x_18); +lean_ctor_set(x_143, 1, x_12); +x_144 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_144, 0, x_143); +lean_ctor_set(x_144, 1, x_14); +x_145 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36; +x_146 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_146, 0, x_144); +lean_ctor_set(x_146, 1, x_145); +x_147 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_147, 0, x_146); +lean_ctor_set(x_147, 1, x_18); if (x_82 == 0) { -lean_object* x_175; -x_175 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53; -x_144 = x_175; -goto block_174; +lean_object* x_185; +x_185 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55; +x_148 = x_185; +goto block_184; } else { -lean_object* x_176; -x_176 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55; -x_144 = x_176; -goto block_174; +lean_object* x_186; +x_186 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57; +x_148 = x_186; +goto block_184; } -block_174: +block_184: { -lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; -x_145 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37; -x_146 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_146, 0, x_145); -lean_ctor_set(x_146, 1, x_144); -x_147 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_147, 0, x_146); -lean_ctor_set_uint8(x_147, sizeof(void*)*1, x_8); -x_148 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_148, 0, x_143); -lean_ctor_set(x_148, 1, x_147); -x_149 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_149, 0, x_148); -lean_ctor_set(x_149, 1, x_12); -x_150 = lean_alloc_ctor(5, 2, 0); +lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; +x_149 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37; +x_150 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_150, 0, x_149); -lean_ctor_set(x_150, 1, x_14); -x_151 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39; +lean_ctor_set(x_150, 1, x_148); +x_151 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_151, 0, x_150); +lean_ctor_set_uint8(x_151, sizeof(void*)*1, x_8); x_152 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_152, 0, x_150); +lean_ctor_set(x_152, 0, x_147); lean_ctor_set(x_152, 1, x_151); x_153 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_153, 0, x_152); -lean_ctor_set(x_153, 1, x_18); +lean_ctor_set(x_153, 1, x_12); x_154 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_154, 0, x_153); -lean_ctor_set(x_154, 1, x_88); -x_155 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_155, 0, x_154); -lean_ctor_set(x_155, 1, x_12); +lean_ctor_set(x_154, 1, x_14); +x_155 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39; x_156 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_14); -x_157 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42; +lean_ctor_set(x_156, 0, x_154); +lean_ctor_set(x_156, 1, x_155); +x_157 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_157, 0, x_156); +lean_ctor_set(x_157, 1, x_18); x_158 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_158, 0, x_156); -lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 0, x_157); +lean_ctor_set(x_158, 1, x_88); x_159 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_159, 0, x_158); -lean_ctor_set(x_159, 1, x_18); +lean_ctor_set(x_159, 1, x_12); x_160 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_160, 0, x_159); -lean_ctor_set(x_160, 1, x_94); -x_161 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_161, 0, x_160); -lean_ctor_set(x_161, 1, x_12); +lean_ctor_set(x_160, 1, x_14); +x_161 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42; x_162 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_162, 0, x_161); -lean_ctor_set(x_162, 1, x_14); -x_163 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44; +lean_ctor_set(x_162, 0, x_160); +lean_ctor_set(x_162, 1, x_161); +x_163 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_163, 0, x_162); +lean_ctor_set(x_163, 1, x_18); x_164 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_164, 0, x_162); -lean_ctor_set(x_164, 1, x_163); +lean_ctor_set(x_164, 0, x_163); +lean_ctor_set(x_164, 1, x_94); x_165 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_165, 0, x_164); -lean_ctor_set(x_165, 1, x_18); +lean_ctor_set(x_165, 1, x_12); x_166 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_166, 0, x_165); -lean_ctor_set(x_166, 1, x_100); -x_167 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49; +lean_ctor_set(x_166, 1, x_14); +x_167 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44; x_168 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_168, 0, x_167); -lean_ctor_set(x_168, 1, x_166); -x_169 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51; +lean_ctor_set(x_168, 0, x_166); +lean_ctor_set(x_168, 1, x_167); +x_169 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_169, 0, x_168); +lean_ctor_set(x_169, 1, x_18); x_170 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_170, 0, x_168); -lean_ctor_set(x_170, 1, x_169); -x_171 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48; -x_172 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_170, 0, x_169); +lean_ctor_set(x_170, 1, x_100); +x_171 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_171, 0, x_170); +lean_ctor_set(x_171, 1, x_12); +x_172 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_172, 0, x_171); -lean_ctor_set(x_172, 1, x_170); -x_173 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_173, 0, x_172); -lean_ctor_set_uint8(x_173, sizeof(void*)*1, x_8); -return x_173; +lean_ctor_set(x_172, 1, x_14); +x_173 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47; +x_174 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_174, 0, x_172); +lean_ctor_set(x_174, 1, x_173); +x_175 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_175, 0, x_174); +lean_ctor_set(x_175, 1, x_18); +x_176 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_176, 0, x_175); +lean_ctor_set(x_176, 1, x_104); +x_177 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51; +x_178 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_178, 0, x_177); +lean_ctor_set(x_178, 1, x_176); +x_179 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53; +x_180 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_180, 0, x_178); +lean_ctor_set(x_180, 1, x_179); +x_181 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50; +x_182 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_182, 0, x_181); +lean_ctor_set(x_182, 1, x_180); +x_183 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_183, 0, x_182); +lean_ctor_set_uint8(x_183, sizeof(void*)*1, x_8); +return x_183; } } } @@ -4600,11 +4389,11 @@ return x_173; } } } -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560_(x_1, x_2); +x_3 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445_(x_1, x_2); lean_dec(x_2); return x_3; } @@ -4613,7 +4402,7 @@ static lean_object* _init_l_Lean_Meta_Grind_instReprENode___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____boxed), 2, 0); return x_1; } } @@ -4645,90 +4434,34 @@ x_3 = lean_box(x_2); return x_3; } } -LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(lean_object* x_1) { +LEAN_EXPORT uint64_t l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1(lean_object* x_1) { _start: { -size_t x_2; uint64_t x_3; -x_2 = lean_ptr_addr(x_1); -x_3 = lean_usize_to_uint64(x_2); -return x_3; +lean_object* x_2; size_t x_3; uint64_t x_4; +x_2 = lean_ctor_get(x_1, 2); +x_3 = lean_ptr_addr(x_2); +x_4 = lean_usize_to_uint64(x_3); +return x_4; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1___boxed(lean_object* x_1) { _start: { uint64_t x_2; lean_object* x_3; -x_2 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_1); +x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1(x_1); lean_dec(x_1); x_3 = lean_box_uint64(x_2); return x_3; } } -LEAN_EXPORT uint64_t l_Lean_Meta_Grind_instHashableENodeKey(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint64_t x_2; -x_2 = l_Lean_Meta_Grind_instHashableENodeKey_unsafe__1(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instHashableENodeKey___boxed(lean_object* x_1) { -_start: -{ -uint64_t x_2; lean_object* x_3; -x_2 = l_Lean_Meta_Grind_instHashableENodeKey(x_1); -lean_dec(x_1); -x_3 = lean_box_uint64(x_2); -return x_3; -} -} -LEAN_EXPORT uint8_t l_Lean_Meta_Grind_instBEqENodeKey(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; -x_3 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_instBEqENodeKey___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint8_t x_3; lean_object* x_4; -x_3 = l_Lean_Meta_Grind_instBEqENodeKey(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; -} -} -LEAN_EXPORT uint64_t l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1(lean_object* x_1) { -_start: -{ -lean_object* x_2; size_t x_3; uint64_t x_4; -x_2 = lean_ctor_get(x_1, 2); -x_3 = lean_ptr_addr(x_2); -x_4 = lean_usize_to_uint64(x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1___boxed(lean_object* x_1) { -_start: -{ -uint64_t x_2; lean_object* x_3; -x_2 = l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot_unsafe__1(x_1); -lean_dec(x_1); -x_3 = lean_box_uint64(x_2); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_findAtAux___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; uint8_t x_7; -x_6 = lean_array_get_size(x_1); -x_7 = lean_nat_dec_lt(x_4, x_6); -lean_dec(x_6); -if (x_7 == 0) +lean_object* x_6; uint8_t x_7; +x_6 = lean_array_get_size(x_1); +x_7 = lean_nat_dec_lt(x_4, x_6); +lean_dec(x_6); +if (x_7 == 0) { lean_object* x_8; lean_dec(x_4); @@ -5130,8 +4863,8 @@ static lean_object* _init_l_Lean_Meta_Grind_congrHash___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; x_3 = l_Lean_Meta_Grind_congrHash___closed__1; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); return x_4; @@ -6195,11 +5928,29 @@ x_1 = l_Lean_Meta_Grind_instInhabitedNewFact___closed__1; return x_1; } } +static lean_object* _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); +return x_1; +} +} +static lean_object* _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} static lean_object* _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1() { _start: { lean_object* x_1; -x_1 = l_Lean_Meta_Grind_canon___closed__2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; return x_1; } } @@ -6207,7 +5958,7 @@ static lean_object* _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_in _start: { lean_object* x_1; -x_1 = l_Lean_Meta_Grind_canon___closed__2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; return x_1; } } @@ -6215,7 +5966,7 @@ static lean_object* _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_in _start: { lean_object* x_1; -x_1 = l_Lean_Meta_Grind_canon___closed__2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; return x_1; } } @@ -6223,22 +5974,34 @@ static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__1() { _start: { lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; +x_2 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(0u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__3() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +x_1 = l_Lean_Meta_Grind_instInhabitedGoal___closed__2; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static size_t _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__3() { +static size_t _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__4() { _start: { lean_object* x_1; size_t x_2; @@ -6247,14 +6010,14 @@ x_2 = lean_usize_of_nat(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__4() { +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; size_t x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_instInhabitedGoal___closed__2; -x_2 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +x_1 = l_Lean_Meta_Grind_instInhabitedGoal___closed__3; +x_2 = l_Lean_Meta_Grind_instInhabitedGoal___closed__2; x_3 = lean_unsigned_to_nat(0u); -x_4 = l_Lean_Meta_Grind_instInhabitedGoal___closed__3; +x_4 = l_Lean_Meta_Grind_instInhabitedGoal___closed__4; x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -6264,11 +6027,28 @@ lean_ctor_set_usize(x_5, 4, x_4); return x_5; } } -static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__5() { +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_instInhabitedGoal___closed__5; +x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; +x_3 = lean_alloc_ctor(0, 7, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +lean_ctor_set(x_3, 2, x_2); +lean_ctor_set(x_3, 3, x_2); +lean_ctor_set(x_3, 4, x_1); +lean_ctor_set(x_3, 5, x_1); +lean_ctor_set(x_3, 6, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_canon___closed__2; +x_1 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; x_2 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedEMatchTheorems___spec__1; x_3 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_3, 0, x_1); @@ -6277,7 +6057,7 @@ lean_ctor_set(x_3, 2, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__6() { +static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__8() { _start: { lean_object* x_1; @@ -6288,43 +6068,48 @@ return x_1; static lean_object* _init_l_Lean_Meta_Grind_instInhabitedGoal() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_1 = lean_box(0); x_2 = lean_box(0); -x_3 = l_Lean_Meta_Grind_canon___closed__2; -x_4 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1; -x_5 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; -x_6 = 0; -x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Lean_Meta_Grind_instInhabitedGoal___closed__4; -x_9 = l_Lean_Meta_Grind_instInhabitedGoal___closed__5; -x_10 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2; -x_11 = l_Lean_Meta_Grind_instInhabitedGoal___closed__6; -x_12 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; -x_13 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__3; -x_14 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_14, 0, x_2); -lean_ctor_set(x_14, 1, x_3); -lean_ctor_set(x_14, 2, x_3); -lean_ctor_set(x_14, 3, x_4); -lean_ctor_set(x_14, 4, x_3); -lean_ctor_set(x_14, 5, x_5); -lean_ctor_set(x_14, 6, x_7); -lean_ctor_set(x_14, 7, x_7); -lean_ctor_set(x_14, 8, x_8); -lean_ctor_set(x_14, 9, x_8); -lean_ctor_set(x_14, 10, x_9); -lean_ctor_set(x_14, 11, x_7); -lean_ctor_set(x_14, 12, x_7); -lean_ctor_set(x_14, 13, x_10); -lean_ctor_set(x_14, 14, x_11); -lean_ctor_set(x_14, 15, x_12); -lean_ctor_set(x_14, 16, x_1); -lean_ctor_set(x_14, 17, x_7); -lean_ctor_set(x_14, 18, x_13); -lean_ctor_set(x_14, 19, x_7); -lean_ctor_set_uint8(x_14, sizeof(void*)*20, x_6); -return x_14; +x_3 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +x_4 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2; +x_5 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1; +x_6 = l_Lean_Meta_Grind_instInhabitedGoal___closed__2; +x_7 = 0; +x_8 = lean_unsigned_to_nat(0u); +x_9 = l_Lean_Meta_Grind_instInhabitedGoal___closed__6; +x_10 = l_Lean_Meta_Grind_instInhabitedGoal___closed__5; +x_11 = l_Lean_Meta_Grind_instInhabitedGoal___closed__7; +x_12 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2; +x_13 = l_Lean_Meta_Grind_instInhabitedGoal___closed__8; +x_14 = l_Lean_PersistentHashMap_empty___at_Lean_KeyedDeclsAttribute_instInhabitedExtensionState___spec__1; +x_15 = l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__3; +x_16 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_16, 0, x_2); +lean_ctor_set(x_16, 1, x_3); +lean_ctor_set(x_16, 2, x_4); +lean_ctor_set(x_16, 3, x_4); +lean_ctor_set(x_16, 4, x_5); +lean_ctor_set(x_16, 5, x_4); +lean_ctor_set(x_16, 6, x_6); +lean_ctor_set(x_16, 7, x_8); +lean_ctor_set(x_16, 8, x_8); +lean_ctor_set(x_16, 9, x_9); +lean_ctor_set(x_16, 10, x_10); +lean_ctor_set(x_16, 11, x_10); +lean_ctor_set(x_16, 12, x_11); +lean_ctor_set(x_16, 13, x_8); +lean_ctor_set(x_16, 14, x_8); +lean_ctor_set(x_16, 15, x_12); +lean_ctor_set(x_16, 16, x_13); +lean_ctor_set(x_16, 17, x_14); +lean_ctor_set(x_16, 18, x_1); +lean_ctor_set(x_16, 19, x_8); +lean_ctor_set(x_16, 20, x_15); +lean_ctor_set(x_16, 21, x_8); +lean_ctor_set(x_16, 22, x_10); +lean_ctor_set_uint8(x_16, sizeof(void*)*23, x_7); +return x_16; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_admit(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { @@ -6770,80 +6555,531 @@ lean_dec(x_2); return x_10; } } -LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_8, 2); -x_12 = l_Lean_isTracingEnabledForCore(x_1, x_11, x_10); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_st_ref_take(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -return x_12; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +lean_ctor_set(x_12, 1, x_16); +x_17 = lean_st_ref_set(x_2, x_12, x_13); +x_18 = lean_ctor_get(x_17, 1); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lean_Meta_Grind_Canon_canon(x_1, x_15, x_6, x_7, x_8, x_9, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); +lean_dec(x_19); +x_22 = lean_ctor_get(x_20, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_20, 1); +lean_inc(x_23); +lean_dec(x_20); +x_24 = lean_st_ref_take(x_2, x_21); +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +x_26 = lean_ctor_get(x_24, 1); +lean_inc(x_26); +lean_dec(x_24); +x_27 = !lean_is_exclusive(x_25); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_28 = lean_ctor_get(x_25, 1); +lean_dec(x_28); +lean_ctor_set(x_25, 1, x_23); +x_29 = lean_st_ref_set(x_2, x_25, x_26); +x_30 = !lean_is_exclusive(x_29); +if (x_30 == 0) +{ +lean_object* x_31; +x_31 = lean_ctor_get(x_29, 0); +lean_dec(x_31); +lean_ctor_set(x_29, 0, x_22); +return x_29; } else { -lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_12, 0); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_inc(x_14); -lean_dec(x_12); -x_16 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_16, 0, x_14); -lean_ctor_set(x_16, 1, x_15); -return x_16; -} +lean_object* x_32; lean_object* x_33; +x_32 = lean_ctor_get(x_29, 1); +lean_inc(x_32); +lean_dec(x_29); +x_33 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_33, 0, x_22); +lean_ctor_set(x_33, 1, x_32); +return x_33; } } -static double _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__1() { -_start: +else { -lean_object* x_1; uint8_t x_2; double x_3; -x_1 = lean_unsigned_to_nat(0u); -x_2 = 0; -x_3 = l_Float_ofScientific(x_1, x_2, x_1); -return x_3; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; +x_34 = lean_ctor_get(x_25, 0); +x_35 = lean_ctor_get(x_25, 2); +x_36 = lean_ctor_get(x_25, 3); +x_37 = lean_ctor_get(x_25, 4); +x_38 = lean_ctor_get(x_25, 5); +x_39 = lean_ctor_get(x_25, 6); +x_40 = lean_ctor_get_uint8(x_25, sizeof(void*)*23); +x_41 = lean_ctor_get(x_25, 7); +x_42 = lean_ctor_get(x_25, 8); +x_43 = lean_ctor_get(x_25, 9); +x_44 = lean_ctor_get(x_25, 10); +x_45 = lean_ctor_get(x_25, 11); +x_46 = lean_ctor_get(x_25, 12); +x_47 = lean_ctor_get(x_25, 13); +x_48 = lean_ctor_get(x_25, 14); +x_49 = lean_ctor_get(x_25, 15); +x_50 = lean_ctor_get(x_25, 16); +x_51 = lean_ctor_get(x_25, 17); +x_52 = lean_ctor_get(x_25, 18); +x_53 = lean_ctor_get(x_25, 19); +x_54 = lean_ctor_get(x_25, 20); +x_55 = lean_ctor_get(x_25, 21); +x_56 = lean_ctor_get(x_25, 22); +lean_inc(x_56); +lean_inc(x_55); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_25); +x_57 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_57, 0, x_34); +lean_ctor_set(x_57, 1, x_23); +lean_ctor_set(x_57, 2, x_35); +lean_ctor_set(x_57, 3, x_36); +lean_ctor_set(x_57, 4, x_37); +lean_ctor_set(x_57, 5, x_38); +lean_ctor_set(x_57, 6, x_39); +lean_ctor_set(x_57, 7, x_41); +lean_ctor_set(x_57, 8, x_42); +lean_ctor_set(x_57, 9, x_43); +lean_ctor_set(x_57, 10, x_44); +lean_ctor_set(x_57, 11, x_45); +lean_ctor_set(x_57, 12, x_46); +lean_ctor_set(x_57, 13, x_47); +lean_ctor_set(x_57, 14, x_48); +lean_ctor_set(x_57, 15, x_49); +lean_ctor_set(x_57, 16, x_50); +lean_ctor_set(x_57, 17, x_51); +lean_ctor_set(x_57, 18, x_52); +lean_ctor_set(x_57, 19, x_53); +lean_ctor_set(x_57, 20, x_54); +lean_ctor_set(x_57, 21, x_55); +lean_ctor_set(x_57, 22, x_56); +lean_ctor_set_uint8(x_57, sizeof(void*)*23, x_40); +x_58 = lean_st_ref_set(x_2, x_57, x_26); +x_59 = lean_ctor_get(x_58, 1); +lean_inc(x_59); +if (lean_is_exclusive(x_58)) { + lean_ctor_release(x_58, 0); + lean_ctor_release(x_58, 1); + x_60 = x_58; +} else { + lean_dec_ref(x_58); + x_60 = lean_box(0); } +if (lean_is_scalar(x_60)) { + x_61 = lean_alloc_ctor(0, 2, 0); +} else { + x_61 = x_60; } -static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__2() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("", 0, 0); -return x_1; +lean_ctor_set(x_61, 0, x_22); +lean_ctor_set(x_61, 1, x_59); +return x_61; } } -static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__3() { -_start: +else { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; +uint8_t x_62; +x_62 = !lean_is_exclusive(x_19); +if (x_62 == 0) +{ +return x_19; +} +else +{ +lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_63 = lean_ctor_get(x_19, 0); +x_64 = lean_ctor_get(x_19, 1); +lean_inc(x_64); +lean_inc(x_63); +lean_dec(x_19); +x_65 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_65, 0, x_63); +lean_ctor_set(x_65, 1, x_64); +return x_65; } } -LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +} +else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_12 = lean_ctor_get(x_9, 5); -x_13 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_7, x_8, x_9, x_10, x_11); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_st_ref_take(x_10, x_15); -x_17 = lean_ctor_get(x_16, 0); -lean_inc(x_17); -x_18 = lean_ctor_get(x_17, 3); -lean_inc(x_18); -x_19 = !lean_is_exclusive(x_16); -if (x_19 == 0) +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_66 = lean_ctor_get(x_12, 0); +x_67 = lean_ctor_get(x_12, 1); +x_68 = lean_ctor_get(x_12, 2); +x_69 = lean_ctor_get(x_12, 3); +x_70 = lean_ctor_get(x_12, 4); +x_71 = lean_ctor_get(x_12, 5); +x_72 = lean_ctor_get(x_12, 6); +x_73 = lean_ctor_get_uint8(x_12, sizeof(void*)*23); +x_74 = lean_ctor_get(x_12, 7); +x_75 = lean_ctor_get(x_12, 8); +x_76 = lean_ctor_get(x_12, 9); +x_77 = lean_ctor_get(x_12, 10); +x_78 = lean_ctor_get(x_12, 11); +x_79 = lean_ctor_get(x_12, 12); +x_80 = lean_ctor_get(x_12, 13); +x_81 = lean_ctor_get(x_12, 14); +x_82 = lean_ctor_get(x_12, 15); +x_83 = lean_ctor_get(x_12, 16); +x_84 = lean_ctor_get(x_12, 17); +x_85 = lean_ctor_get(x_12, 18); +x_86 = lean_ctor_get(x_12, 19); +x_87 = lean_ctor_get(x_12, 20); +x_88 = lean_ctor_get(x_12, 21); +x_89 = lean_ctor_get(x_12, 22); +lean_inc(x_89); +lean_inc(x_88); +lean_inc(x_87); +lean_inc(x_86); +lean_inc(x_85); +lean_inc(x_84); +lean_inc(x_83); +lean_inc(x_82); +lean_inc(x_81); +lean_inc(x_80); +lean_inc(x_79); +lean_inc(x_78); +lean_inc(x_77); +lean_inc(x_76); +lean_inc(x_75); +lean_inc(x_74); +lean_inc(x_72); +lean_inc(x_71); +lean_inc(x_70); +lean_inc(x_69); +lean_inc(x_68); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_12); +x_90 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +x_91 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_91, 0, x_66); +lean_ctor_set(x_91, 1, x_90); +lean_ctor_set(x_91, 2, x_68); +lean_ctor_set(x_91, 3, x_69); +lean_ctor_set(x_91, 4, x_70); +lean_ctor_set(x_91, 5, x_71); +lean_ctor_set(x_91, 6, x_72); +lean_ctor_set(x_91, 7, x_74); +lean_ctor_set(x_91, 8, x_75); +lean_ctor_set(x_91, 9, x_76); +lean_ctor_set(x_91, 10, x_77); +lean_ctor_set(x_91, 11, x_78); +lean_ctor_set(x_91, 12, x_79); +lean_ctor_set(x_91, 13, x_80); +lean_ctor_set(x_91, 14, x_81); +lean_ctor_set(x_91, 15, x_82); +lean_ctor_set(x_91, 16, x_83); +lean_ctor_set(x_91, 17, x_84); +lean_ctor_set(x_91, 18, x_85); +lean_ctor_set(x_91, 19, x_86); +lean_ctor_set(x_91, 20, x_87); +lean_ctor_set(x_91, 21, x_88); +lean_ctor_set(x_91, 22, x_89); +lean_ctor_set_uint8(x_91, sizeof(void*)*23, x_73); +x_92 = lean_st_ref_set(x_2, x_91, x_13); +x_93 = lean_ctor_get(x_92, 1); +lean_inc(x_93); +lean_dec(x_92); +x_94 = l_Lean_Meta_Grind_Canon_canon(x_1, x_67, x_6, x_7, x_8, x_9, x_93); +if (lean_obj_tag(x_94) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_ctor_get(x_16, 1); +lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; uint8_t x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; +x_95 = lean_ctor_get(x_94, 0); +lean_inc(x_95); +x_96 = lean_ctor_get(x_94, 1); +lean_inc(x_96); +lean_dec(x_94); +x_97 = lean_ctor_get(x_95, 0); +lean_inc(x_97); +x_98 = lean_ctor_get(x_95, 1); +lean_inc(x_98); +lean_dec(x_95); +x_99 = lean_st_ref_take(x_2, x_96); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +lean_dec(x_99); +x_102 = lean_ctor_get(x_100, 0); +lean_inc(x_102); +x_103 = lean_ctor_get(x_100, 2); +lean_inc(x_103); +x_104 = lean_ctor_get(x_100, 3); +lean_inc(x_104); +x_105 = lean_ctor_get(x_100, 4); +lean_inc(x_105); +x_106 = lean_ctor_get(x_100, 5); +lean_inc(x_106); +x_107 = lean_ctor_get(x_100, 6); +lean_inc(x_107); +x_108 = lean_ctor_get_uint8(x_100, sizeof(void*)*23); +x_109 = lean_ctor_get(x_100, 7); +lean_inc(x_109); +x_110 = lean_ctor_get(x_100, 8); +lean_inc(x_110); +x_111 = lean_ctor_get(x_100, 9); +lean_inc(x_111); +x_112 = lean_ctor_get(x_100, 10); +lean_inc(x_112); +x_113 = lean_ctor_get(x_100, 11); +lean_inc(x_113); +x_114 = lean_ctor_get(x_100, 12); +lean_inc(x_114); +x_115 = lean_ctor_get(x_100, 13); +lean_inc(x_115); +x_116 = lean_ctor_get(x_100, 14); +lean_inc(x_116); +x_117 = lean_ctor_get(x_100, 15); +lean_inc(x_117); +x_118 = lean_ctor_get(x_100, 16); +lean_inc(x_118); +x_119 = lean_ctor_get(x_100, 17); +lean_inc(x_119); +x_120 = lean_ctor_get(x_100, 18); +lean_inc(x_120); +x_121 = lean_ctor_get(x_100, 19); +lean_inc(x_121); +x_122 = lean_ctor_get(x_100, 20); +lean_inc(x_122); +x_123 = lean_ctor_get(x_100, 21); +lean_inc(x_123); +x_124 = lean_ctor_get(x_100, 22); +lean_inc(x_124); +if (lean_is_exclusive(x_100)) { + lean_ctor_release(x_100, 0); + lean_ctor_release(x_100, 1); + lean_ctor_release(x_100, 2); + lean_ctor_release(x_100, 3); + lean_ctor_release(x_100, 4); + lean_ctor_release(x_100, 5); + lean_ctor_release(x_100, 6); + lean_ctor_release(x_100, 7); + lean_ctor_release(x_100, 8); + lean_ctor_release(x_100, 9); + lean_ctor_release(x_100, 10); + lean_ctor_release(x_100, 11); + lean_ctor_release(x_100, 12); + lean_ctor_release(x_100, 13); + lean_ctor_release(x_100, 14); + lean_ctor_release(x_100, 15); + lean_ctor_release(x_100, 16); + lean_ctor_release(x_100, 17); + lean_ctor_release(x_100, 18); + lean_ctor_release(x_100, 19); + lean_ctor_release(x_100, 20); + lean_ctor_release(x_100, 21); + lean_ctor_release(x_100, 22); + x_125 = x_100; +} else { + lean_dec_ref(x_100); + x_125 = lean_box(0); +} +if (lean_is_scalar(x_125)) { + x_126 = lean_alloc_ctor(0, 23, 1); +} else { + x_126 = x_125; +} +lean_ctor_set(x_126, 0, x_102); +lean_ctor_set(x_126, 1, x_98); +lean_ctor_set(x_126, 2, x_103); +lean_ctor_set(x_126, 3, x_104); +lean_ctor_set(x_126, 4, x_105); +lean_ctor_set(x_126, 5, x_106); +lean_ctor_set(x_126, 6, x_107); +lean_ctor_set(x_126, 7, x_109); +lean_ctor_set(x_126, 8, x_110); +lean_ctor_set(x_126, 9, x_111); +lean_ctor_set(x_126, 10, x_112); +lean_ctor_set(x_126, 11, x_113); +lean_ctor_set(x_126, 12, x_114); +lean_ctor_set(x_126, 13, x_115); +lean_ctor_set(x_126, 14, x_116); +lean_ctor_set(x_126, 15, x_117); +lean_ctor_set(x_126, 16, x_118); +lean_ctor_set(x_126, 17, x_119); +lean_ctor_set(x_126, 18, x_120); +lean_ctor_set(x_126, 19, x_121); +lean_ctor_set(x_126, 20, x_122); +lean_ctor_set(x_126, 21, x_123); +lean_ctor_set(x_126, 22, x_124); +lean_ctor_set_uint8(x_126, sizeof(void*)*23, x_108); +x_127 = lean_st_ref_set(x_2, x_126, x_101); +x_128 = lean_ctor_get(x_127, 1); +lean_inc(x_128); +if (lean_is_exclusive(x_127)) { + lean_ctor_release(x_127, 0); + lean_ctor_release(x_127, 1); + x_129 = x_127; +} else { + lean_dec_ref(x_127); + x_129 = lean_box(0); +} +if (lean_is_scalar(x_129)) { + x_130 = lean_alloc_ctor(0, 2, 0); +} else { + x_130 = x_129; +} +lean_ctor_set(x_130, 0, x_97); +lean_ctor_set(x_130, 1, x_128); +return x_130; +} +else +{ +lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; +x_131 = lean_ctor_get(x_94, 0); +lean_inc(x_131); +x_132 = lean_ctor_get(x_94, 1); +lean_inc(x_132); +if (lean_is_exclusive(x_94)) { + lean_ctor_release(x_94, 0); + lean_ctor_release(x_94, 1); + x_133 = x_94; +} else { + lean_dec_ref(x_94); + x_133 = lean_box(0); +} +if (lean_is_scalar(x_133)) { + x_134 = lean_alloc_ctor(1, 2, 0); +} else { + x_134 = x_133; +} +lean_ctor_set(x_134, 0, x_131); +lean_ctor_set(x_134, 1, x_132); +return x_134; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_canon___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_canon(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; uint8_t x_13; +x_11 = lean_ctor_get(x_8, 2); +x_12 = l_Lean_isTracingEnabledForCore(x_1, x_11, x_10); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) +{ +return x_12; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_12); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +} +static double _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__1() { +_start: +{ +lean_object* x_1; uint8_t x_2; double x_3; +x_1 = lean_unsigned_to_nat(0u); +x_2 = 0; +x_3 = l_Float_ofScientific(x_1, x_2, x_1); +return x_3; +} +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("", 0, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_9, 5); +x_13 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_2, x_7, x_8, x_9, x_10, x_11); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_st_ref_take(x_10, x_15); +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_17, 3); +lean_inc(x_18); +x_19 = !lean_is_exclusive(x_16); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_20 = lean_ctor_get(x_16, 1); x_21 = lean_ctor_get(x_16, 0); lean_dec(x_21); x_22 = !lean_is_exclusive(x_17); @@ -7237,7 +7473,7 @@ static lean_object* _init_l_Lean_Meta_Grind_updateLastTag___closed__1() { { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } @@ -7761,9 +7997,9 @@ static lean_object* _init_l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______cl _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; x_4 = l_Lean_Meta_Grind_doElemTrace__goal_x5b___x5d_______closed__1; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -8035,7 +8271,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__3; @@ -8063,7 +8299,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__6; @@ -8101,7 +8337,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__10; @@ -8121,7 +8357,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__12; @@ -8149,7 +8385,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__15; @@ -8169,7 +8405,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__17; @@ -8224,7 +8460,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__23; @@ -8252,7 +8488,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__26; @@ -8272,7 +8508,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__28; @@ -8300,7 +8536,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__31; @@ -8328,7 +8564,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__34; @@ -8365,7 +8601,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__38; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -8423,7 +8659,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__44; @@ -8462,9 +8698,9 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; -x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7; -x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; +x_2 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7; +x_3 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__46; x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); return x_5; @@ -8523,7 +8759,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__54; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -8565,7 +8801,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__58; @@ -8606,7 +8842,7 @@ x_13 = lean_alloc_ctor(2, 2, 0); lean_ctor_set(x_13, 0, x_7); lean_ctor_set(x_13, 1, x_12); x_14 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__9; -x_15 = l_Lean_Meta_Grind_instInhabitedGoal___closed__1; +x_15 = l_Lean_Meta_Grind_instInhabitedGoal___closed__2; lean_inc(x_7); x_16 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_16, 0, x_7); @@ -8844,7 +9080,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__1; x_3 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___lambda__1___closed__2; x_4 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__3; @@ -8891,7 +9127,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__6; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -8955,7 +9191,7 @@ static lean_object* _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Ty _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6; x_2 = l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__14; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; @@ -11035,10 +11271,10 @@ x_15 = !lean_is_exclusive(x_13); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_16 = lean_ctor_get(x_13, 13); +x_16 = lean_ctor_get(x_13, 15); x_17 = lean_box(0); x_18 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markTheoremInstance___spec__1(x_16, x_1, x_17); -lean_ctor_set(x_13, 13, x_18); +lean_ctor_set(x_13, 15, x_18); x_19 = lean_st_ref_set(x_3, x_13, x_14); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) @@ -11067,15 +11303,15 @@ return x_27; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; lean_object* x_56; lean_object* x_57; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; lean_object* x_59; lean_object* x_60; x_28 = lean_ctor_get(x_13, 0); x_29 = lean_ctor_get(x_13, 1); x_30 = lean_ctor_get(x_13, 2); x_31 = lean_ctor_get(x_13, 3); x_32 = lean_ctor_get(x_13, 4); x_33 = lean_ctor_get(x_13, 5); -x_34 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_35 = lean_ctor_get(x_13, 6); +x_34 = lean_ctor_get(x_13, 6); +x_35 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_36 = lean_ctor_get(x_13, 7); x_37 = lean_ctor_get(x_13, 8); x_38 = lean_ctor_get(x_13, 9); @@ -11089,6 +11325,12 @@ x_45 = lean_ctor_get(x_13, 16); x_46 = lean_ctor_get(x_13, 17); x_47 = lean_ctor_get(x_13, 18); x_48 = lean_ctor_get(x_13, 19); +x_49 = lean_ctor_get(x_13, 20); +x_50 = lean_ctor_get(x_13, 21); +x_51 = lean_ctor_get(x_13, 22); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); @@ -11102,7 +11344,7 @@ lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); lean_inc(x_36); -lean_inc(x_35); +lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); @@ -11110,51 +11352,54 @@ lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_dec(x_13); -x_49 = lean_box(0); -x_50 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markTheoremInstance___spec__1(x_42, x_1, x_49); -x_51 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_51, 0, x_28); -lean_ctor_set(x_51, 1, x_29); -lean_ctor_set(x_51, 2, x_30); -lean_ctor_set(x_51, 3, x_31); -lean_ctor_set(x_51, 4, x_32); -lean_ctor_set(x_51, 5, x_33); -lean_ctor_set(x_51, 6, x_35); -lean_ctor_set(x_51, 7, x_36); -lean_ctor_set(x_51, 8, x_37); -lean_ctor_set(x_51, 9, x_38); -lean_ctor_set(x_51, 10, x_39); -lean_ctor_set(x_51, 11, x_40); -lean_ctor_set(x_51, 12, x_41); -lean_ctor_set(x_51, 13, x_50); -lean_ctor_set(x_51, 14, x_43); -lean_ctor_set(x_51, 15, x_44); -lean_ctor_set(x_51, 16, x_45); -lean_ctor_set(x_51, 17, x_46); -lean_ctor_set(x_51, 18, x_47); -lean_ctor_set(x_51, 19, x_48); -lean_ctor_set_uint8(x_51, sizeof(void*)*20, x_34); -x_52 = lean_st_ref_set(x_3, x_51, x_14); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_54 = x_52; +x_52 = lean_box(0); +x_53 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markTheoremInstance___spec__1(x_44, x_1, x_52); +x_54 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_54, 0, x_28); +lean_ctor_set(x_54, 1, x_29); +lean_ctor_set(x_54, 2, x_30); +lean_ctor_set(x_54, 3, x_31); +lean_ctor_set(x_54, 4, x_32); +lean_ctor_set(x_54, 5, x_33); +lean_ctor_set(x_54, 6, x_34); +lean_ctor_set(x_54, 7, x_36); +lean_ctor_set(x_54, 8, x_37); +lean_ctor_set(x_54, 9, x_38); +lean_ctor_set(x_54, 10, x_39); +lean_ctor_set(x_54, 11, x_40); +lean_ctor_set(x_54, 12, x_41); +lean_ctor_set(x_54, 13, x_42); +lean_ctor_set(x_54, 14, x_43); +lean_ctor_set(x_54, 15, x_53); +lean_ctor_set(x_54, 16, x_45); +lean_ctor_set(x_54, 17, x_46); +lean_ctor_set(x_54, 18, x_47); +lean_ctor_set(x_54, 19, x_48); +lean_ctor_set(x_54, 20, x_49); +lean_ctor_set(x_54, 21, x_50); +lean_ctor_set(x_54, 22, x_51); +lean_ctor_set_uint8(x_54, sizeof(void*)*23, x_35); +x_55 = lean_st_ref_set(x_3, x_54, x_14); +x_56 = lean_ctor_get(x_55, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_57 = x_55; } else { - lean_dec_ref(x_52); - x_54 = lean_box(0); + lean_dec_ref(x_55); + x_57 = lean_box(0); } -x_55 = 1; -x_56 = lean_box(x_55); -if (lean_is_scalar(x_54)) { - x_57 = lean_alloc_ctor(0, 2, 0); +x_58 = 1; +x_59 = lean_box(x_58); +if (lean_is_scalar(x_57)) { + x_60 = lean_alloc_ctor(0, 2, 0); } else { - x_57 = x_54; + x_60 = x_57; } -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_53); -return x_57; +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_56); +return x_60; } } } @@ -11172,7 +11417,7 @@ if (x_14 == 0) lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_ctor_get(x_15, 13); +x_17 = lean_ctor_get(x_15, 15); lean_inc(x_17); lean_dec(x_15); x_18 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_markTheoremInstance___spec__9(x_17, x_12); @@ -11202,7 +11447,7 @@ x_24 = lean_ctor_get(x_13, 1); lean_inc(x_24); lean_inc(x_23); lean_dec(x_13); -x_25 = lean_ctor_get(x_23, 13); +x_25 = lean_ctor_get(x_23, 15); lean_inc(x_25); lean_dec(x_23); x_26 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_markTheoremInstance___spec__9(x_25, x_12); @@ -11534,13 +11779,13 @@ x_16 = !lean_is_exclusive(x_14); if (x_16 == 0) { lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_17 = lean_ctor_get(x_14, 14); +x_17 = lean_ctor_get(x_14, 16); x_18 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_18, 0, x_1); lean_ctor_set(x_18, 1, x_2); lean_ctor_set(x_18, 2, x_3); x_19 = l_Std_Queue_enqueue___rarg(x_18, x_17); -lean_ctor_set(x_14, 14, x_19); +lean_ctor_set(x_14, 16, x_19); x_20 = lean_st_ref_set(x_4, x_14, x_15); x_21 = !lean_is_exclusive(x_20); if (x_21 == 0) @@ -11567,15 +11812,15 @@ return x_26; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; x_27 = lean_ctor_get(x_14, 0); x_28 = lean_ctor_get(x_14, 1); x_29 = lean_ctor_get(x_14, 2); x_30 = lean_ctor_get(x_14, 3); x_31 = lean_ctor_get(x_14, 4); x_32 = lean_ctor_get(x_14, 5); -x_33 = lean_ctor_get_uint8(x_14, sizeof(void*)*20); -x_34 = lean_ctor_get(x_14, 6); +x_33 = lean_ctor_get(x_14, 6); +x_34 = lean_ctor_get_uint8(x_14, sizeof(void*)*23); x_35 = lean_ctor_get(x_14, 7); x_36 = lean_ctor_get(x_14, 8); x_37 = lean_ctor_get(x_14, 9); @@ -11589,6 +11834,12 @@ x_44 = lean_ctor_get(x_14, 16); x_45 = lean_ctor_get(x_14, 17); x_46 = lean_ctor_get(x_14, 18); x_47 = lean_ctor_get(x_14, 19); +x_48 = lean_ctor_get(x_14, 20); +x_49 = lean_ctor_get(x_14, 21); +x_50 = lean_ctor_get(x_14, 22); +lean_inc(x_50); +lean_inc(x_49); +lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); @@ -11602,7 +11853,7 @@ lean_inc(x_38); lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); -lean_inc(x_34); +lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_inc(x_30); @@ -11610,53 +11861,56 @@ lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); lean_dec(x_14); -x_48 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_48, 0, x_1); -lean_ctor_set(x_48, 1, x_2); -lean_ctor_set(x_48, 2, x_3); -x_49 = l_Std_Queue_enqueue___rarg(x_48, x_42); -x_50 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_50, 0, x_27); -lean_ctor_set(x_50, 1, x_28); -lean_ctor_set(x_50, 2, x_29); -lean_ctor_set(x_50, 3, x_30); -lean_ctor_set(x_50, 4, x_31); -lean_ctor_set(x_50, 5, x_32); -lean_ctor_set(x_50, 6, x_34); -lean_ctor_set(x_50, 7, x_35); -lean_ctor_set(x_50, 8, x_36); -lean_ctor_set(x_50, 9, x_37); -lean_ctor_set(x_50, 10, x_38); -lean_ctor_set(x_50, 11, x_39); -lean_ctor_set(x_50, 12, x_40); -lean_ctor_set(x_50, 13, x_41); -lean_ctor_set(x_50, 14, x_49); -lean_ctor_set(x_50, 15, x_43); -lean_ctor_set(x_50, 16, x_44); -lean_ctor_set(x_50, 17, x_45); -lean_ctor_set(x_50, 18, x_46); -lean_ctor_set(x_50, 19, x_47); -lean_ctor_set_uint8(x_50, sizeof(void*)*20, x_33); -x_51 = lean_st_ref_set(x_4, x_50, x_15); -x_52 = lean_ctor_get(x_51, 1); -lean_inc(x_52); -if (lean_is_exclusive(x_51)) { - lean_ctor_release(x_51, 0); - lean_ctor_release(x_51, 1); - x_53 = x_51; +x_51 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_51, 0, x_1); +lean_ctor_set(x_51, 1, x_2); +lean_ctor_set(x_51, 2, x_3); +x_52 = l_Std_Queue_enqueue___rarg(x_51, x_44); +x_53 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_53, 0, x_27); +lean_ctor_set(x_53, 1, x_28); +lean_ctor_set(x_53, 2, x_29); +lean_ctor_set(x_53, 3, x_30); +lean_ctor_set(x_53, 4, x_31); +lean_ctor_set(x_53, 5, x_32); +lean_ctor_set(x_53, 6, x_33); +lean_ctor_set(x_53, 7, x_35); +lean_ctor_set(x_53, 8, x_36); +lean_ctor_set(x_53, 9, x_37); +lean_ctor_set(x_53, 10, x_38); +lean_ctor_set(x_53, 11, x_39); +lean_ctor_set(x_53, 12, x_40); +lean_ctor_set(x_53, 13, x_41); +lean_ctor_set(x_53, 14, x_42); +lean_ctor_set(x_53, 15, x_43); +lean_ctor_set(x_53, 16, x_52); +lean_ctor_set(x_53, 17, x_45); +lean_ctor_set(x_53, 18, x_46); +lean_ctor_set(x_53, 19, x_47); +lean_ctor_set(x_53, 20, x_48); +lean_ctor_set(x_53, 21, x_49); +lean_ctor_set(x_53, 22, x_50); +lean_ctor_set_uint8(x_53, sizeof(void*)*23, x_34); +x_54 = lean_st_ref_set(x_4, x_53, x_15); +x_55 = lean_ctor_get(x_54, 1); +lean_inc(x_55); +if (lean_is_exclusive(x_54)) { + lean_ctor_release(x_54, 0); + lean_ctor_release(x_54, 1); + x_56 = x_54; } else { - lean_dec_ref(x_51); - x_53 = lean_box(0); + lean_dec_ref(x_54); + x_56 = lean_box(0); } -x_54 = lean_box(0); -if (lean_is_scalar(x_53)) { - x_55 = lean_alloc_ctor(0, 2, 0); +x_57 = lean_box(0); +if (lean_is_scalar(x_56)) { + x_58 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_53; + x_58 = x_56; } -lean_ctor_set(x_55, 0, x_54); -lean_ctor_set(x_55, 1, x_52); -return x_55; +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_55); +return x_58; } } } @@ -11694,11 +11948,11 @@ x_18 = !lean_is_exclusive(x_16); if (x_18 == 0) { lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_19 = lean_ctor_get(x_16, 11); +x_19 = lean_ctor_get(x_16, 13); x_20 = lean_unsigned_to_nat(1u); x_21 = lean_nat_add(x_19, x_20); lean_dec(x_19); -lean_ctor_set(x_16, 11, x_21); +lean_ctor_set(x_16, 13, x_21); x_22 = lean_st_ref_set(x_4, x_16, x_17); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) @@ -11725,15 +11979,15 @@ return x_28; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; x_29 = lean_ctor_get(x_16, 0); x_30 = lean_ctor_get(x_16, 1); x_31 = lean_ctor_get(x_16, 2); x_32 = lean_ctor_get(x_16, 3); x_33 = lean_ctor_get(x_16, 4); x_34 = lean_ctor_get(x_16, 5); -x_35 = lean_ctor_get_uint8(x_16, sizeof(void*)*20); -x_36 = lean_ctor_get(x_16, 6); +x_35 = lean_ctor_get(x_16, 6); +x_36 = lean_ctor_get_uint8(x_16, sizeof(void*)*23); x_37 = lean_ctor_get(x_16, 7); x_38 = lean_ctor_get(x_16, 8); x_39 = lean_ctor_get(x_16, 9); @@ -11747,6 +12001,12 @@ x_46 = lean_ctor_get(x_16, 16); x_47 = lean_ctor_get(x_16, 17); x_48 = lean_ctor_get(x_16, 18); x_49 = lean_ctor_get(x_16, 19); +x_50 = lean_ctor_get(x_16, 20); +x_51 = lean_ctor_get(x_16, 21); +x_52 = lean_ctor_get(x_16, 22); +lean_inc(x_52); +lean_inc(x_51); +lean_inc(x_50); lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); @@ -11760,7 +12020,7 @@ lean_inc(x_40); lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); -lean_inc(x_36); +lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); @@ -11768,51 +12028,54 @@ lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_dec(x_16); -x_50 = lean_unsigned_to_nat(1u); -x_51 = lean_nat_add(x_41, x_50); -lean_dec(x_41); -x_52 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_52, 0, x_29); -lean_ctor_set(x_52, 1, x_30); -lean_ctor_set(x_52, 2, x_31); -lean_ctor_set(x_52, 3, x_32); -lean_ctor_set(x_52, 4, x_33); -lean_ctor_set(x_52, 5, x_34); -lean_ctor_set(x_52, 6, x_36); -lean_ctor_set(x_52, 7, x_37); -lean_ctor_set(x_52, 8, x_38); -lean_ctor_set(x_52, 9, x_39); -lean_ctor_set(x_52, 10, x_40); -lean_ctor_set(x_52, 11, x_51); -lean_ctor_set(x_52, 12, x_42); -lean_ctor_set(x_52, 13, x_43); -lean_ctor_set(x_52, 14, x_44); -lean_ctor_set(x_52, 15, x_45); -lean_ctor_set(x_52, 16, x_46); -lean_ctor_set(x_52, 17, x_47); -lean_ctor_set(x_52, 18, x_48); -lean_ctor_set(x_52, 19, x_49); -lean_ctor_set_uint8(x_52, sizeof(void*)*20, x_35); -x_53 = lean_st_ref_set(x_4, x_52, x_17); -x_54 = lean_ctor_get(x_53, 1); -lean_inc(x_54); -if (lean_is_exclusive(x_53)) { - lean_ctor_release(x_53, 0); - lean_ctor_release(x_53, 1); - x_55 = x_53; +x_53 = lean_unsigned_to_nat(1u); +x_54 = lean_nat_add(x_43, x_53); +lean_dec(x_43); +x_55 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_55, 0, x_29); +lean_ctor_set(x_55, 1, x_30); +lean_ctor_set(x_55, 2, x_31); +lean_ctor_set(x_55, 3, x_32); +lean_ctor_set(x_55, 4, x_33); +lean_ctor_set(x_55, 5, x_34); +lean_ctor_set(x_55, 6, x_35); +lean_ctor_set(x_55, 7, x_37); +lean_ctor_set(x_55, 8, x_38); +lean_ctor_set(x_55, 9, x_39); +lean_ctor_set(x_55, 10, x_40); +lean_ctor_set(x_55, 11, x_41); +lean_ctor_set(x_55, 12, x_42); +lean_ctor_set(x_55, 13, x_54); +lean_ctor_set(x_55, 14, x_44); +lean_ctor_set(x_55, 15, x_45); +lean_ctor_set(x_55, 16, x_46); +lean_ctor_set(x_55, 17, x_47); +lean_ctor_set(x_55, 18, x_48); +lean_ctor_set(x_55, 19, x_49); +lean_ctor_set(x_55, 20, x_50); +lean_ctor_set(x_55, 21, x_51); +lean_ctor_set(x_55, 22, x_52); +lean_ctor_set_uint8(x_55, sizeof(void*)*23, x_36); +x_56 = lean_st_ref_set(x_4, x_55, x_17); +x_57 = lean_ctor_get(x_56, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_56)) { + lean_ctor_release(x_56, 0); + lean_ctor_release(x_56, 1); + x_58 = x_56; } else { - lean_dec_ref(x_53); - x_55 = lean_box(0); + lean_dec_ref(x_56); + x_58 = lean_box(0); } -x_56 = lean_box(0); -if (lean_is_scalar(x_55)) { - x_57 = lean_alloc_ctor(0, 2, 0); +x_59 = lean_box(0); +if (lean_is_scalar(x_58)) { + x_60 = lean_alloc_ctor(0, 2, 0); } else { - x_57 = x_55; + x_60 = x_58; } -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_54); -return x_57; +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_57); +return x_60; } } } @@ -11851,7 +12114,7 @@ x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_15, 3); lean_inc(x_16); lean_dec(x_15); -x_17 = lean_ctor_get(x_11, 11); +x_17 = lean_ctor_get(x_11, 13); lean_inc(x_17); lean_dec(x_11); x_18 = lean_nat_dec_le(x_16, x_17); @@ -11872,7 +12135,7 @@ lean_dec(x_13); x_22 = lean_ctor_get(x_20, 3); lean_inc(x_22); lean_dec(x_20); -x_23 = lean_ctor_get(x_11, 11); +x_23 = lean_ctor_get(x_11, 13); lean_inc(x_23); lean_dec(x_11); x_24 = lean_nat_dec_le(x_22, x_23); @@ -11921,7 +12184,7 @@ x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_15, 0); lean_inc(x_16); lean_dec(x_15); -x_17 = lean_ctor_get(x_11, 17); +x_17 = lean_ctor_get(x_11, 19); lean_inc(x_17); lean_dec(x_11); x_18 = lean_nat_dec_le(x_16, x_17); @@ -11942,7 +12205,7 @@ lean_dec(x_13); x_22 = lean_ctor_get(x_20, 0); lean_inc(x_22); lean_dec(x_20); -x_23 = lean_ctor_get(x_11, 17); +x_23 = lean_ctor_get(x_11, 19); lean_inc(x_23); lean_dec(x_11); x_24 = lean_nat_dec_le(x_22, x_23); @@ -11991,7 +12254,7 @@ x_15 = lean_ctor_get(x_13, 0); x_16 = lean_ctor_get(x_15, 1); lean_inc(x_16); lean_dec(x_15); -x_17 = lean_ctor_get(x_11, 12); +x_17 = lean_ctor_get(x_11, 14); lean_inc(x_17); lean_dec(x_11); x_18 = lean_nat_dec_le(x_16, x_17); @@ -12012,7 +12275,7 @@ lean_dec(x_13); x_22 = lean_ctor_get(x_20, 1); lean_inc(x_22); lean_dec(x_20); -x_23 = lean_ctor_get(x_11, 12); +x_23 = lean_ctor_get(x_11, 14); lean_inc(x_23); lean_dec(x_11); x_24 = lean_nat_dec_le(x_22, x_23); @@ -12042,6 +12305,26 @@ lean_dec(x_1); return x_10; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode_x3f(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_ctor_get(x_1, 2); +lean_inc(x_3); +lean_dec(x_1); +x_4 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_3, x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode_x3f___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { @@ -12050,31 +12333,25 @@ x_11 = lean_st_ref_get(x_2, x_10); x_12 = !lean_is_exclusive(x_11); if (x_12 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_13; lean_object* x_14; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -x_15 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_14, x_1); -lean_ctor_set(x_11, 0, x_15); +x_14 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_13, x_1); +lean_ctor_set(x_11, 0, x_14); return x_11; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = lean_ctor_get(x_11, 1); lean_inc(x_16); +lean_inc(x_15); lean_dec(x_11); -x_18 = lean_ctor_get(x_16, 1); -lean_inc(x_18); -lean_dec(x_16); -x_19 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_18, x_1); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_17); -return x_20; +x_17 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_15, x_1); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; } } } @@ -12095,45 +12372,53 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_11 = lean_ctor_get(x_8, 5); -x_12 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_6, x_7, x_8, x_9, x_10); -x_13 = !lean_is_exclusive(x_12); -if (x_13 == 0) +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = lean_ctor_get(x_2, 5); +x_6 = l_Lean_addMessageContextPartial___at_Lean_Core_instAddMessageContextCoreM___spec__1(x_1, x_2, x_3, x_4); +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_12, 0); -lean_inc(x_11); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_11); -lean_ctor_set(x_15, 1, x_14); -lean_ctor_set_tag(x_12, 1); -lean_ctor_set(x_12, 0, x_15); -return x_12; +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_5); +x_9 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_9, 0, x_5); +lean_ctor_set(x_9, 1, x_8); +lean_ctor_set_tag(x_6, 1); +lean_ctor_set(x_6, 0, x_9); +return x_6; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_12, 0); -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_12); +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); lean_inc(x_11); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_11); -lean_ctor_set(x_18, 1, x_16); -x_19 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; +lean_inc(x_10); +lean_dec(x_6); +lean_inc(x_5); +x_12 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_12, 0, x_5); +lean_ctor_set(x_12, 1, x_10); +x_13 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} } } +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg___boxed), 4, 0); +return x_2; } -static lean_object* _init_l_Lean_Meta_Grind_getENode___closed__1() { +} +static lean_object* _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1() { _start: { lean_object* x_1; @@ -12141,16 +12426,16 @@ x_1 = lean_mk_string_unchecked("internal `grind` error, term has not been intern return x_1; } } -static lean_object* _init_l_Lean_Meta_Grind_getENode___closed__2() { +static lean_object* _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_getENode___closed__1; +x_1 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1; x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -static lean_object* _init_l_Lean_Meta_Grind_getENode___closed__3() { +static lean_object* _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -12159,104 +12444,101 @@ x_2 = l_Lean_stringToMessageData(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_11; uint8_t x_12; -x_11 = lean_st_ref_get(x_2, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_5 = l_Lean_indentExpr(x_1); +x_6 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2; +x_7 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_5); +x_8 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3; +x_9 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_9, 0, x_7); +lean_ctor_set(x_9, 1, x_8); +x_10 = l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg(x_9, x_2, x_3, x_4); +return x_10; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr(lean_object* x_1) { +_start: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_15, x_1); -if (lean_obj_tag(x_16) == 0) +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___boxed), 4, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -lean_free_object(x_11); -x_17 = l_Lean_indentExpr(x_1); -x_18 = l_Lean_Meta_Grind_getENode___closed__2; -x_19 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -x_20 = l_Lean_Meta_Grind_getENode___closed__3; -x_21 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1(x_21, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -return x_22; +lean_object* x_5; +x_5 = l_Lean_throwError___at_Lean_Meta_Grind_throwNonInternalizedExpr___spec__1___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { -lean_object* x_23; -lean_dec(x_1); -x_23 = lean_ctor_get(x_16, 0); -lean_inc(x_23); -lean_dec(x_16); -lean_ctor_set(x_11, 0, x_23); -return x_11; +lean_object* x_5; +x_5 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg(x_1, x_2, x_3, x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_5; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_24 = lean_ctor_get(x_11, 0); -x_25 = lean_ctor_get(x_11, 1); -lean_inc(x_25); -lean_inc(x_24); -lean_dec(x_11); -x_26 = lean_ctor_get(x_24, 1); -lean_inc(x_26); -lean_dec(x_24); -x_27 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_26, x_1); -if (lean_obj_tag(x_27) == 0) +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_1, 2); +lean_inc(x_6); +lean_dec(x_1); +x_7 = l_Lean_PersistentHashMap_find_x3f___at___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_hashRoot___spec__1(x_6, x_2); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_28 = l_Lean_indentExpr(x_1); -x_29 = l_Lean_Meta_Grind_getENode___closed__2; -x_30 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_30, 0, x_29); -lean_ctor_set(x_30, 1, x_28); -x_31 = l_Lean_Meta_Grind_getENode___closed__3; -x_32 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -x_33 = l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1(x_32, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_25); -return x_33; +lean_object* x_8; +x_8 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg(x_2, x_3, x_4, x_5); +return x_8; } else { -lean_object* x_34; lean_object* x_35; -lean_dec(x_1); -x_34 = lean_ctor_get(x_27, 0); -lean_inc(x_34); -lean_dec(x_27); -x_35 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_25); -return x_35; -} +lean_object* x_9; lean_object* x_10; +lean_dec(x_2); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_5); +return x_10; } } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENode___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_11; -x_11 = l_Lean_throwError___at_Lean_Meta_Grind_getENode___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Goal_getENode(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -return x_11; +return x_6; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +return x_14; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENode___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -12278,59 +12560,65 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getGeneration(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 8); -lean_inc(x_14); -lean_dec(x_13); -lean_ctor_set(x_11, 0, x_14); -return x_11; +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_16, 8); +lean_inc(x_17); +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_17); +return x_14; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_11, 0); -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_11); -x_17 = lean_ctor_get(x_15, 8); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_18 = lean_ctor_get(x_14, 0); +x_19 = lean_ctor_get(x_14, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_14); +x_20 = lean_ctor_get(x_18, 8); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_20); +lean_ctor_set(x_21, 1, x_19); +return x_21; } } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) +uint8_t x_22; +x_22 = !lean_is_exclusive(x_14); +if (x_22 == 0) { -return x_11; +return x_14; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_11, 0); -x_21 = lean_ctor_get(x_11, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_11); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_14, 0); +x_24 = lean_ctor_get(x_14, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_14); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } @@ -12354,73 +12642,79 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqTrue(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_12, 2); -lean_inc(x_17); -lean_dec(x_12); -x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_17, x_16); -lean_dec(x_16); -lean_dec(x_17); -x_19 = lean_box(x_18); -lean_ctor_set(x_14, 0, x_19); -return x_14; -} -else +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_16); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); +lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_15, 2); lean_inc(x_20); -lean_dec(x_14); -x_22 = lean_ctor_get(x_12, 2); -lean_inc(x_22); -lean_dec(x_12); -x_23 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_22, x_20); +lean_dec(x_15); +x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_20, x_19); +lean_dec(x_19); lean_dec(x_20); -lean_dec(x_22); -x_24 = lean_box(x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_21); -return x_25; +x_22 = lean_box(x_21); +lean_ctor_set(x_17, 0, x_22); +return x_17; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; +x_23 = lean_ctor_get(x_17, 0); +x_24 = lean_ctor_get(x_17, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_17); +x_25 = lean_ctor_get(x_15, 2); +lean_inc(x_25); +lean_dec(x_15); +x_26 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_25, x_23); +lean_dec(x_23); +lean_dec(x_25); +x_27 = lean_box(x_26); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_24); +return x_28; } } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_11); -if (x_26 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -return x_11; +return x_14; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_11, 0); -x_28 = lean_ctor_get(x_11, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_11); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } @@ -12444,73 +12738,79 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isEqFalse(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_13); -x_15 = !lean_is_exclusive(x_14); -if (x_15 == 0) +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; -x_16 = lean_ctor_get(x_14, 0); -x_17 = lean_ctor_get(x_12, 2); -lean_inc(x_17); -lean_dec(x_12); -x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_17, x_16); -lean_dec(x_16); -lean_dec(x_17); -x_19 = lean_box(x_18); -lean_ctor_set(x_14, 0, x_19); -return x_14; -} -else +lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_16); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; -x_20 = lean_ctor_get(x_14, 0); -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); +lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_15, 2); lean_inc(x_20); -lean_dec(x_14); -x_22 = lean_ctor_get(x_12, 2); -lean_inc(x_22); -lean_dec(x_12); -x_23 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_22, x_20); +lean_dec(x_15); +x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_20, x_19); +lean_dec(x_19); lean_dec(x_20); -lean_dec(x_22); -x_24 = lean_box(x_23); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_24); -lean_ctor_set(x_25, 1, x_21); -return x_25; +x_22 = lean_box(x_21); +lean_ctor_set(x_17, 0, x_22); +return x_17; +} +else +{ +lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; +x_23 = lean_ctor_get(x_17, 0); +x_24 = lean_ctor_get(x_17, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_17); +x_25 = lean_ctor_get(x_15, 2); +lean_inc(x_25); +lean_dec(x_15); +x_26 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_25, x_23); +lean_dec(x_23); +lean_dec(x_25); +x_27 = lean_box(x_26); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_24); +return x_28; } } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_11); -if (x_26 == 0) +uint8_t x_29; +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -return x_11; +return x_14; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_11, 0); -x_28 = lean_ctor_get(x_11, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_11); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } } @@ -12538,121 +12838,133 @@ uint8_t x_12; x_12 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_2); if (x_12 == 0) { -lean_object* x_13; -x_13 = l_Lean_Meta_Grind_getENode(x_1, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_13) == 0) -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_13 = lean_st_ref_get(x_3, x_11); x_14 = lean_ctor_get(x_13, 0); lean_inc(x_14); x_15 = lean_ctor_get(x_13, 1); lean_inc(x_15); lean_dec(x_13); -x_16 = l_Lean_Meta_Grind_getENode(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +x_16 = l_Lean_Meta_Grind_Goal_getENode(x_14, x_1, x_9, x_10, x_15); if (lean_obj_tag(x_16) == 0) { -uint8_t x_17; -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_14, 2); -lean_inc(x_19); -lean_dec(x_14); -x_20 = lean_ctor_get(x_18, 2); +lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_17 = lean_ctor_get(x_16, 0); +lean_inc(x_17); +x_18 = lean_ctor_get(x_16, 1); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_st_ref_get(x_3, x_18); +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_19, x_20); -lean_dec(x_20); +x_21 = lean_ctor_get(x_19, 1); +lean_inc(x_21); lean_dec(x_19); -x_22 = lean_box(x_21); -lean_ctor_set(x_16, 0, x_22); -return x_16; -} -else +x_22 = l_Lean_Meta_Grind_Goal_getENode(x_20, x_2, x_9, x_10, x_21); +if (lean_obj_tag(x_22) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; lean_object* x_29; -x_23 = lean_ctor_get(x_16, 0); -x_24 = lean_ctor_get(x_16, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_16); -x_25 = lean_ctor_get(x_14, 2); +uint8_t x_23; +x_23 = !lean_is_exclusive(x_22); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; uint8_t x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_22, 0); +x_25 = lean_ctor_get(x_17, 2); lean_inc(x_25); -lean_dec(x_14); -x_26 = lean_ctor_get(x_23, 2); +lean_dec(x_17); +x_26 = lean_ctor_get(x_24, 2); lean_inc(x_26); -lean_dec(x_23); +lean_dec(x_24); x_27 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_25, x_26); lean_dec(x_26); lean_dec(x_25); x_28 = lean_box(x_27); -x_29 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_29, 0, x_28); -lean_ctor_set(x_29, 1, x_24); -return x_29; +lean_ctor_set(x_22, 0, x_28); +return x_22; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; +x_29 = lean_ctor_get(x_22, 0); +x_30 = lean_ctor_get(x_22, 1); +lean_inc(x_30); +lean_inc(x_29); +lean_dec(x_22); +x_31 = lean_ctor_get(x_17, 2); +lean_inc(x_31); +lean_dec(x_17); +x_32 = lean_ctor_get(x_29, 2); +lean_inc(x_32); +lean_dec(x_29); +x_33 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_31, x_32); +lean_dec(x_32); +lean_dec(x_31); +x_34 = lean_box(x_33); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_34); +lean_ctor_set(x_35, 1, x_30); +return x_35; } } else { -uint8_t x_30; -lean_dec(x_14); -x_30 = !lean_is_exclusive(x_16); -if (x_30 == 0) +uint8_t x_36; +lean_dec(x_17); +x_36 = !lean_is_exclusive(x_22); +if (x_36 == 0) { -return x_16; +return x_22; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_31 = lean_ctor_get(x_16, 0); -x_32 = lean_ctor_get(x_16, 1); -lean_inc(x_32); -lean_inc(x_31); -lean_dec(x_16); -x_33 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_33, 0, x_31); -lean_ctor_set(x_33, 1, x_32); -return x_33; +lean_object* x_37; lean_object* x_38; lean_object* x_39; +x_37 = lean_ctor_get(x_22, 0); +x_38 = lean_ctor_get(x_22, 1); +lean_inc(x_38); +lean_inc(x_37); +lean_dec(x_22); +x_39 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_39, 0, x_37); +lean_ctor_set(x_39, 1, x_38); +return x_39; } } } else { -uint8_t x_34; +uint8_t x_40; lean_dec(x_2); -x_34 = !lean_is_exclusive(x_13); -if (x_34 == 0) +x_40 = !lean_is_exclusive(x_16); +if (x_40 == 0) { -return x_13; +return x_16; } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_13, 0); -x_36 = lean_ctor_get(x_13, 1); -lean_inc(x_36); -lean_inc(x_35); -lean_dec(x_13); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_16, 0); +x_42 = lean_ctor_get(x_16, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_16); +x_43 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_43, 0, x_41); +lean_ctor_set(x_43, 1, x_42); +return x_43; } } } else { -uint8_t x_38; lean_object* x_39; lean_object* x_40; +uint8_t x_44; lean_object* x_45; lean_object* x_46; lean_dec(x_2); lean_dec(x_1); -x_38 = 1; -x_39 = lean_box(x_38); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_11); -return x_40; +x_44 = 1; +x_45 = lean_box(x_44); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_45); +lean_ctor_set(x_46, 1, x_11); +return x_46; } } } @@ -12675,19 +12987,17 @@ return x_12; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Meta_Grind_getENode_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) { -uint8_t x_13; -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +x_14 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_13, x_1); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_14; uint8_t x_15; lean_object* x_16; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); +uint8_t x_15; lean_object* x_16; x_15 = 0; x_16 = lean_box(x_15); lean_ctor_set(x_11, 0, x_16); @@ -12695,58 +13005,55 @@ return x_11; } else { -lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; -x_17 = lean_ctor_get(x_11, 1); +lean_object* x_17; lean_object* x_18; uint8_t x_19; lean_object* x_20; +x_17 = lean_ctor_get(x_14, 0); lean_inc(x_17); -lean_dec(x_11); -x_18 = 0; -x_19 = lean_box(x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_17); -return x_20; -} -} -else -{ -uint8_t x_21; -x_21 = !lean_is_exclusive(x_11); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; -x_22 = lean_ctor_get(x_11, 0); -lean_dec(x_22); -x_23 = lean_ctor_get(x_12, 0); -lean_inc(x_23); -lean_dec(x_12); -x_24 = lean_ctor_get(x_23, 2); -lean_inc(x_24); -lean_dec(x_23); -x_25 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_24, x_1); -lean_dec(x_24); -x_26 = lean_box(x_25); -lean_ctor_set(x_11, 0, x_26); +lean_dec(x_14); +x_18 = lean_ctor_get(x_17, 2); +lean_inc(x_18); +lean_dec(x_17); +x_19 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_18, x_1); +lean_dec(x_18); +x_20 = lean_box(x_19); +lean_ctor_set(x_11, 0, x_20); return x_11; } +} else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; -x_27 = lean_ctor_get(x_11, 1); -lean_inc(x_27); +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_11, 0); +x_22 = lean_ctor_get(x_11, 1); +lean_inc(x_22); +lean_inc(x_21); lean_dec(x_11); -x_28 = lean_ctor_get(x_12, 0); +x_23 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_21, x_1); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; lean_object* x_25; lean_object* x_26; +x_24 = 0; +x_25 = lean_box(x_24); +x_26 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_26, 0, x_25); +lean_ctor_set(x_26, 1, x_22); +return x_26; +} +else +{ +lean_object* x_27; lean_object* x_28; uint8_t x_29; lean_object* x_30; lean_object* x_31; +x_27 = lean_ctor_get(x_23, 0); +lean_inc(x_27); +lean_dec(x_23); +x_28 = lean_ctor_get(x_27, 2); lean_inc(x_28); -lean_dec(x_12); -x_29 = lean_ctor_get(x_28, 2); -lean_inc(x_29); +lean_dec(x_27); +x_29 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_28, x_1); lean_dec(x_28); -x_30 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_29, x_1); -lean_dec(x_29); -x_31 = lean_box(x_30); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_27); -return x_32; +x_30 = lean_box(x_29); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_30); +lean_ctor_set(x_31, 1, x_22); +return x_31; } } } @@ -12768,103 +13075,83 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Meta_Grind_getENode_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = lean_box(0); -lean_ctor_set(x_11, 0, x_15); -return x_11; +lean_object* x_4; +x_4 = lean_box(0); +return x_4; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; -} +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_6, 2); +lean_inc(x_7); +lean_dec(x_6); +lean_ctor_set(x_3, 0, x_7); +return x_3; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) -{ -lean_object* x_20; uint8_t x_21; -x_20 = lean_ctor_get(x_11, 0); -lean_dec(x_20); -x_21 = !lean_is_exclusive(x_12); -if (x_21 == 0) +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 2); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot_x3f___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_22; lean_object* x_23; -x_22 = lean_ctor_get(x_12, 0); -x_23 = lean_ctor_get(x_22, 2); -lean_inc(x_23); -lean_dec(x_22); -lean_ctor_set(x_12, 0, x_23); -return x_11; +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_1, x_2); +lean_dec(x_2); +return x_3; } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_24 = lean_ctor_get(x_12, 0); -lean_inc(x_24); -lean_dec(x_12); -x_25 = lean_ctor_get(x_24, 2); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_11, 0, x_26); +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +x_14 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_13, x_1); +lean_ctor_set(x_11, 0, x_14); return x_11; } -} else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_27 = lean_ctor_get(x_11, 1); -lean_inc(x_27); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_inc(x_15); lean_dec(x_11); -x_28 = lean_ctor_get(x_12, 0); -lean_inc(x_28); -if (lean_is_exclusive(x_12)) { - lean_ctor_release(x_12, 0); - x_29 = x_12; -} else { - lean_dec_ref(x_12); - x_29 = lean_box(0); -} -x_30 = lean_ctor_get(x_28, 2); -lean_inc(x_30); -lean_dec(x_28); -if (lean_is_scalar(x_29)) { - x_31 = lean_alloc_ctor(1, 1, 0); -} else { - x_31 = x_29; -} -lean_ctor_set(x_31, 0, x_30); -x_32 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_27); -return x_32; -} +x_17 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_15, x_1); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; } } } @@ -12885,65 +13172,89 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Goal_getENode(x_1, x_2, x_3, x_4, x_5); +if (lean_obj_tag(x_6) == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 2); -lean_inc(x_14); -lean_dec(x_13); -lean_ctor_set(x_11, 0, x_14); -return x_11; +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_8, 2); +lean_inc(x_9); +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_9); +return x_6; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_11, 0); -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_11); -x_17 = lean_ctor_get(x_15, 2); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_6); +x_12 = lean_ctor_get(x_10, 2); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; } } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) +uint8_t x_14; +x_14 = !lean_is_exclusive(x_6); +if (x_14 == 0) { -return x_11; +return x_6; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_11, 0); -x_21 = lean_ctor_get(x_11, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_11); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_6, 0); +x_16 = lean_ctor_get(x_6, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_6); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Goal_getRoot(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_6; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_getRoot(x_12, x_1, x_8, x_9, x_13); +return x_14; +} } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: @@ -12964,39 +13275,51 @@ return x_11; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getRootENode(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getRoot(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = l_Lean_Meta_Grind_getENode(x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_14; +x_14 = l_Lean_Meta_Grind_Goal_getRoot(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = lean_st_ref_get(x_2, x_16); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +x_20 = l_Lean_Meta_Grind_Goal_getENode(x_18, x_15, x_8, x_9, x_19); +return x_20; } else { -uint8_t x_15; -x_15 = !lean_is_exclusive(x_11); -if (x_15 == 0) +uint8_t x_21; +x_21 = !lean_is_exclusive(x_14); +if (x_21 == 0) { -return x_11; +return x_14; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_11); -x_18 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_18, 0, x_16); -lean_ctor_set(x_18, 1, x_17); -return x_18; +lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_22 = lean_ctor_get(x_14, 0); +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_14); +x_24 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +return x_24; } } } @@ -13017,64 +13340,138 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +lean_object* x_4; +x_4 = lean_box(0); +return x_4; +} +else { -lean_object* x_13; lean_object* x_14; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 1); -lean_inc(x_14); -lean_dec(x_13); -lean_ctor_set(x_11, 0, x_14); -return x_11; +uint8_t x_5; +x_5 = !lean_is_exclusive(x_3); +if (x_5 == 0) +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_3, 0); +x_7 = lean_ctor_get(x_6, 1); +lean_inc(x_7); +lean_dec(x_6); +lean_ctor_set(x_3, 0, x_7); +return x_3; } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_15 = lean_ctor_get(x_11, 0); -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_11); -x_17 = lean_ctor_get(x_15, 1); -lean_inc(x_17); -lean_dec(x_15); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_3, 0); +lean_inc(x_8); +lean_dec(x_3); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +x_10 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_10, 0, x_9); +return x_10; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext_x3f___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getNext_x3f(x_1, x_2); +lean_dec(x_2); +return x_3; +} } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Goal_getENode(x_1, x_2, x_3, x_4, x_5); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_8, 1); +lean_inc(x_9); +lean_dec(x_8); +lean_ctor_set(x_6, 0, x_9); +return x_6; } else { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_10 = lean_ctor_get(x_6, 0); +x_11 = lean_ctor_get(x_6, 1); +lean_inc(x_11); +lean_inc(x_10); +lean_dec(x_6); +x_12 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +lean_dec(x_10); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +return x_13; +} +} +else { -return x_11; +uint8_t x_14; +x_14 = !lean_is_exclusive(x_6); +if (x_14 == 0) +{ +return x_6; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_11, 0); -x_21 = lean_ctor_get(x_11, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_11); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_6, 0); +x_16 = lean_ctor_get(x_6, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_6); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getNext___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +x_6 = l_Lean_Meta_Grind_Goal_getNext(x_1, x_2, x_3, x_4, x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_6; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNext(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = l_Lean_Meta_Grind_Goal_getNext(x_12, x_1, x_8, x_9, x_13); +return x_14; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getNext___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -13216,7 +13613,7 @@ if (x_12 == 0) { lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 1); +x_14 = lean_ctor_get(x_13, 2); lean_inc(x_14); lean_dec(x_13); x_15 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_alreadyInternalized___spec__1(x_14, x_1); @@ -13232,7 +13629,7 @@ x_18 = lean_ctor_get(x_11, 1); lean_inc(x_18); lean_inc(x_17); lean_dec(x_11); -x_19 = lean_ctor_get(x_17, 1); +x_19 = lean_ctor_get(x_17, 2); lean_inc(x_19); lean_dec(x_17); x_20 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_alreadyInternalized___spec__1(x_19, x_1); @@ -13295,74 +13692,66 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTarget_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = l_Lean_Meta_Grind_getENode_x3f(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -if (lean_obj_tag(x_12) == 0) -{ -uint8_t x_13; -x_13 = !lean_is_exclusive(x_11); -if (x_13 == 0) +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getENode_x3f(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -lean_object* x_14; lean_object* x_15; -x_14 = lean_ctor_get(x_11, 0); -lean_dec(x_14); -x_15 = lean_box(0); -lean_ctor_set(x_11, 0, x_15); -return x_11; +lean_object* x_4; +x_4 = lean_box(0); +return x_4; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = lean_ctor_get(x_11, 1); -lean_inc(x_16); -lean_dec(x_11); -x_17 = lean_box(0); -x_18 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_18, 0, x_17); -lean_ctor_set(x_18, 1, x_16); -return x_18; +lean_object* x_5; lean_object* x_6; +x_5 = lean_ctor_get(x_3, 0); +lean_inc(x_5); +lean_dec(x_3); +x_6 = lean_ctor_get(x_5, 4); +lean_inc(x_6); +lean_dec(x_5); +return x_6; } } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getTarget_x3f___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -uint8_t x_19; -x_19 = !lean_is_exclusive(x_11); -if (x_19 == 0) +lean_object* x_3; +x_3 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_1, x_2); +lean_dec(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getTarget_x3f(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_11, 0); -lean_dec(x_20); -x_21 = lean_ctor_get(x_12, 0); -lean_inc(x_21); -lean_dec(x_12); -x_22 = lean_ctor_get(x_21, 4); -lean_inc(x_22); -lean_dec(x_21); -lean_ctor_set(x_11, 0, x_22); +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +x_14 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_13, x_1); +lean_ctor_set(x_11, 0, x_14); return x_11; } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_23 = lean_ctor_get(x_11, 1); -lean_inc(x_23); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_inc(x_15); lean_dec(x_11); -x_24 = lean_ctor_get(x_12, 0); -lean_inc(x_24); -lean_dec(x_12); -x_25 = lean_ctor_get(x_24, 4); -lean_inc(x_25); -lean_dec(x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_23); -return x_26; -} +x_17 = l_Lean_Meta_Grind_Goal_getTarget_x3f(x_15, x_1); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; } } } @@ -13397,14 +13786,14 @@ x_17 = !lean_is_exclusive(x_15); if (x_17 == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_18 = lean_ctor_get(x_15, 5); +x_18 = lean_ctor_get(x_15, 6); x_19 = lean_alloc_ctor(0, 3, 1); lean_ctor_set(x_19, 0, x_1); lean_ctor_set(x_19, 1, x_2); lean_ctor_set(x_19, 2, x_3); lean_ctor_set_uint8(x_19, sizeof(void*)*3, x_4); x_20 = lean_array_push(x_18, x_19); -lean_ctor_set(x_15, 5, x_20); +lean_ctor_set(x_15, 6, x_20); x_21 = lean_st_ref_set(x_5, x_15, x_16); x_22 = !lean_is_exclusive(x_21); if (x_22 == 0) @@ -13431,15 +13820,15 @@ return x_27; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; uint8_t x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; x_28 = lean_ctor_get(x_15, 0); x_29 = lean_ctor_get(x_15, 1); x_30 = lean_ctor_get(x_15, 2); x_31 = lean_ctor_get(x_15, 3); x_32 = lean_ctor_get(x_15, 4); x_33 = lean_ctor_get(x_15, 5); -x_34 = lean_ctor_get_uint8(x_15, sizeof(void*)*20); -x_35 = lean_ctor_get(x_15, 6); +x_34 = lean_ctor_get(x_15, 6); +x_35 = lean_ctor_get_uint8(x_15, sizeof(void*)*23); x_36 = lean_ctor_get(x_15, 7); x_37 = lean_ctor_get(x_15, 8); x_38 = lean_ctor_get(x_15, 9); @@ -13453,6 +13842,12 @@ x_45 = lean_ctor_get(x_15, 16); x_46 = lean_ctor_get(x_15, 17); x_47 = lean_ctor_get(x_15, 18); x_48 = lean_ctor_get(x_15, 19); +x_49 = lean_ctor_get(x_15, 20); +x_50 = lean_ctor_get(x_15, 21); +x_51 = lean_ctor_get(x_15, 22); +lean_inc(x_51); +lean_inc(x_50); +lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); @@ -13466,7 +13861,7 @@ lean_inc(x_39); lean_inc(x_38); lean_inc(x_37); lean_inc(x_36); -lean_inc(x_35); +lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); @@ -13474,54 +13869,57 @@ lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_dec(x_15); -x_49 = lean_alloc_ctor(0, 3, 1); -lean_ctor_set(x_49, 0, x_1); -lean_ctor_set(x_49, 1, x_2); -lean_ctor_set(x_49, 2, x_3); -lean_ctor_set_uint8(x_49, sizeof(void*)*3, x_4); -x_50 = lean_array_push(x_33, x_49); -x_51 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_51, 0, x_28); -lean_ctor_set(x_51, 1, x_29); -lean_ctor_set(x_51, 2, x_30); -lean_ctor_set(x_51, 3, x_31); -lean_ctor_set(x_51, 4, x_32); -lean_ctor_set(x_51, 5, x_50); -lean_ctor_set(x_51, 6, x_35); -lean_ctor_set(x_51, 7, x_36); -lean_ctor_set(x_51, 8, x_37); -lean_ctor_set(x_51, 9, x_38); -lean_ctor_set(x_51, 10, x_39); -lean_ctor_set(x_51, 11, x_40); -lean_ctor_set(x_51, 12, x_41); -lean_ctor_set(x_51, 13, x_42); -lean_ctor_set(x_51, 14, x_43); -lean_ctor_set(x_51, 15, x_44); -lean_ctor_set(x_51, 16, x_45); -lean_ctor_set(x_51, 17, x_46); -lean_ctor_set(x_51, 18, x_47); -lean_ctor_set(x_51, 19, x_48); -lean_ctor_set_uint8(x_51, sizeof(void*)*20, x_34); -x_52 = lean_st_ref_set(x_5, x_51, x_16); -x_53 = lean_ctor_get(x_52, 1); -lean_inc(x_53); -if (lean_is_exclusive(x_52)) { - lean_ctor_release(x_52, 0); - lean_ctor_release(x_52, 1); - x_54 = x_52; +x_52 = lean_alloc_ctor(0, 3, 1); +lean_ctor_set(x_52, 0, x_1); +lean_ctor_set(x_52, 1, x_2); +lean_ctor_set(x_52, 2, x_3); +lean_ctor_set_uint8(x_52, sizeof(void*)*3, x_4); +x_53 = lean_array_push(x_34, x_52); +x_54 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_54, 0, x_28); +lean_ctor_set(x_54, 1, x_29); +lean_ctor_set(x_54, 2, x_30); +lean_ctor_set(x_54, 3, x_31); +lean_ctor_set(x_54, 4, x_32); +lean_ctor_set(x_54, 5, x_33); +lean_ctor_set(x_54, 6, x_53); +lean_ctor_set(x_54, 7, x_36); +lean_ctor_set(x_54, 8, x_37); +lean_ctor_set(x_54, 9, x_38); +lean_ctor_set(x_54, 10, x_39); +lean_ctor_set(x_54, 11, x_40); +lean_ctor_set(x_54, 12, x_41); +lean_ctor_set(x_54, 13, x_42); +lean_ctor_set(x_54, 14, x_43); +lean_ctor_set(x_54, 15, x_44); +lean_ctor_set(x_54, 16, x_45); +lean_ctor_set(x_54, 17, x_46); +lean_ctor_set(x_54, 18, x_47); +lean_ctor_set(x_54, 19, x_48); +lean_ctor_set(x_54, 20, x_49); +lean_ctor_set(x_54, 21, x_50); +lean_ctor_set(x_54, 22, x_51); +lean_ctor_set_uint8(x_54, sizeof(void*)*23, x_35); +x_55 = lean_st_ref_set(x_5, x_54, x_16); +x_56 = lean_ctor_get(x_55, 1); +lean_inc(x_56); +if (lean_is_exclusive(x_55)) { + lean_ctor_release(x_55, 0); + lean_ctor_release(x_55, 1); + x_57 = x_55; } else { - lean_dec_ref(x_52); - x_54 = lean_box(0); + lean_dec_ref(x_55); + x_57 = lean_box(0); } -x_55 = lean_box(0); -if (lean_is_scalar(x_54)) { - x_56 = lean_alloc_ctor(0, 2, 0); +x_58 = lean_box(0); +if (lean_is_scalar(x_57)) { + x_59 = lean_alloc_ctor(0, 2, 0); } else { - x_56 = x_54; + x_59 = x_57; } -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_53); -return x_56; +lean_ctor_set(x_59, 0, x_58); +lean_ctor_set(x_59, 1, x_56); +return x_59; } } } @@ -17407,57 +17805,41 @@ return x_5; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_registerParent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; -x_12 = l_Lean_Meta_Grind_getRoot_x3f(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -x_13 = lean_ctor_get(x_12, 0); -lean_inc(x_13); -if (lean_obj_tag(x_13) == 0) +lean_object* x_12; uint8_t x_13; +x_12 = lean_st_ref_get(x_3, x_11); +x_13 = !lean_is_exclusive(x_12); +if (x_13 == 0) { -uint8_t x_14; -lean_dec(x_1); -x_14 = !lean_is_exclusive(x_12); -if (x_14 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_12, 0); +x_15 = lean_ctor_get(x_12, 1); +x_16 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_14, x_2); +if (lean_obj_tag(x_16) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 0); -lean_dec(x_15); -x_16 = lean_box(0); -lean_ctor_set(x_12, 0, x_16); +lean_object* x_17; +lean_dec(x_1); +x_17 = lean_box(0); +lean_ctor_set(x_12, 0, x_17); return x_12; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_dec(x_12); -x_18 = lean_box(0); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_17); -return x_19; -} -} -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_69; lean_object* x_70; -x_20 = lean_ctor_get(x_12, 1); +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_69; lean_object* x_70; +lean_free_object(x_12); +x_18 = lean_ctor_get(x_16, 0); +lean_inc(x_18); +lean_dec(x_16); +x_19 = lean_st_ref_get(x_3, x_15); +x_20 = lean_ctor_get(x_19, 0); lean_inc(x_20); -lean_dec(x_12); -x_21 = lean_ctor_get(x_13, 0); +x_21 = lean_ctor_get(x_19, 1); lean_inc(x_21); -lean_dec(x_13); -x_22 = lean_st_ref_get(x_3, x_20); -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -x_25 = lean_ctor_get(x_23, 2); -lean_inc(x_25); -lean_dec(x_23); -x_69 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_25, x_21); -x_70 = lean_st_ref_take(x_3, x_24); +lean_dec(x_19); +x_22 = lean_ctor_get(x_20, 3); +lean_inc(x_22); +lean_dec(x_20); +x_69 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_22, x_18); +x_70 = lean_st_ref_take(x_3, x_21); if (lean_obj_tag(x_69) == 0) { lean_object* x_71; lean_object* x_72; lean_object* x_73; @@ -17467,9 +17849,9 @@ x_72 = lean_ctor_get(x_70, 1); lean_inc(x_72); lean_dec(x_70); x_73 = lean_box(0); -x_26 = x_73; -x_27 = x_71; -x_28 = x_72; +x_23 = x_73; +x_24 = x_71; +x_25 = x_72; goto block_68; } else @@ -17483,69 +17865,72 @@ lean_inc(x_75); x_76 = lean_ctor_get(x_70, 1); lean_inc(x_76); lean_dec(x_70); -x_26 = x_74; -x_27 = x_75; -x_28 = x_76; +x_23 = x_74; +x_24 = x_75; +x_25 = x_76; goto block_68; } block_68: { -uint8_t x_29; -x_29 = !lean_is_exclusive(x_27); -if (x_29 == 0) +uint8_t x_26; +x_26 = !lean_is_exclusive(x_24); +if (x_26 == 0) { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_30 = lean_ctor_get(x_27, 2); -x_31 = lean_box(0); -x_32 = l_Lean_RBNode_insert___at_Lean_Meta_Grind_registerParent___spec__1(x_26, x_1, x_31); -x_33 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_30, x_21, x_32); -lean_ctor_set(x_27, 2, x_33); -x_34 = lean_st_ref_set(x_3, x_27, x_28); -x_35 = !lean_is_exclusive(x_34); -if (x_35 == 0) +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; +x_27 = lean_ctor_get(x_24, 3); +x_28 = lean_box(0); +x_29 = l_Lean_RBNode_insert___at_Lean_Meta_Grind_registerParent___spec__1(x_23, x_1, x_28); +x_30 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_27, x_18, x_29); +lean_ctor_set(x_24, 3, x_30); +x_31 = lean_st_ref_set(x_3, x_24, x_25); +x_32 = !lean_is_exclusive(x_31); +if (x_32 == 0) { -lean_object* x_36; -x_36 = lean_ctor_get(x_34, 0); -lean_dec(x_36); -lean_ctor_set(x_34, 0, x_31); -return x_34; +lean_object* x_33; +x_33 = lean_ctor_get(x_31, 0); +lean_dec(x_33); +lean_ctor_set(x_31, 0, x_28); +return x_31; } else { -lean_object* x_37; lean_object* x_38; -x_37 = lean_ctor_get(x_34, 1); -lean_inc(x_37); -lean_dec(x_34); -x_38 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_38, 0, x_31); -lean_ctor_set(x_38, 1, x_37); -return x_38; +lean_object* x_34; lean_object* x_35; +x_34 = lean_ctor_get(x_31, 1); +lean_inc(x_34); +lean_dec(x_31); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_28); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } else { -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; -x_39 = lean_ctor_get(x_27, 0); -x_40 = lean_ctor_get(x_27, 1); -x_41 = lean_ctor_get(x_27, 2); -x_42 = lean_ctor_get(x_27, 3); -x_43 = lean_ctor_get(x_27, 4); -x_44 = lean_ctor_get(x_27, 5); -x_45 = lean_ctor_get_uint8(x_27, sizeof(void*)*20); -x_46 = lean_ctor_get(x_27, 6); -x_47 = lean_ctor_get(x_27, 7); -x_48 = lean_ctor_get(x_27, 8); -x_49 = lean_ctor_get(x_27, 9); -x_50 = lean_ctor_get(x_27, 10); -x_51 = lean_ctor_get(x_27, 11); -x_52 = lean_ctor_get(x_27, 12); -x_53 = lean_ctor_get(x_27, 13); -x_54 = lean_ctor_get(x_27, 14); -x_55 = lean_ctor_get(x_27, 15); -x_56 = lean_ctor_get(x_27, 16); -x_57 = lean_ctor_get(x_27, 17); -x_58 = lean_ctor_get(x_27, 18); -x_59 = lean_ctor_get(x_27, 19); +lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_36 = lean_ctor_get(x_24, 0); +x_37 = lean_ctor_get(x_24, 1); +x_38 = lean_ctor_get(x_24, 2); +x_39 = lean_ctor_get(x_24, 3); +x_40 = lean_ctor_get(x_24, 4); +x_41 = lean_ctor_get(x_24, 5); +x_42 = lean_ctor_get(x_24, 6); +x_43 = lean_ctor_get_uint8(x_24, sizeof(void*)*23); +x_44 = lean_ctor_get(x_24, 7); +x_45 = lean_ctor_get(x_24, 8); +x_46 = lean_ctor_get(x_24, 9); +x_47 = lean_ctor_get(x_24, 10); +x_48 = lean_ctor_get(x_24, 11); +x_49 = lean_ctor_get(x_24, 12); +x_50 = lean_ctor_get(x_24, 13); +x_51 = lean_ctor_get(x_24, 14); +x_52 = lean_ctor_get(x_24, 15); +x_53 = lean_ctor_get(x_24, 16); +x_54 = lean_ctor_get(x_24, 17); +x_55 = lean_ctor_get(x_24, 18); +x_56 = lean_ctor_get(x_24, 19); +x_57 = lean_ctor_get(x_24, 20); +x_58 = lean_ctor_get(x_24, 21); +x_59 = lean_ctor_get(x_24, 22); lean_inc(x_59); lean_inc(x_58); lean_inc(x_57); @@ -17560,39 +17945,45 @@ lean_inc(x_49); lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); +lean_inc(x_45); lean_inc(x_44); -lean_inc(x_43); lean_inc(x_42); lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); -lean_dec(x_27); +lean_inc(x_38); +lean_inc(x_37); +lean_inc(x_36); +lean_dec(x_24); x_60 = lean_box(0); -x_61 = l_Lean_RBNode_insert___at_Lean_Meta_Grind_registerParent___spec__1(x_26, x_1, x_60); -x_62 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_41, x_21, x_61); -x_63 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_63, 0, x_39); -lean_ctor_set(x_63, 1, x_40); -lean_ctor_set(x_63, 2, x_62); -lean_ctor_set(x_63, 3, x_42); -lean_ctor_set(x_63, 4, x_43); -lean_ctor_set(x_63, 5, x_44); -lean_ctor_set(x_63, 6, x_46); -lean_ctor_set(x_63, 7, x_47); -lean_ctor_set(x_63, 8, x_48); -lean_ctor_set(x_63, 9, x_49); -lean_ctor_set(x_63, 10, x_50); -lean_ctor_set(x_63, 11, x_51); -lean_ctor_set(x_63, 12, x_52); -lean_ctor_set(x_63, 13, x_53); -lean_ctor_set(x_63, 14, x_54); -lean_ctor_set(x_63, 15, x_55); -lean_ctor_set(x_63, 16, x_56); -lean_ctor_set(x_63, 17, x_57); -lean_ctor_set(x_63, 18, x_58); -lean_ctor_set(x_63, 19, x_59); -lean_ctor_set_uint8(x_63, sizeof(void*)*20, x_45); -x_64 = lean_st_ref_set(x_3, x_63, x_28); +x_61 = l_Lean_RBNode_insert___at_Lean_Meta_Grind_registerParent___spec__1(x_23, x_1, x_60); +x_62 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_39, x_18, x_61); +x_63 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_63, 0, x_36); +lean_ctor_set(x_63, 1, x_37); +lean_ctor_set(x_63, 2, x_38); +lean_ctor_set(x_63, 3, x_62); +lean_ctor_set(x_63, 4, x_40); +lean_ctor_set(x_63, 5, x_41); +lean_ctor_set(x_63, 6, x_42); +lean_ctor_set(x_63, 7, x_44); +lean_ctor_set(x_63, 8, x_45); +lean_ctor_set(x_63, 9, x_46); +lean_ctor_set(x_63, 10, x_47); +lean_ctor_set(x_63, 11, x_48); +lean_ctor_set(x_63, 12, x_49); +lean_ctor_set(x_63, 13, x_50); +lean_ctor_set(x_63, 14, x_51); +lean_ctor_set(x_63, 15, x_52); +lean_ctor_set(x_63, 16, x_53); +lean_ctor_set(x_63, 17, x_54); +lean_ctor_set(x_63, 18, x_55); +lean_ctor_set(x_63, 19, x_56); +lean_ctor_set(x_63, 20, x_57); +lean_ctor_set(x_63, 21, x_58); +lean_ctor_set(x_63, 22, x_59); +lean_ctor_set_uint8(x_63, sizeof(void*)*23, x_43); +x_64 = lean_st_ref_set(x_3, x_63, x_25); x_65 = lean_ctor_get(x_64, 1); lean_inc(x_65); if (lean_is_exclusive(x_64)) { @@ -17615,6 +18006,206 @@ return x_67; } } } +else +{ +lean_object* x_77; lean_object* x_78; lean_object* x_79; +x_77 = lean_ctor_get(x_12, 0); +x_78 = lean_ctor_get(x_12, 1); +lean_inc(x_78); +lean_inc(x_77); +lean_dec(x_12); +x_79 = l_Lean_Meta_Grind_Goal_getRoot_x3f(x_77, x_2); +if (lean_obj_tag(x_79) == 0) +{ +lean_object* x_80; lean_object* x_81; +lean_dec(x_1); +x_80 = lean_box(0); +x_81 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_78); +return x_81; +} +else +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_124; lean_object* x_125; +x_82 = lean_ctor_get(x_79, 0); +lean_inc(x_82); +lean_dec(x_79); +x_83 = lean_st_ref_get(x_3, x_78); +x_84 = lean_ctor_get(x_83, 0); +lean_inc(x_84); +x_85 = lean_ctor_get(x_83, 1); +lean_inc(x_85); +lean_dec(x_83); +x_86 = lean_ctor_get(x_84, 3); +lean_inc(x_86); +lean_dec(x_84); +x_124 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_86, x_82); +x_125 = lean_st_ref_take(x_3, x_85); +if (lean_obj_tag(x_124) == 0) +{ +lean_object* x_126; lean_object* x_127; lean_object* x_128; +x_126 = lean_ctor_get(x_125, 0); +lean_inc(x_126); +x_127 = lean_ctor_get(x_125, 1); +lean_inc(x_127); +lean_dec(x_125); +x_128 = lean_box(0); +x_87 = x_128; +x_88 = x_126; +x_89 = x_127; +goto block_123; +} +else +{ +lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_ctor_get(x_125, 0); +lean_inc(x_130); +x_131 = lean_ctor_get(x_125, 1); +lean_inc(x_131); +lean_dec(x_125); +x_87 = x_129; +x_88 = x_130; +x_89 = x_131; +goto block_123; +} +block_123: +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; +x_90 = lean_ctor_get(x_88, 0); +lean_inc(x_90); +x_91 = lean_ctor_get(x_88, 1); +lean_inc(x_91); +x_92 = lean_ctor_get(x_88, 2); +lean_inc(x_92); +x_93 = lean_ctor_get(x_88, 3); +lean_inc(x_93); +x_94 = lean_ctor_get(x_88, 4); +lean_inc(x_94); +x_95 = lean_ctor_get(x_88, 5); +lean_inc(x_95); +x_96 = lean_ctor_get(x_88, 6); +lean_inc(x_96); +x_97 = lean_ctor_get_uint8(x_88, sizeof(void*)*23); +x_98 = lean_ctor_get(x_88, 7); +lean_inc(x_98); +x_99 = lean_ctor_get(x_88, 8); +lean_inc(x_99); +x_100 = lean_ctor_get(x_88, 9); +lean_inc(x_100); +x_101 = lean_ctor_get(x_88, 10); +lean_inc(x_101); +x_102 = lean_ctor_get(x_88, 11); +lean_inc(x_102); +x_103 = lean_ctor_get(x_88, 12); +lean_inc(x_103); +x_104 = lean_ctor_get(x_88, 13); +lean_inc(x_104); +x_105 = lean_ctor_get(x_88, 14); +lean_inc(x_105); +x_106 = lean_ctor_get(x_88, 15); +lean_inc(x_106); +x_107 = lean_ctor_get(x_88, 16); +lean_inc(x_107); +x_108 = lean_ctor_get(x_88, 17); +lean_inc(x_108); +x_109 = lean_ctor_get(x_88, 18); +lean_inc(x_109); +x_110 = lean_ctor_get(x_88, 19); +lean_inc(x_110); +x_111 = lean_ctor_get(x_88, 20); +lean_inc(x_111); +x_112 = lean_ctor_get(x_88, 21); +lean_inc(x_112); +x_113 = lean_ctor_get(x_88, 22); +lean_inc(x_113); +if (lean_is_exclusive(x_88)) { + lean_ctor_release(x_88, 0); + lean_ctor_release(x_88, 1); + lean_ctor_release(x_88, 2); + lean_ctor_release(x_88, 3); + lean_ctor_release(x_88, 4); + lean_ctor_release(x_88, 5); + lean_ctor_release(x_88, 6); + lean_ctor_release(x_88, 7); + lean_ctor_release(x_88, 8); + lean_ctor_release(x_88, 9); + lean_ctor_release(x_88, 10); + lean_ctor_release(x_88, 11); + lean_ctor_release(x_88, 12); + lean_ctor_release(x_88, 13); + lean_ctor_release(x_88, 14); + lean_ctor_release(x_88, 15); + lean_ctor_release(x_88, 16); + lean_ctor_release(x_88, 17); + lean_ctor_release(x_88, 18); + lean_ctor_release(x_88, 19); + lean_ctor_release(x_88, 20); + lean_ctor_release(x_88, 21); + lean_ctor_release(x_88, 22); + x_114 = x_88; +} else { + lean_dec_ref(x_88); + x_114 = lean_box(0); +} +x_115 = lean_box(0); +x_116 = l_Lean_RBNode_insert___at_Lean_Meta_Grind_registerParent___spec__1(x_87, x_1, x_115); +x_117 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_93, x_82, x_116); +if (lean_is_scalar(x_114)) { + x_118 = lean_alloc_ctor(0, 23, 1); +} else { + x_118 = x_114; +} +lean_ctor_set(x_118, 0, x_90); +lean_ctor_set(x_118, 1, x_91); +lean_ctor_set(x_118, 2, x_92); +lean_ctor_set(x_118, 3, x_117); +lean_ctor_set(x_118, 4, x_94); +lean_ctor_set(x_118, 5, x_95); +lean_ctor_set(x_118, 6, x_96); +lean_ctor_set(x_118, 7, x_98); +lean_ctor_set(x_118, 8, x_99); +lean_ctor_set(x_118, 9, x_100); +lean_ctor_set(x_118, 10, x_101); +lean_ctor_set(x_118, 11, x_102); +lean_ctor_set(x_118, 12, x_103); +lean_ctor_set(x_118, 13, x_104); +lean_ctor_set(x_118, 14, x_105); +lean_ctor_set(x_118, 15, x_106); +lean_ctor_set(x_118, 16, x_107); +lean_ctor_set(x_118, 17, x_108); +lean_ctor_set(x_118, 18, x_109); +lean_ctor_set(x_118, 19, x_110); +lean_ctor_set(x_118, 20, x_111); +lean_ctor_set(x_118, 21, x_112); +lean_ctor_set(x_118, 22, x_113); +lean_ctor_set_uint8(x_118, sizeof(void*)*23, x_97); +x_119 = lean_st_ref_set(x_3, x_118, x_89); +x_120 = lean_ctor_get(x_119, 1); +lean_inc(x_120); +if (lean_is_exclusive(x_119)) { + lean_ctor_release(x_119, 0); + lean_ctor_release(x_119, 1); + x_121 = x_119; +} else { + lean_dec_ref(x_119); + x_121 = lean_box(0); +} +if (lean_is_scalar(x_121)) { + x_122 = lean_alloc_ctor(0, 2, 0); +} else { + x_122 = x_121; +} +lean_ctor_set(x_122, 0, x_115); +lean_ctor_set(x_122, 1, x_120); +return x_122; +} +} +} +} } LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_insertAux_traverse___at_Lean_Meta_Grind_registerParent___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: @@ -17698,7 +18289,7 @@ if (x_12 == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 2); +x_14 = lean_ctor_get(x_13, 3); lean_inc(x_14); lean_dec(x_13); x_15 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_14, x_1); @@ -17727,7 +18318,7 @@ x_19 = lean_ctor_get(x_11, 1); lean_inc(x_19); lean_inc(x_18); lean_dec(x_11); -x_20 = lean_ctor_get(x_18, 2); +x_20 = lean_ctor_get(x_18, 3); lean_inc(x_20); lean_dec(x_18); x_21 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_20, x_1); @@ -18143,9 +18734,9 @@ x_17 = !lean_is_exclusive(x_15); if (x_17 == 0) { lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_ctor_get(x_15, 2); +x_18 = lean_ctor_get(x_15, 3); x_19 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_getParentsAndReset___spec__1(x_18, x_1); -lean_ctor_set(x_15, 2, x_19); +lean_ctor_set(x_15, 3, x_19); x_20 = lean_st_ref_set(x_2, x_15, x_16); x_21 = !lean_is_exclusive(x_20); if (x_21 == 0) @@ -18170,15 +18761,15 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; x_25 = lean_ctor_get(x_15, 0); x_26 = lean_ctor_get(x_15, 1); x_27 = lean_ctor_get(x_15, 2); x_28 = lean_ctor_get(x_15, 3); x_29 = lean_ctor_get(x_15, 4); x_30 = lean_ctor_get(x_15, 5); -x_31 = lean_ctor_get_uint8(x_15, sizeof(void*)*20); -x_32 = lean_ctor_get(x_15, 6); +x_31 = lean_ctor_get(x_15, 6); +x_32 = lean_ctor_get_uint8(x_15, sizeof(void*)*23); x_33 = lean_ctor_get(x_15, 7); x_34 = lean_ctor_get(x_15, 8); x_35 = lean_ctor_get(x_15, 9); @@ -18192,6 +18783,12 @@ x_42 = lean_ctor_get(x_15, 16); x_43 = lean_ctor_get(x_15, 17); x_44 = lean_ctor_get(x_15, 18); x_45 = lean_ctor_get(x_15, 19); +x_46 = lean_ctor_get(x_15, 20); +x_47 = lean_ctor_get(x_15, 21); +x_48 = lean_ctor_get(x_15, 22); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); @@ -18205,7 +18802,7 @@ lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); +lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); @@ -18213,48 +18810,51 @@ lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_dec(x_15); -x_46 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_getParentsAndReset___spec__1(x_27, x_1); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_25); -lean_ctor_set(x_47, 1, x_26); -lean_ctor_set(x_47, 2, x_46); -lean_ctor_set(x_47, 3, x_28); -lean_ctor_set(x_47, 4, x_29); -lean_ctor_set(x_47, 5, x_30); -lean_ctor_set(x_47, 6, x_32); -lean_ctor_set(x_47, 7, x_33); -lean_ctor_set(x_47, 8, x_34); -lean_ctor_set(x_47, 9, x_35); -lean_ctor_set(x_47, 10, x_36); -lean_ctor_set(x_47, 11, x_37); -lean_ctor_set(x_47, 12, x_38); -lean_ctor_set(x_47, 13, x_39); -lean_ctor_set(x_47, 14, x_40); -lean_ctor_set(x_47, 15, x_41); -lean_ctor_set(x_47, 16, x_42); -lean_ctor_set(x_47, 17, x_43); -lean_ctor_set(x_47, 18, x_44); -lean_ctor_set(x_47, 19, x_45); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_31); -x_48 = lean_st_ref_set(x_2, x_47, x_16); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_49 = l_Lean_PersistentHashMap_erase___at_Lean_Meta_Grind_getParentsAndReset___spec__1(x_28, x_1); +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_25); +lean_ctor_set(x_50, 1, x_26); +lean_ctor_set(x_50, 2, x_27); +lean_ctor_set(x_50, 3, x_49); +lean_ctor_set(x_50, 4, x_29); +lean_ctor_set(x_50, 5, x_30); +lean_ctor_set(x_50, 6, x_31); +lean_ctor_set(x_50, 7, x_33); +lean_ctor_set(x_50, 8, x_34); +lean_ctor_set(x_50, 9, x_35); +lean_ctor_set(x_50, 10, x_36); +lean_ctor_set(x_50, 11, x_37); +lean_ctor_set(x_50, 12, x_38); +lean_ctor_set(x_50, 13, x_39); +lean_ctor_set(x_50, 14, x_40); +lean_ctor_set(x_50, 15, x_41); +lean_ctor_set(x_50, 16, x_42); +lean_ctor_set(x_50, 17, x_43); +lean_ctor_set(x_50, 18, x_44); +lean_ctor_set(x_50, 19, x_45); +lean_ctor_set(x_50, 20, x_46); +lean_ctor_set(x_50, 21, x_47); +lean_ctor_set(x_50, 22, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_32); +x_51 = lean_st_ref_set(x_2, x_50, x_16); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_50; + x_54 = x_53; } -lean_ctor_set(x_51, 0, x_12); -lean_ctor_set(x_51, 1, x_49); -return x_51; +lean_ctor_set(x_54, 0, x_12); +lean_ctor_set(x_54, 1, x_52); +return x_54; } } } @@ -18349,54 +18949,54 @@ goto _start; LEAN_EXPORT lean_object* l_Lean_Meta_Grind_copyParentsTo(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_60; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_63; x_12 = lean_st_ref_get(x_3, x_11); x_13 = lean_ctor_get(x_12, 0); lean_inc(x_13); x_14 = lean_ctor_get(x_12, 1); lean_inc(x_14); lean_dec(x_12); -x_15 = lean_ctor_get(x_13, 2); +x_15 = lean_ctor_get(x_13, 3); lean_inc(x_15); lean_dec(x_13); -x_60 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_15, x_2); -if (lean_obj_tag(x_60) == 0) +x_63 = l_Lean_PersistentHashMap_find_x3f___at_Lean_Meta_Grind_registerParent___spec__7(x_15, x_2); +if (lean_obj_tag(x_63) == 0) { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_61 = lean_box(0); -x_62 = l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1(x_1, x_61, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -x_63 = lean_ctor_get(x_62, 0); -lean_inc(x_63); -x_64 = lean_ctor_get(x_62, 1); -lean_inc(x_64); -lean_dec(x_62); -x_65 = lean_ctor_get(x_63, 0); -lean_inc(x_65); -lean_dec(x_63); -x_16 = x_65; -x_17 = x_64; -goto block_59; +lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_64 = lean_box(0); +x_65 = l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1(x_1, x_64, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +x_66 = lean_ctor_get(x_65, 0); +lean_inc(x_66); +x_67 = lean_ctor_get(x_65, 1); +lean_inc(x_67); +lean_dec(x_65); +x_68 = lean_ctor_get(x_66, 0); +lean_inc(x_68); +lean_dec(x_66); +x_16 = x_68; +x_17 = x_67; +goto block_62; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; -x_66 = lean_ctor_get(x_60, 0); -lean_inc(x_66); -lean_dec(x_60); -x_67 = l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1(x_1, x_66, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); -x_68 = lean_ctor_get(x_67, 0); -lean_inc(x_68); -x_69 = lean_ctor_get(x_67, 1); +lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_69 = lean_ctor_get(x_63, 0); lean_inc(x_69); -lean_dec(x_67); -x_70 = lean_ctor_get(x_68, 0); -lean_inc(x_70); -lean_dec(x_68); -x_16 = x_70; -x_17 = x_69; -goto block_59; +lean_dec(x_63); +x_70 = l_Lean_RBNode_forIn_visit___at_Lean_Meta_Grind_copyParentsTo___spec__1(x_1, x_69, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_14); +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_ctor_get(x_71, 0); +lean_inc(x_73); +lean_dec(x_71); +x_16 = x_73; +x_17 = x_72; +goto block_62; } -block_59: +block_62: { lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; x_18 = lean_st_ref_take(x_3, x_17); @@ -18409,9 +19009,9 @@ x_21 = !lean_is_exclusive(x_19); if (x_21 == 0) { lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_22 = lean_ctor_get(x_19, 2); +x_22 = lean_ctor_get(x_19, 3); x_23 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_22, x_2, x_16); -lean_ctor_set(x_19, 2, x_23); +lean_ctor_set(x_19, 3, x_23); x_24 = lean_st_ref_set(x_3, x_19, x_20); x_25 = !lean_is_exclusive(x_24); if (x_25 == 0) @@ -18438,15 +19038,15 @@ return x_30; } else { -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; x_31 = lean_ctor_get(x_19, 0); x_32 = lean_ctor_get(x_19, 1); x_33 = lean_ctor_get(x_19, 2); x_34 = lean_ctor_get(x_19, 3); x_35 = lean_ctor_get(x_19, 4); x_36 = lean_ctor_get(x_19, 5); -x_37 = lean_ctor_get_uint8(x_19, sizeof(void*)*20); -x_38 = lean_ctor_get(x_19, 6); +x_37 = lean_ctor_get(x_19, 6); +x_38 = lean_ctor_get_uint8(x_19, sizeof(void*)*23); x_39 = lean_ctor_get(x_19, 7); x_40 = lean_ctor_get(x_19, 8); x_41 = lean_ctor_get(x_19, 9); @@ -18460,6 +19060,12 @@ x_48 = lean_ctor_get(x_19, 16); x_49 = lean_ctor_get(x_19, 17); x_50 = lean_ctor_get(x_19, 18); x_51 = lean_ctor_get(x_19, 19); +x_52 = lean_ctor_get(x_19, 20); +x_53 = lean_ctor_get(x_19, 21); +x_54 = lean_ctor_get(x_19, 22); +lean_inc(x_54); +lean_inc(x_53); +lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); lean_inc(x_49); @@ -18473,7 +19079,7 @@ lean_inc(x_42); lean_inc(x_41); lean_inc(x_40); lean_inc(x_39); -lean_inc(x_38); +lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); @@ -18481,49 +19087,52 @@ lean_inc(x_33); lean_inc(x_32); lean_inc(x_31); lean_dec(x_19); -x_52 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_33, x_2, x_16); -x_53 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_53, 0, x_31); -lean_ctor_set(x_53, 1, x_32); -lean_ctor_set(x_53, 2, x_52); -lean_ctor_set(x_53, 3, x_34); -lean_ctor_set(x_53, 4, x_35); -lean_ctor_set(x_53, 5, x_36); -lean_ctor_set(x_53, 6, x_38); -lean_ctor_set(x_53, 7, x_39); -lean_ctor_set(x_53, 8, x_40); -lean_ctor_set(x_53, 9, x_41); -lean_ctor_set(x_53, 10, x_42); -lean_ctor_set(x_53, 11, x_43); -lean_ctor_set(x_53, 12, x_44); -lean_ctor_set(x_53, 13, x_45); -lean_ctor_set(x_53, 14, x_46); -lean_ctor_set(x_53, 15, x_47); -lean_ctor_set(x_53, 16, x_48); -lean_ctor_set(x_53, 17, x_49); -lean_ctor_set(x_53, 18, x_50); -lean_ctor_set(x_53, 19, x_51); -lean_ctor_set_uint8(x_53, sizeof(void*)*20, x_37); -x_54 = lean_st_ref_set(x_3, x_53, x_20); -x_55 = lean_ctor_get(x_54, 1); -lean_inc(x_55); -if (lean_is_exclusive(x_54)) { - lean_ctor_release(x_54, 0); - lean_ctor_release(x_54, 1); - x_56 = x_54; +x_55 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_registerParent___spec__3(x_34, x_2, x_16); +x_56 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_56, 0, x_31); +lean_ctor_set(x_56, 1, x_32); +lean_ctor_set(x_56, 2, x_33); +lean_ctor_set(x_56, 3, x_55); +lean_ctor_set(x_56, 4, x_35); +lean_ctor_set(x_56, 5, x_36); +lean_ctor_set(x_56, 6, x_37); +lean_ctor_set(x_56, 7, x_39); +lean_ctor_set(x_56, 8, x_40); +lean_ctor_set(x_56, 9, x_41); +lean_ctor_set(x_56, 10, x_42); +lean_ctor_set(x_56, 11, x_43); +lean_ctor_set(x_56, 12, x_44); +lean_ctor_set(x_56, 13, x_45); +lean_ctor_set(x_56, 14, x_46); +lean_ctor_set(x_56, 15, x_47); +lean_ctor_set(x_56, 16, x_48); +lean_ctor_set(x_56, 17, x_49); +lean_ctor_set(x_56, 18, x_50); +lean_ctor_set(x_56, 19, x_51); +lean_ctor_set(x_56, 20, x_52); +lean_ctor_set(x_56, 21, x_53); +lean_ctor_set(x_56, 22, x_54); +lean_ctor_set_uint8(x_56, sizeof(void*)*23, x_38); +x_57 = lean_st_ref_set(x_3, x_56, x_20); +x_58 = lean_ctor_get(x_57, 1); +lean_inc(x_58); +if (lean_is_exclusive(x_57)) { + lean_ctor_release(x_57, 0); + lean_ctor_release(x_57, 1); + x_59 = x_57; } else { - lean_dec_ref(x_54); - x_56 = lean_box(0); + lean_dec_ref(x_57); + x_59 = lean_box(0); } -x_57 = lean_box(0); -if (lean_is_scalar(x_56)) { - x_58 = lean_alloc_ctor(0, 2, 0); +x_60 = lean_box(0); +if (lean_is_scalar(x_59)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_58 = x_56; + x_61 = x_59; } -lean_ctor_set(x_58, 0, x_57); -lean_ctor_set(x_58, 1, x_55); -return x_58; +lean_ctor_set(x_61, 0, x_60); +lean_ctor_set(x_61, 1, x_58); +return x_61; } } } @@ -18564,7 +19173,7 @@ LEAN_EXPORT lean_object* l_Lean_Meta_Grind_setENode_unsafe__1___rarg(lean_object _start: { lean_object* x_2; -x_2 = lean_ctor_get(x_1, 3); +x_2 = lean_ctor_get(x_1, 4); lean_inc(x_2); return x_2; } @@ -19112,9 +19721,9 @@ x_15 = !lean_is_exclusive(x_13); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_16 = lean_ctor_get(x_13, 1); +x_16 = lean_ctor_get(x_13, 2); x_17 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_setENode___spec__1(x_16, x_1, x_2); -lean_ctor_set(x_13, 1, x_17); +lean_ctor_set(x_13, 2, x_17); x_18 = lean_st_ref_set(x_3, x_13, x_14); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) @@ -19141,15 +19750,15 @@ return x_24; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; uint8_t x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; x_25 = lean_ctor_get(x_13, 0); x_26 = lean_ctor_get(x_13, 1); x_27 = lean_ctor_get(x_13, 2); x_28 = lean_ctor_get(x_13, 3); x_29 = lean_ctor_get(x_13, 4); x_30 = lean_ctor_get(x_13, 5); -x_31 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_32 = lean_ctor_get(x_13, 6); +x_31 = lean_ctor_get(x_13, 6); +x_32 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_33 = lean_ctor_get(x_13, 7); x_34 = lean_ctor_get(x_13, 8); x_35 = lean_ctor_get(x_13, 9); @@ -19163,6 +19772,12 @@ x_42 = lean_ctor_get(x_13, 16); x_43 = lean_ctor_get(x_13, 17); x_44 = lean_ctor_get(x_13, 18); x_45 = lean_ctor_get(x_13, 19); +x_46 = lean_ctor_get(x_13, 20); +x_47 = lean_ctor_get(x_13, 21); +x_48 = lean_ctor_get(x_13, 22); +lean_inc(x_48); +lean_inc(x_47); +lean_inc(x_46); lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); @@ -19176,7 +19791,7 @@ lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); -lean_inc(x_32); +lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); @@ -19184,49 +19799,52 @@ lean_inc(x_27); lean_inc(x_26); lean_inc(x_25); lean_dec(x_13); -x_46 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_setENode___spec__1(x_26, x_1, x_2); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_25); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_27); -lean_ctor_set(x_47, 3, x_28); -lean_ctor_set(x_47, 4, x_29); -lean_ctor_set(x_47, 5, x_30); -lean_ctor_set(x_47, 6, x_32); -lean_ctor_set(x_47, 7, x_33); -lean_ctor_set(x_47, 8, x_34); -lean_ctor_set(x_47, 9, x_35); -lean_ctor_set(x_47, 10, x_36); -lean_ctor_set(x_47, 11, x_37); -lean_ctor_set(x_47, 12, x_38); -lean_ctor_set(x_47, 13, x_39); -lean_ctor_set(x_47, 14, x_40); -lean_ctor_set(x_47, 15, x_41); -lean_ctor_set(x_47, 16, x_42); -lean_ctor_set(x_47, 17, x_43); -lean_ctor_set(x_47, 18, x_44); -lean_ctor_set(x_47, 19, x_45); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_31); -x_48 = lean_st_ref_set(x_3, x_47, x_14); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; -} else { - lean_dec_ref(x_48); - x_50 = lean_box(0); -} -x_51 = lean_box(0); -if (lean_is_scalar(x_50)) { - x_52 = lean_alloc_ctor(0, 2, 0); +x_49 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_setENode___spec__1(x_27, x_1, x_2); +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_25); +lean_ctor_set(x_50, 1, x_26); +lean_ctor_set(x_50, 2, x_49); +lean_ctor_set(x_50, 3, x_28); +lean_ctor_set(x_50, 4, x_29); +lean_ctor_set(x_50, 5, x_30); +lean_ctor_set(x_50, 6, x_31); +lean_ctor_set(x_50, 7, x_33); +lean_ctor_set(x_50, 8, x_34); +lean_ctor_set(x_50, 9, x_35); +lean_ctor_set(x_50, 10, x_36); +lean_ctor_set(x_50, 11, x_37); +lean_ctor_set(x_50, 12, x_38); +lean_ctor_set(x_50, 13, x_39); +lean_ctor_set(x_50, 14, x_40); +lean_ctor_set(x_50, 15, x_41); +lean_ctor_set(x_50, 16, x_42); +lean_ctor_set(x_50, 17, x_43); +lean_ctor_set(x_50, 18, x_44); +lean_ctor_set(x_50, 19, x_45); +lean_ctor_set(x_50, 20, x_46); +lean_ctor_set(x_50, 21, x_47); +lean_ctor_set(x_50, 22, x_48); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_32); +x_51 = lean_st_ref_set(x_3, x_50, x_14); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - x_52 = x_50; + lean_dec_ref(x_51); + x_53 = lean_box(0); } -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_49); -return x_52; +x_54 = lean_box(0); +if (lean_is_scalar(x_53)) { + x_55 = lean_alloc_ctor(0, 2, 0); +} else { + x_55 = x_53; +} +lean_ctor_set(x_55, 0, x_54); +lean_ctor_set(x_55, 1, x_52); +return x_55; } } } @@ -19288,16 +19906,16 @@ lean_inc(x_19); lean_dec(x_17); x_20 = lean_box(0); x_21 = l_Lean_Expr_isLambda(x_1); -x_22 = lean_ctor_get(x_18, 7); +x_22 = lean_ctor_get(x_18, 8); lean_inc(x_22); lean_dec(x_18); -x_23 = lean_ctor_get(x_15, 6); +x_23 = lean_ctor_get(x_15, 7); lean_inc(x_23); lean_dec(x_15); x_24 = 0; x_25 = lean_unsigned_to_nat(1u); lean_inc_n(x_1, 4); -x_26 = lean_alloc_ctor(0, 10, 5); +x_26 = lean_alloc_ctor(0, 11, 5); lean_ctor_set(x_26, 0, x_1); lean_ctor_set(x_26, 1, x_1); lean_ctor_set(x_26, 2, x_1); @@ -19308,11 +19926,12 @@ lean_ctor_set(x_26, 6, x_25); lean_ctor_set(x_26, 7, x_22); lean_ctor_set(x_26, 8, x_4); lean_ctor_set(x_26, 9, x_23); -lean_ctor_set_uint8(x_26, sizeof(void*)*10, x_24); -lean_ctor_set_uint8(x_26, sizeof(void*)*10 + 1, x_2); -lean_ctor_set_uint8(x_26, sizeof(void*)*10 + 2, x_3); -lean_ctor_set_uint8(x_26, sizeof(void*)*10 + 3, x_21); -lean_ctor_set_uint8(x_26, sizeof(void*)*10 + 4, x_24); +lean_ctor_set(x_26, 10, x_20); +lean_ctor_set_uint8(x_26, sizeof(void*)*11, x_24); +lean_ctor_set_uint8(x_26, sizeof(void*)*11 + 1, x_2); +lean_ctor_set_uint8(x_26, sizeof(void*)*11 + 2, x_3); +lean_ctor_set_uint8(x_26, sizeof(void*)*11 + 3, x_21); +lean_ctor_set_uint8(x_26, sizeof(void*)*11 + 4, x_24); x_27 = l_Lean_Meta_Grind_setENode(x_1, x_26, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_19); x_28 = lean_ctor_get(x_27, 1); lean_inc(x_28); @@ -19327,10 +19946,10 @@ x_32 = !lean_is_exclusive(x_30); if (x_32 == 0) { lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_33 = lean_ctor_get(x_30, 7); +x_33 = lean_ctor_get(x_30, 8); x_34 = lean_nat_add(x_33, x_25); lean_dec(x_33); -lean_ctor_set(x_30, 7, x_34); +lean_ctor_set(x_30, 8, x_34); x_35 = lean_st_ref_set(x_5, x_30, x_31); x_36 = !lean_is_exclusive(x_35); if (x_36 == 0) @@ -19357,15 +19976,15 @@ return x_41; } else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; x_42 = lean_ctor_get(x_30, 0); x_43 = lean_ctor_get(x_30, 1); x_44 = lean_ctor_get(x_30, 2); x_45 = lean_ctor_get(x_30, 3); x_46 = lean_ctor_get(x_30, 4); x_47 = lean_ctor_get(x_30, 5); -x_48 = lean_ctor_get_uint8(x_30, sizeof(void*)*20); -x_49 = lean_ctor_get(x_30, 6); +x_48 = lean_ctor_get(x_30, 6); +x_49 = lean_ctor_get_uint8(x_30, sizeof(void*)*23); x_50 = lean_ctor_get(x_30, 7); x_51 = lean_ctor_get(x_30, 8); x_52 = lean_ctor_get(x_30, 9); @@ -19379,6 +19998,12 @@ x_59 = lean_ctor_get(x_30, 16); x_60 = lean_ctor_get(x_30, 17); x_61 = lean_ctor_get(x_30, 18); x_62 = lean_ctor_get(x_30, 19); +x_63 = lean_ctor_get(x_30, 20); +x_64 = lean_ctor_get(x_30, 21); +x_65 = lean_ctor_get(x_30, 22); +lean_inc(x_65); +lean_inc(x_64); +lean_inc(x_63); lean_inc(x_62); lean_inc(x_61); lean_inc(x_60); @@ -19392,7 +20017,7 @@ lean_inc(x_53); lean_inc(x_52); lean_inc(x_51); lean_inc(x_50); -lean_inc(x_49); +lean_inc(x_48); lean_inc(x_47); lean_inc(x_46); lean_inc(x_45); @@ -19400,50 +20025,53 @@ lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); lean_dec(x_30); -x_63 = lean_nat_add(x_50, x_25); -lean_dec(x_50); -x_64 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_64, 0, x_42); -lean_ctor_set(x_64, 1, x_43); -lean_ctor_set(x_64, 2, x_44); -lean_ctor_set(x_64, 3, x_45); -lean_ctor_set(x_64, 4, x_46); -lean_ctor_set(x_64, 5, x_47); -lean_ctor_set(x_64, 6, x_49); -lean_ctor_set(x_64, 7, x_63); -lean_ctor_set(x_64, 8, x_51); -lean_ctor_set(x_64, 9, x_52); -lean_ctor_set(x_64, 10, x_53); -lean_ctor_set(x_64, 11, x_54); -lean_ctor_set(x_64, 12, x_55); -lean_ctor_set(x_64, 13, x_56); -lean_ctor_set(x_64, 14, x_57); -lean_ctor_set(x_64, 15, x_58); -lean_ctor_set(x_64, 16, x_59); -lean_ctor_set(x_64, 17, x_60); -lean_ctor_set(x_64, 18, x_61); -lean_ctor_set(x_64, 19, x_62); -lean_ctor_set_uint8(x_64, sizeof(void*)*20, x_48); -x_65 = lean_st_ref_set(x_5, x_64, x_31); -x_66 = lean_ctor_get(x_65, 1); -lean_inc(x_66); -if (lean_is_exclusive(x_65)) { - lean_ctor_release(x_65, 0); - lean_ctor_release(x_65, 1); - x_67 = x_65; +x_66 = lean_nat_add(x_51, x_25); +lean_dec(x_51); +x_67 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_67, 0, x_42); +lean_ctor_set(x_67, 1, x_43); +lean_ctor_set(x_67, 2, x_44); +lean_ctor_set(x_67, 3, x_45); +lean_ctor_set(x_67, 4, x_46); +lean_ctor_set(x_67, 5, x_47); +lean_ctor_set(x_67, 6, x_48); +lean_ctor_set(x_67, 7, x_50); +lean_ctor_set(x_67, 8, x_66); +lean_ctor_set(x_67, 9, x_52); +lean_ctor_set(x_67, 10, x_53); +lean_ctor_set(x_67, 11, x_54); +lean_ctor_set(x_67, 12, x_55); +lean_ctor_set(x_67, 13, x_56); +lean_ctor_set(x_67, 14, x_57); +lean_ctor_set(x_67, 15, x_58); +lean_ctor_set(x_67, 16, x_59); +lean_ctor_set(x_67, 17, x_60); +lean_ctor_set(x_67, 18, x_61); +lean_ctor_set(x_67, 19, x_62); +lean_ctor_set(x_67, 20, x_63); +lean_ctor_set(x_67, 21, x_64); +lean_ctor_set(x_67, 22, x_65); +lean_ctor_set_uint8(x_67, sizeof(void*)*23, x_49); +x_68 = lean_st_ref_set(x_5, x_67, x_31); +x_69 = lean_ctor_get(x_68, 1); +lean_inc(x_69); +if (lean_is_exclusive(x_68)) { + lean_ctor_release(x_68, 0); + lean_ctor_release(x_68, 1); + x_70 = x_68; } else { - lean_dec_ref(x_65); - x_67 = lean_box(0); + lean_dec_ref(x_68); + x_70 = lean_box(0); } -x_68 = lean_box(0); -if (lean_is_scalar(x_67)) { - x_69 = lean_alloc_ctor(0, 2, 0); +x_71 = lean_box(0); +if (lean_is_scalar(x_70)) { + x_72 = lean_alloc_ctor(0, 2, 0); } else { - x_69 = x_67; + x_72 = x_70; } -lean_ctor_set(x_69, 0, x_68); -lean_ctor_set(x_69, 1, x_66); -return x_69; +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_69); +return x_72; } } } @@ -19662,324 +20290,341 @@ lean_dec(x_3); return x_12; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_processNewOffsetEq___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -lean_object* x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_ctor_get(x_11, 0); -x_14 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_13); -lean_dec(x_13); -x_15 = lean_box(x_14); -lean_ctor_set(x_11, 0, x_15); -return x_11; +lean_object* x_12; +x_12 = lean_process_new_offset_eq(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Arith_processNewOffsetEqLit___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -lean_object* x_16; lean_object* x_17; uint8_t x_18; lean_object* x_19; lean_object* x_20; -x_16 = lean_ctor_get(x_11, 0); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_11); -x_18 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_16); -lean_dec(x_16); -x_19 = lean_box(x_18); -x_20 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_20, 0, x_19); -lean_ctor_set(x_20, 1, x_17); -return x_20; +lean_object* x_12; +x_12 = lean_process_new_offset_eq_lit(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; } } -else -{ -uint8_t x_21; -x_21 = !lean_is_exclusive(x_11); -if (x_21 == 0) +LEAN_EXPORT uint8_t l_Lean_Meta_Grind_isNatNum___lambda__1(lean_object* x_1) { +_start: { -return x_11; +uint8_t x_2; +x_2 = 0; +return x_2; } -else +} +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1() { +_start: { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_ctor_get(x_11, 0); -x_23 = lean_ctor_get(x_11, 1); -lean_inc(x_23); -lean_inc(x_22); -lean_dec(x_11); -x_24 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_24, 0, x_22); -lean_ctor_set(x_24, 1, x_23); -return x_24; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_isNatNum___lambda__1___boxed), 1, 0); +return x_1; } } +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1; +x_2 = lean_box(0); +x_3 = lean_apply_1(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3() { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_isCongrRoot(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("instOfNatNat", 12, 12); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4() { _start: { -lean_object* x_12; lean_object* x_13; -x_12 = lean_ctor_get(x_1, 3); -lean_inc(x_12); -lean_dec(x_1); -x_13 = l_Lean_Meta_Grind_getCongrRoot(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_13; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum___lambda__2(lean_object* x_1) { _start: { -lean_object* x_11; -lean_inc(x_1); -x_11 = l_Lean_Meta_Grind_getENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) -{ -uint8_t x_12; -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_11, 1); -x_15 = lean_ctor_get(x_13, 3); -lean_inc(x_15); -x_16 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_15, x_1); -lean_dec(x_15); -if (x_16 == 0) -{ -lean_object* x_17; lean_object* x_18; -lean_free_object(x_11); -lean_dec(x_1); -x_17 = lean_box(0); -x_18 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_13, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); -return x_18; -} -else +lean_object* x_2; uint8_t x_3; +x_2 = l_Lean_Expr_cleanupAnnotations(x_1); +x_3 = l_Lean_Expr_isApp(x_2); +if (x_3 == 0) { -lean_dec(x_13); -lean_ctor_set(x_11, 0, x_1); -return x_11; -} +lean_object* x_4; +lean_dec(x_2); +x_4 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; +return x_4; } else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_19 = lean_ctor_get(x_11, 0); -x_20 = lean_ctor_get(x_11, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_11); -x_21 = lean_ctor_get(x_19, 3); -lean_inc(x_21); -x_22 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_21, x_1); -lean_dec(x_21); -if (x_22 == 0) +lean_object* x_5; lean_object* x_6; uint8_t x_7; +x_5 = l_Lean_Expr_appFnCleanup(x_2, lean_box(0)); +x_6 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4; +x_7 = l_Lean_Expr_isConstOf(x_5, x_6); +lean_dec(x_5); +if (x_7 == 0) { -lean_object* x_23; lean_object* x_24; -lean_dec(x_1); -x_23 = lean_box(0); -x_24 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_19, x_23, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_20); -return x_24; +lean_object* x_8; +x_8 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; +return x_8; } else { -lean_object* x_25; -lean_dec(x_19); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_1); -lean_ctor_set(x_25, 1, x_20); -return x_25; +uint8_t x_9; lean_object* x_10; +x_9 = 1; +x_10 = lean_box(x_9); +return x_10; } } } -else -{ -uint8_t x_26; -lean_dec(x_1); -x_26 = !lean_is_exclusive(x_11); -if (x_26 == 0) -{ -return x_11; } -else +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___closed__1() { +_start: { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_11, 0); -x_28 = lean_ctor_get(x_11, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_11); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_isNatNum___lambda__2), 1, 0); +return x_1; } } +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("OfNat", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___closed__3() { _start: { -lean_object* x_12; -x_12 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_12; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("ofNat", 5, 5); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +static lean_object* _init_l_Lean_Meta_Grind_isNatNum___closed__4() { _start: { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_getCongrRoot(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_11; +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Grind_isNatNum___closed__2; +x_2 = l_Lean_Meta_Grind_isNatNum___closed__3; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum(lean_object* x_1) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_ref_get(x_1, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +lean_object* x_2; lean_object* x_3; uint8_t x_4; +x_2 = l_Lean_Meta_Grind_isNatNum___closed__1; +x_3 = l_Lean_Expr_cleanupAnnotations(x_1); +x_4 = l_Lean_Expr_isApp(x_3); +if (x_4 == 0) { -lean_object* x_12; uint8_t x_13; lean_object* x_14; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*20); -lean_dec(x_12); -x_14 = lean_box(x_13); -lean_ctor_set(x_10, 0, x_14); -return x_10; +lean_object* x_5; +lean_dec(x_3); +x_5 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; +return x_5; } else { -lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_inc(x_15); -lean_dec(x_10); -x_17 = lean_ctor_get_uint8(x_15, sizeof(void*)*20); -lean_dec(x_15); -x_18 = lean_box(x_17); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_18); -lean_ctor_set(x_19, 1, x_16); -return x_19; -} -} -} -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = l_Lean_Expr_appArg(x_3, lean_box(0)); +x_7 = l_Lean_Expr_appFnCleanup(x_3, lean_box(0)); +x_8 = l_Lean_Expr_isApp(x_7); +if (x_8 == 0) { -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); +lean_object* x_9; lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_10; -} +x_9 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; +return x_9; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else +{ +lean_object* x_10; uint8_t x_11; +x_10 = l_Lean_Expr_appFnCleanup(x_7, lean_box(0)); +x_11 = l_Lean_Expr_isApp(x_10); +if (x_11 == 0) { lean_object* x_12; -x_12 = lean_grind_mk_eq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_6); +x_12 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; return x_12; } +else +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_13 = l_Lean_Expr_appFnCleanup(x_10, lean_box(0)); +x_14 = l_Lean_Meta_Grind_isNatNum___closed__4; +x_15 = l_Lean_Expr_isConstOf(x_13, x_14); +lean_dec(x_13); +if (x_15 == 0) +{ +lean_object* x_16; +lean_dec(x_6); +x_16 = l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2; +return x_16; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHEqProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +else +{ +lean_object* x_17; +x_17 = lean_apply_1(x_2, x_6); +return x_17; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isNatNum___lambda__1___boxed(lean_object* x_1) { _start: { -lean_object* x_12; -x_12 = lean_grind_mk_heq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -return x_12; +uint8_t x_2; lean_object* x_3; +x_2 = l_Lean_Meta_Grind_isNatNum___lambda__1(x_1); +lean_dec(x_1); +x_3 = lean_box(x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqHEqProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsOffsetTerm(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; -lean_inc(x_10); -lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_2); +lean_object* x_11; lean_inc(x_1); -x_12 = l_Lean_Meta_Grind_hasSameType(x_1, x_2, x_7, x_8, x_9, x_10, x_11); -if (lean_obj_tag(x_12) == 0) +x_11 = l_Lean_Meta_Grind_getRootENode(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) { -lean_object* x_13; uint8_t x_14; -x_13 = lean_ctor_get(x_12, 0); +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_12, 10); lean_inc(x_13); -x_14 = lean_unbox(x_13); -lean_dec(x_13); -if (x_14 == 0) +if (lean_obj_tag(x_13) == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = lean_ctor_get(x_12, 1); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; uint8_t x_25; uint8_t x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_36; uint8_t x_37; +x_14 = lean_ctor_get(x_11, 1); +lean_inc(x_14); +lean_dec(x_11); +x_15 = lean_ctor_get(x_12, 0); lean_inc(x_15); -lean_dec(x_12); -x_16 = lean_grind_mk_heq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); -return x_16; +x_16 = lean_ctor_get(x_12, 1); +lean_inc(x_16); +x_17 = lean_ctor_get(x_12, 2); +lean_inc(x_17); +x_18 = lean_ctor_get(x_12, 3); +lean_inc(x_18); +x_19 = lean_ctor_get(x_12, 4); +lean_inc(x_19); +x_20 = lean_ctor_get(x_12, 5); +lean_inc(x_20); +x_21 = lean_ctor_get_uint8(x_12, sizeof(void*)*11); +x_22 = lean_ctor_get(x_12, 6); +lean_inc(x_22); +x_23 = lean_ctor_get_uint8(x_12, sizeof(void*)*11 + 1); +x_24 = lean_ctor_get_uint8(x_12, sizeof(void*)*11 + 2); +x_25 = lean_ctor_get_uint8(x_12, sizeof(void*)*11 + 3); +x_26 = lean_ctor_get_uint8(x_12, sizeof(void*)*11 + 4); +x_27 = lean_ctor_get(x_12, 7); +lean_inc(x_27); +x_28 = lean_ctor_get(x_12, 8); +lean_inc(x_28); +x_29 = lean_ctor_get(x_12, 9); +lean_inc(x_29); +if (lean_is_exclusive(x_12)) { + lean_ctor_release(x_12, 0); + lean_ctor_release(x_12, 1); + lean_ctor_release(x_12, 2); + lean_ctor_release(x_12, 3); + lean_ctor_release(x_12, 4); + lean_ctor_release(x_12, 5); + lean_ctor_release(x_12, 6); + lean_ctor_release(x_12, 7); + lean_ctor_release(x_12, 8); + lean_ctor_release(x_12, 9); + lean_ctor_release(x_12, 10); + x_30 = x_12; +} else { + lean_dec_ref(x_12); + x_30 = lean_box(0); } -else +lean_inc(x_15); +x_36 = l_Lean_Meta_Grind_isNatNum(x_15); +x_37 = lean_unbox(x_36); +lean_dec(x_36); +if (x_37 == 0) { -lean_object* x_17; lean_object* x_18; -x_17 = lean_ctor_get(x_12, 1); -lean_inc(x_17); -lean_dec(x_12); -x_18 = lean_grind_mk_eq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); -return x_18; +lean_object* x_38; +x_38 = lean_box(0); +x_31 = x_38; +goto block_35; } +else +{ +uint8_t x_39; +x_39 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); +if (x_39 == 0) +{ +lean_object* x_40; +lean_dec(x_30); +lean_dec(x_29); +lean_dec(x_28); +lean_dec(x_27); +lean_dec(x_22); +lean_dec(x_20); +lean_dec(x_19); +lean_dec(x_18); +lean_dec(x_17); +lean_dec(x_16); +x_40 = lean_process_new_offset_eq_lit(x_1, x_15, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); +return x_40; } else { -uint8_t x_19; -lean_dec(x_10); +lean_object* x_41; +x_41 = lean_box(0); +x_31 = x_41; +goto block_35; +} +} +block_35: +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; +lean_dec(x_31); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_1); +lean_inc(x_15); +if (lean_is_scalar(x_30)) { + x_33 = lean_alloc_ctor(0, 11, 5); +} else { + x_33 = x_30; +} +lean_ctor_set(x_33, 0, x_15); +lean_ctor_set(x_33, 1, x_16); +lean_ctor_set(x_33, 2, x_17); +lean_ctor_set(x_33, 3, x_18); +lean_ctor_set(x_33, 4, x_19); +lean_ctor_set(x_33, 5, x_20); +lean_ctor_set(x_33, 6, x_22); +lean_ctor_set(x_33, 7, x_27); +lean_ctor_set(x_33, 8, x_28); +lean_ctor_set(x_33, 9, x_29); +lean_ctor_set(x_33, 10, x_32); +lean_ctor_set_uint8(x_33, sizeof(void*)*11, x_21); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 1, x_23); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 2, x_24); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 3, x_25); +lean_ctor_set_uint8(x_33, sizeof(void*)*11 + 4, x_26); +x_34 = l_Lean_Meta_Grind_setENode(x_15, x_33, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_14); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -19988,290 +20633,253 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_19 = !lean_is_exclusive(x_12); -if (x_19 == 0) -{ -return x_12; +return x_34; +} } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_12, 0); -x_21 = lean_ctor_get(x_12, 1); -lean_inc(x_21); -lean_inc(x_20); +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_dec(x_12); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_20); -lean_ctor_set(x_22, 1, x_21); -return x_22; -} +x_42 = lean_ctor_get(x_11, 1); +lean_inc(x_42); +lean_dec(x_11); +x_43 = lean_ctor_get(x_13, 0); +lean_inc(x_43); +lean_dec(x_13); +x_44 = lean_process_new_offset_eq(x_1, x_43, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_42); +return x_44; } } +else +{ +uint8_t x_45; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_45 = !lean_is_exclusive(x_11); +if (x_45 == 0) +{ +return x_11; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); +lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_46 = lean_ctor_get(x_11, 0); +x_47 = lean_ctor_get(x_11, 1); +lean_inc(x_47); +lean_inc(x_46); lean_dec(x_11); -x_14 = lean_grind_mk_eq_proof(x_1, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_14; +x_48 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_48, 0, x_46); +lean_ctor_set(x_48, 1, x_47); +return x_48; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; -x_11 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_10); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_grind_mk_eq_proof(x_1, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); -return x_14; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = lean_st_ref_take(x_2, x_10); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); x_12 = lean_ctor_get(x_11, 0); lean_inc(x_12); x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); lean_dec(x_11); -x_14 = !lean_is_exclusive(x_12); -if (x_14 == 0) +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) { -uint8_t x_15; lean_object* x_16; uint8_t x_17; -x_15 = 1; -lean_ctor_set_uint8(x_12, sizeof(void*)*20, x_15); -x_16 = lean_st_ref_set(x_2, x_12, x_13); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = lean_ctor_get(x_16, 0); -lean_dec(x_18); -x_19 = lean_box(0); -lean_ctor_set(x_16, 0, x_19); -return x_16; +lean_object* x_16; uint8_t x_17; lean_object* x_18; +x_16 = lean_ctor_get(x_14, 0); +x_17 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_16); +lean_dec(x_16); +x_18 = lean_box(x_17); +lean_ctor_set(x_14, 0, x_18); +return x_14; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_20 = lean_ctor_get(x_16, 1); +lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_14, 0); +x_20 = lean_ctor_get(x_14, 1); lean_inc(x_20); -lean_dec(x_16); -x_21 = lean_box(0); -x_22 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_22, 0, x_21); -lean_ctor_set(x_22, 1, x_20); -return x_22; +lean_inc(x_19); +lean_dec(x_14); +x_21 = l_Lean_Meta_Grind_ENode_isCongrRoot(x_19); +lean_dec(x_19); +x_22 = lean_box(x_21); +x_23 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_23, 0, x_22); +lean_ctor_set(x_23, 1, x_20); +return x_23; } } else { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_23 = lean_ctor_get(x_12, 0); -x_24 = lean_ctor_get(x_12, 1); -x_25 = lean_ctor_get(x_12, 2); -x_26 = lean_ctor_get(x_12, 3); -x_27 = lean_ctor_get(x_12, 4); -x_28 = lean_ctor_get(x_12, 5); -x_29 = lean_ctor_get(x_12, 6); -x_30 = lean_ctor_get(x_12, 7); -x_31 = lean_ctor_get(x_12, 8); -x_32 = lean_ctor_get(x_12, 9); -x_33 = lean_ctor_get(x_12, 10); -x_34 = lean_ctor_get(x_12, 11); -x_35 = lean_ctor_get(x_12, 12); -x_36 = lean_ctor_get(x_12, 13); -x_37 = lean_ctor_get(x_12, 14); -x_38 = lean_ctor_get(x_12, 15); -x_39 = lean_ctor_get(x_12, 16); -x_40 = lean_ctor_get(x_12, 17); -x_41 = lean_ctor_get(x_12, 18); -x_42 = lean_ctor_get(x_12, 19); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); -lean_inc(x_39); -lean_inc(x_38); -lean_inc(x_37); -lean_inc(x_36); -lean_inc(x_35); -lean_inc(x_34); -lean_inc(x_33); -lean_inc(x_32); -lean_inc(x_31); -lean_inc(x_30); -lean_inc(x_29); -lean_inc(x_28); -lean_inc(x_27); +uint8_t x_24; +x_24 = !lean_is_exclusive(x_14); +if (x_24 == 0) +{ +return x_14; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_14, 0); +x_26 = lean_ctor_get(x_14, 1); lean_inc(x_26); lean_inc(x_25); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_12); -x_43 = 1; -x_44 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_44, 0, x_23); -lean_ctor_set(x_44, 1, x_24); -lean_ctor_set(x_44, 2, x_25); -lean_ctor_set(x_44, 3, x_26); -lean_ctor_set(x_44, 4, x_27); -lean_ctor_set(x_44, 5, x_28); -lean_ctor_set(x_44, 6, x_29); -lean_ctor_set(x_44, 7, x_30); -lean_ctor_set(x_44, 8, x_31); -lean_ctor_set(x_44, 9, x_32); -lean_ctor_set(x_44, 10, x_33); -lean_ctor_set(x_44, 11, x_34); -lean_ctor_set(x_44, 12, x_35); -lean_ctor_set(x_44, 13, x_36); -lean_ctor_set(x_44, 14, x_37); -lean_ctor_set(x_44, 15, x_38); -lean_ctor_set(x_44, 16, x_39); -lean_ctor_set(x_44, 17, x_40); -lean_ctor_set(x_44, 18, x_41); -lean_ctor_set(x_44, 19, x_42); -lean_ctor_set_uint8(x_44, sizeof(void*)*20, x_43); -x_45 = lean_st_ref_set(x_2, x_44, x_13); -x_46 = lean_ctor_get(x_45, 1); -lean_inc(x_46); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_47 = x_45; -} else { - lean_dec_ref(x_45); - x_47 = lean_box(0); -} -x_48 = lean_box(0); -if (lean_is_scalar(x_47)) { - x_49 = lean_alloc_ctor(0, 2, 0); -} else { - x_49 = x_47; +lean_dec(x_14); +x_27 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_27, 0, x_25); +lean_ctor_set(x_27, 1, x_26); +return x_27; } -lean_ctor_set(x_49, 0, x_48); -lean_ctor_set(x_49, 1, x_46); -return x_49; } } } -static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__1() { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isCongrRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_markAsInconsistent___lambda__1___boxed), 10, 0); -return x_1; +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_isCongrRoot(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_11; } } -static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__2() { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("closed `", 8, 8); -return x_1; +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_1, 3); +lean_inc(x_12); +lean_dec(x_1); +x_13 = l_Lean_Meta_Grind_getCongrRoot(x_12, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_13; } } -static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_Meta_Grind_markAsInconsistent___closed__2; -x_2 = l_Lean_stringToMessageData(x_1); -return x_2; -} +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +lean_inc(x_1); +x_14 = l_Lean_Meta_Grind_Goal_getENode(x_12, x_1, x_8, x_9, x_13); +if (lean_obj_tag(x_14) == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_14); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_16 = lean_ctor_get(x_14, 0); +x_17 = lean_ctor_get(x_14, 1); +x_18 = lean_ctor_get(x_16, 3); +lean_inc(x_18); +x_19 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_18, x_1); +lean_dec(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +lean_free_object(x_14); +lean_dec(x_1); +x_20 = lean_box(0); +x_21 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_16, x_20, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_17); +return x_21; } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { -_start: +else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_10 = lean_st_ref_get(x_1, x_9); -x_11 = lean_ctor_get(x_10, 0); -lean_inc(x_11); -x_12 = lean_ctor_get_uint8(x_11, sizeof(void*)*20); -lean_dec(x_11); -if (x_12 == 0) +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_1); +return x_14; +} +} +else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_13 = lean_ctor_get(x_10, 1); -lean_inc(x_13); -lean_dec(x_10); -x_14 = l_Lean_Meta_Grind_updateLastTag___closed__1; -x_15 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_14, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -x_16 = !lean_is_exclusive(x_15); -if (x_16 == 0) +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; +x_22 = lean_ctor_get(x_14, 0); +x_23 = lean_ctor_get(x_14, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_14); +x_24 = lean_ctor_get(x_22, 3); +lean_inc(x_24); +x_25 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_24, x_1); +lean_dec(x_24); +if (x_25 == 0) { -lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_17 = lean_ctor_get(x_15, 0); -x_18 = lean_ctor_get(x_15, 1); -x_19 = l_Lean_Meta_Grind_markAsInconsistent___closed__1; -x_20 = lean_unbox(x_17); -lean_dec(x_17); -if (x_20 == 0) +lean_object* x_26; lean_object* x_27; +lean_dec(x_1); +x_26 = lean_box(0); +x_27 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_22, x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +return x_27; +} +else { -lean_object* x_21; lean_object* x_22; -lean_free_object(x_15); -x_21 = lean_box(0); -x_22 = lean_apply_10(x_19, x_21, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_18); -return x_22; +lean_object* x_28; +lean_dec(x_22); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_1); +lean_ctor_set(x_28, 1, x_23); +return x_28; +} +} } else { -lean_object* x_23; uint8_t x_24; -x_23 = lean_st_ref_get(x_1, x_18); -x_24 = !lean_is_exclusive(x_23); -if (x_24 == 0) +uint8_t x_29; +lean_dec(x_1); +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = lean_ctor_get(x_23, 0); -x_26 = lean_ctor_get(x_23, 1); -x_27 = lean_ctor_get(x_25, 0); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_MVarId_getTag(x_27, x_5, x_6, x_7, x_8, x_26); -if (lean_obj_tag(x_28) == 0) +return x_14; +} +else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_29 = lean_ctor_get(x_28, 0); -lean_inc(x_29); -x_30 = lean_ctor_get(x_28, 1); +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); lean_inc(x_30); -lean_dec(x_28); -x_31 = l_Lean_MessageData_ofName(x_29); -x_32 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; -lean_ctor_set_tag(x_23, 7); -lean_ctor_set(x_23, 1, x_31); -lean_ctor_set(x_23, 0, x_32); -x_33 = l_Lean_Meta_Grind_updateLastTag___closed__5; -lean_ctor_set_tag(x_15, 7); -lean_ctor_set(x_15, 1, x_33); -lean_ctor_set(x_15, 0, x_23); -x_34 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_30); -x_35 = lean_ctor_get(x_34, 0); -lean_inc(x_35); -x_36 = lean_ctor_get(x_34, 1); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_apply_10(x_19, x_35, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_36); -return x_37; +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } -else +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_38; -lean_free_object(x_23); -lean_free_object(x_15); +lean_object* x_12; +x_12 = l_Lean_Meta_Grind_getCongrRoot___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -20279,69 +20887,15 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_38 = !lean_is_exclusive(x_28); -if (x_38 == 0) -{ -return x_28; -} -else -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_39 = lean_ctor_get(x_28, 0); -x_40 = lean_ctor_get(x_28, 1); -lean_inc(x_40); -lean_inc(x_39); -lean_dec(x_28); -x_41 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_41, 0, x_39); -lean_ctor_set(x_41, 1, x_40); -return x_41; -} +return x_12; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getCongrRoot___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_42 = lean_ctor_get(x_23, 0); -x_43 = lean_ctor_get(x_23, 1); -lean_inc(x_43); -lean_inc(x_42); -lean_dec(x_23); -x_44 = lean_ctor_get(x_42, 0); -lean_inc(x_44); -lean_dec(x_42); -x_45 = l_Lean_MVarId_getTag(x_44, x_5, x_6, x_7, x_8, x_43); -if (lean_obj_tag(x_45) == 0) -{ -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; -x_46 = lean_ctor_get(x_45, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_45, 1); -lean_inc(x_47); -lean_dec(x_45); -x_48 = l_Lean_MessageData_ofName(x_46); -x_49 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; -x_50 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_48); -x_51 = l_Lean_Meta_Grind_updateLastTag___closed__5; -lean_ctor_set_tag(x_15, 7); -lean_ctor_set(x_15, 1, x_51); -lean_ctor_set(x_15, 0, x_50); -x_52 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_47); -x_53 = lean_ctor_get(x_52, 0); -lean_inc(x_53); -x_54 = lean_ctor_get(x_52, 1); -lean_inc(x_54); -lean_dec(x_52); -x_55 = lean_apply_10(x_19, x_53, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_54); -return x_55; -} -else -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; -lean_free_object(x_15); +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_getCongrRoot(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -20349,104 +20903,48 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_56 = lean_ctor_get(x_45, 0); -lean_inc(x_56); -x_57 = lean_ctor_get(x_45, 1); -lean_inc(x_57); -if (lean_is_exclusive(x_45)) { - lean_ctor_release(x_45, 0); - lean_ctor_release(x_45, 1); - x_58 = x_45; -} else { - lean_dec_ref(x_45); - x_58 = lean_box(0); -} -if (lean_is_scalar(x_58)) { - x_59 = lean_alloc_ctor(1, 2, 0); -} else { - x_59 = x_58; -} -lean_ctor_set(x_59, 0, x_56); -lean_ctor_set(x_59, 1, x_57); -return x_59; -} -} +return x_11; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; -x_60 = lean_ctor_get(x_15, 0); -x_61 = lean_ctor_get(x_15, 1); -lean_inc(x_61); -lean_inc(x_60); -lean_dec(x_15); -x_62 = l_Lean_Meta_Grind_markAsInconsistent___closed__1; -x_63 = lean_unbox(x_60); -lean_dec(x_60); -if (x_63 == 0) +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_64; lean_object* x_65; -x_64 = lean_box(0); -x_65 = lean_apply_10(x_62, x_64, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_61); -return x_65; +lean_object* x_12; uint8_t x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get_uint8(x_12, sizeof(void*)*23); +lean_dec(x_12); +x_14 = lean_box(x_13); +lean_ctor_set(x_10, 0, x_14); +return x_10; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; -x_66 = lean_st_ref_get(x_1, x_61); -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -if (lean_is_exclusive(x_66)) { - lean_ctor_release(x_66, 0); - lean_ctor_release(x_66, 1); - x_69 = x_66; -} else { - lean_dec_ref(x_66); - x_69 = lean_box(0); +lean_object* x_15; lean_object* x_16; uint8_t x_17; lean_object* x_18; lean_object* x_19; +x_15 = lean_ctor_get(x_10, 0); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_10); +x_17 = lean_ctor_get_uint8(x_15, sizeof(void*)*23); +lean_dec(x_15); +x_18 = lean_box(x_17); +x_19 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_19, 0, x_18); +lean_ctor_set(x_19, 1, x_16); +return x_19; } -x_70 = lean_ctor_get(x_67, 0); -lean_inc(x_70); -lean_dec(x_67); -x_71 = l_Lean_MVarId_getTag(x_70, x_5, x_6, x_7, x_8, x_68); -if (lean_obj_tag(x_71) == 0) -{ -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; -x_72 = lean_ctor_get(x_71, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_71, 1); -lean_inc(x_73); -lean_dec(x_71); -x_74 = l_Lean_MessageData_ofName(x_72); -x_75 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; -if (lean_is_scalar(x_69)) { - x_76 = lean_alloc_ctor(7, 2, 0); -} else { - x_76 = x_69; - lean_ctor_set_tag(x_76, 7); } -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_74); -x_77 = l_Lean_Meta_Grind_updateLastTag___closed__5; -x_78 = lean_alloc_ctor(7, 2, 0); -lean_ctor_set(x_78, 0, x_76); -lean_ctor_set(x_78, 1, x_77); -x_79 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_78, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_73); -x_80 = lean_ctor_get(x_79, 0); -lean_inc(x_80); -x_81 = lean_ctor_get(x_79, 1); -lean_inc(x_81); -lean_dec(x_79); -x_82 = lean_apply_10(x_62, x_80, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_81); -return x_82; } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_isInconsistent___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; -lean_dec(x_69); +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_isInconsistent(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -20455,71 +20953,66 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -x_83 = lean_ctor_get(x_71, 0); -lean_inc(x_83); -x_84 = lean_ctor_get(x_71, 1); -lean_inc(x_84); -if (lean_is_exclusive(x_71)) { - lean_ctor_release(x_71, 0); - lean_ctor_release(x_71, 1); - x_85 = x_71; -} else { - lean_dec_ref(x_71); - x_85 = lean_box(0); +return x_10; } -if (lean_is_scalar(x_85)) { - x_86 = lean_alloc_ctor(1, 2, 0); -} else { - x_86 = x_85; } -lean_ctor_set(x_86, 0, x_83); -lean_ctor_set(x_86, 1, x_84); -return x_86; +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = lean_grind_mk_eq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkHEqProof___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = lean_grind_mk_heq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqHEqProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: { -uint8_t x_87; -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_87 = !lean_is_exclusive(x_10); -if (x_87 == 0) +lean_object* x_12; +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_2); +lean_inc(x_1); +x_12 = l_Lean_Meta_Grind_hasSameType(x_1, x_2, x_7, x_8, x_9, x_10, x_11); +if (lean_obj_tag(x_12) == 0) { -lean_object* x_88; lean_object* x_89; -x_88 = lean_ctor_get(x_10, 0); -lean_dec(x_88); -x_89 = lean_box(0); -lean_ctor_set(x_10, 0, x_89); -return x_10; +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_unbox(x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = lean_grind_mk_heq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_15); +return x_16; } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; -x_90 = lean_ctor_get(x_10, 1); -lean_inc(x_90); -lean_dec(x_10); -x_91 = lean_box(0); -x_92 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_90); -return x_92; -} -} +lean_object* x_17; lean_object* x_18; +x_17 = lean_ctor_get(x_12, 1); +lean_inc(x_17); +lean_dec(x_12); +x_18 = lean_grind_mk_eq_proof(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_17); +return x_18; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: +else { -lean_object* x_11; -x_11 = l_Lean_Meta_Grind_markAsInconsistent___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +uint8_t x_19; +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -20529,114 +21022,130 @@ lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); lean_dec(x_1); -return x_11; -} -} -LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; uint8_t x_12; -x_11 = lean_st_ref_get(x_7, x_10); -x_12 = !lean_is_exclusive(x_11); -if (x_12 == 0) +x_19 = !lean_is_exclusive(x_12); +if (x_19 == 0) { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; -x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -lean_dec(x_13); -x_15 = lean_ctor_get(x_14, 7); -lean_inc(x_15); -lean_dec(x_14); -x_16 = l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(x_15, x_1); -x_17 = lean_box(x_16); -lean_ctor_set(x_11, 0, x_17); -return x_11; +return x_12; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; -x_18 = lean_ctor_get(x_11, 0); -x_19 = lean_ctor_get(x_11, 1); -lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_11); -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -lean_dec(x_18); -x_21 = lean_ctor_get(x_20, 7); +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_12, 0); +x_21 = lean_ctor_get(x_12, 1); lean_inc(x_21); -lean_dec(x_20); -x_22 = l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(x_21, x_1); -x_23 = lean_box(x_22); -x_24 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_24, 0, x_23); -lean_ctor_set(x_24, 1, x_19); -return x_24; +lean_inc(x_20); +lean_dec(x_12); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; } } } -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqTrueProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_12 = lean_st_ref_take(x_8, x_11); -x_13 = lean_ctor_get(x_12, 0); +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = l_Lean_Meta_Grind_getTrueExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); lean_inc(x_13); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_12, 1); -lean_inc(x_15); -lean_dec(x_12); -x_16 = !lean_is_exclusive(x_13); -if (x_16 == 0) +lean_dec(x_11); +x_14 = lean_grind_mk_eq_proof(x_1, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_mkEqFalseProof(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_17; uint8_t x_18; -x_17 = lean_ctor_get(x_13, 0); -lean_dec(x_17); -x_18 = !lean_is_exclusive(x_14); -if (x_18 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = l_Lean_Meta_Grind_getFalseExpr___rarg(x_5, x_6, x_7, x_8, x_9, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = lean_grind_mk_eq_proof(x_1, x_12, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_19 = lean_ctor_get(x_14, 7); -x_20 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_19, x_1, x_2); -lean_ctor_set(x_14, 7, x_20); -x_21 = lean_st_ref_set(x_8, x_13, x_15); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_11 = lean_st_ref_take(x_2, x_10); +x_12 = lean_ctor_get(x_11, 0); +lean_inc(x_12); +x_13 = lean_ctor_get(x_11, 1); +lean_inc(x_13); +lean_dec(x_11); +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -lean_object* x_23; lean_object* x_24; -x_23 = lean_ctor_get(x_21, 0); -lean_dec(x_23); -x_24 = lean_box(0); -lean_ctor_set(x_21, 0, x_24); -return x_21; +uint8_t x_15; lean_object* x_16; uint8_t x_17; +x_15 = 1; +lean_ctor_set_uint8(x_12, sizeof(void*)*23, x_15); +x_16 = lean_st_ref_set(x_2, x_12, x_13); +x_17 = !lean_is_exclusive(x_16); +if (x_17 == 0) +{ +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_16, 0); +lean_dec(x_18); +x_19 = lean_box(0); +lean_ctor_set(x_16, 0, x_19); +return x_16; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_21, 1); -lean_inc(x_25); -lean_dec(x_21); -x_26 = lean_box(0); -x_27 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_27, 0, x_26); -lean_ctor_set(x_27, 1, x_25); -return x_27; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_16, 1); +lean_inc(x_20); +lean_dec(x_16); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; } } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_28 = lean_ctor_get(x_14, 0); -x_29 = lean_ctor_get(x_14, 1); -x_30 = lean_ctor_get(x_14, 2); -x_31 = lean_ctor_get(x_14, 3); -x_32 = lean_ctor_get(x_14, 4); -x_33 = lean_ctor_get(x_14, 5); -x_34 = lean_ctor_get(x_14, 6); -x_35 = lean_ctor_get(x_14, 7); -x_36 = lean_ctor_get(x_14, 8); +lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; +x_23 = lean_ctor_get(x_12, 0); +x_24 = lean_ctor_get(x_12, 1); +x_25 = lean_ctor_get(x_12, 2); +x_26 = lean_ctor_get(x_12, 3); +x_27 = lean_ctor_get(x_12, 4); +x_28 = lean_ctor_get(x_12, 5); +x_29 = lean_ctor_get(x_12, 6); +x_30 = lean_ctor_get(x_12, 7); +x_31 = lean_ctor_get(x_12, 8); +x_32 = lean_ctor_get(x_12, 9); +x_33 = lean_ctor_get(x_12, 10); +x_34 = lean_ctor_get(x_12, 11); +x_35 = lean_ctor_get(x_12, 12); +x_36 = lean_ctor_get(x_12, 13); +x_37 = lean_ctor_get(x_12, 14); +x_38 = lean_ctor_get(x_12, 15); +x_39 = lean_ctor_get(x_12, 16); +x_40 = lean_ctor_get(x_12, 17); +x_41 = lean_ctor_get(x_12, 18); +x_42 = lean_ctor_get(x_12, 19); +x_43 = lean_ctor_get(x_12, 20); +x_44 = lean_ctor_get(x_12, 21); +x_45 = lean_ctor_get(x_12, 22); +lean_inc(x_45); +lean_inc(x_44); +lean_inc(x_43); +lean_inc(x_42); +lean_inc(x_41); +lean_inc(x_40); +lean_inc(x_39); +lean_inc(x_38); +lean_inc(x_37); lean_inc(x_36); lean_inc(x_35); lean_inc(x_34); @@ -20646,64 +21155,597 @@ lean_inc(x_31); lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); -lean_dec(x_14); -x_37 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_35, x_1, x_2); -x_38 = lean_alloc_ctor(0, 9, 0); -lean_ctor_set(x_38, 0, x_28); -lean_ctor_set(x_38, 1, x_29); -lean_ctor_set(x_38, 2, x_30); -lean_ctor_set(x_38, 3, x_31); -lean_ctor_set(x_38, 4, x_32); -lean_ctor_set(x_38, 5, x_33); -lean_ctor_set(x_38, 6, x_34); -lean_ctor_set(x_38, 7, x_37); -lean_ctor_set(x_38, 8, x_36); -lean_ctor_set(x_13, 0, x_38); -x_39 = lean_st_ref_set(x_8, x_13, x_15); -x_40 = lean_ctor_get(x_39, 1); -lean_inc(x_40); -if (lean_is_exclusive(x_39)) { - lean_ctor_release(x_39, 0); - lean_ctor_release(x_39, 1); - x_41 = x_39; +lean_inc(x_27); +lean_inc(x_26); +lean_inc(x_25); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_12); +x_46 = 1; +x_47 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_47, 0, x_23); +lean_ctor_set(x_47, 1, x_24); +lean_ctor_set(x_47, 2, x_25); +lean_ctor_set(x_47, 3, x_26); +lean_ctor_set(x_47, 4, x_27); +lean_ctor_set(x_47, 5, x_28); +lean_ctor_set(x_47, 6, x_29); +lean_ctor_set(x_47, 7, x_30); +lean_ctor_set(x_47, 8, x_31); +lean_ctor_set(x_47, 9, x_32); +lean_ctor_set(x_47, 10, x_33); +lean_ctor_set(x_47, 11, x_34); +lean_ctor_set(x_47, 12, x_35); +lean_ctor_set(x_47, 13, x_36); +lean_ctor_set(x_47, 14, x_37); +lean_ctor_set(x_47, 15, x_38); +lean_ctor_set(x_47, 16, x_39); +lean_ctor_set(x_47, 17, x_40); +lean_ctor_set(x_47, 18, x_41); +lean_ctor_set(x_47, 19, x_42); +lean_ctor_set(x_47, 20, x_43); +lean_ctor_set(x_47, 21, x_44); +lean_ctor_set(x_47, 22, x_45); +lean_ctor_set_uint8(x_47, sizeof(void*)*23, x_46); +x_48 = lean_st_ref_set(x_2, x_47, x_13); +x_49 = lean_ctor_get(x_48, 1); +lean_inc(x_49); +if (lean_is_exclusive(x_48)) { + lean_ctor_release(x_48, 0); + lean_ctor_release(x_48, 1); + x_50 = x_48; } else { - lean_dec_ref(x_39); - x_41 = lean_box(0); + lean_dec_ref(x_48); + x_50 = lean_box(0); } -x_42 = lean_box(0); -if (lean_is_scalar(x_41)) { - x_43 = lean_alloc_ctor(0, 2, 0); +x_51 = lean_box(0); +if (lean_is_scalar(x_50)) { + x_52 = lean_alloc_ctor(0, 2, 0); } else { - x_43 = x_41; + x_52 = x_50; } -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_40); -return x_43; +lean_ctor_set(x_52, 0, x_51); +lean_ctor_set(x_52, 1, x_49); +return x_52; } } -else +} +static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__1() { +_start: { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; -x_44 = lean_ctor_get(x_13, 1); -x_45 = lean_ctor_get(x_13, 2); -x_46 = lean_ctor_get(x_13, 3); -x_47 = lean_ctor_get(x_13, 4); -lean_inc(x_47); -lean_inc(x_46); -lean_inc(x_45); -lean_inc(x_44); -lean_dec(x_13); -x_48 = lean_ctor_get(x_14, 0); -lean_inc(x_48); -x_49 = lean_ctor_get(x_14, 1); -lean_inc(x_49); -x_50 = lean_ctor_get(x_14, 2); -lean_inc(x_50); -x_51 = lean_ctor_get(x_14, 3); -lean_inc(x_51); -x_52 = lean_ctor_get(x_14, 4); -lean_inc(x_52); -x_53 = lean_ctor_get(x_14, 5); +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_Meta_Grind_markAsInconsistent___lambda__1___boxed), 10, 0); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("closed `", 8, 8); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Grind_markAsInconsistent___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_Meta_Grind_markAsInconsistent___closed__2; +x_2 = l_Lean_stringToMessageData(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_ctor_get_uint8(x_11, sizeof(void*)*23); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_13 = lean_ctor_get(x_10, 1); +lean_inc(x_13); +lean_dec(x_10); +x_14 = l_Lean_Meta_Grind_updateLastTag___closed__1; +x_15 = l_Lean_isTracingEnabledFor___at_Lean_Meta_Grind_updateLastTag___spec__1(x_14, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); +x_16 = !lean_is_exclusive(x_15); +if (x_16 == 0) +{ +lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_17 = lean_ctor_get(x_15, 0); +x_18 = lean_ctor_get(x_15, 1); +x_19 = l_Lean_Meta_Grind_markAsInconsistent___closed__1; +x_20 = lean_unbox(x_17); +lean_dec(x_17); +if (x_20 == 0) +{ +lean_object* x_21; lean_object* x_22; +lean_free_object(x_15); +x_21 = lean_box(0); +x_22 = lean_apply_10(x_19, x_21, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_18); +return x_22; +} +else +{ +lean_object* x_23; uint8_t x_24; +x_23 = lean_st_ref_get(x_1, x_18); +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_25 = lean_ctor_get(x_23, 0); +x_26 = lean_ctor_get(x_23, 1); +x_27 = lean_ctor_get(x_25, 0); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_MVarId_getTag(x_27, x_5, x_6, x_7, x_8, x_26); +if (lean_obj_tag(x_28) == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_29 = lean_ctor_get(x_28, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_28, 1); +lean_inc(x_30); +lean_dec(x_28); +x_31 = l_Lean_MessageData_ofName(x_29); +x_32 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; +lean_ctor_set_tag(x_23, 7); +lean_ctor_set(x_23, 1, x_31); +lean_ctor_set(x_23, 0, x_32); +x_33 = l_Lean_Meta_Grind_updateLastTag___closed__5; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_33); +lean_ctor_set(x_15, 0, x_23); +x_34 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_30); +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); +x_36 = lean_ctor_get(x_34, 1); +lean_inc(x_36); +lean_dec(x_34); +x_37 = lean_apply_10(x_19, x_35, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_36); +return x_37; +} +else +{ +uint8_t x_38; +lean_free_object(x_23); +lean_free_object(x_15); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_38 = !lean_is_exclusive(x_28); +if (x_38 == 0) +{ +return x_28; +} +else +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; +x_39 = lean_ctor_get(x_28, 0); +x_40 = lean_ctor_get(x_28, 1); +lean_inc(x_40); +lean_inc(x_39); +lean_dec(x_28); +x_41 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_41, 0, x_39); +lean_ctor_set(x_41, 1, x_40); +return x_41; +} +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_42 = lean_ctor_get(x_23, 0); +x_43 = lean_ctor_get(x_23, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_23); +x_44 = lean_ctor_get(x_42, 0); +lean_inc(x_44); +lean_dec(x_42); +x_45 = l_Lean_MVarId_getTag(x_44, x_5, x_6, x_7, x_8, x_43); +if (lean_obj_tag(x_45) == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_46 = lean_ctor_get(x_45, 0); +lean_inc(x_46); +x_47 = lean_ctor_get(x_45, 1); +lean_inc(x_47); +lean_dec(x_45); +x_48 = l_Lean_MessageData_ofName(x_46); +x_49 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; +x_50 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_48); +x_51 = l_Lean_Meta_Grind_updateLastTag___closed__5; +lean_ctor_set_tag(x_15, 7); +lean_ctor_set(x_15, 1, x_51); +lean_ctor_set(x_15, 0, x_50); +x_52 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_15, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_47); +x_53 = lean_ctor_get(x_52, 0); +lean_inc(x_53); +x_54 = lean_ctor_get(x_52, 1); +lean_inc(x_54); +lean_dec(x_52); +x_55 = lean_apply_10(x_19, x_53, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_54); +return x_55; +} +else +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +lean_free_object(x_15); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_56 = lean_ctor_get(x_45, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_45, 1); +lean_inc(x_57); +if (lean_is_exclusive(x_45)) { + lean_ctor_release(x_45, 0); + lean_ctor_release(x_45, 1); + x_58 = x_45; +} else { + lean_dec_ref(x_45); + x_58 = lean_box(0); +} +if (lean_is_scalar(x_58)) { + x_59 = lean_alloc_ctor(1, 2, 0); +} else { + x_59 = x_58; +} +lean_ctor_set(x_59, 0, x_56); +lean_ctor_set(x_59, 1, x_57); +return x_59; +} +} +} +} +else +{ +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_60 = lean_ctor_get(x_15, 0); +x_61 = lean_ctor_get(x_15, 1); +lean_inc(x_61); +lean_inc(x_60); +lean_dec(x_15); +x_62 = l_Lean_Meta_Grind_markAsInconsistent___closed__1; +x_63 = lean_unbox(x_60); +lean_dec(x_60); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_box(0); +x_65 = lean_apply_10(x_62, x_64, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_61); +return x_65; +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +x_66 = lean_st_ref_get(x_1, x_61); +x_67 = lean_ctor_get(x_66, 0); +lean_inc(x_67); +x_68 = lean_ctor_get(x_66, 1); +lean_inc(x_68); +if (lean_is_exclusive(x_66)) { + lean_ctor_release(x_66, 0); + lean_ctor_release(x_66, 1); + x_69 = x_66; +} else { + lean_dec_ref(x_66); + x_69 = lean_box(0); +} +x_70 = lean_ctor_get(x_67, 0); +lean_inc(x_70); +lean_dec(x_67); +x_71 = l_Lean_MVarId_getTag(x_70, x_5, x_6, x_7, x_8, x_68); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; +x_72 = lean_ctor_get(x_71, 0); +lean_inc(x_72); +x_73 = lean_ctor_get(x_71, 1); +lean_inc(x_73); +lean_dec(x_71); +x_74 = l_Lean_MessageData_ofName(x_72); +x_75 = l_Lean_Meta_Grind_markAsInconsistent___closed__3; +if (lean_is_scalar(x_69)) { + x_76 = lean_alloc_ctor(7, 2, 0); +} else { + x_76 = x_69; + lean_ctor_set_tag(x_76, 7); +} +lean_ctor_set(x_76, 0, x_75); +lean_ctor_set(x_76, 1, x_74); +x_77 = l_Lean_Meta_Grind_updateLastTag___closed__5; +x_78 = lean_alloc_ctor(7, 2, 0); +lean_ctor_set(x_78, 0, x_76); +lean_ctor_set(x_78, 1, x_77); +x_79 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2(x_14, x_78, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_73); +x_80 = lean_ctor_get(x_79, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_79, 1); +lean_inc(x_81); +lean_dec(x_79); +x_82 = lean_apply_10(x_62, x_80, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_81); +return x_82; +} +else +{ +lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; +lean_dec(x_69); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_83 = lean_ctor_get(x_71, 0); +lean_inc(x_83); +x_84 = lean_ctor_get(x_71, 1); +lean_inc(x_84); +if (lean_is_exclusive(x_71)) { + lean_ctor_release(x_71, 0); + lean_ctor_release(x_71, 1); + x_85 = x_71; +} else { + lean_dec_ref(x_71); + x_85 = lean_box(0); +} +if (lean_is_scalar(x_85)) { + x_86 = lean_alloc_ctor(1, 2, 0); +} else { + x_86 = x_85; +} +lean_ctor_set(x_86, 0, x_83); +lean_ctor_set(x_86, 1, x_84); +return x_86; +} +} +} +} +else +{ +uint8_t x_87; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_87 = !lean_is_exclusive(x_10); +if (x_87 == 0) +{ +lean_object* x_88; lean_object* x_89; +x_88 = lean_ctor_get(x_10, 0); +lean_dec(x_88); +x_89 = lean_box(0); +lean_ctor_set(x_10, 0, x_89); +return x_10; +} +else +{ +lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_90 = lean_ctor_get(x_10, 1); +lean_inc(x_90); +lean_dec(x_10); +x_91 = lean_box(0); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_90); +return x_92; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_markAsInconsistent___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +x_11 = l_Lean_Meta_Grind_markAsInconsistent___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_7, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +lean_dec(x_13); +x_15 = lean_ctor_get(x_14, 7); +lean_inc(x_15); +lean_dec(x_14); +x_16 = l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(x_15, x_1); +x_17 = lean_box(x_16); +lean_ctor_set(x_11, 0, x_17); +return x_11; +} +else +{ +lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; lean_object* x_24; +x_18 = lean_ctor_get(x_11, 0); +x_19 = lean_ctor_get(x_11, 1); +lean_inc(x_19); +lean_inc(x_18); +lean_dec(x_11); +x_20 = lean_ctor_get(x_18, 0); +lean_inc(x_20); +lean_dec(x_18); +x_21 = lean_ctor_get(x_20, 7); +lean_inc(x_21); +lean_dec(x_20); +x_22 = l_Lean_PersistentHashMap_contains___at_Lean_MVarId_isAssigned___spec__1(x_21, x_1); +x_23 = lean_box(x_22); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_19); +return x_24; +} +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; +x_12 = lean_st_ref_take(x_8, x_11); +x_13 = lean_ctor_get(x_12, 0); +lean_inc(x_13); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_12, 1); +lean_inc(x_15); +lean_dec(x_12); +x_16 = !lean_is_exclusive(x_13); +if (x_16 == 0) +{ +lean_object* x_17; uint8_t x_18; +x_17 = lean_ctor_get(x_13, 0); +lean_dec(x_17); +x_18 = !lean_is_exclusive(x_14); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_14, 7); +x_20 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_19, x_1, x_2); +lean_ctor_set(x_14, 7, x_20); +x_21 = lean_st_ref_set(x_8, x_13, x_15); +x_22 = !lean_is_exclusive(x_21); +if (x_22 == 0) +{ +lean_object* x_23; lean_object* x_24; +x_23 = lean_ctor_get(x_21, 0); +lean_dec(x_23); +x_24 = lean_box(0); +lean_ctor_set(x_21, 0, x_24); +return x_21; +} +else +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_25 = lean_ctor_get(x_21, 1); +lean_inc(x_25); +lean_dec(x_21); +x_26 = lean_box(0); +x_27 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_27, 0, x_26); +lean_ctor_set(x_27, 1, x_25); +return x_27; +} +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_28 = lean_ctor_get(x_14, 0); +x_29 = lean_ctor_get(x_14, 1); +x_30 = lean_ctor_get(x_14, 2); +x_31 = lean_ctor_get(x_14, 3); +x_32 = lean_ctor_get(x_14, 4); +x_33 = lean_ctor_get(x_14, 5); +x_34 = lean_ctor_get(x_14, 6); +x_35 = lean_ctor_get(x_14, 7); +x_36 = lean_ctor_get(x_14, 8); +lean_inc(x_36); +lean_inc(x_35); +lean_inc(x_34); +lean_inc(x_33); +lean_inc(x_32); +lean_inc(x_31); +lean_inc(x_30); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_14); +x_37 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_35, x_1, x_2); +x_38 = lean_alloc_ctor(0, 9, 0); +lean_ctor_set(x_38, 0, x_28); +lean_ctor_set(x_38, 1, x_29); +lean_ctor_set(x_38, 2, x_30); +lean_ctor_set(x_38, 3, x_31); +lean_ctor_set(x_38, 4, x_32); +lean_ctor_set(x_38, 5, x_33); +lean_ctor_set(x_38, 6, x_34); +lean_ctor_set(x_38, 7, x_37); +lean_ctor_set(x_38, 8, x_36); +lean_ctor_set(x_13, 0, x_38); +x_39 = lean_st_ref_set(x_8, x_13, x_15); +x_40 = lean_ctor_get(x_39, 1); +lean_inc(x_40); +if (lean_is_exclusive(x_39)) { + lean_ctor_release(x_39, 0); + lean_ctor_release(x_39, 1); + x_41 = x_39; +} else { + lean_dec_ref(x_39); + x_41 = lean_box(0); +} +x_42 = lean_box(0); +if (lean_is_scalar(x_41)) { + x_43 = lean_alloc_ctor(0, 2, 0); +} else { + x_43 = x_41; +} +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_40); +return x_43; +} +} +else +{ +lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +x_44 = lean_ctor_get(x_13, 1); +x_45 = lean_ctor_get(x_13, 2); +x_46 = lean_ctor_get(x_13, 3); +x_47 = lean_ctor_get(x_13, 4); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); +lean_inc(x_44); +lean_dec(x_13); +x_48 = lean_ctor_get(x_14, 0); +lean_inc(x_48); +x_49 = lean_ctor_get(x_14, 1); +lean_inc(x_49); +x_50 = lean_ctor_get(x_14, 2); +lean_inc(x_50); +x_51 = lean_ctor_get(x_14, 3); +lean_inc(x_51); +x_52 = lean_ctor_get(x_14, 4); +lean_inc(x_52); +x_53 = lean_ctor_get(x_14, 5); lean_inc(x_53); x_54 = lean_ctor_get(x_14, 6); lean_inc(x_54); @@ -20726,166 +21768,579 @@ if (lean_is_exclusive(x_14)) { lean_dec_ref(x_14); x_57 = lean_box(0); } -x_58 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_55, x_1, x_2); -if (lean_is_scalar(x_57)) { - x_59 = lean_alloc_ctor(0, 9, 0); -} else { - x_59 = x_57; +x_58 = l_Lean_PersistentHashMap_insert___at_Lean_MVarId_assign___spec__1(x_55, x_1, x_2); +if (lean_is_scalar(x_57)) { + x_59 = lean_alloc_ctor(0, 9, 0); +} else { + x_59 = x_57; +} +lean_ctor_set(x_59, 0, x_48); +lean_ctor_set(x_59, 1, x_49); +lean_ctor_set(x_59, 2, x_50); +lean_ctor_set(x_59, 3, x_51); +lean_ctor_set(x_59, 4, x_52); +lean_ctor_set(x_59, 5, x_53); +lean_ctor_set(x_59, 6, x_54); +lean_ctor_set(x_59, 7, x_58); +lean_ctor_set(x_59, 8, x_56); +x_60 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_44); +lean_ctor_set(x_60, 2, x_45); +lean_ctor_set(x_60, 3, x_46); +lean_ctor_set(x_60, 4, x_47); +x_61 = lean_st_ref_set(x_8, x_60, x_15); +x_62 = lean_ctor_get(x_61, 1); +lean_inc(x_62); +if (lean_is_exclusive(x_61)) { + lean_ctor_release(x_61, 0); + lean_ctor_release(x_61, 1); + x_63 = x_61; +} else { + lean_dec_ref(x_61); + x_63 = lean_box(0); +} +x_64 = lean_box(0); +if (lean_is_scalar(x_63)) { + x_65 = lean_alloc_ctor(0, 2, 0); +} else { + x_65 = x_63; +} +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set(x_65, 1, x_62); +return x_65; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_closeGoal(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +lean_object* x_11; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_4); +lean_inc(x_3); +lean_inc(x_2); +x_11 = l_Lean_Meta_Grind_markAsInconsistent(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +if (lean_obj_tag(x_11) == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_11, 1); +lean_inc(x_12); +lean_dec(x_11); +x_13 = lean_st_ref_get(x_2, x_12); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_14, 0); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_17, 1); +lean_inc(x_20); +lean_dec(x_17); +lean_inc(x_16); +x_21 = l_Lean_MVarId_getType(x_16, x_6, x_7, x_8, x_9, x_20); +if (lean_obj_tag(x_21) == 0) +{ +lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_22 = lean_ctor_get(x_21, 0); +lean_inc(x_22); +x_23 = lean_ctor_get(x_21, 1); +lean_inc(x_23); +lean_dec(x_21); +lean_inc(x_22); +x_24 = l_Lean_Expr_isFalse(x_22); +if (x_24 == 0) +{ +lean_object* x_25; +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +x_25 = l_Lean_Meta_mkFalseElim(x_22, x_1, x_6, x_7, x_8, x_9, x_23); +if (lean_obj_tag(x_25) == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_25, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_25, 1); +lean_inc(x_27); +lean_dec(x_25); +x_28 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_16, x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_28; +} +else +{ +uint8_t x_29; +lean_dec(x_16); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +x_29 = !lean_is_exclusive(x_25); +if (x_29 == 0) +{ +return x_25; +} +else +{ +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_25, 0); +x_31 = lean_ctor_get(x_25, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_25); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; +} +} +} +else +{ +lean_object* x_33; +lean_dec(x_22); +x_33 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_16, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_33; +} +} +else +{ +uint8_t x_34; +lean_dec(x_16); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_34 = !lean_is_exclusive(x_21); +if (x_34 == 0) +{ +return x_21; +} +else +{ +lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_35 = lean_ctor_get(x_21, 0); +x_36 = lean_ctor_get(x_21, 1); +lean_inc(x_36); +lean_inc(x_35); +lean_dec(x_21); +x_37 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_37, 0, x_35); +lean_ctor_set(x_37, 1, x_36); +return x_37; +} +} +} +else +{ +uint8_t x_38; +lean_dec(x_16); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_38 = !lean_is_exclusive(x_17); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_ctor_get(x_17, 0); +lean_dec(x_39); +x_40 = lean_box(0); +lean_ctor_set(x_17, 0, x_40); +return x_17; +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; +x_41 = lean_ctor_get(x_17, 1); +lean_inc(x_41); +lean_dec(x_17); +x_42 = lean_box(0); +x_43 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_43, 0, x_42); +lean_ctor_set(x_43, 1, x_41); +return x_43; +} } -lean_ctor_set(x_59, 0, x_48); -lean_ctor_set(x_59, 1, x_49); -lean_ctor_set(x_59, 2, x_50); -lean_ctor_set(x_59, 3, x_51); -lean_ctor_set(x_59, 4, x_52); -lean_ctor_set(x_59, 5, x_53); -lean_ctor_set(x_59, 6, x_54); -lean_ctor_set(x_59, 7, x_58); -lean_ctor_set(x_59, 8, x_56); -x_60 = lean_alloc_ctor(0, 5, 0); -lean_ctor_set(x_60, 0, x_59); -lean_ctor_set(x_60, 1, x_44); -lean_ctor_set(x_60, 2, x_45); -lean_ctor_set(x_60, 3, x_46); -lean_ctor_set(x_60, 4, x_47); -x_61 = lean_st_ref_set(x_8, x_60, x_15); -x_62 = lean_ctor_get(x_61, 1); -lean_inc(x_62); -if (lean_is_exclusive(x_61)) { - lean_ctor_release(x_61, 0); - lean_ctor_release(x_61, 1); - x_63 = x_61; -} else { - lean_dec_ref(x_61); - x_63 = lean_box(0); } -x_64 = lean_box(0); -if (lean_is_scalar(x_63)) { - x_65 = lean_alloc_ctor(0, 2, 0); -} else { - x_65 = x_63; +else +{ +uint8_t x_44; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +x_44 = !lean_is_exclusive(x_11); +if (x_44 == 0) +{ +return x_11; } -lean_ctor_set(x_65, 0, x_64); -lean_ctor_set(x_65, 1, x_62); -return x_65; +else +{ +lean_object* x_45; lean_object* x_46; lean_object* x_47; +x_45 = lean_ctor_get(x_11, 0); +x_46 = lean_ctor_get(x_11, 1); +lean_inc(x_46); +lean_inc(x_45); +lean_dec(x_11); +x_47 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_47, 0, x_45); +lean_ctor_set(x_47, 1, x_46); +return x_47; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_closeGoal(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +} +LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; -lean_inc(x_9); +x_11 = l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_11; +} +} +LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +lean_dec(x_3); +return x_12; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_Goal_getENodes___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_PersistentHashMap_foldlMAux___at_Lean_MetavarContext_getExprAssignmentDomain___spec__2___rarg(x_2, x_1, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_4, 0, x_2); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_array_push(x_1, x_4); +return x_5; +} +} +static lean_object* _init_l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___lambda__1), 3, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_2 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1; +x_3 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__3; +x_4 = l_Lean_PersistentHashMap_foldlMAux___at_Lean_MetavarContext_getExprAssignmentDomain___spec__2___rarg(x_2, x_1, x_3); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { +_start: +{ +uint8_t x_4; +x_4 = lean_usize_dec_lt(x_2, x_1); +if (x_4 == 0) +{ +return x_3; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; +x_5 = lean_array_uget(x_3, x_2); +x_6 = lean_unsigned_to_nat(0u); +x_7 = lean_array_uset(x_3, x_2, x_6); +x_8 = lean_ctor_get(x_5, 1); lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -lean_inc(x_5); -lean_inc(x_4); +lean_dec(x_5); +x_9 = 1; +x_10 = lean_usize_add(x_2, x_9); +x_11 = lean_array_uset(x_7, x_2, x_8); +x_2 = x_10; +x_3 = x_11; +goto _start; +} +} +} +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; +x_3 = lean_ctor_get(x_1, 7); +x_4 = lean_ctor_get(x_2, 7); +x_5 = lean_nat_dec_lt(x_3, x_4); +return x_5; +} +} +static lean_object* _init_l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1___boxed), 2, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +x_7 = lean_nat_dec_lt(x_3, x_4); +if (x_7 == 0) +{ +lean_dec(x_3); +return x_2; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_8 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1; lean_inc(x_3); -lean_inc(x_2); -x_11 = l_Lean_Meta_Grind_markAsInconsistent(x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -if (lean_obj_tag(x_11) == 0) +x_9 = l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(x_1, x_2, x_8, x_3, x_4, lean_box(0), lean_box(0)); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_nat_dec_le(x_4, x_10); +if (x_12 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_12 = lean_ctor_get(x_11, 1); -lean_inc(x_12); -lean_dec(x_11); -x_13 = lean_st_ref_get(x_2, x_12); -x_14 = lean_ctor_get(x_13, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_13, 1); -lean_inc(x_15); -lean_dec(x_13); -x_16 = lean_ctor_get(x_14, 0); -lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(x_16, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_15); -x_18 = lean_ctor_get(x_17, 0); -lean_inc(x_18); -x_19 = lean_unbox(x_18); -lean_dec(x_18); -if (x_19 == 0) +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); +x_14 = lean_unsigned_to_nat(1u); +x_15 = lean_nat_add(x_10, x_14); +lean_dec(x_10); +x_2 = x_13; +x_3 = x_15; +x_5 = lean_box(0); +x_6 = lean_box(0); +goto _start; +} +else { -lean_object* x_20; lean_object* x_21; -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_dec(x_17); -lean_inc(x_16); -x_21 = l_Lean_MVarId_getType(x_16, x_6, x_7, x_8, x_9, x_20); -if (lean_obj_tag(x_21) == 0) +lean_dec(x_10); +lean_dec(x_3); +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENodes(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; size_t x_4; size_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_2 = lean_ctor_get(x_1, 2); +x_3 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1(x_2); +x_4 = lean_array_size(x_3); +x_5 = 0; +x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3(x_4, x_5, x_3); +x_7 = lean_array_get_size(x_6); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_7, x_8); +x_10 = lean_unsigned_to_nat(0u); +x_11 = lean_nat_dec_eq(x_7, x_10); +if (x_11 == 0) { -lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_22 = lean_ctor_get(x_21, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_21, 1); -lean_inc(x_23); -lean_dec(x_21); -lean_inc(x_22); -x_24 = l_Lean_Expr_isFalse(x_22); -if (x_24 == 0) +uint8_t x_12; +x_12 = lean_nat_dec_le(x_10, x_9); +if (x_12 == 0) { -lean_object* x_25; +lean_object* x_13; lean_inc(x_9); -lean_inc(x_8); -lean_inc(x_7); -lean_inc(x_6); -x_25 = l_Lean_Meta_mkFalseElim(x_22, x_1, x_6, x_7, x_8, x_9, x_23); -if (lean_obj_tag(x_25) == 0) +x_13 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(x_7, x_6, x_9, x_9, lean_box(0), lean_box(0)); +lean_dec(x_9); +lean_dec(x_7); +return x_13; +} +else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_16, x_26, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_27); +lean_object* x_14; +x_14 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(x_7, x_6, x_10, x_9, lean_box(0), lean_box(0)); lean_dec(x_9); -lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -return x_28; +return x_14; +} } else { -uint8_t x_29; -lean_dec(x_16); lean_dec(x_9); -lean_dec(x_8); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); +return x_6; +} +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_Goal_getENodes___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_Goal_getENodes___spec__2(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1(x_1); +lean_dec(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +size_t x_4; size_t x_5; lean_object* x_6; +x_4 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_29 = !lean_is_exclusive(x_25); -if (x_29 == 0) +x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_Goal_getENodes___spec__3(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +_start: { -return x_25; +uint8_t x_3; lean_object* x_4; +x_3 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___lambda__1(x_1, x_2); +lean_dec(x_2); +lean_dec(x_1); +x_4 = lean_box(x_3); +return x_4; } -else +} +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_30; lean_object* x_31; lean_object* x_32; -x_30 = lean_ctor_get(x_25, 0); -x_31 = lean_ctor_get(x_25, 1); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_25); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_30); -lean_ctor_set(x_32, 1, x_31); -return x_32; +lean_object* x_7; +x_7 = l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4(x_1, x_2, x_3, x_4, x_5, x_6); +lean_dec(x_4); +lean_dec(x_1); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getENodes___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = l_Lean_Meta_Grind_Goal_getENodes(x_1); +lean_dec(x_1); +return x_2; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_10, 0); +x_13 = l_Lean_Meta_Grind_Goal_getENodes(x_12); +lean_dec(x_12); +lean_ctor_set(x_10, 0, x_13); +return x_10; } else { -lean_object* x_33; -lean_dec(x_22); -x_33 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_16, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_23); -lean_dec(x_9); +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_10); +x_16 = l_Lean_Meta_Grind_Goal_getENodes(x_14); +lean_dec(x_14); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); +return x_17; +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Grind_getENodes(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -20893,453 +22348,556 @@ lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -return x_33; +lean_dec(x_1); +return x_10; } } -else +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: { -uint8_t x_34; +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_1, 1); +lean_inc(x_14); +x_15 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_15, 0, x_2); +lean_ctor_set(x_15, 1, x_14); +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_13); +return x_17; +} +} +static lean_object* _init_l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +uint8_t x_14; +x_14 = !lean_is_exclusive(x_4); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; +x_15 = lean_ctor_get(x_4, 1); +x_16 = lean_ctor_get(x_4, 0); lean_dec(x_16); +x_17 = lean_st_ref_get(x_5, x_13); +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +x_19 = lean_ctor_get(x_17, 1); +lean_inc(x_19); +lean_dec(x_17); +lean_inc(x_15); +x_20 = l_Lean_Meta_Grind_Goal_getENode(x_18, x_15, x_11, x_12, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +x_22 = lean_ctor_get(x_20, 1); +lean_inc(x_22); +lean_dec(x_20); +lean_inc(x_2); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_21); +x_23 = lean_apply_10(x_2, x_21, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_22); +if (lean_obj_tag(x_23) == 0) +{ +uint8_t x_24; +x_24 = !lean_is_exclusive(x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_25 = lean_ctor_get(x_23, 1); +x_26 = lean_ctor_get(x_23, 0); +lean_dec(x_26); +x_27 = lean_ctor_get(x_21, 1); +lean_inc(x_27); +x_28 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_27, x_1); +lean_dec(x_27); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +lean_free_object(x_23); +lean_free_object(x_4); +x_29 = lean_box(0); +lean_inc(x_3); +x_30 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(x_21, x_3, x_15, x_29, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_25); +lean_dec(x_15); +lean_dec(x_21); +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = lean_ctor_get(x_31, 0); +lean_inc(x_33); +lean_dec(x_31); +x_4 = x_33; +x_13 = x_32; +goto _start; +} +else +{ +lean_object* x_35; +lean_dec(x_21); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_34 = !lean_is_exclusive(x_21); -if (x_34 == 0) -{ -return x_21; +x_35 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1; +lean_ctor_set(x_4, 0, x_35); +lean_ctor_set(x_23, 0, x_4); +return x_23; +} } else { -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_21, 0); -x_36 = lean_ctor_get(x_21, 1); +lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_36 = lean_ctor_get(x_23, 1); lean_inc(x_36); -lean_inc(x_35); +lean_dec(x_23); +x_37 = lean_ctor_get(x_21, 1); +lean_inc(x_37); +x_38 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_37, x_1); +lean_dec(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_free_object(x_4); +x_39 = lean_box(0); +lean_inc(x_3); +x_40 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(x_21, x_3, x_15, x_39, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_36); +lean_dec(x_15); lean_dec(x_21); -x_37 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_37, 0, x_35); -lean_ctor_set(x_37, 1, x_36); -return x_37; -} -} +x_41 = lean_ctor_get(x_40, 0); +lean_inc(x_41); +x_42 = lean_ctor_get(x_40, 1); +lean_inc(x_42); +lean_dec(x_40); +x_43 = lean_ctor_get(x_41, 0); +lean_inc(x_43); +lean_dec(x_41); +x_4 = x_43; +x_13 = x_42; +goto _start; } else { -uint8_t x_38; -lean_dec(x_16); +lean_object* x_45; lean_object* x_46; +lean_dec(x_21); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_38 = !lean_is_exclusive(x_17); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; -x_39 = lean_ctor_get(x_17, 0); -lean_dec(x_39); -x_40 = lean_box(0); -lean_ctor_set(x_17, 0, x_40); -return x_17; -} -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_41 = lean_ctor_get(x_17, 1); -lean_inc(x_41); -lean_dec(x_17); -x_42 = lean_box(0); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_41); -return x_43; +x_45 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1; +lean_ctor_set(x_4, 0, x_45); +x_46 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_46, 0, x_4); +lean_ctor_set(x_46, 1, x_36); +return x_46; } } } else { -uint8_t x_44; +uint8_t x_47; +lean_dec(x_21); +lean_free_object(x_4); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); -lean_dec(x_1); -x_44 = !lean_is_exclusive(x_11); -if (x_44 == 0) +x_47 = !lean_is_exclusive(x_23); +if (x_47 == 0) { -return x_11; +return x_23; } else { -lean_object* x_45; lean_object* x_46; lean_object* x_47; -x_45 = lean_ctor_get(x_11, 0); -x_46 = lean_ctor_get(x_11, 1); -lean_inc(x_46); -lean_inc(x_45); -lean_dec(x_11); -x_47 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_47, 0, x_45); -lean_ctor_set(x_47, 1, x_46); -return x_47; -} -} -} +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_23, 0); +x_49 = lean_ctor_get(x_23, 1); +lean_inc(x_49); +lean_inc(x_48); +lean_dec(x_23); +x_50 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_50, 0, x_48); +lean_ctor_set(x_50, 1, x_49); +return x_50; } -LEAN_EXPORT lean_object* l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -lean_object* x_11; -x_11 = l_Lean_MVarId_isAssigned___at_Lean_Meta_Grind_closeGoal___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_11; } } -LEAN_EXPORT lean_object* l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { -_start: +else { -lean_object* x_12; -x_12 = l_Lean_MVarId_assign___at_Lean_Meta_Grind_closeGoal___spec__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +uint8_t x_51; +lean_free_object(x_4); +lean_dec(x_15); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); -return x_12; -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_getENodes___spec__2(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +lean_dec(x_2); +x_51 = !lean_is_exclusive(x_20); +if (x_51 == 0) { -lean_object* x_4; -x_4 = l_Lean_PersistentHashMap_foldlMAux___at_Lean_MetavarContext_getExprAssignmentDomain___spec__2___rarg(x_2, x_1, x_3); -return x_4; -} +return x_20; } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +else { -lean_object* x_4; lean_object* x_5; -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_2); -lean_ctor_set(x_4, 1, x_3); -x_5 = lean_array_push(x_1, x_4); -return x_5; -} +lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_52 = lean_ctor_get(x_20, 0); +x_53 = lean_ctor_get(x_20, 1); +lean_inc(x_53); +lean_inc(x_52); +lean_dec(x_20); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_52); +lean_ctor_set(x_54, 1, x_53); +return x_54; } -static lean_object* _init_l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1() { -_start: -{ -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___lambda__1), 3, 0); -return x_1; } } -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1(lean_object* x_1) { -_start: +else { -lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1; -x_3 = l_Lean_addTrace___at_Lean_Meta_Grind_updateLastTag___spec__2___closed__3; -x_4 = l_Lean_PersistentHashMap_foldlMAux___at_Lean_MetavarContext_getExprAssignmentDomain___spec__2___rarg(x_2, x_1, x_3); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3(size_t x_1, size_t x_2, lean_object* x_3) { -_start: +lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_55 = lean_ctor_get(x_4, 1); +lean_inc(x_55); +lean_dec(x_4); +x_56 = lean_st_ref_get(x_5, x_13); +x_57 = lean_ctor_get(x_56, 0); +lean_inc(x_57); +x_58 = lean_ctor_get(x_56, 1); +lean_inc(x_58); +lean_dec(x_56); +lean_inc(x_55); +x_59 = l_Lean_Meta_Grind_Goal_getENode(x_57, x_55, x_11, x_12, x_58); +if (lean_obj_tag(x_59) == 0) { -uint8_t x_4; -x_4 = lean_usize_dec_lt(x_2, x_1); -if (x_4 == 0) +lean_object* x_60; lean_object* x_61; lean_object* x_62; +x_60 = lean_ctor_get(x_59, 0); +lean_inc(x_60); +x_61 = lean_ctor_get(x_59, 1); +lean_inc(x_61); +lean_dec(x_59); +lean_inc(x_2); +lean_inc(x_12); +lean_inc(x_11); +lean_inc(x_10); +lean_inc(x_9); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +lean_inc(x_60); +x_62 = lean_apply_10(x_2, x_60, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_61); +if (lean_obj_tag(x_62) == 0) { -return x_3; +lean_object* x_63; lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_63 = lean_ctor_get(x_62, 1); +lean_inc(x_63); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_64 = x_62; +} else { + lean_dec_ref(x_62); + x_64 = lean_box(0); } -else +x_65 = lean_ctor_get(x_60, 1); +lean_inc(x_65); +x_66 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_65, x_1); +lean_dec(x_65); +if (x_66 == 0) { -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; size_t x_9; size_t x_10; lean_object* x_11; -x_5 = lean_array_uget(x_3, x_2); -x_6 = lean_unsigned_to_nat(0u); -x_7 = lean_array_uset(x_3, x_2, x_6); -x_8 = lean_ctor_get(x_5, 1); -lean_inc(x_8); -lean_dec(x_5); -x_9 = 1; -x_10 = lean_usize_add(x_2, x_9); -x_11 = lean_array_uset(x_7, x_2, x_8); -x_2 = x_10; -x_3 = x_11; +lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; +lean_dec(x_64); +x_67 = lean_box(0); +lean_inc(x_3); +x_68 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(x_60, x_3, x_55, x_67, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_63); +lean_dec(x_55); +lean_dec(x_60); +x_69 = lean_ctor_get(x_68, 0); +lean_inc(x_69); +x_70 = lean_ctor_get(x_68, 1); +lean_inc(x_70); +lean_dec(x_68); +x_71 = lean_ctor_get(x_69, 0); +lean_inc(x_71); +lean_dec(x_69); +x_4 = x_71; +x_13 = x_70; goto _start; } -} -} -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; lean_object* x_4; uint8_t x_5; -x_3 = lean_ctor_get(x_1, 7); -x_4 = lean_ctor_get(x_2, 7); -x_5 = lean_nat_dec_lt(x_3, x_4); -return x_5; -} -} -static lean_object* _init_l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1() { -_start: +else { -lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1___boxed), 2, 0); -return x_1; +lean_object* x_73; lean_object* x_74; lean_object* x_75; +lean_dec(x_60); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_73 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_55); +if (lean_is_scalar(x_64)) { + x_75 = lean_alloc_ctor(0, 2, 0); +} else { + x_75 = x_64; } +lean_ctor_set(x_75, 0, x_74); +lean_ctor_set(x_75, 1, x_63); +return x_75; } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -uint8_t x_7; -x_7 = lean_nat_dec_lt(x_3, x_4); -if (x_7 == 0) -{ -lean_dec(x_3); -return x_2; } else { -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_8 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1; -lean_inc(x_3); -x_9 = l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(x_1, x_2, x_8, x_3, x_4, lean_box(0), lean_box(0)); -x_10 = lean_ctor_get(x_9, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_9, 1); -lean_inc(x_11); -lean_dec(x_9); -x_12 = lean_nat_dec_le(x_4, x_10); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_add(x_10, x_14); +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; +lean_dec(x_60); +lean_dec(x_55); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); -x_2 = x_13; -x_3 = x_15; -x_5 = lean_box(0); -x_6 = lean_box(0); -goto _start; +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +x_76 = lean_ctor_get(x_62, 0); +lean_inc(x_76); +x_77 = lean_ctor_get(x_62, 1); +lean_inc(x_77); +if (lean_is_exclusive(x_62)) { + lean_ctor_release(x_62, 0); + lean_ctor_release(x_62, 1); + x_78 = x_62; +} else { + lean_dec_ref(x_62); + x_78 = lean_box(0); +} +if (lean_is_scalar(x_78)) { + x_79 = lean_alloc_ctor(1, 2, 0); +} else { + x_79 = x_78; +} +lean_ctor_set(x_79, 0, x_76); +lean_ctor_set(x_79, 1, x_77); +return x_79; +} } else { +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; +lean_dec(x_55); +lean_dec(x_12); +lean_dec(x_11); lean_dec(x_10); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_3); -return x_11; +lean_dec(x_2); +x_80 = lean_ctor_get(x_59, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_59, 1); +lean_inc(x_81); +if (lean_is_exclusive(x_59)) { + lean_ctor_release(x_59, 0); + lean_ctor_release(x_59, 1); + x_82 = x_59; +} else { + lean_dec_ref(x_59); + x_82 = lean_box(0); +} +if (lean_is_scalar(x_82)) { + x_83 = lean_alloc_ctor(1, 2, 0); +} else { + x_83 = x_82; } +lean_ctor_set(x_83, 0, x_80); +lean_ctor_set(x_83, 1, x_81); +return x_83; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +} +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_traverseEqc(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { _start: { -lean_object* x_10; uint8_t x_11; -x_10 = lean_st_ref_get(x_1, x_9); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +lean_inc(x_1); +x_13 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_1); +x_14 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1(x_1, x_2, x_12, x_13, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_1); +if (lean_obj_tag(x_14) == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1(x_13); -lean_dec(x_13); -x_15 = lean_array_size(x_14); -x_16 = 0; -x_17 = l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3(x_15, x_16, x_14); -x_18 = lean_array_get_size(x_17); -x_19 = lean_unsigned_to_nat(1u); -x_20 = lean_nat_sub(x_18, x_19); -x_21 = lean_unsigned_to_nat(0u); -x_22 = lean_nat_dec_eq(x_18, x_21); -if (x_22 == 0) +lean_object* x_15; lean_object* x_16; +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_15, 0); +lean_inc(x_16); +lean_dec(x_15); +if (lean_obj_tag(x_16) == 0) { -uint8_t x_23; -x_23 = lean_nat_dec_le(x_21, x_20); -if (x_23 == 0) +uint8_t x_17; +x_17 = !lean_is_exclusive(x_14); +if (x_17 == 0) { -lean_object* x_24; -lean_inc(x_20); -x_24 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_18, x_17, x_20, x_20, lean_box(0), lean_box(0)); -lean_dec(x_20); +lean_object* x_18; lean_object* x_19; +x_18 = lean_ctor_get(x_14, 0); lean_dec(x_18); -lean_ctor_set(x_10, 0, x_24); -return x_10; +x_19 = lean_box(0); +lean_ctor_set(x_14, 0, x_19); +return x_14; } else { -lean_object* x_25; -x_25 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_18, x_17, x_21, x_20, lean_box(0), lean_box(0)); -lean_dec(x_20); -lean_dec(x_18); -lean_ctor_set(x_10, 0, x_25); -return x_10; +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_14, 1); +lean_inc(x_20); +lean_dec(x_14); +x_21 = lean_box(0); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_20); +return x_22; } } else { -lean_dec(x_20); -lean_dec(x_18); -lean_ctor_set(x_10, 0, x_17); -return x_10; -} +uint8_t x_23; +x_23 = !lean_is_exclusive(x_14); +if (x_23 == 0) +{ +lean_object* x_24; lean_object* x_25; +x_24 = lean_ctor_get(x_14, 0); +lean_dec(x_24); +x_25 = lean_ctor_get(x_16, 0); +lean_inc(x_25); +lean_dec(x_16); +lean_ctor_set(x_14, 0, x_25); +return x_14; } else { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; size_t x_30; size_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_26 = lean_ctor_get(x_10, 0); -x_27 = lean_ctor_get(x_10, 1); -lean_inc(x_27); +lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_26 = lean_ctor_get(x_14, 1); lean_inc(x_26); -lean_dec(x_10); -x_28 = lean_ctor_get(x_26, 1); -lean_inc(x_28); -lean_dec(x_26); -x_29 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1(x_28); -lean_dec(x_28); -x_30 = lean_array_size(x_29); -x_31 = 0; -x_32 = l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3(x_30, x_31, x_29); -x_33 = lean_array_get_size(x_32); -x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_nat_sub(x_33, x_34); -x_36 = lean_unsigned_to_nat(0u); -x_37 = lean_nat_dec_eq(x_33, x_36); -if (x_37 == 0) -{ -uint8_t x_38; -x_38 = lean_nat_dec_le(x_36, x_35); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; -lean_inc(x_35); -x_39 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_33, x_32, x_35, x_35, lean_box(0), lean_box(0)); -lean_dec(x_35); -lean_dec(x_33); -x_40 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_27); -return x_40; +lean_dec(x_14); +x_27 = lean_ctor_get(x_16, 0); +lean_inc(x_27); +lean_dec(x_16); +x_28 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_26); +return x_28; } -else -{ -lean_object* x_41; lean_object* x_42; -x_41 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_33, x_32, x_36, x_35, lean_box(0), lean_box(0)); -lean_dec(x_35); -lean_dec(x_33); -x_42 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_42, 0, x_41); -lean_ctor_set(x_42, 1, x_27); -return x_42; } } else { -lean_object* x_43; -lean_dec(x_35); -lean_dec(x_33); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_32); -lean_ctor_set(x_43, 1, x_27); -return x_43; -} -} -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_getENodes___spec__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Lean_PersistentHashMap_foldlM___at_Lean_Meta_Grind_getENodes___spec__2(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___boxed(lean_object* x_1) { -_start: -{ -lean_object* x_2; -x_2 = l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1(x_1); -lean_dec(x_1); -return x_2; -} -} -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: +uint8_t x_29; +x_29 = !lean_is_exclusive(x_14); +if (x_29 == 0) { -size_t x_4; size_t x_5; lean_object* x_6; -x_4 = lean_unbox_usize(x_1); -lean_dec(x_1); -x_5 = lean_unbox_usize(x_2); -lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Meta_Grind_getENodes___spec__3(x_4, x_5, x_3); -return x_6; -} +return x_14; } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { -_start: +else { -uint8_t x_3; lean_object* x_4; -x_3 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___lambda__1(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(x_3); -return x_4; +lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_30 = lean_ctor_get(x_14, 0); +x_31 = lean_ctor_get(x_14, 1); +lean_inc(x_31); +lean_inc(x_30); +lean_dec(x_14); +x_32 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_32, 0, x_30); +lean_ctor_set(x_32, 1, x_31); +return x_32; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_4); -lean_dec(x_1); -return x_7; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getENodes___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { _start: { -lean_object* x_10; -x_10 = l_Lean_Meta_Grind_getENodes(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_object* x_14; +x_14 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_12); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); lean_dec(x_1); -return x_10; +return x_14; +} +} +LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13) { +_start: +{ +lean_object* x_14; +x_14 = l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13); +lean_dec(x_1); +return x_14; } } LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachENode___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { @@ -21682,7 +23240,7 @@ lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; @@ -21789,7 +23347,7 @@ return x_36; } } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_forEachEqc(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_forEachEqcRoot(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; lean_object* x_18; @@ -21803,7 +23361,7 @@ x_14 = lean_box(0); x_15 = lean_array_size(x_12); x_16 = 0; x_17 = lean_box(0); -x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1(x_1, x_12, x_14, x_12, x_15, x_16, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); +x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1(x_1, x_12, x_14, x_12, x_15, x_16, x_17, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_13); lean_dec(x_12); if (lean_obj_tag(x_18) == 0) { @@ -21853,7 +23411,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { size_t x_17; size_t x_18; lean_object* x_19; @@ -21861,7 +23419,7 @@ x_17 = lean_unbox_usize(x_5); lean_dec(x_5); x_18 = lean_unbox_usize(x_6); lean_dec(x_6); -x_19 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqc___spec__1(x_1, x_2, x_3, x_4, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_forEachEqcRoot___spec__1(x_1, x_2, x_3, x_4, x_17, x_18, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -22071,122 +23629,91 @@ x_11 = lean_apply_9(x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); return x_11; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc_go(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_13; -lean_inc(x_2); -x_13 = l_Lean_Meta_Grind_getNext(x_2, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -if (lean_obj_tag(x_13) == 0) -{ -uint8_t x_14; -x_14 = !lean_is_exclusive(x_13); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_15 = lean_ctor_get(x_13, 0); -x_16 = lean_ctor_get(x_13, 1); -x_17 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_17, 0, x_2); -lean_ctor_set(x_17, 1, x_3); -x_18 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_15); -if (x_18 == 0) -{ -lean_free_object(x_13); -x_2 = x_15; -x_3 = x_17; -x_12 = x_16; -goto _start; -} -else +lean_object* x_5; +lean_inc(x_1); +x_5 = l_Lean_Meta_Grind_Goal_getNext_x3f(x_1, x_3); +if (lean_obj_tag(x_5) == 0) { -lean_dec(x_15); -lean_ctor_set(x_13, 0, x_17); -return x_13; -} +lean_dec(x_3); +lean_dec(x_1); +return x_4; } else { -lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_20 = lean_ctor_get(x_13, 0); -x_21 = lean_ctor_get(x_13, 1); -lean_inc(x_21); -lean_inc(x_20); -lean_dec(x_13); -x_22 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_22, 0, x_2); -lean_ctor_set(x_22, 1, x_3); -x_23 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_1, x_20); -if (x_23 == 0) +lean_object* x_6; lean_object* x_7; uint8_t x_8; +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +lean_dec(x_5); +x_7 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_7, 0, x_3); +lean_ctor_set(x_7, 1, x_4); +x_8 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_2, x_6); +if (x_8 == 0) { -x_2 = x_20; -x_3 = x_22; -x_12 = x_21; +x_3 = x_6; +x_4 = x_7; goto _start; } else { -lean_object* x_25; -lean_dec(x_20); -x_25 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_25, 0, x_22); -lean_ctor_set(x_25, 1, x_21); -return x_25; -} -} -} -else -{ -uint8_t x_26; -lean_dec(x_3); -lean_dec(x_2); -x_26 = !lean_is_exclusive(x_13); -if (x_26 == 0) -{ -return x_13; +lean_dec(x_6); +lean_dec(x_1); +return x_7; +} } -else -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_13, 0); -x_28 = lean_ctor_get(x_13, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_13); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l_Lean_Meta_Grind_Goal_getEqc_go(x_1, x_2, x_3, x_4); +lean_dec(x_2); +return x_5; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc_go___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqc(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_13; -x_13 = l_Lean_Meta_Grind_getEqc_go(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_1); -return x_13; +lean_object* x_3; lean_object* x_4; +x_3 = lean_box(0); +lean_inc(x_2); +x_4 = l_Lean_Meta_Grind_Goal_getEqc_go(x_1, x_2, x_2, x_3); +lean_dec(x_2); +return x_4; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; -x_11 = lean_box(0); -lean_inc(x_1); -x_12 = l_Lean_Meta_Grind_getEqc_go(x_1, x_1, x_11, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_1); -return x_12; +lean_object* x_11; uint8_t x_12; +x_11 = lean_st_ref_get(x_2, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; +x_13 = lean_ctor_get(x_11, 0); +x_14 = l_Lean_Meta_Grind_Goal_getEqc(x_13, x_1); +lean_ctor_set(x_11, 0, x_14); +return x_11; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_11, 0); +x_16 = lean_ctor_get(x_11, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_11); +x_17 = l_Lean_Meta_Grind_Goal_getEqc(x_15, x_1); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +return x_18; +} } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqc___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { @@ -22205,171 +23732,110 @@ lean_dec(x_2); return x_11; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, size_t x_4, size_t x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { _start: { -uint8_t x_16; -x_16 = lean_usize_dec_lt(x_5, x_4); -if (x_16 == 0) +uint8_t x_8; +x_8 = lean_usize_dec_lt(x_6, x_5); +if (x_8 == 0) { -lean_object* x_17; -x_17 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_17, 0, x_6); -lean_ctor_set(x_17, 1, x_15); -return x_17; +lean_dec(x_1); +return x_7; } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_18 = lean_array_uget(x_3, x_5); -x_19 = lean_ctor_get(x_18, 2); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 0); -lean_inc(x_20); -lean_dec(x_18); -x_21 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_19, x_20); -lean_dec(x_19); -if (x_21 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_9 = lean_array_uget(x_4, x_6); +x_10 = lean_ctor_get(x_9, 2); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 0); +lean_inc(x_11); +lean_dec(x_9); +x_12 = l_Lean_Meta_Grind_isSameExpr_unsafe__1(x_10, x_11); +lean_dec(x_10); +if (x_12 == 0) { -size_t x_22; size_t x_23; -lean_dec(x_20); -x_22 = 1; -x_23 = lean_usize_add(x_5, x_22); -x_5 = x_23; +size_t x_13; size_t x_14; +lean_dec(x_11); +x_13 = 1; +x_14 = lean_usize_add(x_6, x_13); +x_6 = x_14; goto _start; } else { -lean_object* x_25; -x_25 = l_Lean_Meta_Grind_getEqc(x_20, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -if (lean_obj_tag(x_25) == 0) -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; size_t x_29; size_t x_30; -x_26 = lean_ctor_get(x_25, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_25, 1); -lean_inc(x_27); -lean_dec(x_25); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_26); -lean_ctor_set(x_28, 1, x_6); -x_29 = 1; -x_30 = lean_usize_add(x_5, x_29); -x_5 = x_30; -x_6 = x_28; -x_15 = x_27; +lean_object* x_16; lean_object* x_17; size_t x_18; size_t x_19; +lean_inc(x_1); +x_16 = l_Lean_Meta_Grind_Goal_getEqc(x_1, x_11); +x_17 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_7); +x_18 = 1; +x_19 = lean_usize_add(x_6, x_18); +x_6 = x_19; +x_7 = x_17; goto _start; } -else -{ -uint8_t x_32; -lean_dec(x_6); -x_32 = !lean_is_exclusive(x_25); -if (x_32 == 0) -{ -return x_25; } -else -{ -lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_33 = lean_ctor_get(x_25, 0); -x_34 = lean_ctor_get(x_25, 1); -lean_inc(x_34); -lean_inc(x_33); -lean_dec(x_25); -x_35 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_35, 0, x_33); -lean_ctor_set(x_35, 1, x_34); -return x_35; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Grind_Goal_getEqcs(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; size_t x_5; size_t x_6; lean_object* x_7; +x_2 = lean_box(0); +x_3 = l_Lean_Meta_Grind_Goal_getENodes(x_1); +x_4 = lean_box(0); +x_5 = lean_array_size(x_3); +x_6 = 0; +x_7 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1(x_1, x_3, x_4, x_3, x_5, x_6, x_2); +lean_dec(x_3); +return x_7; } } +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +_start: +{ +size_t x_8; size_t x_9; lean_object* x_10; +x_8 = lean_unbox_usize(x_5); +lean_dec(x_5); +x_9 = lean_unbox_usize(x_6); +lean_dec(x_6); +x_10 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_Goal_getEqcs___spec__1(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_2); +return x_10; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqcs(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; size_t x_15; size_t x_16; lean_object* x_17; -x_10 = lean_box(0); -x_11 = l_Lean_Meta_Grind_getENodes(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -x_12 = lean_ctor_get(x_11, 0); -lean_inc(x_12); -x_13 = lean_ctor_get(x_11, 1); -lean_inc(x_13); -lean_dec(x_11); -x_14 = lean_box(0); -x_15 = lean_array_size(x_12); -x_16 = 0; -x_17 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1(x_12, x_14, x_12, x_15, x_16, x_10, x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_13); -lean_dec(x_12); -if (lean_obj_tag(x_17) == 0) -{ -uint8_t x_18; -x_18 = !lean_is_exclusive(x_17); -if (x_18 == 0) -{ -return x_17; -} -else +lean_object* x_10; uint8_t x_11; +x_10 = lean_st_ref_get(x_1, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; -x_19 = lean_ctor_get(x_17, 0); -x_20 = lean_ctor_get(x_17, 1); -lean_inc(x_20); -lean_inc(x_19); -lean_dec(x_17); -x_21 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -return x_21; -} +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_10, 0); +x_13 = l_Lean_Meta_Grind_Goal_getEqcs(x_12); +lean_ctor_set(x_10, 0, x_13); +return x_10; } else { -uint8_t x_22; -x_22 = !lean_is_exclusive(x_17); -if (x_22 == 0) -{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_14 = lean_ctor_get(x_10, 0); +x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_10); +x_16 = l_Lean_Meta_Grind_Goal_getEqcs(x_14); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_16); +lean_ctor_set(x_17, 1, x_15); return x_17; } -else -{ -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_17, 0); -x_24 = lean_ctor_get(x_17, 1); -lean_inc(x_24); -lean_inc(x_23); -lean_dec(x_17); -x_25 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); -return x_25; -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15) { -_start: -{ -size_t x_16; size_t x_17; lean_object* x_18; -x_16 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_17 = lean_unbox_usize(x_5); -lean_dec(x_5); -x_18 = l_Array_forIn_x27Unsafe_loop___at_Lean_Meta_Grind_getEqcs___spec__1(x_1, x_2, x_3, x_16, x_17, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -return x_18; } } LEAN_EXPORT lean_object* l_Lean_Meta_Grind_getEqcs___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { @@ -22511,7 +23977,7 @@ if (x_12 == 0) { lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; x_13 = lean_ctor_get(x_11, 0); -x_14 = lean_ctor_get(x_13, 18); +x_14 = lean_ctor_get(x_13, 20); lean_inc(x_14); lean_dec(x_13); x_15 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__1(x_14, x_1); @@ -22527,7 +23993,7 @@ x_18 = lean_ctor_get(x_11, 1); lean_inc(x_18); lean_inc(x_17); lean_dec(x_11); -x_19 = lean_ctor_get(x_17, 18); +x_19 = lean_ctor_get(x_17, 20); lean_inc(x_19); lean_dec(x_17); x_20 = l_Lean_PersistentHashMap_contains___at_Lean_Meta_Grind_isResolvedCaseSplit___spec__1(x_19, x_1); @@ -23106,10 +24572,10 @@ x_15 = !lean_is_exclusive(x_13); if (x_15 == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; -x_16 = lean_ctor_get(x_13, 18); +x_16 = lean_ctor_get(x_13, 20); x_17 = lean_box(0); x_18 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__1(x_16, x_1, x_17); -lean_ctor_set(x_13, 18, x_18); +lean_ctor_set(x_13, 20, x_18); x_19 = lean_st_ref_set(x_3, x_13, x_14); x_20 = !lean_is_exclusive(x_19); if (x_20 == 0) @@ -23134,15 +24600,15 @@ return x_23; } else { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; x_24 = lean_ctor_get(x_13, 0); x_25 = lean_ctor_get(x_13, 1); x_26 = lean_ctor_get(x_13, 2); x_27 = lean_ctor_get(x_13, 3); x_28 = lean_ctor_get(x_13, 4); x_29 = lean_ctor_get(x_13, 5); -x_30 = lean_ctor_get_uint8(x_13, sizeof(void*)*20); -x_31 = lean_ctor_get(x_13, 6); +x_30 = lean_ctor_get(x_13, 6); +x_31 = lean_ctor_get_uint8(x_13, sizeof(void*)*23); x_32 = lean_ctor_get(x_13, 7); x_33 = lean_ctor_get(x_13, 8); x_34 = lean_ctor_get(x_13, 9); @@ -23156,6 +24622,12 @@ x_41 = lean_ctor_get(x_13, 16); x_42 = lean_ctor_get(x_13, 17); x_43 = lean_ctor_get(x_13, 18); x_44 = lean_ctor_get(x_13, 19); +x_45 = lean_ctor_get(x_13, 20); +x_46 = lean_ctor_get(x_13, 21); +x_47 = lean_ctor_get(x_13, 22); +lean_inc(x_47); +lean_inc(x_46); +lean_inc(x_45); lean_inc(x_44); lean_inc(x_43); lean_inc(x_42); @@ -23169,7 +24641,7 @@ lean_inc(x_35); lean_inc(x_34); lean_inc(x_33); lean_inc(x_32); -lean_inc(x_31); +lean_inc(x_30); lean_inc(x_29); lean_inc(x_28); lean_inc(x_27); @@ -23177,49 +24649,52 @@ lean_inc(x_26); lean_inc(x_25); lean_inc(x_24); lean_dec(x_13); -x_45 = lean_box(0); -x_46 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__1(x_43, x_1, x_45); -x_47 = lean_alloc_ctor(0, 20, 1); -lean_ctor_set(x_47, 0, x_24); -lean_ctor_set(x_47, 1, x_25); -lean_ctor_set(x_47, 2, x_26); -lean_ctor_set(x_47, 3, x_27); -lean_ctor_set(x_47, 4, x_28); -lean_ctor_set(x_47, 5, x_29); -lean_ctor_set(x_47, 6, x_31); -lean_ctor_set(x_47, 7, x_32); -lean_ctor_set(x_47, 8, x_33); -lean_ctor_set(x_47, 9, x_34); -lean_ctor_set(x_47, 10, x_35); -lean_ctor_set(x_47, 11, x_36); -lean_ctor_set(x_47, 12, x_37); -lean_ctor_set(x_47, 13, x_38); -lean_ctor_set(x_47, 14, x_39); -lean_ctor_set(x_47, 15, x_40); -lean_ctor_set(x_47, 16, x_41); -lean_ctor_set(x_47, 17, x_42); -lean_ctor_set(x_47, 18, x_46); -lean_ctor_set(x_47, 19, x_44); -lean_ctor_set_uint8(x_47, sizeof(void*)*20, x_30); -x_48 = lean_st_ref_set(x_3, x_47, x_14); -x_49 = lean_ctor_get(x_48, 1); -lean_inc(x_49); -if (lean_is_exclusive(x_48)) { - lean_ctor_release(x_48, 0); - lean_ctor_release(x_48, 1); - x_50 = x_48; +x_48 = lean_box(0); +x_49 = l_Lean_PersistentHashMap_insert___at_Lean_Meta_Grind_markCaseSplitAsResolved___spec__1(x_45, x_1, x_48); +x_50 = lean_alloc_ctor(0, 23, 1); +lean_ctor_set(x_50, 0, x_24); +lean_ctor_set(x_50, 1, x_25); +lean_ctor_set(x_50, 2, x_26); +lean_ctor_set(x_50, 3, x_27); +lean_ctor_set(x_50, 4, x_28); +lean_ctor_set(x_50, 5, x_29); +lean_ctor_set(x_50, 6, x_30); +lean_ctor_set(x_50, 7, x_32); +lean_ctor_set(x_50, 8, x_33); +lean_ctor_set(x_50, 9, x_34); +lean_ctor_set(x_50, 10, x_35); +lean_ctor_set(x_50, 11, x_36); +lean_ctor_set(x_50, 12, x_37); +lean_ctor_set(x_50, 13, x_38); +lean_ctor_set(x_50, 14, x_39); +lean_ctor_set(x_50, 15, x_40); +lean_ctor_set(x_50, 16, x_41); +lean_ctor_set(x_50, 17, x_42); +lean_ctor_set(x_50, 18, x_43); +lean_ctor_set(x_50, 19, x_44); +lean_ctor_set(x_50, 20, x_49); +lean_ctor_set(x_50, 21, x_46); +lean_ctor_set(x_50, 22, x_47); +lean_ctor_set_uint8(x_50, sizeof(void*)*23, x_31); +x_51 = lean_st_ref_set(x_3, x_50, x_14); +x_52 = lean_ctor_get(x_51, 1); +lean_inc(x_52); +if (lean_is_exclusive(x_51)) { + lean_ctor_release(x_51, 0); + lean_ctor_release(x_51, 1); + x_53 = x_51; } else { - lean_dec_ref(x_48); - x_50 = lean_box(0); + lean_dec_ref(x_51); + x_53 = lean_box(0); } -if (lean_is_scalar(x_50)) { - x_51 = lean_alloc_ctor(0, 2, 0); +if (lean_is_scalar(x_53)) { + x_54 = lean_alloc_ctor(0, 2, 0); } else { - x_51 = x_50; + x_54 = x_53; } -lean_ctor_set(x_51, 0, x_45); -lean_ctor_set(x_51, 1, x_49); -return x_51; +lean_ctor_set(x_54, 0, x_48); +lean_ctor_set(x_54, 1, x_52); +return x_54; } } } @@ -23243,7 +24718,7 @@ static lean_object* _init_l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__3( _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1; +x_1 = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1; x_2 = l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__1; x_3 = l_Lean_Meta_Grind_markCaseSplitAsResolved___closed__2; x_4 = l_Lean_Name_mkStr3(x_1, x_2, x_3); @@ -23300,7 +24775,7 @@ lean_inc(x_26); lean_dec(x_25); lean_inc(x_1); x_27 = l_Lean_MessageData_ofExpr(x_1); -x_28 = l_Lean_Meta_Grind_getENode___closed__3; +x_28 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3; lean_ctor_set_tag(x_16, 7); lean_ctor_set(x_16, 1, x_27); lean_ctor_set(x_16, 0, x_28); @@ -23357,7 +24832,7 @@ lean_inc(x_40); lean_dec(x_39); lean_inc(x_1); x_41 = l_Lean_MessageData_ofExpr(x_1); -x_42 = l_Lean_Meta_Grind_getENode___closed__3; +x_42 = l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3; x_43 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_43, 0, x_42); lean_ctor_set(x_43, 1, x_41); @@ -23497,8 +24972,10 @@ lean_object* initialize_Lean_Meta_CongrTheorems(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_AbstractNestedProofs(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Simp_Types(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Util(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_ENodeKey(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Canon(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_Attr(uint8_t builtin, lean_object*); +lean_object* initialize_Lean_Meta_Tactic_Grind_Arith_Types(uint8_t builtin, lean_object*); lean_object* initialize_Lean_Meta_Tactic_Grind_EMatchTheorem(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Lean_Meta_Tactic_Grind_Types(uint8_t builtin, lean_object* w) { @@ -23532,12 +25009,18 @@ lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Util(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_ENodeKey(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Canon(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_Attr(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Lean_Meta_Tactic_Grind_Arith_Types(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Lean_Meta_Tactic_Grind_EMatchTheorem(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); @@ -23549,40 +25032,40 @@ l_Lean_Meta_Grind_congrPlaceholderProof___closed__3 = _init_l_Lean_Meta_Grind_co lean_mark_persistent(l_Lean_Meta_Grind_congrPlaceholderProof___closed__3); l_Lean_Meta_Grind_congrPlaceholderProof = _init_l_Lean_Meta_Grind_congrPlaceholderProof(); lean_mark_persistent(l_Lean_Meta_Grind_congrPlaceholderProof); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__1); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__2); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__3); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__4); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__5); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__6); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__7); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__8); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78____closed__9); -if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_78_(lean_io_mk_world()); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__1); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__2); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__3); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__4); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__5); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__6); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__7); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__8); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69____closed__9); +if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_69_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_Grind_grind_debug = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_Grind_grind_debug); lean_dec_ref(res); -}l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__1); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__2); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__3); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__4); -l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5(); -lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118____closed__5); -if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_118_(lean_io_mk_world()); +}l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__1); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__2); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__3); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__4); +l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5 = _init_l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5(); +lean_mark_persistent(l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109____closed__5); +if (builtin) {res = l_Lean_Meta_Grind_initFn____x40_Lean_Meta_Tactic_Grind_Types___hyg_109_(lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; l_Lean_Meta_Grind_grind_debug_proofs = lean_io_result_get_value(res); lean_mark_persistent(l_Lean_Meta_Grind_grind_debug_proofs); @@ -23594,12 +25077,6 @@ l_Lean_Meta_Grind_abstractNestedProofs___closed__2 = _init_l_Lean_Meta_Grind_abs lean_mark_persistent(l_Lean_Meta_Grind_abstractNestedProofs___closed__2); l_Lean_Meta_Grind_abstractNestedProofs___closed__3 = _init_l_Lean_Meta_Grind_abstractNestedProofs___closed__3(); lean_mark_persistent(l_Lean_Meta_Grind_abstractNestedProofs___closed__3); -l_Lean_Meta_Grind_canon___closed__1 = _init_l_Lean_Meta_Grind_canon___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_canon___closed__1); -l_Lean_Meta_Grind_canon___closed__2 = _init_l_Lean_Meta_Grind_canon___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_canon___closed__2); -l_Lean_Meta_Grind_canon___closed__3 = _init_l_Lean_Meta_Grind_canon___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_canon___closed__3); l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__1 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__1(); l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__2 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__2(); l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__3 = _init_l_Lean_PersistentHashMap_insertAux___at_Lean_Meta_Grind_mkHCongrWithArity___spec__2___closed__3(); @@ -23610,116 +25087,120 @@ l_Lean_Meta_Grind_instInhabitedENode___closed__2 = _init_l_Lean_Meta_Grind_instI lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedENode___closed__2); l_Lean_Meta_Grind_instInhabitedENode = _init_l_Lean_Meta_Grind_instInhabitedENode(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedENode); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__1); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__2); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__3); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__4); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__5); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__6); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__7); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__8); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__9); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__10); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__11); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__12); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__13); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__14); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__15); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__16); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__17); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__18); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__19); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__20); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__21); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__22); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__23); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__24); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__25); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__26); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__27); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__28); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__29); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__30); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__31); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__32); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__33); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__34); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__35); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__36); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__37); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__38); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__39); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__40); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__41); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__42); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__43); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__44); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__45); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__46); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__47); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__48); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__49); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__50); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__51); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__52); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__53); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__54); -l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55(); -lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1560____closed__55); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__1); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__2); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__3); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__4); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__5); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__6); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__7); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__8); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__9); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__10); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__11); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__12); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__13); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__14); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__15); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__16); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__17); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__18); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__19); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__20); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__21); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__22); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__23); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__24); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__25); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__26); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__27); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__28); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__29); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__30); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__31); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__32); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__33); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__34); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__35); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__36); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__37); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__38); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__39); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__40); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__41); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__42); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__43); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__44); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__45); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__46); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__47); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__48); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__49); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__50); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__51); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__52); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__53); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__54); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__55); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__56); +l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57 = _init_l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57(); +lean_mark_persistent(l___private_Lean_Meta_Tactic_Grind_Types_0__Lean_Meta_Grind_reprENode____x40_Lean_Meta_Tactic_Grind_Types___hyg_1445____closed__57); l_Lean_Meta_Grind_instReprENode___closed__1 = _init_l_Lean_Meta_Grind_instReprENode___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_instReprENode___closed__1); l_Lean_Meta_Grind_instReprENode = _init_l_Lean_Meta_Grind_instReprENode(); @@ -23742,6 +25223,10 @@ l_Lean_Meta_Grind_instInhabitedNewFact___closed__1 = _init_l_Lean_Meta_Grind_ins lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedNewFact___closed__1); l_Lean_Meta_Grind_instInhabitedNewFact = _init_l_Lean_Meta_Grind_instInhabitedNewFact(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedNewFact); +l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1 = _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1(); +lean_mark_persistent(l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__1); +l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2 = _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2(); +lean_mark_persistent(l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1___closed__2); l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1 = _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1(); lean_mark_persistent(l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__1); l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2 = _init_l_Lean_PersistentHashMap_empty___at_Lean_Meta_Grind_instInhabitedGoal___spec__2(); @@ -23753,12 +25238,16 @@ lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__1); l_Lean_Meta_Grind_instInhabitedGoal___closed__2 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__2); l_Lean_Meta_Grind_instInhabitedGoal___closed__3 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__3); l_Lean_Meta_Grind_instInhabitedGoal___closed__4 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__4(); -lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__4); l_Lean_Meta_Grind_instInhabitedGoal___closed__5 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__5(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__5); l_Lean_Meta_Grind_instInhabitedGoal___closed__6 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__6(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__6); +l_Lean_Meta_Grind_instInhabitedGoal___closed__7 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__7(); +lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__7); +l_Lean_Meta_Grind_instInhabitedGoal___closed__8 = _init_l_Lean_Meta_Grind_instInhabitedGoal___closed__8(); +lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal___closed__8); l_Lean_Meta_Grind_instInhabitedGoal = _init_l_Lean_Meta_Grind_instInhabitedGoal(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedGoal); l_Lean_Meta_Grind_GoalM_run_x27___closed__1 = _init_l_Lean_Meta_Grind_GoalM_run_x27___closed__1(); @@ -23980,23 +25469,41 @@ l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean_ lean_mark_persistent(l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__15); l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__16 = _init_l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__16(); lean_mark_persistent(l_Lean_Meta_Grind___aux__Lean__Meta__Tactic__Grind__Types______macroRules__Lean__Meta__Grind__doElemTrace__goal_x5b___x5d______1___closed__16); -l_Lean_Meta_Grind_getENode___closed__1 = _init_l_Lean_Meta_Grind_getENode___closed__1(); -lean_mark_persistent(l_Lean_Meta_Grind_getENode___closed__1); -l_Lean_Meta_Grind_getENode___closed__2 = _init_l_Lean_Meta_Grind_getENode___closed__2(); -lean_mark_persistent(l_Lean_Meta_Grind_getENode___closed__2); -l_Lean_Meta_Grind_getENode___closed__3 = _init_l_Lean_Meta_Grind_getENode___closed__3(); -lean_mark_persistent(l_Lean_Meta_Grind_getENode___closed__3); +l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1 = _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__1); +l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2 = _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__2); +l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3 = _init_l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_throwNonInternalizedExpr___rarg___closed__3); l_Lean_Meta_Grind_hasSameType___closed__1 = _init_l_Lean_Meta_Grind_hasSameType___closed__1(); +l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1 = _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___lambda__2___closed__1); +l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2 = _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___lambda__2___closed__2); +l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3 = _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___lambda__2___closed__3); +l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4 = _init_l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___lambda__2___closed__4); +l_Lean_Meta_Grind_isNatNum___closed__1 = _init_l_Lean_Meta_Grind_isNatNum___closed__1(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___closed__1); +l_Lean_Meta_Grind_isNatNum___closed__2 = _init_l_Lean_Meta_Grind_isNatNum___closed__2(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___closed__2); +l_Lean_Meta_Grind_isNatNum___closed__3 = _init_l_Lean_Meta_Grind_isNatNum___closed__3(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___closed__3); +l_Lean_Meta_Grind_isNatNum___closed__4 = _init_l_Lean_Meta_Grind_isNatNum___closed__4(); +lean_mark_persistent(l_Lean_Meta_Grind_isNatNum___closed__4); l_Lean_Meta_Grind_markAsInconsistent___closed__1 = _init_l_Lean_Meta_Grind_markAsInconsistent___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_markAsInconsistent___closed__1); l_Lean_Meta_Grind_markAsInconsistent___closed__2 = _init_l_Lean_Meta_Grind_markAsInconsistent___closed__2(); lean_mark_persistent(l_Lean_Meta_Grind_markAsInconsistent___closed__2); l_Lean_Meta_Grind_markAsInconsistent___closed__3 = _init_l_Lean_Meta_Grind_markAsInconsistent___closed__3(); lean_mark_persistent(l_Lean_Meta_Grind_markAsInconsistent___closed__3); -l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1 = _init_l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1(); -lean_mark_persistent(l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_getENodes___spec__1___closed__1); -l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1 = _init_l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Meta_Grind_getENodes___spec__4___closed__1); +l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1 = _init_l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1(); +lean_mark_persistent(l_Lean_PersistentHashMap_toArray___at_Lean_Meta_Grind_Goal_getENodes___spec__1___closed__1); +l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1 = _init_l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Meta_Grind_Goal_getENodes___spec__4___closed__1); +l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1 = _init_l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1(); +lean_mark_persistent(l_Lean_Loop_forIn_loop___at_Lean_Meta_Grind_traverseEqc___spec__1___closed__1); l_Lean_Meta_Grind_instInhabitedMethods___closed__1 = _init_l_Lean_Meta_Grind_instInhabitedMethods___closed__1(); lean_mark_persistent(l_Lean_Meta_Grind_instInhabitedMethods___closed__1); l_Lean_Meta_Grind_instInhabitedMethods = _init_l_Lean_Meta_Grind_instInhabitedMethods(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c index 0f314e09b619..4bbb1f70b851 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c +++ b/stage0/stdlib/Lean/Meta/Tactic/LinearArith/Nat/Simp.c @@ -17,7 +17,6 @@ lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); lean_object* l_Lean_mkNatLit(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__3; lean_object* l_Lean_mkAppN(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__14; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; @@ -29,27 +28,29 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__3; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7; lean_object* l_Lean_mkAppB(lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); +uint8_t l_Lean_Expr_isApp(lean_object*); lean_object* l_Lean_Meta_Linear_Nat_LinearExpr_toExpr(lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__15; +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_LinearCnstr_toArith(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3(size_t, size_t, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1; lean_object* l_Lean_Meta_mkExpectedTypeHint(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearCnstr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__1; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__3; +lean_object* l_Lean_Expr_cleanupAnnotations(lean_object*); lean_object* l_Lean_mkApp4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_withAbstractAtoms___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_mkAdd(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__8; @@ -60,18 +61,16 @@ static lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbs lean_object* l_Lean_Meta_Linear_Nat_ToLinear_run___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10; lean_object* l___private_Lean_CoreM_0__Lean_Core_mkFreshNameImp(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__16; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5; +lean_object* l_Lean_Expr_appArg(lean_object*, lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___closed__2; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20; lean_object* l_Lean_Meta_mkEq(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Lean_Expr_appFnCleanup(lean_object*, lean_object*); lean_object* l_Lean_Meta_Linear_Nat_LinearExpr_toArith(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15; lean_object* l_Lean_Meta_mkLE(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_Linear_Poly_toExpr(lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -85,35 +84,47 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__4 LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls_loop___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Meta_Linear_Nat_reflTrue; +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDeclsD___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__2(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1; lean_object* l_Nat_Linear_Poly_norm(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__17; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__9; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_mkApp3(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2; +uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); lean_object* l_Nat_Linear_PolyCnstr_toExpr(lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2; lean_object* l_Nat_Linear_ExprCnstr_toPoly(lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__5; LEAN_EXPORT lean_object* l_Lean_Meta_withLocalDecls___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__4(lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); extern lean_object* l_Lean_levelOne; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1___closed__11; -static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18; +lean_object* l_Lean_Meta_instantiateMVarsIfMVarApp(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_Linear_Expr_toPoly(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__5; @@ -130,6 +141,7 @@ static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4; static lean_object* l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__2; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__6; static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__2; +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_withLocalDecl___at_Lean_Meta_addPPExplicitToExposeDiff_visit___spec__4___rarg(lean_object*, uint8_t, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Nat_Linear_PolyCnstr_isValid(lean_object*); @@ -143,8 +155,12 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstrac lean_object* l_Lean_Meta_Linear_Nat_ToLinear_toLinearExpr(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2; lean_object* l_Lean_Expr_beta(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstrPos_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2; +static lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3; static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1() { _start: { @@ -2633,205 +2649,629 @@ return x_117; } } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Not", 3, 3); +x_1 = lean_mk_string_unchecked("not_gt_eq", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1; -x_3 = l_Lean_Name_str___override(x_1, x_2); +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3() { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("LE", 2, 2); -return x_1; +lean_object* x_10; uint8_t x_11; +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; +x_11 = l_Lean_Expr_isConstOf(x_4, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +x_13 = lean_box(0); +x_14 = lean_apply_8(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9); +return x_14; } +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_2); +x_15 = lean_unsigned_to_nat(0u); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_15); +x_17 = lean_unsigned_to_nat(2u); +x_18 = lean_nat_sub(x_16, x_17); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_18, x_19); +lean_dec(x_18); +x_21 = l_Lean_Expr_getRevArg_x21(x_3, x_20); +x_22 = lean_unsigned_to_nat(3u); +x_23 = lean_nat_sub(x_16, x_22); +lean_dec(x_16); +x_24 = lean_nat_sub(x_23, x_19); +lean_dec(x_23); +x_25 = l_Lean_Expr_getRevArg_x21(x_3, x_24); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_26 = l_Lean_Meta_mkLE(x_21, x_25, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_27); +x_30 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2; +x_31 = lean_box(0); +x_32 = lean_apply_8(x_1, x_29, x_30, x_31, x_5, x_6, x_7, x_8, x_28); +return x_32; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4() { +else +{ +uint8_t x_33; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_33 = !lean_is_exclusive(x_26); +if (x_33 == 0) +{ +return x_26; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_26, 0); +x_35 = lean_ctor_get(x_26, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_26); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("le", 2, 2); +x_1 = lean_mk_string_unchecked("not_lt_eq", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6() { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("GE", 2, 2); -return x_1; +lean_object* x_10; uint8_t x_11; +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; +x_11 = l_Lean_Expr_isConstOf(x_4, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +x_13 = lean_box(0); +x_14 = lean_apply_8(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9); +return x_14; } +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_2); +x_15 = lean_unsigned_to_nat(0u); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_15); +x_17 = lean_unsigned_to_nat(3u); +x_18 = lean_nat_sub(x_16, x_17); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_18, x_19); +lean_dec(x_18); +x_21 = l_Lean_Expr_getRevArg_x21(x_3, x_20); +x_22 = lean_unsigned_to_nat(2u); +x_23 = lean_nat_sub(x_16, x_22); +lean_dec(x_16); +x_24 = lean_nat_sub(x_23, x_19); +lean_dec(x_23); +x_25 = l_Lean_Expr_getRevArg_x21(x_3, x_24); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_26 = l_Lean_Meta_mkLE(x_21, x_25, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +lean_dec(x_26); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_27); +x_30 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2; +x_31 = lean_box(0); +x_32 = lean_apply_8(x_1, x_29, x_30, x_31, x_5, x_6, x_7, x_8, x_28); +return x_32; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7() { +else +{ +uint8_t x_33; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_33 = !lean_is_exclusive(x_26); +if (x_33 == 0) +{ +return x_26; +} +else +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_34 = lean_ctor_get(x_26, 0); +x_35 = lean_ctor_get(x_26, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_26); +x_36 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_36, 0, x_34); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1u); +x_2 = l_Lean_mkNatLit(x_1); +return x_2; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("ge", 2, 2); +x_1 = lean_mk_string_unchecked("not_ge_eq", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9() { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("LT", 2, 2); -return x_1; +lean_object* x_10; uint8_t x_11; +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; +x_11 = l_Lean_Expr_isConstOf(x_4, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +x_13 = lean_box(0); +x_14 = lean_apply_8(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9); +return x_14; } +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_2); +x_15 = lean_unsigned_to_nat(0u); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_15); +x_17 = lean_unsigned_to_nat(2u); +x_18 = lean_nat_sub(x_16, x_17); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_18, x_19); +lean_dec(x_18); +x_21 = l_Lean_Expr_getRevArg_x21(x_3, x_20); +x_22 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_23 = l_Lean_Meta_mkAdd(x_21, x_22, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_unsigned_to_nat(3u); +x_27 = lean_nat_sub(x_16, x_26); +lean_dec(x_16); +x_28 = lean_nat_sub(x_27, x_19); +lean_dec(x_27); +x_29 = l_Lean_Expr_getRevArg_x21(x_3, x_28); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_30 = l_Lean_Meta_mkLE(x_24, x_29, x_5, x_6, x_7, x_8, x_25); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_31); +x_34 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3; +x_35 = lean_box(0); +x_36 = lean_apply_8(x_1, x_33, x_34, x_35, x_5, x_6, x_7, x_8, x_32); +return x_36; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10() { +else +{ +uint8_t x_37; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_37 = !lean_is_exclusive(x_30); +if (x_37 == 0) +{ +return x_30; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_30, 0); +x_39 = lean_ctor_get(x_30, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_30); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_16); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_23); +if (x_41 == 0) +{ +return x_23; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_23, 0); +x_43 = lean_ctor_get(x_23, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_23); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("lt", 2, 2); +x_1 = lean_mk_string_unchecked("not_le_eq", 9, 9); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12() { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("GT", 2, 2); -return x_1; +lean_object* x_10; uint8_t x_11; +x_10 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__2; +x_11 = l_Lean_Expr_isConstOf(x_4, x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_box(0); +x_13 = lean_box(0); +x_14 = lean_apply_8(x_1, x_2, x_12, x_13, x_5, x_6, x_7, x_8, x_9); +return x_14; } +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; +lean_dec(x_2); +x_15 = lean_unsigned_to_nat(0u); +x_16 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_3, x_15); +x_17 = lean_unsigned_to_nat(3u); +x_18 = lean_nat_sub(x_16, x_17); +x_19 = lean_unsigned_to_nat(1u); +x_20 = lean_nat_sub(x_18, x_19); +lean_dec(x_18); +x_21 = l_Lean_Expr_getRevArg_x21(x_3, x_20); +x_22 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1; +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_23 = l_Lean_Meta_mkAdd(x_21, x_22, x_5, x_6, x_7, x_8, x_9); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_unsigned_to_nat(2u); +x_27 = lean_nat_sub(x_16, x_26); +lean_dec(x_16); +x_28 = lean_nat_sub(x_27, x_19); +lean_dec(x_27); +x_29 = l_Lean_Expr_getRevArg_x21(x_3, x_28); +lean_inc(x_8); +lean_inc(x_7); +lean_inc(x_6); +lean_inc(x_5); +x_30 = l_Lean_Meta_mkLE(x_24, x_29, x_5, x_6, x_7, x_8, x_25); +if (lean_obj_tag(x_30) == 0) +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_30, 1); +lean_inc(x_32); +lean_dec(x_30); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_31); +x_34 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2; +x_35 = lean_box(0); +x_36 = lean_apply_8(x_1, x_33, x_34, x_35, x_5, x_6, x_7, x_8, x_32); +return x_36; } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13() { +else +{ +uint8_t x_37; +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_37 = !lean_is_exclusive(x_30); +if (x_37 == 0) +{ +return x_30; +} +else +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_30, 0); +x_39 = lean_ctor_get(x_30, 1); +lean_inc(x_39); +lean_inc(x_38); +lean_dec(x_30); +x_40 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_40, 0, x_38); +lean_ctor_set(x_40, 1, x_39); +return x_40; +} +} +} +else +{ +uint8_t x_41; +lean_dec(x_16); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_41 = !lean_is_exclusive(x_23); +if (x_41 == 0) +{ +return x_23; +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_42 = lean_ctor_get(x_23, 0); +x_43 = lean_ctor_get(x_23, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_23); +x_44 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +return x_44; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +_start: +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_box(0); +x_10 = lean_box(0); +x_11 = lean_apply_8(x_1, x_2, x_9, x_10, x_4, x_5, x_6, x_7, x_8); +return x_11; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("gt", 2, 2); +x_1 = lean_mk_string_unchecked("Not", 3, 3); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); +x_1 = lean_box(0); +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1; +x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_gt_eq", 9, 9); +x_1 = lean_mk_string_unchecked("GT", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("gt", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__3; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__4; +x_3 = l_Lean_Name_mkStr2(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("LT", 2, 2); +return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_lt_eq", 9, 9); +x_1 = lean_mk_string_unchecked("lt", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17; +x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__6; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__7; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9() { _start: { -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1u); -x_2 = l_Lean_mkNatLit(x_1); -return x_2; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("GE", 2, 2); +return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_ge_eq", 9, 9); +x_1 = lean_mk_string_unchecked("ge", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20; +x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__9; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__10; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12() { _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("not_le_eq", 9, 9); +x_1 = lean_mk_string_unchecked("LE", 2, 2); return x_1; } } -static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23() { +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("le", 2, 2); +return x_1; +} +} +static lean_object* _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Meta_Linear_Nat_withAbstractAtoms___spec__1___lambda__1___closed__1; -x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22; +x_1 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__12; +x_2 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } @@ -2851,402 +3291,223 @@ return x_10; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_11 = l_Lean_Expr_appArg_x21(x_1); x_12 = lean_box(0); -x_13 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5; -x_14 = lean_unsigned_to_nat(4u); -x_15 = l_Lean_Expr_isAppOfArity(x_11, x_13, x_14); -if (x_15 == 0) -{ -lean_object* x_16; uint8_t x_17; -x_16 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8; -x_17 = l_Lean_Expr_isAppOfArity(x_11, x_16, x_14); -if (x_17 == 0) -{ -lean_object* x_18; uint8_t x_19; -x_18 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11; -x_19 = l_Lean_Expr_isAppOfArity(x_11, x_18, x_14); -if (x_19 == 0) -{ -lean_object* x_20; uint8_t x_21; -x_20 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14; -x_21 = l_Lean_Expr_isAppOfArity(x_11, x_20, x_14); -if (x_21 == 0) +lean_inc(x_1); +lean_inc(x_11); +x_13 = lean_alloc_closure((void*)(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___boxed), 11, 3); +lean_closure_set(x_13, 0, x_12); +lean_closure_set(x_13, 1, x_11); +lean_closure_set(x_13, 2, x_1); +lean_inc(x_11); +x_14 = l_Lean_Meta_instantiateMVarsIfMVarApp(x_11, x_2, x_3, x_4, x_5, x_6); +x_15 = lean_ctor_get(x_14, 0); +lean_inc(x_15); +x_16 = lean_ctor_get(x_14, 1); +lean_inc(x_16); +lean_dec(x_14); +x_17 = l_Lean_Expr_cleanupAnnotations(x_15); +x_18 = l_Lean_Expr_isApp(x_17); +if (x_18 == 0) { -lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_22 = lean_box(0); -x_23 = lean_box(0); -x_24 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_22, x_23, x_2, x_3, x_4, x_5, x_6); +lean_object* x_19; lean_object* x_20; lean_object* x_21; +lean_dec(x_17); +lean_dec(x_13); +x_19 = lean_box(0); +x_20 = lean_box(0); +x_21 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_19, x_20, x_2, x_3, x_4, x_5, x_16); lean_dec(x_11); -return x_24; +return x_21; } else { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; -x_25 = lean_unsigned_to_nat(0u); -x_26 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_25); -x_27 = lean_unsigned_to_nat(2u); -x_28 = lean_nat_sub(x_26, x_27); -x_29 = lean_nat_sub(x_28, x_8); -lean_dec(x_28); -x_30 = l_Lean_Expr_getRevArg_x21(x_11, x_29); -x_31 = lean_unsigned_to_nat(3u); -x_32 = lean_nat_sub(x_26, x_31); -lean_dec(x_26); -x_33 = lean_nat_sub(x_32, x_8); -lean_dec(x_32); -x_34 = l_Lean_Expr_getRevArg_x21(x_11, x_33); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_35 = l_Lean_Meta_mkLE(x_30, x_34, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_35) == 0) +lean_object* x_22; uint8_t x_23; +x_22 = l_Lean_Expr_appFnCleanup(x_17, lean_box(0)); +x_23 = l_Lean_Expr_isApp(x_22); +if (x_23 == 0) { -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_36 = lean_ctor_get(x_35, 0); -lean_inc(x_36); -x_37 = lean_ctor_get(x_35, 1); -lean_inc(x_37); -lean_dec(x_35); -x_38 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_38, 0, x_36); -x_39 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16; -x_40 = lean_box(0); -x_41 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_38, x_39, x_40, x_2, x_3, x_4, x_5, x_37); +lean_object* x_24; lean_object* x_25; lean_object* x_26; +lean_dec(x_22); +lean_dec(x_13); +x_24 = lean_box(0); +x_25 = lean_box(0); +x_26 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_24, x_25, x_2, x_3, x_4, x_5, x_16); lean_dec(x_11); -return x_41; +return x_26; } else { -uint8_t x_42; -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_42 = !lean_is_exclusive(x_35); -if (x_42 == 0) -{ -return x_35; -} -else +lean_object* x_27; uint8_t x_28; +x_27 = l_Lean_Expr_appFnCleanup(x_22, lean_box(0)); +x_28 = l_Lean_Expr_isApp(x_27); +if (x_28 == 0) { -lean_object* x_43; lean_object* x_44; lean_object* x_45; -x_43 = lean_ctor_get(x_35, 0); -x_44 = lean_ctor_get(x_35, 1); -lean_inc(x_44); -lean_inc(x_43); -lean_dec(x_35); -x_45 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_45, 0, x_43); -lean_ctor_set(x_45, 1, x_44); -return x_45; -} -} -} +lean_object* x_29; lean_object* x_30; lean_object* x_31; +lean_dec(x_27); +lean_dec(x_13); +x_29 = lean_box(0); +x_30 = lean_box(0); +x_31 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_29, x_30, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_11); +return x_31; } else { -lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_46 = lean_unsigned_to_nat(0u); -x_47 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_46); -x_48 = lean_unsigned_to_nat(3u); -x_49 = lean_nat_sub(x_47, x_48); -x_50 = lean_nat_sub(x_49, x_8); -lean_dec(x_49); -x_51 = l_Lean_Expr_getRevArg_x21(x_11, x_50); -x_52 = lean_unsigned_to_nat(2u); -x_53 = lean_nat_sub(x_47, x_52); -lean_dec(x_47); -x_54 = lean_nat_sub(x_53, x_8); -lean_dec(x_53); -x_55 = l_Lean_Expr_getRevArg_x21(x_11, x_54); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_56 = l_Lean_Meta_mkLE(x_51, x_55, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_56) == 0) +lean_object* x_32; uint8_t x_33; +x_32 = l_Lean_Expr_appFnCleanup(x_27, lean_box(0)); +x_33 = l_Lean_Expr_isApp(x_32); +if (x_33 == 0) { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_57 = lean_ctor_get(x_56, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_56, 1); -lean_inc(x_58); -lean_dec(x_56); -x_59 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_59, 0, x_57); -x_60 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18; -x_61 = lean_box(0); -x_62 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_59, x_60, x_61, x_2, x_3, x_4, x_5, x_58); +lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_32); +lean_dec(x_13); +x_34 = lean_box(0); +x_35 = lean_box(0); +x_36 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_34, x_35, x_2, x_3, x_4, x_5, x_16); lean_dec(x_11); -return x_62; +return x_36; } else { -uint8_t x_63; -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_63 = !lean_is_exclusive(x_56); -if (x_63 == 0) -{ -return x_56; -} -else +lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_37 = l_Lean_Expr_appArg(x_32, lean_box(0)); +x_38 = l_Lean_Expr_appFnCleanup(x_32, lean_box(0)); +x_39 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__5; +x_40 = l_Lean_Expr_isConstOf(x_38, x_39); +if (x_40 == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; -x_64 = lean_ctor_get(x_56, 0); -x_65 = lean_ctor_get(x_56, 1); -lean_inc(x_65); -lean_inc(x_64); -lean_dec(x_56); -x_66 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_66, 0, x_64); -lean_ctor_set(x_66, 1, x_65); -return x_66; -} -} -} -} -else +lean_object* x_41; uint8_t x_42; +x_41 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__8; +x_42 = l_Lean_Expr_isConstOf(x_38, x_41); +if (x_42 == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; -x_67 = lean_unsigned_to_nat(0u); -x_68 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_67); -x_69 = lean_unsigned_to_nat(2u); -x_70 = lean_nat_sub(x_68, x_69); -x_71 = lean_nat_sub(x_70, x_8); -lean_dec(x_70); -x_72 = l_Lean_Expr_getRevArg_x21(x_11, x_71); -x_73 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_74 = l_Lean_Meta_mkAdd(x_72, x_73, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_74) == 0) +lean_object* x_43; uint8_t x_44; +x_43 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__11; +x_44 = l_Lean_Expr_isConstOf(x_38, x_43); +if (x_44 == 0) { -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_75 = lean_ctor_get(x_74, 0); -lean_inc(x_75); -x_76 = lean_ctor_get(x_74, 1); -lean_inc(x_76); -lean_dec(x_74); -x_77 = lean_unsigned_to_nat(3u); -x_78 = lean_nat_sub(x_68, x_77); -lean_dec(x_68); -x_79 = lean_nat_sub(x_78, x_8); -lean_dec(x_78); -x_80 = l_Lean_Expr_getRevArg_x21(x_11, x_79); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_81 = l_Lean_Meta_mkLE(x_75, x_80, x_2, x_3, x_4, x_5, x_76); -if (lean_obj_tag(x_81) == 0) +lean_object* x_45; uint8_t x_46; +x_45 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14; +x_46 = l_Lean_Expr_isConstOf(x_38, x_45); +lean_dec(x_38); +if (x_46 == 0) { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_82 = lean_ctor_get(x_81, 0); -lean_inc(x_82); -x_83 = lean_ctor_get(x_81, 1); -lean_inc(x_83); -lean_dec(x_81); -x_84 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_84, 0, x_82); -x_85 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21; -x_86 = lean_box(0); -x_87 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_84, x_85, x_86, x_2, x_3, x_4, x_5, x_83); +lean_object* x_47; lean_object* x_48; lean_object* x_49; +lean_dec(x_37); +lean_dec(x_13); +x_47 = lean_box(0); +x_48 = lean_box(0); +x_49 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_12, x_47, x_48, x_2, x_3, x_4, x_5, x_16); lean_dec(x_11); -return x_87; +return x_49; } else { -uint8_t x_88; -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_50; lean_dec(x_1); -x_88 = !lean_is_exclusive(x_81); -if (x_88 == 0) -{ -return x_81; +x_50 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5(x_13, x_12, x_11, x_37, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_37); +lean_dec(x_11); +return x_50; +} } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_89 = lean_ctor_get(x_81, 0); -x_90 = lean_ctor_get(x_81, 1); -lean_inc(x_90); -lean_inc(x_89); -lean_dec(x_81); -x_91 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_91, 0, x_89); -lean_ctor_set(x_91, 1, x_90); -return x_91; -} +lean_object* x_51; +lean_dec(x_38); +lean_dec(x_1); +x_51 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4(x_13, x_12, x_11, x_37, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_37); +lean_dec(x_11); +return x_51; } } else { -uint8_t x_92; -lean_dec(x_68); -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_52; +lean_dec(x_38); lean_dec(x_1); -x_92 = !lean_is_exclusive(x_74); -if (x_92 == 0) -{ -return x_74; +x_52 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3(x_13, x_12, x_11, x_37, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_37); +lean_dec(x_11); +return x_52; +} } else { -lean_object* x_93; lean_object* x_94; lean_object* x_95; -x_93 = lean_ctor_get(x_74, 0); -x_94 = lean_ctor_get(x_74, 1); -lean_inc(x_94); -lean_inc(x_93); -lean_dec(x_74); -x_95 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_95, 0, x_93); -lean_ctor_set(x_95, 1, x_94); -return x_95; +lean_object* x_53; +lean_dec(x_38); +lean_dec(x_1); +x_53 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2(x_13, x_12, x_11, x_37, x_2, x_3, x_4, x_5, x_16); +lean_dec(x_37); +lean_dec(x_11); +return x_53; +} } } } } -else -{ -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -x_96 = lean_unsigned_to_nat(0u); -x_97 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_11, x_96); -x_98 = lean_unsigned_to_nat(3u); -x_99 = lean_nat_sub(x_97, x_98); -x_100 = lean_nat_sub(x_99, x_8); -lean_dec(x_99); -x_101 = l_Lean_Expr_getRevArg_x21(x_11, x_100); -x_102 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19; -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_103 = l_Lean_Meta_mkAdd(x_101, x_102, x_2, x_3, x_4, x_5, x_6); -if (lean_obj_tag(x_103) == 0) -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_104 = lean_ctor_get(x_103, 0); -lean_inc(x_104); -x_105 = lean_ctor_get(x_103, 1); -lean_inc(x_105); -lean_dec(x_103); -x_106 = lean_unsigned_to_nat(2u); -x_107 = lean_nat_sub(x_97, x_106); -lean_dec(x_97); -x_108 = lean_nat_sub(x_107, x_8); -lean_dec(x_107); -x_109 = l_Lean_Expr_getRevArg_x21(x_11, x_108); -lean_inc(x_5); -lean_inc(x_4); -lean_inc(x_3); -lean_inc(x_2); -x_110 = l_Lean_Meta_mkLE(x_104, x_109, x_2, x_3, x_4, x_5, x_105); -if (lean_obj_tag(x_110) == 0) -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; -x_111 = lean_ctor_get(x_110, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_110, 1); -lean_inc(x_112); -lean_dec(x_110); -x_113 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_113, 0, x_111); -x_114 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23; -x_115 = lean_box(0); -x_116 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_12, x_11, x_1, x_113, x_114, x_115, x_2, x_3, x_4, x_5, x_112); -lean_dec(x_11); -return x_116; } -else -{ -uint8_t x_117; -lean_dec(x_11); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_117 = !lean_is_exclusive(x_110); -if (x_117 == 0) -{ -return x_110; } -else -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_110, 0); -x_119 = lean_ctor_get(x_110, 1); -lean_inc(x_119); -lean_inc(x_118); -lean_dec(x_110); -x_120 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_120, 0, x_118); -lean_ctor_set(x_120, 1, x_119); -return x_120; } +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +_start: +{ +lean_object* x_12; +x_12 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); +lean_dec(x_6); +lean_dec(x_2); +return x_12; } } -else +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -uint8_t x_121; -lean_dec(x_97); -lean_dec(x_11); -lean_dec(x_5); +lean_object* x_10; +x_10 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); lean_dec(x_4); lean_dec(x_3); -lean_dec(x_2); -lean_dec(x_1); -x_121 = !lean_is_exclusive(x_103); -if (x_121 == 0) -{ -return x_103; +return x_10; } -else +} +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: { -lean_object* x_122; lean_object* x_123; lean_object* x_124; -x_122 = lean_ctor_get(x_103, 0); -x_123 = lean_ctor_get(x_103, 1); -lean_inc(x_123); -lean_inc(x_122); -lean_dec(x_103); -x_124 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_124, 0, x_122); -lean_ctor_set(x_124, 1, x_123); -return x_124; +lean_object* x_10; +x_10 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +_start: +{ +lean_object* x_10; +x_10 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); +lean_dec(x_4); +lean_dec(x_3); +return x_10; } } -LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11) { +LEAN_EXPORT lean_object* l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -lean_object* x_12; -x_12 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11); -lean_dec(x_6); -lean_dec(x_2); -return x_12; +lean_object* x_9; +x_9 = l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +lean_dec(x_3); +return x_9; } } static lean_object* _init_l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1() { @@ -3654,6 +3915,24 @@ l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__5 = _init_l_Lean_Meta lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__5); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__6 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__6(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__1___closed__6); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__2___closed__2); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__3___closed__2); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__2); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__4___closed__3); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__1); +l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2(); +lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___lambda__5___closed__2); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__1); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__2(); @@ -3682,24 +3961,6 @@ l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13 = _init_l_Lean_Meta_Linear_Nat lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__13); l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__14); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__15); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__16); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__17); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__18); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__19); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__20); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__21); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__22); -l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23 = _init_l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23(); -lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpCnstr_x3f___closed__23); l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1 = _init_l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1(); lean_mark_persistent(l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__1); l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__2 = _init_l_Lean_Meta_Linear_Nat_simpExpr_x3f___closed__2(); diff --git a/stage0/stdlib/Lean/Meta/Tactic/Simp/Simproc.c b/stage0/stdlib/Lean/Meta/Tactic/Simp/Simproc.c index fad84975e4f0..3323d5bea3da 100644 --- a/stage0/stdlib/Lean/Meta/Tactic/Simp/Simproc.c +++ b/stage0/stdlib/Lean/Meta/Tactic/Simp/Simproc.c @@ -22243,6 +22243,8 @@ lean_dec(x_3); lean_dec(x_1); x_45 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_46 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_45, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_47 = !lean_is_exclusive(x_46); if (x_47 == 0) { @@ -22279,6 +22281,8 @@ lean_dec(x_3); lean_dec(x_1); x_53 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_54 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_53, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_55 = !lean_is_exclusive(x_54); if (x_55 == 0) { @@ -22314,6 +22318,8 @@ lean_dec(x_3); lean_dec(x_1); x_61 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_62 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_61, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_63 = !lean_is_exclusive(x_62); if (x_63 == 0) { @@ -22353,6 +22359,8 @@ lean_dec(x_3); lean_dec(x_1); x_71 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_72 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_71, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_73 = !lean_is_exclusive(x_72); if (x_73 == 0) { @@ -22418,6 +22426,8 @@ lean_dec(x_3); lean_dec(x_1); x_89 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_90 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_89, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_91 = !lean_is_exclusive(x_90); if (x_91 == 0) { @@ -22451,6 +22461,8 @@ lean_dec(x_3); lean_dec(x_1); x_95 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_96 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_95, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_97 = !lean_is_exclusive(x_96); if (x_97 == 0) { @@ -22483,6 +22495,8 @@ lean_dec(x_3); lean_dec(x_1); x_101 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_102 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_101, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_103 = !lean_is_exclusive(x_102); if (x_103 == 0) { @@ -22514,6 +22528,8 @@ lean_dec(x_3); lean_dec(x_1); x_107 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_108 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_107, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_109 = !lean_is_exclusive(x_108); if (x_109 == 0) { @@ -22544,6 +22560,8 @@ lean_dec(x_3); lean_dec(x_1); x_113 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_114 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_113, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_115 = !lean_is_exclusive(x_114); if (x_115 == 0) { @@ -22574,6 +22592,8 @@ lean_dec(x_3); lean_dec(x_1); x_119 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___closed__6; x_120 = l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(x_119, x_29, x_14, x_4, x_5, x_32); +lean_dec(x_5); +lean_dec(x_4); x_121 = !lean_is_exclusive(x_120); if (x_121 == 0) { @@ -22599,6 +22619,8 @@ goto block_28; else { uint8_t x_125; +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_3); lean_dec(x_1); x_125 = !lean_is_exclusive(x_30); @@ -22689,8 +22711,6 @@ uint8_t x_11; lean_object* x_12; x_11 = lean_unbox(x_4); lean_dec(x_4); x_12 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin___lambda__1(x_1, x_2, x_3, x_11, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_9); -lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); return x_12; @@ -22701,8 +22721,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_ { lean_object* x_7; x_7 = l___private_Lean_Meta_Tactic_Simp_Simproc_0__Lean_Meta_Simp_addBuiltin(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); return x_7; } @@ -22994,8 +23012,6 @@ uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); x_8 = l_Lean_Meta_Simp_initFn____x40_Lean_Meta_Tactic_Simp_Simproc___hyg_6626____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); return x_8; } @@ -23164,8 +23180,6 @@ uint8_t x_7; lean_object* x_8; x_7 = lean_unbox(x_3); lean_dec(x_3); x_8 = l_Lean_Meta_Simp_initFn____x40_Lean_Meta_Tactic_Simp_Simproc___hyg_6701____lambda__1(x_1, x_2, x_7, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_2); return x_8; } diff --git a/stage0/stdlib/Lean/Parser/Extension.c b/stage0/stdlib/Lean/Parser/Extension.c index 231af616156f..9d86a245390d 100644 --- a/stage0/stdlib/Lean/Parser/Extension.c +++ b/stage0/stdlib/Lean/Parser/Extension.c @@ -371,7 +371,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_Parser LEAN_EXPORT lean_object* l___auto____x40_Lean_Parser_Extension___hyg_5878_; static lean_object* l_Lean_Parser_categoryParserFnImpl___closed__6; static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_5925____closed__2; -LEAN_EXPORT lean_object* l_Lean_Parser_declareLeadingBuiltinParser___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_ParserState_mkError(lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_86____closed__10; LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_ParserExtension_OLeanEntry_toEntry(lean_object*, lean_object*, lean_object*, lean_object*); @@ -495,7 +494,6 @@ LEAN_EXPORT lean_object* l_Lean_Parser_instCoeParserParserAliasValue(lean_object static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3784____closed__11; static lean_object* l_Lean_Parser_ParserExtension_addEntryImpl___closed__4; LEAN_EXPORT lean_object* l_Lean_Parser_addBuiltinLeadingParser(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_declareTrailingBuiltinParser___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Parser_instCoeForallParserParserAliasValue(lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_4079____closed__5; LEAN_EXPORT lean_object* l_Lean_Parser_registerParserCategory___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -666,7 +664,6 @@ static lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_throwParser static lean_object* l_Lean_Parser_parserOfStackFn___closed__2; size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_List_foldl___at___private_Lean_Parser_Extension_0__Lean_Parser_withNamespaces___spec__1(uint8_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_Parser_declareBuiltinParser___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Parser_initFn____x40_Lean_Parser_Extension___hyg_3784____closed__17; static lean_object* l_Lean_Parser_categoryParserFnImpl___closed__5; LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_BuiltinParserAttribute_add___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -10845,16 +10842,6 @@ x_20 = l_Lean_declareBuiltin(x_3, x_19, x_5, x_6, x_7); return x_20; } } -LEAN_EXPORT lean_object* l_Lean_Parser_declareBuiltinParser___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { -_start: -{ -lean_object* x_8; -x_8 = l_Lean_Parser_declareBuiltinParser(x_1, x_2, x_3, x_4, x_5, x_6, x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_8; -} -} static lean_object* _init_l_Lean_Parser_declareLeadingBuiltinParser___closed__1() { _start: { @@ -10883,16 +10870,6 @@ x_8 = l_Lean_Parser_declareBuiltinParser(x_7, x_1, x_2, x_3, x_4, x_5, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Parser_declareLeadingBuiltinParser___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Parser_declareLeadingBuiltinParser(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_7; -} -} static lean_object* _init_l_Lean_Parser_declareTrailingBuiltinParser___closed__1() { _start: { @@ -10921,16 +10898,6 @@ x_8 = l_Lean_Parser_declareBuiltinParser(x_7, x_1, x_2, x_3, x_4, x_5, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Lean_Parser_declareTrailingBuiltinParser___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; -x_7 = l_Lean_Parser_declareTrailingBuiltinParser(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_7; -} -} static lean_object* _init_l_Lean_Parser_getParserPriority___closed__1() { _start: { @@ -11051,6 +11018,8 @@ LEAN_EXPORT lean_object* l___private_Lean_Parser_Extension_0__Lean_Parser_Builti _start: { lean_object* x_7; +lean_inc(x_5); +lean_inc(x_4); lean_inc(x_1); x_7 = l_Lean_declareBuiltinDocStringAndRanges(x_1, x_4, x_5, x_6); if (lean_obj_tag(x_7) == 0) @@ -11299,6 +11268,8 @@ return x_55; else { lean_object* x_56; +lean_inc(x_6); +lean_inc(x_5); lean_inc(x_1); lean_inc(x_2); x_56 = l_Lean_Parser_declareLeadingBuiltinParser(x_2, x_1, x_3, x_5, x_6, x_10); @@ -11346,6 +11317,8 @@ else { lean_object* x_64; lean_dec(x_16); +lean_inc(x_6); +lean_inc(x_5); lean_inc(x_1); lean_inc(x_2); x_64 = l_Lean_Parser_declareTrailingBuiltinParser(x_2, x_1, x_3, x_5, x_6, x_10); diff --git a/stage0/stdlib/Lean/ParserCompiler.c b/stage0/stdlib/Lean/ParserCompiler.c index 310dfa5a8fe8..35f7b6a851a9 100644 --- a/stage0/stdlib/Lean/ParserCompiler.c +++ b/stage0/stdlib/Lean/ParserCompiler.c @@ -13,325 +13,310 @@ #ifdef __cplusplus extern "C" { #endif -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16(lean_object*); +static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_const___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4(lean_object*); static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__1___rarg___closed__2; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10(lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_Meta_mkConstWithFreshMVarLevels___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__12; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__15; LEAN_EXPORT lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__1; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36(lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__8; lean_object* l_Lean_ConstantInfo_type(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28(lean_object*); -lean_object* l_Lean_MessageData_toString(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Exception_isInterrupt(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38(lean_object*); uint64_t lean_uint64_lor(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isAppOfArity(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isOptParam(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_sort___override(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_Context_tyName___rarg___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); uint8_t l_Lean_Name_isAnonymous(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Meta_ReduceEval_0__Lean_Meta_evalName(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Parser_registerParserAttributeHook(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45(lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__7; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Attribute_add(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_stringToMessageData(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed(lean_object**); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileEmbeddedParsers___rarg(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__1; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_value_x21(lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Expr_appArg_x21(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_value_x3f(lean_object*, uint8_t); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__10; static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6; LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__5; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileEmbeddedParsers___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__1; lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalContext_getFVar_x21(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); -static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33(lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_throwError___at_Lean_Expr_abstractRangeM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_replace_expr(lean_object*, lean_object*); +lean_object* lean_st_ref_take(lean_object*, lean_object*); lean_object* l_Lean_Expr_getRevArg_x21(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__8; static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7; static uint64_t l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__4; lean_object* l_Lean_Meta_lambdaLetTelescope___at___private_Lean_Meta_InferType_0__Lean_Meta_inferLambdaType___spec__1___rarg(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__5; -lean_object* l_Lean_MessageData_ofFormat(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___boxed(lean_object**); lean_object* l_Lean_Expr_forallE___override(lean_object*, lean_object*, lean_object*, uint8_t); lean_object* l_outOfBounds___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__13; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_st_mk_ref(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_append(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_registerParserCompiler(lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12; extern lean_object* l_Lean_levelZero; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_instInhabitedExpr; static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__5; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_Context_tyName___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20(lean_object*); static uint64_t l_Lean_Meta_reduceEval___at_Lean_ParserCompiler_parserNodeKind_x3f___spec__2___closed__1; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__9; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__2; LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__6; lean_object* l_Lean_Expr_appFn_x21(lean_object*); lean_object* lean_mk_syntax_ident(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ParserCompiler_CombinatorAttribute_getDeclFor_x3f(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7(lean_object*); lean_object* l_Lean_MessageData_ofExpr(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48(lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed(lean_object**); lean_object* l_Lean_Meta_whnfEasyCases___at_Lean_Meta_whnfCore_go___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed(lean_object**); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22(lean_object*); lean_object* l_Lean_evalConstCheck___at_Lean_KeyedDeclsAttribute_init___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed(lean_object**); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__2___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__1___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* l_Lean_Environment_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed(lean_object**); lean_object* l_Lean_Expr_app___override(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_Context_tyName(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49(lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__4; lean_object* l_Lean_Name_mkStr2(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed(lean_object**); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_getConstInfo___at_Lean_registerInitAttrUnsafe___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__7; +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Meta_unfoldDefinition_x3f(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed(lean_object**); uint8_t l_Lean_Expr_isConstOf(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___closed__1; -lean_object* l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_LocalDecl_type(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__2(lean_object*); @@ -340,122 +325,113 @@ static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda lean_object* l_Lean_Expr_getAppFn(lean_object*); LEAN_EXPORT lean_object* l_List_filterTR_loop___at_Lean_ParserCompiler_parserNodeKind_x3f___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__1(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_left(uint64_t, uint64_t); static lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__1___rarg___closed__1; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51(lean_object*); lean_object* l_Lean_Environment_getModuleIdxFor_x3f(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6(lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_reverse___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42(lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14; uint8_t l_Lean_Meta_TransparencyMode_lt(uint8_t, uint8_t); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17(lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__1; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed(lean_object**); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___rarg___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_replaceParserTy(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__11; static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__14; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); -static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16; -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33(lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10(lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__3; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileEmbeddedParsers(lean_object*); -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32(lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__2; lean_object* lean_infer_type(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__8; lean_object* l_Lean_Meta_mkLambdaFVars(lean_object*, lean_object*, uint8_t, uint8_t, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29(lean_object*); uint64_t l_Lean_Meta_TransparencyMode_toUInt64(uint8_t); +lean_object* l_Lean_addAndCompile(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27(lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Expr_isConst(lean_object*); uint8_t l_Lean_Exception_isRuntime(lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__6; static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__16; static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__9; +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_List_enumFrom___rarg(lean_object*, lean_object*); -lean_object* l_Lean_KernelException_toMessageData(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t l___private_Lean_Meta_Basic_0__Lean_Meta_Config_toKey(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26(lean_object*); static lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__3___at_Lean_ParserCompiler_compileParserExpr___spec__4___rarg___closed__1; static lean_object* l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__2; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MessageData_ofName(lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed(lean_object**); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30(lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_parserNodeKind_x3f___closed__2; static lean_object* l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__3; -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___closed__4; -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed(lean_object**); lean_object* l_Lean_throwError___at___private_Lean_Meta_InferType_0__Lean_Meta_inferProjType___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33(lean_object*, lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(lean_object*, uint8_t, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_ParserCompiler_Context_tyName___rarg(lean_object* x_1) { _start: { @@ -3322,45 +3298,7 @@ x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserComp return x_2; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { -_start: -{ -lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_7 = lean_ctor_get(x_4, 5); -x_8 = l_Lean_addMessageContextFull___at_Lean_Meta_instAddMessageContextMetaM___spec__1(x_1, x_2, x_3, x_4, x_5, x_6); -x_9 = !lean_is_exclusive(x_8); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; -x_10 = lean_ctor_get(x_8, 0); -lean_inc(x_7); -x_11 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_11, 0, x_7); -lean_ctor_set(x_11, 1, x_10); -lean_ctor_set_tag(x_8, 1); -lean_ctor_set(x_8, 0, x_11); -return x_8; -} -else -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_ctor_get(x_8, 0); -x_13 = lean_ctor_get(x_8, 1); -lean_inc(x_13); -lean_inc(x_12); -lean_dec(x_8); -lean_inc(x_7); -x_14 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_14, 0, x_7); -lean_ctor_set(x_14, 1, x_12); -x_15 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_13); -return x_15; -} -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -3923,15 +3861,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -4010,15 +3948,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -4097,15 +4035,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -4680,15 +4618,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -5251,15 +5189,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -5822,15 +5760,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -5909,15 +5847,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -5996,15 +5934,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -6579,15 +6517,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -7150,15 +7088,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -7721,15 +7659,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -7808,15 +7746,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -7895,15 +7833,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -8478,15 +8416,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -9049,15 +8987,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -9620,15 +9558,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -9707,15 +9645,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -9794,15 +9732,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -10377,15 +10315,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -10948,15 +10886,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -11519,15 +11457,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -11606,15 +11544,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -11693,15 +11631,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -12276,15 +12214,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -12847,15 +12785,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -13418,15 +13356,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -13505,15 +13443,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -13592,15 +13530,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -14175,15 +14113,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -14746,15 +14684,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -15317,15 +15255,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -15404,15 +15342,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -15491,15 +15429,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -16074,15 +16012,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -16645,15 +16583,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -17216,15 +17154,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -17303,15 +17241,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -17390,15 +17328,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -17973,15 +17911,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -18544,15 +18482,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -19115,15 +19053,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -19202,15 +19140,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(lean_object* x_1, lean_object* x_2, size_t x_3, size_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -19289,15 +19227,15 @@ return x_27; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed), 10, 0); +x_2 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg___boxed), 10, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16, lean_object* x_17) { _start: { lean_object* x_18; uint8_t x_19; @@ -19872,15 +19810,15 @@ return x_114; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed), 17, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed), 17, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -20443,15 +20381,15 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed), 16, 0); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; uint8_t x_18; @@ -21014,11 +20952,11 @@ return x_115; } } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg___boxed), 16, 0); +x_2 = lean_alloc_closure((void*)(l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed), 16, 0); return x_2; } } @@ -21251,544 +21189,93 @@ static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambd _start: { lean_object* x_1; -x_1 = lean_mk_string_unchecked("Attr", 4, 4); +x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); return x_1; } } static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("simple", 6, 6); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__1; +x_2 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; } } static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__1; -x_2 = l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__2; -x_3 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__1; -x_4 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; +x_2 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +return x_2; } } static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4() { _start: { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("null", 4, 4); -return x_1; +lean_object* x_1; lean_object* x_2; +x_1 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; +x_2 = lean_alloc_ctor(0, 6, 0); +lean_ctor_set(x_2, 0, x_1); +lean_ctor_set(x_2, 1, x_1); +lean_ctor_set(x_2, 2, x_1); +lean_ctor_set(x_2, 3, x_1); +lean_ctor_set(x_2, 4, x_1); +lean_ctor_set(x_2, 5, x_1); +return x_2; } } static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Attr", 4, 4); +return x_1; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6() { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) -{ -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; -} -else -{ -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; -} -else -{ -uint8_t x_53; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) -{ -return x_49; -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; -} -} -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; -} -else -{ -uint8_t x_70; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) -{ -return x_66; -} -else -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; -} -} -} -} -} -else -{ -uint8_t x_74; -lean_free_object(x_18); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) -{ -return x_27; -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; -} -} -} -} -else -{ -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) -{ -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_1; +x_1 = lean_mk_string_unchecked("simple", 6, 6); +return x_1; } -else -{ -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) -{ -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) -{ -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; } -else -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) -{ -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; -} -else +static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7() { +_start: { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; -} else { - lean_dec_ref(x_107); - x_113 = lean_box(0); -} -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); -} else { - x_114 = x_113; -} -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__1; +x_2 = l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__2; +x_3 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; +x_4 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; } -else -{ -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; } -else +static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8() { +_start: { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; -} else { - lean_dec_ref(x_124); - x_130 = lean_box(0); -} -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); -} else { - x_131 = x_130; -} -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; -} -} +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; } } -else +static lean_object* _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9() { +_start: { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; -} else { - lean_dec_ref(x_84); - x_134 = lean_box(0); -} -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); -} else { - x_135 = x_134; -} -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; -} -} -} +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { lean_object* x_17; lean_object* x_18; @@ -21820,7 +21307,7 @@ lean_inc(x_5); x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); if (lean_obj_tag(x_23) == 0) { -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; x_24 = lean_ctor_get(x_23, 0); lean_inc(x_24); x_25 = lean_ctor_get(x_23, 1); @@ -21846,122 +21333,1181 @@ lean_ctor_set(x_31, 3, x_28); lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); x_32 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; +} +else +{ +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) +{ +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; +} +else +{ +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; +} +else { -uint8_t x_39; +uint8_t x_94; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) +{ +return x_90; +} +else +{ +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; +} +} +} +else +{ +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) +{ +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; +} +else +{ +uint8_t x_110; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) +{ +return x_106; +} +else +{ +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; +} +} +} +} +} +else +{ +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) +{ +return x_70; +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; +} +} +} +} +else +{ +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); lean_dec(x_5); +if (x_119 == 0) +{ +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; +} +else +{ +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) +{ +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; +} else { + lean_dec_ref(x_144); + x_150 = lean_box(0); +} +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); +} else { + x_151 = x_150; +} +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; +} +else +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; +} else { + lean_dec_ref(x_160); + x_166 = lean_box(0); +} +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); +} else { + x_167 = x_166; +} +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; +} +} +} +} +else { -return x_46; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; +} else { + lean_dec_ref(x_123); + x_170 = lean_box(0); +} +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); +} else { + x_171 = x_170; +} +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; +} +} +} } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) +{ +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_209); + x_215 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_216 = x_215; } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else +{ +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else +{ +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); lean_dec(x_5); -return x_64; +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; +} +else +{ +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} +} +} +} +else +{ +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} +} +} +else +{ +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -21973,29 +22519,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -22006,28 +22552,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -22062,7 +22608,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -22112,7 +22658,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -22146,7 +22692,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -22175,13 +22721,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -22216,7 +22762,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -22266,7 +22812,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -22287,7 +22833,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -22328,217 +22874,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) -{ -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; -} -else -{ -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) -{ -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) -{ -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; -} -else -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); +x_41 = lean_ctor_get(x_36, 2); lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); +x_42 = lean_ctor_get(x_36, 3); lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; +} +else +{ +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_13); +lean_inc(x_12); +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) +{ +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -uint8_t x_53; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) +{ +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) +{ +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; +} +else +{ +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -22546,458 +23217,863 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; +} else { + lean_dec_ref(x_209); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); +} else { + x_216 = x_215; +} +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; +} +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else { -uint8_t x_39; +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else { -return x_46; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); } +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_278); + x_284 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); -lean_dec(x_5); -return x_64; +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} } } else { -uint8_t x_65; -lean_dec(x_19); +uint8_t x_307; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -23008,29 +24084,30 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) { -return x_23; +return x_33; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; } } } else { -uint8_t x_69; +uint8_t x_311; +lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -23041,28 +24118,61 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { -return x_18; +return x_23; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); +lean_dec(x_23); +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } +else +{ +uint8_t x_315; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) +{ +return x_18; } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +else +{ +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_18); +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -23097,7 +24207,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -23147,7 +24257,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -23181,7 +24291,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -23210,13 +24320,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -23251,7 +24361,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -23301,7 +24411,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -23322,7 +24432,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -23363,217 +24473,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -23581,558 +24816,997 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); -lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); -lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -uint8_t x_39; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) { -return x_46; +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; -} +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_209); + x_215 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_216 = x_215; } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); -lean_dec(x_5); -return x_64; -} +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; } else { -uint8_t x_65; -lean_dec(x_19); +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) -{ -return x_23; +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; } -else -{ -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); -lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; } } } else { -uint8_t x_69; +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) -{ -return x_18; +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); } -else -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; } +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_13 = lean_unsigned_to_nat(0u); -x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; -lean_inc(x_14); -x_16 = lean_mk_array(x_14, x_15); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_14, x_17); -lean_dec(x_14); -x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_16, x_18); -x_32 = lean_array_get_size(x_6); -x_33 = lean_array_get_size(x_19); -x_34 = lean_nat_dec_le(x_32, x_33); -if (x_34 == 0) -{ -lean_dec(x_32); -x_20 = x_33; -goto block_31; } else { -lean_dec(x_33); -x_20 = x_32; -goto block_31; -} -block_31: -{ -lean_object* x_21; lean_object* x_22; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; +} +else +{ +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} +} +} +} +else +{ +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} +} +} +else +{ +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} +} +} +else +{ +uint8_t x_311; +lean_dec(x_19); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) +{ +return x_23; +} +else +{ +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); +lean_dec(x_23); +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; +} +} +} +else +{ +uint8_t x_315; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) +{ +return x_18; +} +else +{ +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); +lean_dec(x_18); +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +_start: +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; +x_13 = lean_unsigned_to_nat(0u); +x_14 = l___private_Lean_Expr_0__Lean_Expr_getAppNumArgsAux(x_1, x_13); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___closed__1; +lean_inc(x_14); +x_16 = lean_mk_array(x_14, x_15); +x_17 = lean_unsigned_to_nat(1u); +x_18 = lean_nat_sub(x_14, x_17); +lean_dec(x_14); +x_19 = l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(x_1, x_16, x_18); +x_32 = lean_array_get_size(x_6); +x_33 = lean_array_get_size(x_19); +x_34 = lean_nat_dec_le(x_32, x_33); +if (x_34 == 0) +{ +lean_dec(x_32); +x_20 = x_33; +goto block_31; +} +else +{ +lean_dec(x_33); +x_20 = x_32; +goto block_31; +} +block_31: +{ +lean_object* x_21; lean_object* x_22; x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -24182,7 +25856,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -24216,7 +25890,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -24245,13 +25919,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -24286,7 +25960,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -24336,7 +26010,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -24357,7 +26031,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -24398,217 +26072,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -24616,457 +26415,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; +} else { + lean_dec_ref(x_209); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); +} else { + x_216 = x_215; +} +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; +} +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else { -uint8_t x_39; +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else { -return x_46; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); } +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_278); + x_284 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} +} +} +else +{ +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -25078,29 +27316,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -25111,28 +27349,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -25167,7 +27405,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -25217,7 +27455,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -25251,7 +27489,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -25280,13 +27518,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -25321,7 +27559,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -25371,7 +27609,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -25392,7 +27630,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -25433,217 +27671,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -25651,457 +28014,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; +} else { + lean_dec_ref(x_209); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); +} else { + x_216 = x_215; +} +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; +} +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else { -uint8_t x_39; +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else { -return x_46; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); } +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_278); + x_284 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} +} +} +else +{ +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -26113,29 +28915,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -26146,28 +28948,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -26202,7 +29004,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -26252,7 +29054,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(lean_object* x_1, uint8_t x_2, uint8_t x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { lean_object* x_11; @@ -26307,7 +29109,7 @@ return x_21; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -26341,7 +29143,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -26370,13 +29172,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -26411,7 +29213,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -26461,7 +29263,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -26482,7 +29284,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -26523,217 +29325,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -26741,457 +29668,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; +} else { + lean_dec_ref(x_209); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); +} else { + x_216 = x_215; +} +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; +} +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) { -uint8_t x_39; +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else +{ +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else { -return x_46; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); } +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_278); + x_284 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; +} else { + lean_dec_ref(x_255); + x_305 = lean_box(0); +} +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); +} else { + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} +} +} +} +else +{ +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -27203,29 +30569,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -27236,28 +30602,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -27292,7 +30658,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -27342,7 +30708,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -27376,7 +30742,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -27405,13 +30771,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -27446,7 +30812,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -27496,7 +30862,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -27517,7 +30883,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__33___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -27558,217 +30924,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -27776,457 +31267,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_144); + x_150 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_151 = x_150; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_160); + x_166 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_167 = x_166; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_123); + x_170 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_171 = x_170; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; +} else { + lean_dec_ref(x_209); + x_215 = lean_box(0); +} +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); +} else { + x_216 = x_215; +} +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; +} +} +else +{ +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; +lean_inc(x_15); +lean_inc(x_14); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) { -uint8_t x_39; +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else +{ +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else { -return x_46; +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) +{ +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__34(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; +} +else +{ +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} +} } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_255); + x_305 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -28238,29 +32168,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -28271,28 +32201,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -28327,7 +32257,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -28377,7 +32307,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -28411,7 +32341,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -28440,13 +32370,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -28481,7 +32411,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -28531,7 +32461,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -28552,7 +32482,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -28593,217 +32523,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -28811,457 +32866,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; +} else { + lean_dec_ref(x_144); + x_150 = lean_box(0); +} +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); +} else { + x_151 = x_150; +} +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; +} +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; +} +else +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; +} else { + lean_dec_ref(x_160); + x_166 = lean_box(0); +} +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); +} else { + x_167 = x_166; +} +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; +} +} +} } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; +} else { + lean_dec_ref(x_123); + x_170 = lean_box(0); +} +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); +} else { + x_171 = x_170; +} +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; +} +} +} +} +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); +} +x_183 = l_Lean_Expr_isConst(x_5); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) +{ +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_209); + x_215 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_216 = x_215; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) +lean_inc(x_6); +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) +{ +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; +} +else +{ +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; +} else { + lean_dec_ref(x_225); + x_231 = lean_box(0); +} +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); +} else { + x_232 = x_231; +} +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; +} +} +} +} +else +{ +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; +} else { + lean_dec_ref(x_187); + x_235 = lean_box(0); +} +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); +} else { + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; +} +} +} +} +else +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; +} +else +{ +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) +{ +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) +{ +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else +{ +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_295); + x_301 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_302 = x_301; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_255); + x_305 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; -} -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; + x_306 = x_305; } +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); -lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); -lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +else { -uint8_t x_39; +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) -{ -return x_46; -} -else +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; -} +return x_33; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); -lean_dec(x_15); -lean_dec(x_14); -lean_dec(x_13); -lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; -} else { - lean_dec_ref(x_58); - x_61 = lean_box(0); -} -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); -} else { - x_62 = x_61; -} -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; -} +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; } -else -{ -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); -lean_dec(x_5); -return x_64; } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -29273,29 +33767,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -29306,28 +33800,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -29362,7 +33856,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -29412,7 +33906,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -29446,7 +33940,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -29475,13 +33969,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -29516,7 +34010,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -29566,7 +34060,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -29587,7 +34081,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -29628,217 +34122,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -29846,457 +34465,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) { -return x_27; +return x_70; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_119 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; +} else { + lean_dec_ref(x_144); + x_150 = lean_box(0); +} +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); +} else { + x_151 = x_150; +} +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; +} +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; +} +else +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; +} else { + lean_dec_ref(x_160); + x_166 = lean_box(0); +} +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); +} else { + x_167 = x_166; +} +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; +} +} +} } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; +} else { + lean_dec_ref(x_123); + x_170 = lean_box(0); +} +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); +} else { + x_171 = x_170; +} +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; +} +} +} +} +else +{ +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); +} +x_183 = l_Lean_Expr_isConst(x_5); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +if (x_183 == 0) +{ +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; +} +else +{ +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) +{ +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) +{ +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; +} +else +{ +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) +{ +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; +} +else +{ +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_209); + x_215 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_216 = x_215; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) +lean_inc(x_6); +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_225); + x_231 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_232 = x_231; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_187); + x_235 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_236 = x_235; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; } } } } +else +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); +} +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); -lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) { -uint8_t x_39; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) { -return x_46; +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} +} } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_255); + x_305 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -30308,29 +35366,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -30341,28 +35399,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -30397,7 +35455,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -30447,7 +35505,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; @@ -30481,7 +35539,7 @@ size_t x_17; size_t x_18; lean_object* x_19; x_17 = lean_usize_of_nat(x_12); lean_dec(x_12); x_18 = 0; -x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); +x_19 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(x_1, x_2, x_17, x_18, x_11, x_4, x_5, x_6, x_7, x_8); return x_19; } } @@ -30510,13 +35568,13 @@ size_t x_23; size_t x_24; lean_object* x_25; x_23 = lean_usize_of_nat(x_12); lean_dec(x_12); x_24 = 0; -x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); +x_25 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(x_1, x_2, x_23, x_24, x_11, x_4, x_5, x_6, x_7, x_8); return x_25; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -30551,7 +35609,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -30601,7 +35659,7 @@ return x_30; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, uint8_t x_5, uint8_t x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; @@ -30622,7 +35680,7 @@ lean_inc(x_16); lean_dec(x_14); x_17 = lean_box(x_5); x_18 = lean_box(x_6); -x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57___boxed), 12, 5); +x_19 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48___boxed), 12, 5); lean_closure_set(x_19, 0, x_3); lean_closure_set(x_19, 1, x_4); lean_closure_set(x_19, 2, x_17); @@ -30663,217 +35721,342 @@ return x_25; } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, uint8_t x_7, uint8_t x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -lean_inc(x_3); -x_17 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_1, x_11, x_2, x_3); -x_18 = l_Lean_setEnv___at_Lean_Meta_setInlineAttribute___spec__2(x_17, x_12, x_13, x_14, x_15, x_16); -x_19 = !lean_is_exclusive(x_18); -if (x_19 == 0) +lean_object* x_17; lean_object* x_18; +lean_inc(x_1); +x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_1); +x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); x_20 = lean_ctor_get(x_18, 1); -x_21 = lean_ctor_get(x_18, 0); -lean_dec(x_21); -x_22 = l_Lean_Expr_isConst(x_9); -if (x_22 == 0) +lean_inc(x_20); +lean_dec(x_18); +lean_inc(x_1); +x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47___boxed), 8, 1); +lean_closure_set(x_21, 0, x_1); +x_22 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +lean_inc(x_5); +x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); +if (lean_obj_tag(x_23) == 0) { -lean_object* x_23; lean_object* x_24; -lean_free_object(x_18); -x_23 = lean_box(0); -x_24 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_23, x_12, x_13, x_14, x_15, x_20); -return x_24; +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +lean_dec(x_23); +x_26 = lean_box(0); +lean_inc(x_6); +x_27 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_27, 0, x_6); +lean_ctor_set(x_27, 1, x_26); +lean_ctor_set(x_27, 2, x_24); +lean_inc(x_6); +x_28 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_28, 0, x_6); +lean_ctor_set(x_28, 1, x_26); +x_29 = lean_box(0); +x_30 = 1; +x_31 = lean_alloc_ctor(0, 4, 1); +lean_ctor_set(x_31, 0, x_27); +lean_ctor_set(x_31, 1, x_19); +lean_ctor_set(x_31, 2, x_29); +lean_ctor_set(x_31, 3, x_28); +lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); +x_32 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_32, 0, x_31); +lean_inc(x_15); +lean_inc(x_14); +x_33 = l_Lean_addAndCompile(x_32, x_14, x_15, x_25); +if (lean_obj_tag(x_33) == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; +x_34 = lean_ctor_get(x_33, 1); +lean_inc(x_34); +lean_dec(x_33); +x_35 = lean_st_ref_take(x_15, x_34); +x_36 = lean_ctor_get(x_35, 0); +lean_inc(x_36); +x_37 = lean_ctor_get(x_35, 1); +lean_inc(x_37); +lean_dec(x_35); +x_38 = lean_ctor_get(x_36, 0); +lean_inc(x_38); +lean_inc(x_6); +x_39 = l_Lean_ParserCompiler_CombinatorAttribute_setDeclFor(x_7, x_38, x_8, x_6); +x_40 = lean_ctor_get(x_36, 1); +lean_inc(x_40); +x_41 = lean_ctor_get(x_36, 2); +lean_inc(x_41); +x_42 = lean_ctor_get(x_36, 3); +lean_inc(x_42); +x_43 = lean_ctor_get(x_36, 5); +lean_inc(x_43); +x_44 = lean_ctor_get(x_36, 6); +lean_inc(x_44); +x_45 = lean_ctor_get(x_36, 7); +lean_inc(x_45); +lean_dec(x_36); +x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; +x_47 = lean_alloc_ctor(0, 8, 0); +lean_ctor_set(x_47, 0, x_39); +lean_ctor_set(x_47, 1, x_40); +lean_ctor_set(x_47, 2, x_41); +lean_ctor_set(x_47, 3, x_42); +lean_ctor_set(x_47, 4, x_46); +lean_ctor_set(x_47, 5, x_43); +lean_ctor_set(x_47, 6, x_44); +lean_ctor_set(x_47, 7, x_45); +x_48 = lean_st_ref_set(x_15, x_47, x_37); +x_49 = !lean_is_exclusive(x_48); +if (x_49 == 0) +{ +lean_object* x_50; lean_object* x_51; lean_object* x_52; uint8_t x_53; +x_50 = lean_ctor_get(x_48, 1); +x_51 = lean_ctor_get(x_48, 0); +lean_dec(x_51); +x_52 = lean_st_ref_take(x_13, x_50); +x_53 = !lean_is_exclusive(x_52); +if (x_53 == 0) +{ +lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_54 = lean_ctor_get(x_52, 0); +x_55 = lean_ctor_get(x_52, 1); +x_56 = lean_ctor_get(x_54, 0); +lean_inc(x_56); +x_57 = lean_ctor_get(x_54, 2); +lean_inc(x_57); +x_58 = lean_ctor_get(x_54, 3); +lean_inc(x_58); +x_59 = lean_ctor_get(x_54, 4); +lean_inc(x_59); +lean_dec(x_54); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_61 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_61, 0, x_56); +lean_ctor_set(x_61, 1, x_60); +lean_ctor_set(x_61, 2, x_57); +lean_ctor_set(x_61, 3, x_58); +lean_ctor_set(x_61, 4, x_59); +x_62 = lean_st_ref_set(x_13, x_61, x_55); +x_63 = !lean_is_exclusive(x_62); +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; uint8_t x_66; +x_64 = lean_ctor_get(x_62, 1); +x_65 = lean_ctor_get(x_62, 0); +lean_dec(x_65); +x_66 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_66 == 0) +{ +lean_object* x_67; lean_object* x_68; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_67 = lean_box(0); +x_68 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_67, x_12, x_13, x_14, x_15, x_64); +return x_68; } else { -uint8_t x_25; lean_object* x_26; lean_object* x_27; -x_25 = 0; -x_26 = l_Lean_ConstantInfo_value_x21(x_10, x_25); +lean_object* x_69; lean_object* x_70; +x_69 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_27 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_26, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_27) == 0) +x_70 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_69, x_12, x_13, x_14, x_15, x_64); +if (lean_obj_tag(x_70) == 0) { -lean_object* x_28; -x_28 = lean_ctor_get(x_27, 0); -lean_inc(x_28); -if (lean_obj_tag(x_28) == 0) +lean_object* x_71; +x_71 = lean_ctor_get(x_70, 0); +lean_inc(x_71); +if (lean_obj_tag(x_71) == 0) { -lean_object* x_29; lean_object* x_30; lean_object* x_31; -lean_free_object(x_18); -x_29 = lean_ctor_get(x_27, 1); -lean_inc(x_29); -lean_dec(x_27); -x_30 = lean_box(0); -x_31 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_30, x_12, x_13, x_14, x_15, x_29); -return x_31; +lean_object* x_72; lean_object* x_73; lean_object* x_74; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); +x_72 = lean_ctor_get(x_70, 1); +lean_inc(x_72); +lean_dec(x_70); +x_73 = lean_box(0); +x_74 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_73, x_12, x_13, x_14, x_15, x_72); +return x_74; } else { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_32 = lean_ctor_get(x_27, 1); -lean_inc(x_32); -lean_dec(x_27); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -lean_dec(x_28); -x_34 = lean_mk_syntax_ident(x_33); -lean_inc(x_4); -lean_ctor_set_tag(x_18, 1); -lean_ctor_set(x_18, 1, x_4); -lean_ctor_set(x_18, 0, x_34); -x_35 = lean_array_mk(x_18); -x_36 = lean_box(2); -x_37 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_36); -lean_ctor_set(x_38, 1, x_37); -lean_ctor_set(x_38, 2, x_35); -lean_inc(x_4); -x_39 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_39, 0, x_38); -lean_ctor_set(x_39, 1, x_4); -if (x_7 == 0) +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +x_75 = lean_ctor_get(x_70, 1); +lean_inc(x_75); +lean_dec(x_70); +x_76 = lean_ctor_get(x_71, 0); +lean_inc(x_76); +lean_dec(x_71); +x_77 = lean_mk_syntax_ident(x_76); +lean_ctor_set_tag(x_62, 1); +lean_ctor_set(x_62, 1, x_26); +lean_ctor_set(x_62, 0, x_77); +x_78 = lean_array_mk(x_62); +x_79 = lean_box(2); +x_80 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_79); +lean_ctor_set(x_81, 1, x_80); +lean_ctor_set(x_81, 2, x_78); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_81); +if (x_3 == 0) { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; lean_object* x_49; -x_40 = lean_ctor_get(x_6, 1); -lean_inc(x_40); -x_41 = lean_ctor_get(x_40, 0); -lean_inc(x_41); -lean_dec(x_40); -x_42 = lean_ctor_get(x_41, 1); -lean_inc(x_42); -lean_dec(x_41); -lean_inc(x_42); -x_43 = lean_mk_syntax_ident(x_42); -x_44 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_39); -x_45 = lean_array_mk(x_44); -x_46 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_47 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_47, 0, x_36); -lean_ctor_set(x_47, 1, x_46); -lean_ctor_set(x_47, 2, x_45); -x_48 = 0; +lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; uint8_t x_89; lean_object* x_90; +x_82 = lean_ctor_get(x_1, 1); +lean_inc(x_82); +x_83 = lean_ctor_get(x_82, 0); +lean_inc(x_83); +lean_dec(x_82); +x_84 = lean_ctor_get(x_83, 1); +lean_inc(x_84); +lean_dec(x_83); +lean_inc(x_84); +x_85 = lean_mk_syntax_ident(x_84); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_85); +x_86 = lean_array_mk(x_48); +x_87 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_88 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_88, 0, x_79); +lean_ctor_set(x_88, 1, x_87); +lean_ctor_set(x_88, 2, x_86); +x_89 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_49 = l_Lean_Attribute_add(x_3, x_42, x_47, x_48, x_14, x_15, x_32); -if (lean_obj_tag(x_49) == 0) +lean_inc(x_6); +x_90 = l_Lean_Attribute_add(x_6, x_84, x_88, x_89, x_14, x_15, x_75); +if (lean_obj_tag(x_90) == 0) { -lean_object* x_50; lean_object* x_51; lean_object* x_52; -x_50 = lean_ctor_get(x_49, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_49, 1); -lean_inc(x_51); -lean_dec(x_49); -x_52 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_50, x_12, x_13, x_14, x_15, x_51); -lean_dec(x_50); -return x_52; +lean_object* x_91; lean_object* x_92; lean_object* x_93; +x_91 = lean_ctor_get(x_90, 0); +lean_inc(x_91); +x_92 = lean_ctor_get(x_90, 1); +lean_inc(x_92); +lean_dec(x_90); +x_93 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_91, x_12, x_13, x_14, x_15, x_92); +lean_dec(x_91); +return x_93; } else { -uint8_t x_53; +uint8_t x_94; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_53 = !lean_is_exclusive(x_49); -if (x_53 == 0) +lean_dec(x_1); +x_94 = !lean_is_exclusive(x_90); +if (x_94 == 0) { -return x_49; +return x_90; } else { -lean_object* x_54; lean_object* x_55; lean_object* x_56; -x_54 = lean_ctor_get(x_49, 0); -x_55 = lean_ctor_get(x_49, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_49); -x_56 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_56, 0, x_54); -lean_ctor_set(x_56, 1, x_55); -return x_56; +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_ctor_get(x_90, 0); +x_96 = lean_ctor_get(x_90, 1); +lean_inc(x_96); +lean_inc(x_95); +lean_dec(x_90); +x_97 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_97, 0, x_95); +lean_ctor_set(x_97, 1, x_96); +return x_97; } } } else { -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint8_t x_65; lean_object* x_66; -x_57 = lean_ctor_get(x_6, 1); -lean_inc(x_57); -x_58 = lean_ctor_get(x_57, 0); -lean_inc(x_58); -lean_dec(x_57); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -lean_dec(x_58); -lean_inc(x_59); -x_60 = lean_mk_syntax_ident(x_59); -x_61 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_61, 0, x_60); -lean_ctor_set(x_61, 1, x_39); -x_62 = lean_array_mk(x_61); -x_63 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_36); -lean_ctor_set(x_64, 1, x_63); -lean_ctor_set(x_64, 2, x_62); -x_65 = 0; +lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; lean_object* x_106; +x_98 = lean_ctor_get(x_1, 1); +lean_inc(x_98); +x_99 = lean_ctor_get(x_98, 0); +lean_inc(x_99); +lean_dec(x_98); +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +lean_dec(x_99); +lean_inc(x_100); +x_101 = lean_mk_syntax_ident(x_100); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_101); +x_102 = lean_array_mk(x_48); +x_103 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_104 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_104, 0, x_79); +lean_ctor_set(x_104, 1, x_103); +lean_ctor_set(x_104, 2, x_102); +x_105 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_66 = l_Lean_Attribute_add(x_3, x_59, x_64, x_65, x_14, x_15, x_32); -if (lean_obj_tag(x_66) == 0) +lean_inc(x_6); +x_106 = l_Lean_Attribute_add(x_6, x_100, x_104, x_105, x_14, x_15, x_75); +if (lean_obj_tag(x_106) == 0) { -lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_67 = lean_ctor_get(x_66, 0); -lean_inc(x_67); -x_68 = lean_ctor_get(x_66, 1); -lean_inc(x_68); -lean_dec(x_66); -x_69 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_67, x_12, x_13, x_14, x_15, x_68); -lean_dec(x_67); -return x_69; +lean_object* x_107; lean_object* x_108; lean_object* x_109; +x_107 = lean_ctor_get(x_106, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_106, 1); +lean_inc(x_108); +lean_dec(x_106); +x_109 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_107, x_12, x_13, x_14, x_15, x_108); +lean_dec(x_107); +return x_109; } else { -uint8_t x_70; +uint8_t x_110; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_70 = !lean_is_exclusive(x_66); -if (x_70 == 0) +lean_dec(x_1); +x_110 = !lean_is_exclusive(x_106); +if (x_110 == 0) { -return x_66; +return x_106; } else { -lean_object* x_71; lean_object* x_72; lean_object* x_73; -x_71 = lean_ctor_get(x_66, 0); -x_72 = lean_ctor_get(x_66, 1); -lean_inc(x_72); -lean_inc(x_71); -lean_dec(x_66); -x_73 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_73, 0, x_71); -lean_ctor_set(x_73, 1, x_72); -return x_73; +lean_object* x_111; lean_object* x_112; lean_object* x_113; +x_111 = lean_ctor_get(x_106, 0); +x_112 = lean_ctor_get(x_106, 1); +lean_inc(x_112); +lean_inc(x_111); +lean_dec(x_106); +x_113 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_113, 0, x_111); +lean_ctor_set(x_113, 1, x_112); +return x_113; } } } @@ -30881,457 +36064,896 @@ return x_73; } else { -uint8_t x_74; -lean_free_object(x_18); +uint8_t x_114; +lean_free_object(x_62); +lean_free_object(x_52); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); +lean_dec(x_1); +x_114 = !lean_is_exclusive(x_70); +if (x_114 == 0) +{ +return x_70; +} +else +{ +lean_object* x_115; lean_object* x_116; lean_object* x_117; +x_115 = lean_ctor_get(x_70, 0); +x_116 = lean_ctor_get(x_70, 1); +lean_inc(x_116); +lean_inc(x_115); +lean_dec(x_70); +x_117 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_117, 0, x_115); +lean_ctor_set(x_117, 1, x_116); +return x_117; +} +} +} +} +else +{ +lean_object* x_118; uint8_t x_119; +x_118 = lean_ctor_get(x_62, 1); +lean_inc(x_118); +lean_dec(x_62); +x_119 = l_Lean_Expr_isConst(x_5); lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_74 = !lean_is_exclusive(x_27); -if (x_74 == 0) +if (x_119 == 0) { -return x_27; +lean_object* x_120; lean_object* x_121; +lean_free_object(x_52); +lean_free_object(x_48); +x_120 = lean_box(0); +x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_120, x_12, x_13, x_14, x_15, x_118); +return x_121; } else { -lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_75 = lean_ctor_get(x_27, 0); -x_76 = lean_ctor_get(x_27, 1); -lean_inc(x_76); -lean_inc(x_75); -lean_dec(x_27); -x_77 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_77, 0, x_75); -lean_ctor_set(x_77, 1, x_76); -return x_77; +lean_object* x_122; lean_object* x_123; +x_122 = l_Lean_ConstantInfo_value_x21(x_10, x_22); +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_13); +lean_inc(x_12); +x_123 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_122, x_12, x_13, x_14, x_15, x_118); +if (lean_obj_tag(x_123) == 0) +{ +lean_object* x_124; +x_124 = lean_ctor_get(x_123, 0); +lean_inc(x_124); +if (lean_obj_tag(x_124) == 0) +{ +lean_object* x_125; lean_object* x_126; lean_object* x_127; +lean_free_object(x_52); +lean_free_object(x_48); +x_125 = lean_ctor_get(x_123, 1); +lean_inc(x_125); +lean_dec(x_123); +x_126 = lean_box(0); +x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_126, x_12, x_13, x_14, x_15, x_125); +return x_127; +} +else +{ +lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +x_128 = lean_ctor_get(x_123, 1); +lean_inc(x_128); +lean_dec(x_123); +x_129 = lean_ctor_get(x_124, 0); +lean_inc(x_129); +lean_dec(x_124); +x_130 = lean_mk_syntax_ident(x_129); +x_131 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_131, 0, x_130); +lean_ctor_set(x_131, 1, x_26); +x_132 = lean_array_mk(x_131); +x_133 = lean_box(2); +x_134 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_135 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_135, 0, x_133); +lean_ctor_set(x_135, 1, x_134); +lean_ctor_set(x_135, 2, x_132); +lean_ctor_set_tag(x_52, 1); +lean_ctor_set(x_52, 1, x_26); +lean_ctor_set(x_52, 0, x_135); +if (x_3 == 0) +{ +lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; uint8_t x_143; lean_object* x_144; +x_136 = lean_ctor_get(x_1, 1); +lean_inc(x_136); +x_137 = lean_ctor_get(x_136, 0); +lean_inc(x_137); +lean_dec(x_136); +x_138 = lean_ctor_get(x_137, 1); +lean_inc(x_138); +lean_dec(x_137); +lean_inc(x_138); +x_139 = lean_mk_syntax_ident(x_138); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_139); +x_140 = lean_array_mk(x_48); +x_141 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_142 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_142, 0, x_133); +lean_ctor_set(x_142, 1, x_141); +lean_ctor_set(x_142, 2, x_140); +x_143 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_144 = l_Lean_Attribute_add(x_6, x_138, x_142, x_143, x_14, x_15, x_128); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; lean_object* x_146; lean_object* x_147; +x_145 = lean_ctor_get(x_144, 0); +lean_inc(x_145); +x_146 = lean_ctor_get(x_144, 1); +lean_inc(x_146); +lean_dec(x_144); +x_147 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_145, x_12, x_13, x_14, x_15, x_146); +lean_dec(x_145); +return x_147; +} +else +{ +lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_148 = lean_ctor_get(x_144, 0); +lean_inc(x_148); +x_149 = lean_ctor_get(x_144, 1); +lean_inc(x_149); +if (lean_is_exclusive(x_144)) { + lean_ctor_release(x_144, 0); + lean_ctor_release(x_144, 1); + x_150 = x_144; +} else { + lean_dec_ref(x_144); + x_150 = lean_box(0); +} +if (lean_is_scalar(x_150)) { + x_151 = lean_alloc_ctor(1, 2, 0); +} else { + x_151 = x_150; +} +lean_ctor_set(x_151, 0, x_148); +lean_ctor_set(x_151, 1, x_149); +return x_151; +} +} +else +{ +lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; uint8_t x_159; lean_object* x_160; +x_152 = lean_ctor_get(x_1, 1); +lean_inc(x_152); +x_153 = lean_ctor_get(x_152, 0); +lean_inc(x_153); +lean_dec(x_152); +x_154 = lean_ctor_get(x_153, 0); +lean_inc(x_154); +lean_dec(x_153); +lean_inc(x_154); +x_155 = lean_mk_syntax_ident(x_154); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_52); +lean_ctor_set(x_48, 0, x_155); +x_156 = lean_array_mk(x_48); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_158 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_158, 0, x_133); +lean_ctor_set(x_158, 1, x_157); +lean_ctor_set(x_158, 2, x_156); +x_159 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_160 = l_Lean_Attribute_add(x_6, x_154, x_158, x_159, x_14, x_15, x_128); +if (lean_obj_tag(x_160) == 0) +{ +lean_object* x_161; lean_object* x_162; lean_object* x_163; +x_161 = lean_ctor_get(x_160, 0); +lean_inc(x_161); +x_162 = lean_ctor_get(x_160, 1); +lean_inc(x_162); +lean_dec(x_160); +x_163 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_161, x_12, x_13, x_14, x_15, x_162); +lean_dec(x_161); +return x_163; +} +else +{ +lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_164 = lean_ctor_get(x_160, 0); +lean_inc(x_164); +x_165 = lean_ctor_get(x_160, 1); +lean_inc(x_165); +if (lean_is_exclusive(x_160)) { + lean_ctor_release(x_160, 0); + lean_ctor_release(x_160, 1); + x_166 = x_160; +} else { + lean_dec_ref(x_160); + x_166 = lean_box(0); +} +if (lean_is_scalar(x_166)) { + x_167 = lean_alloc_ctor(1, 2, 0); +} else { + x_167 = x_166; +} +lean_ctor_set(x_167, 0, x_164); +lean_ctor_set(x_167, 1, x_165); +return x_167; +} +} +} +} +else +{ +lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; +lean_free_object(x_52); +lean_free_object(x_48); +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_168 = lean_ctor_get(x_123, 0); +lean_inc(x_168); +x_169 = lean_ctor_get(x_123, 1); +lean_inc(x_169); +if (lean_is_exclusive(x_123)) { + lean_ctor_release(x_123, 0); + lean_ctor_release(x_123, 1); + x_170 = x_123; +} else { + lean_dec_ref(x_123); + x_170 = lean_box(0); +} +if (lean_is_scalar(x_170)) { + x_171 = lean_alloc_ctor(1, 2, 0); +} else { + x_171 = x_170; +} +lean_ctor_set(x_171, 0, x_168); +lean_ctor_set(x_171, 1, x_169); +return x_171; } } } } else { -lean_object* x_78; uint8_t x_79; -x_78 = lean_ctor_get(x_18, 1); -lean_inc(x_78); -lean_dec(x_18); -x_79 = l_Lean_Expr_isConst(x_9); -if (x_79 == 0) +lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; uint8_t x_183; +x_172 = lean_ctor_get(x_52, 0); +x_173 = lean_ctor_get(x_52, 1); +lean_inc(x_173); +lean_inc(x_172); +lean_dec(x_52); +x_174 = lean_ctor_get(x_172, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_172, 2); +lean_inc(x_175); +x_176 = lean_ctor_get(x_172, 3); +lean_inc(x_176); +x_177 = lean_ctor_get(x_172, 4); +lean_inc(x_177); +lean_dec(x_172); +x_178 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_179 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_179, 0, x_174); +lean_ctor_set(x_179, 1, x_178); +lean_ctor_set(x_179, 2, x_175); +lean_ctor_set(x_179, 3, x_176); +lean_ctor_set(x_179, 4, x_177); +x_180 = lean_st_ref_set(x_13, x_179, x_173); +x_181 = lean_ctor_get(x_180, 1); +lean_inc(x_181); +if (lean_is_exclusive(x_180)) { + lean_ctor_release(x_180, 0); + lean_ctor_release(x_180, 1); + x_182 = x_180; +} else { + lean_dec_ref(x_180); + x_182 = lean_box(0); +} +x_183 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_183 == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = lean_box(0); -x_81 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_80, x_12, x_13, x_14, x_15, x_78); -return x_81; +lean_object* x_184; lean_object* x_185; +lean_dec(x_182); +lean_free_object(x_48); +x_184 = lean_box(0); +x_185 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_184, x_12, x_13, x_14, x_15, x_181); +return x_185; } else { -uint8_t x_82; lean_object* x_83; lean_object* x_84; -x_82 = 0; -x_83 = l_Lean_ConstantInfo_value_x21(x_10, x_82); +lean_object* x_186; lean_object* x_187; +x_186 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -x_84 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_83, x_12, x_13, x_14, x_15, x_78); -if (lean_obj_tag(x_84) == 0) +x_187 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_186, x_12, x_13, x_14, x_15, x_181); +if (lean_obj_tag(x_187) == 0) { -lean_object* x_85; -x_85 = lean_ctor_get(x_84, 0); -lean_inc(x_85); -if (lean_obj_tag(x_85) == 0) +lean_object* x_188; +x_188 = lean_ctor_get(x_187, 0); +lean_inc(x_188); +if (lean_obj_tag(x_188) == 0) { -lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_86 = lean_ctor_get(x_84, 1); -lean_inc(x_86); -lean_dec(x_84); -x_87 = lean_box(0); -x_88 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_87, x_12, x_13, x_14, x_15, x_86); -return x_88; +lean_object* x_189; lean_object* x_190; lean_object* x_191; +lean_dec(x_182); +lean_free_object(x_48); +x_189 = lean_ctor_get(x_187, 1); +lean_inc(x_189); +lean_dec(x_187); +x_190 = lean_box(0); +x_191 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_190, x_12, x_13, x_14, x_15, x_189); +return x_191; } else { -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; -x_89 = lean_ctor_get(x_84, 1); -lean_inc(x_89); -lean_dec(x_84); -x_90 = lean_ctor_get(x_85, 0); -lean_inc(x_90); -lean_dec(x_85); -x_91 = lean_mk_syntax_ident(x_90); -lean_inc(x_4); -x_92 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_92, 0, x_91); -lean_ctor_set(x_92, 1, x_4); -x_93 = lean_array_mk(x_92); -x_94 = lean_box(2); -x_95 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5; -x_96 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_96, 0, x_94); -lean_ctor_set(x_96, 1, x_95); -lean_ctor_set(x_96, 2, x_93); -lean_inc(x_4); -x_97 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_97, 0, x_96); -lean_ctor_set(x_97, 1, x_4); -if (x_7 == 0) +lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_192 = lean_ctor_get(x_187, 1); +lean_inc(x_192); +lean_dec(x_187); +x_193 = lean_ctor_get(x_188, 0); +lean_inc(x_193); +lean_dec(x_188); +x_194 = lean_mk_syntax_ident(x_193); +if (lean_is_scalar(x_182)) { + x_195 = lean_alloc_ctor(1, 2, 0); +} else { + x_195 = x_182; + lean_ctor_set_tag(x_195, 1); +} +lean_ctor_set(x_195, 0, x_194); +lean_ctor_set(x_195, 1, x_26); +x_196 = lean_array_mk(x_195); +x_197 = lean_box(2); +x_198 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_199 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_199, 0, x_197); +lean_ctor_set(x_199, 1, x_198); +lean_ctor_set(x_199, 2, x_196); +x_200 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_200, 0, x_199); +lean_ctor_set(x_200, 1, x_26); +if (x_3 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; lean_object* x_107; -x_98 = lean_ctor_get(x_6, 1); -lean_inc(x_98); -x_99 = lean_ctor_get(x_98, 0); -lean_inc(x_99); -lean_dec(x_98); -x_100 = lean_ctor_get(x_99, 1); -lean_inc(x_100); -lean_dec(x_99); -lean_inc(x_100); -x_101 = lean_mk_syntax_ident(x_100); -x_102 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_102, 0, x_101); -lean_ctor_set(x_102, 1, x_97); -x_103 = lean_array_mk(x_102); -x_104 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_105 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_105, 0, x_94); -lean_ctor_set(x_105, 1, x_104); -lean_ctor_set(x_105, 2, x_103); -x_106 = 0; +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; uint8_t x_208; lean_object* x_209; +x_201 = lean_ctor_get(x_1, 1); +lean_inc(x_201); +x_202 = lean_ctor_get(x_201, 0); +lean_inc(x_202); +lean_dec(x_201); +x_203 = lean_ctor_get(x_202, 1); +lean_inc(x_203); +lean_dec(x_202); +lean_inc(x_203); +x_204 = lean_mk_syntax_ident(x_203); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_204); +x_205 = lean_array_mk(x_48); +x_206 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_207 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_207, 0, x_197); +lean_ctor_set(x_207, 1, x_206); +lean_ctor_set(x_207, 2, x_205); +x_208 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_107 = l_Lean_Attribute_add(x_3, x_100, x_105, x_106, x_14, x_15, x_89); -if (lean_obj_tag(x_107) == 0) +lean_inc(x_6); +x_209 = l_Lean_Attribute_add(x_6, x_203, x_207, x_208, x_14, x_15, x_192); +if (lean_obj_tag(x_209) == 0) { -lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_108 = lean_ctor_get(x_107, 0); -lean_inc(x_108); -x_109 = lean_ctor_get(x_107, 1); -lean_inc(x_109); -lean_dec(x_107); -x_110 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_108, x_12, x_13, x_14, x_15, x_109); -lean_dec(x_108); -return x_110; +lean_object* x_210; lean_object* x_211; lean_object* x_212; +x_210 = lean_ctor_get(x_209, 0); +lean_inc(x_210); +x_211 = lean_ctor_get(x_209, 1); +lean_inc(x_211); +lean_dec(x_209); +x_212 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_210, x_12, x_13, x_14, x_15, x_211); +lean_dec(x_210); +return x_212; } else { -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; +lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_111 = lean_ctor_get(x_107, 0); -lean_inc(x_111); -x_112 = lean_ctor_get(x_107, 1); -lean_inc(x_112); -if (lean_is_exclusive(x_107)) { - lean_ctor_release(x_107, 0); - lean_ctor_release(x_107, 1); - x_113 = x_107; +lean_dec(x_1); +x_213 = lean_ctor_get(x_209, 0); +lean_inc(x_213); +x_214 = lean_ctor_get(x_209, 1); +lean_inc(x_214); +if (lean_is_exclusive(x_209)) { + lean_ctor_release(x_209, 0); + lean_ctor_release(x_209, 1); + x_215 = x_209; } else { - lean_dec_ref(x_107); - x_113 = lean_box(0); + lean_dec_ref(x_209); + x_215 = lean_box(0); } -if (lean_is_scalar(x_113)) { - x_114 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_215)) { + x_216 = lean_alloc_ctor(1, 2, 0); } else { - x_114 = x_113; + x_216 = x_215; } -lean_ctor_set(x_114, 0, x_111); -lean_ctor_set(x_114, 1, x_112); -return x_114; +lean_ctor_set(x_216, 0, x_213); +lean_ctor_set(x_216, 1, x_214); +return x_216; } } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint8_t x_123; lean_object* x_124; -x_115 = lean_ctor_get(x_6, 1); -lean_inc(x_115); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -lean_dec(x_115); -x_117 = lean_ctor_get(x_116, 0); -lean_inc(x_117); -lean_dec(x_116); -lean_inc(x_117); -x_118 = lean_mk_syntax_ident(x_117); -x_119 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_97); -x_120 = lean_array_mk(x_119); -x_121 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__3; -x_122 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_122, 0, x_94); -lean_ctor_set(x_122, 1, x_121); -lean_ctor_set(x_122, 2, x_120); -x_123 = 0; +lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; lean_object* x_222; lean_object* x_223; uint8_t x_224; lean_object* x_225; +x_217 = lean_ctor_get(x_1, 1); +lean_inc(x_217); +x_218 = lean_ctor_get(x_217, 0); +lean_inc(x_218); +lean_dec(x_217); +x_219 = lean_ctor_get(x_218, 0); +lean_inc(x_219); +lean_dec(x_218); +lean_inc(x_219); +x_220 = lean_mk_syntax_ident(x_219); +lean_ctor_set_tag(x_48, 1); +lean_ctor_set(x_48, 1, x_200); +lean_ctor_set(x_48, 0, x_220); +x_221 = lean_array_mk(x_48); +x_222 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_223 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_223, 0, x_197); +lean_ctor_set(x_223, 1, x_222); +lean_ctor_set(x_223, 2, x_221); +x_224 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_3); -x_124 = l_Lean_Attribute_add(x_3, x_117, x_122, x_123, x_14, x_15, x_89); -if (lean_obj_tag(x_124) == 0) +lean_inc(x_6); +x_225 = l_Lean_Attribute_add(x_6, x_219, x_223, x_224, x_14, x_15, x_192); +if (lean_obj_tag(x_225) == 0) { -lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_125 = lean_ctor_get(x_124, 0); -lean_inc(x_125); -x_126 = lean_ctor_get(x_124, 1); -lean_inc(x_126); -lean_dec(x_124); -x_127 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_3, x_4, x_5, x_6, x_7, x_8, x_125, x_12, x_13, x_14, x_15, x_126); -lean_dec(x_125); -return x_127; +lean_object* x_226; lean_object* x_227; lean_object* x_228; +x_226 = lean_ctor_get(x_225, 0); +lean_inc(x_226); +x_227 = lean_ctor_get(x_225, 1); +lean_inc(x_227); +lean_dec(x_225); +x_228 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_226, x_12, x_13, x_14, x_15, x_227); +lean_dec(x_226); +return x_228; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +lean_object* x_229; lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_128 = lean_ctor_get(x_124, 0); -lean_inc(x_128); -x_129 = lean_ctor_get(x_124, 1); -lean_inc(x_129); -if (lean_is_exclusive(x_124)) { - lean_ctor_release(x_124, 0); - lean_ctor_release(x_124, 1); - x_130 = x_124; +lean_dec(x_1); +x_229 = lean_ctor_get(x_225, 0); +lean_inc(x_229); +x_230 = lean_ctor_get(x_225, 1); +lean_inc(x_230); +if (lean_is_exclusive(x_225)) { + lean_ctor_release(x_225, 0); + lean_ctor_release(x_225, 1); + x_231 = x_225; } else { - lean_dec_ref(x_124); - x_130 = lean_box(0); + lean_dec_ref(x_225); + x_231 = lean_box(0); } -if (lean_is_scalar(x_130)) { - x_131 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_231)) { + x_232 = lean_alloc_ctor(1, 2, 0); } else { - x_131 = x_130; + x_232 = x_231; } -lean_ctor_set(x_131, 0, x_128); -lean_ctor_set(x_131, 1, x_129); -return x_131; +lean_ctor_set(x_232, 0, x_229); +lean_ctor_set(x_232, 1, x_230); +return x_232; } } } } else { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; +lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; +lean_dec(x_182); +lean_free_object(x_48); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); +lean_dec(x_9); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -lean_dec(x_3); -x_132 = lean_ctor_get(x_84, 0); -lean_inc(x_132); -x_133 = lean_ctor_get(x_84, 1); -lean_inc(x_133); -if (lean_is_exclusive(x_84)) { - lean_ctor_release(x_84, 0); - lean_ctor_release(x_84, 1); - x_134 = x_84; +lean_dec(x_1); +x_233 = lean_ctor_get(x_187, 0); +lean_inc(x_233); +x_234 = lean_ctor_get(x_187, 1); +lean_inc(x_234); +if (lean_is_exclusive(x_187)) { + lean_ctor_release(x_187, 0); + lean_ctor_release(x_187, 1); + x_235 = x_187; } else { - lean_dec_ref(x_84); - x_134 = lean_box(0); + lean_dec_ref(x_187); + x_235 = lean_box(0); } -if (lean_is_scalar(x_134)) { - x_135 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_235)) { + x_236 = lean_alloc_ctor(1, 2, 0); } else { - x_135 = x_134; + x_236 = x_235; +} +lean_ctor_set(x_236, 0, x_233); +lean_ctor_set(x_236, 1, x_234); +return x_236; } -lean_ctor_set(x_135, 0, x_132); -lean_ctor_set(x_135, 1, x_133); -return x_135; } } } +else +{ +lean_object* x_237; lean_object* x_238; lean_object* x_239; lean_object* x_240; lean_object* x_241; lean_object* x_242; lean_object* x_243; lean_object* x_244; lean_object* x_245; lean_object* x_246; lean_object* x_247; lean_object* x_248; lean_object* x_249; lean_object* x_250; uint8_t x_251; +x_237 = lean_ctor_get(x_48, 1); +lean_inc(x_237); +lean_dec(x_48); +x_238 = lean_st_ref_take(x_13, x_237); +x_239 = lean_ctor_get(x_238, 0); +lean_inc(x_239); +x_240 = lean_ctor_get(x_238, 1); +lean_inc(x_240); +if (lean_is_exclusive(x_238)) { + lean_ctor_release(x_238, 0); + lean_ctor_release(x_238, 1); + x_241 = x_238; +} else { + lean_dec_ref(x_238); + x_241 = lean_box(0); +} +x_242 = lean_ctor_get(x_239, 0); +lean_inc(x_242); +x_243 = lean_ctor_get(x_239, 2); +lean_inc(x_243); +x_244 = lean_ctor_get(x_239, 3); +lean_inc(x_244); +x_245 = lean_ctor_get(x_239, 4); +lean_inc(x_245); +lean_dec(x_239); +x_246 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_247 = lean_alloc_ctor(0, 5, 0); +lean_ctor_set(x_247, 0, x_242); +lean_ctor_set(x_247, 1, x_246); +lean_ctor_set(x_247, 2, x_243); +lean_ctor_set(x_247, 3, x_244); +lean_ctor_set(x_247, 4, x_245); +x_248 = lean_st_ref_set(x_13, x_247, x_240); +x_249 = lean_ctor_get(x_248, 1); +lean_inc(x_249); +if (lean_is_exclusive(x_248)) { + lean_ctor_release(x_248, 0); + lean_ctor_release(x_248, 1); + x_250 = x_248; +} else { + lean_dec_ref(x_248); + x_250 = lean_box(0); } +x_251 = l_Lean_Expr_isConst(x_5); +lean_dec(x_5); +if (x_251 == 0) +{ +lean_object* x_252; lean_object* x_253; +lean_dec(x_250); +lean_dec(x_241); +x_252 = lean_box(0); +x_253 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_252, x_12, x_13, x_14, x_15, x_249); +return x_253; } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: +else { -lean_object* x_17; lean_object* x_18; -lean_inc(x_1); -x_17 = l_Lean_ParserCompiler_replaceParserTy___rarg(x_1, x_2); +lean_object* x_254; lean_object* x_255; +x_254 = l_Lean_ConstantInfo_value_x21(x_10, x_22); lean_inc(x_15); lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); -lean_inc(x_1); -x_18 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_3, x_4, x_17, x_12, x_13, x_14, x_15, x_16); -if (lean_obj_tag(x_18) == 0) +x_255 = l_Lean_ParserCompiler_parserNodeKind_x3f(x_254, x_12, x_13, x_14, x_15, x_249); +if (lean_obj_tag(x_255) == 0) { -lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; lean_object* x_23; -x_19 = lean_ctor_get(x_18, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_18, 1); -lean_inc(x_20); -lean_dec(x_18); -lean_inc(x_1); -x_21 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56___boxed), 8, 1); -lean_closure_set(x_21, 0, x_1); -x_22 = 0; +lean_object* x_256; +x_256 = lean_ctor_get(x_255, 0); +lean_inc(x_256); +if (lean_obj_tag(x_256) == 0) +{ +lean_object* x_257; lean_object* x_258; lean_object* x_259; +lean_dec(x_250); +lean_dec(x_241); +x_257 = lean_ctor_get(x_255, 1); +lean_inc(x_257); +lean_dec(x_255); +x_258 = lean_box(0); +x_259 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_258, x_12, x_13, x_14, x_15, x_257); +return x_259; +} +else +{ +lean_object* x_260; lean_object* x_261; lean_object* x_262; lean_object* x_263; lean_object* x_264; lean_object* x_265; lean_object* x_266; lean_object* x_267; lean_object* x_268; +x_260 = lean_ctor_get(x_255, 1); +lean_inc(x_260); +lean_dec(x_255); +x_261 = lean_ctor_get(x_256, 0); +lean_inc(x_261); +lean_dec(x_256); +x_262 = lean_mk_syntax_ident(x_261); +if (lean_is_scalar(x_250)) { + x_263 = lean_alloc_ctor(1, 2, 0); +} else { + x_263 = x_250; + lean_ctor_set_tag(x_263, 1); +} +lean_ctor_set(x_263, 0, x_262); +lean_ctor_set(x_263, 1, x_26); +x_264 = lean_array_mk(x_263); +x_265 = lean_box(2); +x_266 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9; +x_267 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_267, 0, x_265); +lean_ctor_set(x_267, 1, x_266); +lean_ctor_set(x_267, 2, x_264); +if (lean_is_scalar(x_241)) { + x_268 = lean_alloc_ctor(1, 2, 0); +} else { + x_268 = x_241; + lean_ctor_set_tag(x_268, 1); +} +lean_ctor_set(x_268, 0, x_267); +lean_ctor_set(x_268, 1, x_26); +if (x_3 == 0) +{ +lean_object* x_269; lean_object* x_270; lean_object* x_271; lean_object* x_272; lean_object* x_273; lean_object* x_274; lean_object* x_275; lean_object* x_276; uint8_t x_277; lean_object* x_278; +x_269 = lean_ctor_get(x_1, 1); +lean_inc(x_269); +x_270 = lean_ctor_get(x_269, 0); +lean_inc(x_270); +lean_dec(x_269); +x_271 = lean_ctor_get(x_270, 1); +lean_inc(x_271); +lean_dec(x_270); +lean_inc(x_271); +x_272 = lean_mk_syntax_ident(x_271); +x_273 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_273, 0, x_272); +lean_ctor_set(x_273, 1, x_268); +x_274 = lean_array_mk(x_273); +x_275 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_276 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_276, 0, x_265); +lean_ctor_set(x_276, 1, x_275); +lean_ctor_set(x_276, 2, x_274); +x_277 = 0; lean_inc(x_15); lean_inc(x_14); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_5); -x_23 = l_Lean_Meta_forallTelescope___at_Lean_Meta_mapForallTelescope_x27___spec__1___rarg(x_5, x_21, x_22, x_12, x_13, x_14, x_15, x_20); -if (lean_obj_tag(x_23) == 0) -{ -lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; -x_24 = lean_ctor_get(x_23, 0); -lean_inc(x_24); -x_25 = lean_ctor_get(x_23, 1); -lean_inc(x_25); -lean_dec(x_23); -x_26 = lean_box(0); -lean_inc(x_6); -x_27 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_27, 0, x_6); -lean_ctor_set(x_27, 1, x_26); -lean_ctor_set(x_27, 2, x_24); lean_inc(x_6); -x_28 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_28, 0, x_6); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_box(0); -x_30 = 1; -x_31 = lean_alloc_ctor(0, 4, 1); -lean_ctor_set(x_31, 0, x_27); -lean_ctor_set(x_31, 1, x_19); -lean_ctor_set(x_31, 2, x_29); -lean_ctor_set(x_31, 3, x_28); -lean_ctor_set_uint8(x_31, sizeof(void*)*4, x_30); -x_32 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_32, 0, x_31); -x_33 = lean_st_ref_get(x_15, x_25); -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_ctor_get(x_34, 0); -lean_inc(x_36); -lean_dec(x_34); -x_37 = lean_box(0); -x_38 = l_Lean_Environment_addAndCompile(x_36, x_26, x_32, x_37); -if (lean_obj_tag(x_38) == 0) +x_278 = l_Lean_Attribute_add(x_6, x_271, x_276, x_277, x_14, x_15, x_260); +if (lean_obj_tag(x_278) == 0) { -uint8_t x_39; -lean_dec(x_9); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -x_39 = !lean_is_exclusive(x_38); -if (x_39 == 0) +lean_object* x_279; lean_object* x_280; lean_object* x_281; +x_279 = lean_ctor_get(x_278, 0); +lean_inc(x_279); +x_280 = lean_ctor_get(x_278, 1); +lean_inc(x_280); +lean_dec(x_278); +x_281 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_279, x_12, x_13, x_14, x_15, x_280); +lean_dec(x_279); +return x_281; +} +else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_38, 0); -x_41 = l_Lean_KernelException_toMessageData(x_40, x_26); -x_42 = l_Lean_MessageData_toString(x_41, x_35); -x_43 = lean_ctor_get(x_42, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_42, 1); -lean_inc(x_44); -lean_dec(x_42); -lean_ctor_set_tag(x_38, 3); -lean_ctor_set(x_38, 0, x_43); -x_45 = l_Lean_MessageData_ofFormat(x_38); -x_46 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_45, x_12, x_13, x_14, x_15, x_44); +lean_object* x_282; lean_object* x_283; lean_object* x_284; lean_object* x_285; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_47 = !lean_is_exclusive(x_46); -if (x_47 == 0) +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_282 = lean_ctor_get(x_278, 0); +lean_inc(x_282); +x_283 = lean_ctor_get(x_278, 1); +lean_inc(x_283); +if (lean_is_exclusive(x_278)) { + lean_ctor_release(x_278, 0); + lean_ctor_release(x_278, 1); + x_284 = x_278; +} else { + lean_dec_ref(x_278); + x_284 = lean_box(0); +} +if (lean_is_scalar(x_284)) { + x_285 = lean_alloc_ctor(1, 2, 0); +} else { + x_285 = x_284; +} +lean_ctor_set(x_285, 0, x_282); +lean_ctor_set(x_285, 1, x_283); +return x_285; +} +} +else +{ +lean_object* x_286; lean_object* x_287; lean_object* x_288; lean_object* x_289; lean_object* x_290; lean_object* x_291; lean_object* x_292; lean_object* x_293; uint8_t x_294; lean_object* x_295; +x_286 = lean_ctor_get(x_1, 1); +lean_inc(x_286); +x_287 = lean_ctor_get(x_286, 0); +lean_inc(x_287); +lean_dec(x_286); +x_288 = lean_ctor_get(x_287, 0); +lean_inc(x_288); +lean_dec(x_287); +lean_inc(x_288); +x_289 = lean_mk_syntax_ident(x_288); +x_290 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_290, 0, x_289); +lean_ctor_set(x_290, 1, x_268); +x_291 = lean_array_mk(x_290); +x_292 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7; +x_293 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_293, 0, x_265); +lean_ctor_set(x_293, 1, x_292); +lean_ctor_set(x_293, 2, x_291); +x_294 = 0; +lean_inc(x_15); +lean_inc(x_14); +lean_inc(x_6); +x_295 = l_Lean_Attribute_add(x_6, x_288, x_293, x_294, x_14, x_15, x_260); +if (lean_obj_tag(x_295) == 0) { -return x_46; +lean_object* x_296; lean_object* x_297; lean_object* x_298; +x_296 = lean_ctor_get(x_295, 0); +lean_inc(x_296); +x_297 = lean_ctor_get(x_295, 1); +lean_inc(x_297); +lean_dec(x_295); +x_298 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_6, x_26, x_9, x_1, x_3, x_4, x_296, x_12, x_13, x_14, x_15, x_297); +lean_dec(x_296); +return x_298; } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_48 = lean_ctor_get(x_46, 0); -x_49 = lean_ctor_get(x_46, 1); -lean_inc(x_49); -lean_inc(x_48); -lean_dec(x_46); -x_50 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_50, 0, x_48); -lean_ctor_set(x_50, 1, x_49); -return x_50; +lean_object* x_299; lean_object* x_300; lean_object* x_301; lean_object* x_302; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_299 = lean_ctor_get(x_295, 0); +lean_inc(x_299); +x_300 = lean_ctor_get(x_295, 1); +lean_inc(x_300); +if (lean_is_exclusive(x_295)) { + lean_ctor_release(x_295, 0); + lean_ctor_release(x_295, 1); + x_301 = x_295; +} else { + lean_dec_ref(x_295); + x_301 = lean_box(0); +} +if (lean_is_scalar(x_301)) { + x_302 = lean_alloc_ctor(1, 2, 0); +} else { + x_302 = x_301; +} +lean_ctor_set(x_302, 0, x_299); +lean_ctor_set(x_302, 1, x_300); +return x_302; +} +} } } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; -x_51 = lean_ctor_get(x_38, 0); -lean_inc(x_51); -lean_dec(x_38); -x_52 = l_Lean_KernelException_toMessageData(x_51, x_26); -x_53 = l_Lean_MessageData_toString(x_52, x_35); -x_54 = lean_ctor_get(x_53, 0); -lean_inc(x_54); -x_55 = lean_ctor_get(x_53, 1); -lean_inc(x_55); -lean_dec(x_53); -x_56 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_56, 0, x_54); -x_57 = l_Lean_MessageData_ofFormat(x_56); -x_58 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_57, x_12, x_13, x_14, x_15, x_55); +lean_object* x_303; lean_object* x_304; lean_object* x_305; lean_object* x_306; +lean_dec(x_250); +lean_dec(x_241); lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); -x_59 = lean_ctor_get(x_58, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_58, 1); -lean_inc(x_60); -if (lean_is_exclusive(x_58)) { - lean_ctor_release(x_58, 0); - lean_ctor_release(x_58, 1); - x_61 = x_58; +lean_dec(x_9); +lean_dec(x_6); +lean_dec(x_1); +x_303 = lean_ctor_get(x_255, 0); +lean_inc(x_303); +x_304 = lean_ctor_get(x_255, 1); +lean_inc(x_304); +if (lean_is_exclusive(x_255)) { + lean_ctor_release(x_255, 0); + lean_ctor_release(x_255, 1); + x_305 = x_255; } else { - lean_dec_ref(x_58); - x_61 = lean_box(0); + lean_dec_ref(x_255); + x_305 = lean_box(0); } -if (lean_is_scalar(x_61)) { - x_62 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_305)) { + x_306 = lean_alloc_ctor(1, 2, 0); } else { - x_62 = x_61; + x_306 = x_305; +} +lean_ctor_set(x_306, 0, x_303); +lean_ctor_set(x_306, 1, x_304); +return x_306; +} } -lean_ctor_set(x_62, 0, x_59); -lean_ctor_set(x_62, 1, x_60); -return x_62; } } else { -lean_object* x_63; lean_object* x_64; -x_63 = lean_ctor_get(x_38, 0); -lean_inc(x_63); -lean_dec(x_38); -x_64 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59(x_7, x_8, x_6, x_26, x_9, x_1, x_3, x_4, x_5, x_10, x_63, x_12, x_13, x_14, x_15, x_35); +uint8_t x_307; +lean_dec(x_15); +lean_dec(x_14); +lean_dec(x_13); +lean_dec(x_12); +lean_dec(x_9); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); -return x_64; +lean_dec(x_1); +x_307 = !lean_is_exclusive(x_33); +if (x_307 == 0) +{ +return x_33; +} +else +{ +lean_object* x_308; lean_object* x_309; lean_object* x_310; +x_308 = lean_ctor_get(x_33, 0); +x_309 = lean_ctor_get(x_33, 1); +lean_inc(x_309); +lean_inc(x_308); +lean_dec(x_33); +x_310 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_310, 0, x_308); +lean_ctor_set(x_310, 1, x_309); +return x_310; +} } } else { -uint8_t x_65; +uint8_t x_311; lean_dec(x_19); lean_dec(x_15); lean_dec(x_14); @@ -31343,29 +36965,29 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_65 = !lean_is_exclusive(x_23); -if (x_65 == 0) +x_311 = !lean_is_exclusive(x_23); +if (x_311 == 0) { return x_23; } else { -lean_object* x_66; lean_object* x_67; lean_object* x_68; -x_66 = lean_ctor_get(x_23, 0); -x_67 = lean_ctor_get(x_23, 1); -lean_inc(x_67); -lean_inc(x_66); +lean_object* x_312; lean_object* x_313; lean_object* x_314; +x_312 = lean_ctor_get(x_23, 0); +x_313 = lean_ctor_get(x_23, 1); +lean_inc(x_313); +lean_inc(x_312); lean_dec(x_23); -x_68 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_68, 0, x_66); -lean_ctor_set(x_68, 1, x_67); -return x_68; +x_314 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_314, 0, x_312); +lean_ctor_set(x_314, 1, x_313); +return x_314; } } } else { -uint8_t x_69; +uint8_t x_315; lean_dec(x_15); lean_dec(x_14); lean_dec(x_13); @@ -31376,28 +36998,28 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_1); -x_69 = !lean_is_exclusive(x_18); -if (x_69 == 0) +x_315 = !lean_is_exclusive(x_18); +if (x_315 == 0) { return x_18; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_70 = lean_ctor_get(x_18, 0); -x_71 = lean_ctor_get(x_18, 1); -lean_inc(x_71); -lean_inc(x_70); +lean_object* x_316; lean_object* x_317; lean_object* x_318; +x_316 = lean_ctor_get(x_18, 0); +x_317 = lean_ctor_get(x_18, 1); +lean_inc(x_317); +lean_inc(x_316); lean_dec(x_18); -x_72 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_72, 0, x_70); -lean_ctor_set(x_72, 1, x_71); -return x_72; +x_318 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_318, 0, x_316); +lean_ctor_set(x_318, 1, x_317); +return x_318; } } } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51(lean_object* x_1, lean_object* x_2, uint8_t x_3, uint8_t x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_32; lean_object* x_33; uint8_t x_34; @@ -31432,7 +37054,7 @@ x_21 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_21, 0, x_13); lean_ctor_set(x_21, 1, x_20); lean_ctor_set(x_21, 2, x_17); -x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); +x_22 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(x_2, x_3, x_4, x_6, x_19, x_21, x_21, x_5, x_13, lean_box(0), lean_box(0), x_8, x_9, x_10, x_11, x_12); lean_dec(x_21); lean_dec(x_19); if (lean_obj_tag(x_22) == 0) @@ -31883,7 +37505,7 @@ if (lean_obj_tag(x_46) == 0) lean_object* x_47; lean_object* x_48; lean_dec(x_18); x_47 = lean_box(0); -x_48 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(x_1, x_45, x_2, x_3, x_27, x_23, x_20, x_14, x_11, x_25, x_47, x_5, x_6, x_7, x_8, x_32); +x_48 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(x_1, x_45, x_2, x_3, x_27, x_23, x_20, x_14, x_11, x_25, x_47, x_5, x_6, x_7, x_8, x_32); lean_dec(x_25); lean_dec(x_45); return x_48; @@ -31944,7 +37566,7 @@ else lean_object* x_59; lean_object* x_60; lean_dec(x_18); x_59 = lean_box(0); -x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(x_1, x_45, x_2, x_3, x_27, x_23, x_20, x_14, x_11, x_25, x_59, x_5, x_6, x_7, x_8, x_32); +x_60 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(x_1, x_45, x_2, x_3, x_27, x_23, x_20, x_14, x_11, x_25, x_59, x_5, x_6, x_7, x_8, x_32); lean_dec(x_25); lean_dec(x_45); return x_60; @@ -32053,7 +37675,7 @@ lean_inc(x_101); lean_dec(x_99); x_102 = lean_box(x_2); x_103 = lean_box(x_3); -x_104 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed), 12, 5); +x_104 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5___boxed), 12, 5); lean_closure_set(x_104, 0, x_11); lean_closure_set(x_104, 1, x_1); lean_closure_set(x_104, 2, x_102); @@ -32392,7 +38014,7 @@ if (lean_obj_tag(x_155) == 0) lean_object* x_156; lean_object* x_157; lean_dec(x_127); x_156 = lean_box(0); -x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(x_1, x_154, x_2, x_3, x_136, x_132, x_129, x_123, x_11, x_134, x_156, x_5, x_6, x_7, x_8, x_141); +x_157 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_1, x_154, x_2, x_3, x_136, x_132, x_129, x_123, x_11, x_134, x_156, x_5, x_6, x_7, x_8, x_141); lean_dec(x_134); lean_dec(x_154); return x_157; @@ -32453,7 +38075,7 @@ else lean_object* x_168; lean_object* x_169; lean_dec(x_127); x_168 = lean_box(0); -x_169 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(x_1, x_154, x_2, x_3, x_136, x_132, x_129, x_123, x_11, x_134, x_168, x_5, x_6, x_7, x_8, x_141); +x_169 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_1, x_154, x_2, x_3, x_136, x_132, x_129, x_123, x_11, x_134, x_168, x_5, x_6, x_7, x_8, x_141); lean_dec(x_134); lean_dec(x_154); return x_169; @@ -32562,7 +38184,7 @@ lean_inc(x_210); lean_dec(x_208); x_211 = lean_box(x_2); x_212 = lean_box(x_3); -x_213 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12___boxed), 12, 5); +x_213 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10___boxed), 12, 5); lean_closure_set(x_213, 0, x_11); lean_closure_set(x_213, 1, x_1); lean_closure_set(x_213, 2, x_211); @@ -32873,7 +38495,7 @@ if (lean_obj_tag(x_260) == 0) lean_object* x_261; lean_object* x_262; lean_dec(x_232); x_261 = lean_box(0); -x_262 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(x_1, x_259, x_2, x_3, x_241, x_237, x_234, x_228, x_11, x_239, x_261, x_5, x_6, x_7, x_8, x_246); +x_262 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(x_1, x_259, x_2, x_3, x_241, x_237, x_234, x_228, x_11, x_239, x_261, x_5, x_6, x_7, x_8, x_246); lean_dec(x_239); lean_dec(x_259); return x_262; @@ -32934,7 +38556,7 @@ else lean_object* x_273; lean_object* x_274; lean_dec(x_232); x_273 = lean_box(0); -x_274 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(x_1, x_259, x_2, x_3, x_241, x_237, x_234, x_228, x_11, x_239, x_273, x_5, x_6, x_7, x_8, x_246); +x_274 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(x_1, x_259, x_2, x_3, x_241, x_237, x_234, x_228, x_11, x_239, x_273, x_5, x_6, x_7, x_8, x_246); lean_dec(x_239); lean_dec(x_259); return x_274; @@ -33043,7 +38665,7 @@ lean_inc(x_315); lean_dec(x_313); x_316 = lean_box(x_2); x_317 = lean_box(x_3); -x_318 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18___boxed), 12, 5); +x_318 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15___boxed), 12, 5); lean_closure_set(x_318, 0, x_11); lean_closure_set(x_318, 1, x_1); lean_closure_set(x_318, 2, x_316); @@ -33354,7 +38976,7 @@ if (lean_obj_tag(x_365) == 0) lean_object* x_366; lean_object* x_367; lean_dec(x_337); x_366 = lean_box(0); -x_367 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_1, x_364, x_2, x_3, x_346, x_342, x_339, x_333, x_11, x_344, x_366, x_5, x_6, x_7, x_8, x_351); +x_367 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(x_1, x_364, x_2, x_3, x_346, x_342, x_339, x_333, x_11, x_344, x_366, x_5, x_6, x_7, x_8, x_351); lean_dec(x_344); lean_dec(x_364); return x_367; @@ -33415,7 +39037,7 @@ else lean_object* x_378; lean_object* x_379; lean_dec(x_337); x_378 = lean_box(0); -x_379 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_1, x_364, x_2, x_3, x_346, x_342, x_339, x_333, x_11, x_344, x_378, x_5, x_6, x_7, x_8, x_351); +x_379 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(x_1, x_364, x_2, x_3, x_346, x_342, x_339, x_333, x_11, x_344, x_378, x_5, x_6, x_7, x_8, x_351); lean_dec(x_344); lean_dec(x_364); return x_379; @@ -33524,7 +39146,7 @@ lean_inc(x_420); lean_dec(x_418); x_421 = lean_box(x_2); x_422 = lean_box(x_3); -x_423 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24___boxed), 12, 5); +x_423 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20___boxed), 12, 5); lean_closure_set(x_423, 0, x_11); lean_closure_set(x_423, 1, x_1); lean_closure_set(x_423, 2, x_421); @@ -33835,7 +39457,7 @@ if (lean_obj_tag(x_470) == 0) lean_object* x_471; lean_object* x_472; lean_dec(x_442); x_471 = lean_box(0); -x_472 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_1, x_469, x_2, x_3, x_451, x_447, x_444, x_438, x_11, x_449, x_471, x_5, x_6, x_7, x_8, x_456); +x_472 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(x_1, x_469, x_2, x_3, x_451, x_447, x_444, x_438, x_11, x_449, x_471, x_5, x_6, x_7, x_8, x_456); lean_dec(x_449); lean_dec(x_469); return x_472; @@ -33896,7 +39518,7 @@ else lean_object* x_483; lean_object* x_484; lean_dec(x_442); x_483 = lean_box(0); -x_484 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_1, x_469, x_2, x_3, x_451, x_447, x_444, x_438, x_11, x_449, x_483, x_5, x_6, x_7, x_8, x_456); +x_484 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(x_1, x_469, x_2, x_3, x_451, x_447, x_444, x_438, x_11, x_449, x_483, x_5, x_6, x_7, x_8, x_456); lean_dec(x_449); lean_dec(x_469); return x_484; @@ -34005,7 +39627,7 @@ lean_inc(x_525); lean_dec(x_523); x_526 = lean_box(x_2); x_527 = lean_box(x_3); -x_528 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30___boxed), 12, 5); +x_528 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed), 12, 5); lean_closure_set(x_528, 0, x_11); lean_closure_set(x_528, 1, x_1); lean_closure_set(x_528, 2, x_526); @@ -34076,7 +39698,7 @@ lean_inc(x_541); lean_dec(x_10); x_542 = lean_box(x_2); x_543 = lean_box(x_3); -x_544 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed), 10, 3); +x_544 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed), 10, 3); lean_closure_set(x_544, 0, x_1); lean_closure_set(x_544, 1, x_542); lean_closure_set(x_544, 2, x_543); @@ -34332,7 +39954,7 @@ if (lean_obj_tag(x_581) == 0) lean_object* x_582; lean_object* x_583; lean_dec(x_553); x_582 = lean_box(0); -x_583 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(x_1, x_580, x_2, x_3, x_562, x_558, x_555, x_549, x_11, x_560, x_582, x_5, x_6, x_7, x_8, x_567); +x_583 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(x_1, x_580, x_2, x_3, x_562, x_558, x_555, x_549, x_11, x_560, x_582, x_5, x_6, x_7, x_8, x_567); lean_dec(x_560); lean_dec(x_580); return x_583; @@ -34393,7 +40015,7 @@ else lean_object* x_594; lean_object* x_595; lean_dec(x_553); x_594 = lean_box(0); -x_595 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(x_1, x_580, x_2, x_3, x_562, x_558, x_555, x_549, x_11, x_560, x_594, x_5, x_6, x_7, x_8, x_567); +x_595 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(x_1, x_580, x_2, x_3, x_562, x_558, x_555, x_549, x_11, x_560, x_594, x_5, x_6, x_7, x_8, x_567); lean_dec(x_560); lean_dec(x_580); return x_595; @@ -34502,7 +40124,7 @@ lean_inc(x_636); lean_dec(x_634); x_637 = lean_box(x_2); x_638 = lean_box(x_3); -x_639 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed), 12, 5); +x_639 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed), 12, 5); lean_closure_set(x_639, 0, x_11); lean_closure_set(x_639, 1, x_1); lean_closure_set(x_639, 2, x_637); @@ -34813,7 +40435,7 @@ if (lean_obj_tag(x_686) == 0) lean_object* x_687; lean_object* x_688; lean_dec(x_658); x_687 = lean_box(0); -x_688 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(x_1, x_685, x_2, x_3, x_667, x_663, x_660, x_654, x_11, x_665, x_687, x_5, x_6, x_7, x_8, x_672); +x_688 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(x_1, x_685, x_2, x_3, x_667, x_663, x_660, x_654, x_11, x_665, x_687, x_5, x_6, x_7, x_8, x_672); lean_dec(x_665); lean_dec(x_685); return x_688; @@ -34874,7 +40496,7 @@ else lean_object* x_699; lean_object* x_700; lean_dec(x_658); x_699 = lean_box(0); -x_700 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(x_1, x_685, x_2, x_3, x_667, x_663, x_660, x_654, x_11, x_665, x_699, x_5, x_6, x_7, x_8, x_672); +x_700 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(x_1, x_685, x_2, x_3, x_667, x_663, x_660, x_654, x_11, x_665, x_699, x_5, x_6, x_7, x_8, x_672); lean_dec(x_665); lean_dec(x_685); return x_700; @@ -34983,7 +40605,7 @@ lean_inc(x_741); lean_dec(x_739); x_742 = lean_box(x_2); x_743 = lean_box(x_3); -x_744 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43___boxed), 12, 5); +x_744 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36___boxed), 12, 5); lean_closure_set(x_744, 0, x_11); lean_closure_set(x_744, 1, x_1); lean_closure_set(x_744, 2, x_742); @@ -35294,7 +40916,7 @@ if (lean_obj_tag(x_791) == 0) lean_object* x_792; lean_object* x_793; lean_dec(x_763); x_792 = lean_box(0); -x_793 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(x_1, x_790, x_2, x_3, x_772, x_768, x_765, x_759, x_11, x_770, x_792, x_5, x_6, x_7, x_8, x_777); +x_793 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_1, x_790, x_2, x_3, x_772, x_768, x_765, x_759, x_11, x_770, x_792, x_5, x_6, x_7, x_8, x_777); lean_dec(x_770); lean_dec(x_790); return x_793; @@ -35355,7 +40977,7 @@ else lean_object* x_804; lean_object* x_805; lean_dec(x_763); x_804 = lean_box(0); -x_805 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(x_1, x_790, x_2, x_3, x_772, x_768, x_765, x_759, x_11, x_770, x_804, x_5, x_6, x_7, x_8, x_777); +x_805 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_1, x_790, x_2, x_3, x_772, x_768, x_765, x_759, x_11, x_770, x_804, x_5, x_6, x_7, x_8, x_777); lean_dec(x_770); lean_dec(x_790); return x_805; @@ -35464,7 +41086,7 @@ lean_inc(x_846); lean_dec(x_844); x_847 = lean_box(x_2); x_848 = lean_box(x_3); -x_849 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49___boxed), 12, 5); +x_849 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41___boxed), 12, 5); lean_closure_set(x_849, 0, x_11); lean_closure_set(x_849, 1, x_1); lean_closure_set(x_849, 2, x_847); @@ -35775,7 +41397,7 @@ if (lean_obj_tag(x_896) == 0) lean_object* x_897; lean_object* x_898; lean_dec(x_868); x_897 = lean_box(0); -x_898 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54(x_1, x_895, x_2, x_3, x_877, x_873, x_870, x_864, x_11, x_875, x_897, x_5, x_6, x_7, x_8, x_882); +x_898 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(x_1, x_895, x_2, x_3, x_877, x_873, x_870, x_864, x_11, x_875, x_897, x_5, x_6, x_7, x_8, x_882); lean_dec(x_875); lean_dec(x_895); return x_898; @@ -35836,7 +41458,7 @@ else lean_object* x_909; lean_object* x_910; lean_dec(x_868); x_909 = lean_box(0); -x_910 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54(x_1, x_895, x_2, x_3, x_877, x_873, x_870, x_864, x_11, x_875, x_909, x_5, x_6, x_7, x_8, x_882); +x_910 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(x_1, x_895, x_2, x_3, x_877, x_873, x_870, x_864, x_11, x_875, x_909, x_5, x_6, x_7, x_8, x_882); lean_dec(x_875); lean_dec(x_895); return x_910; @@ -35945,7 +41567,7 @@ lean_inc(x_951); lean_dec(x_949); x_952 = lean_box(x_2); x_953 = lean_box(x_3); -x_954 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55___boxed), 12, 5); +x_954 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46___boxed), 12, 5); lean_closure_set(x_954, 0, x_11); lean_closure_set(x_954, 1, x_1); lean_closure_set(x_954, 2, x_952); @@ -36256,7 +41878,7 @@ if (lean_obj_tag(x_1001) == 0) lean_object* x_1002; lean_object* x_1003; lean_dec(x_973); x_1002 = lean_box(0); -x_1003 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60(x_1, x_1000, x_2, x_3, x_982, x_978, x_975, x_969, x_11, x_980, x_1002, x_5, x_6, x_7, x_8, x_987); +x_1003 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(x_1, x_1000, x_2, x_3, x_982, x_978, x_975, x_969, x_11, x_980, x_1002, x_5, x_6, x_7, x_8, x_987); lean_dec(x_980); lean_dec(x_1000); return x_1003; @@ -36317,7 +41939,7 @@ else lean_object* x_1014; lean_object* x_1015; lean_dec(x_973); x_1014 = lean_box(0); -x_1015 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60(x_1, x_1000, x_2, x_3, x_982, x_978, x_975, x_969, x_11, x_980, x_1014, x_5, x_6, x_7, x_8, x_987); +x_1015 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(x_1, x_1000, x_2, x_3, x_982, x_978, x_975, x_969, x_11, x_980, x_1014, x_5, x_6, x_7, x_8, x_987); lean_dec(x_980); lean_dec(x_1000); return x_1015; @@ -36426,7 +42048,7 @@ lean_inc(x_1056); lean_dec(x_1054); x_1057 = lean_box(x_2); x_1058 = lean_box(x_3); -x_1059 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61___boxed), 12, 5); +x_1059 = lean_alloc_closure((void*)(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51___boxed), 12, 5); lean_closure_set(x_1059, 0, x_11); lean_closure_set(x_1059, 1, x_1); lean_closure_set(x_1059, 2, x_1057); @@ -36628,19 +42250,82 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { -lean_object* x_7; -x_7 = l_Lean_throwError___at_Lean_ParserCompiler_compileParserExpr___spec__5(x_1, x_2, x_3, x_4, x_5, x_6); +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__5___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); -return x_7; +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox(x_3); +lean_dec(x_3); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36648,7 +42333,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__6___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__8___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36656,7 +42341,23 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36664,12 +42365,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__7___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36677,12 +42378,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__8___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -36707,7 +42408,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -36715,7 +42416,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36723,7 +42424,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__9___at_Lean_ParserCompiler_compileParserExpr___spec__10___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__13___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36731,7 +42432,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36739,7 +42440,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__11___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36747,7 +42448,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36755,12 +42456,194 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__12___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox(x_3); +lean_dec(x_3); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_20; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__18___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +lean_dec(x_2); +return x_13; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed(lean_object** _args) { +lean_object* x_1 = _args[0]; +lean_object* x_2 = _args[1]; +lean_object* x_3 = _args[2]; +lean_object* x_4 = _args[3]; +lean_object* x_5 = _args[4]; +lean_object* x_6 = _args[5]; +lean_object* x_7 = _args[6]; +lean_object* x_8 = _args[7]; +lean_object* x_9 = _args[8]; +lean_object* x_10 = _args[9]; +lean_object* x_11 = _args[10]; +lean_object* x_12 = _args[11]; +lean_object* x_13 = _args[12]; +lean_object* x_14 = _args[13]; +lean_object* x_15 = _args[14]; +lean_object* x_16 = _args[15]; +lean_object* x_17 = _args[16]; +_start: +{ +uint8_t x_18; uint8_t x_19; lean_object* x_20; +x_18 = lean_unbox(x_2); +lean_dec(x_2); +x_19 = lean_unbox(x_3); +lean_dec(x_3); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +return x_20; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__23___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +_start: +{ +uint8_t x_17; uint8_t x_18; lean_object* x_19; +x_17 = lean_unbox(x_2); +lean_dec(x_2); +x_18 = lean_unbox(x_3); +lean_dec(x_3); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_4); +return x_19; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +_start: +{ +size_t x_11; size_t x_12; lean_object* x_13; +x_11 = lean_unbox_usize(x_3); +lean_dec(x_3); +x_12 = lean_unbox_usize(x_4); +lean_dec(x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36768,12 +42651,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__13___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -36798,7 +42681,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -36806,7 +42689,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36814,7 +42697,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__14___at_Lean_ParserCompiler_compileParserExpr___spec__15___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__28___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36822,7 +42705,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36830,7 +42713,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__16___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36838,7 +42721,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36846,12 +42729,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__17___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36859,12 +42742,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__18___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -36889,7 +42772,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -36897,7 +42780,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36905,7 +42788,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__19___at_Lean_ParserCompiler_compileParserExpr___spec__20___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__33___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36913,7 +42796,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36921,7 +42804,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__21___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -36929,7 +42812,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36937,12 +42820,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__22___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -36950,12 +42833,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__23___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -36980,7 +42863,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -36988,7 +42871,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -36996,7 +42879,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__24___at_Lean_ParserCompiler_compileParserExpr___spec__25___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__38___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37004,7 +42887,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37012,7 +42895,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__26___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37020,7 +42903,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -37028,12 +42911,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__27___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -37041,12 +42924,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__28___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -37071,7 +42954,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -37079,7 +42962,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37087,7 +42970,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__29___at_Lean_ParserCompiler_compileParserExpr___spec__30___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__43___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37095,7 +42978,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37103,7 +42986,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__31___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37111,7 +42994,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -37119,12 +43002,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__32___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -37132,12 +43015,12 @@ x_11 = lean_unbox_usize(x_3); lean_dec(x_3); x_12 = lean_unbox_usize(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__33___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); +x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); return x_13; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg___boxed(lean_object** _args) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed(lean_object** _args) { lean_object* x_1 = _args[0]; lean_object* x_2 = _args[1]; lean_object* x_3 = _args[2]; @@ -37162,7 +43045,7 @@ x_18 = lean_unbox(x_2); lean_dec(x_2); x_19 = lean_unbox(x_3); lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); +x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); @@ -37170,7 +43053,7 @@ lean_dec(x_5); return x_20; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37178,7 +43061,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__34___at_Lean_ParserCompiler_compileParserExpr___spec__35___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__48___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37186,7 +43069,7 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37194,7 +43077,7 @@ x_17 = lean_unbox(x_2); lean_dec(x_2); x_18 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__36___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); @@ -37202,290 +43085,149 @@ lean_dec(x_4); return x_19; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); +lean_object* x_9; +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__37___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); -return x_13; +return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_3); lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); +x_14 = lean_unbox(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__38___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -_start: -{ -uint8_t x_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_unbox(x_2); -lean_dec(x_2); -x_19 = lean_unbox(x_3); -lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_8); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -return x_20; +return x_15; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); -lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__39___at_Lean_ParserCompiler_compileParserExpr___spec__40___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -lean_dec(x_6); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_5); lean_dec(x_5); -lean_dec(x_4); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); -lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__41___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); +x_14 = lean_unbox(x_6); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__42___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); -lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__43___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_13; -} -} -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; -_start: -{ -uint8_t x_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_unbox(x_2); -lean_dec(x_2); -x_19 = lean_unbox(x_3); -lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_8); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); -return x_20; +return x_15; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); +x_17 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__44___at_Lean_ParserCompiler_compileParserExpr___spec__45___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +x_18 = lean_unbox(x_4); lean_dec(x_4); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__46___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_19; +return x_15; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); +lean_object* x_9; +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); -lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__47___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_2); -return x_13; +return x_9; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -size_t x_11; size_t x_12; lean_object* x_13; -x_11 = lean_unbox_usize(x_3); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_3); lean_dec(x_3); -x_12 = lean_unbox_usize(x_4); +x_14 = lean_unbox(x_4); lean_dec(x_4); -x_13 = l_Array_foldrMUnsafe_fold___at_Lean_ParserCompiler_compileParserExpr___spec__48___rarg(x_1, x_2, x_11, x_12, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_2); -return x_13; +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); +lean_dec(x_6); +return x_15; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg___boxed(lean_object** _args) { -lean_object* x_1 = _args[0]; -lean_object* x_2 = _args[1]; -lean_object* x_3 = _args[2]; -lean_object* x_4 = _args[3]; -lean_object* x_5 = _args[4]; -lean_object* x_6 = _args[5]; -lean_object* x_7 = _args[6]; -lean_object* x_8 = _args[7]; -lean_object* x_9 = _args[8]; -lean_object* x_10 = _args[9]; -lean_object* x_11 = _args[10]; -lean_object* x_12 = _args[11]; -lean_object* x_13 = _args[12]; -lean_object* x_14 = _args[13]; -lean_object* x_15 = _args[14]; -lean_object* x_16 = _args[15]; -lean_object* x_17 = _args[16]; +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_18; uint8_t x_19; lean_object* x_20; -x_18 = lean_unbox(x_2); -lean_dec(x_2); -x_19 = lean_unbox(x_3); -lean_dec(x_3); -x_20 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___rarg(x_1, x_18, x_19, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16, x_17); -lean_dec(x_8); -lean_dec(x_7); -lean_dec(x_6); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_5); lean_dec(x_5); -return x_20; +x_14 = lean_unbox(x_6); +lean_dec(x_6); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +lean_dec(x_7); +return x_15; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); +x_17 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__49___at_Lean_ParserCompiler_compileParserExpr___spec__50___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_7); -lean_dec(x_6); -lean_dec(x_5); +x_18 = lean_unbox(x_4); lean_dec(x_4); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +lean_dec(x_11); +lean_dec(x_10); +lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_2); -lean_dec(x_2); -x_18 = lean_unbox(x_3); +uint8_t x_13; uint8_t x_14; lean_object* x_15; +x_13 = lean_unbox(x_3); lean_dec(x_3); -x_19 = l_Std_Range_forIn_x27_loop___at_Lean_ParserCompiler_compileParserExpr___spec__51___rarg(x_1, x_17, x_18, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_14 = lean_unbox(x_4); +lean_dec(x_4); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_4); -return x_19; +return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37493,13 +43235,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__2(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37507,26 +43249,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__3(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37534,14 +43262,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__5(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37549,23 +43277,23 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__6(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__7(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37573,13 +43301,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__8(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37587,26 +43315,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__9(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__10(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37614,14 +43328,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__11(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37629,23 +43343,23 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__12(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__13(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37653,13 +43367,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__14(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37667,26 +43381,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__15(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__16(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37694,38 +43394,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__17(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_3); -lean_dec(x_3); -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__18(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -lean_dec(x_6); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__19(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -lean_dec(x_2); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37733,79 +43409,36 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__20(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_5); -lean_dec(x_5); -x_14 = lean_unbox(x_6); -lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__21(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__22(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_3); -lean_dec(x_3); -x_18 = lean_unbox(x_4); -lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__23(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_11); -lean_dec(x_10); +uint8_t x_11; uint8_t x_12; lean_object* x_13; +x_11 = lean_unbox(x_2); lean_dec(x_2); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_3); +x_12 = lean_unbox(x_3); lean_dec(x_3); -x_14 = lean_unbox(x_4); +x_13 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__24(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -lean_dec(x_6); -return x_15; +return x_13; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__25(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37813,13 +43446,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__26(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37827,26 +43460,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__27(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__28(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -37854,14 +43473,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__29(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -37869,25 +43488,12 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__30(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { -_start: -{ -uint8_t x_11; uint8_t x_12; lean_object* x_13; -x_11 = lean_unbox(x_2); -lean_dec(x_2); -x_12 = lean_unbox(x_3); -lean_dec(x_3); -x_13 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__31(x_1, x_11, x_12, x_4, x_5, x_6, x_7, x_8, x_9, x_10); -lean_dec(x_4); -return x_13; -} -} LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__32___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { @@ -37929,112 +43535,18 @@ LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_3); -lean_dec(x_3); -x_18 = lean_unbox(x_4); -lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_11); -lean_dec(x_10); -lean_dec(x_2); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_3); -lean_dec(x_3); -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -lean_dec(x_6); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { -_start: -{ -lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); -lean_dec(x_3); -lean_dec(x_2); -return x_9; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_3); -lean_dec(x_3); -x_14 = lean_unbox(x_4); -lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -lean_dec(x_6); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { -_start: -{ -uint8_t x_13; uint8_t x_14; lean_object* x_15; -x_13 = lean_unbox(x_5); -lean_dec(x_5); -x_14 = lean_unbox(x_6); -lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_7); -return x_15; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__35(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38042,23 +43554,23 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__36(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__37(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38066,13 +43578,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__38(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38080,26 +43592,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__39(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -38107,14 +43605,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__40(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38122,23 +43620,23 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__41(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__42(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38146,13 +43644,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__43(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38160,26 +43658,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__52(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__44(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__53(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -38187,14 +43671,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__54(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__45(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38202,23 +43686,23 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__55(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__46(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { lean_object* x_9; -x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__56(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); +x_9 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__47(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8); lean_dec(x_3); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38226,13 +43710,13 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__57(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__48(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38240,26 +43724,12 @@ x_13 = lean_unbox(x_5); lean_dec(x_5); x_14 = lean_unbox(x_6); lean_dec(x_6); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__58(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__49(x_1, x_2, x_3, x_4, x_13, x_14, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); return x_15; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { -_start: -{ -uint8_t x_17; uint8_t x_18; lean_object* x_19; -x_17 = lean_unbox(x_7); -lean_dec(x_7); -x_18 = lean_unbox(x_8); -lean_dec(x_8); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__59(x_1, x_2, x_3, x_4, x_5, x_6, x_17, x_18, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); -lean_dec(x_10); -lean_dec(x_9); -return x_19; -} -} -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12, lean_object* x_13, lean_object* x_14, lean_object* x_15, lean_object* x_16) { _start: { uint8_t x_17; uint8_t x_18; lean_object* x_19; @@ -38267,14 +43737,14 @@ x_17 = lean_unbox(x_3); lean_dec(x_3); x_18 = lean_unbox(x_4); lean_dec(x_4); -x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__60(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); +x_19 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__50(x_1, x_2, x_17, x_18, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12, x_13, x_14, x_15, x_16); lean_dec(x_11); lean_dec(x_10); lean_dec(x_2); return x_19; } } -LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { +LEAN_EXPORT lean_object* l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10, lean_object* x_11, lean_object* x_12) { _start: { uint8_t x_13; uint8_t x_14; lean_object* x_15; @@ -38282,7 +43752,7 @@ x_13 = lean_unbox(x_3); lean_dec(x_3); x_14 = lean_unbox(x_4); lean_dec(x_4); -x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__61(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); +x_15 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__51(x_1, x_2, x_13, x_14, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); lean_dec(x_7); lean_dec(x_6); return x_15; @@ -38687,47 +44157,29 @@ return x_2; static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__5() { _start: { -lean_object* x_1; -x_1 = l_Lean_PersistentHashMap_mkEmptyEntriesArray(lean_box(0), lean_box(0)); -return x_1; -} -} -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__5; -x_2 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7() { -_start: -{ lean_object* x_1; lean_object* x_2; x_1 = lean_unsigned_to_nat(32u); x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__8() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7; +x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__5; x_2 = lean_alloc_ctor(0, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7() { _start: { size_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_1 = 5; -x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__8; -x_3 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7; +x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; +x_3 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__5; x_4 = lean_unsigned_to_nat(0u); x_5 = lean_alloc_ctor(0, 4, sizeof(size_t)*1); lean_ctor_set(x_5, 0, x_2); @@ -38738,19 +44190,19 @@ lean_ctor_set_usize(x_5, 4, x_1); return x_5; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; -x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9; +x_1 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; +x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__11() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9() { _start: { lean_object* x_1; lean_object* x_2; @@ -38759,7 +44211,7 @@ x_2 = lean_array_mk(x_1); return x_2; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; uint64_t x_4; uint8_t x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; @@ -38768,8 +44220,8 @@ x_2 = lean_box(0); x_3 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__3; x_4 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__4; x_5 = 0; -x_6 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10; -x_7 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__11; +x_6 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__8; +x_7 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9; x_8 = lean_unsigned_to_nat(0u); x_9 = lean_alloc_ctor(0, 7, 11); lean_ctor_set(x_9, 0, x_3); @@ -38786,12 +44238,12 @@ lean_ctor_set_uint8(x_9, sizeof(void*)*7 + 10, x_5); return x_9; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_unsigned_to_nat(0u); -x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; +x_2 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; x_3 = lean_alloc_ctor(0, 9, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_1); @@ -38805,26 +44257,11 @@ lean_ctor_set(x_3, 8, x_2); return x_3; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; -x_2 = lean_alloc_ctor(0, 6, 0); -lean_ctor_set(x_2, 0, x_1); -lean_ctor_set(x_2, 1, x_1); -lean_ctor_set(x_2, 2, x_1); -lean_ctor_set(x_2, 3, x_1); -lean_ctor_set(x_2, 4, x_1); -lean_ctor_set(x_2, 5, x_1); -return x_2; -} -} -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__6; +x_1 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__2; x_2 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_2, 0, x_1); lean_ctor_set(x_2, 1, x_1); @@ -38833,15 +44270,15 @@ lean_ctor_set(x_2, 3, x_1); return x_2; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_1 = lean_box(0); -x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13; -x_3 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14; -x_4 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__9; -x_5 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15; +x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__11; +x_3 = l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4; +x_4 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__7; +x_5 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12; x_6 = lean_alloc_ctor(0, 5, 0); lean_ctor_set(x_6, 0, x_2); lean_ctor_set(x_6, 1, x_3); @@ -38851,7 +44288,7 @@ lean_ctor_set(x_6, 4, x_5); return x_6; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14() { _start: { lean_object* x_1; @@ -38859,12 +44296,12 @@ x_1 = lean_mk_string_unchecked("TrailingParserDescr", 19, 19); return x_1; } } -static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18() { +static lean_object* _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Lean_ParserCompiler_replaceParserTy___rarg___lambda__1___closed__1; -x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17; +x_2 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14; x_3 = l_Lean_Name_mkStr2(x_1, x_2); return x_3; } @@ -38890,7 +44327,7 @@ x_66 = l_Lean_Expr_isConstOf(x_11, x_65); if (x_66 == 0) { lean_object* x_67; uint8_t x_68; -x_67 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18; +x_67 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15; x_68 = l_Lean_Expr_isConstOf(x_11, x_67); lean_dec(x_11); if (x_68 == 0) @@ -38899,14 +44336,14 @@ uint8_t x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_obje x_69 = l_Lean_Name_isAnonymous(x_2); x_70 = lean_box(0); x_71 = l_Lean_Expr_const___override(x_3, x_70); -x_72 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16; +x_72 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13; x_73 = lean_st_mk_ref(x_72, x_10); x_74 = lean_ctor_get(x_73, 0); lean_inc(x_74); x_75 = lean_ctor_get(x_73, 1); lean_inc(x_75); lean_dec(x_73); -x_76 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12; +x_76 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10; lean_inc(x_74); x_77 = l_Lean_ParserCompiler_compileParserExpr___rarg(x_1, x_4, x_69, x_71, x_76, x_74, x_5, x_6, x_75); if (lean_obj_tag(x_77) == 0) @@ -39019,7 +44456,7 @@ if (x_41 == 0) lean_object* x_42; lean_object* x_43; lean_free_object(x_34); lean_dec(x_38); -x_42 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18; +x_42 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15; x_43 = l_Lean_evalConstCheck___at_Lean_KeyedDeclsAttribute_init___spec__1___rarg(x_42, x_3, x_5, x_6, x_39); if (lean_obj_tag(x_43) == 0) { @@ -39094,7 +44531,7 @@ if (x_53 == 0) { lean_object* x_54; lean_object* x_55; lean_dec(x_50); -x_54 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18; +x_54 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15; x_55 = l_Lean_evalConstCheck___at_Lean_KeyedDeclsAttribute_init___spec__1___rarg(x_54, x_3, x_5, x_6, x_51); if (lean_obj_tag(x_55) == 0) { @@ -39166,14 +44603,14 @@ return x_63; block_32: { lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; -x_15 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16; +x_15 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__13; x_16 = lean_st_mk_ref(x_15, x_14); x_17 = lean_ctor_get(x_16, 0); lean_inc(x_17); x_18 = lean_ctor_get(x_16, 1); lean_inc(x_18); lean_dec(x_16); -x_19 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__12; +x_19 = l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__10; lean_inc(x_17); x_20 = l_Lean_ParserCompiler_compileEmbeddedParsers___rarg(x_1, x_4, x_13, x_19, x_17, x_5, x_6, x_18); if (lean_obj_tag(x_20) == 0) @@ -39360,6 +44797,14 @@ l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4 = _init_l lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__4); l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5(); lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__5); +l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6(); +lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__6); +l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7(); +lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__7); +l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8(); +lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__8); +l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9(); +lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___lambda__4___closed__9); l_Lean_ParserCompiler_compileParserExpr___rarg___closed__1 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___closed__1(); lean_mark_persistent(l_Lean_ParserCompiler_compileParserExpr___rarg___closed__1); l_Lean_ParserCompiler_compileParserExpr___rarg___closed__2 = _init_l_Lean_ParserCompiler_compileParserExpr___rarg___closed__2(); @@ -39421,12 +44866,6 @@ l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14 = _ lean_mark_persistent(l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__14); l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15 = _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15(); lean_mark_persistent(l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__15); -l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16 = _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16(); -lean_mark_persistent(l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__16); -l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17 = _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17(); -lean_mark_persistent(l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__17); -l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18 = _init_l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18(); -lean_mark_persistent(l_Lean_ParserCompiler_registerParserCompiler___rarg___lambda__1___closed__18); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Lean/Server/CodeActions/Attr.c b/stage0/stdlib/Lean/Server/CodeActions/Attr.c index 2b407fdc244d..6edba648a534 100644 --- a/stage0/stdlib/Lean/Server/CodeActions/Attr.c +++ b/stage0/stdlib/Lean/Server/CodeActions/Attr.c @@ -185,7 +185,6 @@ LEAN_EXPORT lean_object* l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions static lean_object* l_Lean_CodeAction_instInhabitedCommandCodeActions___closed__1; static lean_object* l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions_Attr___hyg_297____closed__22; static lean_object* l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions_Attr___hyg_83____closed__4; -LEAN_EXPORT lean_object* l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_ToExpr_0__Lean_List_toExprAux___at___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin___closed__19; LEAN_EXPORT lean_object* l_Lean_CodeAction_insertBuiltin(lean_object*, lean_object*, lean_object*); @@ -4026,16 +4025,6 @@ lean_dec(x_1); return x_4; } } -LEAN_EXPORT lean_object* l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; -x_6 = l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); -return x_6; -} -} LEAN_EXPORT lean_object* l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions_Attr___hyg_1441____lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { @@ -4135,8 +4124,6 @@ if (lean_obj_tag(x_24) == 0) lean_object* x_25; lean_free_object(x_19); x_25 = l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin(x_2, x_17, x_4, x_5, x_22); -lean_dec(x_5); -lean_dec(x_4); return x_25; } else @@ -4169,8 +4156,6 @@ if (lean_obj_tag(x_30) == 0) { lean_object* x_31; x_31 = l___private_Lean_Server_CodeActions_Attr_0__Lean_CodeAction_addBuiltin(x_2, x_17, x_4, x_5, x_28); -lean_dec(x_5); -lean_dec(x_4); return x_31; } else @@ -4340,8 +4325,6 @@ LEAN_EXPORT lean_object* l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions { lean_object* x_7; x_7 = l_Lean_CodeAction_initFn____x40_Lean_Server_CodeActions_Attr___hyg_1441____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); return x_7; } diff --git a/stage0/stdlib/Lean/Server/CodeActions/Basic.c b/stage0/stdlib/Lean/Server/CodeActions/Basic.c index d628a224785e..91bede81cf67 100644 --- a/stage0/stdlib/Lean/Server/CodeActions/Basic.c +++ b/stage0/stdlib/Lean/Server/CodeActions/Basic.c @@ -41,7 +41,6 @@ lean_object* l_Lean_Json_mkObj(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_CodeAction_getFileSource_x21___closed__2; lean_object* l_Lean_ConstantInfo_type(lean_object*); -lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_fromJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_125____closed__11; LEAN_EXPORT lean_object* l_Lean_Server_instFromJsonCodeActionResolveData; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____closed__20; @@ -209,6 +208,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_handleCodeActionResolve___closed__3; static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____closed__21; +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__2___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517_(lean_object*); static lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____closed__14; @@ -423,7 +423,7 @@ x_24 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_24, 0, x_7); lean_ctor_set(x_24, 1, x_23); x_25 = l___private_Lean_Server_CodeActions_Basic_0__Lean_Server_toJsonCodeActionResolveData____x40_Lean_Server_CodeActions_Basic___hyg_59____closed__5; -x_26 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_24, x_25); +x_26 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_24, x_25); x_27 = l_Lean_Json_mkObj(x_26); return x_27; } @@ -1475,6 +1475,8 @@ x_17 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_17, 0, x_15); lean_ctor_set(x_17, 1, x_16); x_18 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_17, x_4, x_5, x_9); +lean_dec(x_5); +lean_dec(x_4); x_19 = !lean_is_exclusive(x_18); if (x_19 == 0) { @@ -1506,6 +1508,8 @@ return x_24; else { uint8_t x_25; +lean_dec(x_5); +lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); x_25 = !lean_is_exclusive(x_7); @@ -1574,6 +1578,7 @@ x_16 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_16, 0, x_14); lean_ctor_set(x_16, 1, x_15); x_17 = l_Lean_throwError___at_Lean_registerTagAttribute___spec__1(x_16, x_5, x_6, x_9); +lean_dec(x_6); lean_dec(x_5); x_18 = !lean_is_exclusive(x_17); if (x_18 == 0) @@ -1599,13 +1604,13 @@ else lean_object* x_22; lean_object* x_23; x_22 = lean_box(0); x_23 = l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__2(x_2, x_1, x_22, x_5, x_6, x_9); -lean_dec(x_5); return x_23; } } else { uint8_t x_24; +lean_dec(x_6); lean_dec(x_5); lean_dec(x_2); lean_dec(x_1); @@ -2166,8 +2171,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Bas { lean_object* x_6; x_6 = l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__1(x_1, x_2, x_3, x_4, x_5); -lean_dec(x_4); -lean_dec(x_3); lean_dec(x_2); return x_6; } @@ -2177,8 +2180,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Bas { lean_object* x_7; x_7 = l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6); -lean_dec(x_5); -lean_dec(x_4); lean_dec(x_3); return x_7; } @@ -2190,7 +2191,6 @@ uint8_t x_8; lean_object* x_9; x_8 = lean_unbox(x_4); lean_dec(x_4); x_9 = l_Lean_Server_initFn____x40_Lean_Server_CodeActions_Basic___hyg_517____lambda__3(x_1, x_2, x_3, x_8, x_5, x_6, x_7); -lean_dec(x_6); return x_9; } } diff --git a/stage0/stdlib/Lean/Server/Completion.c b/stage0/stdlib/Lean/Server/Completion.c index 1418b57b0551..464040b6b82a 100644 --- a/stage0/stdlib/Lean/Server/Completion.c +++ b/stage0/stdlib/Lean/Server/Completion.c @@ -16,136 +16,135 @@ extern "C" { static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__6; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2___boxed__const__1; lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; uint32_t lean_string_utf8_get(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__3(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__30; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__3___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__31; extern lean_object* l_Lean_Lsp_instHashableMarkupContent; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(lean_object*, size_t, size_t, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__3; uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(lean_object*, lean_object*); static lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___closed__1; uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); lean_object* l_Array_instBEq___rarg___boxed(lean_object*, lean_object*, lean_object*); +static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1; size_t lean_uint64_to_usize(uint64_t); lean_object* l_Lean_Server_Completion_idCompletion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__21; lean_object* l_Lean_Server_Completion_optionCompletion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___lambda__1(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___lambda__1___boxed(lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__20; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__2; lean_object* lean_array_fget(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Lsp_instDecidableEqCompletionItemKind___boxed(lean_object*, lean_object*); +static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__22; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(lean_object*, lean_object*); uint8_t lean_float_decLt(double, double); uint64_t l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1704_(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint64_t lean_string_hash(lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); lean_object* lean_string_utf8_set(lean_object*, lean_object*, uint32_t); lean_object* l_Std_DHashMap_Internal_AssocList_map_go___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__25; uint8_t lean_string_dec_eq(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(lean_object*); lean_object* l_instBEqProd___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__19; -static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2___boxed(lean_object*, lean_object*); lean_object* l_instHashableArray___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(size_t, size_t, lean_object*); size_t lean_usize_of_nat(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(lean_object*, size_t, size_t, lean_object*); uint8_t lean_string_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__1___lambda__1(lean_object*, lean_object*, lean_object*); lean_object* l_Char_toLower(uint32_t); -static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1; LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___lambda__1(lean_object*, lean_object*); lean_object* lean_string_utf8_next(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instHashableInsertReplaceEdit; LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___lambda__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__15; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12___boxed(lean_object*); lean_object* lean_string_mk(lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__12; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__1___closed__1; +static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___lambda__1___boxed(lean_object*, lean_object*); lean_object* l_outOfBounds___rarg(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___boxed(lean_object*); extern lean_object* l_instHashableString; +static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1; +static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3; LEAN_EXPORT lean_object* l_Array_mapFinIdxM_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__1; -static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3; lean_object* l_Lean_Server_Completion_tacticCompletion(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__13; LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts(lean_object*); uint8_t lean_string_utf8_at_end(lean_object*, lean_object*); -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(lean_object*, size_t, size_t, uint64_t); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__10; uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(lean_object*, lean_object*); lean_object* l_panic___at_String_fromUTF8_x21___spec__1(lean_object*); lean_object* l_List_replicateTR___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_String_mapAux___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__1(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__33; -static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__9; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__7; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(lean_object*, lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems(lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__29; +LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(lean_object*, size_t, size_t, uint64_t); extern lean_object* l_Lean_Lsp_instInhabitedCompletionItem; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3___boxed(lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems(lean_object*); +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Lsp_instDecidableEqCompletionItemTag___boxed(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__16; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__26; lean_object* l_Array_append___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(size_t, size_t, lean_object*); -static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(lean_object*, size_t, size_t, lean_object*); uint64_t l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(lean_object*); extern lean_object* l_Lean_Lsp_instHashableCompletionItemKind; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__27; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____rarg(lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(lean_object*, lean_object*); +static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; +static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__5; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__1___lambda__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_instHashableOption___rarg___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19(lean_object*, size_t, size_t, lean_object*); lean_object* lean_string_length(lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__8; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7(lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__24; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___lambda__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -158,26 +157,27 @@ LEAN_EXPORT lean_object* l_Lean_Server_Completion_find_x3f(lean_object*, lean_ob LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__18; lean_object* lean_nat_mul(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10___boxed(lean_object*); uint64_t l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1169_(uint8_t); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__17; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__14; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(lean_object*, lean_object*); extern lean_object* l_Lean_Server_Completion_instInhabitedScoredCompletionItem; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__32; size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); lean_object* l_Lean_Server_Completion_findPrioritizedCompletionPartitionsAt(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_Completion_dotCompletion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8(lean_object*); size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__23; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_assignSortTexts___spec__2(lean_object*, size_t, size_t, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); lean_object* l_Lean_Server_Completion_dotIdCompletion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Lsp_instDecidableEqMarkupContent___boxed(lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); @@ -185,183 +185,20 @@ LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completio uint8_t lean_nat_dec_le(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); lean_object* l_Lean_Server_Completion_fieldIdCompletion(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instBEqInsertReplaceEdit; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8(lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__4; extern lean_object* l_Lean_Lsp_instHashableCompletionItemTag; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); lean_object* l___private_Init_Data_Repr_0__Nat_reprFast(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1(lean_object*, lean_object*); lean_object* l_instDecidableEqString___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); +static lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2; uint8_t l_Array_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -lean_dec(x_1); -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -x_6 = lean_ctor_get(x_2, 2); -lean_inc(x_6); -lean_dec(x_2); -x_7 = lean_ctor_get(x_4, 0); -lean_inc(x_7); -x_8 = lean_ctor_get(x_4, 1); -lean_inc(x_8); -lean_dec(x_4); -x_9 = lean_ctor_get(x_1, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_1, 1); -lean_inc(x_10); -x_11 = lean_string_dec_eq(x_7, x_9); -lean_dec(x_9); -lean_dec(x_7); -if (x_11 == 0) -{ -lean_dec(x_10); -lean_dec(x_8); -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_13 = lean_ctor_get(x_8, 0); -lean_inc(x_13); -x_14 = lean_ctor_get(x_8, 1); -lean_inc(x_14); -lean_dec(x_8); -x_15 = lean_ctor_get(x_10, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_10, 1); -lean_inc(x_16); -lean_dec(x_10); -x_17 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_13, x_15); -lean_dec(x_15); -lean_dec(x_13); -if (x_17 == 0) -{ -lean_dec(x_16); -lean_dec(x_14); -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; -x_19 = lean_ctor_get(x_14, 0); -lean_inc(x_19); -x_20 = lean_ctor_get(x_14, 1); -lean_inc(x_20); -lean_dec(x_14); -x_21 = lean_ctor_get(x_16, 0); -lean_inc(x_21); -x_22 = lean_ctor_get(x_16, 1); -lean_inc(x_22); -lean_dec(x_16); -x_23 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_19, x_21); -lean_dec(x_21); -lean_dec(x_19); -if (x_23 == 0) -{ -lean_dec(x_22); -lean_dec(x_20); -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; -x_25 = lean_ctor_get(x_20, 0); -lean_inc(x_25); -x_26 = lean_ctor_get(x_20, 1); -lean_inc(x_26); -lean_dec(x_20); -x_27 = lean_ctor_get(x_22, 0); -lean_inc(x_27); -x_28 = lean_ctor_get(x_22, 1); -lean_inc(x_28); -lean_dec(x_22); -x_29 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_25, x_27); -if (x_29 == 0) -{ -lean_dec(x_28); -lean_dec(x_26); -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_31 = lean_ctor_get(x_26, 0); -lean_inc(x_31); -x_32 = lean_ctor_get(x_26, 1); -lean_inc(x_32); -lean_dec(x_26); -x_33 = lean_ctor_get(x_28, 0); -lean_inc(x_33); -x_34 = lean_ctor_get(x_28, 1); -lean_inc(x_34); -lean_dec(x_28); -x_35 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_31, x_33); -lean_dec(x_33); -lean_dec(x_31); -if (x_35 == 0) -{ -lean_dec(x_34); -lean_dec(x_32); -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -uint8_t x_37; -x_37 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_32, x_34); -lean_dec(x_34); -lean_dec(x_32); -if (x_37 == 0) -{ -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_39; -lean_dec(x_6); -lean_dec(x_1); -x_39 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_39, 0, x_5); -return x_39; -} -} -} -} -} -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -515,7 +352,7 @@ return x_38; } } } -LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(lean_object* x_1, size_t x_2, size_t x_3, uint64_t x_4) { +LEAN_EXPORT uint64_t l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(lean_object* x_1, size_t x_2, size_t x_3, uint64_t x_4) { _start: { uint8_t x_5; @@ -537,7 +374,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -620,7 +457,7 @@ goto _start; } } } -static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1() { +static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1() { _start: { uint64_t x_1; uint64_t x_2; @@ -629,7 +466,7 @@ x_2 = lean_uint64_mix_hash(x_1, x_1); return x_2; } } -static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2() { +static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2() { _start: { uint64_t x_1; uint64_t x_2; uint64_t x_3; @@ -639,17 +476,17 @@ x_3 = lean_uint64_mix_hash(x_1, x_2); return x_3; } } -static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3() { +static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3() { _start: { uint64_t x_1; uint64_t x_2; uint64_t x_3; x_1 = 11; -x_2 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; +x_2 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; x_3 = lean_uint64_mix_hash(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -828,7 +665,7 @@ if (lean_obj_tag(x_33) == 0) if (lean_obj_tag(x_34) == 0) { uint64_t x_35; uint64_t x_36; uint64_t x_37; uint64_t x_38; uint64_t x_39; -x_35 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1; +x_35 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1; x_36 = lean_uint64_mix_hash(x_32, x_35); x_37 = lean_uint64_mix_hash(x_31, x_36); x_38 = lean_uint64_mix_hash(x_28, x_37); @@ -874,7 +711,7 @@ lean_dec(x_50); if (lean_obj_tag(x_34) == 0) { uint64_t x_56; uint64_t x_57; uint64_t x_58; uint64_t x_59; uint64_t x_60; -x_56 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3; +x_56 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3; x_57 = lean_uint64_mix_hash(x_32, x_56); x_58 = lean_uint64_mix_hash(x_31, x_57); x_59 = lean_uint64_mix_hash(x_28, x_58); @@ -891,7 +728,7 @@ lean_dec(x_34); x_62 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_61); lean_dec(x_61); x_63 = lean_uint64_mix_hash(x_62, x_55); -x_64 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; +x_64 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; x_65 = lean_uint64_mix_hash(x_64, x_63); x_66 = lean_uint64_mix_hash(x_32, x_65); x_67 = lean_uint64_mix_hash(x_31, x_66); @@ -912,7 +749,7 @@ lean_dec(x_50); if (lean_obj_tag(x_34) == 0) { uint64_t x_71; uint64_t x_72; uint64_t x_73; uint64_t x_74; uint64_t x_75; -x_71 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3; +x_71 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3; x_72 = lean_uint64_mix_hash(x_32, x_71); x_73 = lean_uint64_mix_hash(x_31, x_72); x_74 = lean_uint64_mix_hash(x_28, x_73); @@ -929,7 +766,7 @@ lean_dec(x_34); x_77 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_76); lean_dec(x_76); x_78 = lean_uint64_mix_hash(x_77, x_55); -x_79 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; +x_79 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; x_80 = lean_uint64_mix_hash(x_79, x_78); x_81 = lean_uint64_mix_hash(x_32, x_80); x_82 = lean_uint64_mix_hash(x_31, x_81); @@ -945,7 +782,7 @@ size_t x_85; size_t x_86; uint64_t x_87; uint64_t x_88; x_85 = 0; x_86 = lean_usize_of_nat(x_52); lean_dec(x_52); -x_87 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(x_50, x_85, x_86, x_51); +x_87 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(x_50, x_85, x_86, x_51); lean_dec(x_50); x_88 = lean_uint64_mix_hash(x_87, x_55); if (lean_obj_tag(x_34) == 0) @@ -986,7 +823,7 @@ goto block_24; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -1005,7 +842,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -1016,7 +853,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -1027,167 +864,200 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_4; -lean_dec(x_2); -lean_dec(x_1); +lean_object* x_4; lean_object* x_5; x_4 = lean_box(0); -return x_4; +x_5 = lean_apply_1(x_2, x_4); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; } else { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_6 = lean_ctor_get(x_3, 0); -x_7 = lean_ctor_get(x_3, 1); -x_8 = lean_ctor_get(x_3, 2); -x_9 = lean_ctor_get(x_6, 0); -lean_inc(x_9); -x_10 = lean_ctor_get(x_6, 1); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 0); -lean_inc(x_11); -x_12 = lean_ctor_get(x_1, 1); -lean_inc(x_12); -x_13 = lean_string_dec_eq(x_9, x_11); -lean_dec(x_11); -lean_dec(x_9); -if (x_13 == 0) -{ -lean_object* x_14; -lean_dec(x_12); -lean_dec(x_10); -x_14 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_14); -return x_3; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_7); +lean_ctor_set(x_9, 2, x_8); +return x_9; +} } else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_15 = lean_ctor_get(x_10, 0); +uint8_t x_10; +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +x_13 = lean_ctor_get(x_3, 2); +x_14 = lean_ctor_get(x_11, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_11, 1); lean_inc(x_15); -x_16 = lean_ctor_get(x_10, 1); +x_16 = lean_ctor_get(x_1, 0); lean_inc(x_16); -lean_dec(x_10); -x_17 = lean_ctor_get(x_12, 0); +x_17 = lean_ctor_get(x_1, 1); lean_inc(x_17); -x_18 = lean_ctor_get(x_12, 1); -lean_inc(x_18); -lean_dec(x_12); -x_19 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_15, x_17); +x_18 = lean_string_dec_eq(x_14, x_16); +lean_dec(x_16); +lean_dec(x_14); +if (x_18 == 0) +{ +lean_object* x_19; lean_dec(x_17); lean_dec(x_15); -if (x_19 == 0) -{ -lean_object* x_20; -lean_dec(x_18); -lean_dec(x_16); -x_20 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_20); +x_19 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_19); return x_3; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; uint8_t x_25; -x_21 = lean_ctor_get(x_16, 0); +lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; +x_20 = lean_ctor_get(x_15, 0); +lean_inc(x_20); +x_21 = lean_ctor_get(x_15, 1); lean_inc(x_21); -x_22 = lean_ctor_get(x_16, 1); +lean_dec(x_15); +x_22 = lean_ctor_get(x_17, 0); lean_inc(x_22); -lean_dec(x_16); -x_23 = lean_ctor_get(x_18, 0); +x_23 = lean_ctor_get(x_17, 1); lean_inc(x_23); -x_24 = lean_ctor_get(x_18, 1); -lean_inc(x_24); -lean_dec(x_18); -x_25 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_21, x_23); +lean_dec(x_17); +x_24 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_20, x_22); +lean_dec(x_22); +lean_dec(x_20); +if (x_24 == 0) +{ +lean_object* x_25; lean_dec(x_23); lean_dec(x_21); -if (x_25 == 0) -{ -lean_object* x_26; -lean_dec(x_24); -lean_dec(x_22); -x_26 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_26); +x_25 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_25); return x_3; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; -x_27 = lean_ctor_get(x_22, 0); +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_21, 0); +lean_inc(x_26); +x_27 = lean_ctor_get(x_21, 1); lean_inc(x_27); -x_28 = lean_ctor_get(x_22, 1); +lean_dec(x_21); +x_28 = lean_ctor_get(x_23, 0); lean_inc(x_28); -lean_dec(x_22); -x_29 = lean_ctor_get(x_24, 0); +x_29 = lean_ctor_get(x_23, 1); lean_inc(x_29); -x_30 = lean_ctor_get(x_24, 1); -lean_inc(x_30); -lean_dec(x_24); -x_31 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_27, x_29); -if (x_31 == 0) -{ -lean_object* x_32; -lean_dec(x_30); +lean_dec(x_23); +x_30 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_26, x_28); lean_dec(x_28); -x_32 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_32); +lean_dec(x_26); +if (x_30 == 0) +{ +lean_object* x_31; +lean_dec(x_29); +lean_dec(x_27); +x_31 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_31); return x_3; } else { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; -x_33 = lean_ctor_get(x_28, 0); +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; +x_32 = lean_ctor_get(x_27, 0); +lean_inc(x_32); +x_33 = lean_ctor_get(x_27, 1); lean_inc(x_33); -x_34 = lean_ctor_get(x_28, 1); +lean_dec(x_27); +x_34 = lean_ctor_get(x_29, 0); lean_inc(x_34); -lean_dec(x_28); -x_35 = lean_ctor_get(x_30, 0); +x_35 = lean_ctor_get(x_29, 1); lean_inc(x_35); -x_36 = lean_ctor_get(x_30, 1); -lean_inc(x_36); -lean_dec(x_30); -x_37 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_33, x_35); +lean_dec(x_29); +x_36 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_32, x_34); +if (x_36 == 0) +{ +lean_object* x_37; lean_dec(x_35); lean_dec(x_33); -if (x_37 == 0) +x_37 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_37); +return x_3; +} +else { -lean_object* x_38; -lean_dec(x_36); -lean_dec(x_34); -x_38 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_38); +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_38 = lean_ctor_get(x_33, 0); +lean_inc(x_38); +x_39 = lean_ctor_get(x_33, 1); +lean_inc(x_39); +lean_dec(x_33); +x_40 = lean_ctor_get(x_35, 0); +lean_inc(x_40); +x_41 = lean_ctor_get(x_35, 1); +lean_inc(x_41); +lean_dec(x_35); +x_42 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_38, x_40); +lean_dec(x_40); +lean_dec(x_38); +if (x_42 == 0) +{ +lean_object* x_43; +lean_dec(x_41); +lean_dec(x_39); +x_43 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_43); return x_3; } else { -uint8_t x_39; -x_39 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_34, x_36); -lean_dec(x_36); -lean_dec(x_34); -if (x_39 == 0) +uint8_t x_44; +x_44 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_39, x_41); +lean_dec(x_41); +lean_dec(x_39); +if (x_44 == 0) { -lean_object* x_40; -x_40 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_40); +lean_object* x_45; +x_45 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_45); return x_3; } else { -lean_dec(x_7); -lean_dec(x_6); -lean_ctor_set(x_3, 1, x_2); +lean_object* x_46; lean_object* x_47; +lean_dec(x_11); +x_46 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_46, 0, x_12); +x_47 = lean_apply_1(x_2, x_46); +if (lean_obj_tag(x_47) == 0) +{ +lean_free_object(x_3); +lean_dec(x_1); +return x_13; +} +else +{ +lean_object* x_48; +x_48 = lean_ctor_get(x_47, 0); +lean_inc(x_48); +lean_dec(x_47); +lean_ctor_set(x_3, 1, x_48); lean_ctor_set(x_3, 0, x_1); return x_3; } @@ -1197,175 +1067,189 @@ return x_3; } } } -else -{ -lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_41 = lean_ctor_get(x_3, 0); -x_42 = lean_ctor_get(x_3, 1); -x_43 = lean_ctor_get(x_3, 2); -lean_inc(x_43); -lean_inc(x_42); -lean_inc(x_41); -lean_dec(x_3); -x_44 = lean_ctor_get(x_41, 0); -lean_inc(x_44); -x_45 = lean_ctor_get(x_41, 1); -lean_inc(x_45); -x_46 = lean_ctor_get(x_1, 0); -lean_inc(x_46); -x_47 = lean_ctor_get(x_1, 1); -lean_inc(x_47); -x_48 = lean_string_dec_eq(x_44, x_46); -lean_dec(x_46); -lean_dec(x_44); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; -lean_dec(x_47); -lean_dec(x_45); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_50 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_50, 0, x_41); -lean_ctor_set(x_50, 1, x_42); -lean_ctor_set(x_50, 2, x_49); -return x_50; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_55; -x_51 = lean_ctor_get(x_45, 0); +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; +x_49 = lean_ctor_get(x_3, 0); +x_50 = lean_ctor_get(x_3, 1); +x_51 = lean_ctor_get(x_3, 2); lean_inc(x_51); -x_52 = lean_ctor_get(x_45, 1); -lean_inc(x_52); -lean_dec(x_45); -x_53 = lean_ctor_get(x_47, 0); +lean_inc(x_50); +lean_inc(x_49); +lean_dec(x_3); +x_52 = lean_ctor_get(x_49, 0); +lean_inc(x_52); +x_53 = lean_ctor_get(x_49, 1); lean_inc(x_53); -x_54 = lean_ctor_get(x_47, 1); +x_54 = lean_ctor_get(x_1, 0); lean_inc(x_54); -lean_dec(x_47); -x_55 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_51, x_53); -lean_dec(x_53); -lean_dec(x_51); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; +x_55 = lean_ctor_get(x_1, 1); +lean_inc(x_55); +x_56 = lean_string_dec_eq(x_52, x_54); lean_dec(x_54); lean_dec(x_52); -x_56 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_57 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_57, 0, x_41); -lean_ctor_set(x_57, 1, x_42); -lean_ctor_set(x_57, 2, x_56); -return x_57; +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; +lean_dec(x_55); +lean_dec(x_53); +x_57 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_58 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_58, 0, x_49); +lean_ctor_set(x_58, 1, x_50); +lean_ctor_set(x_58, 2, x_57); +return x_58; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; -x_58 = lean_ctor_get(x_52, 0); -lean_inc(x_58); -x_59 = lean_ctor_get(x_52, 1); +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; uint8_t x_63; +x_59 = lean_ctor_get(x_53, 0); lean_inc(x_59); -lean_dec(x_52); -x_60 = lean_ctor_get(x_54, 0); +x_60 = lean_ctor_get(x_53, 1); lean_inc(x_60); -x_61 = lean_ctor_get(x_54, 1); +lean_dec(x_53); +x_61 = lean_ctor_get(x_55, 0); lean_inc(x_61); -lean_dec(x_54); -x_62 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_58, x_60); -lean_dec(x_60); -lean_dec(x_58); -if (x_62 == 0) -{ -lean_object* x_63; lean_object* x_64; +x_62 = lean_ctor_get(x_55, 1); +lean_inc(x_62); +lean_dec(x_55); +x_63 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_59, x_61); lean_dec(x_61); lean_dec(x_59); -x_63 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_41); -lean_ctor_set(x_64, 1, x_42); -lean_ctor_set(x_64, 2, x_63); -return x_64; +if (x_63 == 0) +{ +lean_object* x_64; lean_object* x_65; +lean_dec(x_62); +lean_dec(x_60); +x_64 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_65 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_65, 0, x_49); +lean_ctor_set(x_65, 1, x_50); +lean_ctor_set(x_65, 2, x_64); +return x_65; } else { -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; -x_65 = lean_ctor_get(x_59, 0); -lean_inc(x_65); -x_66 = lean_ctor_get(x_59, 1); +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_66 = lean_ctor_get(x_60, 0); lean_inc(x_66); -lean_dec(x_59); -x_67 = lean_ctor_get(x_61, 0); +x_67 = lean_ctor_get(x_60, 1); lean_inc(x_67); -x_68 = lean_ctor_get(x_61, 1); +lean_dec(x_60); +x_68 = lean_ctor_get(x_62, 0); lean_inc(x_68); -lean_dec(x_61); -x_69 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_65, x_67); -if (x_69 == 0) -{ -lean_object* x_70; lean_object* x_71; +x_69 = lean_ctor_get(x_62, 1); +lean_inc(x_69); +lean_dec(x_62); +x_70 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_66, x_68); lean_dec(x_68); lean_dec(x_66); -x_70 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_71 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_71, 0, x_41); -lean_ctor_set(x_71, 1, x_42); -lean_ctor_set(x_71, 2, x_70); -return x_71; +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; +lean_dec(x_69); +lean_dec(x_67); +x_71 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_49); +lean_ctor_set(x_72, 1, x_50); +lean_ctor_set(x_72, 2, x_71); +return x_72; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_72 = lean_ctor_get(x_66, 0); -lean_inc(x_72); -x_73 = lean_ctor_get(x_66, 1); +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; +x_73 = lean_ctor_get(x_67, 0); lean_inc(x_73); -lean_dec(x_66); -x_74 = lean_ctor_get(x_68, 0); +x_74 = lean_ctor_get(x_67, 1); lean_inc(x_74); -x_75 = lean_ctor_get(x_68, 1); +lean_dec(x_67); +x_75 = lean_ctor_get(x_69, 0); lean_inc(x_75); -lean_dec(x_68); -x_76 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_72, x_74); -lean_dec(x_74); -lean_dec(x_72); -if (x_76 == 0) +x_76 = lean_ctor_get(x_69, 1); +lean_inc(x_76); +lean_dec(x_69); +x_77 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_73, x_75); +if (x_77 == 0) { -lean_object* x_77; lean_object* x_78; -lean_dec(x_75); -lean_dec(x_73); -x_77 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_78 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_78, 0, x_41); -lean_ctor_set(x_78, 1, x_42); -lean_ctor_set(x_78, 2, x_77); -return x_78; +lean_object* x_78; lean_object* x_79; +lean_dec(x_76); +lean_dec(x_74); +x_78 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_79 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_79, 0, x_49); +lean_ctor_set(x_79, 1, x_50); +lean_ctor_set(x_79, 2, x_78); +return x_79; } else { -uint8_t x_79; -x_79 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_73, x_75); -lean_dec(x_75); -lean_dec(x_73); -if (x_79 == 0) +lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +x_81 = lean_ctor_get(x_74, 1); +lean_inc(x_81); +lean_dec(x_74); +x_82 = lean_ctor_get(x_76, 0); +lean_inc(x_82); +x_83 = lean_ctor_get(x_76, 1); +lean_inc(x_83); +lean_dec(x_76); +x_84 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_80, x_82); +lean_dec(x_82); +lean_dec(x_80); +if (x_84 == 0) +{ +lean_object* x_85; lean_object* x_86; +lean_dec(x_83); +lean_dec(x_81); +x_85 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_86 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_86, 0, x_49); +lean_ctor_set(x_86, 1, x_50); +lean_ctor_set(x_86, 2, x_85); +return x_86; +} +else +{ +uint8_t x_87; +x_87 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_81, x_83); +lean_dec(x_83); +lean_dec(x_81); +if (x_87 == 0) +{ +lean_object* x_88; lean_object* x_89; +x_88 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_1, x_2, x_51); +x_89 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_89, 0, x_49); +lean_ctor_set(x_89, 1, x_50); +lean_ctor_set(x_89, 2, x_88); +return x_89; +} +else +{ +lean_object* x_90; lean_object* x_91; +lean_dec(x_49); +x_90 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_90, 0, x_50); +x_91 = lean_apply_1(x_2, x_90); +if (lean_obj_tag(x_91) == 0) { -lean_object* x_80; lean_object* x_81; -x_80 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_43); -x_81 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_81, 0, x_41); -lean_ctor_set(x_81, 1, x_42); -lean_ctor_set(x_81, 2, x_80); -return x_81; +lean_dec(x_1); +return x_51; } else { -lean_object* x_82; -lean_dec(x_42); -lean_dec(x_41); -x_82 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_82, 0, x_1); -lean_ctor_set(x_82, 1, x_2); -lean_ctor_set(x_82, 2, x_43); -return x_82; +lean_object* x_92; lean_object* x_93; +x_92 = lean_ctor_get(x_91, 0); +lean_inc(x_92); +lean_dec(x_91); +x_93 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_93, 0, x_1); +lean_ctor_set(x_93, 1, x_92); +lean_ctor_set(x_93, 2, x_51); +return x_93; } } } @@ -1376,356 +1260,63 @@ return x_82; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -lean_dec(x_1); -x_3 = lean_box(0); -return x_3; } -else -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = lean_ctor_get(x_5, 0); -lean_inc(x_8); -x_9 = lean_ctor_get(x_5, 1); -lean_inc(x_9); -x_10 = lean_ctor_get(x_1, 0); -lean_inc(x_10); -x_11 = lean_ctor_get(x_1, 1); -lean_inc(x_11); -x_12 = lean_string_dec_eq(x_8, x_10); -lean_dec(x_10); -lean_dec(x_8); -if (x_12 == 0) +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8(lean_object* x_1) { +_start: { -lean_object* x_13; -lean_dec(x_11); -lean_dec(x_9); -x_13 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_13); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg), 3, 0); return x_2; } -else -{ -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; -x_14 = lean_ctor_get(x_9, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_9, 1); -lean_inc(x_15); -lean_dec(x_9); -x_16 = lean_ctor_get(x_11, 0); -lean_inc(x_16); -x_17 = lean_ctor_get(x_11, 1); -lean_inc(x_17); -lean_dec(x_11); -x_18 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_14, x_16); -lean_dec(x_16); -lean_dec(x_14); -if (x_18 == 0) -{ -lean_object* x_19; -lean_dec(x_17); -lean_dec(x_15); -x_19 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_19); -return x_2; } -else -{ -lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; uint8_t x_24; -x_20 = lean_ctor_get(x_15, 0); -lean_inc(x_20); -x_21 = lean_ctor_get(x_15, 1); -lean_inc(x_21); -lean_dec(x_15); -x_22 = lean_ctor_get(x_17, 0); -lean_inc(x_22); -x_23 = lean_ctor_get(x_17, 1); -lean_inc(x_23); -lean_dec(x_17); -x_24 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_20, x_22); -lean_dec(x_22); -lean_dec(x_20); -if (x_24 == 0) +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1() { +_start: { -lean_object* x_25; -lean_dec(x_23); -lean_dec(x_21); -x_25 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_25); +lean_object* x_1; lean_object* x_2; +x_1 = lean_box(0); +x_2 = lean_array_mk(x_1); return x_2; } -else -{ -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; -x_26 = lean_ctor_get(x_21, 0); -lean_inc(x_26); -x_27 = lean_ctor_get(x_21, 1); -lean_inc(x_27); -lean_dec(x_21); -x_28 = lean_ctor_get(x_23, 0); -lean_inc(x_28); -x_29 = lean_ctor_get(x_23, 1); -lean_inc(x_29); -lean_dec(x_23); -x_30 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_26, x_28); -if (x_30 == 0) -{ -lean_object* x_31; -lean_dec(x_29); -lean_dec(x_27); -x_31 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_31); -return x_2; } -else +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; uint8_t x_36; -x_32 = lean_ctor_get(x_27, 0); -lean_inc(x_32); -x_33 = lean_ctor_get(x_27, 1); -lean_inc(x_33); -lean_dec(x_27); -x_34 = lean_ctor_get(x_29, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_29, 1); -lean_inc(x_35); -lean_dec(x_29); -x_36 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_32, x_34); -lean_dec(x_34); -lean_dec(x_32); -if (x_36 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_37; -lean_dec(x_35); -lean_dec(x_33); -x_37 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_37); -return x_2; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -uint8_t x_38; -x_38 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_33, x_35); -lean_dec(x_35); -lean_dec(x_33); -if (x_38 == 0) +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) { -lean_object* x_39; -x_39 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_7); -lean_ctor_set(x_2, 2, x_39); +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); return x_2; } else { -lean_free_object(x_2); -lean_dec(x_6); -lean_dec(x_5); -lean_dec(x_1); -return x_7; -} -} -} -} -} -} -} -else -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; -x_40 = lean_ctor_get(x_2, 0); -x_41 = lean_ctor_get(x_2, 1); -x_42 = lean_ctor_get(x_2, 2); -lean_inc(x_42); -lean_inc(x_41); -lean_inc(x_40); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); lean_dec(x_2); -x_43 = lean_ctor_get(x_40, 0); -lean_inc(x_43); -x_44 = lean_ctor_get(x_40, 1); -lean_inc(x_44); -x_45 = lean_ctor_get(x_1, 0); -lean_inc(x_45); -x_46 = lean_ctor_get(x_1, 1); -lean_inc(x_46); -x_47 = lean_string_dec_eq(x_43, x_45); -lean_dec(x_45); -lean_dec(x_43); -if (x_47 == 0) -{ -lean_object* x_48; lean_object* x_49; -lean_dec(x_46); -lean_dec(x_44); -x_48 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_49 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_49, 0, x_40); -lean_ctor_set(x_49, 1, x_41); -lean_ctor_set(x_49, 2, x_48); -return x_49; -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_50 = lean_ctor_get(x_44, 0); -lean_inc(x_50); -x_51 = lean_ctor_get(x_44, 1); -lean_inc(x_51); -lean_dec(x_44); -x_52 = lean_ctor_get(x_46, 0); -lean_inc(x_52); -x_53 = lean_ctor_get(x_46, 1); -lean_inc(x_53); -lean_dec(x_46); -x_54 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__4(x_50, x_52); -lean_dec(x_52); -lean_dec(x_50); -if (x_54 == 0) -{ -lean_object* x_55; lean_object* x_56; -lean_dec(x_53); -lean_dec(x_51); -x_55 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_56 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_56, 0, x_40); -lean_ctor_set(x_56, 1, x_41); -lean_ctor_set(x_56, 2, x_55); -return x_56; -} -else -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; -x_57 = lean_ctor_get(x_51, 0); -lean_inc(x_57); -x_58 = lean_ctor_get(x_51, 1); -lean_inc(x_58); -lean_dec(x_51); -x_59 = lean_ctor_get(x_53, 0); -lean_inc(x_59); -x_60 = lean_ctor_get(x_53, 1); -lean_inc(x_60); -lean_dec(x_53); -x_61 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(x_57, x_59); -lean_dec(x_59); -lean_dec(x_57); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; -lean_dec(x_60); -lean_dec(x_58); -x_62 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_63 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_63, 0, x_40); -lean_ctor_set(x_63, 1, x_41); -lean_ctor_set(x_63, 2, x_62); -return x_63; -} -else -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; -x_64 = lean_ctor_get(x_58, 0); -lean_inc(x_64); -x_65 = lean_ctor_get(x_58, 1); -lean_inc(x_65); -lean_dec(x_58); -x_66 = lean_ctor_get(x_60, 0); -lean_inc(x_66); -x_67 = lean_ctor_get(x_60, 1); -lean_inc(x_67); -lean_dec(x_60); -x_68 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__3(x_64, x_66); -if (x_68 == 0) -{ -lean_object* x_69; lean_object* x_70; -lean_dec(x_67); -lean_dec(x_65); -x_69 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_40); -lean_ctor_set(x_70, 1, x_41); -lean_ctor_set(x_70, 2, x_69); -return x_70; -} -else -{ -lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; -x_71 = lean_ctor_get(x_65, 0); -lean_inc(x_71); -x_72 = lean_ctor_get(x_65, 1); -lean_inc(x_72); -lean_dec(x_65); -x_73 = lean_ctor_get(x_67, 0); -lean_inc(x_73); -x_74 = lean_ctor_get(x_67, 1); -lean_inc(x_74); -lean_dec(x_67); -x_75 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__6(x_71, x_73); -lean_dec(x_73); -lean_dec(x_71); -if (x_75 == 0) -{ -lean_object* x_76; lean_object* x_77; -lean_dec(x_74); -lean_dec(x_72); -x_76 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_77 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_77, 0, x_40); -lean_ctor_set(x_77, 1, x_41); -lean_ctor_set(x_77, 2, x_76); -return x_77; -} -else -{ -uint8_t x_78; -x_78 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__2(x_72, x_74); -lean_dec(x_74); -lean_dec(x_72); -if (x_78 == 0) -{ -lean_object* x_79; lean_object* x_80; -x_79 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1, x_42); -x_80 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_80, 0, x_40); -lean_ctor_set(x_80, 1, x_41); -lean_ctor_set(x_80, 2, x_79); -return x_80; -} -else -{ -lean_dec(x_41); -lean_dec(x_40); -lean_dec(x_1); -return x_42; -} -} -} -} -} -} -} -} +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -1738,110 +1329,108 @@ return x_10; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; uint64_t x_23; lean_object* x_131; lean_object* x_132; uint64_t x_133; uint64_t x_134; lean_object* x_135; lean_object* x_136; lean_object* x_230; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; size_t x_21; size_t x_22; size_t x_23; uint64_t x_24; lean_object* x_65; lean_object* x_66; uint64_t x_67; uint64_t x_68; lean_object* x_69; lean_object* x_70; lean_object* x_164; x_12 = lean_array_uget(x_7, x_9); lean_inc(x_1); lean_inc(x_12); x_13 = lean_apply_1(x_1, x_12); -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +x_14 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1), 2, 1); +lean_closure_set(x_14, 0, x_12); +x_15 = lean_ctor_get(x_10, 0); lean_inc(x_15); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); if (lean_is_exclusive(x_10)) { lean_ctor_release(x_10, 0); lean_ctor_release(x_10, 1); - x_16 = x_10; + x_17 = x_10; } else { lean_dec_ref(x_10); - x_16 = lean_box(0); + x_17 = lean_box(0); } -x_17 = lean_array_get_size(x_15); -x_18 = 32; -x_19 = 16; -x_20 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_21 = 1; -x_22 = lean_usize_sub(x_20, x_21); -x_131 = lean_ctor_get(x_13, 0); -lean_inc(x_131); -x_132 = lean_ctor_get(x_13, 1); -lean_inc(x_132); -x_133 = lean_string_hash(x_131); -lean_dec(x_131); -x_230 = lean_ctor_get(x_132, 0); -lean_inc(x_230); -if (lean_obj_tag(x_230) == 0) -{ -lean_object* x_231; uint64_t x_232; lean_object* x_233; lean_object* x_234; -x_231 = lean_ctor_get(x_132, 1); -lean_inc(x_231); -lean_dec(x_132); -x_232 = 11; -x_233 = lean_ctor_get(x_231, 0); -lean_inc(x_233); -x_234 = lean_ctor_get(x_231, 1); -lean_inc(x_234); -lean_dec(x_231); -x_134 = x_232; -x_135 = x_233; -x_136 = x_234; -goto block_229; +x_18 = lean_array_get_size(x_16); +x_19 = 32; +x_20 = 16; +x_21 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_65 = lean_ctor_get(x_13, 0); +lean_inc(x_65); +x_66 = lean_ctor_get(x_13, 1); +lean_inc(x_66); +x_67 = lean_string_hash(x_65); +lean_dec(x_65); +x_164 = lean_ctor_get(x_66, 0); +lean_inc(x_164); +if (lean_obj_tag(x_164) == 0) +{ +lean_object* x_165; uint64_t x_166; lean_object* x_167; lean_object* x_168; +x_165 = lean_ctor_get(x_66, 1); +lean_inc(x_165); +lean_dec(x_66); +x_166 = 11; +x_167 = lean_ctor_get(x_165, 0); +lean_inc(x_167); +x_168 = lean_ctor_get(x_165, 1); +lean_inc(x_168); +lean_dec(x_165); +x_68 = x_166; +x_69 = x_167; +x_70 = x_168; +goto block_163; } else { -lean_object* x_235; lean_object* x_236; uint64_t x_237; uint64_t x_238; uint64_t x_239; lean_object* x_240; lean_object* x_241; -x_235 = lean_ctor_get(x_132, 1); -lean_inc(x_235); -lean_dec(x_132); -x_236 = lean_ctor_get(x_230, 0); -lean_inc(x_236); -lean_dec(x_230); -x_237 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1704_(x_236); -lean_dec(x_236); -x_238 = 13; -x_239 = lean_uint64_mix_hash(x_237, x_238); -x_240 = lean_ctor_get(x_235, 0); -lean_inc(x_240); -x_241 = lean_ctor_get(x_235, 1); -lean_inc(x_241); -lean_dec(x_235); -x_134 = x_239; -x_135 = x_240; -x_136 = x_241; -goto block_229; -} -block_130: -{ -uint64_t x_24; uint64_t x_25; uint64_t x_26; uint64_t x_27; size_t x_28; size_t x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_uint64_shift_right(x_23, x_18); -x_25 = lean_uint64_xor(x_23, x_24); -x_26 = lean_uint64_shift_right(x_25, x_19); -x_27 = lean_uint64_xor(x_25, x_26); -x_28 = lean_uint64_to_usize(x_27); -x_29 = lean_usize_land(x_28, x_22); -x_30 = lean_array_uget(x_15, x_29); -lean_inc(x_30); -lean_inc(x_13); -x_31 = l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(x_13, x_30); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_32 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; -x_33 = lean_array_push(x_32, x_12); -lean_inc(x_30); +lean_object* x_169; lean_object* x_170; uint64_t x_171; uint64_t x_172; uint64_t x_173; lean_object* x_174; lean_object* x_175; +x_169 = lean_ctor_get(x_66, 1); +lean_inc(x_169); +lean_dec(x_66); +x_170 = lean_ctor_get(x_164, 0); +lean_inc(x_170); +lean_dec(x_164); +x_171 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashInsertReplaceEdit____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1704_(x_170); +lean_dec(x_170); +x_172 = 13; +x_173 = lean_uint64_mix_hash(x_171, x_172); +x_174 = lean_ctor_get(x_169, 0); +lean_inc(x_174); +x_175 = lean_ctor_get(x_169, 1); +lean_inc(x_175); +lean_dec(x_169); +x_68 = x_173; +x_69 = x_174; +x_70 = x_175; +goto block_163; +} +block_64: +{ +uint64_t x_25; uint64_t x_26; uint64_t x_27; uint64_t x_28; size_t x_29; size_t x_30; lean_object* x_31; uint8_t x_32; +x_25 = lean_uint64_shift_right(x_24, x_19); +x_26 = lean_uint64_xor(x_24, x_25); +x_27 = lean_uint64_shift_right(x_26, x_20); +x_28 = lean_uint64_xor(x_26, x_27); +x_29 = lean_uint64_to_usize(x_28); +x_30 = lean_usize_land(x_29, x_23); +x_31 = lean_array_uget(x_16, x_30); +lean_inc(x_31); lean_inc(x_13); -x_34 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_13, x_30); -if (x_34 == 0) +x_32 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(x_13, x_31); +if (x_32 == 0) { -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_nat_add(x_14, x_35); +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_dec(x_14); +x_33 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; +x_34 = lean_array_push(x_33, x_12); +x_35 = lean_unsigned_to_nat(1u); +x_36 = lean_nat_add(x_15, x_35); +lean_dec(x_15); x_37 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_37, 0, x_13); -lean_ctor_set(x_37, 1, x_33); -lean_ctor_set(x_37, 2, x_30); -x_38 = lean_array_uset(x_15, x_29, x_37); +lean_ctor_set(x_37, 1, x_34); +lean_ctor_set(x_37, 2, x_31); +x_38 = lean_array_uset(x_16, x_30, x_37); x_39 = lean_unsigned_to_nat(4u); x_40 = lean_nat_mul(x_36, x_39); x_41 = lean_unsigned_to_nat(3u); @@ -1854,15 +1443,15 @@ lean_dec(x_42); if (x_44 == 0) { lean_object* x_45; lean_object* x_46; size_t x_47; -x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(x_38); -if (lean_is_scalar(x_16)) { +x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_38); +if (lean_is_scalar(x_17)) { x_46 = lean_alloc_ctor(0, 2, 0); } else { - x_46 = x_16; + x_46 = x_17; } lean_ctor_set(x_46, 0, x_36); lean_ctor_set(x_46, 1, x_45); -x_47 = lean_usize_add(x_9, x_21); +x_47 = lean_usize_add(x_9, x_22); x_9 = x_47; x_10 = x_46; goto _start; @@ -1870,14 +1459,14 @@ goto _start; else { lean_object* x_49; size_t x_50; -if (lean_is_scalar(x_16)) { +if (lean_is_scalar(x_17)) { x_49 = lean_alloc_ctor(0, 2, 0); } else { - x_49 = x_16; + x_49 = x_17; } lean_ctor_set(x_49, 0, x_36); lean_ctor_set(x_49, 1, x_38); -x_50 = lean_usize_add(x_9, x_21); +x_50 = lean_usize_add(x_9, x_22); x_9 = x_50; x_10 = x_49; goto _start; @@ -1885,447 +1474,274 @@ goto _start; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; size_t x_56; +lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; +lean_dec(x_12); lean_inc(x_5); -x_52 = lean_array_uset(x_15, x_29, x_5); -x_53 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_13, x_33, x_30); -x_54 = lean_array_uset(x_52, x_29, x_53); -if (lean_is_scalar(x_16)) { - x_55 = lean_alloc_ctor(0, 2, 0); -} else { - x_55 = x_16; -} -lean_ctor_set(x_55, 0, x_14); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_usize_add(x_9, x_21); -x_9 = x_56; -x_10 = x_55; -goto _start; -} -} -else -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_122; -x_58 = lean_ctor_get(x_31, 0); -lean_inc(x_58); -lean_dec(x_31); -x_59 = lean_array_push(x_58, x_12); -lean_inc(x_30); +x_52 = lean_array_uset(x_16, x_30, x_5); lean_inc(x_13); -x_122 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_13, x_30); -if (x_122 == 0) +x_53 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___rarg(x_13, x_14, x_31); +lean_inc(x_53); +x_54 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(x_13, x_53); +x_55 = lean_array_uset(x_52, x_30, x_53); +if (x_54 == 0) { -lean_object* x_123; -lean_dec(x_30); -if (lean_is_scalar(x_16)) { - x_123 = lean_alloc_ctor(0, 2, 0); +lean_object* x_56; lean_object* x_57; lean_object* x_58; size_t x_59; +x_56 = lean_unsigned_to_nat(1u); +x_57 = lean_nat_sub(x_15, x_56); +lean_dec(x_15); +if (lean_is_scalar(x_17)) { + x_58 = lean_alloc_ctor(0, 2, 0); } else { - x_123 = x_16; + x_58 = x_17; } -lean_ctor_set(x_123, 0, x_14); -lean_ctor_set(x_123, 1, x_15); -x_60 = x_123; -goto block_121; +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_55); +x_59 = lean_usize_add(x_9, x_22); +x_9 = x_59; +x_10 = x_58; +goto _start; } else { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -lean_inc(x_5); -x_124 = lean_array_uset(x_15, x_29, x_5); -x_125 = lean_unsigned_to_nat(1u); -x_126 = lean_nat_sub(x_14, x_125); -lean_dec(x_14); -lean_inc(x_13); -x_127 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_13, x_30); -x_128 = lean_array_uset(x_124, x_29, x_127); -if (lean_is_scalar(x_16)) { - x_129 = lean_alloc_ctor(0, 2, 0); +lean_object* x_61; size_t x_62; +if (lean_is_scalar(x_17)) { + x_61 = lean_alloc_ctor(0, 2, 0); } else { - x_129 = x_16; -} -lean_ctor_set(x_129, 0, x_126); -lean_ctor_set(x_129, 1, x_128); -x_60 = x_129; -goto block_121; -} -block_121: -{ -uint8_t x_61; -x_61 = !lean_is_exclusive(x_60); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; size_t x_65; size_t x_66; size_t x_67; lean_object* x_68; uint8_t x_69; -x_62 = lean_ctor_get(x_60, 0); -x_63 = lean_ctor_get(x_60, 1); -x_64 = lean_array_get_size(x_63); -x_65 = lean_usize_of_nat(x_64); -lean_dec(x_64); -x_66 = lean_usize_sub(x_65, x_21); -x_67 = lean_usize_land(x_28, x_66); -x_68 = lean_array_uget(x_63, x_67); -lean_inc(x_68); -lean_inc(x_13); -x_69 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_13, x_68); -if (x_69 == 0) -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; -x_70 = lean_unsigned_to_nat(1u); -x_71 = lean_nat_add(x_62, x_70); -lean_dec(x_62); -x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_13); -lean_ctor_set(x_72, 1, x_59); -lean_ctor_set(x_72, 2, x_68); -x_73 = lean_array_uset(x_63, x_67, x_72); -x_74 = lean_unsigned_to_nat(4u); -x_75 = lean_nat_mul(x_71, x_74); -x_76 = lean_unsigned_to_nat(3u); -x_77 = lean_nat_div(x_75, x_76); -lean_dec(x_75); -x_78 = lean_array_get_size(x_73); -x_79 = lean_nat_dec_le(x_77, x_78); -lean_dec(x_78); -lean_dec(x_77); -if (x_79 == 0) -{ -lean_object* x_80; size_t x_81; -x_80 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(x_73); -lean_ctor_set(x_60, 1, x_80); -lean_ctor_set(x_60, 0, x_71); -x_81 = lean_usize_add(x_9, x_21); -x_9 = x_81; -x_10 = x_60; -goto _start; + x_61 = x_17; } -else -{ -size_t x_83; -lean_ctor_set(x_60, 1, x_73); -lean_ctor_set(x_60, 0, x_71); -x_83 = lean_usize_add(x_9, x_21); -x_9 = x_83; -x_10 = x_60; +lean_ctor_set(x_61, 0, x_15); +lean_ctor_set(x_61, 1, x_55); +x_62 = lean_usize_add(x_9, x_22); +x_9 = x_62; +x_10 = x_61; goto _start; } } -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; size_t x_88; -lean_inc(x_5); -x_85 = lean_array_uset(x_63, x_67, x_5); -x_86 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_13, x_59, x_68); -x_87 = lean_array_uset(x_85, x_67, x_86); -lean_ctor_set(x_60, 1, x_87); -x_88 = lean_usize_add(x_9, x_21); -x_9 = x_88; -x_10 = x_60; -goto _start; -} } -else +block_163: { -lean_object* x_90; lean_object* x_91; lean_object* x_92; size_t x_93; size_t x_94; size_t x_95; lean_object* x_96; uint8_t x_97; -x_90 = lean_ctor_get(x_60, 0); -x_91 = lean_ctor_get(x_60, 1); -lean_inc(x_91); -lean_inc(x_90); -lean_dec(x_60); -x_92 = lean_array_get_size(x_91); -x_93 = lean_usize_of_nat(x_92); -lean_dec(x_92); -x_94 = lean_usize_sub(x_93, x_21); -x_95 = lean_usize_land(x_28, x_94); -x_96 = lean_array_uget(x_91, x_95); -lean_inc(x_96); -lean_inc(x_13); -x_97 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_13, x_96); -if (x_97 == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; -x_98 = lean_unsigned_to_nat(1u); -x_99 = lean_nat_add(x_90, x_98); -lean_dec(x_90); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_13); -lean_ctor_set(x_100, 1, x_59); -lean_ctor_set(x_100, 2, x_96); -x_101 = lean_array_uset(x_91, x_95, x_100); -x_102 = lean_unsigned_to_nat(4u); -x_103 = lean_nat_mul(x_99, x_102); -x_104 = lean_unsigned_to_nat(3u); -x_105 = lean_nat_div(x_103, x_104); -lean_dec(x_103); -x_106 = lean_array_get_size(x_101); -x_107 = lean_nat_dec_le(x_105, x_106); -lean_dec(x_106); -lean_dec(x_105); -if (x_107 == 0) -{ -lean_object* x_108; lean_object* x_109; size_t x_110; -x_108 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__4(x_101); -x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_99); -lean_ctor_set(x_109, 1, x_108); -x_110 = lean_usize_add(x_9, x_21); -x_9 = x_110; -x_10 = x_109; -goto _start; -} -else +uint64_t x_71; +if (lean_obj_tag(x_69) == 0) { -lean_object* x_112; size_t x_113; -x_112 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_112, 0, x_99); -lean_ctor_set(x_112, 1, x_101); -x_113 = lean_usize_add(x_9, x_21); -x_9 = x_113; -x_10 = x_112; -goto _start; -} +uint64_t x_158; +x_158 = 11; +x_71 = x_158; +goto block_157; } else { -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; size_t x_119; -lean_inc(x_5); -x_115 = lean_array_uset(x_91, x_95, x_5); -x_116 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_13, x_59, x_96); -x_117 = lean_array_uset(x_115, x_95, x_116); -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_90); -lean_ctor_set(x_118, 1, x_117); -x_119 = lean_usize_add(x_9, x_21); -x_9 = x_119; -x_10 = x_118; -goto _start; -} -} -} -} +lean_object* x_159; uint64_t x_160; uint64_t x_161; uint64_t x_162; +x_159 = lean_ctor_get(x_69, 0); +lean_inc(x_159); +lean_dec(x_69); +x_160 = lean_string_hash(x_159); +lean_dec(x_159); +x_161 = 13; +x_162 = lean_uint64_mix_hash(x_160, x_161); +x_71 = x_162; +goto block_157; +} +block_157: +{ +uint64_t x_72; lean_object* x_73; lean_object* x_74; lean_object* x_144; +x_144 = lean_ctor_get(x_70, 0); +lean_inc(x_144); +if (lean_obj_tag(x_144) == 0) +{ +lean_object* x_145; uint64_t x_146; lean_object* x_147; lean_object* x_148; +x_145 = lean_ctor_get(x_70, 1); +lean_inc(x_145); +lean_dec(x_70); +x_146 = 11; +x_147 = lean_ctor_get(x_145, 0); +lean_inc(x_147); +x_148 = lean_ctor_get(x_145, 1); +lean_inc(x_148); +lean_dec(x_145); +x_72 = x_146; +x_73 = x_147; +x_74 = x_148; +goto block_143; +} +else +{ +lean_object* x_149; lean_object* x_150; uint8_t x_151; uint64_t x_152; uint64_t x_153; uint64_t x_154; lean_object* x_155; lean_object* x_156; +x_149 = lean_ctor_get(x_70, 1); +lean_inc(x_149); +lean_dec(x_70); +x_150 = lean_ctor_get(x_144, 0); +lean_inc(x_150); +lean_dec(x_144); +x_151 = lean_unbox(x_150); +lean_dec(x_150); +x_152 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1169_(x_151); +x_153 = 13; +x_154 = lean_uint64_mix_hash(x_152, x_153); +x_155 = lean_ctor_get(x_149, 0); +lean_inc(x_155); +x_156 = lean_ctor_get(x_149, 1); +lean_inc(x_156); +lean_dec(x_149); +x_72 = x_154; +x_73 = x_155; +x_74 = x_156; +goto block_143; } -block_229: -{ -uint64_t x_137; -if (lean_obj_tag(x_135) == 0) +block_143: { -uint64_t x_224; -x_224 = 11; -x_137 = x_224; -goto block_223; -} -else +if (lean_obj_tag(x_73) == 0) { -lean_object* x_225; uint64_t x_226; uint64_t x_227; uint64_t x_228; -x_225 = lean_ctor_get(x_135, 0); -lean_inc(x_225); -lean_dec(x_135); -x_226 = lean_string_hash(x_225); -lean_dec(x_225); -x_227 = 13; -x_228 = lean_uint64_mix_hash(x_226, x_227); -x_137 = x_228; -goto block_223; -} -block_223: -{ -uint64_t x_138; lean_object* x_139; lean_object* x_140; lean_object* x_210; -x_210 = lean_ctor_get(x_136, 0); -lean_inc(x_210); -if (lean_obj_tag(x_210) == 0) -{ -lean_object* x_211; uint64_t x_212; lean_object* x_213; lean_object* x_214; -x_211 = lean_ctor_get(x_136, 1); -lean_inc(x_211); -lean_dec(x_136); -x_212 = 11; -x_213 = lean_ctor_get(x_211, 0); -lean_inc(x_213); -x_214 = lean_ctor_get(x_211, 1); -lean_inc(x_214); -lean_dec(x_211); -x_138 = x_212; -x_139 = x_213; -x_140 = x_214; -goto block_209; -} -else +if (lean_obj_tag(x_74) == 0) { -lean_object* x_215; lean_object* x_216; uint8_t x_217; uint64_t x_218; uint64_t x_219; uint64_t x_220; lean_object* x_221; lean_object* x_222; -x_215 = lean_ctor_get(x_136, 1); -lean_inc(x_215); -lean_dec(x_136); -x_216 = lean_ctor_get(x_210, 0); -lean_inc(x_216); -lean_dec(x_210); -x_217 = lean_unbox(x_216); -lean_dec(x_216); -x_218 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCompletionItemKind____x40_Lean_Data_Lsp_LanguageFeatures___hyg_1169_(x_217); -x_219 = 13; -x_220 = lean_uint64_mix_hash(x_218, x_219); -x_221 = lean_ctor_get(x_215, 0); -lean_inc(x_221); -x_222 = lean_ctor_get(x_215, 1); -lean_inc(x_222); -lean_dec(x_215); -x_138 = x_220; -x_139 = x_221; -x_140 = x_222; -goto block_209; -} -block_209: -{ -if (lean_obj_tag(x_139) == 0) -{ -if (lean_obj_tag(x_140) == 0) -{ -uint64_t x_141; uint64_t x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; -x_141 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1; -x_142 = lean_uint64_mix_hash(x_138, x_141); -x_143 = lean_uint64_mix_hash(x_137, x_142); -x_144 = lean_uint64_mix_hash(x_134, x_143); -x_145 = lean_uint64_mix_hash(x_133, x_144); -x_23 = x_145; -goto block_130; +uint64_t x_75; uint64_t x_76; uint64_t x_77; uint64_t x_78; uint64_t x_79; +x_75 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1; +x_76 = lean_uint64_mix_hash(x_72, x_75); +x_77 = lean_uint64_mix_hash(x_71, x_76); +x_78 = lean_uint64_mix_hash(x_68, x_77); +x_79 = lean_uint64_mix_hash(x_67, x_78); +x_24 = x_79; +goto block_64; } else { -lean_object* x_146; uint64_t x_147; uint64_t x_148; uint64_t x_149; uint64_t x_150; uint64_t x_151; uint64_t x_152; uint64_t x_153; uint64_t x_154; uint64_t x_155; -x_146 = lean_ctor_get(x_140, 0); -lean_inc(x_146); -lean_dec(x_140); -x_147 = 11; -x_148 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_146); -lean_dec(x_146); -x_149 = 13; -x_150 = lean_uint64_mix_hash(x_148, x_149); -x_151 = lean_uint64_mix_hash(x_147, x_150); -x_152 = lean_uint64_mix_hash(x_138, x_151); -x_153 = lean_uint64_mix_hash(x_137, x_152); -x_154 = lean_uint64_mix_hash(x_134, x_153); -x_155 = lean_uint64_mix_hash(x_133, x_154); -x_23 = x_155; -goto block_130; +lean_object* x_80; uint64_t x_81; uint64_t x_82; uint64_t x_83; uint64_t x_84; uint64_t x_85; uint64_t x_86; uint64_t x_87; uint64_t x_88; uint64_t x_89; +x_80 = lean_ctor_get(x_74, 0); +lean_inc(x_80); +lean_dec(x_74); +x_81 = 11; +x_82 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_80); +lean_dec(x_80); +x_83 = 13; +x_84 = lean_uint64_mix_hash(x_82, x_83); +x_85 = lean_uint64_mix_hash(x_81, x_84); +x_86 = lean_uint64_mix_hash(x_72, x_85); +x_87 = lean_uint64_mix_hash(x_71, x_86); +x_88 = lean_uint64_mix_hash(x_68, x_87); +x_89 = lean_uint64_mix_hash(x_67, x_88); +x_24 = x_89; +goto block_64; } } else { -lean_object* x_156; uint64_t x_157; lean_object* x_158; lean_object* x_159; uint8_t x_160; uint64_t x_161; -x_156 = lean_ctor_get(x_139, 0); -lean_inc(x_156); -lean_dec(x_139); -x_157 = 7; -x_158 = lean_array_get_size(x_156); -x_159 = lean_unsigned_to_nat(0u); -x_160 = lean_nat_dec_lt(x_159, x_158); -x_161 = 13; -if (x_160 == 0) +lean_object* x_90; uint64_t x_91; lean_object* x_92; lean_object* x_93; uint8_t x_94; uint64_t x_95; +x_90 = lean_ctor_get(x_73, 0); +lean_inc(x_90); +lean_dec(x_73); +x_91 = 7; +x_92 = lean_array_get_size(x_90); +x_93 = lean_unsigned_to_nat(0u); +x_94 = lean_nat_dec_lt(x_93, x_92); +x_95 = 13; +if (x_94 == 0) { -lean_dec(x_158); -lean_dec(x_156); -if (lean_obj_tag(x_140) == 0) +lean_dec(x_92); +lean_dec(x_90); +if (lean_obj_tag(x_74) == 0) { -uint64_t x_162; uint64_t x_163; uint64_t x_164; uint64_t x_165; uint64_t x_166; -x_162 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3; -x_163 = lean_uint64_mix_hash(x_138, x_162); -x_164 = lean_uint64_mix_hash(x_137, x_163); -x_165 = lean_uint64_mix_hash(x_134, x_164); -x_166 = lean_uint64_mix_hash(x_133, x_165); -x_23 = x_166; -goto block_130; +uint64_t x_96; uint64_t x_97; uint64_t x_98; uint64_t x_99; uint64_t x_100; +x_96 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3; +x_97 = lean_uint64_mix_hash(x_72, x_96); +x_98 = lean_uint64_mix_hash(x_71, x_97); +x_99 = lean_uint64_mix_hash(x_68, x_98); +x_100 = lean_uint64_mix_hash(x_67, x_99); +x_24 = x_100; +goto block_64; } else { -lean_object* x_167; uint64_t x_168; uint64_t x_169; uint64_t x_170; uint64_t x_171; uint64_t x_172; uint64_t x_173; uint64_t x_174; uint64_t x_175; -x_167 = lean_ctor_get(x_140, 0); -lean_inc(x_167); -lean_dec(x_140); -x_168 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_167); -lean_dec(x_167); -x_169 = lean_uint64_mix_hash(x_168, x_161); -x_170 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; -x_171 = lean_uint64_mix_hash(x_170, x_169); -x_172 = lean_uint64_mix_hash(x_138, x_171); -x_173 = lean_uint64_mix_hash(x_137, x_172); -x_174 = lean_uint64_mix_hash(x_134, x_173); -x_175 = lean_uint64_mix_hash(x_133, x_174); -x_23 = x_175; -goto block_130; +lean_object* x_101; uint64_t x_102; uint64_t x_103; uint64_t x_104; uint64_t x_105; uint64_t x_106; uint64_t x_107; uint64_t x_108; uint64_t x_109; +x_101 = lean_ctor_get(x_74, 0); +lean_inc(x_101); +lean_dec(x_74); +x_102 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_101); +lean_dec(x_101); +x_103 = lean_uint64_mix_hash(x_102, x_95); +x_104 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; +x_105 = lean_uint64_mix_hash(x_104, x_103); +x_106 = lean_uint64_mix_hash(x_72, x_105); +x_107 = lean_uint64_mix_hash(x_71, x_106); +x_108 = lean_uint64_mix_hash(x_68, x_107); +x_109 = lean_uint64_mix_hash(x_67, x_108); +x_24 = x_109; +goto block_64; } } else { -uint8_t x_176; -x_176 = lean_nat_dec_le(x_158, x_158); -if (x_176 == 0) +uint8_t x_110; +x_110 = lean_nat_dec_le(x_92, x_92); +if (x_110 == 0) { -lean_dec(x_158); -lean_dec(x_156); -if (lean_obj_tag(x_140) == 0) +lean_dec(x_92); +lean_dec(x_90); +if (lean_obj_tag(x_74) == 0) { -uint64_t x_177; uint64_t x_178; uint64_t x_179; uint64_t x_180; uint64_t x_181; -x_177 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3; -x_178 = lean_uint64_mix_hash(x_138, x_177); -x_179 = lean_uint64_mix_hash(x_137, x_178); -x_180 = lean_uint64_mix_hash(x_134, x_179); -x_181 = lean_uint64_mix_hash(x_133, x_180); -x_23 = x_181; -goto block_130; +uint64_t x_111; uint64_t x_112; uint64_t x_113; uint64_t x_114; uint64_t x_115; +x_111 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3; +x_112 = lean_uint64_mix_hash(x_72, x_111); +x_113 = lean_uint64_mix_hash(x_71, x_112); +x_114 = lean_uint64_mix_hash(x_68, x_113); +x_115 = lean_uint64_mix_hash(x_67, x_114); +x_24 = x_115; +goto block_64; } else { -lean_object* x_182; uint64_t x_183; uint64_t x_184; uint64_t x_185; uint64_t x_186; uint64_t x_187; uint64_t x_188; uint64_t x_189; uint64_t x_190; -x_182 = lean_ctor_get(x_140, 0); -lean_inc(x_182); -lean_dec(x_140); -x_183 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_182); -lean_dec(x_182); -x_184 = lean_uint64_mix_hash(x_183, x_161); -x_185 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2; -x_186 = lean_uint64_mix_hash(x_185, x_184); -x_187 = lean_uint64_mix_hash(x_138, x_186); -x_188 = lean_uint64_mix_hash(x_137, x_187); -x_189 = lean_uint64_mix_hash(x_134, x_188); -x_190 = lean_uint64_mix_hash(x_133, x_189); -x_23 = x_190; -goto block_130; +lean_object* x_116; uint64_t x_117; uint64_t x_118; uint64_t x_119; uint64_t x_120; uint64_t x_121; uint64_t x_122; uint64_t x_123; uint64_t x_124; +x_116 = lean_ctor_get(x_74, 0); +lean_inc(x_116); +lean_dec(x_74); +x_117 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_116); +lean_dec(x_116); +x_118 = lean_uint64_mix_hash(x_117, x_95); +x_119 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2; +x_120 = lean_uint64_mix_hash(x_119, x_118); +x_121 = lean_uint64_mix_hash(x_72, x_120); +x_122 = lean_uint64_mix_hash(x_71, x_121); +x_123 = lean_uint64_mix_hash(x_68, x_122); +x_124 = lean_uint64_mix_hash(x_67, x_123); +x_24 = x_124; +goto block_64; } } else { -size_t x_191; size_t x_192; uint64_t x_193; uint64_t x_194; -x_191 = 0; -x_192 = lean_usize_of_nat(x_158); -lean_dec(x_158); -x_193 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(x_156, x_191, x_192, x_157); -lean_dec(x_156); -x_194 = lean_uint64_mix_hash(x_193, x_161); -if (lean_obj_tag(x_140) == 0) -{ -uint64_t x_195; uint64_t x_196; uint64_t x_197; uint64_t x_198; uint64_t x_199; uint64_t x_200; -x_195 = 11; -x_196 = lean_uint64_mix_hash(x_194, x_195); -x_197 = lean_uint64_mix_hash(x_138, x_196); -x_198 = lean_uint64_mix_hash(x_137, x_197); -x_199 = lean_uint64_mix_hash(x_134, x_198); -x_200 = lean_uint64_mix_hash(x_133, x_199); -x_23 = x_200; -goto block_130; +size_t x_125; size_t x_126; uint64_t x_127; uint64_t x_128; +x_125 = 0; +x_126 = lean_usize_of_nat(x_92); +lean_dec(x_92); +x_127 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(x_90, x_125, x_126, x_91); +lean_dec(x_90); +x_128 = lean_uint64_mix_hash(x_127, x_95); +if (lean_obj_tag(x_74) == 0) +{ +uint64_t x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; uint64_t x_133; uint64_t x_134; +x_129 = 11; +x_130 = lean_uint64_mix_hash(x_128, x_129); +x_131 = lean_uint64_mix_hash(x_72, x_130); +x_132 = lean_uint64_mix_hash(x_71, x_131); +x_133 = lean_uint64_mix_hash(x_68, x_132); +x_134 = lean_uint64_mix_hash(x_67, x_133); +x_24 = x_134; +goto block_64; } else { -lean_object* x_201; uint64_t x_202; uint64_t x_203; uint64_t x_204; uint64_t x_205; uint64_t x_206; uint64_t x_207; uint64_t x_208; -x_201 = lean_ctor_get(x_140, 0); -lean_inc(x_201); -lean_dec(x_140); -x_202 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_201); -lean_dec(x_201); -x_203 = lean_uint64_mix_hash(x_202, x_161); -x_204 = lean_uint64_mix_hash(x_194, x_203); -x_205 = lean_uint64_mix_hash(x_138, x_204); -x_206 = lean_uint64_mix_hash(x_137, x_205); -x_207 = lean_uint64_mix_hash(x_134, x_206); -x_208 = lean_uint64_mix_hash(x_133, x_207); -x_23 = x_208; -goto block_130; +lean_object* x_135; uint64_t x_136; uint64_t x_137; uint64_t x_138; uint64_t x_139; uint64_t x_140; uint64_t x_141; uint64_t x_142; +x_135 = lean_ctor_get(x_74, 0); +lean_inc(x_135); +lean_dec(x_74); +x_136 = l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashMarkupContent____x40_Lean_Data_Lsp_Basic___hyg_6277_(x_135); +lean_dec(x_135); +x_137 = lean_uint64_mix_hash(x_136, x_95); +x_138 = lean_uint64_mix_hash(x_128, x_137); +x_139 = lean_uint64_mix_hash(x_72, x_138); +x_140 = lean_uint64_mix_hash(x_71, x_139); +x_141 = lean_uint64_mix_hash(x_68, x_140); +x_142 = lean_uint64_mix_hash(x_67, x_141); +x_24 = x_142; +goto block_64; } } } @@ -2691,11 +2107,11 @@ x_6 = 0; x_7 = l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__19; x_8 = l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__30; x_9 = l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__33; -x_10 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(x_1, x_2, x_7, x_8, x_3, x_4, x_2, x_5, x_6, x_9); +x_10 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_7, x_8, x_3, x_4, x_2, x_5, x_6, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -2729,7 +2145,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; uint8_t x_4; @@ -2775,7 +2191,7 @@ size_t x_12; size_t x_13; lean_object* x_14; lean_object* x_15; x_12 = 1; x_13 = lean_usize_of_nat(x_2); lean_dec(x_2); -x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(x_1, x_12, x_13, x_6); +x_14 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(x_1, x_12, x_13, x_6); x_15 = lean_alloc_ctor(1, 1, 0); lean_ctor_set(x_15, 0, x_14); return x_15; @@ -2784,7 +2200,7 @@ return x_15; } } } -LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(lean_object* x_1) { +LEAN_EXPORT lean_object* l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; @@ -2793,7 +2209,7 @@ x_3 = lean_panic_fn(x_2, x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2815,7 +2231,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -2843,7 +2259,7 @@ goto _start; } } } -static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1() { +static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1() { _start: { lean_object* x_1; @@ -2851,7 +2267,7 @@ x_1 = lean_mk_string_unchecked("Init.Data.Option.BasicAux", 25, 25); return x_1; } } -static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2() { +static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2() { _start: { lean_object* x_1; @@ -2859,7 +2275,7 @@ x_1 = lean_mk_string_unchecked("Option.get!", 11, 11); return x_1; } } -static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3() { +static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3() { _start: { lean_object* x_1; @@ -2867,20 +2283,20 @@ x_1 = lean_mk_string_unchecked("value is none", 13, 13); return x_1; } } -static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4() { +static lean_object* _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; -x_1 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1; -x_2 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2; +x_1 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1; +x_2 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2; x_3 = lean_unsigned_to_nat(16u); x_4 = lean_unsigned_to_nat(14u); -x_5 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3; +x_5 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3; x_6 = l___private_Init_Util_0__mkPanicMessageWithDecl(x_1, x_2, x_3, x_4, x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2896,13 +2312,13 @@ if (x_3 == 0) lean_object* x_4; lean_object* x_5; lean_object* x_6; x_4 = lean_ctor_get(x_2, 1); x_5 = lean_ctor_get(x_2, 2); -x_6 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(x_4); +x_6 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_4); lean_dec(x_4); if (lean_obj_tag(x_6) == 0) { lean_object* x_7; lean_object* x_8; -x_7 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; -x_8 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(x_7); +x_7 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; +x_8 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(x_7); lean_ctor_set(x_2, 2, x_1); lean_ctor_set(x_2, 1, x_8); x_1 = x_2; @@ -2932,13 +2348,13 @@ lean_inc(x_14); lean_inc(x_13); lean_inc(x_12); lean_dec(x_2); -x_15 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(x_13); +x_15 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_13); lean_dec(x_13); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_16 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; -x_17 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(x_16); +x_16 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; +x_17 = l_panic___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(x_16); x_18 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_18, 0, x_12); lean_ctor_set(x_18, 1, x_17); @@ -2965,7 +2381,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -2981,7 +2397,7 @@ x_5 = lean_array_uget(x_3, x_2); x_6 = lean_unsigned_to_nat(0u); x_7 = lean_array_uset(x_3, x_2, x_6); x_8 = lean_box(0); -x_9 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18(x_8, x_5); +x_9 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(x_8, x_5); x_10 = 1; x_11 = lean_usize_add(x_2, x_10); x_12 = lean_array_uset(x_7, x_2, x_9); @@ -2991,7 +2407,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -3000,7 +2416,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(x_4, x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); x_2 = x_9; @@ -3067,7 +2483,7 @@ lean_inc(x_4); lean_dec(x_3); x_5 = lean_array_size(x_4); x_6 = 0; -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(x_5, x_6, x_4); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(x_5, x_6, x_4); x_8 = lean_array_get_size(x_7); x_9 = lean_unsigned_to_nat(0u); x_10 = lean_nat_dec_lt(x_9, x_8); @@ -3076,7 +2492,7 @@ if (x_10 == 0) lean_object* x_11; lean_dec(x_8); lean_dec(x_7); -x_11 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; +x_11 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; return x_11; } else @@ -3088,7 +2504,7 @@ if (x_12 == 0) lean_object* x_13; lean_dec(x_8); lean_dec(x_7); -x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; +x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; return x_13; } else @@ -3096,24 +2512,24 @@ else size_t x_14; lean_object* x_15; lean_object* x_16; x_14 = lean_usize_of_nat(x_8); lean_dec(x_8); -x_15 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; -x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19(x_7, x_6, x_14, x_15); +x_15 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; +x_16 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(x_7, x_6, x_14, x_15); lean_dec(x_7); return x_16; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__2(x_1, x_2); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; uint64_t x_7; uint64_t x_8; lean_object* x_9; @@ -3123,13 +2539,13 @@ x_6 = lean_unbox_usize(x_3); lean_dec(x_3); x_7 = lean_unbox_uint64(x_4); lean_dec(x_4); -x_8 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6(x_1, x_5, x_6, x_7); +x_8 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__5(x_1, x_5, x_6, x_7); lean_dec(x_1); x_9 = lean_box_uint64(x_8); return x_9; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -3137,7 +2553,7 @@ x_11 = lean_unbox_usize(x_8); lean_dec(x_8); x_12 = lean_unbox_usize(x_9); lean_dec(x_9); -x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); +x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); @@ -3155,7 +2571,7 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -3163,21 +2579,21 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__13(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12___boxed(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10___boxed(lean_object* x_1) { _start: { lean_object* x_2; -x_2 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__12(x_1); +x_2 = l_Array_getMax_x3f___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__10(x_1); lean_dec(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -3185,11 +2601,11 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16(x_1, x_5, x_6, x_4); +x_7 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14(x_1, x_5, x_6, x_4); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -3197,11 +2613,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__14___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__15(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -3209,7 +2625,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__19(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__17(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -3571,7 +2987,7 @@ x_12 = lean_usize_add(x_3, x_11); if (lean_obj_tag(x_10) == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_13 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; +x_13 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; x_14 = l_panic___at_String_fromUTF8_x21___spec__1(x_13); x_15 = lean_string_length(x_14); x_16 = lean_nat_sub(x_1, x_15); @@ -3660,7 +3076,7 @@ x_53 = lean_usize_add(x_3, x_52); if (lean_obj_tag(x_49) == 0) { lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; -x_54 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; +x_54 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; x_55 = l_panic___at_String_fromUTF8_x21___spec__1(x_54); x_56 = lean_string_length(x_55); x_57 = lean_nat_sub(x_1, x_56); @@ -3757,7 +3173,7 @@ lean_dec(x_14); if (lean_obj_tag(x_15) == 0) { lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_16 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; +x_16 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; x_17 = l_panic___at_String_fromUTF8_x21___spec__1(x_16); x_18 = lean_string_length(x_17); lean_dec(x_17); @@ -3789,7 +3205,7 @@ lean_dec(x_23); if (lean_obj_tag(x_24) == 0) { lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_25 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4; +x_25 = l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4; x_26 = l_panic___at_String_fromUTF8_x21___spec__1(x_25); x_27 = lean_string_length(x_26); lean_dec(x_26); @@ -3827,7 +3243,7 @@ return x_4; else { lean_object* x_5; -x_5 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; +x_5 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; return x_5; } } @@ -4456,7 +3872,7 @@ x_8 = l_Lean_Server_Completion_findPrioritizedCompletionPartitionsAt(x_2, x_3, x x_9 = lean_box(0); x_10 = lean_array_size(x_8); x_11 = 0; -x_12 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1; +x_12 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1; x_13 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Completion_find_x3f___spec__2(x_1, x_6, x_8, x_12, x_9, x_8, x_10, x_11, x_12, x_7); lean_dec(x_8); if (lean_obj_tag(x_13) == 0) @@ -4578,11 +3994,11 @@ lean_dec_ref(res); res = initialize_Std_Data_HashMap(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); -l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__1(); -l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__2(); -l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__8___closed__3(); -l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__11___closed__1); +l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__1(); +l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__2(); +l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__6___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__7___closed__3(); +l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__9___lambda__1___closed__1); l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__1 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__1(); lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__1); l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__2 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__2(); @@ -4649,14 +4065,14 @@ l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completi lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__32); l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__33 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__33(); lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__1___closed__33); -l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1(); -lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__1); -l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2(); -lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__2); -l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3(); -lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__3); -l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4(); -lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__18___closed__4); +l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1(); +lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__1); +l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2(); +lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__2); +l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3(); +lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__3); +l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4 = _init_l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4(); +lean_mark_persistent(l_Std_DHashMap_Internal_AssocList_map_go___at___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___spec__16___closed__4); l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___closed__1 = _init_l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___closed__1(); lean_mark_persistent(l___private_Lean_Server_Completion_0__Lean_Server_Completion_filterDuplicateCompletionItems___closed__1); l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___closed__1 = _init_l_Array_qsort_sort___at___private_Lean_Server_Completion_0__Lean_Server_Completion_sortCompletionItems___spec__2___closed__1(); diff --git a/stage0/stdlib/Lean/Server/Completion/CompletionInfoSelection.c b/stage0/stdlib/Lean/Server/Completion/CompletionInfoSelection.c index 1b09d68e0440..4900cb308b56 100644 --- a/stage0/stdlib/Lean/Server/Completion/CompletionInfoSelection.c +++ b/stage0/stdlib/Lean/Server/Completion/CompletionInfoSelection.c @@ -17,31 +17,29 @@ LEAN_EXPORT lean_object* l_Array_groupByKey___at___private_Lean_Server_Completio LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__2___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___lambda__1(lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__1(lean_object*, lean_object*, size_t, size_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9___boxed(lean_object*, lean_object*); lean_object* l_instBEqOfDecidableEq___rarg(lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_Lean_Meta_addPPExplicitToExposeDiff_visit___spec__2(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__7; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__11; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2___boxed(lean_object*, lean_object*); uint64_t lean_uint64_of_nat(lean_object*); uint64_t lean_uint64_mix_hash(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_FileMap_toPosition(lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__6; LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_push(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(lean_object*, size_t, size_t, lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6(lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Server_Completion_findSyntheticCompletions(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos(lean_object*); lean_object* l_Lean_Elab_Info_size_x3f(lean_object*); @@ -57,51 +55,47 @@ LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go(lean_ LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos_eq___boxed(lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(size_t, size_t, lean_object*); lean_object* l_Lean_Elab_Info_tailPos_x3f(lean_object*); -LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1(lean_object*, lean_object*); uint8_t lean_expr_eqv(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__1; uint64_t lean_uint64_shift_right(uint64_t, uint64_t); -static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2; lean_object* lean_nat_div(lean_object*, lean_object*); lean_object* l_instDecidableEqPos___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instHashableBool___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_anyMUnsafe_any___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14(lean_object*, size_t, size_t, lean_object*); lean_object* l_instDecidableEqBool___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__2___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__3___closed__2; static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__8; -static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7(lean_object*); lean_object* l_instHashableProd___rarg___boxed(lean_object*, lean_object*, lean_object*); uint8_t lean_name_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2; +static uint64_t l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1; +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(lean_object*, lean_object*); lean_object* l_Array_zipWithIndex___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__3; LEAN_EXPORT lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(lean_object*, lean_object*); lean_object* l_panic___at_Lean_Parser_ParserState_mkUnexpectedTokenErrors___spec__1(lean_object*); lean_object* l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__12; static lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__3___closed__3; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_instHashableOption___rarg___boxed(lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt___lambda__1(lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); -static lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__4; uint8_t l_List_beq___at___private_Init_Meta_0__Lean_Syntax_beqPreresolved____x40_Init_Meta___hyg_2878____spec__1(lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); @@ -109,36 +103,40 @@ static lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__ lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); lean_object* l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1___boxed(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findPrioritizedCompletionPartitionsAt(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); uint8_t l_Lean_Syntax_eqWithInfo(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___boxed(lean_object*); lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_Completion_findCompletionInfosAt___closed__1; lean_object* l_Lean_Elab_Info_pos_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__10; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); lean_object* l_instHashablePos___boxed(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(lean_object*, lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(size_t, size_t, lean_object*); uint8_t l_Lean_Elab_Info_occursInOrOnBoundary(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Completion_findCompletionInfosAt_go___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos_eq(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__13; +static lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11___boxed(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); uint8_t l_Array_isEmpty___rarg(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos_eq(lean_object* x_1, lean_object* x_2) { @@ -958,95 +956,7 @@ lean_dec(x_1); return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_ctor_get(x_4, 0); -x_6 = lean_unbox(x_5); -if (x_6 == 0) -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_ctor_get(x_1, 0); -x_8 = lean_unbox(x_7); -if (x_8 == 0) -{ -lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_9 = lean_ctor_get(x_2, 1); -x_10 = lean_ctor_get(x_2, 2); -x_11 = lean_ctor_get(x_4, 1); -x_12 = lean_ctor_get(x_1, 1); -x_13 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_11, x_12); -if (x_13 == 0) -{ -x_2 = x_10; -goto _start; -} -else -{ -lean_object* x_15; -lean_inc(x_9); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_9); -return x_15; -} -} -else -{ -lean_object* x_16; -x_16 = lean_ctor_get(x_2, 2); -x_2 = x_16; -goto _start; -} -} -else -{ -lean_object* x_18; uint8_t x_19; -x_18 = lean_ctor_get(x_1, 0); -x_19 = lean_unbox(x_18); -if (x_19 == 0) -{ -lean_object* x_20; -x_20 = lean_ctor_get(x_2, 2); -x_2 = x_20; -goto _start; -} -else -{ -lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; -x_22 = lean_ctor_get(x_2, 1); -x_23 = lean_ctor_get(x_2, 2); -x_24 = lean_ctor_get(x_4, 1); -x_25 = lean_ctor_get(x_1, 1); -x_26 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_24, x_25); -if (x_26 == 0) -{ -x_2 = x_23; -goto _start; -} -else -{ -lean_object* x_28; -lean_inc(x_22); -x_28 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_28, 0, x_22); -return x_28; -} -} -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -1128,7 +1038,7 @@ return x_26; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -1211,7 +1121,7 @@ goto _start; } } } -static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1() { +static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1() { _start: { uint64_t x_1; uint64_t x_2; uint64_t x_3; @@ -1221,7 +1131,7 @@ x_3 = lean_uint64_mix_hash(x_1, x_2); return x_3; } } -static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2() { +static uint64_t _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2() { _start: { uint64_t x_1; uint64_t x_2; @@ -1230,7 +1140,7 @@ x_2 = lean_uint64_mix_hash(x_1, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -1274,7 +1184,7 @@ lean_inc(x_27); if (lean_obj_tag(x_27) == 0) { uint64_t x_28; -x_28 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1; +x_28 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1; x_13 = x_28; goto block_24; } @@ -1301,7 +1211,7 @@ lean_inc(x_34); if (lean_obj_tag(x_34) == 0) { uint64_t x_35; -x_35 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2; +x_35 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2; x_13 = x_35; goto block_24; } @@ -1347,7 +1257,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -1366,7 +1276,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -1377,7 +1287,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -1388,471 +1298,378 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_4; -lean_dec(x_2); -lean_dec(x_1); +lean_object* x_4; lean_object* x_5; x_4 = lean_box(0); -return x_4; -} -else +x_5 = lean_apply_1(x_2, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_5 = lean_ctor_get(x_3, 0); -lean_inc(x_5); -x_6 = lean_ctor_get(x_5, 0); -lean_inc(x_6); -x_7 = lean_unbox(x_6); -lean_dec(x_6); -if (x_7 == 0) -{ -lean_object* x_8; uint8_t x_9; -x_8 = lean_ctor_get(x_1, 0); -lean_inc(x_8); -x_9 = lean_unbox(x_8); -lean_dec(x_8); -if (x_9 == 0) -{ -uint8_t x_10; -x_10 = !lean_is_exclusive(x_3); -if (x_10 == 0) -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; -x_11 = lean_ctor_get(x_3, 1); -x_12 = lean_ctor_get(x_3, 2); -x_13 = lean_ctor_get(x_3, 0); -lean_dec(x_13); -x_14 = lean_ctor_get(x_5, 1); -lean_inc(x_14); -x_15 = lean_ctor_get(x_1, 1); -lean_inc(x_15); -x_16 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_14, x_15); -lean_dec(x_15); -lean_dec(x_14); -if (x_16 == 0) -{ -lean_object* x_17; -x_17 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_12); -lean_ctor_set(x_3, 2, x_17); -return x_3; +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; } else { -lean_dec(x_11); +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); lean_dec(x_5); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_1); -return x_3; +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_7); +lean_ctor_set(x_9, 2, x_8); +return x_9; } } else { -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_18 = lean_ctor_get(x_3, 1); -x_19 = lean_ctor_get(x_3, 2); +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_3, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_10, 0); +lean_inc(x_11); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; uint8_t x_14; +x_13 = lean_ctor_get(x_1, 0); +lean_inc(x_13); +x_14 = lean_unbox(x_13); +lean_dec(x_13); +if (x_14 == 0) +{ +uint8_t x_15; +x_15 = !lean_is_exclusive(x_3); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_16 = lean_ctor_get(x_3, 1); +x_17 = lean_ctor_get(x_3, 2); +x_18 = lean_ctor_get(x_3, 0); +lean_dec(x_18); +x_19 = lean_ctor_get(x_10, 1); lean_inc(x_19); -lean_inc(x_18); -lean_dec(x_3); -x_20 = lean_ctor_get(x_5, 1); +x_20 = lean_ctor_get(x_1, 1); lean_inc(x_20); -x_21 = lean_ctor_get(x_1, 1); -lean_inc(x_21); -x_22 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_20, x_21); -lean_dec(x_21); +x_21 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_19, x_20); lean_dec(x_20); -if (x_22 == 0) +lean_dec(x_19); +if (x_21 == 0) +{ +lean_object* x_22; +x_22 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_17); +lean_ctor_set(x_3, 2, x_22); +return x_3; +} +else { lean_object* x_23; lean_object* x_24; -x_23 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_19); -x_24 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_24, 0, x_5); -lean_ctor_set(x_24, 1, x_18); -lean_ctor_set(x_24, 2, x_23); -return x_24; +lean_dec(x_10); +x_23 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_23, 0, x_16); +x_24 = lean_apply_1(x_2, x_23); +if (lean_obj_tag(x_24) == 0) +{ +lean_free_object(x_3); +lean_dec(x_1); +return x_17; } else { lean_object* x_25; -lean_dec(x_18); -lean_dec(x_5); -x_25 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_25, 0, x_1); -lean_ctor_set(x_25, 1, x_2); -lean_ctor_set(x_25, 2, x_19); -return x_25; +x_25 = lean_ctor_get(x_24, 0); +lean_inc(x_25); +lean_dec(x_24); +lean_ctor_set(x_3, 1, x_25); +lean_ctor_set(x_3, 0, x_1); +return x_3; } } } else { -uint8_t x_26; -x_26 = !lean_is_exclusive(x_3); -if (x_26 == 0) -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +x_26 = lean_ctor_get(x_3, 1); x_27 = lean_ctor_get(x_3, 2); -x_28 = lean_ctor_get(x_3, 0); +lean_inc(x_27); +lean_inc(x_26); +lean_dec(x_3); +x_28 = lean_ctor_get(x_10, 1); +lean_inc(x_28); +x_29 = lean_ctor_get(x_1, 1); +lean_inc(x_29); +x_30 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_28, x_29); +lean_dec(x_29); lean_dec(x_28); -x_29 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_27); -lean_ctor_set(x_3, 2, x_29); -return x_3; +if (x_30 == 0) +{ +lean_object* x_31; lean_object* x_32; +x_31 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_27); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_10); +lean_ctor_set(x_32, 1, x_26); +lean_ctor_set(x_32, 2, x_31); +return x_32; } else { -lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_3, 1); -x_31 = lean_ctor_get(x_3, 2); -lean_inc(x_31); -lean_inc(x_30); -lean_dec(x_3); -x_32 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_31); -x_33 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_33, 0, x_5); -lean_ctor_set(x_33, 1, x_30); -lean_ctor_set(x_33, 2, x_32); -return x_33; -} -} +lean_object* x_33; lean_object* x_34; +lean_dec(x_10); +x_33 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_33, 0, x_26); +x_34 = lean_apply_1(x_2, x_33); +if (lean_obj_tag(x_34) == 0) +{ +lean_dec(x_1); +return x_27; } else { -lean_object* x_34; uint8_t x_35; -x_34 = lean_ctor_get(x_1, 0); -lean_inc(x_34); -x_35 = lean_unbox(x_34); +lean_object* x_35; lean_object* x_36; +x_35 = lean_ctor_get(x_34, 0); +lean_inc(x_35); lean_dec(x_34); -if (x_35 == 0) +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_1); +lean_ctor_set(x_36, 1, x_35); +lean_ctor_set(x_36, 2, x_27); +return x_36; +} +} +} +} +else { -uint8_t x_36; -x_36 = !lean_is_exclusive(x_3); -if (x_36 == 0) +uint8_t x_37; +x_37 = !lean_is_exclusive(x_3); +if (x_37 == 0) { -lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_37 = lean_ctor_get(x_3, 2); -x_38 = lean_ctor_get(x_3, 0); -lean_dec(x_38); -x_39 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_37); -lean_ctor_set(x_3, 2, x_39); +lean_object* x_38; lean_object* x_39; lean_object* x_40; +x_38 = lean_ctor_get(x_3, 2); +x_39 = lean_ctor_get(x_3, 0); +lean_dec(x_39); +x_40 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_38); +lean_ctor_set(x_3, 2, x_40); return x_3; } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; -x_40 = lean_ctor_get(x_3, 1); -x_41 = lean_ctor_get(x_3, 2); +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; +x_41 = lean_ctor_get(x_3, 1); +x_42 = lean_ctor_get(x_3, 2); +lean_inc(x_42); lean_inc(x_41); -lean_inc(x_40); lean_dec(x_3); -x_42 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_41); -x_43 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_43, 0, x_5); -lean_ctor_set(x_43, 1, x_40); -lean_ctor_set(x_43, 2, x_42); -return x_43; +x_43 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_42); +x_44 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_44, 0, x_10); +lean_ctor_set(x_44, 1, x_41); +lean_ctor_set(x_44, 2, x_43); +return x_44; } } -else -{ -uint8_t x_44; -x_44 = !lean_is_exclusive(x_3); -if (x_44 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; -x_45 = lean_ctor_get(x_3, 1); -x_46 = lean_ctor_get(x_3, 2); -x_47 = lean_ctor_get(x_3, 0); -lean_dec(x_47); -x_48 = lean_ctor_get(x_5, 1); -lean_inc(x_48); -x_49 = lean_ctor_get(x_1, 1); -lean_inc(x_49); -x_50 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_48, x_49); -lean_dec(x_49); -lean_dec(x_48); -if (x_50 == 0) -{ -lean_object* x_51; -x_51 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_46); -lean_ctor_set(x_3, 2, x_51); -return x_3; } else { +lean_object* x_45; uint8_t x_46; +x_45 = lean_ctor_get(x_1, 0); +lean_inc(x_45); +x_46 = lean_unbox(x_45); lean_dec(x_45); -lean_dec(x_5); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_1); +if (x_46 == 0) +{ +uint8_t x_47; +x_47 = !lean_is_exclusive(x_3); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_ctor_get(x_3, 2); +x_49 = lean_ctor_get(x_3, 0); +lean_dec(x_49); +x_50 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_48); +lean_ctor_set(x_3, 2, x_50); return x_3; } -} else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_56; -x_52 = lean_ctor_get(x_3, 1); -x_53 = lean_ctor_get(x_3, 2); -lean_inc(x_53); +lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_51 = lean_ctor_get(x_3, 1); +x_52 = lean_ctor_get(x_3, 2); lean_inc(x_52); +lean_inc(x_51); lean_dec(x_3); -x_54 = lean_ctor_get(x_5, 1); -lean_inc(x_54); -x_55 = lean_ctor_get(x_1, 1); -lean_inc(x_55); -x_56 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_54, x_55); -lean_dec(x_55); -lean_dec(x_54); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; -x_57 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_53); -x_58 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_58, 0, x_5); -lean_ctor_set(x_58, 1, x_52); -lean_ctor_set(x_58, 2, x_57); -return x_58; -} -else -{ -lean_object* x_59; -lean_dec(x_52); -lean_dec(x_5); -x_59 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_59, 0, x_1); -lean_ctor_set(x_59, 1, x_2); -lean_ctor_set(x_59, 2, x_53); -return x_59; -} -} -} -} -} +x_53 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_52); +x_54 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_54, 0, x_10); +lean_ctor_set(x_54, 1, x_51); +lean_ctor_set(x_54, 2, x_53); +return x_54; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +uint8_t x_55; +x_55 = !lean_is_exclusive(x_3); +if (x_55 == 0) { -lean_object* x_3; -x_3 = lean_box(0); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; +x_56 = lean_ctor_get(x_3, 1); +x_57 = lean_ctor_get(x_3, 2); +x_58 = lean_ctor_get(x_3, 0); +lean_dec(x_58); +x_59 = lean_ctor_get(x_10, 1); +lean_inc(x_59); +x_60 = lean_ctor_get(x_1, 1); +lean_inc(x_60); +x_61 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_59, x_60); +lean_dec(x_60); +lean_dec(x_59); +if (x_61 == 0) +{ +lean_object* x_62; +x_62 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_57); +lean_ctor_set(x_3, 2, x_62); return x_3; } else { -lean_object* x_4; lean_object* x_5; uint8_t x_6; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_4, 0); -lean_inc(x_5); -x_6 = lean_unbox(x_5); -lean_dec(x_5); -if (x_6 == 0) -{ -lean_object* x_7; uint8_t x_8; -x_7 = lean_ctor_get(x_1, 0); -x_8 = lean_unbox(x_7); -if (x_8 == 0) -{ -uint8_t x_9; -x_9 = !lean_is_exclusive(x_2); -if (x_9 == 0) -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; -x_10 = lean_ctor_get(x_2, 1); -x_11 = lean_ctor_get(x_2, 2); -x_12 = lean_ctor_get(x_2, 0); -lean_dec(x_12); -x_13 = lean_ctor_get(x_4, 1); -lean_inc(x_13); -x_14 = lean_ctor_get(x_1, 1); -x_15 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_13, x_14); -lean_dec(x_13); -if (x_15 == 0) +lean_object* x_63; lean_object* x_64; +lean_dec(x_10); +x_63 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_63, 0, x_56); +x_64 = lean_apply_1(x_2, x_63); +if (lean_obj_tag(x_64) == 0) { -lean_object* x_16; -x_16 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_11); -lean_ctor_set(x_2, 2, x_16); -return x_2; +lean_free_object(x_3); +lean_dec(x_1); +return x_57; } else { -lean_free_object(x_2); -lean_dec(x_10); -lean_dec(x_4); -return x_11; +lean_object* x_65; +x_65 = lean_ctor_get(x_64, 0); +lean_inc(x_65); +lean_dec(x_64); +lean_ctor_set(x_3, 1, x_65); +lean_ctor_set(x_3, 0, x_1); +return x_3; } } -else -{ -lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; uint8_t x_21; -x_17 = lean_ctor_get(x_2, 1); -x_18 = lean_ctor_get(x_2, 2); -lean_inc(x_18); -lean_inc(x_17); -lean_dec(x_2); -x_19 = lean_ctor_get(x_4, 1); -lean_inc(x_19); -x_20 = lean_ctor_get(x_1, 1); -x_21 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_19, x_20); -lean_dec(x_19); -if (x_21 == 0) -{ -lean_object* x_22; lean_object* x_23; -x_22 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_18); -x_23 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_23, 0, x_4); -lean_ctor_set(x_23, 1, x_17); -lean_ctor_set(x_23, 2, x_22); -return x_23; } else { -lean_dec(x_17); -lean_dec(x_4); -return x_18; -} -} +lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; uint8_t x_70; +x_66 = lean_ctor_get(x_3, 1); +x_67 = lean_ctor_get(x_3, 2); +lean_inc(x_67); +lean_inc(x_66); +lean_dec(x_3); +x_68 = lean_ctor_get(x_10, 1); +lean_inc(x_68); +x_69 = lean_ctor_get(x_1, 1); +lean_inc(x_69); +x_70 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_68, x_69); +lean_dec(x_69); +lean_dec(x_68); +if (x_70 == 0) +{ +lean_object* x_71; lean_object* x_72; +x_71 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_1, x_2, x_67); +x_72 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_72, 0, x_10); +lean_ctor_set(x_72, 1, x_66); +lean_ctor_set(x_72, 2, x_71); +return x_72; } else { -uint8_t x_24; -x_24 = !lean_is_exclusive(x_2); -if (x_24 == 0) +lean_object* x_73; lean_object* x_74; +lean_dec(x_10); +x_73 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_73, 0, x_66); +x_74 = lean_apply_1(x_2, x_73); +if (lean_obj_tag(x_74) == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; -x_25 = lean_ctor_get(x_2, 2); -x_26 = lean_ctor_get(x_2, 0); -lean_dec(x_26); -x_27 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_25); -lean_ctor_set(x_2, 2, x_27); -return x_2; +lean_dec(x_1); +return x_67; } else { -lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; -x_28 = lean_ctor_get(x_2, 1); -x_29 = lean_ctor_get(x_2, 2); -lean_inc(x_29); -lean_inc(x_28); -lean_dec(x_2); -x_30 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_29); -x_31 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_31, 0, x_4); -lean_ctor_set(x_31, 1, x_28); -lean_ctor_set(x_31, 2, x_30); -return x_31; +lean_object* x_75; lean_object* x_76; +x_75 = lean_ctor_get(x_74, 0); +lean_inc(x_75); +lean_dec(x_74); +x_76 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_76, 0, x_1); +lean_ctor_set(x_76, 1, x_75); +lean_ctor_set(x_76, 2, x_67); +return x_76; } } } -else -{ -lean_object* x_32; uint8_t x_33; -x_32 = lean_ctor_get(x_1, 0); -x_33 = lean_unbox(x_32); -if (x_33 == 0) -{ -uint8_t x_34; -x_34 = !lean_is_exclusive(x_2); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_35 = lean_ctor_get(x_2, 2); -x_36 = lean_ctor_get(x_2, 0); -lean_dec(x_36); -x_37 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_35); -lean_ctor_set(x_2, 2, x_37); -return x_2; } -else -{ -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -x_38 = lean_ctor_get(x_2, 1); -x_39 = lean_ctor_get(x_2, 2); -lean_inc(x_39); -lean_inc(x_38); -lean_dec(x_2); -x_40 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_39); -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_4); -lean_ctor_set(x_41, 1, x_38); -lean_ctor_set(x_41, 2, x_40); -return x_41; } } -else -{ -uint8_t x_42; -x_42 = !lean_is_exclusive(x_2); -if (x_42 == 0) +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7(lean_object* x_1) { +_start: { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -x_43 = lean_ctor_get(x_2, 1); -x_44 = lean_ctor_get(x_2, 2); -x_45 = lean_ctor_get(x_2, 0); -lean_dec(x_45); -x_46 = lean_ctor_get(x_4, 1); -lean_inc(x_46); -x_47 = lean_ctor_get(x_1, 1); -x_48 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_46, x_47); -lean_dec(x_46); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_44); -lean_ctor_set(x_2, 2, x_49); +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg), 3, 0); return x_2; } -else -{ -lean_free_object(x_2); -lean_dec(x_43); -lean_dec(x_4); -return x_44; } +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; uint8_t x_54; -x_50 = lean_ctor_get(x_2, 1); -x_51 = lean_ctor_get(x_2, 2); -lean_inc(x_51); -lean_inc(x_50); -lean_dec(x_2); -x_52 = lean_ctor_get(x_4, 1); -lean_inc(x_52); -x_53 = lean_ctor_get(x_1, 1); -x_54 = l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at_System_FilePath_parent___spec__1(x_52, x_53); -lean_dec(x_52); -if (x_54 == 0) +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) { -lean_object* x_55; lean_object* x_56; -x_55 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_51); -x_56 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_56, 0, x_4); -lean_ctor_set(x_56, 1, x_50); -lean_ctor_set(x_56, 2, x_55); -return x_56; +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); +return x_2; } else { -lean_dec(x_50); -lean_dec(x_4); -return x_51; -} -} -} +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { _start: { uint8_t x_11; @@ -1865,117 +1682,117 @@ return x_10; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; size_t x_20; size_t x_21; size_t x_22; uint64_t x_23; lean_object* x_131; uint8_t x_132; +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; size_t x_21; size_t x_22; size_t x_23; uint64_t x_24; lean_object* x_65; uint8_t x_66; x_12 = lean_array_uget(x_7, x_9); lean_inc(x_1); lean_inc(x_12); x_13 = lean_apply_1(x_1, x_12); -x_14 = lean_ctor_get(x_10, 0); -lean_inc(x_14); -x_15 = lean_ctor_get(x_10, 1); +lean_inc(x_12); +x_14 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8___lambda__1), 2, 1); +lean_closure_set(x_14, 0, x_12); +x_15 = lean_ctor_get(x_10, 0); lean_inc(x_15); +x_16 = lean_ctor_get(x_10, 1); +lean_inc(x_16); if (lean_is_exclusive(x_10)) { lean_ctor_release(x_10, 0); lean_ctor_release(x_10, 1); - x_16 = x_10; + x_17 = x_10; } else { lean_dec_ref(x_10); - x_16 = lean_box(0); + x_17 = lean_box(0); } -x_17 = lean_array_get_size(x_15); -x_18 = 32; -x_19 = 16; -x_20 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_21 = 1; -x_22 = lean_usize_sub(x_20, x_21); -x_131 = lean_ctor_get(x_13, 0); -lean_inc(x_131); -x_132 = lean_unbox(x_131); -lean_dec(x_131); -if (x_132 == 0) -{ -lean_object* x_133; -x_133 = lean_ctor_get(x_13, 1); -lean_inc(x_133); -if (lean_obj_tag(x_133) == 0) -{ -uint64_t x_134; -x_134 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1; -x_23 = x_134; -goto block_130; -} -else -{ -lean_object* x_135; uint64_t x_136; uint64_t x_137; uint64_t x_138; uint64_t x_139; -x_135 = lean_ctor_get(x_133, 0); -lean_inc(x_135); -lean_dec(x_133); -x_136 = 13; -x_137 = lean_uint64_of_nat(x_135); -lean_dec(x_135); -x_138 = lean_uint64_mix_hash(x_137, x_136); -x_139 = lean_uint64_mix_hash(x_136, x_138); -x_23 = x_139; -goto block_130; -} -} -else -{ -lean_object* x_140; -x_140 = lean_ctor_get(x_13, 1); -lean_inc(x_140); -if (lean_obj_tag(x_140) == 0) -{ -uint64_t x_141; -x_141 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2; -x_23 = x_141; -goto block_130; -} -else -{ -lean_object* x_142; uint64_t x_143; uint64_t x_144; uint64_t x_145; uint64_t x_146; uint64_t x_147; -x_142 = lean_ctor_get(x_140, 0); -lean_inc(x_142); -lean_dec(x_140); -x_143 = 11; -x_144 = lean_uint64_of_nat(x_142); -lean_dec(x_142); -x_145 = 13; -x_146 = lean_uint64_mix_hash(x_144, x_145); -x_147 = lean_uint64_mix_hash(x_143, x_146); -x_23 = x_147; -goto block_130; -} -} -block_130: -{ -uint64_t x_24; uint64_t x_25; uint64_t x_26; uint64_t x_27; size_t x_28; size_t x_29; lean_object* x_30; lean_object* x_31; -x_24 = lean_uint64_shift_right(x_23, x_18); -x_25 = lean_uint64_xor(x_23, x_24); -x_26 = lean_uint64_shift_right(x_25, x_19); -x_27 = lean_uint64_xor(x_25, x_26); -x_28 = lean_uint64_to_usize(x_27); -x_29 = lean_usize_land(x_28, x_22); -x_30 = lean_array_uget(x_15, x_29); -x_31 = l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(x_13, x_30); -if (lean_obj_tag(x_31) == 0) -{ -lean_object* x_32; lean_object* x_33; uint8_t x_34; -x_32 = l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___closed__1; -x_33 = lean_array_push(x_32, x_12); -x_34 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_13, x_30); -if (x_34 == 0) -{ -lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; -x_35 = lean_unsigned_to_nat(1u); -x_36 = lean_nat_add(x_14, x_35); +x_18 = lean_array_get_size(x_16); +x_19 = 32; +x_20 = 16; +x_21 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_22 = 1; +x_23 = lean_usize_sub(x_21, x_22); +x_65 = lean_ctor_get(x_13, 0); +lean_inc(x_65); +x_66 = lean_unbox(x_65); +lean_dec(x_65); +if (x_66 == 0) +{ +lean_object* x_67; +x_67 = lean_ctor_get(x_13, 1); +lean_inc(x_67); +if (lean_obj_tag(x_67) == 0) +{ +uint64_t x_68; +x_68 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1; +x_24 = x_68; +goto block_64; +} +else +{ +lean_object* x_69; uint64_t x_70; uint64_t x_71; uint64_t x_72; uint64_t x_73; +x_69 = lean_ctor_get(x_67, 0); +lean_inc(x_69); +lean_dec(x_67); +x_70 = 13; +x_71 = lean_uint64_of_nat(x_69); +lean_dec(x_69); +x_72 = lean_uint64_mix_hash(x_71, x_70); +x_73 = lean_uint64_mix_hash(x_70, x_72); +x_24 = x_73; +goto block_64; +} +} +else +{ +lean_object* x_74; +x_74 = lean_ctor_get(x_13, 1); +lean_inc(x_74); +if (lean_obj_tag(x_74) == 0) +{ +uint64_t x_75; +x_75 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2; +x_24 = x_75; +goto block_64; +} +else +{ +lean_object* x_76; uint64_t x_77; uint64_t x_78; uint64_t x_79; uint64_t x_80; uint64_t x_81; +x_76 = lean_ctor_get(x_74, 0); +lean_inc(x_76); +lean_dec(x_74); +x_77 = 11; +x_78 = lean_uint64_of_nat(x_76); +lean_dec(x_76); +x_79 = 13; +x_80 = lean_uint64_mix_hash(x_78, x_79); +x_81 = lean_uint64_mix_hash(x_77, x_80); +x_24 = x_81; +goto block_64; +} +} +block_64: +{ +uint64_t x_25; uint64_t x_26; uint64_t x_27; uint64_t x_28; size_t x_29; size_t x_30; lean_object* x_31; uint8_t x_32; +x_25 = lean_uint64_shift_right(x_24, x_19); +x_26 = lean_uint64_xor(x_24, x_25); +x_27 = lean_uint64_shift_right(x_26, x_20); +x_28 = lean_uint64_xor(x_26, x_27); +x_29 = lean_uint64_to_usize(x_28); +x_30 = lean_usize_land(x_29, x_23); +x_31 = lean_array_uget(x_16, x_30); +x_32 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(x_13, x_31); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; lean_dec(x_14); +x_33 = l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___closed__1; +x_34 = lean_array_push(x_33, x_12); +x_35 = lean_unsigned_to_nat(1u); +x_36 = lean_nat_add(x_15, x_35); +lean_dec(x_15); x_37 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_37, 0, x_13); -lean_ctor_set(x_37, 1, x_33); -lean_ctor_set(x_37, 2, x_30); -x_38 = lean_array_uset(x_15, x_29, x_37); +lean_ctor_set(x_37, 1, x_34); +lean_ctor_set(x_37, 2, x_31); +x_38 = lean_array_uset(x_16, x_30, x_37); x_39 = lean_unsigned_to_nat(4u); x_40 = lean_nat_mul(x_36, x_39); x_41 = lean_unsigned_to_nat(3u); @@ -1988,15 +1805,15 @@ lean_dec(x_42); if (x_44 == 0) { lean_object* x_45; lean_object* x_46; size_t x_47; -x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(x_38); -if (lean_is_scalar(x_16)) { +x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_38); +if (lean_is_scalar(x_17)) { x_46 = lean_alloc_ctor(0, 2, 0); } else { - x_46 = x_16; + x_46 = x_17; } lean_ctor_set(x_46, 0, x_36); lean_ctor_set(x_46, 1, x_45); -x_47 = lean_usize_add(x_9, x_21); +x_47 = lean_usize_add(x_9, x_22); x_9 = x_47; x_10 = x_46; goto _start; @@ -2004,14 +1821,14 @@ goto _start; else { lean_object* x_49; size_t x_50; -if (lean_is_scalar(x_16)) { +if (lean_is_scalar(x_17)) { x_49 = lean_alloc_ctor(0, 2, 0); } else { - x_49 = x_16; + x_49 = x_17; } lean_ctor_set(x_49, 0, x_36); lean_ctor_set(x_49, 1, x_38); -x_50 = lean_usize_add(x_9, x_21); +x_50 = lean_usize_add(x_9, x_22); x_9 = x_50; x_10 = x_49; goto _start; @@ -2019,210 +1836,46 @@ goto _start; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; size_t x_56; +lean_object* x_52; lean_object* x_53; uint8_t x_54; lean_object* x_55; +lean_dec(x_12); lean_inc(x_5); -x_52 = lean_array_uset(x_15, x_29, x_5); -x_53 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_13, x_33, x_30); -x_54 = lean_array_uset(x_52, x_29, x_53); -if (lean_is_scalar(x_16)) { - x_55 = lean_alloc_ctor(0, 2, 0); -} else { - x_55 = x_16; -} -lean_ctor_set(x_55, 0, x_14); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_usize_add(x_9, x_21); -x_9 = x_56; -x_10 = x_55; -goto _start; -} -} -else -{ -lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_122; -x_58 = lean_ctor_get(x_31, 0); -lean_inc(x_58); -lean_dec(x_31); -x_59 = lean_array_push(x_58, x_12); -x_122 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_13, x_30); -if (x_122 == 0) -{ -lean_object* x_123; -lean_dec(x_30); -if (lean_is_scalar(x_16)) { - x_123 = lean_alloc_ctor(0, 2, 0); -} else { - x_123 = x_16; -} -lean_ctor_set(x_123, 0, x_14); -lean_ctor_set(x_123, 1, x_15); -x_60 = x_123; -goto block_121; -} -else +x_52 = lean_array_uset(x_16, x_30, x_5); +lean_inc(x_13); +x_53 = l_Std_DHashMap_Internal_AssocList_Const_alter___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___rarg(x_13, x_14, x_31); +x_54 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(x_13, x_53); +lean_dec(x_13); +x_55 = lean_array_uset(x_52, x_30, x_53); +if (x_54 == 0) { -lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -lean_inc(x_5); -x_124 = lean_array_uset(x_15, x_29, x_5); -x_125 = lean_unsigned_to_nat(1u); -x_126 = lean_nat_sub(x_14, x_125); -lean_dec(x_14); -x_127 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_13, x_30); -x_128 = lean_array_uset(x_124, x_29, x_127); -if (lean_is_scalar(x_16)) { - x_129 = lean_alloc_ctor(0, 2, 0); +lean_object* x_56; lean_object* x_57; lean_object* x_58; size_t x_59; +x_56 = lean_unsigned_to_nat(1u); +x_57 = lean_nat_sub(x_15, x_56); +lean_dec(x_15); +if (lean_is_scalar(x_17)) { + x_58 = lean_alloc_ctor(0, 2, 0); } else { - x_129 = x_16; -} -lean_ctor_set(x_129, 0, x_126); -lean_ctor_set(x_129, 1, x_128); -x_60 = x_129; -goto block_121; -} -block_121: -{ -uint8_t x_61; -x_61 = !lean_is_exclusive(x_60); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; size_t x_65; size_t x_66; size_t x_67; lean_object* x_68; uint8_t x_69; -x_62 = lean_ctor_get(x_60, 0); -x_63 = lean_ctor_get(x_60, 1); -x_64 = lean_array_get_size(x_63); -x_65 = lean_usize_of_nat(x_64); -lean_dec(x_64); -x_66 = lean_usize_sub(x_65, x_21); -x_67 = lean_usize_land(x_28, x_66); -x_68 = lean_array_uget(x_63, x_67); -x_69 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_13, x_68); -if (x_69 == 0) -{ -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; uint8_t x_79; -x_70 = lean_unsigned_to_nat(1u); -x_71 = lean_nat_add(x_62, x_70); -lean_dec(x_62); -x_72 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_72, 0, x_13); -lean_ctor_set(x_72, 1, x_59); -lean_ctor_set(x_72, 2, x_68); -x_73 = lean_array_uset(x_63, x_67, x_72); -x_74 = lean_unsigned_to_nat(4u); -x_75 = lean_nat_mul(x_71, x_74); -x_76 = lean_unsigned_to_nat(3u); -x_77 = lean_nat_div(x_75, x_76); -lean_dec(x_75); -x_78 = lean_array_get_size(x_73); -x_79 = lean_nat_dec_le(x_77, x_78); -lean_dec(x_78); -lean_dec(x_77); -if (x_79 == 0) -{ -lean_object* x_80; size_t x_81; -x_80 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(x_73); -lean_ctor_set(x_60, 1, x_80); -lean_ctor_set(x_60, 0, x_71); -x_81 = lean_usize_add(x_9, x_21); -x_9 = x_81; -x_10 = x_60; -goto _start; + x_58 = x_17; } -else -{ -size_t x_83; -lean_ctor_set(x_60, 1, x_73); -lean_ctor_set(x_60, 0, x_71); -x_83 = lean_usize_add(x_9, x_21); -x_9 = x_83; -x_10 = x_60; -goto _start; -} -} -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; size_t x_88; -lean_inc(x_5); -x_85 = lean_array_uset(x_63, x_67, x_5); -x_86 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_13, x_59, x_68); -x_87 = lean_array_uset(x_85, x_67, x_86); -lean_ctor_set(x_60, 1, x_87); -x_88 = lean_usize_add(x_9, x_21); -x_9 = x_88; -x_10 = x_60; -goto _start; -} -} -else -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; size_t x_93; size_t x_94; size_t x_95; lean_object* x_96; uint8_t x_97; -x_90 = lean_ctor_get(x_60, 0); -x_91 = lean_ctor_get(x_60, 1); -lean_inc(x_91); -lean_inc(x_90); -lean_dec(x_60); -x_92 = lean_array_get_size(x_91); -x_93 = lean_usize_of_nat(x_92); -lean_dec(x_92); -x_94 = lean_usize_sub(x_93, x_21); -x_95 = lean_usize_land(x_28, x_94); -x_96 = lean_array_uget(x_91, x_95); -x_97 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_13, x_96); -if (x_97 == 0) -{ -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; uint8_t x_107; -x_98 = lean_unsigned_to_nat(1u); -x_99 = lean_nat_add(x_90, x_98); -lean_dec(x_90); -x_100 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_100, 0, x_13); -lean_ctor_set(x_100, 1, x_59); -lean_ctor_set(x_100, 2, x_96); -x_101 = lean_array_uset(x_91, x_95, x_100); -x_102 = lean_unsigned_to_nat(4u); -x_103 = lean_nat_mul(x_99, x_102); -x_104 = lean_unsigned_to_nat(3u); -x_105 = lean_nat_div(x_103, x_104); -lean_dec(x_103); -x_106 = lean_array_get_size(x_101); -x_107 = lean_nat_dec_le(x_105, x_106); -lean_dec(x_106); -lean_dec(x_105); -if (x_107 == 0) -{ -lean_object* x_108; lean_object* x_109; size_t x_110; -x_108 = l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__4(x_101); -x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_99); -lean_ctor_set(x_109, 1, x_108); -x_110 = lean_usize_add(x_9, x_21); -x_9 = x_110; -x_10 = x_109; +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_55); +x_59 = lean_usize_add(x_9, x_22); +x_9 = x_59; +x_10 = x_58; goto _start; } else { -lean_object* x_112; size_t x_113; -x_112 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_112, 0, x_99); -lean_ctor_set(x_112, 1, x_101); -x_113 = lean_usize_add(x_9, x_21); -x_9 = x_113; -x_10 = x_112; -goto _start; -} +lean_object* x_61; size_t x_62; +if (lean_is_scalar(x_17)) { + x_61 = lean_alloc_ctor(0, 2, 0); +} else { + x_61 = x_17; } -else -{ -lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; size_t x_119; -lean_inc(x_5); -x_115 = lean_array_uset(x_91, x_95, x_5); -x_116 = l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_13, x_59, x_96); -x_117 = lean_array_uset(x_115, x_95, x_116); -x_118 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_118, 0, x_90); -lean_ctor_set(x_118, 1, x_117); -x_119 = lean_usize_add(x_9, x_21); -x_9 = x_119; -x_10 = x_118; +lean_ctor_set(x_61, 0, x_15); +lean_ctor_set(x_61, 1, x_55); +x_62 = lean_usize_add(x_9, x_22); +x_9 = x_62; +x_10 = x_61; goto _start; } } @@ -2230,8 +1883,6 @@ goto _start; } } } -} -} static lean_object* _init_l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__1() { _start: { @@ -2371,11 +2022,11 @@ x_6 = 0; x_7 = l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__6; x_8 = l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__10; x_9 = l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__13; -x_10 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_1, x_2, x_7, x_8, x_3, x_4, x_2, x_5, x_6, x_9); +x_10 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_7, x_8, x_3, x_4, x_2, x_5, x_6, x_9); return x_10; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -2400,7 +2051,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; @@ -2497,15 +2148,15 @@ return x_29; } } } -static lean_object* _init_l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -2518,7 +2169,7 @@ return x_2; else { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_8 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1; +x_8 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1; lean_inc(x_3); x_9 = l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(x_1, x_2, x_8, x_3, x_4, lean_box(0), lean_box(0)); x_10 = lean_ctor_get(x_9, 0); @@ -2530,7 +2181,7 @@ x_12 = lean_nat_dec_le(x_4, x_10); if (x_12 == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); +x_13 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); x_14 = lean_unsigned_to_nat(1u); x_15 = lean_nat_add(x_10, x_14); lean_dec(x_10); @@ -2549,7 +2200,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -2576,7 +2227,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -2585,7 +2236,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -2727,7 +2378,7 @@ size_t x_27; lean_object* x_28; lean_object* x_29; x_27 = lean_usize_of_nat(x_5); lean_dec(x_5); x_28 = l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_filterDuplicateCompletionInfos___closed__1; -x_29 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14(x_4, x_8, x_27, x_28); +x_29 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_4, x_8, x_27, x_28); lean_dec(x_4); x_9 = x_29; goto block_23; @@ -2748,21 +2399,21 @@ if (x_14 == 0) { lean_object* x_15; size_t x_16; lean_object* x_17; lean_inc(x_12); -x_15 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_10, x_9, x_12, x_12, lean_box(0), lean_box(0)); +x_15 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_10, x_9, x_12, x_12, lean_box(0), lean_box(0)); lean_dec(x_12); lean_dec(x_10); x_16 = lean_array_size(x_15); -x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(x_16, x_8, x_15); +x_17 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_16, x_8, x_15); return x_17; } else { lean_object* x_18; size_t x_19; lean_object* x_20; -x_18 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_10, x_9, x_6, x_12, lean_box(0), lean_box(0)); +x_18 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_10, x_9, x_6, x_12, lean_box(0), lean_box(0)); lean_dec(x_12); lean_dec(x_10); x_19 = lean_array_size(x_18); -x_20 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(x_19, x_8, x_18); +x_20 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_19, x_8, x_18); return x_20; } } @@ -2772,43 +2423,24 @@ size_t x_21; lean_object* x_22; lean_dec(x_12); lean_dec(x_10); x_21 = lean_array_size(x_9); -x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(x_21, x_8, x_9); +x_22 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_21, x_8, x_9); return x_22; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__2(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_erase___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -2816,7 +2448,7 @@ x_11 = lean_unbox_usize(x_8); lean_dec(x_8); x_12 = lean_unbox_usize(x_9); lean_dec(x_9); -x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); +x_13 = l_Array_forIn_x27Unsafe_loop___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); @@ -2834,37 +2466,37 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__9(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___lambda__1(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -2872,11 +2504,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__13(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__11(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -2884,7 +2516,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__14(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -2931,8 +2563,8 @@ l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__3___closed__4 = _ini lean_mark_persistent(l_Lean_Server_Completion_findCompletionInfosAt_go___lambda__3___closed__4); l_Lean_Server_Completion_findCompletionInfosAt___closed__1 = _init_l_Lean_Server_Completion_findCompletionInfosAt___closed__1(); lean_mark_persistent(l_Lean_Server_Completion_findCompletionInfosAt___closed__1); -l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__1(); -l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__7___closed__2(); +l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__1(); +l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2 = _init_l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__5___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__6___closed__2(); l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__1 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__1(); lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__1); l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__2 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__2(); @@ -2959,8 +2591,8 @@ l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__12); l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__13 = _init_l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__13(); lean_mark_persistent(l_Array_groupByKey___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__1___closed__13); -l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1 = _init_l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__12___closed__1); +l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1 = _init_l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___spec__10___closed__1); l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___closed__1 = _init_l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___closed__1(); lean_mark_persistent(l___private_Lean_Server_Completion_CompletionInfoSelection_0__Lean_Server_Completion_computePrioritizedCompletionPartitions___closed__1); return lean_io_result_mk_ok(lean_box(0)); diff --git a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c index fe4458f93206..d2f6edf35d0e 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c +++ b/stage0/stdlib/Lean/Server/FileWorker/RequestHandling.c @@ -21,6 +21,7 @@ LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Server_FileWorker_computeDeltaL static lean_object* l_Array_groupByKey___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_collectInfoBasedSemanticTokens(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__17___lambda__2(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__18(lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__16(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__13___lambda__4___closed__1; @@ -50,7 +51,6 @@ static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_Fil lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSemanticTokens____x40_Lean_Data_Lsp_LanguageFeatures___hyg_10571_(lean_object*); lean_object* l_Lean_Server_Snapshots_Snapshot_infoTree(lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonDocumentSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4717_(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10___boxed(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_collectSyntaxBasedSemanticTokens(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_run___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -83,7 +83,6 @@ static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePla static lean_object* l_List_mapM_loop___at_Lean_Server_FileWorker_getInteractiveGoals___spec__2___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens_run(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__1; -lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(lean_object*, lean_object*); uint64_t l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_hashPosition____x40_Lean_Data_Lsp_Basic___hyg_180_(lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__4___lambda__3___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__21___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); @@ -102,6 +101,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_NamespaceEntry_finish___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Server_FileWorker_keywordSemanticTokenMap___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__24___lambda__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__21___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -232,6 +232,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__ static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__7; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__7___lambda__2___closed__2; static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__14; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleCompletionItemResolve(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__11(lean_object*, lean_object*, size_t, size_t); @@ -239,6 +240,7 @@ uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_filterDuplicateSemanticTokens___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_findSomeM_x3f___at_Lean_Server_FileWorker_handleHover___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___closed__2; static lean_object* l_List_findSomeM_x3f___at_Lean_Server_FileWorker_handleHover___spec__2___closed__1; static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__18; @@ -248,17 +250,16 @@ static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymb LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__37___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols_popStack(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__15(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Lean_PersistentArray_anyMAux___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__10(lean_object*, lean_object*); uint64_t l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_hashRefIdent____x40_Lean_Data_Lsp_Internal___hyg_158_(lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__4; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__19(lean_object*, lean_object*, lean_object*); uint8_t l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_beqPosition____x40_Lean_Data_Lsp_Basic___hyg_41_(lean_object*, lean_object*); lean_object* l_Lean_Server_RequestM_findInfoTreeAtPosWithTrailingWhitespace(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__17; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__2(lean_object*, lean_object*, lean_object*); static lean_object* l_List_mapM_loop___at_Lean_Server_FileWorker_getInteractiveGoals___spec__2___closed__3; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_FileWorker_computeDeltaLspSemanticTokens___spec__2___lambda__1___boxed(lean_object*, lean_object*); @@ -331,7 +332,6 @@ LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleHover___lambda__2(lean_object LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__2___boxed(lean_object*, lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonFoldingRange____x40_Lean_Data_Lsp_LanguageFeatures___hyg_10800_(lean_object*); uint8_t lean_uint32_dec_le(uint32_t, uint32_t); lean_object* l_Lean_RBNode_setBlack___rarg(lean_object*); @@ -390,6 +390,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lamb static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1___closed__1; static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__9___closed__8; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7___lambda__1(lean_object*, lean_object*); lean_object* l_IO_sleep(uint32_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__13___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_instHashableAbsoluteLspSemanticToken; @@ -438,7 +439,6 @@ lean_object* l_Lean_PersistentHashMap_insert___at_Lean_Server_registerLspRequest LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleHover___lambda__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__9___closed__4; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentHighlight___lambda__2(lean_object*, size_t, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonSemanticTokensRangeParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_10284_(lean_object*); LEAN_EXPORT lean_object* l_Lean_PersistentArray_anyMAux___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__2___boxed(lean_object*, lean_object*); @@ -452,7 +452,6 @@ LEAN_EXPORT uint8_t l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_S lean_object* l_Lean_Expr_constName_x3f(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__17___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Option_bindM___at_Lean_Server_FileWorker_getInteractiveTermGoal___spec__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange(lean_object*); @@ -481,7 +480,6 @@ lean_object* l_Array_mapMUnsafe_map___at_Lean_Lsp_instToJsonDocumentSymbol_go___ lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__8(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_MapDeclarationExtension_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__11(lean_object*); lean_object* l_Lean_Server_locationLinksFromDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -494,7 +492,6 @@ lean_object* l_Lean_Syntax_getArg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_liftExcept___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__15(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Lean_Syntax_matchesNull(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_anyMUnsafe_any___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__12(lean_object*, lean_object*, size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_instToJsonAbsoluteLspSemanticToken; static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__3; @@ -505,6 +502,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokens___lambda_ LEAN_EXPORT uint8_t l_Lean_Server_FileWorker_handleHover___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDefinition___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics_waitLoop___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -523,6 +521,7 @@ static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___lambda__1___close static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1___lambda__3(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__35(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(lean_object*, lean_object*); extern lean_object* l_Std_Format_defWidth; static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__2; LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at_Lean_Server_FileWorker_keywordSemanticTokenMap___spec__1(lean_object*, lean_object*, uint8_t); @@ -532,7 +531,7 @@ static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_S LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRangeFromSyntax___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__34___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); @@ -560,6 +559,7 @@ lean_object* l_Lean_Meta_isInstance(lean_object*, lean_object*, lean_object*, le static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__11; static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__1(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__3___closed__2; lean_object* l_IO_AsyncList_waitUntil___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); @@ -573,6 +573,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Serve LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__30___lambda__2(lean_object*); static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__21; +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__13; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_collectSyntaxBasedSemanticTokens___spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__3; @@ -624,8 +625,8 @@ lean_object* l_List_drop___rarg(lean_object*, lean_object*); lean_object* l_Lean_Syntax_findStack_x3f(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__13; LEAN_EXPORT lean_object* l_List_mapTR_loop___at_Lean_Server_FileWorker_handleDocumentSymbol___spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleWaitForDiagnostics___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__17___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_List_findSomeM_x3f___at_Lean_Server_FileWorker_handleHover___spec__2___closed__3; @@ -652,6 +653,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_parseRequestParams___at_Lean_Server_FileW LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__4___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__14; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__30___lambda__4___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_NamespaceEntry_finish___closed__4; static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__12; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__30(lean_object*, lean_object*, lean_object*); @@ -718,6 +720,7 @@ lean_object* l_String_intercalate(lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__3(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -726,8 +729,6 @@ static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_Fil static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__5; static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__14; static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__10___lambda__3___closed__1; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handleDocumentHighlight___spec__4(size_t, size_t, lean_object*); @@ -742,9 +743,7 @@ static lean_object* l_Array_groupByKey___at_Lean_Server_FileWorker_filterDuplica LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__11___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__10___lambda__5(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__34___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(lean_object*); static lean_object* l_Lean_Server_FileWorker_keywordSemanticTokenMap___closed__3; lean_object* lean_array_uget(lean_object*, size_t); lean_object* l_Lean_Elab_Info_lctx(lean_object*); @@ -773,7 +772,6 @@ lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_o lean_object* l_IO_AsyncList_getFinishedPrefix___rarg(lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__9___closed__3; static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__8; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__15; lean_object* l___private_Lean_Expr_0__Lean_Expr_getAppArgsAux(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -782,9 +780,9 @@ static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_Fil static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1___lambda__3___closed__2; static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__11; LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__34___lambda__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__13___lambda__1(lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addCommandRange___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_collectInfoBasedSemanticTokens___lambda__1(lean_object*, lean_object*); @@ -792,7 +790,6 @@ uint8_t l_Lean_PersistentHashMap_contains___at_Lean_Server_registerLspRequestHan LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_locationLinksOfInfo___spec__14(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__27___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleSemanticTokensFull___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); static lean_object* l_Lean_Server_FileWorker_handlePlainGoal___closed__3; static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__24; @@ -819,6 +816,7 @@ static lean_object* l_Lean_Server_FileWorker_collectInfoBasedSemanticTokens___cl static lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_handleDocumentHighlight_highlightReturn_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleFoldingRange_isImport___closed__5; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_handlePlainGoal___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at_Lean_Server_FileWorker_keywordSemanticTokenMap___spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__6___closed__3; @@ -857,6 +855,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleFoldingRange_addRange(le static lean_object* l_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____closed__22; lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__7___lambda__4___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6(lean_object*); static lean_object* l_Lean_Server_FileWorker_noHighlightKinds___closed__3; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_handleDocumentSymbol_toDocumentSymbols___lambda__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Array_contains___at_Lean_Server_FileWorker_collectSyntaxBasedSemanticTokens___spec__4(lean_object*, lean_object*); @@ -870,7 +869,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__ static lean_object* l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_fromJsonAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8962____closed__5; LEAN_EXPORT lean_object* l_Lean_Server_FileWorker_locationLinksOfInfo___lambda__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__27___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_pure___at_Lean_Server_FileWorker_handleHover___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerLspRequestHandler___at_Lean_Server_FileWorker_initFn____x40_Lean_Server_FileWorker_RequestHandling___hyg_12951____spec__1___lambda__3___closed__1; @@ -24415,7 +24413,7 @@ x_20 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_20, 0, x_7); lean_ctor_set(x_20, 1, x_19); x_21 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_22 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_20, x_21); +x_22 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_20, x_21); x_23 = l_Lean_Json_mkObj(x_22); return x_23; } @@ -24636,39 +24634,7 @@ lean_dec(x_2); return x_5; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_ctor_get(x_2, 2); -x_7 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_4, x_1); -if (x_7 == 0) -{ -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_9; -lean_inc(x_5); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_5); -return x_9; -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -24697,7 +24663,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -24771,7 +24737,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -24790,7 +24756,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -24801,7 +24767,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -24812,151 +24778,179 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_4; -lean_dec(x_2); -lean_dec(x_1); +lean_object* x_4; lean_object* x_5; x_4 = lean_box(0); -return x_4; -} -else -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_3, 0); -x_7 = lean_ctor_get(x_3, 1); -x_8 = lean_ctor_get(x_3, 2); -x_9 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_6, x_1); -if (x_9 == 0) +x_5 = lean_apply_1(x_2, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_10); -return x_3; +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; } else { -lean_dec(x_7); -lean_dec(x_6); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_1); -return x_3; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_7); +lean_ctor_set(x_9, 2, x_8); +return x_9; } } else { +uint8_t x_10; +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_11 = lean_ctor_get(x_3, 0); x_12 = lean_ctor_get(x_3, 1); x_13 = lean_ctor_get(x_3, 2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_3); x_14 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_11, x_1); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_1, x_2, x_13); -x_16 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_16, 0, x_11); -lean_ctor_set(x_16, 1, x_12); -lean_ctor_set(x_16, 2, x_15); -return x_16; +lean_object* x_15; +x_15 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_15); +return x_3; } else { -lean_object* x_17; -lean_dec(x_12); +lean_object* x_16; lean_object* x_17; lean_dec(x_11); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_2); -lean_ctor_set(x_17, 2, x_13); -return x_17; -} +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_12); +x_17 = lean_apply_1(x_2, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_free_object(x_3); +lean_dec(x_1); +return x_13; } +else +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +lean_dec(x_17); +lean_ctor_set(x_3, 1, x_18); +lean_ctor_set(x_3, 0, x_1); +return x_3; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_3, 0); +x_20 = lean_ctor_get(x_3, 1); +x_21 = lean_ctor_get(x_3, 2); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_3); +x_22 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_19, x_1); +if (x_22 == 0) { -lean_object* x_3; -x_3 = lean_box(0); -return x_3; +lean_object* x_23; lean_object* x_24; +x_23 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(x_1, x_2, x_21); +x_24 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_20); +lean_ctor_set(x_24, 2, x_23); +return x_24; } else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_5, x_1); -if (x_8 == 0) +lean_object* x_25; lean_object* x_26; +lean_dec(x_19); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_20); +x_26 = lean_apply_1(x_2, x_25); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_9; -x_9 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_1, x_7); -lean_ctor_set(x_2, 2, x_9); -return x_2; +lean_dec(x_1); +return x_21; } else { -lean_free_object(x_2); -lean_dec(x_6); -lean_dec(x_5); -return x_7; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +lean_dec(x_26); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_1); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set(x_28, 2, x_21); +return x_28; } } -else +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6(lean_object* x_1) { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -x_12 = lean_ctor_get(x_2, 2); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_2); -x_13 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_beqAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8822_(x_10, x_1); -if (x_13 == 0) +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_14; lean_object* x_15; -x_14 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_1, x_12); -x_15 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_11); -lean_ctor_set(x_15, 2, x_14); -return x_15; +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -lean_dec(x_11); -lean_dec(x_10); -return x_12; +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); +return x_2; } +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -24969,50 +24963,50 @@ return x_8; } else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; x_10 = lean_array_uget(x_5, x_7); lean_inc(x_1); lean_inc(x_10); x_11 = lean_apply_1(x_1, x_10); -x_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; -x_13 = lean_ctor_get(x_8, 0); -x_14 = lean_ctor_get(x_8, 1); -x_15 = lean_array_get_size(x_14); -x_16 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_hashAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8912_(x_11); -x_17 = 32; -x_18 = lean_uint64_shift_right(x_16, x_17); -x_19 = lean_uint64_xor(x_16, x_18); -x_20 = 16; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = lean_uint64_to_usize(x_22); -x_24 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_25 = 1; -x_26 = lean_usize_sub(x_24, x_25); -x_27 = lean_usize_land(x_23, x_26); -x_28 = lean_array_uget(x_14, x_27); -x_29 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_28); -if (lean_obj_tag(x_29) == 0) +lean_inc(x_10); +x_12 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7___lambda__1), 2, 1); +lean_closure_set(x_12, 0, x_10); +x_13 = !lean_is_exclusive(x_8); +if (x_13 == 0) { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_31 = lean_array_push(x_30, x_10); -x_32 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_28); -if (x_32 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_8, 0); +x_15 = lean_ctor_get(x_8, 1); +x_16 = lean_array_get_size(x_15); +x_17 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_hashAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8912_(x_11); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_29); +if (x_30 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_dec(x_12); +x_31 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; +x_32 = lean_array_push(x_31, x_10); x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_nat_add(x_13, x_33); -lean_dec(x_13); +x_34 = lean_nat_add(x_14, x_33); +lean_dec(x_14); x_35 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_35, 0, x_11); -lean_ctor_set(x_35, 1, x_31); -lean_ctor_set(x_35, 2, x_28); -x_36 = lean_array_uset(x_14, x_27, x_35); +lean_ctor_set(x_35, 1, x_32); +lean_ctor_set(x_35, 2, x_29); +x_36 = lean_array_uset(x_15, x_28, x_35); x_37 = lean_unsigned_to_nat(4u); x_38 = lean_nat_mul(x_34, x_37); x_39 = lean_unsigned_to_nat(3u); @@ -25025,10 +25019,10 @@ lean_dec(x_40); if (x_42 == 0) { lean_object* x_43; size_t x_44; -x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_36); +x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_36); lean_ctor_set(x_8, 1, x_43); lean_ctor_set(x_8, 0, x_34); -x_44 = lean_usize_add(x_7, x_25); +x_44 = lean_usize_add(x_7, x_26); x_7 = x_44; goto _start; } @@ -25037,418 +25031,149 @@ else size_t x_46; lean_ctor_set(x_8, 1, x_36); lean_ctor_set(x_8, 0, x_34); -x_46 = lean_usize_add(x_7, x_25); +x_46 = lean_usize_add(x_7, x_26); x_7 = x_46; goto _start; } } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; size_t x_51; -lean_inc(x_3); -x_48 = lean_array_uset(x_14, x_27, x_3); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_11, x_31, x_28); -x_50 = lean_array_uset(x_48, x_27, x_49); -lean_ctor_set(x_8, 1, x_50); -x_51 = lean_usize_add(x_7, x_25); -x_7 = x_51; -goto _start; -} -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_117; -x_53 = lean_ctor_get(x_29, 0); -lean_inc(x_53); -lean_dec(x_29); -x_54 = lean_array_push(x_53, x_10); -x_117 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_28); -if (x_117 == 0) -{ -lean_dec(x_28); -x_55 = x_8; -goto block_116; -} -else -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_inc(x_3); -x_118 = lean_array_uset(x_14, x_27, x_3); -x_119 = lean_unsigned_to_nat(1u); -x_120 = lean_nat_sub(x_13, x_119); -lean_dec(x_13); -x_121 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_11, x_28); -x_122 = lean_array_uset(x_118, x_27, x_121); -lean_ctor_set(x_8, 1, x_122); -lean_ctor_set(x_8, 0, x_120); -x_55 = x_8; -goto block_116; -} -block_116: -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; size_t x_62; lean_object* x_63; uint8_t x_64; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_ctor_get(x_55, 1); -x_59 = lean_array_get_size(x_58); -x_60 = lean_usize_of_nat(x_59); -lean_dec(x_59); -x_61 = lean_usize_sub(x_60, x_25); -x_62 = lean_usize_land(x_23, x_61); -x_63 = lean_array_uget(x_58, x_62); -x_64 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_63); -if (x_64 == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_nat_add(x_57, x_65); -lean_dec(x_57); -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_11); -lean_ctor_set(x_67, 1, x_54); -lean_ctor_set(x_67, 2, x_63); -x_68 = lean_array_uset(x_58, x_62, x_67); -x_69 = lean_unsigned_to_nat(4u); -x_70 = lean_nat_mul(x_66, x_69); -x_71 = lean_unsigned_to_nat(3u); -x_72 = lean_nat_div(x_70, x_71); -lean_dec(x_70); -x_73 = lean_array_get_size(x_68); -x_74 = lean_nat_dec_le(x_72, x_73); -lean_dec(x_73); -lean_dec(x_72); -if (x_74 == 0) -{ -lean_object* x_75; size_t x_76; -x_75 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_68); -lean_ctor_set(x_55, 1, x_75); -lean_ctor_set(x_55, 0, x_66); -x_76 = lean_usize_add(x_7, x_25); -x_7 = x_76; -x_8 = x_55; -goto _start; -} -else -{ -size_t x_78; -lean_ctor_set(x_55, 1, x_68); -lean_ctor_set(x_55, 0, x_66); -x_78 = lean_usize_add(x_7, x_25); -x_7 = x_78; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; size_t x_83; +lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +lean_dec(x_10); lean_inc(x_3); -x_80 = lean_array_uset(x_58, x_62, x_3); -x_81 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_11, x_54, x_63); -x_82 = lean_array_uset(x_80, x_62, x_81); -lean_ctor_set(x_55, 1, x_82); -x_83 = lean_usize_add(x_7, x_25); -x_7 = x_83; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; size_t x_88; size_t x_89; size_t x_90; lean_object* x_91; uint8_t x_92; -x_85 = lean_ctor_get(x_55, 0); -x_86 = lean_ctor_get(x_55, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_55); -x_87 = lean_array_get_size(x_86); -x_88 = lean_usize_of_nat(x_87); -lean_dec(x_87); -x_89 = lean_usize_sub(x_88, x_25); -x_90 = lean_usize_land(x_23, x_89); -x_91 = lean_array_uget(x_86, x_90); -x_92 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_91); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_93 = lean_unsigned_to_nat(1u); -x_94 = lean_nat_add(x_85, x_93); -lean_dec(x_85); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_11); -lean_ctor_set(x_95, 1, x_54); -lean_ctor_set(x_95, 2, x_91); -x_96 = lean_array_uset(x_86, x_90, x_95); -x_97 = lean_unsigned_to_nat(4u); -x_98 = lean_nat_mul(x_94, x_97); -x_99 = lean_unsigned_to_nat(3u); -x_100 = lean_nat_div(x_98, x_99); -lean_dec(x_98); -x_101 = lean_array_get_size(x_96); -x_102 = lean_nat_dec_le(x_100, x_101); -lean_dec(x_101); -lean_dec(x_100); -if (x_102 == 0) -{ -lean_object* x_103; lean_object* x_104; size_t x_105; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_96); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_94); -lean_ctor_set(x_104, 1, x_103); -x_105 = lean_usize_add(x_7, x_25); -x_7 = x_105; -x_8 = x_104; -goto _start; -} -else +x_48 = lean_array_uset(x_15, x_28, x_3); +lean_inc(x_11); +x_49 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(x_11, x_12, x_29); +x_50 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_49); +lean_dec(x_11); +x_51 = lean_array_uset(x_48, x_28, x_49); +if (x_50 == 0) { -lean_object* x_107; size_t x_108; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_94); -lean_ctor_set(x_107, 1, x_96); -x_108 = lean_usize_add(x_7, x_25); -x_7 = x_108; -x_8 = x_107; +lean_object* x_52; lean_object* x_53; size_t x_54; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_sub(x_14, x_52); +lean_dec(x_14); +lean_ctor_set(x_8, 1, x_51); +lean_ctor_set(x_8, 0, x_53); +x_54 = lean_usize_add(x_7, x_26); +x_7 = x_54; goto _start; } -} else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; size_t x_114; -lean_inc(x_3); -x_110 = lean_array_uset(x_86, x_90, x_3); -x_111 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_11, x_54, x_91); -x_112 = lean_array_uset(x_110, x_90, x_111); -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_85); -lean_ctor_set(x_113, 1, x_112); -x_114 = lean_usize_add(x_7, x_25); -x_7 = x_114; -x_8 = x_113; +size_t x_56; +lean_ctor_set(x_8, 1, x_51); +x_56 = lean_usize_add(x_7, x_26); +x_7 = x_56; goto _start; } } } -} -} else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; uint64_t x_126; uint64_t x_127; uint64_t x_128; uint64_t x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; size_t x_133; size_t x_134; size_t x_135; size_t x_136; size_t x_137; lean_object* x_138; lean_object* x_139; -x_123 = lean_ctor_get(x_8, 0); -x_124 = lean_ctor_get(x_8, 1); -lean_inc(x_124); -lean_inc(x_123); +lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; size_t x_68; size_t x_69; size_t x_70; size_t x_71; size_t x_72; lean_object* x_73; uint8_t x_74; +x_58 = lean_ctor_get(x_8, 0); +x_59 = lean_ctor_get(x_8, 1); +lean_inc(x_59); +lean_inc(x_58); lean_dec(x_8); -x_125 = lean_array_get_size(x_124); -x_126 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_hashAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8912_(x_11); -x_127 = 32; -x_128 = lean_uint64_shift_right(x_126, x_127); -x_129 = lean_uint64_xor(x_126, x_128); -x_130 = 16; -x_131 = lean_uint64_shift_right(x_129, x_130); -x_132 = lean_uint64_xor(x_129, x_131); -x_133 = lean_uint64_to_usize(x_132); -x_134 = lean_usize_of_nat(x_125); -lean_dec(x_125); -x_135 = 1; -x_136 = lean_usize_sub(x_134, x_135); -x_137 = lean_usize_land(x_133, x_136); -x_138 = lean_array_uget(x_124, x_137); -x_139 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_138); -if (lean_obj_tag(x_139) == 0) -{ -lean_object* x_140; lean_object* x_141; uint8_t x_142; -x_140 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_141 = lean_array_push(x_140, x_10); -x_142 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_138); -if (x_142 == 0) +x_60 = lean_array_get_size(x_59); +x_61 = l___private_Lean_Server_FileWorker_RequestHandling_0__Lean_Server_FileWorker_hashAbsoluteLspSemanticToken____x40_Lean_Server_FileWorker_RequestHandling___hyg_8912_(x_11); +x_62 = 32; +x_63 = lean_uint64_shift_right(x_61, x_62); +x_64 = lean_uint64_xor(x_61, x_63); +x_65 = 16; +x_66 = lean_uint64_shift_right(x_64, x_65); +x_67 = lean_uint64_xor(x_64, x_66); +x_68 = lean_uint64_to_usize(x_67); +x_69 = lean_usize_of_nat(x_60); +lean_dec(x_60); +x_70 = 1; +x_71 = lean_usize_sub(x_69, x_70); +x_72 = lean_usize_land(x_68, x_71); +x_73 = lean_array_uget(x_59, x_72); +x_74 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_73); +if (x_74 == 0) { -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; -x_143 = lean_unsigned_to_nat(1u); -x_144 = lean_nat_add(x_123, x_143); -lean_dec(x_123); -x_145 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_145, 0, x_11); -lean_ctor_set(x_145, 1, x_141); -lean_ctor_set(x_145, 2, x_138); -x_146 = lean_array_uset(x_124, x_137, x_145); -x_147 = lean_unsigned_to_nat(4u); -x_148 = lean_nat_mul(x_144, x_147); -x_149 = lean_unsigned_to_nat(3u); -x_150 = lean_nat_div(x_148, x_149); -lean_dec(x_148); -x_151 = lean_array_get_size(x_146); -x_152 = lean_nat_dec_le(x_150, x_151); -lean_dec(x_151); -lean_dec(x_150); -if (x_152 == 0) -{ -lean_object* x_153; lean_object* x_154; size_t x_155; -x_153 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_146); -x_154 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_154, 0, x_144); -lean_ctor_set(x_154, 1, x_153); -x_155 = lean_usize_add(x_7, x_135); -x_7 = x_155; -x_8 = x_154; -goto _start; -} -else +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +lean_dec(x_12); +x_75 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; +x_76 = lean_array_push(x_75, x_10); +x_77 = lean_unsigned_to_nat(1u); +x_78 = lean_nat_add(x_58, x_77); +lean_dec(x_58); +x_79 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_79, 0, x_11); +lean_ctor_set(x_79, 1, x_76); +lean_ctor_set(x_79, 2, x_73); +x_80 = lean_array_uset(x_59, x_72, x_79); +x_81 = lean_unsigned_to_nat(4u); +x_82 = lean_nat_mul(x_78, x_81); +x_83 = lean_unsigned_to_nat(3u); +x_84 = lean_nat_div(x_82, x_83); +lean_dec(x_82); +x_85 = lean_array_get_size(x_80); +x_86 = lean_nat_dec_le(x_84, x_85); +lean_dec(x_85); +lean_dec(x_84); +if (x_86 == 0) { -lean_object* x_157; size_t x_158; -x_157 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_157, 0, x_144); -lean_ctor_set(x_157, 1, x_146); -x_158 = lean_usize_add(x_7, x_135); -x_7 = x_158; -x_8 = x_157; +lean_object* x_87; lean_object* x_88; size_t x_89; +x_87 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_80); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_78); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_7, x_70); +x_7 = x_89; +x_8 = x_88; goto _start; } -} else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; size_t x_164; -lean_inc(x_3); -x_160 = lean_array_uset(x_124, x_137, x_3); -x_161 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_11, x_141, x_138); -x_162 = lean_array_uset(x_160, x_137, x_161); -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_123); -lean_ctor_set(x_163, 1, x_162); -x_164 = lean_usize_add(x_7, x_135); -x_7 = x_164; -x_8 = x_163; +lean_object* x_91; size_t x_92; +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_78); +lean_ctor_set(x_91, 1, x_80); +x_92 = lean_usize_add(x_7, x_70); +x_7 = x_92; +x_8 = x_91; goto _start; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_202; -x_166 = lean_ctor_get(x_139, 0); -lean_inc(x_166); -lean_dec(x_139); -x_167 = lean_array_push(x_166, x_10); -x_202 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_138); -if (x_202 == 0) -{ -lean_object* x_203; -lean_dec(x_138); -x_203 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_203, 0, x_123); -lean_ctor_set(x_203, 1, x_124); -x_168 = x_203; -goto block_201; -} -else -{ -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; +lean_object* x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; +lean_dec(x_10); lean_inc(x_3); -x_204 = lean_array_uset(x_124, x_137, x_3); -x_205 = lean_unsigned_to_nat(1u); -x_206 = lean_nat_sub(x_123, x_205); -lean_dec(x_123); -x_207 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_11, x_138); -x_208 = lean_array_uset(x_204, x_137, x_207); -x_209 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_209, 0, x_206); -lean_ctor_set(x_209, 1, x_208); -x_168 = x_209; -goto block_201; -} -block_201: -{ -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; size_t x_173; size_t x_174; size_t x_175; lean_object* x_176; uint8_t x_177; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -x_170 = lean_ctor_get(x_168, 1); -lean_inc(x_170); -if (lean_is_exclusive(x_168)) { - lean_ctor_release(x_168, 0); - lean_ctor_release(x_168, 1); - x_171 = x_168; -} else { - lean_dec_ref(x_168); - x_171 = lean_box(0); -} -x_172 = lean_array_get_size(x_170); -x_173 = lean_usize_of_nat(x_172); -lean_dec(x_172); -x_174 = lean_usize_sub(x_173, x_135); -x_175 = lean_usize_land(x_133, x_174); -x_176 = lean_array_uget(x_170, x_175); -x_177 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_11, x_176); -if (x_177 == 0) -{ -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; -x_178 = lean_unsigned_to_nat(1u); -x_179 = lean_nat_add(x_169, x_178); -lean_dec(x_169); -x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_11); -lean_ctor_set(x_180, 1, x_167); -lean_ctor_set(x_180, 2, x_176); -x_181 = lean_array_uset(x_170, x_175, x_180); -x_182 = lean_unsigned_to_nat(4u); -x_183 = lean_nat_mul(x_179, x_182); -x_184 = lean_unsigned_to_nat(3u); -x_185 = lean_nat_div(x_183, x_184); -lean_dec(x_183); -x_186 = lean_array_get_size(x_181); -x_187 = lean_nat_dec_le(x_185, x_186); -lean_dec(x_186); -lean_dec(x_185); -if (x_187 == 0) -{ -lean_object* x_188; lean_object* x_189; size_t x_190; -x_188 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__4(x_181); -if (lean_is_scalar(x_171)) { - x_189 = lean_alloc_ctor(0, 2, 0); -} else { - x_189 = x_171; -} -lean_ctor_set(x_189, 0, x_179); -lean_ctor_set(x_189, 1, x_188); -x_190 = lean_usize_add(x_7, x_135); -x_7 = x_190; -x_8 = x_189; -goto _start; -} -else +x_94 = lean_array_uset(x_59, x_72, x_3); +lean_inc(x_11); +x_95 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__6___rarg(x_11, x_12, x_73); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_11, x_95); +lean_dec(x_11); +x_97 = lean_array_uset(x_94, x_72, x_95); +if (x_96 == 0) { -lean_object* x_192; size_t x_193; -if (lean_is_scalar(x_171)) { - x_192 = lean_alloc_ctor(0, 2, 0); -} else { - x_192 = x_171; -} -lean_ctor_set(x_192, 0, x_179); -lean_ctor_set(x_192, 1, x_181); -x_193 = lean_usize_add(x_7, x_135); -x_7 = x_193; -x_8 = x_192; +lean_object* x_98; lean_object* x_99; lean_object* x_100; size_t x_101; +x_98 = lean_unsigned_to_nat(1u); +x_99 = lean_nat_sub(x_58, x_98); +lean_dec(x_58); +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_99); +lean_ctor_set(x_100, 1, x_97); +x_101 = lean_usize_add(x_7, x_70); +x_7 = x_101; +x_8 = x_100; goto _start; } -} else { -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; size_t x_199; -lean_inc(x_3); -x_195 = lean_array_uset(x_170, x_175, x_3); -x_196 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_11, x_167, x_176); -x_197 = lean_array_uset(x_195, x_175, x_196); -if (lean_is_scalar(x_171)) { - x_198 = lean_alloc_ctor(0, 2, 0); -} else { - x_198 = x_171; -} -lean_ctor_set(x_198, 0, x_169); -lean_ctor_set(x_198, 1, x_197); -x_199 = lean_usize_add(x_7, x_135); -x_7 = x_199; -x_8 = x_198; +lean_object* x_103; size_t x_104; +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_58); +lean_ctor_set(x_103, 1, x_97); +x_104 = lean_usize_add(x_7, x_70); +x_7 = x_104; +x_8 = x_103; goto _start; } } @@ -25456,7 +25181,6 @@ goto _start; } } } -} static lean_object* _init_l_Array_groupByKey___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__1___closed__1() { _start: { @@ -25498,11 +25222,11 @@ x_4 = lean_box(0); x_5 = lean_array_size(x_2); x_6 = 0; x_7 = l_Array_groupByKey___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__1___closed__3; -x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); +x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -25527,7 +25251,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -25554,7 +25278,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -25563,7 +25287,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -25614,7 +25338,7 @@ lean_dec(x_5); lean_dec(x_4); x_9 = l_Lean_Server_FileWorker_filterDuplicateSemanticTokens___closed__2; x_10 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(x_9, x_8, x_10); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_9, x_8, x_10); return x_11; } else @@ -25628,7 +25352,7 @@ lean_dec(x_5); lean_dec(x_4); x_13 = l_Lean_Server_FileWorker_filterDuplicateSemanticTokens___closed__2; x_14 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(x_13, x_8, x_14); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_13, x_8, x_14); return x_15; } else @@ -25637,46 +25361,27 @@ size_t x_16; lean_object* x_17; lean_object* x_18; size_t x_19; lean_object* x_2 x_16 = lean_usize_of_nat(x_5); lean_dec(x_5); x_17 = l_Lean_Server_FileWorker_locationLinksOfInfo_extractInstances___closed__1; -x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12(x_4, x_8, x_16, x_17); +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(x_4, x_8, x_16, x_17); lean_dec(x_4); x_19 = lean_array_size(x_18); -x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(x_19, x_8, x_18); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_19, x_8, x_18); return x_20; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__2(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_1, x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { size_t x_9; size_t x_10; lean_object* x_11; @@ -25684,7 +25389,7 @@ x_9 = lean_unbox_usize(x_6); lean_dec(x_6); x_10 = lean_unbox_usize(x_7); lean_dec(x_7); -x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__7(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -25700,16 +25405,16 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__8(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -25717,11 +25422,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__11(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__9(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -25729,7 +25434,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__12(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_FileWorker_filterDuplicateSemanticTokens___spec__10(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } diff --git a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c index 574afa69119f..62f33233650e 100644 --- a/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c +++ b/stage0/stdlib/Lean/Server/FileWorker/WidgetRequests.c @@ -47,7 +47,6 @@ static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Wi LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_58____lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1389_(lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLineRange____x40_Lean_Data_Lsp_Extra___hyg_2944_(lean_object*); -lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_instInhabitedMsgToInteractive___closed__1; LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1945____lambda__3(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_registerBuiltinRpcProcedure___at_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_394____spec__1___lambda__2___closed__2; @@ -214,6 +213,7 @@ static lean_object* l_Lean_Widget_instInhabitedInfoPopup___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204_(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1755_(lean_object*); lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableInteractiveHypothesisBundle_dec____x40_Lean_Widget_InteractiveGoal___hyg_5____spec__1(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_520____closed__14; static lean_object* l_Lean_Widget_initFn____x40_Lean_Server_FileWorker_WidgetRequests___hyg_1409____closed__2; static lean_object* l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_520____closed__13; @@ -769,7 +769,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -803,7 +803,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_21); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } @@ -1710,7 +1710,7 @@ x_17 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_17, 0, x_8); lean_ctor_set(x_17, 1, x_16); x_18 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_19 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_17, x_18); +x_19 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_17, x_18); x_20 = l_Lean_Json_mkObj(x_19); return x_20; } @@ -4400,7 +4400,7 @@ x_5 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_5, 0, x_3); lean_ctor_set(x_5, 1, x_4); x_6 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_7 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_5, x_6); +x_7 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_5, x_6); x_8 = l_Lean_Json_mkObj(x_7); return x_8; } @@ -4635,7 +4635,7 @@ x_12 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_12, 0, x_7); lean_ctor_set(x_12, 1, x_11); x_13 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_14 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_12, x_13); +x_14 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_12, x_13); x_15 = l_Lean_Json_mkObj(x_14); return x_15; } @@ -4669,7 +4669,7 @@ x_26 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_26, 0, x_21); lean_ctor_set(x_26, 1, x_25); x_27 = l___private_Lean_Server_FileWorker_WidgetRequests_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Server_FileWorker_WidgetRequests___hyg_204____closed__1; -x_28 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_26, x_27); +x_28 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_26, x_27); x_29 = l_Lean_Json_mkObj(x_28); return x_29; } diff --git a/stage0/stdlib/Lean/Server/Watchdog.c b/stage0/stdlib/Lean/Server/Watchdog.c index 0b97fb0addb0..451bbfdbeec8 100644 --- a/stage0/stdlib/Lean/Server/Watchdog.c +++ b/stage0/stdlib/Lean/Server/Watchdog.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__2(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_JsonNumber_fromNat(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_References_definitionsMatching___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__19(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__10(lean_object*, lean_object*, lean_object*); @@ -28,7 +29,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___rarg(lean_object*, static lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleRename___spec__13___closed__2; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonReferenceParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4098_(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleRequest___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___closed__11; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__7; @@ -49,6 +49,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__31; lean_object* l_IO_throwServerError___rarg(lean_object*, lean_object*); lean_object* lean_mk_empty_array_with_capacity(lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Server_References_findAt(lean_object*, lean_object*, lean_object*, uint8_t); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleWorkspaceSymbol___spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCrash___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -64,12 +65,16 @@ lean_object* l___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelPara LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_ImportData_update___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__3___closed__1; static lean_object* l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_startFileWorker___spec__4(lean_object*); lean_object* l_System_FilePath_join(lean_object*, lean_object*); lean_object* lean_private_to_user_name(lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Json_mkObj(lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__3___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__40; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__16; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__2(lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_557_(lean_object*); @@ -81,6 +86,7 @@ LEAN_EXPORT uint8_t l_Lean_Server_Watchdog_ImportData_update___lambda__1(lean_ob LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_ServerRequestData_trackOutboundRequest(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__16(size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___lambda__1(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__6; static double l_Lean_Server_Watchdog_handleWorkspaceSymbol___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__3___boxed(lean_object*, lean_object*, lean_object*); @@ -96,7 +102,6 @@ lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonLeanDidOpenTextDo LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleResponseError(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__8; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__4___boxed(lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages___closed__1; @@ -104,6 +109,7 @@ lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonSymbol lean_object* lean_io_as_task(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__5(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__1___boxed(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcConnectParams____x40_Lean_Data_Lsp_Extra___hyg_1823_(lean_object*); @@ -129,6 +135,7 @@ static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__9; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_forwardNotification___at_Lean_Server_Watchdog_handleNotification___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_FileWorker_errorPendingRequests___spec__1(lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__6(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(lean_object*, size_t, size_t, lean_object*); lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_toJsonDidChangeWatchedFilesRegistrationOptions____x40_Lean_Data_Lsp_Workspace___hyg_457_(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_runClientTask___closed__1; @@ -146,7 +153,6 @@ static lean_object* l_Lean_Json_toStructured_x3f___at___private_Lean_Server_Watc LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Server_Watchdog_updateFileWorkers___spec__2(lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instOrdPosition; static lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleDidSave___spec__2___lambda__1___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2___boxed(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__30; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__2___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__4(lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -174,10 +180,12 @@ lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Referenc LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_runClientTask___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_RBNode_balLeft___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__18; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); uint8_t l___private_Lean_Data_JsonRpc_0__Lean_JsonRpc_ordRequestID____x40_Lean_Data_JsonRpc___hyg_126_(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__12; static lean_object* l_Lean_Server_Watchdog_startLoadingReferences___closed__1; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_startFileWorker___closed__4; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__20___boxed(lean_object*, lean_object*, lean_object*); uint64_t lean_string_hash(lean_object*); @@ -211,7 +219,6 @@ uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_StateRefT_x27_get___at_Lean_Server_Watchdog_FileWorker_waitForProc___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_handleRename___closed__1; static lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_ImportData_update___spec__11___closed__3; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__11; LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -234,17 +241,16 @@ static lean_object* l_IO_FS_Stream_readLspRequestAs___at_Lean_Server_Watchdog_in LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_forwardNotification___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__39; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__63; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2___boxed(lean_object*, lean_object*); lean_object* l_Lean_Server_mkPublishDiagnosticsNotification(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__42; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleDidChange(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__14(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___spec__2(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at_Lean_Server_Watchdog_updateFileWorkers___spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_killProcAndWait(lean_object*, lean_object*); lean_object* lean_get_stdout(lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__10; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_waitForProc___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_process_child_wait(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -265,13 +271,11 @@ lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_toJsonLeanStaleDepen uint8_t lean_string_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_del___at_Lean_Server_Watchdog_ImportData_update___spec__6(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__14; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(size_t, size_t, lean_object*); lean_object* l_Lean_Json_opt___at___private_Lean_Widget_InteractiveCode_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveCode___hyg_552____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_waitForProc(lean_object*, lean_object*); lean_object* lean_task_pure(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_del___at_Lean_Server_Watchdog_FileWorker_erasePendingRequest___spec__2(lean_object*, lean_object*); lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Lsp_ModuleRefs_findAt___spec__4(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__19; static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__5; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__62; @@ -305,13 +309,13 @@ lean_object* l_Lean_RBNode_setBlack___rarg(lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__25; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__52; lean_object* lean_nat_to_int(lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__9; LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_handleNotification___spec__8(lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___boxed(lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleReference___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(lean_object*, lean_object*, lean_object*); lean_object* l_IO_FS_Stream_readLspMessage(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_erase___at_Lean_Server_Watchdog_FileWorker_erasePendingRequest___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspRequest___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__3(lean_object*, lean_object*, lean_object*); @@ -328,9 +332,9 @@ static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__1; static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__10; static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__10; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_eraseFileWorker(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_del___at_Lean_Server_Watchdog_eraseFileWorker___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_CrashOrigin_noConfusion(lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_ImportData_update___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__46; static lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__5___closed__1; @@ -341,14 +345,12 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleDidSave(lean_object*, lean LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_forwardRequestToWorker___spec__3(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_notifyAboutStaleDependency(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_wait_any(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at_Lean_Server_Watchdog_ImportData_update___spec__9(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_fromJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_124_(lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__26; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__2; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__8(lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_ImportData_update(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_findWorkerPath___lambda__2___boxed(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_mkFileProgressAtPosNotification(lean_object*, lean_object*, uint8_t); @@ -366,17 +368,16 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_han LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__9___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_st_ref_get(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__11___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__11(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_insert___at_Lean_Server_Watchdog_ServerRequestData_trackOutboundRequest___spec__1(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_References_removeWorkerRefs(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__4; LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_handleRequest___spec__2(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_forwardNotification(lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* lean_server_watchdog_main(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleDidSave___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__36; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); lean_object* l_Lean_Server_routeLspRequest(lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__19; lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidChangeTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_585_(lean_object*); @@ -428,7 +429,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__4___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_findCore___at_Lean_Server_Watchdog_handleDidSave___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__5; LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_handleRequest___spec__12(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_forwardNotification___at_Lean_Server_Watchdog_handleNotification___spec__5(lean_object*, lean_object*, lean_object*, lean_object*); @@ -482,18 +482,16 @@ static lean_object* l_Lean_Server_Watchdog_startFileWorker___closed__1; static lean_object* l_Lean_Server_Watchdog_watchdogMain___closed__1; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__3; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__22; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_startFileWorker___spec__2(lean_object*); lean_object* l_System_SearchPath_searchModuleNameOfUri(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_startFileWorker___closed__7; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__1___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_handleRequest___lambda__1___closed__4; LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_handleNotification___spec__3___boxed(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mainLoop___closed__2; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11___boxed(lean_object*, lean_object*); lean_object* l_Lean_Server_References_removeIlean(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8___boxed(lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_fromJsonWorkspaceSymbolParams____x40_Lean_Data_Lsp_LanguageFeatures___hyg_4321_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__12(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_FS_Stream_readLspNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__1(lean_object*, lean_object*, lean_object*); @@ -512,6 +510,7 @@ static lean_object* l_Lean_Server_Watchdog_findWorkerPath___closed__2; static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__14; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__10(size_t, size_t, lean_object*); lean_object* l_Array_append___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___closed__5; LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_handleNotification___spec__3(lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___closed__8; @@ -519,7 +518,6 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_findWorkerPath___lambda__2(lean_ static lean_object* l_Lean_Server_Watchdog_handleNotification___closed__6; static lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__5___closed__1; static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__6; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleRequest(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_tryWriteMessage___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_mainLoop___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); @@ -533,12 +531,10 @@ static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__10; double l_Float_ofScientific(lean_object*, uint8_t, lean_object*); static lean_object* l_Lean_Server_Watchdog_handleRequest___lambda__1___closed__12; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(lean_object*, lean_object*); lean_object* l_Array_extract___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Server_Watchdog_findFileWorker_x3f___spec__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_stdout(lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___closed__4; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(lean_object*, lean_object*); lean_object* l_Lean_Server_References_definitionOf_x3f(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_startFileWorker___closed__8; static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__8; @@ -560,7 +556,6 @@ LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_shu LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_erasePendingRequest(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_ImportData_update___closed__1; lean_object* l_IO_FS_Stream_writeLspMessage(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__1___boxed(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__32; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_findDefinitions(lean_object*, lean_object*, lean_object*); @@ -577,7 +572,6 @@ static lean_object* l_Lean_Loop_forIn_loop___at_Lean_Server_Watchdog_initAndRunW static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__5; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleRename___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_searchModuleNameOfFileName(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handlePrepareRename(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__10; @@ -596,6 +590,7 @@ LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_ lean_object* l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_toJsonCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_6912_(lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(lean_object*, lean_object*, lean_object*); uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x40_Init_Data_Option_Basic___hyg_159____at___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCompletionItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_2497____spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_tryDischargeQueuedMessages(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_ReaderT_bind___at_Lean_Server_Watchdog_FileWorker_waitForProc___spec__2(lean_object*, lean_object*); @@ -623,6 +618,7 @@ extern lean_object* l_Lean_Lsp_SemanticTokenModifier_names; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams(lean_object*); static lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__7___closed__2; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_tryWriteMessage___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8___boxed(lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__21; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_ImportData_eraseImportsOf(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCrash(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); @@ -640,6 +636,7 @@ static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_ static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__11; uint8_t l_String_isPrefixOf(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__13; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_handleRename___lambda__1___closed__2; static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__3; LEAN_EXPORT lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop(lean_object*, lean_object*, lean_object*); @@ -650,7 +647,6 @@ uint64_t l_Lean_Name_hash___override(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleDidSave___spec__3(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_io_basemutex_unlock(lean_object*, lean_object*); static lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11(lean_object*, lean_object*); lean_object* lean_io_exit(uint8_t, lean_object*); static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__9; static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__12; @@ -675,9 +671,9 @@ static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_for LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__6(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_forwardRequestToWorker___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__59; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__8; lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(lean_object*); static lean_object* l_Lean_Server_Watchdog_parseParams___rarg___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_ImportData_update___lambda__1___boxed(lean_object*, lean_object*); @@ -699,19 +695,18 @@ static lean_object* l_Lean_Server_Watchdog_handleRequest___lambda__1___closed__1 lean_object* l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_runClientTask___closed__2; LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_mainLoop___spec__2___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_shutdown___spec__2(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__13___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_killProcAndWait___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_toJsonRpcReleaseParams____x40_Lean_Data_Lsp_Extra___hyg_2505_(lean_object*); lean_object* l___private_Lean_Data_Lsp_Workspace_0__Lean_Lsp_fromJsonDidChangeWatchedFilesParams____x40_Lean_Data_Lsp_Workspace___hyg_816_(lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleRename___spec__8(lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Lsp_Extra_0__Lean_Lsp_fromJsonRpcCallParams____x40_Lean_Data_Lsp_Extra___hyg_2014____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleCancelRequest___spec__3___closed__2; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleRename___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__12; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleRequest___spec__8(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_handleCancelRequest___spec__3___closed__1; static lean_object* l_Lean_Server_Watchdog_terminateFileWorker___closed__1; @@ -730,10 +725,8 @@ size_t lean_usize_sub(size_t, size_t); lean_object* l___private_Lean_Data_Lsp_TextSync_0__Lean_Lsp_fromJsonDidSaveTextDocumentParams____x40_Lean_Data_Lsp_TextSync___hyg_754_(lean_object*); lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Watchdog_handleNotification___spec__13___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_ImportData_update___spec__11(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__7; -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_findCore___at_Lean_Server_Watchdog_handleDidSave___spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__16; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -746,11 +739,9 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_shutdown(lean_object*, lean_obje size_t lean_usize_add(size_t, size_t); static lean_object* l_Lean_Server_Watchdog_handleRequest___lambda__1___closed__8; LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_handleRequest___spec__15(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13(lean_object*, size_t, size_t, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__53; LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_mainLoop___closed__1; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__9; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleRename___spec__14(lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__3___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -758,6 +749,7 @@ LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_parseParams___at_Lean_Server_Wat LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_CallHierarchyItemData_fromItem_x3f(lean_object*); lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonInitializeResult____x40_Lean_Data_Lsp_InitShutdown___hyg_928_(lean_object*); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_errorPendingRequests(lean_object*, lean_object*, uint8_t, lean_object*, lean_object*); size_t lean_array_size(lean_object*); @@ -778,11 +770,9 @@ static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fro static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdog___closed__3; static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__4; lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Lean_Server_Watchdog_initAndRunWatchdogAux___closed__19; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_CrashOrigin_noConfusion___rarg(uint8_t, uint8_t, lean_object*); lean_object* l_IO_FS_Stream_putStrLn(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleDidClose(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_startLoadingReferences(lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_tryDischargeQueuedMessages___closed__1; @@ -796,7 +786,6 @@ static lean_object* l_Lean_Server_Watchdog_handleDidOpen___closed__1; static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_fromJsonCallHierarchyItemData____x40_Lean_Server_Watchdog___hyg_4173____closed__7; static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__19; LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Server_Watchdog_forwardRequestToWorker___spec__2(lean_object*, lean_object*, lean_object*); -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__7; lean_object* l___private_Lean_Data_Lsp_Internal_0__Lean_Lsp_fromJsonLeanImportClosureParams____x40_Lean_Data_Lsp_Internal___hyg_2094_(lean_object*); lean_object* l___private_Lean_Data_Lsp_Client_0__Lean_Lsp_toJsonRegistrationParams____x40_Lean_Data_Lsp_Client___hyg_258_(lean_object*); @@ -806,6 +795,7 @@ static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_ LEAN_EXPORT lean_object* l_IO_FS_Stream_writeLspResponse___at_Lean_Server_Watchdog_handleRequest___spec__9(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleRequest___spec__10___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_callHierarchyItemOf_x3f(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_Server_References_finalizeWorkerRefs(lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_Lean_Lsp_instInhabitedCallHierarchyOutgoingCall; LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleCancelRequest(lean_object*, lean_object*, lean_object*); @@ -825,6 +815,7 @@ LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handleWork static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__64; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__2(lean_object*, size_t, size_t, lean_object*); static lean_object* l_IO_FS_Stream_readNotificationAs___at_Lean_Server_Watchdog_initAndRunWatchdogAux___spec__2___closed__43; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__10; lean_object* l___private_Lean_Data_Lsp_InitShutdown_0__Lean_Lsp_toJsonInitializeParams____x40_Lean_Data_Lsp_InitShutdown___hyg_523_(lean_object*); @@ -849,6 +840,7 @@ static lean_object* l_Lean_Server_Watchdog_mkLeanServerCapabilities___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__9(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* l___private_Lean_Data_Lsp_Communication_0__IO_FS_Stream_readLspHeader(lean_object*, lean_object*); lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_ins___at_Lean_Server_Watchdog_ImportData_update___spec__10(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_forIn_visit___at_Lean_Server_Watchdog_FileWorker_errorPendingRequests___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_FileWorker_waitForProc___closed__1; @@ -863,12 +855,14 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Serv lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__7___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Server_Watchdog_handleRename___lambda__1___closed__3; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleIleanInfoUpdate(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_erase___at_Lean_Server_Watchdog_ImportData_update___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handlePrepareCallHierarchy___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleDidChangeWatchedFiles___spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(lean_object*); lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonLocation____x40_Lean_Data_Lsp_Basic___hyg_895_(lean_object*); LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__5(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_SearchPath_findAllWithExt(lean_object*, lean_object*, lean_object*); @@ -880,15 +874,14 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_ lean_object* l_instDecidableEqString___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Server_Watchdog_0__Lean_Server_Watchdog_forwardMessages_loop___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_toStructured_x3f___at_Lean_Server_Watchdog_handleNotification___spec__6(lean_object*); size_t lean_usize_land(size_t, size_t); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_FileWorker_errorPendingRequests___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_IO_FS_Stream_readRequestAs___at_Lean_Server_Watchdog_initAndRunWatchdog___spec__2___closed__2; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_del___at_Lean_Server_Watchdog_ServerRequestData_translateInboundResponse___spec__3(lean_object*, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at_Lean_Lsp_instFromJsonInitializeParams___spec__3(lean_object*, lean_object*); lean_object* l_Lean_Server_maybeTee(lean_object*, uint8_t, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__4___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Server_Watchdog_handleResponseError___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_filterMapM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls___spec__3___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -19264,39 +19257,7 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_ctor_get(x_2, 2); -x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_4, x_1); -if (x_7 == 0) -{ -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_9; -lean_inc(x_5); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_5); -return x_9; -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -19325,7 +19286,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -19399,7 +19360,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -19418,7 +19379,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -19429,7 +19390,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -19440,151 +19401,179 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_4; -lean_dec(x_2); -lean_dec(x_1); +lean_object* x_4; lean_object* x_5; x_4 = lean_box(0); -return x_4; -} -else -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_3, 0); -x_7 = lean_ctor_get(x_3, 1); -x_8 = lean_ctor_get(x_3, 2); -x_9 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_6, x_1); -if (x_9 == 0) +x_5 = lean_apply_1(x_2, x_4); +if (lean_obj_tag(x_5) == 0) { -lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_10); -return x_3; +lean_object* x_6; +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; } else { -lean_dec(x_7); -lean_dec(x_6); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_1); -return x_3; +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_box(0); +x_9 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_9, 0, x_1); +lean_ctor_set(x_9, 1, x_7); +lean_ctor_set(x_9, 2, x_8); +return x_9; } } else { +uint8_t x_10; +x_10 = !lean_is_exclusive(x_3); +if (x_10 == 0) +{ lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_11 = lean_ctor_get(x_3, 0); x_12 = lean_ctor_get(x_3, 1); x_13 = lean_ctor_get(x_3, 2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_3); x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_11, x_1); if (x_14 == 0) { -lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_1, x_2, x_13); -x_16 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_16, 0, x_11); -lean_ctor_set(x_16, 1, x_12); -lean_ctor_set(x_16, 2, x_15); -return x_16; +lean_object* x_15; +x_15 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_1, x_2, x_13); +lean_ctor_set(x_3, 2, x_15); +return x_3; } else { -lean_object* x_17; -lean_dec(x_12); +lean_object* x_16; lean_object* x_17; lean_dec(x_11); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_2); -lean_ctor_set(x_17, 2, x_13); -return x_17; -} +x_16 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_16, 0, x_12); +x_17 = lean_apply_1(x_2, x_16); +if (lean_obj_tag(x_17) == 0) +{ +lean_free_object(x_3); +lean_dec(x_1); +return x_13; } +else +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_17, 0); +lean_inc(x_18); +lean_dec(x_17); +lean_ctor_set(x_3, 1, x_18); +lean_ctor_set(x_3, 0, x_1); +return x_3; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(lean_object* x_1, lean_object* x_2) { -_start: +else { -if (lean_obj_tag(x_2) == 0) +lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; +x_19 = lean_ctor_get(x_3, 0); +x_20 = lean_ctor_get(x_3, 1); +x_21 = lean_ctor_get(x_3, 2); +lean_inc(x_21); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_3); +x_22 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_19, x_1); +if (x_22 == 0) { -lean_object* x_3; -x_3 = lean_box(0); -return x_3; +lean_object* x_23; lean_object* x_24; +x_23 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_1, x_2, x_21); +x_24 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_24, 0, x_19); +lean_ctor_set(x_24, 1, x_20); +lean_ctor_set(x_24, 2, x_23); +return x_24; } else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_5, x_1); -if (x_8 == 0) +lean_object* x_25; lean_object* x_26; +lean_dec(x_19); +x_25 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_25, 0, x_20); +x_26 = lean_apply_1(x_2, x_25); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_9; -x_9 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_1, x_7); -lean_ctor_set(x_2, 2, x_9); -return x_2; +lean_dec(x_1); +return x_21; } else { -lean_free_object(x_2); -lean_dec(x_6); -lean_dec(x_5); -return x_7; +lean_object* x_27; lean_object* x_28; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +lean_dec(x_26); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_1); +lean_ctor_set(x_28, 1, x_27); +lean_ctor_set(x_28, 2, x_21); +return x_28; } } -else +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6(lean_object* x_1) { +_start: { -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -x_12 = lean_ctor_get(x_2, 2); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_2); -x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_10, x_1); -if (x_13 == 0) +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_14; lean_object* x_15; -x_14 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_1, x_12); -x_15 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_11); -lean_ctor_set(x_15, 2, x_14); -return x_15; +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -lean_dec(x_11); -lean_dec(x_10); -return x_12; +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); +return x_2; } +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -19597,50 +19586,50 @@ return x_8; } else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; x_10 = lean_array_uget(x_5, x_7); lean_inc(x_1); lean_inc(x_10); x_11 = lean_apply_1(x_1, x_10); -x_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; -x_13 = lean_ctor_get(x_8, 0); -x_14 = lean_ctor_get(x_8, 1); -x_15 = lean_array_get_size(x_14); -x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); -x_17 = 32; -x_18 = lean_uint64_shift_right(x_16, x_17); -x_19 = lean_uint64_xor(x_16, x_18); -x_20 = 16; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = lean_uint64_to_usize(x_22); -x_24 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_25 = 1; -x_26 = lean_usize_sub(x_24, x_25); -x_27 = lean_usize_land(x_23, x_26); -x_28 = lean_array_uget(x_14, x_27); -x_29 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_28); -if (lean_obj_tag(x_29) == 0) +lean_inc(x_10); +x_12 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___lambda__1), 2, 1); +lean_closure_set(x_12, 0, x_10); +x_13 = !lean_is_exclusive(x_8); +if (x_13 == 0) { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_31 = lean_array_push(x_30, x_10); -x_32 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_28); -if (x_32 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_8, 0); +x_15 = lean_ctor_get(x_8, 1); +x_16 = lean_array_get_size(x_15); +x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_29); +if (x_30 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_dec(x_12); +x_31 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +x_32 = lean_array_push(x_31, x_10); x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_nat_add(x_13, x_33); -lean_dec(x_13); +x_34 = lean_nat_add(x_14, x_33); +lean_dec(x_14); x_35 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_35, 0, x_11); -lean_ctor_set(x_35, 1, x_31); -lean_ctor_set(x_35, 2, x_28); -x_36 = lean_array_uset(x_14, x_27, x_35); +lean_ctor_set(x_35, 1, x_32); +lean_ctor_set(x_35, 2, x_29); +x_36 = lean_array_uset(x_15, x_28, x_35); x_37 = lean_unsigned_to_nat(4u); x_38 = lean_nat_mul(x_34, x_37); x_39 = lean_unsigned_to_nat(3u); @@ -19653,10 +19642,10 @@ lean_dec(x_40); if (x_42 == 0) { lean_object* x_43; size_t x_44; -x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_36); +x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_36); lean_ctor_set(x_8, 1, x_43); lean_ctor_set(x_8, 0, x_34); -x_44 = lean_usize_add(x_7, x_25); +x_44 = lean_usize_add(x_7, x_26); x_7 = x_44; goto _start; } @@ -19665,418 +19654,149 @@ else size_t x_46; lean_ctor_set(x_8, 1, x_36); lean_ctor_set(x_8, 0, x_34); -x_46 = lean_usize_add(x_7, x_25); +x_46 = lean_usize_add(x_7, x_26); x_7 = x_46; goto _start; } } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; size_t x_51; -lean_inc(x_3); -x_48 = lean_array_uset(x_14, x_27, x_3); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_11, x_31, x_28); -x_50 = lean_array_uset(x_48, x_27, x_49); -lean_ctor_set(x_8, 1, x_50); -x_51 = lean_usize_add(x_7, x_25); -x_7 = x_51; -goto _start; -} -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_117; -x_53 = lean_ctor_get(x_29, 0); -lean_inc(x_53); -lean_dec(x_29); -x_54 = lean_array_push(x_53, x_10); -x_117 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_28); -if (x_117 == 0) -{ -lean_dec(x_28); -x_55 = x_8; -goto block_116; -} -else -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_inc(x_3); -x_118 = lean_array_uset(x_14, x_27, x_3); -x_119 = lean_unsigned_to_nat(1u); -x_120 = lean_nat_sub(x_13, x_119); -lean_dec(x_13); -x_121 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_11, x_28); -x_122 = lean_array_uset(x_118, x_27, x_121); -lean_ctor_set(x_8, 1, x_122); -lean_ctor_set(x_8, 0, x_120); -x_55 = x_8; -goto block_116; -} -block_116: -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; size_t x_62; lean_object* x_63; uint8_t x_64; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_ctor_get(x_55, 1); -x_59 = lean_array_get_size(x_58); -x_60 = lean_usize_of_nat(x_59); -lean_dec(x_59); -x_61 = lean_usize_sub(x_60, x_25); -x_62 = lean_usize_land(x_23, x_61); -x_63 = lean_array_uget(x_58, x_62); -x_64 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_63); -if (x_64 == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_nat_add(x_57, x_65); -lean_dec(x_57); -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_11); -lean_ctor_set(x_67, 1, x_54); -lean_ctor_set(x_67, 2, x_63); -x_68 = lean_array_uset(x_58, x_62, x_67); -x_69 = lean_unsigned_to_nat(4u); -x_70 = lean_nat_mul(x_66, x_69); -x_71 = lean_unsigned_to_nat(3u); -x_72 = lean_nat_div(x_70, x_71); -lean_dec(x_70); -x_73 = lean_array_get_size(x_68); -x_74 = lean_nat_dec_le(x_72, x_73); -lean_dec(x_73); -lean_dec(x_72); -if (x_74 == 0) -{ -lean_object* x_75; size_t x_76; -x_75 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_68); -lean_ctor_set(x_55, 1, x_75); -lean_ctor_set(x_55, 0, x_66); -x_76 = lean_usize_add(x_7, x_25); -x_7 = x_76; -x_8 = x_55; -goto _start; -} -else -{ -size_t x_78; -lean_ctor_set(x_55, 1, x_68); -lean_ctor_set(x_55, 0, x_66); -x_78 = lean_usize_add(x_7, x_25); -x_7 = x_78; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; size_t x_83; +lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +lean_dec(x_10); lean_inc(x_3); -x_80 = lean_array_uset(x_58, x_62, x_3); -x_81 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_11, x_54, x_63); -x_82 = lean_array_uset(x_80, x_62, x_81); -lean_ctor_set(x_55, 1, x_82); -x_83 = lean_usize_add(x_7, x_25); -x_7 = x_83; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; size_t x_88; size_t x_89; size_t x_90; lean_object* x_91; uint8_t x_92; -x_85 = lean_ctor_get(x_55, 0); -x_86 = lean_ctor_get(x_55, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_55); -x_87 = lean_array_get_size(x_86); -x_88 = lean_usize_of_nat(x_87); -lean_dec(x_87); -x_89 = lean_usize_sub(x_88, x_25); -x_90 = lean_usize_land(x_23, x_89); -x_91 = lean_array_uget(x_86, x_90); -x_92 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_91); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_93 = lean_unsigned_to_nat(1u); -x_94 = lean_nat_add(x_85, x_93); -lean_dec(x_85); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_11); -lean_ctor_set(x_95, 1, x_54); -lean_ctor_set(x_95, 2, x_91); -x_96 = lean_array_uset(x_86, x_90, x_95); -x_97 = lean_unsigned_to_nat(4u); -x_98 = lean_nat_mul(x_94, x_97); -x_99 = lean_unsigned_to_nat(3u); -x_100 = lean_nat_div(x_98, x_99); -lean_dec(x_98); -x_101 = lean_array_get_size(x_96); -x_102 = lean_nat_dec_le(x_100, x_101); -lean_dec(x_101); -lean_dec(x_100); -if (x_102 == 0) -{ -lean_object* x_103; lean_object* x_104; size_t x_105; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_96); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_94); -lean_ctor_set(x_104, 1, x_103); -x_105 = lean_usize_add(x_7, x_25); -x_7 = x_105; -x_8 = x_104; -goto _start; -} -else +x_48 = lean_array_uset(x_15, x_28, x_3); +lean_inc(x_11); +x_49 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_11, x_12, x_29); +x_50 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_49); +lean_dec(x_11); +x_51 = lean_array_uset(x_48, x_28, x_49); +if (x_50 == 0) { -lean_object* x_107; size_t x_108; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_94); -lean_ctor_set(x_107, 1, x_96); -x_108 = lean_usize_add(x_7, x_25); -x_7 = x_108; -x_8 = x_107; +lean_object* x_52; lean_object* x_53; size_t x_54; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_sub(x_14, x_52); +lean_dec(x_14); +lean_ctor_set(x_8, 1, x_51); +lean_ctor_set(x_8, 0, x_53); +x_54 = lean_usize_add(x_7, x_26); +x_7 = x_54; goto _start; } -} else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; size_t x_114; -lean_inc(x_3); -x_110 = lean_array_uset(x_86, x_90, x_3); -x_111 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_11, x_54, x_91); -x_112 = lean_array_uset(x_110, x_90, x_111); -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_85); -lean_ctor_set(x_113, 1, x_112); -x_114 = lean_usize_add(x_7, x_25); -x_7 = x_114; -x_8 = x_113; +size_t x_56; +lean_ctor_set(x_8, 1, x_51); +x_56 = lean_usize_add(x_7, x_26); +x_7 = x_56; goto _start; } } } -} -} else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; uint64_t x_126; uint64_t x_127; uint64_t x_128; uint64_t x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; size_t x_133; size_t x_134; size_t x_135; size_t x_136; size_t x_137; lean_object* x_138; lean_object* x_139; -x_123 = lean_ctor_get(x_8, 0); -x_124 = lean_ctor_get(x_8, 1); -lean_inc(x_124); -lean_inc(x_123); +lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; size_t x_68; size_t x_69; size_t x_70; size_t x_71; size_t x_72; lean_object* x_73; uint8_t x_74; +x_58 = lean_ctor_get(x_8, 0); +x_59 = lean_ctor_get(x_8, 1); +lean_inc(x_59); +lean_inc(x_58); lean_dec(x_8); -x_125 = lean_array_get_size(x_124); -x_126 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); -x_127 = 32; -x_128 = lean_uint64_shift_right(x_126, x_127); -x_129 = lean_uint64_xor(x_126, x_128); -x_130 = 16; -x_131 = lean_uint64_shift_right(x_129, x_130); -x_132 = lean_uint64_xor(x_129, x_131); -x_133 = lean_uint64_to_usize(x_132); -x_134 = lean_usize_of_nat(x_125); -lean_dec(x_125); -x_135 = 1; -x_136 = lean_usize_sub(x_134, x_135); -x_137 = lean_usize_land(x_133, x_136); -x_138 = lean_array_uget(x_124, x_137); -x_139 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_138); -if (lean_obj_tag(x_139) == 0) -{ -lean_object* x_140; lean_object* x_141; uint8_t x_142; -x_140 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_141 = lean_array_push(x_140, x_10); -x_142 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_138); -if (x_142 == 0) -{ -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; -x_143 = lean_unsigned_to_nat(1u); -x_144 = lean_nat_add(x_123, x_143); -lean_dec(x_123); -x_145 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_145, 0, x_11); -lean_ctor_set(x_145, 1, x_141); -lean_ctor_set(x_145, 2, x_138); -x_146 = lean_array_uset(x_124, x_137, x_145); -x_147 = lean_unsigned_to_nat(4u); -x_148 = lean_nat_mul(x_144, x_147); -x_149 = lean_unsigned_to_nat(3u); -x_150 = lean_nat_div(x_148, x_149); -lean_dec(x_148); -x_151 = lean_array_get_size(x_146); -x_152 = lean_nat_dec_le(x_150, x_151); -lean_dec(x_151); -lean_dec(x_150); -if (x_152 == 0) +x_60 = lean_array_get_size(x_59); +x_61 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); +x_62 = 32; +x_63 = lean_uint64_shift_right(x_61, x_62); +x_64 = lean_uint64_xor(x_61, x_63); +x_65 = 16; +x_66 = lean_uint64_shift_right(x_64, x_65); +x_67 = lean_uint64_xor(x_64, x_66); +x_68 = lean_uint64_to_usize(x_67); +x_69 = lean_usize_of_nat(x_60); +lean_dec(x_60); +x_70 = 1; +x_71 = lean_usize_sub(x_69, x_70); +x_72 = lean_usize_land(x_68, x_71); +x_73 = lean_array_uget(x_59, x_72); +x_74 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_73); +if (x_74 == 0) { -lean_object* x_153; lean_object* x_154; size_t x_155; -x_153 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_146); -x_154 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_154, 0, x_144); -lean_ctor_set(x_154, 1, x_153); -x_155 = lean_usize_add(x_7, x_135); -x_7 = x_155; -x_8 = x_154; -goto _start; -} -else +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +lean_dec(x_12); +x_75 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +x_76 = lean_array_push(x_75, x_10); +x_77 = lean_unsigned_to_nat(1u); +x_78 = lean_nat_add(x_58, x_77); +lean_dec(x_58); +x_79 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_79, 0, x_11); +lean_ctor_set(x_79, 1, x_76); +lean_ctor_set(x_79, 2, x_73); +x_80 = lean_array_uset(x_59, x_72, x_79); +x_81 = lean_unsigned_to_nat(4u); +x_82 = lean_nat_mul(x_78, x_81); +x_83 = lean_unsigned_to_nat(3u); +x_84 = lean_nat_div(x_82, x_83); +lean_dec(x_82); +x_85 = lean_array_get_size(x_80); +x_86 = lean_nat_dec_le(x_84, x_85); +lean_dec(x_85); +lean_dec(x_84); +if (x_86 == 0) { -lean_object* x_157; size_t x_158; -x_157 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_157, 0, x_144); -lean_ctor_set(x_157, 1, x_146); -x_158 = lean_usize_add(x_7, x_135); -x_7 = x_158; -x_8 = x_157; +lean_object* x_87; lean_object* x_88; size_t x_89; +x_87 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_80); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_78); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_7, x_70); +x_7 = x_89; +x_8 = x_88; goto _start; } -} else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; size_t x_164; -lean_inc(x_3); -x_160 = lean_array_uset(x_124, x_137, x_3); -x_161 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_11, x_141, x_138); -x_162 = lean_array_uset(x_160, x_137, x_161); -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_123); -lean_ctor_set(x_163, 1, x_162); -x_164 = lean_usize_add(x_7, x_135); -x_7 = x_164; -x_8 = x_163; +lean_object* x_91; size_t x_92; +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_78); +lean_ctor_set(x_91, 1, x_80); +x_92 = lean_usize_add(x_7, x_70); +x_7 = x_92; +x_8 = x_91; goto _start; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_202; -x_166 = lean_ctor_get(x_139, 0); -lean_inc(x_166); -lean_dec(x_139); -x_167 = lean_array_push(x_166, x_10); -x_202 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_138); -if (x_202 == 0) -{ -lean_object* x_203; -lean_dec(x_138); -x_203 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_203, 0, x_123); -lean_ctor_set(x_203, 1, x_124); -x_168 = x_203; -goto block_201; -} -else -{ -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; +lean_object* x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; +lean_dec(x_10); lean_inc(x_3); -x_204 = lean_array_uset(x_124, x_137, x_3); -x_205 = lean_unsigned_to_nat(1u); -x_206 = lean_nat_sub(x_123, x_205); -lean_dec(x_123); -x_207 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_11, x_138); -x_208 = lean_array_uset(x_204, x_137, x_207); -x_209 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_209, 0, x_206); -lean_ctor_set(x_209, 1, x_208); -x_168 = x_209; -goto block_201; -} -block_201: -{ -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; size_t x_173; size_t x_174; size_t x_175; lean_object* x_176; uint8_t x_177; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -x_170 = lean_ctor_get(x_168, 1); -lean_inc(x_170); -if (lean_is_exclusive(x_168)) { - lean_ctor_release(x_168, 0); - lean_ctor_release(x_168, 1); - x_171 = x_168; -} else { - lean_dec_ref(x_168); - x_171 = lean_box(0); -} -x_172 = lean_array_get_size(x_170); -x_173 = lean_usize_of_nat(x_172); -lean_dec(x_172); -x_174 = lean_usize_sub(x_173, x_135); -x_175 = lean_usize_land(x_133, x_174); -x_176 = lean_array_uget(x_170, x_175); -x_177 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_11, x_176); -if (x_177 == 0) -{ -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; -x_178 = lean_unsigned_to_nat(1u); -x_179 = lean_nat_add(x_169, x_178); -lean_dec(x_169); -x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_11); -lean_ctor_set(x_180, 1, x_167); -lean_ctor_set(x_180, 2, x_176); -x_181 = lean_array_uset(x_170, x_175, x_180); -x_182 = lean_unsigned_to_nat(4u); -x_183 = lean_nat_mul(x_179, x_182); -x_184 = lean_unsigned_to_nat(3u); -x_185 = lean_nat_div(x_183, x_184); -lean_dec(x_183); -x_186 = lean_array_get_size(x_181); -x_187 = lean_nat_dec_le(x_185, x_186); -lean_dec(x_186); -lean_dec(x_185); -if (x_187 == 0) -{ -lean_object* x_188; lean_object* x_189; size_t x_190; -x_188 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__4(x_181); -if (lean_is_scalar(x_171)) { - x_189 = lean_alloc_ctor(0, 2, 0); -} else { - x_189 = x_171; -} -lean_ctor_set(x_189, 0, x_179); -lean_ctor_set(x_189, 1, x_188); -x_190 = lean_usize_add(x_7, x_135); -x_7 = x_190; -x_8 = x_189; -goto _start; -} -else +x_94 = lean_array_uset(x_59, x_72, x_3); +lean_inc(x_11); +x_95 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_11, x_12, x_73); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_11, x_95); +lean_dec(x_11); +x_97 = lean_array_uset(x_94, x_72, x_95); +if (x_96 == 0) { -lean_object* x_192; size_t x_193; -if (lean_is_scalar(x_171)) { - x_192 = lean_alloc_ctor(0, 2, 0); -} else { - x_192 = x_171; -} -lean_ctor_set(x_192, 0, x_179); -lean_ctor_set(x_192, 1, x_181); -x_193 = lean_usize_add(x_7, x_135); -x_7 = x_193; -x_8 = x_192; +lean_object* x_98; lean_object* x_99; lean_object* x_100; size_t x_101; +x_98 = lean_unsigned_to_nat(1u); +x_99 = lean_nat_sub(x_58, x_98); +lean_dec(x_58); +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_99); +lean_ctor_set(x_100, 1, x_97); +x_101 = lean_usize_add(x_7, x_70); +x_7 = x_101; +x_8 = x_100; goto _start; } -} else { -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; size_t x_199; -lean_inc(x_3); -x_195 = lean_array_uset(x_170, x_175, x_3); -x_196 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_11, x_167, x_176); -x_197 = lean_array_uset(x_195, x_175, x_196); -if (lean_is_scalar(x_171)) { - x_198 = lean_alloc_ctor(0, 2, 0); -} else { - x_198 = x_171; -} -lean_ctor_set(x_198, 0, x_169); -lean_ctor_set(x_198, 1, x_197); -x_199 = lean_usize_add(x_7, x_135); -x_7 = x_199; -x_8 = x_198; +lean_object* x_103; size_t x_104; +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_58); +lean_ctor_set(x_103, 1, x_97); +x_104 = lean_usize_add(x_7, x_70); +x_7 = x_104; +x_8 = x_103; goto _start; } } @@ -20084,7 +19804,6 @@ goto _start; } } } -} static lean_object* _init_l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__1() { _start: { @@ -20126,11 +19845,11 @@ x_4 = lean_box(0); x_5 = lean_array_size(x_2); x_6 = 0; x_7 = l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__3; -x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); +x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -20156,7 +19875,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -20181,7 +19900,7 @@ goto _start; } } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1() { _start: { lean_object* x_1; lean_object* x_2; @@ -20190,7 +19909,7 @@ x_2 = lean_mk_empty_array_with_capacity(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -20225,7 +19944,7 @@ if (x_15 == 0) lean_object* x_16; lean_object* x_17; lean_object* x_18; x_16 = lean_ctor_get(x_14, 1); lean_dec(x_16); -x_17 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_17 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; lean_ctor_set(x_14, 1, x_17); x_18 = lean_array_uset(x_7, x_2, x_14); x_2 = x_9; @@ -20238,7 +19957,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_20 = lean_ctor_get(x_14, 0); lean_inc(x_20); lean_dec(x_14); -x_21 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_21 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); @@ -20264,7 +19983,7 @@ if (x_28 == 0) lean_object* x_29; lean_object* x_30; lean_dec(x_11); lean_dec(x_10); -x_29 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_29 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; lean_ctor_set(x_25, 1, x_29); x_30 = lean_array_uset(x_7, x_2, x_25); x_2 = x_9; @@ -20277,8 +19996,8 @@ size_t x_32; size_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_3 x_32 = 0; x_33 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_34 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; -x_35 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_10, x_32, x_33, x_34); +x_34 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; +x_35 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_10, x_32, x_33, x_34); lean_dec(x_10); lean_ctor_set(x_25, 1, x_35); x_36 = lean_array_uset(x_7, x_2, x_25); @@ -20299,7 +20018,7 @@ if (x_39 == 0) lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_dec(x_11); lean_dec(x_10); -x_40 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_40 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; x_41 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_41, 0, x_38); lean_ctor_set(x_41, 1, x_40); @@ -20314,8 +20033,8 @@ size_t x_44; size_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_4 x_44 = 0; x_45 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_46 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; -x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_10, x_44, x_45, x_46); +x_46 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; +x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_10, x_44, x_45, x_46); lean_dec(x_10); x_48 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_48, 0, x_38); @@ -20330,7 +20049,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -20339,7 +20058,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -20399,7 +20118,7 @@ lean_dec(x_5); lean_dec(x_4); x_9 = l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2; x_10 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(x_9, x_8, x_10); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_9, x_8, x_10); return x_11; } else @@ -20413,7 +20132,7 @@ lean_dec(x_5); lean_dec(x_4); x_13 = l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2; x_14 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(x_13, x_8, x_14); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_13, x_8, x_14); return x_15; } else @@ -20422,46 +20141,27 @@ size_t x_16; lean_object* x_17; lean_object* x_18; size_t x_19; lean_object* x_2 x_16 = lean_usize_of_nat(x_5); lean_dec(x_5); x_17 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13(x_4, x_8, x_16, x_17); +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(x_4, x_8, x_16, x_17); lean_dec(x_4); x_19 = lean_array_size(x_18); -x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(x_19, x_8, x_18); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_19, x_8, x_18); return x_20; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__2(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_1, x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { size_t x_9; size_t x_10; lean_object* x_11; @@ -20469,7 +20169,7 @@ x_9 = lean_unbox_usize(x_6); lean_dec(x_6); x_10 = lean_unbox_usize(x_7); lean_dec(x_7); -x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -20485,7 +20185,7 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -20493,21 +20193,21 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__8(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__9(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -20515,11 +20215,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -20527,7 +20227,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__13(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__11(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -22089,39 +21789,7 @@ lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint8_t x_7; -x_4 = lean_ctor_get(x_2, 0); -x_5 = lean_ctor_get(x_2, 1); -x_6 = lean_ctor_get(x_2, 2); -x_7 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_4, x_1); -if (x_7 == 0) -{ -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_9; -lean_inc(x_5); -x_9 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_9, 0, x_5); -return x_9; -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -22150,7 +21818,7 @@ return x_8; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -22224,7 +21892,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -22243,7 +21911,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -22254,7 +21922,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -22265,151 +21933,11 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -if (lean_obj_tag(x_3) == 0) -{ -lean_object* x_4; -lean_dec(x_2); -lean_dec(x_1); -x_4 = lean_box(0); -return x_4; -} -else -{ -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; -x_6 = lean_ctor_get(x_3, 0); -x_7 = lean_ctor_get(x_3, 1); -x_8 = lean_ctor_get(x_3, 2); -x_9 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_6, x_1); -if (x_9 == 0) -{ -lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_10); -return x_3; -} -else -{ -lean_dec(x_7); -lean_dec(x_6); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_1); -return x_3; -} -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_11 = lean_ctor_get(x_3, 0); -x_12 = lean_ctor_get(x_3, 1); -x_13 = lean_ctor_get(x_3, 2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); -lean_dec(x_3); -x_14 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_11, x_1); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; -x_15 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_1, x_2, x_13); -x_16 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_16, 0, x_11); -lean_ctor_set(x_16, 1, x_12); -lean_ctor_set(x_16, 2, x_15); -return x_16; -} -else -{ -lean_object* x_17; -lean_dec(x_12); -lean_dec(x_11); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_1); -lean_ctor_set(x_17, 1, x_2); -lean_ctor_set(x_17, 2, x_13); -return x_17; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(lean_object* x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_5, x_1); -if (x_8 == 0) -{ -lean_object* x_9; -x_9 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_1, x_7); -lean_ctor_set(x_2, 2, x_9); -return x_2; -} -else -{ -lean_free_object(x_2); -lean_dec(x_6); -lean_dec(x_5); -return x_7; -} -} -else -{ -lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_10 = lean_ctor_get(x_2, 0); -x_11 = lean_ctor_get(x_2, 1); -x_12 = lean_ctor_get(x_2, 2); -lean_inc(x_12); -lean_inc(x_11); -lean_inc(x_10); -lean_dec(x_2); -x_13 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_beqCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7018_(x_10, x_1); -if (x_13 == 0) -{ -lean_object* x_14; lean_object* x_15; -x_14 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_1, x_12); -x_15 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_15, 0, x_10); -lean_ctor_set(x_15, 1, x_11); -lean_ctor_set(x_15, 2, x_14); -return x_15; -} -else -{ -lean_dec(x_11); -lean_dec(x_10); -return x_12; -} -} -} -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, size_t x_6, size_t x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -22422,50 +21950,50 @@ return x_8; } else { -lean_object* x_10; lean_object* x_11; uint8_t x_12; +lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; x_10 = lean_array_uget(x_5, x_7); lean_inc(x_1); lean_inc(x_10); x_11 = lean_apply_1(x_1, x_10); -x_12 = !lean_is_exclusive(x_8); -if (x_12 == 0) -{ -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; size_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; lean_object* x_28; lean_object* x_29; -x_13 = lean_ctor_get(x_8, 0); -x_14 = lean_ctor_get(x_8, 1); -x_15 = lean_array_get_size(x_14); -x_16 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); -x_17 = 32; -x_18 = lean_uint64_shift_right(x_16, x_17); -x_19 = lean_uint64_xor(x_16, x_18); -x_20 = 16; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = lean_uint64_to_usize(x_22); -x_24 = lean_usize_of_nat(x_15); -lean_dec(x_15); -x_25 = 1; -x_26 = lean_usize_sub(x_24, x_25); -x_27 = lean_usize_land(x_23, x_26); -x_28 = lean_array_uget(x_14, x_27); -x_29 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_28); -if (lean_obj_tag(x_29) == 0) +lean_inc(x_10); +x_12 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__7___lambda__1), 2, 1); +lean_closure_set(x_12, 0, x_10); +x_13 = !lean_is_exclusive(x_8); +if (x_13 == 0) { -lean_object* x_30; lean_object* x_31; uint8_t x_32; -x_30 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_31 = lean_array_push(x_30, x_10); -x_32 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_28); -if (x_32 == 0) +lean_object* x_14; lean_object* x_15; lean_object* x_16; uint64_t x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; uint8_t x_30; +x_14 = lean_ctor_get(x_8, 0); +x_15 = lean_ctor_get(x_8, 1); +x_16 = lean_array_get_size(x_15); +x_17 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); +x_18 = 32; +x_19 = lean_uint64_shift_right(x_17, x_18); +x_20 = lean_uint64_xor(x_17, x_19); +x_21 = 16; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = lean_uint64_to_usize(x_23); +x_25 = lean_usize_of_nat(x_16); +lean_dec(x_16); +x_26 = 1; +x_27 = lean_usize_sub(x_25, x_26); +x_28 = lean_usize_land(x_24, x_27); +x_29 = lean_array_uget(x_15, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_29); +if (x_30 == 0) { -lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +lean_dec(x_12); +x_31 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +x_32 = lean_array_push(x_31, x_10); x_33 = lean_unsigned_to_nat(1u); -x_34 = lean_nat_add(x_13, x_33); -lean_dec(x_13); +x_34 = lean_nat_add(x_14, x_33); +lean_dec(x_14); x_35 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_35, 0, x_11); -lean_ctor_set(x_35, 1, x_31); -lean_ctor_set(x_35, 2, x_28); -x_36 = lean_array_uset(x_14, x_27, x_35); +lean_ctor_set(x_35, 1, x_32); +lean_ctor_set(x_35, 2, x_29); +x_36 = lean_array_uset(x_15, x_28, x_35); x_37 = lean_unsigned_to_nat(4u); x_38 = lean_nat_mul(x_34, x_37); x_39 = lean_unsigned_to_nat(3u); @@ -22478,10 +22006,10 @@ lean_dec(x_40); if (x_42 == 0) { lean_object* x_43; size_t x_44; -x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_36); +x_43 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_36); lean_ctor_set(x_8, 1, x_43); lean_ctor_set(x_8, 0, x_34); -x_44 = lean_usize_add(x_7, x_25); +x_44 = lean_usize_add(x_7, x_26); x_7 = x_44; goto _start; } @@ -22490,418 +22018,149 @@ else size_t x_46; lean_ctor_set(x_8, 1, x_36); lean_ctor_set(x_8, 0, x_34); -x_46 = lean_usize_add(x_7, x_25); +x_46 = lean_usize_add(x_7, x_26); x_7 = x_46; goto _start; } } else { -lean_object* x_48; lean_object* x_49; lean_object* x_50; size_t x_51; -lean_inc(x_3); -x_48 = lean_array_uset(x_14, x_27, x_3); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_11, x_31, x_28); -x_50 = lean_array_uset(x_48, x_27, x_49); -lean_ctor_set(x_8, 1, x_50); -x_51 = lean_usize_add(x_7, x_25); -x_7 = x_51; -goto _start; -} -} -else -{ -lean_object* x_53; lean_object* x_54; lean_object* x_55; uint8_t x_117; -x_53 = lean_ctor_get(x_29, 0); -lean_inc(x_53); -lean_dec(x_29); -x_54 = lean_array_push(x_53, x_10); -x_117 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_28); -if (x_117 == 0) -{ -lean_dec(x_28); -x_55 = x_8; -goto block_116; -} -else -{ -lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -lean_inc(x_3); -x_118 = lean_array_uset(x_14, x_27, x_3); -x_119 = lean_unsigned_to_nat(1u); -x_120 = lean_nat_sub(x_13, x_119); -lean_dec(x_13); -x_121 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_11, x_28); -x_122 = lean_array_uset(x_118, x_27, x_121); -lean_ctor_set(x_8, 1, x_122); -lean_ctor_set(x_8, 0, x_120); -x_55 = x_8; -goto block_116; -} -block_116: -{ -uint8_t x_56; -x_56 = !lean_is_exclusive(x_55); -if (x_56 == 0) -{ -lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; size_t x_62; lean_object* x_63; uint8_t x_64; -x_57 = lean_ctor_get(x_55, 0); -x_58 = lean_ctor_get(x_55, 1); -x_59 = lean_array_get_size(x_58); -x_60 = lean_usize_of_nat(x_59); -lean_dec(x_59); -x_61 = lean_usize_sub(x_60, x_25); -x_62 = lean_usize_land(x_23, x_61); -x_63 = lean_array_uget(x_58, x_62); -x_64 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_63); -if (x_64 == 0) -{ -lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; uint8_t x_74; -x_65 = lean_unsigned_to_nat(1u); -x_66 = lean_nat_add(x_57, x_65); -lean_dec(x_57); -x_67 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_67, 0, x_11); -lean_ctor_set(x_67, 1, x_54); -lean_ctor_set(x_67, 2, x_63); -x_68 = lean_array_uset(x_58, x_62, x_67); -x_69 = lean_unsigned_to_nat(4u); -x_70 = lean_nat_mul(x_66, x_69); -x_71 = lean_unsigned_to_nat(3u); -x_72 = lean_nat_div(x_70, x_71); -lean_dec(x_70); -x_73 = lean_array_get_size(x_68); -x_74 = lean_nat_dec_le(x_72, x_73); -lean_dec(x_73); -lean_dec(x_72); -if (x_74 == 0) -{ -lean_object* x_75; size_t x_76; -x_75 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_68); -lean_ctor_set(x_55, 1, x_75); -lean_ctor_set(x_55, 0, x_66); -x_76 = lean_usize_add(x_7, x_25); -x_7 = x_76; -x_8 = x_55; -goto _start; -} -else -{ -size_t x_78; -lean_ctor_set(x_55, 1, x_68); -lean_ctor_set(x_55, 0, x_66); -x_78 = lean_usize_add(x_7, x_25); -x_7 = x_78; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_80; lean_object* x_81; lean_object* x_82; size_t x_83; +lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +lean_dec(x_10); lean_inc(x_3); -x_80 = lean_array_uset(x_58, x_62, x_3); -x_81 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_11, x_54, x_63); -x_82 = lean_array_uset(x_80, x_62, x_81); -lean_ctor_set(x_55, 1, x_82); -x_83 = lean_usize_add(x_7, x_25); -x_7 = x_83; -x_8 = x_55; -goto _start; -} -} -else -{ -lean_object* x_85; lean_object* x_86; lean_object* x_87; size_t x_88; size_t x_89; size_t x_90; lean_object* x_91; uint8_t x_92; -x_85 = lean_ctor_get(x_55, 0); -x_86 = lean_ctor_get(x_55, 1); -lean_inc(x_86); -lean_inc(x_85); -lean_dec(x_55); -x_87 = lean_array_get_size(x_86); -x_88 = lean_usize_of_nat(x_87); -lean_dec(x_87); -x_89 = lean_usize_sub(x_88, x_25); -x_90 = lean_usize_land(x_23, x_89); -x_91 = lean_array_uget(x_86, x_90); -x_92 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_91); -if (x_92 == 0) -{ -lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; uint8_t x_102; -x_93 = lean_unsigned_to_nat(1u); -x_94 = lean_nat_add(x_85, x_93); -lean_dec(x_85); -x_95 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_95, 0, x_11); -lean_ctor_set(x_95, 1, x_54); -lean_ctor_set(x_95, 2, x_91); -x_96 = lean_array_uset(x_86, x_90, x_95); -x_97 = lean_unsigned_to_nat(4u); -x_98 = lean_nat_mul(x_94, x_97); -x_99 = lean_unsigned_to_nat(3u); -x_100 = lean_nat_div(x_98, x_99); -lean_dec(x_98); -x_101 = lean_array_get_size(x_96); -x_102 = lean_nat_dec_le(x_100, x_101); -lean_dec(x_101); -lean_dec(x_100); -if (x_102 == 0) -{ -lean_object* x_103; lean_object* x_104; size_t x_105; -x_103 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_96); -x_104 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_104, 0, x_94); -lean_ctor_set(x_104, 1, x_103); -x_105 = lean_usize_add(x_7, x_25); -x_7 = x_105; -x_8 = x_104; -goto _start; -} -else +x_48 = lean_array_uset(x_15, x_28, x_3); +lean_inc(x_11); +x_49 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_11, x_12, x_29); +x_50 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_49); +lean_dec(x_11); +x_51 = lean_array_uset(x_48, x_28, x_49); +if (x_50 == 0) { -lean_object* x_107; size_t x_108; -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_94); -lean_ctor_set(x_107, 1, x_96); -x_108 = lean_usize_add(x_7, x_25); -x_7 = x_108; -x_8 = x_107; +lean_object* x_52; lean_object* x_53; size_t x_54; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_sub(x_14, x_52); +lean_dec(x_14); +lean_ctor_set(x_8, 1, x_51); +lean_ctor_set(x_8, 0, x_53); +x_54 = lean_usize_add(x_7, x_26); +x_7 = x_54; goto _start; } -} else { -lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; size_t x_114; -lean_inc(x_3); -x_110 = lean_array_uset(x_86, x_90, x_3); -x_111 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_11, x_54, x_91); -x_112 = lean_array_uset(x_110, x_90, x_111); -x_113 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_113, 0, x_85); -lean_ctor_set(x_113, 1, x_112); -x_114 = lean_usize_add(x_7, x_25); -x_7 = x_114; -x_8 = x_113; +size_t x_56; +lean_ctor_set(x_8, 1, x_51); +x_56 = lean_usize_add(x_7, x_26); +x_7 = x_56; goto _start; } } } -} -} else { -lean_object* x_123; lean_object* x_124; lean_object* x_125; uint64_t x_126; uint64_t x_127; uint64_t x_128; uint64_t x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; size_t x_133; size_t x_134; size_t x_135; size_t x_136; size_t x_137; lean_object* x_138; lean_object* x_139; -x_123 = lean_ctor_get(x_8, 0); -x_124 = lean_ctor_get(x_8, 1); -lean_inc(x_124); -lean_inc(x_123); +lean_object* x_58; lean_object* x_59; lean_object* x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; size_t x_68; size_t x_69; size_t x_70; size_t x_71; size_t x_72; lean_object* x_73; uint8_t x_74; +x_58 = lean_ctor_get(x_8, 0); +x_59 = lean_ctor_get(x_8, 1); +lean_inc(x_59); +lean_inc(x_58); lean_dec(x_8); -x_125 = lean_array_get_size(x_124); -x_126 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); -x_127 = 32; -x_128 = lean_uint64_shift_right(x_126, x_127); -x_129 = lean_uint64_xor(x_126, x_128); -x_130 = 16; -x_131 = lean_uint64_shift_right(x_129, x_130); -x_132 = lean_uint64_xor(x_129, x_131); -x_133 = lean_uint64_to_usize(x_132); -x_134 = lean_usize_of_nat(x_125); -lean_dec(x_125); -x_135 = 1; -x_136 = lean_usize_sub(x_134, x_135); -x_137 = lean_usize_land(x_133, x_136); -x_138 = lean_array_uget(x_124, x_137); -x_139 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_138); -if (lean_obj_tag(x_139) == 0) -{ -lean_object* x_140; lean_object* x_141; uint8_t x_142; -x_140 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_141 = lean_array_push(x_140, x_10); -x_142 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_138); -if (x_142 == 0) -{ -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; uint8_t x_152; -x_143 = lean_unsigned_to_nat(1u); -x_144 = lean_nat_add(x_123, x_143); -lean_dec(x_123); -x_145 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_145, 0, x_11); -lean_ctor_set(x_145, 1, x_141); -lean_ctor_set(x_145, 2, x_138); -x_146 = lean_array_uset(x_124, x_137, x_145); -x_147 = lean_unsigned_to_nat(4u); -x_148 = lean_nat_mul(x_144, x_147); -x_149 = lean_unsigned_to_nat(3u); -x_150 = lean_nat_div(x_148, x_149); -lean_dec(x_148); -x_151 = lean_array_get_size(x_146); -x_152 = lean_nat_dec_le(x_150, x_151); -lean_dec(x_151); -lean_dec(x_150); -if (x_152 == 0) +x_60 = lean_array_get_size(x_59); +x_61 = l___private_Lean_Data_Lsp_LanguageFeatures_0__Lean_Lsp_hashCallHierarchyItem____x40_Lean_Data_Lsp_LanguageFeatures___hyg_7188_(x_11); +x_62 = 32; +x_63 = lean_uint64_shift_right(x_61, x_62); +x_64 = lean_uint64_xor(x_61, x_63); +x_65 = 16; +x_66 = lean_uint64_shift_right(x_64, x_65); +x_67 = lean_uint64_xor(x_64, x_66); +x_68 = lean_uint64_to_usize(x_67); +x_69 = lean_usize_of_nat(x_60); +lean_dec(x_60); +x_70 = 1; +x_71 = lean_usize_sub(x_69, x_70); +x_72 = lean_usize_land(x_68, x_71); +x_73 = lean_array_uget(x_59, x_72); +x_74 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_73); +if (x_74 == 0) { -lean_object* x_153; lean_object* x_154; size_t x_155; -x_153 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_146); -x_154 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_154, 0, x_144); -lean_ctor_set(x_154, 1, x_153); -x_155 = lean_usize_add(x_7, x_135); -x_7 = x_155; -x_8 = x_154; -goto _start; -} -else +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; uint8_t x_86; +lean_dec(x_12); +x_75 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; +x_76 = lean_array_push(x_75, x_10); +x_77 = lean_unsigned_to_nat(1u); +x_78 = lean_nat_add(x_58, x_77); +lean_dec(x_58); +x_79 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_79, 0, x_11); +lean_ctor_set(x_79, 1, x_76); +lean_ctor_set(x_79, 2, x_73); +x_80 = lean_array_uset(x_59, x_72, x_79); +x_81 = lean_unsigned_to_nat(4u); +x_82 = lean_nat_mul(x_78, x_81); +x_83 = lean_unsigned_to_nat(3u); +x_84 = lean_nat_div(x_82, x_83); +lean_dec(x_82); +x_85 = lean_array_get_size(x_80); +x_86 = lean_nat_dec_le(x_84, x_85); +lean_dec(x_85); +lean_dec(x_84); +if (x_86 == 0) { -lean_object* x_157; size_t x_158; -x_157 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_157, 0, x_144); -lean_ctor_set(x_157, 1, x_146); -x_158 = lean_usize_add(x_7, x_135); -x_7 = x_158; -x_8 = x_157; +lean_object* x_87; lean_object* x_88; size_t x_89; +x_87 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_80); +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_78); +lean_ctor_set(x_88, 1, x_87); +x_89 = lean_usize_add(x_7, x_70); +x_7 = x_89; +x_8 = x_88; goto _start; } -} else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; size_t x_164; -lean_inc(x_3); -x_160 = lean_array_uset(x_124, x_137, x_3); -x_161 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_11, x_141, x_138); -x_162 = lean_array_uset(x_160, x_137, x_161); -x_163 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_163, 0, x_123); -lean_ctor_set(x_163, 1, x_162); -x_164 = lean_usize_add(x_7, x_135); -x_7 = x_164; -x_8 = x_163; +lean_object* x_91; size_t x_92; +x_91 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_91, 0, x_78); +lean_ctor_set(x_91, 1, x_80); +x_92 = lean_usize_add(x_7, x_70); +x_7 = x_92; +x_8 = x_91; goto _start; } } else { -lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_202; -x_166 = lean_ctor_get(x_139, 0); -lean_inc(x_166); -lean_dec(x_139); -x_167 = lean_array_push(x_166, x_10); -x_202 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_138); -if (x_202 == 0) -{ -lean_object* x_203; -lean_dec(x_138); -x_203 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_203, 0, x_123); -lean_ctor_set(x_203, 1, x_124); -x_168 = x_203; -goto block_201; -} -else -{ -lean_object* x_204; lean_object* x_205; lean_object* x_206; lean_object* x_207; lean_object* x_208; lean_object* x_209; +lean_object* x_94; lean_object* x_95; uint8_t x_96; lean_object* x_97; +lean_dec(x_10); lean_inc(x_3); -x_204 = lean_array_uset(x_124, x_137, x_3); -x_205 = lean_unsigned_to_nat(1u); -x_206 = lean_nat_sub(x_123, x_205); -lean_dec(x_123); -x_207 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_11, x_138); -x_208 = lean_array_uset(x_204, x_137, x_207); -x_209 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_209, 0, x_206); -lean_ctor_set(x_209, 1, x_208); -x_168 = x_209; -goto block_201; -} -block_201: -{ -lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; size_t x_173; size_t x_174; size_t x_175; lean_object* x_176; uint8_t x_177; -x_169 = lean_ctor_get(x_168, 0); -lean_inc(x_169); -x_170 = lean_ctor_get(x_168, 1); -lean_inc(x_170); -if (lean_is_exclusive(x_168)) { - lean_ctor_release(x_168, 0); - lean_ctor_release(x_168, 1); - x_171 = x_168; -} else { - lean_dec_ref(x_168); - x_171 = lean_box(0); -} -x_172 = lean_array_get_size(x_170); -x_173 = lean_usize_of_nat(x_172); -lean_dec(x_172); -x_174 = lean_usize_sub(x_173, x_135); -x_175 = lean_usize_land(x_133, x_174); -x_176 = lean_array_uget(x_170, x_175); -x_177 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_11, x_176); -if (x_177 == 0) -{ -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; uint8_t x_187; -x_178 = lean_unsigned_to_nat(1u); -x_179 = lean_nat_add(x_169, x_178); -lean_dec(x_169); -x_180 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_180, 0, x_11); -lean_ctor_set(x_180, 1, x_167); -lean_ctor_set(x_180, 2, x_176); -x_181 = lean_array_uset(x_170, x_175, x_180); -x_182 = lean_unsigned_to_nat(4u); -x_183 = lean_nat_mul(x_179, x_182); -x_184 = lean_unsigned_to_nat(3u); -x_185 = lean_nat_div(x_183, x_184); -lean_dec(x_183); -x_186 = lean_array_get_size(x_181); -x_187 = lean_nat_dec_le(x_185, x_186); -lean_dec(x_186); -lean_dec(x_185); -if (x_187 == 0) -{ -lean_object* x_188; lean_object* x_189; size_t x_190; -x_188 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__4(x_181); -if (lean_is_scalar(x_171)) { - x_189 = lean_alloc_ctor(0, 2, 0); -} else { - x_189 = x_171; -} -lean_ctor_set(x_189, 0, x_179); -lean_ctor_set(x_189, 1, x_188); -x_190 = lean_usize_add(x_7, x_135); -x_7 = x_190; -x_8 = x_189; -goto _start; -} -else +x_94 = lean_array_uset(x_59, x_72, x_3); +lean_inc(x_11); +x_95 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__6___rarg(x_11, x_12, x_73); +x_96 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_11, x_95); +lean_dec(x_11); +x_97 = lean_array_uset(x_94, x_72, x_95); +if (x_96 == 0) { -lean_object* x_192; size_t x_193; -if (lean_is_scalar(x_171)) { - x_192 = lean_alloc_ctor(0, 2, 0); -} else { - x_192 = x_171; -} -lean_ctor_set(x_192, 0, x_179); -lean_ctor_set(x_192, 1, x_181); -x_193 = lean_usize_add(x_7, x_135); -x_7 = x_193; -x_8 = x_192; +lean_object* x_98; lean_object* x_99; lean_object* x_100; size_t x_101; +x_98 = lean_unsigned_to_nat(1u); +x_99 = lean_nat_sub(x_58, x_98); +lean_dec(x_58); +x_100 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_100, 0, x_99); +lean_ctor_set(x_100, 1, x_97); +x_101 = lean_usize_add(x_7, x_70); +x_7 = x_101; +x_8 = x_100; goto _start; } -} else { -lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; size_t x_199; -lean_inc(x_3); -x_195 = lean_array_uset(x_170, x_175, x_3); -x_196 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_11, x_167, x_176); -x_197 = lean_array_uset(x_195, x_175, x_196); -if (lean_is_scalar(x_171)) { - x_198 = lean_alloc_ctor(0, 2, 0); -} else { - x_198 = x_171; -} -lean_ctor_set(x_198, 0, x_169); -lean_ctor_set(x_198, 1, x_197); -x_199 = lean_usize_add(x_7, x_135); -x_7 = x_199; -x_8 = x_198; +lean_object* x_103; size_t x_104; +x_103 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_103, 0, x_58); +lean_ctor_set(x_103, 1, x_97); +x_104 = lean_usize_add(x_7, x_70); +x_7 = x_104; +x_8 = x_103; goto _start; } } @@ -22909,7 +22168,6 @@ goto _start; } } } -} LEAN_EXPORT lean_object* l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -22919,11 +22177,11 @@ x_4 = lean_box(0); x_5 = lean_array_size(x_2); x_6 = 0; x_7 = l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__3; -x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); +x_8 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(x_1, x_2, x_3, x_4, x_2, x_5, x_6, x_7); return x_8; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -22949,7 +22207,7 @@ return x_4; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -22974,7 +22232,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -23009,7 +22267,7 @@ if (x_15 == 0) lean_object* x_16; lean_object* x_17; lean_object* x_18; x_16 = lean_ctor_get(x_14, 1); lean_dec(x_16); -x_17 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_17 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; lean_ctor_set(x_14, 1, x_17); x_18 = lean_array_uset(x_7, x_2, x_14); x_2 = x_9; @@ -23022,7 +22280,7 @@ lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; x_20 = lean_ctor_get(x_14, 0); lean_inc(x_20); lean_dec(x_14); -x_21 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_21 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; x_22 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_22, 0, x_20); lean_ctor_set(x_22, 1, x_21); @@ -23048,7 +22306,7 @@ if (x_28 == 0) lean_object* x_29; lean_object* x_30; lean_dec(x_11); lean_dec(x_10); -x_29 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_29 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; lean_ctor_set(x_25, 1, x_29); x_30 = lean_array_uset(x_7, x_2, x_25); x_2 = x_9; @@ -23061,8 +22319,8 @@ size_t x_32; size_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_3 x_32 = 0; x_33 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_34 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; -x_35 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(x_10, x_32, x_33, x_34); +x_34 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; +x_35 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_10, x_32, x_33, x_34); lean_dec(x_10); lean_ctor_set(x_25, 1, x_35); x_36 = lean_array_uset(x_7, x_2, x_25); @@ -23083,7 +22341,7 @@ if (x_39 == 0) lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_dec(x_11); lean_dec(x_10); -x_40 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; +x_40 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; x_41 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_41, 0, x_38); lean_ctor_set(x_41, 1, x_40); @@ -23098,8 +22356,8 @@ size_t x_44; size_t x_45; lean_object* x_46; lean_object* x_47; lean_object* x_4 x_44 = 0; x_45 = lean_usize_of_nat(x_11); lean_dec(x_11); -x_46 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1; -x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(x_10, x_44, x_45, x_46); +x_46 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1; +x_47 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_10, x_44, x_45, x_46); lean_dec(x_10); x_48 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_48, 0, x_38); @@ -23114,7 +22372,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -23123,7 +22381,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -23174,7 +22432,7 @@ lean_dec(x_5); lean_dec(x_4); x_9 = l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2; x_10 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(x_9, x_8, x_10); +x_11 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_9, x_8, x_10); return x_11; } else @@ -23188,7 +22446,7 @@ lean_dec(x_5); lean_dec(x_4); x_13 = l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2; x_14 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(x_13, x_8, x_14); +x_15 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_13, x_8, x_14); return x_15; } else @@ -23197,46 +22455,27 @@ size_t x_16; lean_object* x_17; lean_object* x_18; size_t x_19; lean_object* x_2 x_16 = lean_usize_of_nat(x_5); lean_dec(x_5); x_17 = l_Lean_Server_Watchdog_FileWorker_queuedMsgs___closed__1; -x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13(x_4, x_8, x_16, x_17); +x_18 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(x_4, x_8, x_16, x_17); lean_dec(x_4); x_19 = lean_array_size(x_18); -x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(x_19, x_8, x_18); +x_20 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_19, x_8, x_18); return x_20; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_1, x_2); -lean_dec(x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__3(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__2(x_1, x_2); lean_dec(x_2); lean_dec(x_1); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_1, x_2); -lean_dec(x_1); -return x_3; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { size_t x_9; size_t x_10; lean_object* x_11; @@ -23244,7 +22483,7 @@ x_9 = lean_unbox_usize(x_6); lean_dec(x_6); x_10 = lean_unbox_usize(x_7); lean_dec(x_7); -x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); +x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__6(x_1, x_2, x_3, x_4, x_5, x_9, x_10, x_8); lean_dec(x_5); lean_dec(x_4); lean_dec(x_2); @@ -23260,7 +22499,7 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -23268,21 +22507,21 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__7(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__11(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__8(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -23290,11 +22529,11 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__12(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__9(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -23302,7 +22541,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__13(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Server_Watchdog_handleCallHierarchyOutgoingCalls_collapseSameOutgoingCalls___spec__10(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -53715,8 +52954,8 @@ l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_co lean_mark_persistent(l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__2); l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__3 = _init_l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__3(); lean_mark_persistent(l_Array_groupByKey___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__1___closed__3); -l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__12___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___spec__10___closed__1); l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__1 = _init_l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__1(); lean_mark_persistent(l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__1); l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2 = _init_l_Lean_Server_Watchdog_handleCallHierarchyIncomingCalls_collapseSameIncomingCalls___closed__2(); diff --git a/stage0/stdlib/Lean/Util/Path.c b/stage0/stdlib/Lean/Util/Path.c index c5fb239629fb..c16ddb5009b6 100644 --- a/stage0/stdlib/Lean/Util/Path.c +++ b/stage0/stdlib/Lean/Util/Path.c @@ -42,6 +42,7 @@ LEAN_EXPORT lean_object* l_List_findM_x3f___at_Lean_SearchPath_findWithExt___spe static lean_object* l_Lean_modToFilePath_go___closed__3; static lean_object* l_Lean_findSysroot___lambda__1___closed__2; static lean_object* l_Lean_SearchPath_findAllWithExt___closed__1; +LEAN_EXPORT lean_object* l_Lean_findLean___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_getLibDir___closed__4; lean_object* l_System_FilePath_withExtension(lean_object*, lean_object*); lean_object* lean_io_getenv(lean_object*, lean_object*); @@ -115,6 +116,7 @@ static lean_object* l_Lean_moduleNameOfFileName___lambda__2___closed__1; extern uint32_t l_System_FilePath_pathSeparator; lean_object* l_Array_append___rarg(lean_object*, lean_object*); static lean_object* l_Lean_getBuildDir___closed__3; +static lean_object* l_Lean_findLean___closed__1; static lean_object* l_Lean_moduleNameOfFileName___lambda__2___closed__2; LEAN_EXPORT lean_object* l_Lean_moduleNameOfFileName___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); @@ -163,6 +165,7 @@ lean_object* lean_io_current_dir(lean_object*); static uint8_t l_Lean_getLibDir___closed__2; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); +LEAN_EXPORT lean_object* l_Lean_findLean(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_moduleNameOfFileName___lambda__3___closed__4; lean_object* lean_st_ref_set(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_modToFilePath(lean_object*, lean_object*, lean_object*); @@ -2191,6 +2194,140 @@ lean_dec(x_1); return x_3; } } +static lean_object* _init_l_Lean_findLean___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked(".lean' in the search path entries:\n", 35, 35); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Lean_findLean(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l_Array_forIn_x27Unsafe_loop___at_Lean_forEachModuleInDir___spec__2___rarg___lambda__5___closed__1; +lean_inc(x_1); +x_5 = l_Lean_SearchPath_findWithExt(x_1, x_4, x_2, x_3); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_8 = lean_ctor_get(x_5, 0); +lean_dec(x_8); +x_9 = l_Lean_Name_getRoot(x_2); +x_10 = 0; +x_11 = l_Lean_SearchPath_findWithExt___closed__1; +x_12 = l_Lean_Name_toString(x_9, x_10, x_11); +x_13 = l_Lean_findOLean___closed__2; +x_14 = lean_string_append(x_13, x_12); +x_15 = l_Lean_findOLean___closed__3; +x_16 = lean_string_append(x_14, x_15); +x_17 = lean_string_append(x_16, x_12); +x_18 = l_Lean_findOLean___closed__4; +x_19 = lean_string_append(x_17, x_18); +x_20 = lean_string_append(x_19, x_12); +lean_dec(x_12); +x_21 = l_Lean_findLean___closed__1; +x_22 = lean_string_append(x_20, x_21); +x_23 = lean_box(0); +x_24 = l_List_mapTR_loop___at_System_SearchPath_toString___spec__1(x_1, x_23); +x_25 = l_Lean_findOLean___closed__6; +x_26 = l_String_intercalate(x_25, x_24); +x_27 = lean_string_append(x_22, x_26); +lean_dec(x_26); +x_28 = l_Array_forIn_x27Unsafe_loop___at_Lean_forEachModuleInDir___spec__2___rarg___lambda__5___closed__3; +x_29 = lean_string_append(x_27, x_28); +x_30 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set_tag(x_5, 1); +lean_ctor_set(x_5, 0, x_30); +return x_5; +} +else +{ +lean_object* x_31; lean_object* x_32; uint8_t x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; +x_31 = lean_ctor_get(x_5, 1); +lean_inc(x_31); +lean_dec(x_5); +x_32 = l_Lean_Name_getRoot(x_2); +x_33 = 0; +x_34 = l_Lean_SearchPath_findWithExt___closed__1; +x_35 = l_Lean_Name_toString(x_32, x_33, x_34); +x_36 = l_Lean_findOLean___closed__2; +x_37 = lean_string_append(x_36, x_35); +x_38 = l_Lean_findOLean___closed__3; +x_39 = lean_string_append(x_37, x_38); +x_40 = lean_string_append(x_39, x_35); +x_41 = l_Lean_findOLean___closed__4; +x_42 = lean_string_append(x_40, x_41); +x_43 = lean_string_append(x_42, x_35); +lean_dec(x_35); +x_44 = l_Lean_findLean___closed__1; +x_45 = lean_string_append(x_43, x_44); +x_46 = lean_box(0); +x_47 = l_List_mapTR_loop___at_System_SearchPath_toString___spec__1(x_1, x_46); +x_48 = l_Lean_findOLean___closed__6; +x_49 = l_String_intercalate(x_48, x_47); +x_50 = lean_string_append(x_45, x_49); +lean_dec(x_49); +x_51 = l_Array_forIn_x27Unsafe_loop___at_Lean_forEachModuleInDir___spec__2___rarg___lambda__5___closed__3; +x_52 = lean_string_append(x_50, x_51); +x_53 = lean_alloc_ctor(18, 1, 0); +lean_ctor_set(x_53, 0, x_52); +x_54 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_54, 0, x_53); +lean_ctor_set(x_54, 1, x_31); +return x_54; +} +} +else +{ +uint8_t x_55; +lean_dec(x_1); +x_55 = !lean_is_exclusive(x_5); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; +x_56 = lean_ctor_get(x_5, 0); +lean_dec(x_56); +x_57 = lean_ctor_get(x_6, 0); +lean_inc(x_57); +lean_dec(x_6); +lean_ctor_set(x_5, 0, x_57); +return x_5; +} +else +{ +lean_object* x_58; lean_object* x_59; lean_object* x_60; +x_58 = lean_ctor_get(x_5, 1); +lean_inc(x_58); +lean_dec(x_5); +x_59 = lean_ctor_get(x_6, 0); +lean_inc(x_59); +lean_dec(x_6); +x_60 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_60, 0, x_59); +lean_ctor_set(x_60, 1, x_58); +return x_60; +} +} +} +} +LEAN_EXPORT lean_object* l_Lean_findLean___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Lean_findLean(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} LEAN_EXPORT lean_object* l_List_foldl___at_Lean_moduleNameOfFileName___spec__1(lean_object* x_1, lean_object* x_2) { _start: { @@ -3072,6 +3209,8 @@ l_Lean_findOLean___closed__5 = _init_l_Lean_findOLean___closed__5(); lean_mark_persistent(l_Lean_findOLean___closed__5); l_Lean_findOLean___closed__6 = _init_l_Lean_findOLean___closed__6(); lean_mark_persistent(l_Lean_findOLean___closed__6); +l_Lean_findLean___closed__1 = _init_l_Lean_findLean___closed__1(); +lean_mark_persistent(l_Lean_findLean___closed__1); l_Lean_moduleNameOfFileName___lambda__2___closed__1 = _init_l_Lean_moduleNameOfFileName___lambda__2___closed__1(); lean_mark_persistent(l_Lean_moduleNameOfFileName___lambda__2___closed__1); l_Lean_moduleNameOfFileName___lambda__2___closed__2 = _init_l_Lean_moduleNameOfFileName___lambda__2___closed__2(); diff --git a/stage0/stdlib/Lean/Util/Profiler.c b/stage0/stdlib/Lean/Util/Profiler.c index 4fbee4f47ca5..6ebd52f5d0cd 100644 --- a/stage0/stdlib/Lean/Util/Profiler.c +++ b/stage0/stdlib/Lean/Util/Profiler.c @@ -20,10 +20,12 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_col LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__23___boxed__const__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__14___boxed__const__1; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3731_(lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__17(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__6; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__21(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(uint64_t, lean_object*, lean_object*); static double l_Lean_Firefox_instFromJsonMilliseconds___closed__7; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__5; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__37___boxed(lean_object*, lean_object*); @@ -31,7 +33,6 @@ lean_object* lean_format_pretty(lean_object*, lean_object*, lean_object*, lean_o static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__7; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__19; LEAN_EXPORT lean_object* l_Lean_Firefox_instInhabitedFrameTable; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__30___boxed__const__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__20(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__27; @@ -57,7 +58,7 @@ LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Util_Pro static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__16; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____spec__3(lean_object*, lean_object*); static lean_object* l_Lean_Firefox_Thread_new___closed__1; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Firefox_Thread_new___closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__15; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____spec__1___boxed(lean_object*, lean_object*); @@ -79,7 +80,7 @@ lean_object* l_Lean_Json_mkObj(lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonProfileMeta; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586____closed__8; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__14; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17(lean_object*, double, lean_object*, double, size_t, size_t, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9(size_t, size_t, lean_object*); lean_object* l_Lean_PersistentArray_toArray___rarg(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__5; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonRawMarkerTable; @@ -97,8 +98,6 @@ LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJson LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__12___boxed__const__1; double lean_float_div(double, double); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__5(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__6___at_Lean_Firefox_Profile_export___spec__7(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__6(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Firefox_Profile_collide___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__9; uint64_t lean_uint64_of_nat(lean_object*); @@ -114,11 +113,13 @@ size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___lambda__1___boxed(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__42; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__41; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__38; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__16; +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1(lean_object*, lean_object*); lean_object* l_Lean_Name_toString(lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__11___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__12(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__29___boxed__const__1; lean_object* l_Array_findIdx_x3f_loop___rarg(lean_object*, lean_object*, lean_object*); @@ -135,6 +136,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrame static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__1; LEAN_EXPORT uint64_t l_Lean_Firefox_Profile_export___lambda__1(lean_object*); lean_object* lean_mk_array(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14___boxed(lean_object*, lean_object*); uint8_t lean_uint64_dec_lt(uint64_t, uint64_t); static lean_object* l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__4; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__41; @@ -142,8 +144,10 @@ uint8_t lean_usize_dec_eq(size_t, size_t); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__32; lean_object* l_Lean_JsonNumber_fromFloat_x3f(double); static lean_object* l_Lean_Firefox_instFromJsonSampleUnits___closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____spec__2(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__18; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonStackTable; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__17; @@ -154,7 +158,6 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Pr static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__1(lean_object*, lean_object*); LEAN_EXPORT double l_Lean_Firefox_instCoeFloatMicroseconds(double); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static double l_Lean_Firefox_instFromJsonMilliseconds___closed__6; lean_object* lean_array_fget(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__34___boxed__const__1; @@ -168,7 +171,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStack LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__6; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonMilliseconds(double); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__21; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__14; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__2; @@ -192,6 +194,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThrea static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__29; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__8; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____spec__2___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__5(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonFrameTable____x40_Lean_Util_Profiler___hyg_3307____spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__3___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850_(lean_object*); @@ -227,6 +230,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThrea LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__1___boxed(lean_object*, lean_object*); uint8_t lean_string_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__2___boxed(lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1(double, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__41; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfileMeta____x40_Lean_Util_Profiler___hyg_1116_(lean_object*); static lean_object* l_Lean_Firefox_categories___closed__7; @@ -234,27 +238,26 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfi static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__21; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__13; static lean_object* l_Lean_Firefox_instToJsonThread___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16___boxed(lean_object*, lean_object*); double lean_float_negate(double); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__34(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__36___boxed(lean_object*, lean_object*); lean_object* lean_string_utf8_byte_size(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__3(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__16(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__18; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__20; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__11; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); extern lean_object* l_instInhabitedNat; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonSamplesTable; static lean_object* l_Lean_Firefox_Profile_export___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__15(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____spec__1___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__34; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__11; static lean_object* l_Lean_Firefox_instToJsonRawMarkerTable___closed__1; static lean_object* l_Lean_Firefox_instInhabitedFrameTable___closed__1; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(uint64_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__5___at_Lean_Firefox_Profile_export___spec__6(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586____closed__10; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__32(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -267,11 +270,9 @@ lean_object* l_Lean_Name_mkStr3(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__22; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__15; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__41(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__9(lean_object*); static lean_object* l_Lean_Firefox_instToJsonSampleUnits___closed__1; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____spec__2___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__47; size_t lean_usize_of_nat(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__35; @@ -279,16 +280,19 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrame LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__2___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__3; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____spec__1___boxed(lean_object*, lean_object*); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2; static lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__13___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__15; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__2(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__1; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__19; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfile____x40_Lean_Util_Profiler___hyg_4847____spec__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonRawMarkerTable___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__6; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__26___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586____closed__7; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__21; @@ -309,8 +313,7 @@ static lean_object* l_Lean_Firefox_instToJsonFuncTable___closed__1; lean_object* lean_nat_to_int(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfileMeta____x40_Lean_Util_Profiler___hyg_1116____spec__1(size_t, size_t, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__38; -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1(double, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__21; lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____spec__4(size_t, size_t, lean_object*); @@ -325,7 +328,6 @@ static lean_object* l_Lean_Firefox_categories___closed__8; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__22; double lean_uint64_to_float(uint64_t); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__25; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__18___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__30; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__3; @@ -336,7 +338,6 @@ LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profile lean_object* l_Lean_MessageData_ofFormat(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__27; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__25(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__5(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__28; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__43; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__27___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -345,9 +346,7 @@ lean_object* lean_uint64_to_nat(uint64_t); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__14; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__21; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1; lean_object* l_outOfBounds___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Firefox_categories___closed__6; @@ -360,60 +359,58 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Pr static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__25; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__4; static lean_object* l_Lean_Firefox_categories___closed__2; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__25; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___lambda__2___closed__4; LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonSampleUnits; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__34; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfile____x40_Lean_Util_Profiler___hyg_4847_(lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(uint64_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__14; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__4(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__37; static lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__3; -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(uint64_t, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonProfile___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__30; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__26; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonSampleUnits____x40_Lean_Util_Profiler___hyg_617____boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__24(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Firefox_categories___closed__10; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__11; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16(size_t, size_t, lean_object*); lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Message_0__Lean_fromJsonBaseMessage____x40_Lean_Message___hyg_2877____spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonMilliseconds___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__13(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__31___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__17; -static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_collideThreads___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonMicroseconds___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__36(lean_object*, lean_object*); lean_object* l_Lean_Name_getRoot(lean_object*); lean_object* lean_io_mono_nanos_now(lean_object*); static lean_object* l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__3; -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__36; static lean_object* l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__12; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__9; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonThread___closed__1; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586_(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__22; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__12; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1939____spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__18___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_collideThreads_collideStacks(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonMicroseconds(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__3(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__15; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__39; -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__24___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__15; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____spec__3___boxed(lean_object*, lean_object*, lean_object*); @@ -421,6 +418,8 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_P extern lean_object* l_String_instInhabited; lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__12; +static lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15(lean_object*, double, lean_object*, double, size_t, size_t, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__4; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__12; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__38; @@ -441,23 +440,24 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCateg static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__34; LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonProfileMeta; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702_(lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonFuncTable; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__28(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__4; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__36; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__36; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(lean_object*); LEAN_EXPORT double l_Lean_Firefox_instOfScientificMicroseconds(lean_object*, uint8_t, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__23; LEAN_EXPORT lean_object* l_Lean_Firefox_Profile_export___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__38; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__5; LEAN_EXPORT double l_Lean_Firefox_instCoeFloatMilliseconds(double); +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonFrameTable____x40_Lean_Util_Profiler___hyg_3307_(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__33; static lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__4; static lean_object* l_Lean_Firefox_instInhabitedFrameTable___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__4(lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__1; static lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____spec__1___closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__24; @@ -468,6 +468,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncT LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__4___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__43; extern lean_object* l_Std_Format_defWidth; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9___boxed(lean_object*, lean_object*, lean_object*); static double l_Lean_Firefox_instInhabitedMilliseconds___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__3; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__4(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -476,6 +477,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCateg static lean_object* l_Lean_Firefox_categories___closed__3; static double l_Lean_Firefox_instFromJsonMilliseconds___closed__10; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___lambda__2___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__13; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_getFirstStart_x3f___lambda__2___closed__3; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__6; @@ -487,10 +489,11 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at___privat static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__20; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__23(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__7___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_Profile_export___lambda__1___boxed(lean_object*); lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Trace_0__Lean_addTraceNode___spec__1(size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1939_(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonStackTable____x40_Lean_Util_Profiler___hyg_1526____spec__2___boxed(lean_object*, lean_object*, lean_object*); @@ -523,7 +526,6 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_P static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__24; lean_object* l_Array_mapMUnsafe_map___at_Lean_Server_instRpcEncodableArray___spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonProfileMeta____x40_Lean_Util_Profiler___hyg_1116____spec__1___boxed(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__19; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonFuncTable____x40_Lean_Util_Profiler___hyg_2483____spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_collideThreads_collideSamples___spec__1___boxed__const__1; @@ -539,13 +541,12 @@ LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Pr LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__38(lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__7; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonFrameTable; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__28___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__4; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__34; +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT double l_Lean_Firefox_instAddMilliseconds(double, double); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(uint64_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__46; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__27___boxed__const__1; @@ -560,6 +561,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThrea static lean_object* l_Lean_Firefox_instToJsonProfile___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__14; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__20___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace(uint8_t, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__20; @@ -567,6 +569,7 @@ uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonCategory; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_collide___spec__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonFrameTable____x40_Lean_Util_Profiler___hyg_3307____spec__1___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__27; LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_collide___spec__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonCategory; @@ -576,7 +579,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThrea LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonResourceTable; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__19; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__5; -static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4; +static lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__25; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__32; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__13; @@ -591,6 +594,7 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncT static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__15; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____spec__1(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__24; +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Range_forIn_x27_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_collideThreads_collideSamples___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__29; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__22___boxed__const__1; @@ -603,7 +607,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncT static lean_object* l_Lean_Firefox_Thread_new___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__5___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__6(lean_object*, lean_object*); lean_object* lean_array_set(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____spec__2___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586____closed__6; uint8_t lean_float_beq(double, double); @@ -613,9 +616,11 @@ static lean_object* l_Lean_Firefox_instFromJsonSamplesTable___closed__1; LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____spec__2___boxed(lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__44; +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__16; LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776_(lean_object*); LEAN_EXPORT uint8_t l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____lambda__1(lean_object*); +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__46; LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonMilliseconds(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__12; @@ -649,15 +654,14 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStack static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__17; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__2; lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Data_Position_0__Lean_fromJsonPosition____x40_Lean_Data_Position___hyg_289____spec__1(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2(uint64_t, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__42; uint8_t lean_uint64_dec_eq(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__13___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__13; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonFrameTable; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__23___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_sub(size_t, size_t); +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3; lean_object* lean_array_mk(lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instFromJsonFuncTable; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__36; @@ -671,7 +675,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMa static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__12; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__12; size_t lean_usize_add(size_t, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__33; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__10; static lean_object* l_Lean_Firefox_Profile_collide___closed__6; @@ -689,8 +692,6 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonResou static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__4; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__19(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uget(lean_object*, size_t); -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__40; size_t lean_array_size(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__7; @@ -701,7 +702,6 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_P static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__24; static lean_object* l_Lean_Firefox_Profile_collide___closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__28; -static lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1; LEAN_EXPORT lean_object* l_Lean_Firefox_instOfScientificMicroseconds___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__23; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonResourceTable____x40_Lean_Util_Profiler___hyg_3825____closed__6; @@ -731,7 +731,6 @@ lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l_Lean_Firefox_instFromJsonMilliseconds___closed__2; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__21___boxed__const__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__12; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____spec__3___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -743,8 +742,8 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampl static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__23; lean_object* lean_int_neg(lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSamplesTable____x40_Lean_Util_Profiler___hyg_1677____closed__23; +static lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__18; -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFuncTable____x40_Lean_Util_Profiler___hyg_2143____closed__37; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonRawMarkerTable____x40_Lean_Util_Profiler___hyg_3586____closed__5; @@ -763,7 +762,6 @@ lean_object* l_Lean_Json_getObjValAs_x3f___at___private_Lean_Message_0__Lean_fro static lean_object* l_Lean_Firefox_instToJsonCategory___closed__1; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__9; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__9; -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonThread____x40_Lean_Util_Profiler___hyg_4084____closed__26; lean_object* lean_nat_add(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____closed__14; @@ -780,7 +778,7 @@ LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_beqOption____x4 LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_collideThreads_collideSamples___boxed(lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__16; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__2; -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_instDecidableEqUInt64___boxed(lean_object*, lean_object*); lean_object* l_Lean_Json_pretty(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonCategory____x40_Lean_Util_Profiler___hyg_230____lambda__1___boxed(lean_object*); @@ -802,7 +800,9 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampl static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonFrameTable____x40_Lean_Util_Profiler___hyg_2850____closed__7; LEAN_EXPORT lean_object* l_Lean_Firefox_instToJsonProfile; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__2___closed__2; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7(lean_object*); static lean_object* l_Lean_Firefox_instToJsonProfileMeta___closed__1; +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(double, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__10; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonStackTable____x40_Lean_Util_Profiler___hyg_1303____closed__14; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__22___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -816,10 +816,8 @@ static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfi static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonSampleUnits____x40_Lean_Util_Profiler___hyg_472____closed__17; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___spec__35___boxed__const__1; lean_object* l_Lean_MessageData_format(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_collide___spec__1(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Lean_Firefox_instCoeFloatMicroseconds___boxed(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13(lean_object*, size_t, size_t, lean_object*); size_t lean_usize_land(size_t, size_t); static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfile____x40_Lean_Util_Profiler___hyg_4702____closed__2; static lean_object* l___private_Lean_Util_Profiler_0__Lean_Firefox_fromJsonProfileMeta____x40_Lean_Util_Profiler___hyg_776____closed__35; @@ -46347,46 +46345,7 @@ lean_ctor_set_uint8(x_11, sizeof(void*)*9, x_3); return x_11; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2(uint64_t x_1, lean_object* x_2) { -_start: -{ -if (lean_obj_tag(x_2) == 0) -{ -lean_object* x_3; -x_3 = lean_box(0); -return x_3; -} -else -{ -lean_object* x_4; lean_object* x_5; lean_object* x_6; uint64_t x_7; uint8_t x_8; -x_4 = lean_ctor_get(x_2, 0); -lean_inc(x_4); -x_5 = lean_ctor_get(x_2, 1); -lean_inc(x_5); -x_6 = lean_ctor_get(x_2, 2); -lean_inc(x_6); -lean_dec(x_2); -x_7 = lean_unbox_uint64(x_4); -lean_dec(x_4); -x_8 = lean_uint64_dec_eq(x_7, x_1); -if (x_8 == 0) -{ -lean_dec(x_5); -x_2 = x_6; -goto _start; -} -else -{ -lean_object* x_10; -lean_dec(x_6); -x_10 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_10, 0, x_5); -return x_10; -} -} -} -} -LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(uint64_t x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(uint64_t x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -46421,7 +46380,7 @@ return x_9; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__6(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) @@ -46504,7 +46463,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__6___at_Lean_Firefox_Profile_export___spec__7(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__5___at_Lean_Firefox_Profile_export___spec__6(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -46580,7 +46539,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__5(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__4(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; uint8_t x_5; @@ -46599,7 +46558,7 @@ lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_obj x_6 = lean_array_fget(x_2, x_1); x_7 = lean_box(0); x_8 = lean_array_fset(x_2, x_1, x_7); -x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__6___at_Lean_Firefox_Profile_export___spec__7(x_3, x_6); +x_9 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__5___at_Lean_Firefox_Profile_export___spec__6(x_3, x_6); x_10 = lean_unsigned_to_nat(1u); x_11 = lean_nat_add(x_1, x_10); lean_dec(x_1); @@ -46610,7 +46569,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(lean_object* x_1) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__3(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; @@ -46621,157 +46580,181 @@ lean_dec(x_2); x_5 = lean_box(0); x_6 = lean_mk_array(x_4, x_5); x_7 = lean_unsigned_to_nat(0u); -x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__5(x_7, x_1, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_expand_go___at_Lean_Firefox_Profile_export___spec__4(x_7, x_1, x_6); return x_8; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(uint64_t x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(uint64_t x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_3) == 0) { -lean_object* x_4; -lean_dec(x_2); +lean_object* x_4; lean_object* x_5; x_4 = lean_box(0); -return x_4; +x_5 = lean_apply_1(x_2, x_4); +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; +x_6 = lean_box(0); +return x_6; } else { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_5, 0); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_box(0); +x_9 = lean_box_uint64(x_1); +x_10 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_7); +lean_ctor_set(x_10, 2, x_8); +return x_10; +} +} +else { -lean_object* x_6; lean_object* x_7; lean_object* x_8; uint64_t x_9; uint8_t x_10; -x_6 = lean_ctor_get(x_3, 0); -x_7 = lean_ctor_get(x_3, 1); -x_8 = lean_ctor_get(x_3, 2); -x_9 = lean_unbox_uint64(x_6); -x_10 = lean_uint64_dec_eq(x_9, x_1); -if (x_10 == 0) +uint8_t x_11; +x_11 = !lean_is_exclusive(x_3); +if (x_11 == 0) { -lean_object* x_11; -x_11 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_1, x_2, x_8); -lean_ctor_set(x_3, 2, x_11); +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint64_t x_15; uint8_t x_16; +x_12 = lean_ctor_get(x_3, 0); +x_13 = lean_ctor_get(x_3, 1); +x_14 = lean_ctor_get(x_3, 2); +x_15 = lean_unbox_uint64(x_12); +x_16 = lean_uint64_dec_eq(x_15, x_1); +if (x_16 == 0) +{ +lean_object* x_17; +x_17 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(x_1, x_2, x_14); +lean_ctor_set(x_3, 2, x_17); return x_3; } else { -lean_object* x_12; -lean_dec(x_7); -lean_dec(x_6); -x_12 = lean_box_uint64(x_1); -lean_ctor_set(x_3, 1, x_2); -lean_ctor_set(x_3, 0, x_12); +lean_object* x_18; lean_object* x_19; +lean_dec(x_12); +x_18 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_18, 0, x_13); +x_19 = lean_apply_1(x_2, x_18); +if (lean_obj_tag(x_19) == 0) +{ +lean_free_object(x_3); +return x_14; +} +else +{ +lean_object* x_20; lean_object* x_21; +x_20 = lean_ctor_get(x_19, 0); +lean_inc(x_20); +lean_dec(x_19); +x_21 = lean_box_uint64(x_1); +lean_ctor_set(x_3, 1, x_20); +lean_ctor_set(x_3, 0, x_21); return x_3; } } +} else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; uint64_t x_16; uint8_t x_17; -x_13 = lean_ctor_get(x_3, 0); -x_14 = lean_ctor_get(x_3, 1); -x_15 = lean_ctor_get(x_3, 2); -lean_inc(x_15); -lean_inc(x_14); -lean_inc(x_13); +lean_object* x_22; lean_object* x_23; lean_object* x_24; uint64_t x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_3, 0); +x_23 = lean_ctor_get(x_3, 1); +x_24 = lean_ctor_get(x_3, 2); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); lean_dec(x_3); -x_16 = lean_unbox_uint64(x_13); -x_17 = lean_uint64_dec_eq(x_16, x_1); -if (x_17 == 0) +x_25 = lean_unbox_uint64(x_22); +x_26 = lean_uint64_dec_eq(x_25, x_1); +if (x_26 == 0) { -lean_object* x_18; lean_object* x_19; -x_18 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_1, x_2, x_15); -x_19 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_19, 0, x_13); -lean_ctor_set(x_19, 1, x_14); -lean_ctor_set(x_19, 2, x_18); -return x_19; +lean_object* x_27; lean_object* x_28; +x_27 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(x_1, x_2, x_24); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_27); +return x_28; } else { -lean_object* x_20; lean_object* x_21; -lean_dec(x_14); -lean_dec(x_13); -x_20 = lean_box_uint64(x_1); -x_21 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_21, 0, x_20); -lean_ctor_set(x_21, 1, x_2); -lean_ctor_set(x_21, 2, x_15); -return x_21; +lean_object* x_29; lean_object* x_30; +lean_dec(x_22); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_23); +x_30 = lean_apply_1(x_2, x_29); +if (lean_obj_tag(x_30) == 0) +{ +return x_24; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_box_uint64(x_1); +x_33 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_31); +lean_ctor_set(x_33, 2, x_24); +return x_33; +} } } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(uint64_t x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg___boxed), 3, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) { -lean_object* x_3; -x_3 = lean_box(0); -return x_3; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_2); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; uint64_t x_8; uint8_t x_9; -x_5 = lean_ctor_get(x_2, 0); -x_6 = lean_ctor_get(x_2, 1); -x_7 = lean_ctor_get(x_2, 2); -x_8 = lean_unbox_uint64(x_5); -x_9 = lean_uint64_dec_eq(x_8, x_1); -if (x_9 == 0) +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) { -lean_object* x_10; -x_10 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(x_1, x_7); -lean_ctor_set(x_2, 2, x_10); +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); return x_2; } else { -lean_free_object(x_2); -lean_dec(x_6); -lean_dec(x_5); -return x_7; -} -} -else -{ -lean_object* x_11; lean_object* x_12; lean_object* x_13; uint64_t x_14; uint8_t x_15; -x_11 = lean_ctor_get(x_2, 0); -x_12 = lean_ctor_get(x_2, 1); -x_13 = lean_ctor_get(x_2, 2); -lean_inc(x_13); -lean_inc(x_12); -lean_inc(x_11); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); lean_dec(x_2); -x_14 = lean_unbox_uint64(x_11); -x_15 = lean_uint64_dec_eq(x_14, x_1); -if (x_15 == 0) -{ -lean_object* x_16; lean_object* x_17; -x_16 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(x_1, x_13); -x_17 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_17, 0, x_11); -lean_ctor_set(x_17, 1, x_12); -lean_ctor_set(x_17, 2, x_16); -return x_17; -} -else -{ -lean_dec(x_12); -lean_dec(x_11); -return x_13; -} +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, size_t x_7, size_t x_8, lean_object* x_9) { _start: { uint8_t x_10; @@ -46784,54 +46767,53 @@ return x_9; } else { -lean_object* x_11; lean_object* x_12; uint64_t x_13; uint8_t x_14; +lean_object* x_11; lean_object* x_12; uint64_t x_13; lean_object* x_14; uint8_t x_15; x_11 = lean_array_uget(x_6, x_8); lean_inc(x_1); lean_inc(x_11); x_12 = lean_apply_1(x_1, x_11); x_13 = lean_unbox_uint64(x_12); lean_dec(x_12); -x_14 = !lean_is_exclusive(x_9); -if (x_14 == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; size_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; -x_15 = lean_ctor_get(x_9, 0); -x_16 = lean_ctor_get(x_9, 1); -x_17 = lean_array_get_size(x_16); -x_18 = 32; -x_19 = lean_uint64_shift_right(x_13, x_18); -x_20 = lean_uint64_xor(x_13, x_19); -x_21 = 16; -x_22 = lean_uint64_shift_right(x_20, x_21); -x_23 = lean_uint64_xor(x_20, x_22); -x_24 = lean_uint64_to_usize(x_23); -x_25 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_26 = 1; -x_27 = lean_usize_sub(x_25, x_26); -x_28 = lean_usize_land(x_24, x_27); -x_29 = lean_array_uget(x_16, x_28); -lean_inc(x_29); -x_30 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2(x_13, x_29); -if (lean_obj_tag(x_30) == 0) +lean_inc(x_11); +x_14 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8___lambda__1), 2, 1); +lean_closure_set(x_14, 0, x_11); +x_15 = !lean_is_exclusive(x_9); +if (x_15 == 0) { -lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_31 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; -x_32 = lean_array_push(x_31, x_11); -lean_inc(x_29); -x_33 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_29); -if (x_33 == 0) +lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; lean_object* x_30; uint8_t x_31; +x_16 = lean_ctor_get(x_9, 0); +x_17 = lean_ctor_get(x_9, 1); +x_18 = lean_array_get_size(x_17); +x_19 = 32; +x_20 = lean_uint64_shift_right(x_13, x_19); +x_21 = lean_uint64_xor(x_13, x_20); +x_22 = 16; +x_23 = lean_uint64_shift_right(x_21, x_22); +x_24 = lean_uint64_xor(x_21, x_23); +x_25 = lean_uint64_to_usize(x_24); +x_26 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_27 = 1; +x_28 = lean_usize_sub(x_26, x_27); +x_29 = lean_usize_land(x_25, x_28); +x_30 = lean_array_uget(x_17, x_29); +lean_inc(x_30); +x_31 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(x_13, x_30); +if (x_31 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; uint8_t x_44; +lean_dec(x_14); +x_32 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; +x_33 = lean_array_push(x_32, x_11); x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_nat_add(x_15, x_34); -lean_dec(x_15); +x_35 = lean_nat_add(x_16, x_34); +lean_dec(x_16); x_36 = lean_box_uint64(x_13); x_37 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_37, 0, x_36); -lean_ctor_set(x_37, 1, x_32); -lean_ctor_set(x_37, 2, x_29); -x_38 = lean_array_uset(x_16, x_28, x_37); +lean_ctor_set(x_37, 1, x_33); +lean_ctor_set(x_37, 2, x_30); +x_38 = lean_array_uset(x_17, x_29, x_37); x_39 = lean_unsigned_to_nat(4u); x_40 = lean_nat_mul(x_35, x_39); x_41 = lean_unsigned_to_nat(3u); @@ -46844,10 +46826,10 @@ lean_dec(x_42); if (x_44 == 0) { lean_object* x_45; size_t x_46; -x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(x_38); +x_45 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__3(x_38); lean_ctor_set(x_9, 1, x_45); lean_ctor_set(x_9, 0, x_35); -x_46 = lean_usize_add(x_8, x_26); +x_46 = lean_usize_add(x_8, x_27); x_8 = x_46; goto _start; } @@ -46856,428 +46838,148 @@ else size_t x_48; lean_ctor_set(x_9, 1, x_38); lean_ctor_set(x_9, 0, x_35); -x_48 = lean_usize_add(x_8, x_26); +x_48 = lean_usize_add(x_8, x_27); x_8 = x_48; goto _start; } } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; size_t x_53; -lean_inc(x_4); -x_50 = lean_array_uset(x_16, x_28, x_4); -x_51 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_13, x_32, x_29); -x_52 = lean_array_uset(x_50, x_28, x_51); -lean_ctor_set(x_9, 1, x_52); -x_53 = lean_usize_add(x_8, x_26); -x_8 = x_53; -goto _start; -} -} -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_121; -x_55 = lean_ctor_get(x_30, 0); -lean_inc(x_55); -lean_dec(x_30); -x_56 = lean_array_push(x_55, x_11); -lean_inc(x_29); -x_121 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_29); -if (x_121 == 0) -{ -lean_dec(x_29); -x_57 = x_9; -goto block_120; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; -lean_inc(x_4); -x_122 = lean_array_uset(x_16, x_28, x_4); -x_123 = lean_unsigned_to_nat(1u); -x_124 = lean_nat_sub(x_15, x_123); -lean_dec(x_15); -x_125 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(x_13, x_29); -x_126 = lean_array_uset(x_122, x_28, x_125); -lean_ctor_set(x_9, 1, x_126); -lean_ctor_set(x_9, 0, x_124); -x_57 = x_9; -goto block_120; -} -block_120: -{ -uint8_t x_58; -x_58 = !lean_is_exclusive(x_57); -if (x_58 == 0) -{ -lean_object* x_59; lean_object* x_60; lean_object* x_61; size_t x_62; size_t x_63; size_t x_64; lean_object* x_65; uint8_t x_66; -x_59 = lean_ctor_get(x_57, 0); -x_60 = lean_ctor_get(x_57, 1); -x_61 = lean_array_get_size(x_60); -x_62 = lean_usize_of_nat(x_61); -lean_dec(x_61); -x_63 = lean_usize_sub(x_62, x_26); -x_64 = lean_usize_land(x_24, x_63); -x_65 = lean_array_uget(x_60, x_64); -lean_inc(x_65); -x_66 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_65); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; -x_67 = lean_unsigned_to_nat(1u); -x_68 = lean_nat_add(x_59, x_67); -lean_dec(x_59); -x_69 = lean_box_uint64(x_13); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_69); -lean_ctor_set(x_70, 1, x_56); -lean_ctor_set(x_70, 2, x_65); -x_71 = lean_array_uset(x_60, x_64, x_70); -x_72 = lean_unsigned_to_nat(4u); -x_73 = lean_nat_mul(x_68, x_72); -x_74 = lean_unsigned_to_nat(3u); -x_75 = lean_nat_div(x_73, x_74); -lean_dec(x_73); -x_76 = lean_array_get_size(x_71); -x_77 = lean_nat_dec_le(x_75, x_76); -lean_dec(x_76); -lean_dec(x_75); -if (x_77 == 0) -{ -lean_object* x_78; size_t x_79; -x_78 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(x_71); -lean_ctor_set(x_57, 1, x_78); -lean_ctor_set(x_57, 0, x_68); -x_79 = lean_usize_add(x_8, x_26); -x_8 = x_79; -x_9 = x_57; -goto _start; -} -else -{ -size_t x_81; -lean_ctor_set(x_57, 1, x_71); -lean_ctor_set(x_57, 0, x_68); -x_81 = lean_usize_add(x_8, x_26); -x_8 = x_81; -x_9 = x_57; -goto _start; -} -} -else -{ -lean_object* x_83; lean_object* x_84; lean_object* x_85; size_t x_86; +lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; +lean_dec(x_11); lean_inc(x_4); -x_83 = lean_array_uset(x_60, x_64, x_4); -x_84 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_13, x_56, x_65); -x_85 = lean_array_uset(x_83, x_64, x_84); -lean_ctor_set(x_57, 1, x_85); -x_86 = lean_usize_add(x_8, x_26); -x_8 = x_86; -x_9 = x_57; -goto _start; -} -} -else -{ -lean_object* x_88; lean_object* x_89; lean_object* x_90; size_t x_91; size_t x_92; size_t x_93; lean_object* x_94; uint8_t x_95; -x_88 = lean_ctor_get(x_57, 0); -x_89 = lean_ctor_get(x_57, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_57); -x_90 = lean_array_get_size(x_89); -x_91 = lean_usize_of_nat(x_90); -lean_dec(x_90); -x_92 = lean_usize_sub(x_91, x_26); -x_93 = lean_usize_land(x_24, x_92); -x_94 = lean_array_uget(x_89, x_93); -lean_inc(x_94); -x_95 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_94); -if (x_95 == 0) -{ -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; uint8_t x_106; -x_96 = lean_unsigned_to_nat(1u); -x_97 = lean_nat_add(x_88, x_96); -lean_dec(x_88); -x_98 = lean_box_uint64(x_13); -x_99 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_56); -lean_ctor_set(x_99, 2, x_94); -x_100 = lean_array_uset(x_89, x_93, x_99); -x_101 = lean_unsigned_to_nat(4u); -x_102 = lean_nat_mul(x_97, x_101); -x_103 = lean_unsigned_to_nat(3u); -x_104 = lean_nat_div(x_102, x_103); -lean_dec(x_102); -x_105 = lean_array_get_size(x_100); -x_106 = lean_nat_dec_le(x_104, x_105); -lean_dec(x_105); -lean_dec(x_104); -if (x_106 == 0) -{ -lean_object* x_107; lean_object* x_108; size_t x_109; -x_107 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(x_100); -x_108 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_108, 0, x_97); -lean_ctor_set(x_108, 1, x_107); -x_109 = lean_usize_add(x_8, x_26); -x_8 = x_109; -x_9 = x_108; -goto _start; -} -else +x_50 = lean_array_uset(x_17, x_29, x_4); +x_51 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(x_13, x_14, x_30); +lean_inc(x_51); +x_52 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(x_13, x_51); +x_53 = lean_array_uset(x_50, x_29, x_51); +if (x_52 == 0) { -lean_object* x_111; size_t x_112; -x_111 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_111, 0, x_97); -lean_ctor_set(x_111, 1, x_100); -x_112 = lean_usize_add(x_8, x_26); -x_8 = x_112; -x_9 = x_111; +lean_object* x_54; lean_object* x_55; size_t x_56; +x_54 = lean_unsigned_to_nat(1u); +x_55 = lean_nat_sub(x_16, x_54); +lean_dec(x_16); +lean_ctor_set(x_9, 1, x_53); +lean_ctor_set(x_9, 0, x_55); +x_56 = lean_usize_add(x_8, x_27); +x_8 = x_56; goto _start; } -} else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; size_t x_118; -lean_inc(x_4); -x_114 = lean_array_uset(x_89, x_93, x_4); -x_115 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_13, x_56, x_94); -x_116 = lean_array_uset(x_114, x_93, x_115); -x_117 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_117, 0, x_88); -lean_ctor_set(x_117, 1, x_116); -x_118 = lean_usize_add(x_8, x_26); -x_8 = x_118; -x_9 = x_117; +size_t x_58; +lean_ctor_set(x_9, 1, x_53); +x_58 = lean_usize_add(x_8, x_27); +x_8 = x_58; goto _start; } } } -} -} else { -lean_object* x_127; lean_object* x_128; lean_object* x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; uint64_t x_133; uint64_t x_134; uint64_t x_135; size_t x_136; size_t x_137; size_t x_138; size_t x_139; size_t x_140; lean_object* x_141; lean_object* x_142; -x_127 = lean_ctor_get(x_9, 0); -x_128 = lean_ctor_get(x_9, 1); -lean_inc(x_128); -lean_inc(x_127); +lean_object* x_60; lean_object* x_61; lean_object* x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; uint64_t x_68; size_t x_69; size_t x_70; size_t x_71; size_t x_72; size_t x_73; lean_object* x_74; uint8_t x_75; +x_60 = lean_ctor_get(x_9, 0); +x_61 = lean_ctor_get(x_9, 1); +lean_inc(x_61); +lean_inc(x_60); lean_dec(x_9); -x_129 = lean_array_get_size(x_128); -x_130 = 32; -x_131 = lean_uint64_shift_right(x_13, x_130); -x_132 = lean_uint64_xor(x_13, x_131); -x_133 = 16; -x_134 = lean_uint64_shift_right(x_132, x_133); -x_135 = lean_uint64_xor(x_132, x_134); -x_136 = lean_uint64_to_usize(x_135); -x_137 = lean_usize_of_nat(x_129); -lean_dec(x_129); -x_138 = 1; -x_139 = lean_usize_sub(x_137, x_138); -x_140 = lean_usize_land(x_136, x_139); -x_141 = lean_array_uget(x_128, x_140); -lean_inc(x_141); -x_142 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2(x_13, x_141); -if (lean_obj_tag(x_142) == 0) -{ -lean_object* x_143; lean_object* x_144; uint8_t x_145; -x_143 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; -x_144 = lean_array_push(x_143, x_11); -lean_inc(x_141); -x_145 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_141); -if (x_145 == 0) +x_62 = lean_array_get_size(x_61); +x_63 = 32; +x_64 = lean_uint64_shift_right(x_13, x_63); +x_65 = lean_uint64_xor(x_13, x_64); +x_66 = 16; +x_67 = lean_uint64_shift_right(x_65, x_66); +x_68 = lean_uint64_xor(x_65, x_67); +x_69 = lean_uint64_to_usize(x_68); +x_70 = lean_usize_of_nat(x_62); +lean_dec(x_62); +x_71 = 1; +x_72 = lean_usize_sub(x_70, x_71); +x_73 = lean_usize_land(x_69, x_72); +x_74 = lean_array_uget(x_61, x_73); +lean_inc(x_74); +x_75 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(x_13, x_74); +if (x_75 == 0) { -lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; -x_146 = lean_unsigned_to_nat(1u); -x_147 = lean_nat_add(x_127, x_146); -lean_dec(x_127); -x_148 = lean_box_uint64(x_13); -x_149 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_149, 0, x_148); -lean_ctor_set(x_149, 1, x_144); -lean_ctor_set(x_149, 2, x_141); -x_150 = lean_array_uset(x_128, x_140, x_149); -x_151 = lean_unsigned_to_nat(4u); -x_152 = lean_nat_mul(x_147, x_151); -x_153 = lean_unsigned_to_nat(3u); -x_154 = lean_nat_div(x_152, x_153); -lean_dec(x_152); -x_155 = lean_array_get_size(x_150); -x_156 = lean_nat_dec_le(x_154, x_155); -lean_dec(x_155); -lean_dec(x_154); -if (x_156 == 0) -{ -lean_object* x_157; lean_object* x_158; size_t x_159; -x_157 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(x_150); -x_158 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_158, 0, x_147); -lean_ctor_set(x_158, 1, x_157); -x_159 = lean_usize_add(x_8, x_138); -x_8 = x_159; -x_9 = x_158; -goto _start; -} -else +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; uint8_t x_88; +lean_dec(x_14); +x_76 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; +x_77 = lean_array_push(x_76, x_11); +x_78 = lean_unsigned_to_nat(1u); +x_79 = lean_nat_add(x_60, x_78); +lean_dec(x_60); +x_80 = lean_box_uint64(x_13); +x_81 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_81, 0, x_80); +lean_ctor_set(x_81, 1, x_77); +lean_ctor_set(x_81, 2, x_74); +x_82 = lean_array_uset(x_61, x_73, x_81); +x_83 = lean_unsigned_to_nat(4u); +x_84 = lean_nat_mul(x_79, x_83); +x_85 = lean_unsigned_to_nat(3u); +x_86 = lean_nat_div(x_84, x_85); +lean_dec(x_84); +x_87 = lean_array_get_size(x_82); +x_88 = lean_nat_dec_le(x_86, x_87); +lean_dec(x_87); +lean_dec(x_86); +if (x_88 == 0) { -lean_object* x_161; size_t x_162; -x_161 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_161, 0, x_147); -lean_ctor_set(x_161, 1, x_150); -x_162 = lean_usize_add(x_8, x_138); -x_8 = x_162; -x_9 = x_161; +lean_object* x_89; lean_object* x_90; size_t x_91; +x_89 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__3(x_82); +x_90 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_90, 0, x_79); +lean_ctor_set(x_90, 1, x_89); +x_91 = lean_usize_add(x_8, x_71); +x_8 = x_91; +x_9 = x_90; goto _start; } -} else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; size_t x_168; -lean_inc(x_4); -x_164 = lean_array_uset(x_128, x_140, x_4); -x_165 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_13, x_144, x_141); -x_166 = lean_array_uset(x_164, x_140, x_165); -x_167 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_167, 0, x_127); -lean_ctor_set(x_167, 1, x_166); -x_168 = lean_usize_add(x_8, x_138); -x_8 = x_168; -x_9 = x_167; +lean_object* x_93; size_t x_94; +x_93 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_93, 0, x_79); +lean_ctor_set(x_93, 1, x_82); +x_94 = lean_usize_add(x_8, x_71); +x_8 = x_94; +x_9 = x_93; goto _start; } } else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; uint8_t x_207; -x_170 = lean_ctor_get(x_142, 0); -lean_inc(x_170); -lean_dec(x_142); -x_171 = lean_array_push(x_170, x_11); -lean_inc(x_141); -x_207 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_141); -if (x_207 == 0) -{ -lean_object* x_208; -lean_dec(x_141); -x_208 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_208, 0, x_127); -lean_ctor_set(x_208, 1, x_128); -x_172 = x_208; -goto block_206; -} -else -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; +lean_object* x_96; lean_object* x_97; uint8_t x_98; lean_object* x_99; +lean_dec(x_11); lean_inc(x_4); -x_209 = lean_array_uset(x_128, x_140, x_4); -x_210 = lean_unsigned_to_nat(1u); -x_211 = lean_nat_sub(x_127, x_210); -lean_dec(x_127); -x_212 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(x_13, x_141); -x_213 = lean_array_uset(x_209, x_140, x_212); -x_214 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_214, 0, x_211); -lean_ctor_set(x_214, 1, x_213); -x_172 = x_214; -goto block_206; -} -block_206: -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; size_t x_177; size_t x_178; size_t x_179; lean_object* x_180; uint8_t x_181; -x_173 = lean_ctor_get(x_172, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_172, 1); -lean_inc(x_174); -if (lean_is_exclusive(x_172)) { - lean_ctor_release(x_172, 0); - lean_ctor_release(x_172, 1); - x_175 = x_172; -} else { - lean_dec_ref(x_172); - x_175 = lean_box(0); -} -x_176 = lean_array_get_size(x_174); -x_177 = lean_usize_of_nat(x_176); -lean_dec(x_176); -x_178 = lean_usize_sub(x_177, x_138); -x_179 = lean_usize_land(x_136, x_178); -x_180 = lean_array_uget(x_174, x_179); -lean_inc(x_180); -x_181 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_13, x_180); -if (x_181 == 0) -{ -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; uint8_t x_192; -x_182 = lean_unsigned_to_nat(1u); -x_183 = lean_nat_add(x_173, x_182); -lean_dec(x_173); -x_184 = lean_box_uint64(x_13); -x_185 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_185, 0, x_184); -lean_ctor_set(x_185, 1, x_171); -lean_ctor_set(x_185, 2, x_180); -x_186 = lean_array_uset(x_174, x_179, x_185); -x_187 = lean_unsigned_to_nat(4u); -x_188 = lean_nat_mul(x_183, x_187); -x_189 = lean_unsigned_to_nat(3u); -x_190 = lean_nat_div(x_188, x_189); -lean_dec(x_188); -x_191 = lean_array_get_size(x_186); -x_192 = lean_nat_dec_le(x_190, x_191); -lean_dec(x_191); -lean_dec(x_190); -if (x_192 == 0) -{ -lean_object* x_193; lean_object* x_194; size_t x_195; -x_193 = l_Std_DHashMap_Internal_Raw_u2080_expand___at_Lean_Firefox_Profile_export___spec__4(x_186); -if (lean_is_scalar(x_175)) { - x_194 = lean_alloc_ctor(0, 2, 0); -} else { - x_194 = x_175; -} -lean_ctor_set(x_194, 0, x_183); -lean_ctor_set(x_194, 1, x_193); -x_195 = lean_usize_add(x_8, x_138); -x_8 = x_195; -x_9 = x_194; -goto _start; -} -else +x_96 = lean_array_uset(x_61, x_73, x_4); +x_97 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(x_13, x_14, x_74); +lean_inc(x_97); +x_98 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(x_13, x_97); +x_99 = lean_array_uset(x_96, x_73, x_97); +if (x_98 == 0) { -lean_object* x_197; size_t x_198; -if (lean_is_scalar(x_175)) { - x_197 = lean_alloc_ctor(0, 2, 0); -} else { - x_197 = x_175; -} -lean_ctor_set(x_197, 0, x_183); -lean_ctor_set(x_197, 1, x_186); -x_198 = lean_usize_add(x_8, x_138); -x_8 = x_198; -x_9 = x_197; +lean_object* x_100; lean_object* x_101; lean_object* x_102; size_t x_103; +x_100 = lean_unsigned_to_nat(1u); +x_101 = lean_nat_sub(x_60, x_100); +lean_dec(x_60); +x_102 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_102, 0, x_101); +lean_ctor_set(x_102, 1, x_99); +x_103 = lean_usize_add(x_8, x_71); +x_8 = x_103; +x_9 = x_102; goto _start; } -} else { -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; size_t x_204; -lean_inc(x_4); -x_200 = lean_array_uset(x_174, x_179, x_4); -x_201 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_13, x_171, x_180); -x_202 = lean_array_uset(x_200, x_179, x_201); -if (lean_is_scalar(x_175)) { - x_203 = lean_alloc_ctor(0, 2, 0); -} else { - x_203 = x_175; -} -lean_ctor_set(x_203, 0, x_173); -lean_ctor_set(x_203, 1, x_202); -x_204 = lean_usize_add(x_8, x_138); -x_8 = x_204; -x_9 = x_203; +lean_object* x_105; size_t x_106; +x_105 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_60); +lean_ctor_set(x_105, 1, x_99); +x_106 = lean_usize_add(x_8, x_71); +x_8 = x_106; +x_9 = x_105; goto _start; } } @@ -47285,7 +46987,6 @@ goto _start; } } } -} static lean_object* _init_l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__1() { _start: { @@ -47346,11 +47047,11 @@ x_5 = lean_array_size(x_2); x_6 = 0; x_7 = l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__2; x_8 = l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__5; -x_9 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(x_1, x_2, x_7, x_3, x_4, x_2, x_5, x_6, x_8); +x_9 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8(x_1, x_2, x_7, x_3, x_4, x_2, x_5, x_6, x_8); return x_9; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -47379,7 +47080,7 @@ goto _start; } } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1() { _start: { lean_object* x_1; @@ -47387,11 +47088,11 @@ x_1 = l_Lean_trace_profiler_output_pp; return x_1; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; uint8_t x_7; lean_object* x_8; uint8_t x_9; -x_6 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1; +x_6 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1; x_7 = l_Lean_Option_get___at___private_Lean_Util_Profile_0__Lean_get__profiler___spec__1(x_1, x_6); x_8 = l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace(x_7, x_3, x_2, x_5); x_9 = !lean_is_exclusive(x_8); @@ -47421,7 +47122,7 @@ return x_15; } } } -static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1() { +static lean_object* _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1() { _start: { double x_1; lean_object* x_2; @@ -47430,7 +47131,7 @@ x_2 = lean_box_float(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -47466,7 +47167,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); x_19 = lean_box(0); -x_20 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_11, x_7, x_19, x_8); +x_20 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_11, x_7, x_19, x_8); x_21 = lean_ctor_get(x_20, 0); lean_inc(x_21); x_22 = lean_ctor_get(x_20, 1); @@ -47494,7 +47195,7 @@ lean_dec(x_14); lean_dec(x_13); lean_dec(x_12); x_28 = lean_box(0); -x_29 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_11, x_7, x_28, x_8); +x_29 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_11, x_7, x_28, x_8); x_30 = lean_ctor_get(x_29, 0); lean_inc(x_30); x_31 = lean_ctor_get(x_29, 1); @@ -47551,15 +47252,15 @@ x_55 = lean_box_float(x_54); x_56 = lean_array_push(x_52, x_55); x_57 = lean_ctor_get(x_43, 2); lean_inc(x_57); -x_58 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_58 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_59 = lean_array_push(x_57, x_58); -x_60 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_60 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_61 = lean_array_push(x_59, x_60); x_62 = lean_ctor_get(x_43, 4); lean_inc(x_62); -x_63 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_63 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_64 = lean_array_push(x_62, x_63); -x_65 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_65 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_66 = lean_array_push(x_64, x_65); x_67 = lean_ctor_get(x_43, 5); lean_inc(x_67); @@ -47577,7 +47278,7 @@ lean_ctor_set(x_71, 4, x_66); lean_ctor_set(x_71, 5, x_69); lean_ctor_set(x_12, 2, x_71); x_72 = lean_box(0); -x_73 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_11, x_7, x_72, x_8); +x_73 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_11, x_7, x_72, x_8); x_74 = lean_ctor_get(x_73, 0); lean_inc(x_74); x_75 = lean_ctor_get(x_73, 1); @@ -47634,15 +47335,15 @@ x_101 = lean_box_float(x_100); x_102 = lean_array_push(x_98, x_101); x_103 = lean_ctor_get(x_83, 2); lean_inc(x_103); -x_104 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_104 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_105 = lean_array_push(x_103, x_104); -x_106 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_106 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_107 = lean_array_push(x_105, x_106); x_108 = lean_ctor_get(x_83, 4); lean_inc(x_108); -x_109 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_109 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_110 = lean_array_push(x_108, x_109); -x_111 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_111 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_112 = lean_array_push(x_110, x_111); x_113 = lean_ctor_get(x_83, 5); lean_inc(x_113); @@ -47671,7 +47372,7 @@ lean_ctor_set(x_118, 8, x_89); lean_ctor_set_uint8(x_118, sizeof(void*)*9, x_82); lean_ctor_set(x_7, 0, x_118); x_119 = lean_box(0); -x_120 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_11, x_7, x_119, x_8); +x_120 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_11, x_7, x_119, x_8); x_121 = lean_ctor_get(x_120, 0); lean_inc(x_121); x_122 = lean_ctor_get(x_120, 1); @@ -47747,15 +47448,15 @@ x_150 = lean_box_float(x_149); x_151 = lean_array_push(x_147, x_150); x_152 = lean_ctor_get(x_131, 2); lean_inc(x_152); -x_153 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_153 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_154 = lean_array_push(x_152, x_153); -x_155 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_155 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_156 = lean_array_push(x_154, x_155); x_157 = lean_ctor_get(x_131, 4); lean_inc(x_157); -x_158 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_158 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_159 = lean_array_push(x_157, x_158); -x_160 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1; +x_160 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1; x_161 = lean_array_push(x_159, x_160); x_162 = lean_ctor_get(x_131, 5); lean_inc(x_162); @@ -47793,7 +47494,7 @@ lean_ctor_set(x_168, 2, x_14); lean_ctor_set(x_168, 3, x_15); lean_ctor_set_float(x_168, sizeof(void*)*4, x_16); x_169 = lean_box(0); -x_170 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_11, x_168, x_169, x_8); +x_170 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_11, x_168, x_169, x_8); x_171 = lean_ctor_get(x_170, 0); lean_inc(x_171); x_172 = lean_ctor_get(x_170, 1); @@ -47814,7 +47515,7 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -47837,7 +47538,7 @@ return x_4; } } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1(double x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1(double x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; lean_object* x_5; lean_object* x_6; @@ -47984,12 +47685,12 @@ return x_38; } } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(double x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(double x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; uint8_t x_10; x_8 = lean_box_float(x_1); -x_9 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1___boxed), 3, 1); +x_9 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed), 3, 1); lean_closure_set(x_9, 0, x_8); x_10 = lean_nat_dec_lt(x_4, x_5); if (x_10 == 0) @@ -48012,7 +47713,7 @@ x_14 = lean_nat_dec_le(x_5, x_12); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(x_1, x_2, x_13, x_4, x_12, lean_box(0), lean_box(0)); +x_15 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(x_1, x_2, x_13, x_4, x_12, lean_box(0), lean_box(0)); x_16 = lean_unsigned_to_nat(1u); x_17 = lean_nat_add(x_12, x_16); lean_dec(x_12); @@ -48031,12 +47732,12 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(double x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(double x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { lean_object* x_8; lean_object* x_9; uint8_t x_10; x_8 = lean_box_float(x_1); -x_9 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1___boxed), 3, 1); +x_9 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed), 3, 1); lean_closure_set(x_9, 0, x_8); x_10 = lean_nat_dec_lt(x_4, x_5); if (x_10 == 0) @@ -48059,7 +47760,7 @@ x_14 = lean_nat_dec_le(x_5, x_12); if (x_14 == 0) { lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(x_1, x_2, x_13, x_4, x_12, lean_box(0), lean_box(0)); +x_15 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(x_1, x_2, x_13, x_4, x_12, lean_box(0), lean_box(0)); x_16 = lean_unsigned_to_nat(1u); x_17 = lean_nat_add(x_12, x_16); lean_dec(x_12); @@ -48078,7 +47779,7 @@ return x_13; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14(lean_object* x_1, lean_object* x_2) { _start: { if (lean_obj_tag(x_2) == 0) @@ -48103,13 +47804,13 @@ goto _start; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(lean_object* x_1, size_t x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; size_t x_8; lean_object* x_9; uint8_t x_10; x_7 = lean_box(0); x_8 = lean_array_size(x_4); -x_9 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12(x_1, x_4, x_7, x_4, x_8, x_2, x_3, x_6); +x_9 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(x_1, x_4, x_7, x_4, x_8, x_2, x_3, x_6); x_10 = !lean_is_exclusive(x_9); if (x_10 == 0) { @@ -48130,7 +47831,7 @@ return x_13; } } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1() { _start: { lean_object* x_1; @@ -48138,17 +47839,17 @@ x_1 = lean_mk_string_unchecked("runFrontend", 11, 11); return x_1; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1; +x_2 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3() { _start: { lean_object* x_1; lean_object* x_2; @@ -48158,16 +47859,16 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4() { +static lean_object* _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3; +x_1 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3; x_2 = l_Lean_MessageData_ofFormat(x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17(lean_object* x_1, double x_2, lean_object* x_3, double x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15(lean_object* x_1, double x_2, lean_object* x_3, double x_4, size_t x_5, size_t x_6, lean_object* x_7, lean_object* x_8) { _start: { uint8_t x_9; @@ -48204,7 +47905,7 @@ x_18 = lean_unbox_uint64(x_14); x_19 = lean_uint64_dec_eq(x_18, x_17); x_20 = lean_array_size(x_15); x_21 = 0; -x_22 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11(x_20, x_21, x_15); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9(x_20, x_21, x_15); x_23 = lean_array_get_size(x_22); x_24 = lean_unsigned_to_nat(1u); x_25 = lean_nat_sub(x_23, x_24); @@ -48259,7 +47960,7 @@ if (x_75 == 0) { lean_object* x_76; lean_inc(x_25); -x_76 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(x_34, x_23, x_22, x_25, x_25, lean_box(0), lean_box(0)); +x_76 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(x_34, x_23, x_22, x_25, x_25, lean_box(0), lean_box(0)); lean_dec(x_25); lean_dec(x_23); x_65 = x_76; @@ -48268,7 +47969,7 @@ goto block_74; else { lean_object* x_77; -x_77 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(x_34, x_23, x_22, x_12, x_25, lean_box(0), lean_box(0)); +x_77 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(x_34, x_23, x_22, x_12, x_25, lean_box(0), lean_box(0)); lean_dec(x_25); lean_dec(x_23); x_65 = x_77; @@ -48292,7 +47993,7 @@ if (x_19 == 0) lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; size_t x_43; size_t x_44; lean_object* x_45; lean_dec(x_16); x_39 = lean_box(0); -x_40 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_3, x_21, x_35, x_38, x_39, x_8); +x_40 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(x_3, x_21, x_35, x_38, x_39, x_8); lean_dec(x_38); x_41 = lean_ctor_get(x_40, 0); lean_inc(x_41); @@ -48310,7 +48011,7 @@ goto _start; else { lean_object* x_47; uint8_t x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; size_t x_60; size_t x_61; lean_object* x_62; -x_47 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2; +x_47 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2; x_48 = 1; x_49 = l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__3___closed__1; x_50 = lean_alloc_ctor(0, 2, 17); @@ -48319,7 +48020,7 @@ lean_ctor_set(x_50, 1, x_49); lean_ctor_set_float(x_50, sizeof(void*)*2, x_2); lean_ctor_set_float(x_50, sizeof(void*)*2 + 8, x_4); lean_ctor_set_uint8(x_50, sizeof(void*)*2 + 16, x_48); -x_51 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4; +x_51 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4; x_52 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_52, 0, x_50); lean_ctor_set(x_52, 1, x_51); @@ -48335,7 +48036,7 @@ lean_ctor_set(x_54, 0, x_52); lean_ctor_set(x_54, 1, x_53); x_55 = lean_array_mk(x_54); x_56 = lean_box(0); -x_57 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_3, x_21, x_35, x_55, x_56, x_8); +x_57 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(x_3, x_21, x_35, x_55, x_56, x_8); lean_dec(x_55); x_58 = lean_ctor_get(x_57, 0); lean_inc(x_58); @@ -48384,7 +48085,7 @@ size_t x_71; lean_object* x_72; lean_object* x_73; x_71 = lean_usize_of_nat(x_66); lean_dec(x_66); x_72 = l_Lean_Firefox_instInhabitedFrameTable___closed__1; -x_73 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13(x_65, x_21, x_71, x_72); +x_73 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11(x_65, x_21, x_71, x_72); lean_dec(x_65); x_36 = x_73; goto block_64; @@ -48438,7 +48139,7 @@ if (x_129 == 0) { lean_object* x_130; lean_inc(x_25); -x_130 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(x_88, x_23, x_22, x_25, x_25, lean_box(0), lean_box(0)); +x_130 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(x_88, x_23, x_22, x_25, x_25, lean_box(0), lean_box(0)); lean_dec(x_25); lean_dec(x_23); x_119 = x_130; @@ -48447,7 +48148,7 @@ goto block_128; else { lean_object* x_131; -x_131 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(x_88, x_23, x_22, x_12, x_25, lean_box(0), lean_box(0)); +x_131 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(x_88, x_23, x_22, x_12, x_25, lean_box(0), lean_box(0)); lean_dec(x_25); lean_dec(x_23); x_119 = x_131; @@ -48471,7 +48172,7 @@ if (x_19 == 0) lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; size_t x_97; size_t x_98; lean_object* x_99; lean_dec(x_16); x_93 = lean_box(0); -x_94 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_3, x_21, x_89, x_92, x_93, x_8); +x_94 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(x_3, x_21, x_89, x_92, x_93, x_8); lean_dec(x_92); x_95 = lean_ctor_get(x_94, 0); lean_inc(x_95); @@ -48489,7 +48190,7 @@ goto _start; else { lean_object* x_101; uint8_t x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; lean_object* x_113; size_t x_114; size_t x_115; lean_object* x_116; -x_101 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2; +x_101 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2; x_102 = 1; x_103 = l___private_Lean_Util_Profiler_0__Lean_Firefox_addTrace_go___lambda__3___closed__1; x_104 = lean_alloc_ctor(0, 2, 17); @@ -48498,7 +48199,7 @@ lean_ctor_set(x_104, 1, x_103); lean_ctor_set_float(x_104, sizeof(void*)*2, x_2); lean_ctor_set_float(x_104, sizeof(void*)*2 + 8, x_4); lean_ctor_set_uint8(x_104, sizeof(void*)*2 + 16, x_102); -x_105 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4; +x_105 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4; x_106 = lean_alloc_ctor(9, 3, 0); lean_ctor_set(x_106, 0, x_104); lean_ctor_set(x_106, 1, x_105); @@ -48514,7 +48215,7 @@ lean_ctor_set(x_108, 0, x_106); lean_ctor_set(x_108, 1, x_107); x_109 = lean_array_mk(x_108); x_110 = lean_box(0); -x_111 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_3, x_21, x_89, x_109, x_110, x_8); +x_111 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(x_3, x_21, x_89, x_109, x_110, x_8); lean_dec(x_109); x_112 = lean_ctor_get(x_111, 0); lean_inc(x_112); @@ -48563,7 +48264,7 @@ size_t x_125; lean_object* x_126; lean_object* x_127; x_125 = lean_usize_of_nat(x_120); lean_dec(x_120); x_126 = l_Lean_Firefox_instInhabitedFrameTable___closed__1; -x_127 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13(x_119, x_21, x_125, x_126); +x_127 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11(x_119, x_21, x_125, x_126); lean_dec(x_119); x_90 = x_127; goto block_118; @@ -48575,7 +48276,7 @@ goto block_118; } } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18(size_t x_1, size_t x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16(size_t x_1, size_t x_2, lean_object* x_3) { _start: { uint8_t x_4; @@ -48602,7 +48303,7 @@ goto _start; } } } -LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT uint8_t l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; uint64_t x_5; uint64_t x_6; uint8_t x_7; @@ -48620,15 +48321,15 @@ x_7 = lean_uint64_dec_lt(x_5, x_6); return x_7; } } -static lean_object* _init_l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1() { +static lean_object* _init_l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1() { _start: { lean_object* x_1; -x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1___boxed), 2, 0); +x_1 = lean_alloc_closure((void*)(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1___boxed), 2, 0); return x_1; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { uint8_t x_7; @@ -48641,7 +48342,7 @@ return x_2; else { lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; -x_8 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1; +x_8 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1; lean_inc(x_3); x_9 = l___private_Init_Data_Array_QSort_0__Array_qpartition___rarg(x_1, x_2, x_8, x_3, x_4, lean_box(0), lean_box(0)); x_10 = lean_ctor_get(x_9, 0); @@ -48653,7 +48354,7 @@ x_12 = lean_nat_dec_le(x_4, x_10); if (x_12 == 0) { lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_13 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); +x_13 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(x_1, x_11, x_3, x_10, lean_box(0), lean_box(0)); x_14 = lean_unsigned_to_nat(1u); x_15 = lean_nat_add(x_10, x_14); lean_dec(x_10); @@ -48672,7 +48373,7 @@ return x_11; } } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18(lean_object* x_1, size_t x_2, size_t x_3, lean_object* x_4) { _start: { uint8_t x_5; @@ -48681,7 +48382,7 @@ if (x_5 == 0) { lean_object* x_6; lean_object* x_7; size_t x_8; size_t x_9; x_6 = lean_array_uget(x_1, x_2); -x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16(x_4, x_6); +x_7 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14(x_4, x_6); lean_dec(x_6); x_8 = 1; x_9 = lean_usize_add(x_2, x_8); @@ -48820,7 +48521,7 @@ size_t x_67; lean_object* x_68; lean_object* x_69; x_67 = lean_usize_of_nat(x_17); lean_dec(x_17); x_68 = l___private_Lean_Util_Profiler_0__Lean_Firefox_toJsonCategory____x40_Lean_Util_Profiler___hyg_375____closed__1; -x_69 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20(x_16, x_19, x_67, x_68); +x_69 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18(x_16, x_19, x_67, x_68); lean_dec(x_16); x_55 = x_69; goto block_63; @@ -48830,7 +48531,7 @@ goto block_63; { size_t x_21; lean_object* x_22; uint8_t x_23; x_21 = lean_array_size(x_20); -x_22 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17(x_1, x_2, x_4, x_15, x_21, x_19, x_20, x_10); +x_22 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15(x_1, x_2, x_4, x_15, x_21, x_19, x_20, x_10); x_23 = !lean_is_exclusive(x_22); if (x_23 == 0) { @@ -48855,7 +48556,7 @@ lean_ctor_set(x_34, 5, x_29); lean_ctor_set(x_34, 6, x_30); lean_ctor_set(x_34, 7, x_31); x_35 = lean_array_size(x_24); -x_36 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18(x_35, x_19, x_24); +x_36 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16(x_35, x_19, x_24); x_37 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_37, 0, x_34); lean_ctor_set(x_37, 1, x_30); @@ -48890,7 +48591,7 @@ lean_ctor_set(x_49, 5, x_44); lean_ctor_set(x_49, 6, x_45); lean_ctor_set(x_49, 7, x_46); x_50 = lean_array_size(x_38); -x_51 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18(x_50, x_19, x_38); +x_51 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16(x_50, x_19, x_38); x_52 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_52, 0, x_49); lean_ctor_set(x_52, 1, x_45); @@ -48916,7 +48617,7 @@ if (x_60 == 0) { lean_object* x_61; lean_inc(x_58); -x_61 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(x_56, x_55, x_58, x_58, lean_box(0), lean_box(0)); +x_61 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(x_56, x_55, x_58, x_58, lean_box(0), lean_box(0)); lean_dec(x_58); lean_dec(x_56); x_20 = x_61; @@ -48925,7 +48626,7 @@ goto block_54; else { lean_object* x_62; -x_62 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(x_56, x_55, x_12, x_58, lean_box(0), lean_box(0)); +x_62 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(x_56, x_55, x_12, x_58, lean_box(0), lean_box(0)); lean_dec(x_58); lean_dec(x_56); x_20 = x_62; @@ -48942,48 +48643,28 @@ goto block_54; } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint64_t x_3; lean_object* x_4; -x_3 = lean_unbox_uint64(x_1); -lean_dec(x_1); -x_4 = l_Std_DHashMap_Internal_AssocList_get_x3f___at_Lean_Firefox_Profile_export___spec__2(x_3, x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint64_t x_3; uint8_t x_4; lean_object* x_5; x_3 = lean_unbox_uint64(x_1); lean_dec(x_1); -x_4 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__3(x_3, x_2); +x_4 = l_Std_DHashMap_Internal_AssocList_contains___at_Lean_Firefox_Profile_export___spec__2(x_3, x_2); x_5 = lean_box(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { uint64_t x_4; lean_object* x_5; x_4 = lean_unbox_uint64(x_1); lean_dec(x_1); -x_5 = l_Std_DHashMap_Internal_AssocList_replace___at_Lean_Firefox_Profile_export___spec__8(x_4, x_2, x_3); +x_5 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Lean_Firefox_Profile_export___spec__7___rarg(x_4, x_2, x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9___boxed(lean_object* x_1, lean_object* x_2) { -_start: -{ -uint64_t x_3; lean_object* x_4; -x_3 = lean_unbox_uint64(x_1); -lean_dec(x_1); -x_4 = l_Std_DHashMap_Internal_AssocList_erase___at_Lean_Firefox_Profile_export___spec__9(x_3, x_2); -return x_4; -} -} -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9) { _start: { size_t x_10; size_t x_11; lean_object* x_12; @@ -48991,7 +48672,7 @@ x_10 = lean_unbox_usize(x_7); lean_dec(x_7); x_11 = lean_unbox_usize(x_8); lean_dec(x_8); -x_12 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(x_1, x_2, x_3, x_4, x_5, x_6, x_10, x_11, x_9); +x_12 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__8(x_1, x_2, x_3, x_4, x_5, x_6, x_10, x_11, x_9); lean_dec(x_6); lean_dec(x_5); lean_dec(x_3); @@ -49008,7 +48689,7 @@ lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -49016,21 +48697,21 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__11(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__9(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; -x_6 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_1, x_2, x_3, x_4, x_5); +x_6 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1(x_1, x_2, x_3, x_4, x_5); lean_dec(x_4); lean_dec(x_1); return x_6; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { size_t x_9; size_t x_10; lean_object* x_11; @@ -49038,7 +48719,7 @@ x_9 = lean_unbox_usize(x_5); lean_dec(x_5); x_10 = lean_unbox_usize(x_6); lean_dec(x_6); -x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12(x_1, x_2, x_3, x_4, x_9, x_10, x_7, x_8); +x_11 = l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10(x_1, x_2, x_3, x_4, x_9, x_10, x_7, x_8); lean_dec(x_4); lean_dec(x_3); lean_dec(x_2); @@ -49046,7 +48727,7 @@ lean_dec(x_1); return x_11; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -49054,71 +48735,71 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__13(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__11(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { double x_4; uint8_t x_5; lean_object* x_6; x_4 = lean_unbox_float(x_1); lean_dec(x_1); -x_5 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___lambda__1(x_4, x_2, x_3); +x_5 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___lambda__1(x_4, x_2, x_3); lean_dec(x_3); lean_dec(x_2); x_6 = lean_box(x_5); return x_6; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { double x_8; lean_object* x_9; x_8 = lean_unbox_float(x_1); lean_dec(x_1); -x_9 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__14(x_8, x_2, x_3, x_4, x_5, x_6, x_7); +x_9 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__12(x_8, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_5); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { double x_8; lean_object* x_9; x_8 = lean_unbox_float(x_1); lean_dec(x_1); -x_9 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__15(x_8, x_2, x_3, x_4, x_5, x_6, x_7); +x_9 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__13(x_8, x_2, x_3, x_4, x_5, x_6, x_7); lean_dec(x_5); lean_dec(x_2); return x_9; } } -LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14___boxed(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__16(x_1, x_2); +x_3 = l_Std_DHashMap_Internal_AssocList_foldlM___at_Lean_Firefox_Profile_export___spec__14(x_1, x_2); lean_dec(x_2); return x_3; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { size_t x_7; lean_object* x_8; x_7 = lean_unbox_usize(x_2); lean_dec(x_2); -x_8 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_1, x_7, x_3, x_4, x_5, x_6); +x_8 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___lambda__1(x_1, x_7, x_3, x_4, x_5, x_6); lean_dec(x_5); lean_dec(x_4); lean_dec(x_1); return x_8; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8) { _start: { double x_9; double x_10; size_t x_11; size_t x_12; lean_object* x_13; @@ -49130,12 +48811,12 @@ x_11 = lean_unbox_usize(x_5); lean_dec(x_5); x_12 = lean_unbox_usize(x_6); lean_dec(x_6); -x_13 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17(x_1, x_9, x_3, x_10, x_11, x_12, x_7, x_8); +x_13 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15(x_1, x_9, x_3, x_10, x_11, x_12, x_7, x_8); lean_dec(x_3); return x_13; } } -LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { size_t x_4; size_t x_5; lean_object* x_6; @@ -49143,30 +48824,30 @@ x_4 = lean_unbox_usize(x_1); lean_dec(x_1); x_5 = lean_unbox_usize(x_2); lean_dec(x_2); -x_6 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__18(x_4, x_5, x_3); +x_6 = l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__16(x_4, x_5, x_3); return x_6; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1___boxed(lean_object* x_1, lean_object* x_2) { _start: { uint8_t x_3; lean_object* x_4; -x_3 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___lambda__1(x_1, x_2); +x_3 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___lambda__1(x_1, x_2); x_4 = lean_box(x_3); return x_4; } } -LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +LEAN_EXPORT lean_object* l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { lean_object* x_7; -x_7 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19(x_1, x_2, x_3, x_4, x_5, x_6); +x_7 = l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17(x_1, x_2, x_3, x_4, x_5, x_6); lean_dec(x_4); lean_dec(x_1); return x_7; } } -LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { size_t x_5; size_t x_6; lean_object* x_7; @@ -49174,7 +48855,7 @@ x_5 = lean_unbox_usize(x_2); lean_dec(x_2); x_6 = lean_unbox_usize(x_3); lean_dec(x_3); -x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__20(x_1, x_5, x_6, x_4); +x_7 = l_Array_foldlMUnsafe_fold___at_Lean_Firefox_Profile_export___spec__18(x_1, x_5, x_6, x_4); lean_dec(x_1); return x_7; } @@ -54679,20 +54360,20 @@ l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__4 = _ini lean_mark_persistent(l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__4); l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__5 = _init_l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__5(); lean_mark_persistent(l_Array_groupByKey___at_Lean_Firefox_Profile_export___spec__1___closed__5); -l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___lambda__1___closed__1); -l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1(); -lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__12___boxed__const__1); -l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__1); -l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__2); -l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__3); -l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4(); -lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__17___closed__4); -l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1 = _init_l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1(); -lean_mark_persistent(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__19___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___lambda__1___closed__1); +l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1 = _init_l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1(); +lean_mark_persistent(l_Array_forIn_x27Unsafe_loop___at_Lean_Firefox_Profile_export___spec__10___boxed__const__1); +l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__1); +l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__2); +l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__3); +l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4 = _init_l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4(); +lean_mark_persistent(l_Array_mapMUnsafe_map___at_Lean_Firefox_Profile_export___spec__15___closed__4); +l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1 = _init_l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1(); +lean_mark_persistent(l_Array_qsort_sort___at_Lean_Firefox_Profile_export___spec__17___closed__1); l_Lean_Firefox_Profile_export___closed__1 = _init_l_Lean_Firefox_Profile_export___closed__1(); lean_mark_persistent(l_Lean_Firefox_Profile_export___closed__1); l_Lean_Firefox_Profile_export___closed__2 = _init_l_Lean_Firefox_Profile_export___closed__2(); diff --git a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c index fd8a9afeea8f..e549a78eff73 100644 --- a/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c +++ b/stage0/stdlib/Lean/Widget/InteractiveDiagnostic.c @@ -287,7 +287,6 @@ static lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_fromJsonCommand____x40_Lean_Data_Lsp_Basic___hyg_1498____spec__3(size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableDiagnosticWith_dec____x40_Lean_Widget_InteractiveDiagnostic___hyg_1853____spec__6(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_msgToInteractiveAux_go___spec__5___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -lean_object* lean_string_length(lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_fromJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_769____lambda__2___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Lean_Widget_InteractiveDiagnostic_0__Lean_Widget_toJsonRpcEncodablePacket____x40_Lean_Widget_InteractiveDiagnostic___hyg_210_(lean_object*); static lean_object* l_Array_mapMUnsafe_map___at_Lean_Widget_instRpcEncodableDiagnosticWith_enc____x40_Lean_Widget_InteractiveDiagnostic___hyg_1853____spec__2___closed__4; @@ -24035,7 +24034,7 @@ return x_22; LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractive_fmtToTT___lambda__3(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_59; uint8_t x_60; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; lean_object* x_57; uint8_t x_58; x_6 = lean_ctor_get(x_3, 0); lean_inc(x_6); x_7 = lean_ctor_get(x_3, 1); @@ -24048,666 +24047,663 @@ if (lean_is_exclusive(x_3)) { lean_dec_ref(x_3); x_8 = lean_box(0); } -x_59 = lean_array_get_size(x_1); -x_60 = lean_nat_dec_lt(x_6, x_59); -lean_dec(x_59); -if (x_60 == 0) +x_57 = lean_array_get_size(x_2); +x_58 = lean_nat_dec_lt(x_6, x_57); +lean_dec(x_57); +if (x_58 == 0) { -lean_object* x_61; lean_object* x_62; +lean_object* x_59; lean_object* x_60; lean_dec(x_6); -x_61 = l_Lean_Widget_instInhabitedEmbedFmt; -x_62 = l_outOfBounds___rarg(x_61); -switch (lean_obj_tag(x_62)) { +x_59 = l_Lean_Widget_instInhabitedEmbedFmt; +x_60 = l_outOfBounds___rarg(x_59); +switch (lean_obj_tag(x_60)) { case 0: { -uint8_t x_63; +uint8_t x_61; lean_dec(x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_63 = !lean_is_exclusive(x_62); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_64 = lean_ctor_get(x_62, 0); -x_65 = lean_ctor_get(x_62, 1); -x_66 = l_Lean_Widget_tagCodeInfos_go(x_64, x_65, x_4); -x_67 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_67, 0, x_66); -x_68 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -lean_ctor_set_tag(x_62, 2); -lean_ctor_set(x_62, 1, x_68); -lean_ctor_set(x_62, 0, x_67); -x_69 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_69, 0, x_62); -lean_ctor_set(x_69, 1, x_5); -return x_69; +x_61 = !lean_is_exclusive(x_60); +if (x_61 == 0) +{ +lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; +x_62 = lean_ctor_get(x_60, 0); +x_63 = lean_ctor_get(x_60, 1); +x_64 = l_Lean_Widget_tagCodeInfos_go(x_62, x_63, x_4); +x_65 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_65, 0, x_64); +x_66 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +lean_ctor_set_tag(x_60, 2); +lean_ctor_set(x_60, 1, x_66); +lean_ctor_set(x_60, 0, x_65); +x_67 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_67, 0, x_60); +lean_ctor_set(x_67, 1, x_5); +return x_67; } else { -lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_70 = lean_ctor_get(x_62, 0); -x_71 = lean_ctor_get(x_62, 1); -lean_inc(x_71); -lean_inc(x_70); -lean_dec(x_62); -x_72 = l_Lean_Widget_tagCodeInfos_go(x_70, x_71, x_4); -x_73 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_73, 0, x_72); -x_74 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_75 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_75, 0, x_73); -lean_ctor_set(x_75, 1, x_74); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_5); -return x_76; +lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; +x_68 = lean_ctor_get(x_60, 0); +x_69 = lean_ctor_get(x_60, 1); +lean_inc(x_69); +lean_inc(x_68); +lean_dec(x_60); +x_70 = l_Lean_Widget_tagCodeInfos_go(x_68, x_69, x_4); +x_71 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_71, 0, x_70); +x_72 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_73 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_73, 0, x_71); +lean_ctor_set(x_73, 1, x_72); +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_73); +lean_ctor_set(x_74, 1, x_5); +return x_74; } } case 1: { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; +lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_dec(x_8); lean_dec(x_7); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_77 = lean_ctor_get(x_62, 0); +x_75 = lean_ctor_get(x_60, 0); +lean_inc(x_75); +x_76 = lean_ctor_get(x_60, 1); +lean_inc(x_76); +x_77 = lean_ctor_get(x_60, 2); lean_inc(x_77); -x_78 = lean_ctor_get(x_62, 1); -lean_inc(x_78); -x_79 = lean_ctor_get(x_62, 2); -lean_inc(x_79); -lean_dec(x_62); -x_80 = lean_alloc_closure((void*)(l_Lean_Widget_msgToInteractive_fmtToTT___lambda__2), 6, 1); -lean_closure_set(x_80, 0, x_79); -x_81 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_77, x_78, x_80, x_5); -return x_81; +lean_dec(x_60); +x_78 = lean_alloc_closure((void*)(l_Lean_Widget_msgToInteractive_fmtToTT___lambda__2), 6, 1); +lean_closure_set(x_78, 0, x_77); +x_79 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_75, x_76, x_78, x_5); +return x_79; } case 2: { -uint8_t x_82; +uint8_t x_80; lean_dec(x_8); lean_dec(x_4); -lean_dec(x_2); -x_82 = !lean_is_exclusive(x_62); -if (x_82 == 0) +lean_dec(x_1); +x_80 = !lean_is_exclusive(x_60); +if (x_80 == 0) { -lean_object* x_83; lean_object* x_84; lean_object* x_85; -x_83 = lean_ctor_get(x_62, 0); -x_84 = lean_ctor_get(x_62, 1); -x_85 = l_Lean_Widget_msgToInteractive_fmtToTT(x_1, x_84, x_7, x_5); -if (lean_obj_tag(x_85) == 0) +lean_object* x_81; lean_object* x_82; lean_object* x_83; +x_81 = lean_ctor_get(x_60, 0); +x_82 = lean_ctor_get(x_60, 1); +x_83 = l_Lean_Widget_msgToInteractive_fmtToTT(x_2, x_82, x_7, x_5); +if (lean_obj_tag(x_83) == 0) { -uint8_t x_86; -x_86 = !lean_is_exclusive(x_85); -if (x_86 == 0) +uint8_t x_84; +x_84 = !lean_is_exclusive(x_83); +if (x_84 == 0) { -lean_object* x_87; lean_object* x_88; lean_object* x_89; -x_87 = lean_ctor_get(x_85, 0); -lean_ctor_set(x_62, 1, x_87); -x_88 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_89 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_89, 0, x_62); -lean_ctor_set(x_89, 1, x_88); -lean_ctor_set(x_85, 0, x_89); -return x_85; +lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_85 = lean_ctor_get(x_83, 0); +lean_ctor_set(x_60, 1, x_85); +x_86 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_87 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_87, 0, x_60); +lean_ctor_set(x_87, 1, x_86); +lean_ctor_set(x_83, 0, x_87); +return x_83; } else { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; -x_90 = lean_ctor_get(x_85, 0); -x_91 = lean_ctor_get(x_85, 1); -lean_inc(x_91); -lean_inc(x_90); -lean_dec(x_85); -lean_ctor_set(x_62, 1, x_90); -x_92 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_93 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_93, 0, x_62); -lean_ctor_set(x_93, 1, x_92); -x_94 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_94, 0, x_93); -lean_ctor_set(x_94, 1, x_91); -return x_94; +lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; +x_88 = lean_ctor_get(x_83, 0); +x_89 = lean_ctor_get(x_83, 1); +lean_inc(x_89); +lean_inc(x_88); +lean_dec(x_83); +lean_ctor_set(x_60, 1, x_88); +x_90 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_91 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_91, 0, x_60); +lean_ctor_set(x_91, 1, x_90); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_91); +lean_ctor_set(x_92, 1, x_89); +return x_92; } } else { -uint8_t x_95; -lean_free_object(x_62); -lean_dec(x_83); -x_95 = !lean_is_exclusive(x_85); -if (x_95 == 0) +uint8_t x_93; +lean_free_object(x_60); +lean_dec(x_81); +x_93 = !lean_is_exclusive(x_83); +if (x_93 == 0) { -return x_85; +return x_83; } else { -lean_object* x_96; lean_object* x_97; lean_object* x_98; -x_96 = lean_ctor_get(x_85, 0); -x_97 = lean_ctor_get(x_85, 1); -lean_inc(x_97); -lean_inc(x_96); -lean_dec(x_85); -x_98 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_98, 0, x_96); -lean_ctor_set(x_98, 1, x_97); -return x_98; +lean_object* x_94; lean_object* x_95; lean_object* x_96; +x_94 = lean_ctor_get(x_83, 0); +x_95 = lean_ctor_get(x_83, 1); +lean_inc(x_95); +lean_inc(x_94); +lean_dec(x_83); +x_96 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_96, 0, x_94); +lean_ctor_set(x_96, 1, x_95); +return x_96; } } } else { -lean_object* x_99; lean_object* x_100; lean_object* x_101; -x_99 = lean_ctor_get(x_62, 0); -x_100 = lean_ctor_get(x_62, 1); -lean_inc(x_100); -lean_inc(x_99); -lean_dec(x_62); -x_101 = l_Lean_Widget_msgToInteractive_fmtToTT(x_1, x_100, x_7, x_5); -if (lean_obj_tag(x_101) == 0) +lean_object* x_97; lean_object* x_98; lean_object* x_99; +x_97 = lean_ctor_get(x_60, 0); +x_98 = lean_ctor_get(x_60, 1); +lean_inc(x_98); +lean_inc(x_97); +lean_dec(x_60); +x_99 = l_Lean_Widget_msgToInteractive_fmtToTT(x_2, x_98, x_7, x_5); +if (lean_obj_tag(x_99) == 0) { -lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; -x_102 = lean_ctor_get(x_101, 0); -lean_inc(x_102); -x_103 = lean_ctor_get(x_101, 1); -lean_inc(x_103); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_104 = x_101; -} else { - lean_dec_ref(x_101); - x_104 = lean_box(0); -} +lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; +x_100 = lean_ctor_get(x_99, 0); +lean_inc(x_100); +x_101 = lean_ctor_get(x_99, 1); +lean_inc(x_101); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_102 = x_99; +} else { + lean_dec_ref(x_99); + x_102 = lean_box(0); +} +x_103 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_103, 0, x_97); +lean_ctor_set(x_103, 1, x_100); +x_104 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; x_105 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_105, 0, x_99); -lean_ctor_set(x_105, 1, x_102); -x_106 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_107 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -if (lean_is_scalar(x_104)) { - x_108 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_105, 0, x_103); +lean_ctor_set(x_105, 1, x_104); +if (lean_is_scalar(x_102)) { + x_106 = lean_alloc_ctor(0, 2, 0); } else { - x_108 = x_104; + x_106 = x_102; } -lean_ctor_set(x_108, 0, x_107); -lean_ctor_set(x_108, 1, x_103); -return x_108; +lean_ctor_set(x_106, 0, x_105); +lean_ctor_set(x_106, 1, x_101); +return x_106; } else { -lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -lean_dec(x_99); -x_109 = lean_ctor_get(x_101, 0); -lean_inc(x_109); -x_110 = lean_ctor_get(x_101, 1); -lean_inc(x_110); -if (lean_is_exclusive(x_101)) { - lean_ctor_release(x_101, 0); - lean_ctor_release(x_101, 1); - x_111 = x_101; +lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; +lean_dec(x_97); +x_107 = lean_ctor_get(x_99, 0); +lean_inc(x_107); +x_108 = lean_ctor_get(x_99, 1); +lean_inc(x_108); +if (lean_is_exclusive(x_99)) { + lean_ctor_release(x_99, 0); + lean_ctor_release(x_99, 1); + x_109 = x_99; } else { - lean_dec_ref(x_101); - x_111 = lean_box(0); + lean_dec_ref(x_99); + x_109 = lean_box(0); } -if (lean_is_scalar(x_111)) { - x_112 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_109)) { + x_110 = lean_alloc_ctor(1, 2, 0); } else { - x_112 = x_111; + x_110 = x_109; } -lean_ctor_set(x_112, 0, x_109); -lean_ctor_set(x_112, 1, x_110); -return x_112; +lean_ctor_set(x_110, 0, x_107); +lean_ctor_set(x_110, 1, x_108); +return x_110; } } } case 3: { -lean_object* x_113; lean_object* x_114; uint8_t x_115; lean_object* x_116; -x_113 = lean_ctor_get(x_62, 0); -lean_inc(x_113); -x_114 = lean_ctor_get(x_62, 1); +lean_object* x_111; lean_object* x_112; uint8_t x_113; lean_object* x_114; +lean_dec(x_4); +x_111 = lean_ctor_get(x_60, 0); +lean_inc(x_111); +x_112 = lean_ctor_get(x_60, 1); +lean_inc(x_112); +x_113 = lean_ctor_get_uint8(x_60, sizeof(void*)*3); +x_114 = lean_ctor_get(x_60, 2); lean_inc(x_114); -x_115 = lean_ctor_get_uint8(x_62, sizeof(void*)*3); -x_116 = lean_ctor_get(x_62, 2); -lean_inc(x_116); -lean_dec(x_62); -x_9 = x_113; -x_10 = x_114; -x_11 = x_115; -x_12 = x_116; -goto block_58; +lean_dec(x_60); +x_9 = x_111; +x_10 = x_112; +x_11 = x_113; +x_12 = x_114; +goto block_56; } default: { -lean_object* x_117; lean_object* x_118; lean_object* x_119; +lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_dec(x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_117 = l_Lean_Widget_TaggedText_stripTags___rarg(x_4); -x_118 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_118, 0, x_117); -x_119 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_119, 0, x_118); -lean_ctor_set(x_119, 1, x_5); -return x_119; +x_115 = l_Lean_Widget_TaggedText_stripTags___rarg(x_4); +x_116 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_116, 0, x_115); +x_117 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_117, 0, x_116); +lean_ctor_set(x_117, 1, x_5); +return x_117; } } } else { -lean_object* x_120; -x_120 = lean_array_fget(x_1, x_6); +lean_object* x_118; +x_118 = lean_array_fget(x_2, x_6); lean_dec(x_6); -switch (lean_obj_tag(x_120)) { +switch (lean_obj_tag(x_118)) { case 0: { -uint8_t x_121; +uint8_t x_119; lean_dec(x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_121 = !lean_is_exclusive(x_120); -if (x_121 == 0) +x_119 = !lean_is_exclusive(x_118); +if (x_119 == 0) { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_122 = lean_ctor_get(x_120, 0); -x_123 = lean_ctor_get(x_120, 1); -x_124 = l_Lean_Widget_tagCodeInfos_go(x_122, x_123, x_4); -x_125 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_125, 0, x_124); -x_126 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -lean_ctor_set_tag(x_120, 2); -lean_ctor_set(x_120, 1, x_126); -lean_ctor_set(x_120, 0, x_125); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_120); -lean_ctor_set(x_127, 1, x_5); -return x_127; +lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; +x_120 = lean_ctor_get(x_118, 0); +x_121 = lean_ctor_get(x_118, 1); +x_122 = l_Lean_Widget_tagCodeInfos_go(x_120, x_121, x_4); +x_123 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_123, 0, x_122); +x_124 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +lean_ctor_set_tag(x_118, 2); +lean_ctor_set(x_118, 1, x_124); +lean_ctor_set(x_118, 0, x_123); +x_125 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_125, 0, x_118); +lean_ctor_set(x_125, 1, x_5); +return x_125; } else { -lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; -x_128 = lean_ctor_get(x_120, 0); -x_129 = lean_ctor_get(x_120, 1); -lean_inc(x_129); -lean_inc(x_128); -lean_dec(x_120); -x_130 = l_Lean_Widget_tagCodeInfos_go(x_128, x_129, x_4); -x_131 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_131, 0, x_130); -x_132 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_133 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_133, 0, x_131); -lean_ctor_set(x_133, 1, x_132); -x_134 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_134, 0, x_133); -lean_ctor_set(x_134, 1, x_5); -return x_134; +lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; +x_126 = lean_ctor_get(x_118, 0); +x_127 = lean_ctor_get(x_118, 1); +lean_inc(x_127); +lean_inc(x_126); +lean_dec(x_118); +x_128 = l_Lean_Widget_tagCodeInfos_go(x_126, x_127, x_4); +x_129 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_129, 0, x_128); +x_130 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_131 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_131, 0, x_129); +lean_ctor_set(x_131, 1, x_130); +x_132 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_132, 0, x_131); +lean_ctor_set(x_132, 1, x_5); +return x_132; } } case 1: { -lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; +lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_dec(x_8); lean_dec(x_7); lean_dec(x_4); lean_dec(x_2); lean_dec(x_1); -x_135 = lean_ctor_get(x_120, 0); +x_133 = lean_ctor_get(x_118, 0); +lean_inc(x_133); +x_134 = lean_ctor_get(x_118, 1); +lean_inc(x_134); +x_135 = lean_ctor_get(x_118, 2); lean_inc(x_135); -x_136 = lean_ctor_get(x_120, 1); -lean_inc(x_136); -x_137 = lean_ctor_get(x_120, 2); -lean_inc(x_137); -lean_dec(x_120); -x_138 = lean_alloc_closure((void*)(l_Lean_Widget_msgToInteractive_fmtToTT___lambda__2), 6, 1); -lean_closure_set(x_138, 0, x_137); -x_139 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_135, x_136, x_138, x_5); -return x_139; +lean_dec(x_118); +x_136 = lean_alloc_closure((void*)(l_Lean_Widget_msgToInteractive_fmtToTT___lambda__2), 6, 1); +lean_closure_set(x_136, 0, x_135); +x_137 = l_Lean_Elab_ContextInfo_runMetaM___rarg(x_133, x_134, x_136, x_5); +return x_137; } case 2: { -uint8_t x_140; +uint8_t x_138; lean_dec(x_8); lean_dec(x_4); -lean_dec(x_2); -x_140 = !lean_is_exclusive(x_120); -if (x_140 == 0) -{ -lean_object* x_141; lean_object* x_142; lean_object* x_143; -x_141 = lean_ctor_get(x_120, 0); -x_142 = lean_ctor_get(x_120, 1); -x_143 = l_Lean_Widget_msgToInteractive_fmtToTT(x_1, x_142, x_7, x_5); -if (lean_obj_tag(x_143) == 0) -{ -uint8_t x_144; -x_144 = !lean_is_exclusive(x_143); -if (x_144 == 0) -{ -lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_145 = lean_ctor_get(x_143, 0); -lean_ctor_set(x_120, 1, x_145); -x_146 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_147 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_147, 0, x_120); -lean_ctor_set(x_147, 1, x_146); -lean_ctor_set(x_143, 0, x_147); -return x_143; +lean_dec(x_1); +x_138 = !lean_is_exclusive(x_118); +if (x_138 == 0) +{ +lean_object* x_139; lean_object* x_140; lean_object* x_141; +x_139 = lean_ctor_get(x_118, 0); +x_140 = lean_ctor_get(x_118, 1); +x_141 = l_Lean_Widget_msgToInteractive_fmtToTT(x_2, x_140, x_7, x_5); +if (lean_obj_tag(x_141) == 0) +{ +uint8_t x_142; +x_142 = !lean_is_exclusive(x_141); +if (x_142 == 0) +{ +lean_object* x_143; lean_object* x_144; lean_object* x_145; +x_143 = lean_ctor_get(x_141, 0); +lean_ctor_set(x_118, 1, x_143); +x_144 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_145 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_145, 0, x_118); +lean_ctor_set(x_145, 1, x_144); +lean_ctor_set(x_141, 0, x_145); +return x_141; } else { -lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; -x_148 = lean_ctor_get(x_143, 0); -x_149 = lean_ctor_get(x_143, 1); -lean_inc(x_149); -lean_inc(x_148); -lean_dec(x_143); -lean_ctor_set(x_120, 1, x_148); -x_150 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_151 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_151, 0, x_120); -lean_ctor_set(x_151, 1, x_150); -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_151); -lean_ctor_set(x_152, 1, x_149); -return x_152; +lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; +x_146 = lean_ctor_get(x_141, 0); +x_147 = lean_ctor_get(x_141, 1); +lean_inc(x_147); +lean_inc(x_146); +lean_dec(x_141); +lean_ctor_set(x_118, 1, x_146); +x_148 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; +x_149 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_149, 0, x_118); +lean_ctor_set(x_149, 1, x_148); +x_150 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_150, 0, x_149); +lean_ctor_set(x_150, 1, x_147); +return x_150; } } else { -uint8_t x_153; -lean_free_object(x_120); -lean_dec(x_141); -x_153 = !lean_is_exclusive(x_143); -if (x_153 == 0) +uint8_t x_151; +lean_free_object(x_118); +lean_dec(x_139); +x_151 = !lean_is_exclusive(x_141); +if (x_151 == 0) { -return x_143; +return x_141; } else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; -x_154 = lean_ctor_get(x_143, 0); -x_155 = lean_ctor_get(x_143, 1); -lean_inc(x_155); -lean_inc(x_154); -lean_dec(x_143); -x_156 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_156, 0, x_154); -lean_ctor_set(x_156, 1, x_155); -return x_156; +lean_object* x_152; lean_object* x_153; lean_object* x_154; +x_152 = lean_ctor_get(x_141, 0); +x_153 = lean_ctor_get(x_141, 1); +lean_inc(x_153); +lean_inc(x_152); +lean_dec(x_141); +x_154 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_154, 0, x_152); +lean_ctor_set(x_154, 1, x_153); +return x_154; } } } else { -lean_object* x_157; lean_object* x_158; lean_object* x_159; -x_157 = lean_ctor_get(x_120, 0); -x_158 = lean_ctor_get(x_120, 1); -lean_inc(x_158); -lean_inc(x_157); -lean_dec(x_120); -x_159 = l_Lean_Widget_msgToInteractive_fmtToTT(x_1, x_158, x_7, x_5); -if (lean_obj_tag(x_159) == 0) +lean_object* x_155; lean_object* x_156; lean_object* x_157; +x_155 = lean_ctor_get(x_118, 0); +x_156 = lean_ctor_get(x_118, 1); +lean_inc(x_156); +lean_inc(x_155); +lean_dec(x_118); +x_157 = l_Lean_Widget_msgToInteractive_fmtToTT(x_2, x_156, x_7, x_5); +if (lean_obj_tag(x_157) == 0) { -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; -x_160 = lean_ctor_get(x_159, 0); -lean_inc(x_160); -x_161 = lean_ctor_get(x_159, 1); -lean_inc(x_161); -if (lean_is_exclusive(x_159)) { - lean_ctor_release(x_159, 0); - lean_ctor_release(x_159, 1); - x_162 = x_159; -} else { - lean_dec_ref(x_159); - x_162 = lean_box(0); -} +lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; +x_158 = lean_ctor_get(x_157, 0); +lean_inc(x_158); +x_159 = lean_ctor_get(x_157, 1); +lean_inc(x_159); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_160 = x_157; +} else { + lean_dec_ref(x_157); + x_160 = lean_box(0); +} +x_161 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_161, 0, x_155); +lean_ctor_set(x_161, 1, x_158); +x_162 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; x_163 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_163, 0, x_157); -lean_ctor_set(x_163, 1, x_160); -x_164 = l_Lean_Widget_instInhabitedMsgEmbed___closed__2; -x_165 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_165, 0, x_163); -lean_ctor_set(x_165, 1, x_164); -if (lean_is_scalar(x_162)) { - x_166 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_163, 0, x_161); +lean_ctor_set(x_163, 1, x_162); +if (lean_is_scalar(x_160)) { + x_164 = lean_alloc_ctor(0, 2, 0); } else { - x_166 = x_162; + x_164 = x_160; } -lean_ctor_set(x_166, 0, x_165); -lean_ctor_set(x_166, 1, x_161); -return x_166; +lean_ctor_set(x_164, 0, x_163); +lean_ctor_set(x_164, 1, x_159); +return x_164; } else { -lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; -lean_dec(x_157); -x_167 = lean_ctor_get(x_159, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_159, 1); -lean_inc(x_168); -if (lean_is_exclusive(x_159)) { - lean_ctor_release(x_159, 0); - lean_ctor_release(x_159, 1); - x_169 = x_159; +lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; +lean_dec(x_155); +x_165 = lean_ctor_get(x_157, 0); +lean_inc(x_165); +x_166 = lean_ctor_get(x_157, 1); +lean_inc(x_166); +if (lean_is_exclusive(x_157)) { + lean_ctor_release(x_157, 0); + lean_ctor_release(x_157, 1); + x_167 = x_157; } else { - lean_dec_ref(x_159); - x_169 = lean_box(0); + lean_dec_ref(x_157); + x_167 = lean_box(0); } -if (lean_is_scalar(x_169)) { - x_170 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_167)) { + x_168 = lean_alloc_ctor(1, 2, 0); } else { - x_170 = x_169; + x_168 = x_167; } -lean_ctor_set(x_170, 0, x_167); -lean_ctor_set(x_170, 1, x_168); -return x_170; +lean_ctor_set(x_168, 0, x_165); +lean_ctor_set(x_168, 1, x_166); +return x_168; } } } case 3: { -lean_object* x_171; lean_object* x_172; uint8_t x_173; lean_object* x_174; -x_171 = lean_ctor_get(x_120, 0); -lean_inc(x_171); -x_172 = lean_ctor_get(x_120, 1); +lean_object* x_169; lean_object* x_170; uint8_t x_171; lean_object* x_172; +lean_dec(x_4); +x_169 = lean_ctor_get(x_118, 0); +lean_inc(x_169); +x_170 = lean_ctor_get(x_118, 1); +lean_inc(x_170); +x_171 = lean_ctor_get_uint8(x_118, sizeof(void*)*3); +x_172 = lean_ctor_get(x_118, 2); lean_inc(x_172); -x_173 = lean_ctor_get_uint8(x_120, sizeof(void*)*3); -x_174 = lean_ctor_get(x_120, 2); -lean_inc(x_174); -lean_dec(x_120); -x_9 = x_171; -x_10 = x_172; -x_11 = x_173; -x_12 = x_174; -goto block_58; +lean_dec(x_118); +x_9 = x_169; +x_10 = x_170; +x_11 = x_171; +x_12 = x_172; +goto block_56; } default: { -lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_dec(x_8); lean_dec(x_7); lean_dec(x_2); lean_dec(x_1); -x_175 = l_Lean_Widget_TaggedText_stripTags___rarg(x_4); -x_176 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_176, 0, x_175); -x_177 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_177, 0, x_176); -lean_ctor_set(x_177, 1, x_5); -return x_177; +x_173 = l_Lean_Widget_TaggedText_stripTags___rarg(x_4); +x_174 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_174, 0, x_173); +x_175 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_175, 0, x_174); +lean_ctor_set(x_175, 1, x_5); +return x_175; } } } -block_58: +block_56: { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_13 = l_Lean_Widget_TaggedText_stripTags___rarg(x_4); -x_14 = lean_string_length(x_13); -lean_dec(x_13); -x_15 = lean_nat_add(x_7, x_14); -lean_dec(x_14); +lean_object* x_13; +x_13 = lean_nat_add(x_1, x_7); lean_dec(x_7); -x_16 = lean_unsigned_to_nat(2u); -x_17 = lean_nat_sub(x_15, x_16); -lean_dec(x_15); if (lean_obj_tag(x_12) == 0) { -uint8_t x_18; +uint8_t x_14; lean_dec(x_8); -x_18 = !lean_is_exclusive(x_12); -if (x_18 == 0) +x_14 = !lean_is_exclusive(x_12); +if (x_14 == 0) { -lean_object* x_19; size_t x_20; size_t x_21; lean_object* x_22; -x_19 = lean_ctor_get(x_12, 0); -x_20 = lean_array_size(x_19); -x_21 = 0; -lean_inc(x_1); -x_22 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__1(x_1, x_17, x_20, x_21, x_19, x_5); -if (lean_obj_tag(x_22) == 0) +lean_object* x_15; size_t x_16; size_t x_17; lean_object* x_18; +x_15 = lean_ctor_get(x_12, 0); +x_16 = lean_array_size(x_15); +x_17 = 0; +lean_inc(x_2); +x_18 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__1(x_2, x_13, x_16, x_17, x_15, x_5); +if (lean_obj_tag(x_18) == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; -x_23 = lean_ctor_get(x_22, 0); -lean_inc(x_23); -x_24 = lean_ctor_get(x_22, 1); -lean_inc(x_24); -lean_dec(x_22); -lean_ctor_set(x_12, 0, x_23); -x_25 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_1, x_10, x_17, x_2, x_9, x_11, x_12, x_24); -return x_25; +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_18, 0); +lean_inc(x_19); +x_20 = lean_ctor_get(x_18, 1); +lean_inc(x_20); +lean_dec(x_18); +lean_ctor_set(x_12, 0, x_19); +x_21 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_2, x_10, x_13, x_1, x_9, x_11, x_12, x_20); +return x_21; } else { -uint8_t x_26; +uint8_t x_22; lean_free_object(x_12); -lean_dec(x_17); +lean_dec(x_13); lean_dec(x_10); lean_dec(x_9); lean_dec(x_2); lean_dec(x_1); -x_26 = !lean_is_exclusive(x_22); -if (x_26 == 0) +x_22 = !lean_is_exclusive(x_18); +if (x_22 == 0) { -return x_22; +return x_18; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; -x_27 = lean_ctor_get(x_22, 0); -x_28 = lean_ctor_get(x_22, 1); -lean_inc(x_28); -lean_inc(x_27); -lean_dec(x_22); -x_29 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_29, 0, x_27); -lean_ctor_set(x_29, 1, x_28); -return x_29; +lean_object* x_23; lean_object* x_24; lean_object* x_25; +x_23 = lean_ctor_get(x_18, 0); +x_24 = lean_ctor_get(x_18, 1); +lean_inc(x_24); +lean_inc(x_23); +lean_dec(x_18); +x_25 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_25, 0, x_23); +lean_ctor_set(x_25, 1, x_24); +return x_25; } } } else { -lean_object* x_30; size_t x_31; size_t x_32; lean_object* x_33; -x_30 = lean_ctor_get(x_12, 0); -lean_inc(x_30); +lean_object* x_26; size_t x_27; size_t x_28; lean_object* x_29; +x_26 = lean_ctor_get(x_12, 0); +lean_inc(x_26); lean_dec(x_12); -x_31 = lean_array_size(x_30); -x_32 = 0; -lean_inc(x_1); -x_33 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__1(x_1, x_17, x_31, x_32, x_30, x_5); -if (lean_obj_tag(x_33) == 0) +x_27 = lean_array_size(x_26); +x_28 = 0; +lean_inc(x_2); +x_29 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__1(x_2, x_13, x_27, x_28, x_26, x_5); +if (lean_obj_tag(x_29) == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; -x_34 = lean_ctor_get(x_33, 0); -lean_inc(x_34); -x_35 = lean_ctor_get(x_33, 1); -lean_inc(x_35); -lean_dec(x_33); -x_36 = lean_alloc_ctor(0, 1, 0); -lean_ctor_set(x_36, 0, x_34); -x_37 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_1, x_10, x_17, x_2, x_9, x_11, x_36, x_35); -return x_37; +lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_30 = lean_ctor_get(x_29, 0); +lean_inc(x_30); +x_31 = lean_ctor_get(x_29, 1); +lean_inc(x_31); +lean_dec(x_29); +x_32 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_32, 0, x_30); +x_33 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_2, x_10, x_13, x_1, x_9, x_11, x_32, x_31); +return x_33; } else { -lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; -lean_dec(x_17); +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +lean_dec(x_13); lean_dec(x_10); lean_dec(x_9); lean_dec(x_2); lean_dec(x_1); -x_38 = lean_ctor_get(x_33, 0); -lean_inc(x_38); -x_39 = lean_ctor_get(x_33, 1); -lean_inc(x_39); -if (lean_is_exclusive(x_33)) { - lean_ctor_release(x_33, 0); - lean_ctor_release(x_33, 1); - x_40 = x_33; +x_34 = lean_ctor_get(x_29, 0); +lean_inc(x_34); +x_35 = lean_ctor_get(x_29, 1); +lean_inc(x_35); +if (lean_is_exclusive(x_29)) { + lean_ctor_release(x_29, 0); + lean_ctor_release(x_29, 1); + x_36 = x_29; } else { - lean_dec_ref(x_33); - x_40 = lean_box(0); + lean_dec_ref(x_29); + x_36 = lean_box(0); } -if (lean_is_scalar(x_40)) { - x_41 = lean_alloc_ctor(1, 2, 0); +if (lean_is_scalar(x_36)) { + x_37 = lean_alloc_ctor(1, 2, 0); } else { - x_41 = x_40; + x_37 = x_36; } -lean_ctor_set(x_41, 0, x_38); -lean_ctor_set(x_41, 1, x_39); -return x_41; +lean_ctor_set(x_37, 0, x_34); +lean_ctor_set(x_37, 1, x_35); +return x_37; } } } else { -uint8_t x_42; -x_42 = !lean_is_exclusive(x_12); -if (x_42 == 0) +uint8_t x_38; +x_38 = !lean_is_exclusive(x_12); +if (x_38 == 0) { -lean_object* x_43; lean_object* x_44; size_t x_45; size_t x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_43 = lean_ctor_get(x_12, 0); -x_44 = lean_nat_add(x_17, x_16); -x_45 = lean_array_size(x_43); -x_46 = 0; -x_47 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__2(x_45, x_46, x_43); +lean_object* x_39; lean_object* x_40; lean_object* x_41; size_t x_42; size_t x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; +x_39 = lean_ctor_get(x_12, 0); +x_40 = lean_unsigned_to_nat(2u); +x_41 = lean_nat_add(x_13, x_40); +x_42 = lean_array_size(x_39); +x_43 = 0; +x_44 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__2(x_42, x_43, x_39); if (lean_is_scalar(x_8)) { - x_48 = lean_alloc_ctor(0, 2, 0); + x_45 = lean_alloc_ctor(0, 2, 0); } else { - x_48 = x_8; + x_45 = x_8; } -lean_ctor_set(x_48, 0, x_44); -lean_ctor_set(x_48, 1, x_47); -lean_ctor_set(x_12, 0, x_48); -x_49 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_1, x_10, x_17, x_2, x_9, x_11, x_12, x_5); -return x_49; +lean_ctor_set(x_45, 0, x_41); +lean_ctor_set(x_45, 1, x_44); +lean_ctor_set(x_12, 0, x_45); +x_46 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_2, x_10, x_13, x_1, x_9, x_11, x_12, x_5); +return x_46; } else { -lean_object* x_50; lean_object* x_51; size_t x_52; size_t x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_50 = lean_ctor_get(x_12, 0); -lean_inc(x_50); +lean_object* x_47; lean_object* x_48; lean_object* x_49; size_t x_50; size_t x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; +x_47 = lean_ctor_get(x_12, 0); +lean_inc(x_47); lean_dec(x_12); -x_51 = lean_nat_add(x_17, x_16); -x_52 = lean_array_size(x_50); -x_53 = 0; -x_54 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__2(x_52, x_53, x_50); +x_48 = lean_unsigned_to_nat(2u); +x_49 = lean_nat_add(x_13, x_48); +x_50 = lean_array_size(x_47); +x_51 = 0; +x_52 = l_Array_mapMUnsafe_map___at_Lean_Widget_msgToInteractive_fmtToTT___spec__2(x_50, x_51, x_47); if (lean_is_scalar(x_8)) { - x_55 = lean_alloc_ctor(0, 2, 0); + x_53 = lean_alloc_ctor(0, 2, 0); } else { - x_55 = x_8; + x_53 = x_8; } -lean_ctor_set(x_55, 0, x_51); -lean_ctor_set(x_55, 1, x_54); -x_56 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_56, 0, x_55); -x_57 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_1, x_10, x_17, x_2, x_9, x_11, x_56, x_5); -return x_57; +lean_ctor_set(x_53, 0, x_49); +lean_ctor_set(x_53, 1, x_52); +x_54 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_54, 0, x_53); +x_55 = l_Lean_Widget_msgToInteractive_fmtToTT___lambda__1(x_2, x_10, x_13, x_1, x_9, x_11, x_54, x_5); +return x_55; } } } @@ -24719,8 +24715,8 @@ LEAN_EXPORT lean_object* l_Lean_Widget_msgToInteractive_fmtToTT(lean_object* x_1 lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_inc(x_3); x_5 = lean_alloc_closure((void*)(l_Lean_Widget_msgToInteractive_fmtToTT___lambda__3), 5, 2); -lean_closure_set(x_5, 0, x_1); -lean_closure_set(x_5, 1, x_3); +lean_closure_set(x_5, 0, x_3); +lean_closure_set(x_5, 1, x_1); x_6 = l_Std_Format_defWidth; x_7 = l_Lean_Widget_TaggedText_prettyTagged(x_2, x_3, x_6); x_8 = l_Lean_Widget_TaggedText_rewriteM___at_Lean_Widget_msgToInteractive_fmtToTT___spec__3(x_5, x_7, x_4); diff --git a/stage0/stdlib/Lean/Widget/UserWidget.c b/stage0/stdlib/Lean/Widget/UserWidget.c index e542b76a81c0..72a1cba1d5eb 100644 --- a/stage0/stdlib/Lean/Widget/UserWidget.c +++ b/stage0/stdlib/Lean/Widget/UserWidget.c @@ -67,7 +67,6 @@ static lean_object* l___private_Lean_Widget_UserWidget_0__Lean_Widget_fromJsonRp lean_object* l___private_Lean_Data_Lsp_Basic_0__Lean_Lsp_toJsonRange____x40_Lean_Data_Lsp_Basic___hyg_557_(lean_object*); LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*, lean_object*, lean_object*); lean_object* l_Lean_ConstantInfo_type(lean_object*); -lean_object* l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(lean_object*, lean_object*); static lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; static lean_object* l_Lean_Widget_showPanelWidgetsCmd___closed__3; extern lean_object* l_Lean_maxRecDepthErrorMessage; @@ -459,6 +458,7 @@ static lean_object* l_Lean_ScopedEnvExtension_add___at_Lean_Widget_elabShowPanel LEAN_EXPORT lean_object* l___private_Lean_Widget_UserWidget_0__Lean_Widget_evalModuleUnsafe(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Lean_Widget_showPanelWidgetsCmd___closed__2; lean_object* l_MonadExcept_ofExcept___at_Lean_Widget_instRpcEncodableInteractiveHypothesisBundle_dec____x40_Lean_Widget_InteractiveGoal___hyg_5____spec__1(lean_object*, lean_object*); +lean_object* l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Lean_RBNode_find___at_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____spec__3___boxed(lean_object*, lean_object*); static lean_object* l_Lean_Widget_widgetInstanceSpec___closed__16; static lean_object* l_Lean_Widget_elabWidgetInstanceSpecAux___closed__4; @@ -6370,7 +6370,6 @@ if (lean_obj_tag(x_17) == 0) lean_object* x_18; lean_object* x_19; x_18 = lean_box(0); x_19 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__1(x_1, x_2, x_3, x_18, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_10); return x_19; } else @@ -6404,7 +6403,6 @@ x_31 = lean_ctor_get(x_29, 1); lean_inc(x_31); lean_dec(x_29); x_32 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__1(x_1, x_2, x_3, x_30, x_8, x_9, x_10, x_11, x_31); -lean_dec(x_10); lean_dec(x_30); return x_32; } @@ -6432,7 +6430,6 @@ x_42 = lean_ctor_get(x_40, 1); lean_inc(x_42); lean_dec(x_40); x_43 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__1(x_1, x_2, x_3, x_41, x_8, x_9, x_10, x_11, x_42); -lean_dec(x_10); lean_dec(x_41); return x_43; } @@ -6518,7 +6515,6 @@ lean_inc(x_23); lean_dec(x_21); x_24 = lean_box(0); x_25 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__2(x_2, x_1, x_10, x_3, x_23, x_18, x_24, x_5, x_6, x_7, x_8, x_22); -lean_dec(x_8); lean_dec(x_6); lean_dec(x_5); lean_dec(x_23); @@ -8055,8 +8051,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hy { lean_object* x_10; x_10 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__1(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9); -lean_dec(x_8); -lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); @@ -8068,7 +8062,6 @@ LEAN_EXPORT lean_object* l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hy { lean_object* x_13; x_13 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__2(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_8, x_9, x_10, x_11, x_12); -lean_dec(x_11); lean_dec(x_9); lean_dec(x_8); lean_dec(x_7); @@ -8201,7 +8194,7 @@ x_15 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_15, 0, x_8); lean_ctor_set(x_15, 1, x_14); x_16 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_17 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_15, x_16); +x_17 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_15, x_16); x_18 = l_Lean_Json_mkObj(x_17); return x_18; } @@ -8536,7 +8529,7 @@ x_7 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_7, 0, x_6); lean_ctor_set(x_7, 1, x_5); x_8 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_9 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_7, x_8); +x_9 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_7, x_8); x_10 = l_Lean_Json_mkObj(x_9); return x_10; } @@ -18894,7 +18887,7 @@ x_14 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_14, 0, x_8); lean_ctor_set(x_14, 1, x_13); x_15 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_16 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_14, x_15); +x_16 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_14, x_15); x_17 = l_Lean_Json_mkObj(x_16); return x_17; } @@ -18932,7 +18925,7 @@ x_30 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_30, 0, x_24); lean_ctor_set(x_30, 1, x_29); x_31 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_32 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_30, x_31); +x_32 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_30, x_31); x_33 = l_Lean_Json_mkObj(x_32); return x_33; } @@ -19956,7 +19949,7 @@ x_25 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_25, 0, x_10); lean_ctor_set(x_25, 1, x_24); x_26 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_27 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_25, x_26); +x_27 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_25, x_26); x_28 = l_Lean_Json_mkObj(x_27); return x_28; } @@ -21627,7 +21620,7 @@ x_6 = lean_alloc_ctor(1, 2, 0); lean_ctor_set(x_6, 0, x_5); lean_ctor_set(x_6, 1, x_4); x_7 = l_Lean_Widget_initFn____x40_Lean_Widget_UserWidget___hyg_240____lambda__4___closed__9; -x_8 = l_List_flatMapTR_go___at___private_Lean_Data_Lsp_CancelParams_0__Lean_Lsp_toJsonCancelParams____x40_Lean_Data_Lsp_CancelParams___hyg_86____spec__1(x_6, x_7); +x_8 = l_List_flatMapTR_go___at___private_Lean_Util_Paths_0__Lean_toJsonLeanPaths____x40_Lean_Util_Paths___hyg_40____spec__2(x_6, x_7); x_9 = l_Lean_Json_mkObj(x_8); return x_9; } diff --git a/stage0/stdlib/Std/Data/DHashMap/Basic.c b/stage0/stdlib/Std/Data/DHashMap/Basic.c index 7748588e1b1c..87194600669d 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Basic.c +++ b/stage0/stdlib/Std/Data/DHashMap/Basic.c @@ -18,6 +18,7 @@ LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_DHashMap_forIn___ LEAN_EXPORT lean_object* l_Std_DHashMap_keys___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Std_DHashMap_instRepr___spec__9___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_toArray___rarg___boxed(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_DHashMap_instRepr___spec__15___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_DHashMap_Const_toList___spec__3___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Const_toArray___spec__1___rarg___boxed(lean_object*, lean_object*); @@ -65,6 +66,7 @@ uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_List_foldl___at_Std_DHashMap_instRepr___spec__5___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_ofList(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_filter___spec__2(lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_instInhabited___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static size_t l_Std_DHashMap_instSingletonSigma___rarg___closed__3; LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_fold___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -86,12 +88,14 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_union___spe LEAN_EXPORT lean_object* l_Std_DHashMap_empty___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_DHashMap_values___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_getKey_x21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_alter(lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_filter___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Std_DHashMap_instRepr___spec__19(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_length___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Format_joinSep___at_Std_DHashMap_instRepr___spec__13(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_empty(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_instEmptyCollection___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_instSingletonSigma___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_valuesArray(lean_object*, lean_object*, lean_object*, lean_object*); @@ -179,6 +183,7 @@ uint8_t l_Std_DHashMap_Internal_AssocList_contains___rarg(lean_object*, lean_obj lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_toArray___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_forM___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Const_get_x3f(lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_replace___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -266,6 +271,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_instForMSig LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_DHashMap_Const_unitOfArray___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldrM___at_Std_DHashMap_keys___spec__1___rarg___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_repr___at_Std_DHashMap_instRepr___spec__16___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_modify(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Const_insertMany___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Const_toArray___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_foldM___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -287,6 +293,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_containsThenInsertIfNew___rarg(lean_obje LEAN_EXPORT lean_object* l_Std_DHashMap_Const_getThenInsertIfNew_x3f(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_numBuckets___rarg(lean_object*); lean_object* lean_string_length(lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_repr___at_Std_DHashMap_instRepr___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldrM___at_Std_DHashMap_values___spec__1___rarg___boxed(lean_object*, lean_object*); @@ -368,6 +375,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_DHashMap_instRepr___ static lean_object* l_List_repr___at_Std_DHashMap_instRepr___spec__2___rarg___closed__8; LEAN_EXPORT lean_object* l_Std_DHashMap_Const_toList___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Const_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_keysArray___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); static lean_object* l_List_repr___at_Std_DHashMap_instRepr___spec__2___rarg___closed__7; @@ -6770,13 +6778,12 @@ return x_5; LEAN_EXPORT lean_object* l_Std_DHashMap_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; x_7 = lean_ctor_get(x_4, 0); lean_inc(x_7); x_8 = lean_ctor_get(x_4, 1); lean_inc(x_8); x_9 = lean_array_get_size(x_8); -lean_inc(x_2); lean_inc(x_5); x_10 = lean_apply_1(x_2, x_5); x_11 = lean_unbox_uint64(x_10); @@ -6797,15 +6804,14 @@ x_23 = lean_array_uget(x_8, x_22); lean_inc(x_23); lean_inc(x_5); lean_inc(x_1); -x_24 = l_Std_DHashMap_Internal_AssocList_getCast_x3f___rarg(x_1, lean_box(0), x_5, x_23); -if (lean_obj_tag(x_24) == 0) +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) { lean_dec(x_23); lean_dec(x_8); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); -lean_dec(x_2); lean_dec(x_1); return x_4; } @@ -6815,331 +6821,128 @@ uint8_t x_25; x_25 = !lean_is_exclusive(x_4); if (x_25 == 0) { -lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_82; +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; x_26 = lean_ctor_get(x_4, 1); lean_dec(x_26); x_27 = lean_ctor_get(x_4, 0); lean_dec(x_27); -x_28 = lean_ctor_get(x_24, 0); -lean_inc(x_28); -lean_dec(x_24); -x_29 = lean_apply_1(x_6, x_28); -lean_inc(x_23); -lean_inc(x_5); -lean_inc(x_1); -x_82 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_82 == 0) -{ -lean_dec(x_23); -x_30 = x_4; -goto block_81; -} -else -{ -lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_83 = lean_box(0); -x_84 = lean_array_uset(x_8, x_22, x_83); -x_85 = lean_unsigned_to_nat(1u); -x_86 = lean_nat_sub(x_7, x_85); -lean_dec(x_7); -lean_inc(x_5); -lean_inc(x_1); -x_87 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_88 = lean_array_uset(x_84, x_22, x_87); -lean_ctor_set(x_4, 1, x_88); -lean_ctor_set(x_4, 0, x_86); -x_30 = x_4; -goto block_81; -} -block_81: -{ -uint8_t x_31; -x_31 = !lean_is_exclusive(x_30); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; size_t x_35; size_t x_36; size_t x_37; lean_object* x_38; uint8_t x_39; -x_32 = lean_ctor_get(x_30, 0); -x_33 = lean_ctor_get(x_30, 1); -x_34 = lean_array_get_size(x_33); -x_35 = lean_usize_of_nat(x_34); -lean_dec(x_34); -x_36 = lean_usize_sub(x_35, x_20); -x_37 = lean_usize_land(x_18, x_36); -x_38 = lean_array_uget(x_33, x_37); -lean_inc(x_38); -lean_inc(x_5); -lean_inc(x_1); -x_39 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_38); -if (x_39 == 0) -{ -lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; uint8_t x_49; -lean_dec(x_1); -x_40 = lean_unsigned_to_nat(1u); -x_41 = lean_nat_add(x_32, x_40); -lean_dec(x_32); -x_42 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_42, 0, x_5); -lean_ctor_set(x_42, 1, x_29); -lean_ctor_set(x_42, 2, x_38); -x_43 = lean_array_uset(x_33, x_37, x_42); -x_44 = lean_unsigned_to_nat(4u); -x_45 = lean_nat_mul(x_41, x_44); -x_46 = lean_unsigned_to_nat(3u); -x_47 = lean_nat_div(x_45, x_46); -lean_dec(x_45); -x_48 = lean_array_get_size(x_43); -x_49 = lean_nat_dec_le(x_47, x_48); -lean_dec(x_48); -lean_dec(x_47); -if (x_49 == 0) -{ -lean_object* x_50; -x_50 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_43); -lean_ctor_set(x_30, 1, x_50); -lean_ctor_set(x_30, 0, x_41); -return x_30; +x_28 = lean_box(0); +x_29 = lean_array_uset(x_8, x_22, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_31 = lean_array_uset(x_29, x_22, x_30); +lean_ctor_set(x_4, 1, x_31); +return x_4; } else { -lean_dec(x_2); -lean_ctor_set(x_30, 1, x_43); -lean_ctor_set(x_30, 0, x_41); -return x_30; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_4); +x_32 = lean_box(0); +x_33 = lean_array_uset(x_8, x_22, x_32); +x_34 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_35 = lean_array_uset(x_33, x_22, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_7); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } -else -{ -lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; -lean_dec(x_2); -x_51 = lean_box(0); -x_52 = lean_array_uset(x_33, x_37, x_51); -x_53 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_29, x_38); -x_54 = lean_array_uset(x_52, x_37, x_53); -lean_ctor_set(x_30, 1, x_54); -return x_30; } } -else -{ -lean_object* x_55; lean_object* x_56; lean_object* x_57; size_t x_58; size_t x_59; size_t x_60; lean_object* x_61; uint8_t x_62; -x_55 = lean_ctor_get(x_30, 0); -x_56 = lean_ctor_get(x_30, 1); -lean_inc(x_56); -lean_inc(x_55); -lean_dec(x_30); -x_57 = lean_array_get_size(x_56); -x_58 = lean_usize_of_nat(x_57); -lean_dec(x_57); -x_59 = lean_usize_sub(x_58, x_20); -x_60 = lean_usize_land(x_18, x_59); -x_61 = lean_array_uget(x_56, x_60); -lean_inc(x_61); -lean_inc(x_5); -lean_inc(x_1); -x_62 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_61); -if (x_62 == 0) -{ -lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; uint8_t x_72; -lean_dec(x_1); -x_63 = lean_unsigned_to_nat(1u); -x_64 = lean_nat_add(x_55, x_63); -lean_dec(x_55); -x_65 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_65, 0, x_5); -lean_ctor_set(x_65, 1, x_29); -lean_ctor_set(x_65, 2, x_61); -x_66 = lean_array_uset(x_56, x_60, x_65); -x_67 = lean_unsigned_to_nat(4u); -x_68 = lean_nat_mul(x_64, x_67); -x_69 = lean_unsigned_to_nat(3u); -x_70 = lean_nat_div(x_68, x_69); -lean_dec(x_68); -x_71 = lean_array_get_size(x_66); -x_72 = lean_nat_dec_le(x_70, x_71); -lean_dec(x_71); -lean_dec(x_70); -if (x_72 == 0) -{ -lean_object* x_73; lean_object* x_74; -x_73 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_66); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_64); -lean_ctor_set(x_74, 1, x_73); -return x_74; -} -else -{ -lean_object* x_75; -lean_dec(x_2); -x_75 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_75, 0, x_64); -lean_ctor_set(x_75, 1, x_66); -return x_75; -} -} -else +LEAN_EXPORT lean_object* l_Std_DHashMap_modify(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -lean_dec(x_2); -x_76 = lean_box(0); -x_77 = lean_array_uset(x_56, x_60, x_76); -x_78 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_29, x_61); -x_79 = lean_array_uset(x_77, x_60, x_78); -x_80 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_80, 0, x_55); -lean_ctor_set(x_80, 1, x_79); -return x_80; -} -} +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_modify___rarg), 6, 0); +return x_3; } } -else +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -lean_object* x_89; lean_object* x_90; lean_object* x_91; uint8_t x_120; -lean_dec(x_4); -x_89 = lean_ctor_get(x_24, 0); -lean_inc(x_89); -lean_dec(x_24); -x_90 = lean_apply_1(x_6, x_89); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_5); +x_10 = lean_apply_1(x_2, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); lean_inc(x_23); lean_inc(x_5); lean_inc(x_1); -x_120 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_120 == 0) +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) { -lean_object* x_121; lean_dec(x_23); -x_121 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_121, 0, x_7); -lean_ctor_set(x_121, 1, x_8); -x_91 = x_121; -goto block_119; -} -else -{ -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_122 = lean_box(0); -x_123 = lean_array_uset(x_8, x_22, x_122); -x_124 = lean_unsigned_to_nat(1u); -x_125 = lean_nat_sub(x_7, x_124); +lean_dec(x_8); lean_dec(x_7); -lean_inc(x_5); -lean_inc(x_1); -x_126 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_127 = lean_array_uset(x_123, x_22, x_126); -x_128 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_128, 0, x_125); -lean_ctor_set(x_128, 1, x_127); -x_91 = x_128; -goto block_119; -} -block_119: -{ -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; size_t x_96; size_t x_97; size_t x_98; lean_object* x_99; uint8_t x_100; -x_92 = lean_ctor_get(x_91, 0); -lean_inc(x_92); -x_93 = lean_ctor_get(x_91, 1); -lean_inc(x_93); -if (lean_is_exclusive(x_91)) { - lean_ctor_release(x_91, 0); - lean_ctor_release(x_91, 1); - x_94 = x_91; -} else { - lean_dec_ref(x_91); - x_94 = lean_box(0); -} -x_95 = lean_array_get_size(x_93); -x_96 = lean_usize_of_nat(x_95); -lean_dec(x_95); -x_97 = lean_usize_sub(x_96, x_20); -x_98 = lean_usize_land(x_18, x_97); -x_99 = lean_array_uget(x_93, x_98); -lean_inc(x_99); -lean_inc(x_5); -lean_inc(x_1); -x_100 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_99); -if (x_100 == 0) -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; uint8_t x_110; +lean_dec(x_6); +lean_dec(x_5); lean_dec(x_1); -x_101 = lean_unsigned_to_nat(1u); -x_102 = lean_nat_add(x_92, x_101); -lean_dec(x_92); -x_103 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_103, 0, x_5); -lean_ctor_set(x_103, 1, x_90); -lean_ctor_set(x_103, 2, x_99); -x_104 = lean_array_uset(x_93, x_98, x_103); -x_105 = lean_unsigned_to_nat(4u); -x_106 = lean_nat_mul(x_102, x_105); -x_107 = lean_unsigned_to_nat(3u); -x_108 = lean_nat_div(x_106, x_107); -lean_dec(x_106); -x_109 = lean_array_get_size(x_104); -x_110 = lean_nat_dec_le(x_108, x_109); -lean_dec(x_109); -lean_dec(x_108); -if (x_110 == 0) -{ -lean_object* x_111; lean_object* x_112; -x_111 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_104); -if (lean_is_scalar(x_94)) { - x_112 = lean_alloc_ctor(0, 2, 0); -} else { - x_112 = x_94; -} -lean_ctor_set(x_112, 0, x_102); -lean_ctor_set(x_112, 1, x_111); -return x_112; +return x_4; } else { -lean_object* x_113; -lean_dec(x_2); -if (lean_is_scalar(x_94)) { - x_113 = lean_alloc_ctor(0, 2, 0); -} else { - x_113 = x_94; -} -lean_ctor_set(x_113, 0, x_102); -lean_ctor_set(x_113, 1, x_104); -return x_113; -} +uint8_t x_25; +x_25 = !lean_is_exclusive(x_4); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_26 = lean_ctor_get(x_4, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_4, 0); +lean_dec(x_27); +x_28 = lean_box(0); +x_29 = lean_array_uset(x_8, x_22, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_31 = lean_array_uset(x_29, x_22, x_30); +lean_ctor_set(x_4, 1, x_31); +return x_4; } else { -lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -lean_dec(x_2); -x_114 = lean_box(0); -x_115 = lean_array_uset(x_93, x_98, x_114); -x_116 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_90, x_99); -x_117 = lean_array_uset(x_115, x_98, x_116); -if (lean_is_scalar(x_94)) { - x_118 = lean_alloc_ctor(0, 2, 0); -} else { - x_118 = x_94; -} -lean_ctor_set(x_118, 0, x_92); -lean_ctor_set(x_118, 1, x_117); -return x_118; -} -} +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_4); +x_32 = lean_box(0); +x_33 = lean_array_uset(x_8, x_22, x_32); +x_34 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_35 = lean_array_uset(x_33, x_22, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_7); +lean_ctor_set(x_36, 1, x_35); +return x_36; } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_modify(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_modify(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_modify___rarg), 6, 0); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Const_modify___rarg), 6, 0); +return x_2; } } LEAN_EXPORT lean_object* l_Std_DHashMap_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { _start: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; lean_object* x_24; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; x_7 = lean_ctor_get(x_4, 0); lean_inc(x_7); x_8 = lean_ctor_get(x_4, 1); @@ -7166,10 +6969,11 @@ x_23 = lean_array_uget(x_8, x_22); lean_inc(x_23); lean_inc(x_5); lean_inc(x_1); -x_24 = l_Std_DHashMap_Internal_AssocList_getCast_x3f___rarg(x_1, lean_box(0), x_5, x_23); -if (lean_obj_tag(x_24) == 0) +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) { lean_object* x_25; lean_object* x_26; +lean_dec(x_1); x_25 = lean_box(0); x_26 = lean_apply_1(x_6, x_25); if (lean_obj_tag(x_26) == 0) @@ -7179,7 +6983,6 @@ lean_dec(x_8); lean_dec(x_7); lean_dec(x_5); lean_dec(x_2); -lean_dec(x_1); return x_4; } else @@ -7188,7 +6991,7 @@ uint8_t x_27; x_27 = !lean_is_exclusive(x_4); if (x_27 == 0) { -lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; x_28 = lean_ctor_get(x_4, 1); lean_dec(x_28); x_29 = lean_ctor_get(x_4, 0); @@ -7196,709 +6999,378 @@ lean_dec(x_29); x_30 = lean_ctor_get(x_26, 0); lean_inc(x_30); lean_dec(x_26); -lean_inc(x_23); -lean_inc(x_5); -lean_inc(x_1); -x_31 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_31 == 0) -{ -lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; uint8_t x_41; -lean_dec(x_1); -x_32 = lean_unsigned_to_nat(1u); -x_33 = lean_nat_add(x_7, x_32); +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_7, x_31); lean_dec(x_7); -x_34 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_34, 0, x_5); -lean_ctor_set(x_34, 1, x_30); -lean_ctor_set(x_34, 2, x_23); -x_35 = lean_array_uset(x_8, x_22, x_34); -x_36 = lean_unsigned_to_nat(4u); -x_37 = lean_nat_mul(x_33, x_36); -x_38 = lean_unsigned_to_nat(3u); -x_39 = lean_nat_div(x_37, x_38); -lean_dec(x_37); -x_40 = lean_array_get_size(x_35); -x_41 = lean_nat_dec_le(x_39, x_40); -lean_dec(x_40); +x_33 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_33, 1, x_30); +lean_ctor_set(x_33, 2, x_23); +x_34 = lean_array_uset(x_8, x_22, x_33); +x_35 = lean_unsigned_to_nat(4u); +x_36 = lean_nat_mul(x_32, x_35); +x_37 = lean_unsigned_to_nat(3u); +x_38 = lean_nat_div(x_36, x_37); +lean_dec(x_36); +x_39 = lean_array_get_size(x_34); +x_40 = lean_nat_dec_le(x_38, x_39); lean_dec(x_39); -if (x_41 == 0) -{ -lean_object* x_42; -x_42 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_35); -lean_ctor_set(x_4, 1, x_42); -lean_ctor_set(x_4, 0, x_33); -return x_4; -} -else +lean_dec(x_38); +if (x_40 == 0) { -lean_dec(x_2); -lean_ctor_set(x_4, 1, x_35); -lean_ctor_set(x_4, 0, x_33); +lean_object* x_41; +x_41 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_34); +lean_ctor_set(x_4, 1, x_41); +lean_ctor_set(x_4, 0, x_32); return x_4; } -} else { -lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_dec(x_2); -x_43 = lean_box(0); -x_44 = lean_array_uset(x_8, x_22, x_43); -x_45 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_30, x_23); -x_46 = lean_array_uset(x_44, x_22, x_45); -lean_ctor_set(x_4, 1, x_46); +lean_ctor_set(x_4, 1, x_34); +lean_ctor_set(x_4, 0, x_32); return x_4; } } else { -lean_object* x_47; uint8_t x_48; +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_dec(x_4); -x_47 = lean_ctor_get(x_26, 0); -lean_inc(x_47); +x_42 = lean_ctor_get(x_26, 0); +lean_inc(x_42); lean_dec(x_26); -lean_inc(x_23); -lean_inc(x_5); -lean_inc(x_1); -x_48 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_48 == 0) -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; uint8_t x_58; -lean_dec(x_1); -x_49 = lean_unsigned_to_nat(1u); -x_50 = lean_nat_add(x_7, x_49); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_7, x_43); lean_dec(x_7); -x_51 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_51, 0, x_5); -lean_ctor_set(x_51, 1, x_47); -lean_ctor_set(x_51, 2, x_23); -x_52 = lean_array_uset(x_8, x_22, x_51); -x_53 = lean_unsigned_to_nat(4u); -x_54 = lean_nat_mul(x_50, x_53); -x_55 = lean_unsigned_to_nat(3u); -x_56 = lean_nat_div(x_54, x_55); -lean_dec(x_54); -x_57 = lean_array_get_size(x_52); -x_58 = lean_nat_dec_le(x_56, x_57); -lean_dec(x_57); -lean_dec(x_56); -if (x_58 == 0) -{ -lean_object* x_59; lean_object* x_60; -x_59 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_52); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_50); -lean_ctor_set(x_60, 1, x_59); -return x_60; -} -else +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_5); +lean_ctor_set(x_45, 1, x_42); +lean_ctor_set(x_45, 2, x_23); +x_46 = lean_array_uset(x_8, x_22, x_45); +x_47 = lean_unsigned_to_nat(4u); +x_48 = lean_nat_mul(x_44, x_47); +x_49 = lean_unsigned_to_nat(3u); +x_50 = lean_nat_div(x_48, x_49); +lean_dec(x_48); +x_51 = lean_array_get_size(x_46); +x_52 = lean_nat_dec_le(x_50, x_51); +lean_dec(x_51); +lean_dec(x_50); +if (x_52 == 0) { -lean_object* x_61; -lean_dec(x_2); -x_61 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_61, 0, x_50); -lean_ctor_set(x_61, 1, x_52); -return x_61; -} +lean_object* x_53; lean_object* x_54; +x_53 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_46); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_44); +lean_ctor_set(x_54, 1, x_53); +return x_54; } else { -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; +lean_object* x_55; lean_dec(x_2); -x_62 = lean_box(0); -x_63 = lean_array_uset(x_8, x_22, x_62); -x_64 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_47, x_23); -x_65 = lean_array_uset(x_63, x_22, x_64); -x_66 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_66, 0, x_7); -lean_ctor_set(x_66, 1, x_65); -return x_66; +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_44); +lean_ctor_set(x_55, 1, x_46); +return x_55; } } } } else { -uint8_t x_67; -x_67 = !lean_is_exclusive(x_4); -if (x_67 == 0) -{ -lean_object* x_68; lean_object* x_69; uint8_t x_70; -x_68 = lean_ctor_get(x_4, 1); -lean_dec(x_68); -x_69 = lean_ctor_get(x_4, 0); -lean_dec(x_69); -x_70 = !lean_is_exclusive(x_24); -if (x_70 == 0) -{ -lean_object* x_71; -x_71 = lean_apply_1(x_6, x_24); -if (lean_obj_tag(x_71) == 0) -{ -uint8_t x_72; +uint8_t x_56; lean_dec(x_2); -lean_inc(x_23); +x_56 = !lean_is_exclusive(x_4); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; +x_57 = lean_ctor_get(x_4, 1); +lean_dec(x_57); +x_58 = lean_ctor_get(x_4, 0); +lean_dec(x_58); +x_59 = lean_box(0); +x_60 = lean_array_uset(x_8, x_22, x_59); lean_inc(x_5); lean_inc(x_1); -x_72 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_72 == 0) +x_61 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_61); +x_62 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_61); +x_63 = lean_array_uset(x_60, x_22, x_61); +if (x_62 == 0) { -lean_dec(x_23); -lean_dec(x_5); -lean_dec(x_1); +lean_object* x_64; lean_object* x_65; +x_64 = lean_unsigned_to_nat(1u); +x_65 = lean_nat_sub(x_7, x_64); +lean_dec(x_7); +lean_ctor_set(x_4, 1, x_63); +lean_ctor_set(x_4, 0, x_65); return x_4; } else { -lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; -x_73 = lean_box(0); -x_74 = lean_array_uset(x_8, x_22, x_73); -x_75 = lean_unsigned_to_nat(1u); -x_76 = lean_nat_sub(x_7, x_75); -lean_dec(x_7); -x_77 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_78 = lean_array_uset(x_74, x_22, x_77); -lean_ctor_set(x_4, 1, x_78); -lean_ctor_set(x_4, 0, x_76); +lean_ctor_set(x_4, 1, x_63); return x_4; } } else { -lean_object* x_79; lean_object* x_80; uint8_t x_132; -x_79 = lean_ctor_get(x_71, 0); -lean_inc(x_79); -lean_dec(x_71); -lean_inc(x_23); +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; +lean_dec(x_4); +x_66 = lean_box(0); +x_67 = lean_array_uset(x_8, x_22, x_66); lean_inc(x_5); lean_inc(x_1); -x_132 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_132 == 0) -{ -lean_dec(x_23); -x_80 = x_4; -goto block_131; -} -else -{ -lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; -x_133 = lean_box(0); -x_134 = lean_array_uset(x_8, x_22, x_133); -x_135 = lean_unsigned_to_nat(1u); -x_136 = lean_nat_sub(x_7, x_135); +x_68 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_68); +x_69 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_68); +x_70 = lean_array_uset(x_67, x_22, x_68); +if (x_69 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_unsigned_to_nat(1u); +x_72 = lean_nat_sub(x_7, x_71); lean_dec(x_7); -lean_inc(x_5); -lean_inc(x_1); -x_137 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_138 = lean_array_uset(x_134, x_22, x_137); -lean_ctor_set(x_4, 1, x_138); -lean_ctor_set(x_4, 0, x_136); -x_80 = x_4; -goto block_131; -} -block_131: -{ -uint8_t x_81; -x_81 = !lean_is_exclusive(x_80); -if (x_81 == 0) -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; size_t x_85; size_t x_86; size_t x_87; lean_object* x_88; uint8_t x_89; -x_82 = lean_ctor_get(x_80, 0); -x_83 = lean_ctor_get(x_80, 1); -x_84 = lean_array_get_size(x_83); -x_85 = lean_usize_of_nat(x_84); -lean_dec(x_84); -x_86 = lean_usize_sub(x_85, x_20); -x_87 = lean_usize_land(x_18, x_86); -x_88 = lean_array_uget(x_83, x_87); -lean_inc(x_88); -lean_inc(x_5); -lean_inc(x_1); -x_89 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_88); -if (x_89 == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; -lean_dec(x_1); -x_90 = lean_unsigned_to_nat(1u); -x_91 = lean_nat_add(x_82, x_90); -lean_dec(x_82); -x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_5); -lean_ctor_set(x_92, 1, x_79); -lean_ctor_set(x_92, 2, x_88); -x_93 = lean_array_uset(x_83, x_87, x_92); -x_94 = lean_unsigned_to_nat(4u); -x_95 = lean_nat_mul(x_91, x_94); -x_96 = lean_unsigned_to_nat(3u); -x_97 = lean_nat_div(x_95, x_96); -lean_dec(x_95); -x_98 = lean_array_get_size(x_93); -x_99 = lean_nat_dec_le(x_97, x_98); -lean_dec(x_98); -lean_dec(x_97); -if (x_99 == 0) -{ -lean_object* x_100; -x_100 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_93); -lean_ctor_set(x_80, 1, x_100); -lean_ctor_set(x_80, 0, x_91); -return x_80; +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; } else { -lean_dec(x_2); -lean_ctor_set(x_80, 1, x_93); -lean_ctor_set(x_80, 0, x_91); -return x_80; -} +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_7); +lean_ctor_set(x_74, 1, x_70); +return x_74; } -else -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; -lean_dec(x_2); -x_101 = lean_box(0); -x_102 = lean_array_uset(x_83, x_87, x_101); -x_103 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_79, x_88); -x_104 = lean_array_uset(x_102, x_87, x_103); -lean_ctor_set(x_80, 1, x_104); -return x_80; } } -else -{ -lean_object* x_105; lean_object* x_106; lean_object* x_107; size_t x_108; size_t x_109; size_t x_110; lean_object* x_111; uint8_t x_112; -x_105 = lean_ctor_get(x_80, 0); -x_106 = lean_ctor_get(x_80, 1); -lean_inc(x_106); -lean_inc(x_105); -lean_dec(x_80); -x_107 = lean_array_get_size(x_106); -x_108 = lean_usize_of_nat(x_107); -lean_dec(x_107); -x_109 = lean_usize_sub(x_108, x_20); -x_110 = lean_usize_land(x_18, x_109); -x_111 = lean_array_uget(x_106, x_110); -lean_inc(x_111); -lean_inc(x_5); -lean_inc(x_1); -x_112 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_111); -if (x_112 == 0) -{ -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; uint8_t x_122; -lean_dec(x_1); -x_113 = lean_unsigned_to_nat(1u); -x_114 = lean_nat_add(x_105, x_113); -lean_dec(x_105); -x_115 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_115, 0, x_5); -lean_ctor_set(x_115, 1, x_79); -lean_ctor_set(x_115, 2, x_111); -x_116 = lean_array_uset(x_106, x_110, x_115); -x_117 = lean_unsigned_to_nat(4u); -x_118 = lean_nat_mul(x_114, x_117); -x_119 = lean_unsigned_to_nat(3u); -x_120 = lean_nat_div(x_118, x_119); -lean_dec(x_118); -x_121 = lean_array_get_size(x_116); -x_122 = lean_nat_dec_le(x_120, x_121); -lean_dec(x_121); -lean_dec(x_120); -if (x_122 == 0) -{ -lean_object* x_123; lean_object* x_124; -x_123 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_116); -x_124 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_124, 0, x_114); -lean_ctor_set(x_124, 1, x_123); -return x_124; -} -else -{ -lean_object* x_125; -lean_dec(x_2); -x_125 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_125, 0, x_114); -lean_ctor_set(x_125, 1, x_116); -return x_125; } } -else +LEAN_EXPORT lean_object* l_Std_DHashMap_alter(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; -lean_dec(x_2); -x_126 = lean_box(0); -x_127 = lean_array_uset(x_106, x_110, x_126); -x_128 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_79, x_111); -x_129 = lean_array_uset(x_127, x_110, x_128); -x_130 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_130, 0, x_105); -lean_ctor_set(x_130, 1, x_129); -return x_130; -} -} -} +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_alter___rarg), 6, 0); +return x_3; } } -else -{ -lean_object* x_139; lean_object* x_140; lean_object* x_141; -x_139 = lean_ctor_get(x_24, 0); -lean_inc(x_139); -lean_dec(x_24); -x_140 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_140, 0, x_139); -x_141 = lean_apply_1(x_6, x_140); -if (lean_obj_tag(x_141) == 0) +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: { -uint8_t x_142; -lean_dec(x_2); +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_2); +lean_inc(x_5); +x_10 = lean_apply_1(x_2, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); lean_inc(x_23); lean_inc(x_5); lean_inc(x_1); -x_142 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_142 == 0) +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) { -lean_dec(x_23); -lean_dec(x_5); +lean_object* x_25; lean_object* x_26; lean_dec(x_1); -return x_4; -} -else +x_25 = lean_box(0); +x_26 = lean_apply_1(x_6, x_25); +if (lean_obj_tag(x_26) == 0) { -lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; -x_143 = lean_box(0); -x_144 = lean_array_uset(x_8, x_22, x_143); -x_145 = lean_unsigned_to_nat(1u); -x_146 = lean_nat_sub(x_7, x_145); +lean_dec(x_23); +lean_dec(x_8); lean_dec(x_7); -x_147 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_148 = lean_array_uset(x_144, x_22, x_147); -lean_ctor_set(x_4, 1, x_148); -lean_ctor_set(x_4, 0, x_146); +lean_dec(x_5); +lean_dec(x_2); return x_4; } -} else { -lean_object* x_149; lean_object* x_150; uint8_t x_179; -x_149 = lean_ctor_get(x_141, 0); -lean_inc(x_149); -lean_dec(x_141); -lean_inc(x_23); -lean_inc(x_5); -lean_inc(x_1); -x_179 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_179 == 0) -{ -lean_dec(x_23); -x_150 = x_4; -goto block_178; -} -else +uint8_t x_27; +x_27 = !lean_is_exclusive(x_4); +if (x_27 == 0) { -lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; -x_180 = lean_box(0); -x_181 = lean_array_uset(x_8, x_22, x_180); -x_182 = lean_unsigned_to_nat(1u); -x_183 = lean_nat_sub(x_7, x_182); +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_28 = lean_ctor_get(x_4, 1); +lean_dec(x_28); +x_29 = lean_ctor_get(x_4, 0); +lean_dec(x_29); +x_30 = lean_ctor_get(x_26, 0); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_7, x_31); lean_dec(x_7); -lean_inc(x_5); -lean_inc(x_1); -x_184 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_185 = lean_array_uset(x_181, x_22, x_184); -lean_ctor_set(x_4, 1, x_185); -lean_ctor_set(x_4, 0, x_183); -x_150 = x_4; -goto block_178; -} -block_178: -{ -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; size_t x_155; size_t x_156; size_t x_157; lean_object* x_158; uint8_t x_159; -x_151 = lean_ctor_get(x_150, 0); -lean_inc(x_151); -x_152 = lean_ctor_get(x_150, 1); -lean_inc(x_152); -if (lean_is_exclusive(x_150)) { - lean_ctor_release(x_150, 0); - lean_ctor_release(x_150, 1); - x_153 = x_150; -} else { - lean_dec_ref(x_150); - x_153 = lean_box(0); -} -x_154 = lean_array_get_size(x_152); -x_155 = lean_usize_of_nat(x_154); -lean_dec(x_154); -x_156 = lean_usize_sub(x_155, x_20); -x_157 = lean_usize_land(x_18, x_156); -x_158 = lean_array_uget(x_152, x_157); -lean_inc(x_158); -lean_inc(x_5); -lean_inc(x_1); -x_159 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_158); -if (x_159 == 0) -{ -lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; uint8_t x_169; -lean_dec(x_1); -x_160 = lean_unsigned_to_nat(1u); -x_161 = lean_nat_add(x_151, x_160); -lean_dec(x_151); -x_162 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_162, 0, x_5); -lean_ctor_set(x_162, 1, x_149); -lean_ctor_set(x_162, 2, x_158); -x_163 = lean_array_uset(x_152, x_157, x_162); -x_164 = lean_unsigned_to_nat(4u); -x_165 = lean_nat_mul(x_161, x_164); -x_166 = lean_unsigned_to_nat(3u); -x_167 = lean_nat_div(x_165, x_166); -lean_dec(x_165); -x_168 = lean_array_get_size(x_163); -x_169 = lean_nat_dec_le(x_167, x_168); -lean_dec(x_168); -lean_dec(x_167); -if (x_169 == 0) +x_33 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_33, 1, x_30); +lean_ctor_set(x_33, 2, x_23); +x_34 = lean_array_uset(x_8, x_22, x_33); +x_35 = lean_unsigned_to_nat(4u); +x_36 = lean_nat_mul(x_32, x_35); +x_37 = lean_unsigned_to_nat(3u); +x_38 = lean_nat_div(x_36, x_37); +lean_dec(x_36); +x_39 = lean_array_get_size(x_34); +x_40 = lean_nat_dec_le(x_38, x_39); +lean_dec(x_39); +lean_dec(x_38); +if (x_40 == 0) { -lean_object* x_170; lean_object* x_171; -x_170 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_163); -if (lean_is_scalar(x_153)) { - x_171 = lean_alloc_ctor(0, 2, 0); -} else { - x_171 = x_153; -} -lean_ctor_set(x_171, 0, x_161); -lean_ctor_set(x_171, 1, x_170); -return x_171; +lean_object* x_41; +x_41 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_34); +lean_ctor_set(x_4, 1, x_41); +lean_ctor_set(x_4, 0, x_32); +return x_4; } else { -lean_object* x_172; lean_dec(x_2); -if (lean_is_scalar(x_153)) { - x_172 = lean_alloc_ctor(0, 2, 0); -} else { - x_172 = x_153; +lean_ctor_set(x_4, 1, x_34); +lean_ctor_set(x_4, 0, x_32); +return x_4; } -lean_ctor_set(x_172, 0, x_161); -lean_ctor_set(x_172, 1, x_163); -return x_172; } +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +lean_dec(x_4); +x_42 = lean_ctor_get(x_26, 0); +lean_inc(x_42); +lean_dec(x_26); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_7, x_43); +lean_dec(x_7); +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_5); +lean_ctor_set(x_45, 1, x_42); +lean_ctor_set(x_45, 2, x_23); +x_46 = lean_array_uset(x_8, x_22, x_45); +x_47 = lean_unsigned_to_nat(4u); +x_48 = lean_nat_mul(x_44, x_47); +x_49 = lean_unsigned_to_nat(3u); +x_50 = lean_nat_div(x_48, x_49); +lean_dec(x_48); +x_51 = lean_array_get_size(x_46); +x_52 = lean_nat_dec_le(x_50, x_51); +lean_dec(x_51); +lean_dec(x_50); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_46); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_44); +lean_ctor_set(x_54, 1, x_53); +return x_54; } else { -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; +lean_object* x_55; lean_dec(x_2); -x_173 = lean_box(0); -x_174 = lean_array_uset(x_152, x_157, x_173); -x_175 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_149, x_158); -x_176 = lean_array_uset(x_174, x_157, x_175); -if (lean_is_scalar(x_153)) { - x_177 = lean_alloc_ctor(0, 2, 0); -} else { - x_177 = x_153; -} -lean_ctor_set(x_177, 0, x_151); -lean_ctor_set(x_177, 1, x_176); -return x_177; -} +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_44); +lean_ctor_set(x_55, 1, x_46); +return x_55; } } } } else { -lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; -lean_dec(x_4); -x_186 = lean_ctor_get(x_24, 0); -lean_inc(x_186); -if (lean_is_exclusive(x_24)) { - lean_ctor_release(x_24, 0); - x_187 = x_24; -} else { - lean_dec_ref(x_24); - x_187 = lean_box(0); -} -if (lean_is_scalar(x_187)) { - x_188 = lean_alloc_ctor(1, 1, 0); -} else { - x_188 = x_187; -} -lean_ctor_set(x_188, 0, x_186); -x_189 = lean_apply_1(x_6, x_188); -if (lean_obj_tag(x_189) == 0) -{ -uint8_t x_190; +uint8_t x_56; lean_dec(x_2); -lean_inc(x_23); +x_56 = !lean_is_exclusive(x_4); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; +x_57 = lean_ctor_get(x_4, 1); +lean_dec(x_57); +x_58 = lean_ctor_get(x_4, 0); +lean_dec(x_58); +x_59 = lean_box(0); +x_60 = lean_array_uset(x_8, x_22, x_59); lean_inc(x_5); lean_inc(x_1); -x_190 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_190 == 0) +x_61 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_61); +x_62 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_61); +x_63 = lean_array_uset(x_60, x_22, x_61); +if (x_62 == 0) { -lean_object* x_191; -lean_dec(x_23); -lean_dec(x_5); -lean_dec(x_1); -x_191 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_191, 0, x_7); -lean_ctor_set(x_191, 1, x_8); -return x_191; +lean_object* x_64; lean_object* x_65; +x_64 = lean_unsigned_to_nat(1u); +x_65 = lean_nat_sub(x_7, x_64); +lean_dec(x_7); +lean_ctor_set(x_4, 1, x_63); +lean_ctor_set(x_4, 0, x_65); +return x_4; } else { -lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_192 = lean_box(0); -x_193 = lean_array_uset(x_8, x_22, x_192); -x_194 = lean_unsigned_to_nat(1u); -x_195 = lean_nat_sub(x_7, x_194); -lean_dec(x_7); -x_196 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_197 = lean_array_uset(x_193, x_22, x_196); -x_198 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_198, 0, x_195); -lean_ctor_set(x_198, 1, x_197); -return x_198; +lean_ctor_set(x_4, 1, x_63); +return x_4; } } else { -lean_object* x_199; lean_object* x_200; uint8_t x_229; -x_199 = lean_ctor_get(x_189, 0); -lean_inc(x_199); -lean_dec(x_189); -lean_inc(x_23); +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; +lean_dec(x_4); +x_66 = lean_box(0); +x_67 = lean_array_uset(x_8, x_22, x_66); lean_inc(x_5); lean_inc(x_1); -x_229 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); -if (x_229 == 0) -{ -lean_object* x_230; -lean_dec(x_23); -x_230 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_230, 0, x_7); -lean_ctor_set(x_230, 1, x_8); -x_200 = x_230; -goto block_228; -} -else -{ -lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; lean_object* x_237; -x_231 = lean_box(0); -x_232 = lean_array_uset(x_8, x_22, x_231); -x_233 = lean_unsigned_to_nat(1u); -x_234 = lean_nat_sub(x_7, x_233); +x_68 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_68); +x_69 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_68); +x_70 = lean_array_uset(x_67, x_22, x_68); +if (x_69 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_unsigned_to_nat(1u); +x_72 = lean_nat_sub(x_7, x_71); lean_dec(x_7); -lean_inc(x_5); -lean_inc(x_1); -x_235 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_5, x_23); -x_236 = lean_array_uset(x_232, x_22, x_235); -x_237 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_237, 0, x_234); -lean_ctor_set(x_237, 1, x_236); -x_200 = x_237; -goto block_228; -} -block_228: -{ -lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; size_t x_205; size_t x_206; size_t x_207; lean_object* x_208; uint8_t x_209; -x_201 = lean_ctor_get(x_200, 0); -lean_inc(x_201); -x_202 = lean_ctor_get(x_200, 1); -lean_inc(x_202); -if (lean_is_exclusive(x_200)) { - lean_ctor_release(x_200, 0); - lean_ctor_release(x_200, 1); - x_203 = x_200; -} else { - lean_dec_ref(x_200); - x_203 = lean_box(0); -} -x_204 = lean_array_get_size(x_202); -x_205 = lean_usize_of_nat(x_204); -lean_dec(x_204); -x_206 = lean_usize_sub(x_205, x_20); -x_207 = lean_usize_land(x_18, x_206); -x_208 = lean_array_uget(x_202, x_207); -lean_inc(x_208); -lean_inc(x_5); -lean_inc(x_1); -x_209 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_208); -if (x_209 == 0) -{ -lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; lean_object* x_218; uint8_t x_219; -lean_dec(x_1); -x_210 = lean_unsigned_to_nat(1u); -x_211 = lean_nat_add(x_201, x_210); -lean_dec(x_201); -x_212 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_212, 0, x_5); -lean_ctor_set(x_212, 1, x_199); -lean_ctor_set(x_212, 2, x_208); -x_213 = lean_array_uset(x_202, x_207, x_212); -x_214 = lean_unsigned_to_nat(4u); -x_215 = lean_nat_mul(x_211, x_214); -x_216 = lean_unsigned_to_nat(3u); -x_217 = lean_nat_div(x_215, x_216); -lean_dec(x_215); -x_218 = lean_array_get_size(x_213); -x_219 = lean_nat_dec_le(x_217, x_218); -lean_dec(x_218); -lean_dec(x_217); -if (x_219 == 0) -{ -lean_object* x_220; lean_object* x_221; -x_220 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_213); -if (lean_is_scalar(x_203)) { - x_221 = lean_alloc_ctor(0, 2, 0); -} else { - x_221 = x_203; -} -lean_ctor_set(x_221, 0, x_211); -lean_ctor_set(x_221, 1, x_220); -return x_221; -} -else -{ -lean_object* x_222; -lean_dec(x_2); -if (lean_is_scalar(x_203)) { - x_222 = lean_alloc_ctor(0, 2, 0); -} else { - x_222 = x_203; -} -lean_ctor_set(x_222, 0, x_211); -lean_ctor_set(x_222, 1, x_213); -return x_222; -} +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; } else { -lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; lean_object* x_227; -lean_dec(x_2); -x_223 = lean_box(0); -x_224 = lean_array_uset(x_202, x_207, x_223); -x_225 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_5, x_199, x_208); -x_226 = lean_array_uset(x_224, x_207, x_225); -if (lean_is_scalar(x_203)) { - x_227 = lean_alloc_ctor(0, 2, 0); -} else { - x_227 = x_203; -} -lean_ctor_set(x_227, 0, x_201); -lean_ctor_set(x_227, 1, x_226); -return x_227; -} -} +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_7); +lean_ctor_set(x_74, 1, x_70); +return x_74; } } } } } -LEAN_EXPORT lean_object* l_Std_DHashMap_alter(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Const_alter(lean_object* x_1) { _start: { -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_alter___rarg), 6, 0); -return x_3; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Const_alter___rarg), 6, 0); +return x_2; } } LEAN_EXPORT lean_object* l_Std_DHashMap_insertMany___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Basic.c b/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Basic.c index 380d4a75685d..2d916e19a257 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Basic.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Basic.c @@ -27,6 +27,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD___rarg(lean_obje LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_length___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getD(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldr___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldl___rarg(lean_object*, lean_object*, lean_object*); @@ -35,9 +36,12 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21(lean_object*, LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldl(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_length___spec__1___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_map_go___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_modify(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg___closed__2; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x21___rarg___closed__1; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_length___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_filter_go(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_filterMap_go___rarg(lean_object*, lean_object*, lean_object*); @@ -74,15 +78,18 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_filterMap___rarg(lean LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_contains___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x21(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_alter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_forM___spec__1___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_replace(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getCastD(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getCast(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_forM___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forM(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getKeyD___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_filter___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldr(lean_object*, lean_object*, lean_object*); @@ -91,6 +98,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_get(lean_object*, lea LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getCast___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x21___rarg___closed__4; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_erase(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forM___rarg(lean_object*, lean_object*, lean_object*); @@ -1601,6 +1609,484 @@ x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_erase___rarg) return x_3; } } +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; +} +else +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_8 = lean_ctor_get(x_5, 0); +x_9 = lean_ctor_get(x_5, 1); +x_10 = lean_ctor_get(x_5, 2); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_8); +x_11 = lean_apply_2(x_1, x_8, x_3); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_3, x_4, x_10); +lean_ctor_set(x_5, 2, x_13); +return x_5; +} +else +{ +lean_object* x_14; +lean_dec(x_8); +lean_dec(x_1); +x_14 = lean_apply_1(x_4, x_9); +lean_ctor_set(x_5, 1, x_14); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_5, 0); +x_16 = lean_ctor_get(x_5, 1); +x_17 = lean_ctor_get(x_5, 2); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_5); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_15); +x_18 = lean_apply_2(x_1, x_15, x_3); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_3, x_4, x_17); +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_15); +lean_ctor_set(x_21, 1, x_16); +lean_ctor_set(x_21, 2, x_20); +return x_21; +} +else +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_15); +lean_dec(x_1); +x_22 = lean_apply_1(x_4, x_16); +x_23 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 2, x_17); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_modify(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_modify___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(0); +x_7 = lean_apply_1(x_4, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +lean_dec(x_3); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_9); +lean_ctor_set(x_11, 2, x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_5); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_5, 0); +x_14 = lean_ctor_get(x_5, 1); +x_15 = lean_ctor_get(x_5, 2); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_13); +x_16 = lean_apply_2(x_1, x_13, x_3); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_3, x_4, x_15); +lean_ctor_set(x_5, 2, x_18); +return x_5; +} +else +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_13); +lean_dec(x_1); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_14); +x_20 = lean_apply_1(x_4, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_free_object(x_5); +lean_dec(x_3); +return x_15; +} +else +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +lean_dec(x_20); +lean_ctor_set(x_5, 1, x_21); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_5, 0); +x_23 = lean_ctor_get(x_5, 1); +x_24 = lean_ctor_get(x_5, 2); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_5); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_22); +x_25 = lean_apply_2(x_1, x_22, x_3); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_3, x_4, x_24); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_27); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_22); +lean_dec(x_1); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_23); +x_30 = lean_apply_1(x_4, x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_dec(x_3); +return x_24; +} +else +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_24); +return x_32; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_alter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_alter___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +x_6 = lean_box(0); +return x_6; +} +else +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_8 = lean_ctor_get(x_5, 0); +x_9 = lean_ctor_get(x_5, 1); +x_10 = lean_ctor_get(x_5, 2); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_8); +x_11 = lean_apply_2(x_1, x_8, x_3); +x_12 = lean_unbox(x_11); +lean_dec(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_3, x_4, x_10); +lean_ctor_set(x_5, 2, x_13); +return x_5; +} +else +{ +lean_object* x_14; +lean_dec(x_8); +lean_dec(x_1); +x_14 = lean_apply_1(x_4, x_9); +lean_ctor_set(x_5, 1, x_14); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_15 = lean_ctor_get(x_5, 0); +x_16 = lean_ctor_get(x_5, 1); +x_17 = lean_ctor_get(x_5, 2); +lean_inc(x_17); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_5); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_15); +x_18 = lean_apply_2(x_1, x_15, x_3); +x_19 = lean_unbox(x_18); +lean_dec(x_18); +if (x_19 == 0) +{ +lean_object* x_20; lean_object* x_21; +x_20 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_3, x_4, x_17); +x_21 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_21, 0, x_15); +lean_ctor_set(x_21, 1, x_16); +lean_ctor_set(x_21, 2, x_20); +return x_21; +} +else +{ +lean_object* x_22; lean_object* x_23; +lean_dec(x_15); +lean_dec(x_1); +x_22 = lean_apply_1(x_4, x_16); +x_23 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_23, 0, x_3); +lean_ctor_set(x_23, 1, x_22); +lean_ctor_set(x_23, 2, x_17); +return x_23; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_modify___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +if (lean_obj_tag(x_5) == 0) +{ +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(0); +x_7 = lean_apply_1(x_4, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +lean_dec(x_3); +x_8 = lean_box(0); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_9); +lean_ctor_set(x_11, 2, x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_5); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_5, 0); +x_14 = lean_ctor_get(x_5, 1); +x_15 = lean_ctor_get(x_5, 2); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_13); +x_16 = lean_apply_2(x_1, x_13, x_3); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_3, x_4, x_15); +lean_ctor_set(x_5, 2, x_18); +return x_5; +} +else +{ +lean_object* x_19; lean_object* x_20; +lean_dec(x_13); +lean_dec(x_1); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_14); +x_20 = lean_apply_1(x_4, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_free_object(x_5); +lean_dec(x_3); +return x_15; +} +else +{ +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +lean_dec(x_20); +lean_ctor_set(x_5, 1, x_21); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_5, 0); +x_23 = lean_ctor_get(x_5, 1); +x_24 = lean_ctor_get(x_5, 2); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_5); +lean_inc(x_1); +lean_inc(x_3); +lean_inc(x_22); +x_25 = lean_apply_2(x_1, x_22, x_3); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_3, x_4, x_24); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_27); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_22); +lean_dec(x_1); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_23); +x_30 = lean_apply_1(x_4, x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_dec(x_3); +return x_24; +} +else +{ +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_24); +return x_32; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___rarg), 5, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_filterMap_go___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Lemmas.c b/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Lemmas.c index cd971b779939..7644c69f4f90 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Lemmas.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/AssocList/Lemmas.c @@ -13,30 +13,37 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_getEntry_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_getEntry_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_foldlM_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__List_filterMap_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_toList_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__List_filterMap_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_toList_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__List_filterMap_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_toList_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_getCast_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_getCast_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_getCast_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_get_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_getEntry_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_foldlM_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_foldlM_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -263,7 +270,7 @@ lean_dec(x_3); return x_6; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -283,28 +290,28 @@ return x_5; } } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg___boxed), 3, 0); +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg___boxed), 3, 0); return x_5; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___rarg(x_1, x_2, x_3); +x_4 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___rarg(x_1, x_2, x_3); lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_filterMap_go_match__1_splitter(x_1, x_2, x_3, x_4); +x_5 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_alter_match__1_splitter(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } @@ -346,6 +353,89 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed), 3, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_AssocList_Lemmas_0__Std_DHashMap_Internal_AssocList_Const_alter_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} lean_object* initialize_Std_Data_DHashMap_Internal_AssocList_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_DHashMap_Internal_List_Associative(uint8_t builtin, lean_object*); static bool _G_initialized = false; diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c index 68e2b9af34bb..586b97d25191 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/Defs.c @@ -16,6 +16,7 @@ extern "C" { LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_empty___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_computeSize___rarg(lean_object*); @@ -25,6 +26,7 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Ra LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getD___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_contains(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify(lean_object*); size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -35,6 +37,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f(lean_objec LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_reinsertAux(lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_fget(lean_object*, lean_object*); lean_object* lean_array_fset(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -45,6 +48,7 @@ lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_length___spec__1___rarg(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_map_go___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filter___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_map___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_map___spec__1(lean_object*, lean_object*, lean_object*); @@ -58,6 +62,7 @@ LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListMo size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_DHashMap_Internal_Raw_u2080_contains___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_getD(lean_object*, lean_object*); @@ -75,6 +80,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expandIfNecessary___r LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insertMany___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filterMap___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_to_list(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_containsThenInsertIfNew(lean_object*, lean_object*); @@ -102,9 +108,12 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insertMany___rarg(lea LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_computeSize___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_insertManyIfNewUnit___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_filterMap___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter(lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter(lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKeyD(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080_map___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD(lean_object*, lean_object*); @@ -115,6 +124,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f___rarg___b LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expandIfNecessary___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_toListModel___rarg___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_toListModel(lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); @@ -151,10 +161,12 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(lean_ob lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_List_flatMapTR_go___at_Std_DHashMap_Internal_toListModel___spec__1(lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Raw_u2080_filterMap___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_Raw_u2080_filter___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_filter_go___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_containsThenInsertIfNew___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); @@ -855,6 +867,604 @@ x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_insert___rarg return x_3; } } +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_5); +x_10 = lean_apply_1(x_2, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); +lean_inc(x_23); +lean_inc(x_5); +lean_inc(x_1); +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) +{ +lean_dec(x_23); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_4; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_4); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_26 = lean_ctor_get(x_4, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_4, 0); +lean_dec(x_27); +x_28 = lean_box(0); +x_29 = lean_array_uset(x_8, x_22, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_31 = lean_array_uset(x_29, x_22, x_30); +lean_ctor_set(x_4, 1, x_31); +return x_4; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_4); +x_32 = lean_box(0); +x_33 = lean_array_uset(x_8, x_22, x_32); +x_34 = l_Std_DHashMap_Internal_AssocList_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_35 = lean_array_uset(x_33, x_22, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_7); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_modify___rarg), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_5); +x_10 = lean_apply_1(x_3, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); +lean_inc(x_23); +lean_inc(x_5); +lean_inc(x_1); +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) +{ +lean_dec(x_23); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_6); +lean_dec(x_5); +lean_dec(x_1); +return x_4; +} +else +{ +uint8_t x_25; +x_25 = !lean_is_exclusive(x_4); +if (x_25 == 0) +{ +lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; +x_26 = lean_ctor_get(x_4, 1); +lean_dec(x_26); +x_27 = lean_ctor_get(x_4, 0); +lean_dec(x_27); +x_28 = lean_box(0); +x_29 = lean_array_uset(x_8, x_22, x_28); +x_30 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_31 = lean_array_uset(x_29, x_22, x_30); +lean_ctor_set(x_4, 1, x_31); +return x_4; +} +else +{ +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +lean_dec(x_4); +x_32 = lean_box(0); +x_33 = lean_array_uset(x_8, x_22, x_32); +x_34 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_5, x_6, x_23); +x_35 = lean_array_uset(x_33, x_22, x_34); +x_36 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_36, 0, x_7); +lean_ctor_set(x_36, 1, x_35); +return x_36; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_Const_modify___rarg), 6, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_2); +lean_inc(x_5); +x_10 = lean_apply_1(x_2, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); +lean_inc(x_23); +lean_inc(x_5); +lean_inc(x_1); +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_1); +x_25 = lean_box(0); +x_26 = lean_apply_1(x_6, x_25); +if (lean_obj_tag(x_26) == 0) +{ +lean_dec(x_23); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_2); +return x_4; +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_4); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_28 = lean_ctor_get(x_4, 1); +lean_dec(x_28); +x_29 = lean_ctor_get(x_4, 0); +lean_dec(x_29); +x_30 = lean_ctor_get(x_26, 0); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_7, x_31); +lean_dec(x_7); +x_33 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_33, 1, x_30); +lean_ctor_set(x_33, 2, x_23); +x_34 = lean_array_uset(x_8, x_22, x_33); +x_35 = lean_unsigned_to_nat(4u); +x_36 = lean_nat_mul(x_32, x_35); +x_37 = lean_unsigned_to_nat(3u); +x_38 = lean_nat_div(x_36, x_37); +lean_dec(x_36); +x_39 = lean_array_get_size(x_34); +x_40 = lean_nat_dec_le(x_38, x_39); +lean_dec(x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; +x_41 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_34); +lean_ctor_set(x_4, 1, x_41); +lean_ctor_set(x_4, 0, x_32); +return x_4; +} +else +{ +lean_dec(x_2); +lean_ctor_set(x_4, 1, x_34); +lean_ctor_set(x_4, 0, x_32); +return x_4; +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +lean_dec(x_4); +x_42 = lean_ctor_get(x_26, 0); +lean_inc(x_42); +lean_dec(x_26); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_7, x_43); +lean_dec(x_7); +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_5); +lean_ctor_set(x_45, 1, x_42); +lean_ctor_set(x_45, 2, x_23); +x_46 = lean_array_uset(x_8, x_22, x_45); +x_47 = lean_unsigned_to_nat(4u); +x_48 = lean_nat_mul(x_44, x_47); +x_49 = lean_unsigned_to_nat(3u); +x_50 = lean_nat_div(x_48, x_49); +lean_dec(x_48); +x_51 = lean_array_get_size(x_46); +x_52 = lean_nat_dec_le(x_50, x_51); +lean_dec(x_51); +lean_dec(x_50); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_46); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_44); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +else +{ +lean_object* x_55; +lean_dec(x_2); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_44); +lean_ctor_set(x_55, 1, x_46); +return x_55; +} +} +} +} +else +{ +uint8_t x_56; +lean_dec(x_2); +x_56 = !lean_is_exclusive(x_4); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; +x_57 = lean_ctor_get(x_4, 1); +lean_dec(x_57); +x_58 = lean_ctor_get(x_4, 0); +lean_dec(x_58); +x_59 = lean_box(0); +x_60 = lean_array_uset(x_8, x_22, x_59); +lean_inc(x_5); +lean_inc(x_1); +x_61 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_61); +x_62 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_61); +x_63 = lean_array_uset(x_60, x_22, x_61); +if (x_62 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_unsigned_to_nat(1u); +x_65 = lean_nat_sub(x_7, x_64); +lean_dec(x_7); +lean_ctor_set(x_4, 1, x_63); +lean_ctor_set(x_4, 0, x_65); +return x_4; +} +else +{ +lean_ctor_set(x_4, 1, x_63); +return x_4; +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; +lean_dec(x_4); +x_66 = lean_box(0); +x_67 = lean_array_uset(x_8, x_22, x_66); +lean_inc(x_5); +lean_inc(x_1); +x_68 = l_Std_DHashMap_Internal_AssocList_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_68); +x_69 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_68); +x_70 = lean_array_uset(x_67, x_22, x_68); +if (x_69 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_unsigned_to_nat(1u); +x_72 = lean_nat_sub(x_7, x_71); +lean_dec(x_7); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; +} +else +{ +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_7); +lean_ctor_set(x_74, 1, x_70); +return x_74; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_alter___rarg), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; uint64_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; size_t x_22; lean_object* x_23; uint8_t x_24; +x_7 = lean_ctor_get(x_4, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_4, 1); +lean_inc(x_8); +x_9 = lean_array_get_size(x_8); +lean_inc(x_2); +lean_inc(x_5); +x_10 = lean_apply_1(x_2, x_5); +x_11 = lean_unbox_uint64(x_10); +lean_dec(x_10); +x_12 = 32; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = 16; +x_16 = lean_uint64_shift_right(x_14, x_15); +x_17 = lean_uint64_xor(x_14, x_16); +x_18 = lean_uint64_to_usize(x_17); +x_19 = lean_usize_of_nat(x_9); +lean_dec(x_9); +x_20 = 1; +x_21 = lean_usize_sub(x_19, x_20); +x_22 = lean_usize_land(x_18, x_21); +x_23 = lean_array_uget(x_8, x_22); +lean_inc(x_23); +lean_inc(x_5); +lean_inc(x_1); +x_24 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_23); +if (x_24 == 0) +{ +lean_object* x_25; lean_object* x_26; +lean_dec(x_1); +x_25 = lean_box(0); +x_26 = lean_apply_1(x_6, x_25); +if (lean_obj_tag(x_26) == 0) +{ +lean_dec(x_23); +lean_dec(x_8); +lean_dec(x_7); +lean_dec(x_5); +lean_dec(x_2); +return x_4; +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_4); +if (x_27 == 0) +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; +x_28 = lean_ctor_get(x_4, 1); +lean_dec(x_28); +x_29 = lean_ctor_get(x_4, 0); +lean_dec(x_29); +x_30 = lean_ctor_get(x_26, 0); +lean_inc(x_30); +lean_dec(x_26); +x_31 = lean_unsigned_to_nat(1u); +x_32 = lean_nat_add(x_7, x_31); +lean_dec(x_7); +x_33 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_33, 0, x_5); +lean_ctor_set(x_33, 1, x_30); +lean_ctor_set(x_33, 2, x_23); +x_34 = lean_array_uset(x_8, x_22, x_33); +x_35 = lean_unsigned_to_nat(4u); +x_36 = lean_nat_mul(x_32, x_35); +x_37 = lean_unsigned_to_nat(3u); +x_38 = lean_nat_div(x_36, x_37); +lean_dec(x_36); +x_39 = lean_array_get_size(x_34); +x_40 = lean_nat_dec_le(x_38, x_39); +lean_dec(x_39); +lean_dec(x_38); +if (x_40 == 0) +{ +lean_object* x_41; +x_41 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_34); +lean_ctor_set(x_4, 1, x_41); +lean_ctor_set(x_4, 0, x_32); +return x_4; +} +else +{ +lean_dec(x_2); +lean_ctor_set(x_4, 1, x_34); +lean_ctor_set(x_4, 0, x_32); +return x_4; +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; +lean_dec(x_4); +x_42 = lean_ctor_get(x_26, 0); +lean_inc(x_42); +lean_dec(x_26); +x_43 = lean_unsigned_to_nat(1u); +x_44 = lean_nat_add(x_7, x_43); +lean_dec(x_7); +x_45 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_45, 0, x_5); +lean_ctor_set(x_45, 1, x_42); +lean_ctor_set(x_45, 2, x_23); +x_46 = lean_array_uset(x_8, x_22, x_45); +x_47 = lean_unsigned_to_nat(4u); +x_48 = lean_nat_mul(x_44, x_47); +x_49 = lean_unsigned_to_nat(3u); +x_50 = lean_nat_div(x_48, x_49); +lean_dec(x_48); +x_51 = lean_array_get_size(x_46); +x_52 = lean_nat_dec_le(x_50, x_51); +lean_dec(x_51); +lean_dec(x_50); +if (x_52 == 0) +{ +lean_object* x_53; lean_object* x_54; +x_53 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_46); +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_44); +lean_ctor_set(x_54, 1, x_53); +return x_54; +} +else +{ +lean_object* x_55; +lean_dec(x_2); +x_55 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_55, 0, x_44); +lean_ctor_set(x_55, 1, x_46); +return x_55; +} +} +} +} +else +{ +uint8_t x_56; +lean_dec(x_2); +x_56 = !lean_is_exclusive(x_4); +if (x_56 == 0) +{ +lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; uint8_t x_62; lean_object* x_63; +x_57 = lean_ctor_get(x_4, 1); +lean_dec(x_57); +x_58 = lean_ctor_get(x_4, 0); +lean_dec(x_58); +x_59 = lean_box(0); +x_60 = lean_array_uset(x_8, x_22, x_59); +lean_inc(x_5); +lean_inc(x_1); +x_61 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_61); +x_62 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_61); +x_63 = lean_array_uset(x_60, x_22, x_61); +if (x_62 == 0) +{ +lean_object* x_64; lean_object* x_65; +x_64 = lean_unsigned_to_nat(1u); +x_65 = lean_nat_sub(x_7, x_64); +lean_dec(x_7); +lean_ctor_set(x_4, 1, x_63); +lean_ctor_set(x_4, 0, x_65); +return x_4; +} +else +{ +lean_ctor_set(x_4, 1, x_63); +return x_4; +} +} +else +{ +lean_object* x_66; lean_object* x_67; lean_object* x_68; uint8_t x_69; lean_object* x_70; +lean_dec(x_4); +x_66 = lean_box(0); +x_67 = lean_array_uset(x_8, x_22, x_66); +lean_inc(x_5); +lean_inc(x_1); +x_68 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_5, x_6, x_23); +lean_inc(x_68); +x_69 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_5, x_68); +x_70 = lean_array_uset(x_67, x_22, x_68); +if (x_69 == 0) +{ +lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_71 = lean_unsigned_to_nat(1u); +x_72 = lean_nat_sub(x_7, x_71); +lean_dec(x_7); +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set(x_73, 1, x_70); +return x_73; +} +else +{ +lean_object* x_74; +x_74 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_74, 0, x_7); +lean_ctor_set(x_74, 1, x_70); +return x_74; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_Const_alter___rarg), 6, 0); +return x_2; +} +} LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_containsThenInsert___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/List/Associative.c b/stage0/stdlib/Std/Data/DHashMap/Internal/List/Associative.c index 50700b3dd4c4..4f31c8855900 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/List/Associative.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/List/Associative.c @@ -14,27 +14,36 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueD___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__List_filterMap_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueD(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCastD___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_eraseKey___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_insertEntryIfNew___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_alterKey(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_List_getValueCast_x21___rarg___closed__4; LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__List_filterMap_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey_x21(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_List_getValueCast_x21___rarg___closed__3; +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_alterKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_getValue_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_alterKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValue_x3f___rarg(lean_object*, lean_object*, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValue(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCast___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_getEntry_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCast(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCast_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_replaceEntry___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_List_getValueCast_x21___rarg___closed__2; static lean_object* l_Std_DHashMap_Internal_List_getValueCast_x21___rarg___closed__1; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey_x3f(lean_object*, lean_object*); @@ -47,10 +56,13 @@ LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_containsKey___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_getEntry_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_modifyKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCast_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getEntry(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_alterKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_insertEntryIfNew(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_modifyKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCastD(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValue_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_getValue_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); @@ -60,9 +72,12 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValue_x21___rarg(lean_o LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKeyD___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCastD___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_insertEntry(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_modifyKey(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getEntry___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValue___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_modifyKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getKeyD___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_getValueCast_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__List_filterMap_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_containsKey(lean_object*, lean_object*); @@ -1265,6 +1280,227 @@ lean_dec(x_2); return x_4; } } +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_alterKey___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_1); +x_6 = l_Std_DHashMap_Internal_List_getValueCast_x3f___rarg(x_1, lean_box(0), x_3, x_5); +x_7 = lean_apply_1(x_4, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +x_8 = l_Std_DHashMap_Internal_List_eraseKey___rarg(x_1, x_3, x_5); +return x_8; +} +else +{ +lean_object* x_9; lean_object* x_10; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_DHashMap_Internal_List_insertEntry___rarg(x_1, x_3, x_9, x_5); +return x_10; +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_alterKey(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_List_alterKey___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed), 3, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_alterKey_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_modifyKey___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_1); +x_6 = l_Std_DHashMap_Internal_List_getValueCast_x3f___rarg(x_1, lean_box(0), x_3, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_apply_1(x_4, x_7); +x_9 = l_Std_DHashMap_Internal_List_replaceEntry___rarg(x_1, x_3, x_8, x_5); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_modifyKey(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_List_modifyKey___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_alterKey___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; lean_object* x_6; +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_5 = l_Std_DHashMap_Internal_List_getValue_x3f___rarg(x_1, x_2, x_4); +x_6 = lean_apply_1(x_3, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; +x_7 = l_Std_DHashMap_Internal_List_eraseKey___rarg(x_1, x_2, x_4); +return x_7; +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_6, 0); +lean_inc(x_8); +lean_dec(x_6); +x_9 = l_Std_DHashMap_Internal_List_insertEntry___rarg(x_1, x_2, x_8, x_4); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_alterKey(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_List_Const_alterKey___rarg), 4, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_List_Associative_0__Std_DHashMap_Internal_List_Const_alterKey_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_modifyKey___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; +lean_inc(x_5); +lean_inc(x_3); +lean_inc(x_1); +x_6 = l_Std_DHashMap_Internal_List_getValue_x3f___rarg(x_1, x_3, x_5); +if (lean_obj_tag(x_6) == 0) +{ +lean_dec(x_4); +lean_dec(x_3); +lean_dec(x_1); +return x_5; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +lean_dec(x_6); +x_8 = lean_apply_1(x_4, x_7); +x_9 = l_Std_DHashMap_Internal_List_replaceEntry___rarg(x_1, x_3, x_8, x_5); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_List_Const_modifyKey(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_List_Const_modifyKey___rarg), 5, 0); +return x_3; +} +} lean_object* initialize_Init_Data_BEq(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_Nat_Simproc(uint8_t builtin, lean_object*); lean_object* initialize_Init_Data_List_Perm(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/Model.c b/stage0/stdlib/Std/Data/DHashMap/Internal/Model.c index eaeefc2c92cc..9837c49256f9 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/Model.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/Model.c @@ -14,8 +14,11 @@ extern "C" { #endif LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_replace_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_erase_u2098aux___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_map_u2098___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_erase_u2098aux___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_replace_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap_u2098(lean_object*, lean_object*, lean_object*); @@ -25,56 +28,73 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD_u2098___rarg(lea LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_uint64_to_usize(uint64_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_replace_u2098___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x21_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filter_u2098___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insertIfNew_u2098(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_map___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_cons_u2098___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_updateAllBuckets___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_cons_u2098(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x3f_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_withComputedSize___rarg(lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_DHashMap_Internal_AssocList_length___spec__1___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg___closed__4; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_map_u2098(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x21_u2098(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_getD_u2098(lean_object*, lean_object*); lean_object* l_panic___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_withComputedSize___spec__1(lean_object*, lean_object*); uint64_t lean_uint64_shift_right(uint64_t, uint64_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_erase_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg(size_t, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_getD_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_bucket___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insert_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filter_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_expandIfNecessary_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insert_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_cons_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_withComputedSize___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Option_map___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_erase_u2098aux(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKeyD_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t l_Std_DHashMap_Internal_AssocList_contains___rarg(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_replace___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_erase_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_contains_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg___closed__2; lean_object* l___private_Init_Util_0__mkPanicMessageWithDecl(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_insertIfNew_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -85,33 +105,39 @@ lean_object* l_Std_DHashMap_Internal_AssocList_filterMap___rarg(lean_object*, le LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKeyD_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x21_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x3f_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter(lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getCast_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg(size_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateAllBuckets___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_erase_u2098aux___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg___boxed(lean_object*, lean_object*); uint8_t lean_nat_dec_lt(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_getD_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_bucket(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_expandIfNecessary_match__1_splitter___rarg(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg___closed__1; -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_withComputedSize(lean_object*, lean_object*); uint64_t lean_uint64_xor(uint64_t, uint64_t); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_mul(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_bucket___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x21_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_filter___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_replace_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_updateAllBuckets___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); size_t lean_usize_sub(size_t, size_t); lean_object* l_Std_DHashMap_Internal_AssocList_getCast___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -122,14 +148,17 @@ lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_u2098___rarg(lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_u2098(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD_u2098(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_x21_u2098(lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg___boxed(lean_object*, lean_object*); lean_object* lean_nat_add(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getD_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -137,12 +166,14 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateAllBuckets(lean_object*, LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x3f_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_array_uset(lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_DHashMap_Internal_withComputedSize___spec__1___rarg(lean_object*, size_t, size_t, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(lean_object*, lean_object*, lean_object*); size_t lean_usize_land(size_t, size_t); lean_object* l_Std_DHashMap_Internal_AssocList_erase___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket(lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080_get_x21_u2098___rarg___closed__3; LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_getKey_u2098___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_bucket___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { @@ -1168,6 +1199,922 @@ x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_erase_u2098__ return x_3; } } +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; size_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_6 = lean_array_get_size(x_2); +x_7 = lean_apply_1(x_1, x_4); +x_8 = lean_unbox_uint64(x_7); +lean_dec(x_7); +x_9 = 32; +x_10 = lean_uint64_shift_right(x_8, x_9); +x_11 = lean_uint64_xor(x_8, x_10); +x_12 = 16; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = lean_uint64_to_usize(x_14); +x_16 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_17 = 1; +x_18 = lean_usize_sub(x_16, x_17); +x_19 = lean_usize_land(x_15, x_18); +x_20 = lean_array_uget(x_2, x_19); +x_21 = lean_apply_1(x_5, x_20); +x_22 = lean_array_uset(x_2, x_19, x_21); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +lean_inc(x_5); +lean_inc(x_2); +lean_inc(x_1); +x_7 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_4, x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_1); +x_8 = lean_box(0); +x_9 = lean_apply_1(x_6, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_dec(x_5); +lean_dec(x_2); +return x_4; +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +lean_inc(x_2); +x_11 = l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg(x_2, x_4, x_5, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_unsigned_to_nat(4u); +x_16 = lean_nat_mul(x_13, x_15); +x_17 = lean_unsigned_to_nat(3u); +x_18 = lean_nat_div(x_16, x_17); +lean_dec(x_16); +x_19 = lean_array_get_size(x_14); +x_20 = lean_nat_dec_le(x_18, x_19); +lean_dec(x_19); +lean_dec(x_18); +if (x_20 == 0) +{ +lean_object* x_21; +x_21 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_14); +lean_ctor_set(x_11, 1, x_21); +return x_11; +} +else +{ +lean_dec(x_2); +return x_11; +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_22 = lean_ctor_get(x_11, 0); +x_23 = lean_ctor_get(x_11, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_11); +x_24 = lean_unsigned_to_nat(4u); +x_25 = lean_nat_mul(x_22, x_24); +x_26 = lean_unsigned_to_nat(3u); +x_27 = lean_nat_div(x_25, x_26); +lean_dec(x_25); +x_28 = lean_array_get_size(x_23); +x_29 = lean_nat_dec_le(x_27, x_28); +lean_dec(x_28); +lean_dec(x_27); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_23); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_22); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +else +{ +lean_object* x_32; +lean_dec(x_2); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_22); +lean_ctor_set(x_32, 1, x_23); +return x_32; +} +} +} +} +else +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_4); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_34 = lean_ctor_get(x_4, 0); +x_35 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_inc(x_1); +x_36 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_alter___rarg), 5, 4); +lean_closure_set(x_36, 0, x_1); +lean_closure_set(x_36, 1, lean_box(0)); +lean_closure_set(x_36, 2, x_5); +lean_closure_set(x_36, 3, x_6); +lean_inc(x_5); +lean_inc(x_2); +x_37 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1___rarg(x_2, x_35, lean_box(0), x_5, x_36); +lean_inc(x_37); +x_38 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_37); +x_39 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_38, x_5); +lean_dec(x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +x_40 = lean_unsigned_to_nat(1u); +x_41 = lean_nat_sub(x_34, x_40); +lean_dec(x_34); +lean_ctor_set(x_4, 1, x_37); +lean_ctor_set(x_4, 0, x_41); +return x_4; +} +else +{ +lean_ctor_set(x_4, 1, x_37); +return x_4; +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_42 = lean_ctor_get(x_4, 0); +x_43 = lean_ctor_get(x_4, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_4); +lean_inc(x_5); +lean_inc(x_1); +x_44 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_alter___rarg), 5, 4); +lean_closure_set(x_44, 0, x_1); +lean_closure_set(x_44, 1, lean_box(0)); +lean_closure_set(x_44, 2, x_5); +lean_closure_set(x_44, 3, x_6); +lean_inc(x_5); +lean_inc(x_2); +x_45 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_alter_u2098___spec__1___rarg(x_2, x_43, lean_box(0), x_5, x_44); +lean_inc(x_45); +x_46 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_45); +x_47 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_46, x_5); +lean_dec(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_unsigned_to_nat(1u); +x_49 = lean_nat_sub(x_42, x_48); +lean_dec(x_42); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_45); +return x_50; +} +else +{ +lean_object* x_51; +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_42); +lean_ctor_set(x_51, 1, x_45); +return x_51; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___rarg), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; size_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_6 = lean_array_get_size(x_2); +x_7 = lean_apply_1(x_1, x_4); +x_8 = lean_unbox_uint64(x_7); +lean_dec(x_7); +x_9 = 32; +x_10 = lean_uint64_shift_right(x_8, x_9); +x_11 = lean_uint64_xor(x_8, x_10); +x_12 = 16; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = lean_uint64_to_usize(x_14); +x_16 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_17 = 1; +x_18 = lean_usize_sub(x_16, x_17); +x_19 = lean_usize_land(x_15, x_18); +x_20 = lean_array_uget(x_2, x_19); +x_21 = lean_apply_1(x_5, x_20); +x_22 = lean_array_uset(x_2, x_19, x_21); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +uint8_t x_7; +lean_inc(x_5); +lean_inc(x_2); +lean_inc(x_1); +x_7 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_4, x_5); +if (x_7 == 0) +{ +lean_object* x_8; lean_object* x_9; +lean_dec(x_1); +x_8 = lean_box(0); +x_9 = lean_apply_1(x_6, x_8); +if (lean_obj_tag(x_9) == 0) +{ +lean_dec(x_5); +lean_dec(x_2); +return x_4; +} +else +{ +lean_object* x_10; lean_object* x_11; uint8_t x_12; +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +lean_dec(x_9); +lean_inc(x_2); +x_11 = l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg(x_2, x_4, x_5, x_10); +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; +x_13 = lean_ctor_get(x_11, 0); +x_14 = lean_ctor_get(x_11, 1); +x_15 = lean_unsigned_to_nat(4u); +x_16 = lean_nat_mul(x_13, x_15); +x_17 = lean_unsigned_to_nat(3u); +x_18 = lean_nat_div(x_16, x_17); +lean_dec(x_16); +x_19 = lean_array_get_size(x_14); +x_20 = lean_nat_dec_le(x_18, x_19); +lean_dec(x_19); +lean_dec(x_18); +if (x_20 == 0) +{ +lean_object* x_21; +x_21 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_14); +lean_ctor_set(x_11, 1, x_21); +return x_11; +} +else +{ +lean_dec(x_2); +return x_11; +} +} +else +{ +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; uint8_t x_29; +x_22 = lean_ctor_get(x_11, 0); +x_23 = lean_ctor_get(x_11, 1); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_11); +x_24 = lean_unsigned_to_nat(4u); +x_25 = lean_nat_mul(x_22, x_24); +x_26 = lean_unsigned_to_nat(3u); +x_27 = lean_nat_div(x_25, x_26); +lean_dec(x_25); +x_28 = lean_array_get_size(x_23); +x_29 = lean_nat_dec_le(x_27, x_28); +lean_dec(x_28); +lean_dec(x_27); +if (x_29 == 0) +{ +lean_object* x_30; lean_object* x_31; +x_30 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_23); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_22); +lean_ctor_set(x_31, 1, x_30); +return x_31; +} +else +{ +lean_object* x_32; +lean_dec(x_2); +x_32 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_32, 0, x_22); +lean_ctor_set(x_32, 1, x_23); +return x_32; +} +} +} +} +else +{ +uint8_t x_33; +x_33 = !lean_is_exclusive(x_4); +if (x_33 == 0) +{ +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; +x_34 = lean_ctor_get(x_4, 0); +x_35 = lean_ctor_get(x_4, 1); +lean_inc(x_5); +lean_inc(x_1); +x_36 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_alter___rarg), 5, 4); +lean_closure_set(x_36, 0, x_1); +lean_closure_set(x_36, 1, lean_box(0)); +lean_closure_set(x_36, 2, x_5); +lean_closure_set(x_36, 3, x_6); +lean_inc(x_5); +lean_inc(x_2); +x_37 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2___rarg(x_2, x_35, lean_box(0), x_5, x_36); +lean_inc(x_37); +x_38 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_37); +x_39 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_38, x_5); +lean_dec(x_38); +if (x_39 == 0) +{ +lean_object* x_40; lean_object* x_41; +x_40 = lean_unsigned_to_nat(1u); +x_41 = lean_nat_sub(x_34, x_40); +lean_dec(x_34); +lean_ctor_set(x_4, 1, x_37); +lean_ctor_set(x_4, 0, x_41); +return x_4; +} +else +{ +lean_ctor_set(x_4, 1, x_37); +return x_4; +} +} +else +{ +lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; uint8_t x_47; +x_42 = lean_ctor_get(x_4, 0); +x_43 = lean_ctor_get(x_4, 1); +lean_inc(x_43); +lean_inc(x_42); +lean_dec(x_4); +lean_inc(x_5); +lean_inc(x_1); +x_44 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_alter___rarg), 5, 4); +lean_closure_set(x_44, 0, x_1); +lean_closure_set(x_44, 1, lean_box(0)); +lean_closure_set(x_44, 2, x_5); +lean_closure_set(x_44, 3, x_6); +lean_inc(x_5); +lean_inc(x_2); +x_45 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__2___rarg(x_2, x_43, lean_box(0), x_5, x_44); +lean_inc(x_45); +x_46 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_45); +x_47 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_46, x_5); +lean_dec(x_46); +if (x_47 == 0) +{ +lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_48 = lean_unsigned_to_nat(1u); +x_49 = lean_nat_sub(x_42, x_48); +lean_dec(x_42); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_45); +return x_50; +} +else +{ +lean_object* x_51; +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_42); +lean_ctor_set(x_51, 1, x_45); +return x_51; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1___rarg), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify_u2098___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6) { +_start: +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_alloc_closure((void*)(l_Option_map___rarg), 2, 1); +lean_closure_set(x_7, 0, x_6); +x_8 = l_Std_DHashMap_Internal_Raw_u2080_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_modify_u2098___spec__1___rarg(x_1, x_2, lean_box(0), x_4, x_5, x_7); +return x_8; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_modify_u2098(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_modify_u2098___rarg), 6, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; size_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_6 = lean_array_get_size(x_2); +x_7 = lean_apply_1(x_1, x_4); +x_8 = lean_unbox_uint64(x_7); +lean_dec(x_7); +x_9 = 32; +x_10 = lean_uint64_shift_right(x_8, x_9); +x_11 = lean_uint64_xor(x_8, x_10); +x_12 = 16; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = lean_uint64_to_usize(x_14); +x_16 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_17 = 1; +x_18 = lean_usize_sub(x_16, x_17); +x_19 = lean_usize_land(x_15, x_18); +x_20 = lean_array_uget(x_2, x_19); +x_21 = lean_apply_1(x_5, x_20); +x_22 = lean_array_uset(x_2, x_19, x_21); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_6 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_3, x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +lean_dec(x_1); +x_7 = lean_box(0); +x_8 = lean_apply_1(x_5, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_dec(x_4); +lean_dec(x_2); +return x_3; +} +else +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +lean_inc(x_2); +x_10 = l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg(x_2, x_3, x_4, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_unsigned_to_nat(4u); +x_15 = lean_nat_mul(x_12, x_14); +x_16 = lean_unsigned_to_nat(3u); +x_17 = lean_nat_div(x_15, x_16); +lean_dec(x_15); +x_18 = lean_array_get_size(x_13); +x_19 = lean_nat_dec_le(x_17, x_18); +lean_dec(x_18); +lean_dec(x_17); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_13); +lean_ctor_set(x_10, 1, x_20); +return x_10; +} +else +{ +lean_dec(x_2); +return x_10; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_10, 0); +x_22 = lean_ctor_get(x_10, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_10); +x_23 = lean_unsigned_to_nat(4u); +x_24 = lean_nat_mul(x_21, x_23); +x_25 = lean_unsigned_to_nat(3u); +x_26 = lean_nat_div(x_24, x_25); +lean_dec(x_24); +x_27 = lean_array_get_size(x_22); +x_28 = lean_nat_dec_le(x_26, x_27); +lean_dec(x_27); +lean_dec(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_22); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_21); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +else +{ +lean_object* x_31; +lean_dec(x_2); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_21); +lean_ctor_set(x_31, 1, x_22); +return x_31; +} +} +} +} +else +{ +uint8_t x_32; +x_32 = !lean_is_exclusive(x_3); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_33 = lean_ctor_get(x_3, 0); +x_34 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_inc(x_1); +x_35 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___rarg), 5, 4); +lean_closure_set(x_35, 0, x_1); +lean_closure_set(x_35, 1, lean_box(0)); +lean_closure_set(x_35, 2, x_4); +lean_closure_set(x_35, 3, x_5); +lean_inc(x_4); +lean_inc(x_2); +x_36 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1___rarg(x_2, x_34, lean_box(0), x_4, x_35); +lean_inc(x_36); +x_37 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_36); +x_38 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_37, x_4); +lean_dec(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_unsigned_to_nat(1u); +x_40 = lean_nat_sub(x_33, x_39); +lean_dec(x_33); +lean_ctor_set(x_3, 1, x_36); +lean_ctor_set(x_3, 0, x_40); +return x_3; +} +else +{ +lean_ctor_set(x_3, 1, x_36); +return x_3; +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_41 = lean_ctor_get(x_3, 0); +x_42 = lean_ctor_get(x_3, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_3); +lean_inc(x_4); +lean_inc(x_1); +x_43 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___rarg), 5, 4); +lean_closure_set(x_43, 0, x_1); +lean_closure_set(x_43, 1, lean_box(0)); +lean_closure_set(x_43, 2, x_4); +lean_closure_set(x_43, 3, x_5); +lean_inc(x_4); +lean_inc(x_2); +x_44 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___spec__1___rarg(x_2, x_42, lean_box(0), x_4, x_43); +lean_inc(x_44); +x_45 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_44); +x_46 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_45, x_4); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_unsigned_to_nat(1u); +x_48 = lean_nat_sub(x_41, x_47); +lean_dec(x_41); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_44); +return x_49; +} +else +{ +lean_object* x_50; +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_41); +lean_ctor_set(x_50, 1, x_44); +return x_50; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; uint64_t x_8; uint64_t x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; size_t x_15; size_t x_16; size_t x_17; size_t x_18; size_t x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_6 = lean_array_get_size(x_2); +x_7 = lean_apply_1(x_1, x_4); +x_8 = lean_unbox_uint64(x_7); +lean_dec(x_7); +x_9 = 32; +x_10 = lean_uint64_shift_right(x_8, x_9); +x_11 = lean_uint64_xor(x_8, x_10); +x_12 = 16; +x_13 = lean_uint64_shift_right(x_11, x_12); +x_14 = lean_uint64_xor(x_11, x_13); +x_15 = lean_uint64_to_usize(x_14); +x_16 = lean_usize_of_nat(x_6); +lean_dec(x_6); +x_17 = 1; +x_18 = lean_usize_sub(x_16, x_17); +x_19 = lean_usize_land(x_15, x_18); +x_20 = lean_array_uget(x_2, x_19); +x_21 = lean_apply_1(x_5, x_20); +x_22 = lean_array_uset(x_2, x_19, x_21); +return x_22; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +uint8_t x_6; +lean_inc(x_4); +lean_inc(x_2); +lean_inc(x_1); +x_6 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_3, x_4); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +lean_dec(x_1); +x_7 = lean_box(0); +x_8 = lean_apply_1(x_5, x_7); +if (lean_obj_tag(x_8) == 0) +{ +lean_dec(x_4); +lean_dec(x_2); +return x_3; +} +else +{ +lean_object* x_9; lean_object* x_10; uint8_t x_11; +x_9 = lean_ctor_get(x_8, 0); +lean_inc(x_9); +lean_dec(x_8); +lean_inc(x_2); +x_10 = l_Std_DHashMap_Internal_Raw_u2080_cons_u2098___rarg(x_2, x_3, x_4, x_9); +x_11 = !lean_is_exclusive(x_10); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint8_t x_19; +x_12 = lean_ctor_get(x_10, 0); +x_13 = lean_ctor_get(x_10, 1); +x_14 = lean_unsigned_to_nat(4u); +x_15 = lean_nat_mul(x_12, x_14); +x_16 = lean_unsigned_to_nat(3u); +x_17 = lean_nat_div(x_15, x_16); +lean_dec(x_15); +x_18 = lean_array_get_size(x_13); +x_19 = lean_nat_dec_le(x_17, x_18); +lean_dec(x_18); +lean_dec(x_17); +if (x_19 == 0) +{ +lean_object* x_20; +x_20 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_13); +lean_ctor_set(x_10, 1, x_20); +return x_10; +} +else +{ +lean_dec(x_2); +return x_10; +} +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; uint8_t x_28; +x_21 = lean_ctor_get(x_10, 0); +x_22 = lean_ctor_get(x_10, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_10); +x_23 = lean_unsigned_to_nat(4u); +x_24 = lean_nat_mul(x_21, x_23); +x_25 = lean_unsigned_to_nat(3u); +x_26 = lean_nat_div(x_24, x_25); +lean_dec(x_24); +x_27 = lean_array_get_size(x_22); +x_28 = lean_nat_dec_le(x_26, x_27); +lean_dec(x_27); +lean_dec(x_26); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +x_29 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_22); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_21); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +else +{ +lean_object* x_31; +lean_dec(x_2); +x_31 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_31, 0, x_21); +lean_ctor_set(x_31, 1, x_22); +return x_31; +} +} +} +} +else +{ +uint8_t x_32; +x_32 = !lean_is_exclusive(x_3); +if (x_32 == 0) +{ +lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; uint8_t x_38; +x_33 = lean_ctor_get(x_3, 0); +x_34 = lean_ctor_get(x_3, 1); +lean_inc(x_4); +lean_inc(x_1); +x_35 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___rarg), 5, 4); +lean_closure_set(x_35, 0, x_1); +lean_closure_set(x_35, 1, lean_box(0)); +lean_closure_set(x_35, 2, x_4); +lean_closure_set(x_35, 3, x_5); +lean_inc(x_4); +lean_inc(x_2); +x_36 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2___rarg(x_2, x_34, lean_box(0), x_4, x_35); +lean_inc(x_36); +x_37 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_36); +x_38 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_37, x_4); +lean_dec(x_37); +if (x_38 == 0) +{ +lean_object* x_39; lean_object* x_40; +x_39 = lean_unsigned_to_nat(1u); +x_40 = lean_nat_sub(x_33, x_39); +lean_dec(x_33); +lean_ctor_set(x_3, 1, x_36); +lean_ctor_set(x_3, 0, x_40); +return x_3; +} +else +{ +lean_ctor_set(x_3, 1, x_36); +return x_3; +} +} +else +{ +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; uint8_t x_46; +x_41 = lean_ctor_get(x_3, 0); +x_42 = lean_ctor_get(x_3, 1); +lean_inc(x_42); +lean_inc(x_41); +lean_dec(x_3); +lean_inc(x_4); +lean_inc(x_1); +x_43 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___rarg), 5, 4); +lean_closure_set(x_43, 0, x_1); +lean_closure_set(x_43, 1, lean_box(0)); +lean_closure_set(x_43, 2, x_4); +lean_closure_set(x_43, 3, x_5); +lean_inc(x_4); +lean_inc(x_2); +x_44 = l_Std_DHashMap_Internal_updateBucket___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__2___rarg(x_2, x_42, lean_box(0), x_4, x_43); +lean_inc(x_44); +x_45 = l_Std_DHashMap_Internal_withComputedSize___rarg(x_44); +x_46 = l_Std_DHashMap_Internal_Raw_u2080_contains_u2098___rarg(x_1, x_2, x_45, x_4); +lean_dec(x_45); +if (x_46 == 0) +{ +lean_object* x_47; lean_object* x_48; lean_object* x_49; +x_47 = lean_unsigned_to_nat(1u); +x_48 = lean_nat_sub(x_41, x_47); +lean_dec(x_41); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_44); +return x_49; +} +else +{ +lean_object* x_50; +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_41); +lean_ctor_set(x_50, 1, x_44); +return x_50; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1___rarg), 5, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +_start: +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_alloc_closure((void*)(l_Option_map___rarg), 2, 1); +lean_closure_set(x_6, 0, x_5); +x_7 = l_Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098___at_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___spec__1___rarg(x_1, x_2, x_3, x_4, x_6); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_Raw_u2080_Const_modify_u2098___rarg), 5, 0); +return x_3; +} +} LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_Raw_u2080_filterMap_u2098___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -1408,74 +2355,146 @@ x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0_ return x_4; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg(size_t x_1, lean_object* x_2) { _start: { -if (lean_obj_tag(x_1) == 0) +lean_object* x_3; lean_object* x_4; +x_3 = lean_box_usize(x_1); +x_4 = lean_apply_2(x_2, x_3, lean_box(0)); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg___boxed), 2, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +size_t x_3; lean_object* x_4; +x_3 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___rarg(x_3, x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: { +lean_object* x_5; +x_5 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__1_splitter(x_1, x_2, x_3, x_4); lean_dec(x_3); -lean_inc(x_2); -return x_2; +return x_5; } -else +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_4; lean_object* x_5; -x_4 = lean_ctor_get(x_1, 0); +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_ctor_get(x_1, 0); +lean_inc(x_3); +x_4 = lean_ctor_get(x_1, 1); lean_inc(x_4); lean_dec(x_1); -x_5 = lean_apply_1(x_3, x_4); +x_5 = lean_apply_3(x_2, x_3, x_4, lean_box(0)); return x_5; } } +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg), 2, 0); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg(size_t x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; +x_3 = lean_box_usize(x_1); +x_4 = lean_apply_2(x_2, x_3, lean_box(0)); +return x_4; +} } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed), 3, 0); +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg___boxed), 2, 0); return x_5; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_4; -x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___rarg(x_1, x_2, x_3); -lean_dec(x_2); +size_t x_3; lean_object* x_4; +x_3 = lean_unbox_usize(x_1); +lean_dec(x_1); +x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___rarg(x_3, x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { lean_object* x_5; -x_5 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_getThenInsertIfNew_x3f_match__1_splitter(x_1, x_2, x_3, x_4); +x_5 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__1_splitter(x_1, x_2, x_3, x_4); lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); -x_4 = lean_ctor_get(x_1, 1); +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); lean_inc(x_4); lean_dec(x_1); -x_5 = lean_apply_3(x_2, x_3, x_4, lean_box(0)); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg___boxed), 3, 0); return x_5; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg), 2, 0); +x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); return x_4; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_alter_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { if (lean_obj_tag(x_1) == 0) @@ -1495,19 +2514,19 @@ return x_5; } } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed), 3, 0); +x_3 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg___boxed), 3, 0); return x_3; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_getThenInsertIfNew_x3f_match__1_splitter___rarg(x_1, x_2, x_3); +x_4 = l___private_Std_Data_DHashMap_Internal_Model_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_match__1_splitter___rarg(x_1, x_2, x_3); lean_dec(x_2); return x_4; } diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/RawLemmas.c b/stage0/stdlib/Std/Data/DHashMap/Internal/RawLemmas.c index a11483f10184..7ce9e8e4b6f5 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/RawLemmas.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/RawLemmas.c @@ -29,6 +29,7 @@ static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHas static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticWf__trivial__1___closed__20; lean_object* lean_mk_empty_array_with_capacity(lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticEmpty__1___closed__1; +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_queryNames___closed__1; static lean_object* l_Std_DHashMap_Internal_Raw_u2080_tacticWf__trivial___closed__6; static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticEmpty__1___closed__22; @@ -163,7 +164,6 @@ static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticWf__trivial__1___closed__64; static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_congrNames___closed__67; static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_congrNames___closed__25; -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_mapMUnsafe_map___at_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticSimp__to__modelUsing____1___spec__7(lean_object*, size_t, size_t, lean_object*); static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_queryNames___closed__49; static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_congrNames___closed__45; @@ -173,6 +173,7 @@ static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap static lean_object* l_Std_DHashMap_Internal_Raw_u2080_tacticWf__trivial___closed__2; static lean_object* l_Std_DHashMap_Internal_Raw_u2080_tacticEmpty___closed__5; static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_queryNames___closed__50; +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg(lean_object*, lean_object*); static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_queryNames___closed__18; static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_queryNames___closed__46; static lean_object* l_Std_DHashMap_Internal_Raw_u2080_tacticSimp__to__modelUsing_____closed__6; @@ -329,7 +330,6 @@ static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHas static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticEmpty__1___closed__19; lean_object* l_Lean_Syntax_node8(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_DHashMap_Internal_Raw_u2080___aux__Std__Data__DHashMap__Internal__RawLemmas______macroRules__Std__DHashMap__Internal__Raw_u2080__tacticWf__trivial__1___closed__38; -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg(lean_object*, lean_object*); static lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_congrNames___closed__75; lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); @@ -5648,7 +5648,7 @@ x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_RawLemma return x_4; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; @@ -5661,11 +5661,11 @@ x_5 = lean_apply_3(x_2, x_3, x_4, lean_box(0)); return x_5; } } -LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { lean_object* x_4; -x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_get_x3f_match__2_splitter___rarg), 2, 0); +x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_RawLemmas_0__Std_DHashMap_Internal_Raw_u2080_Const_modify_match__2_splitter___rarg), 2, 0); return x_4; } } diff --git a/stage0/stdlib/Std/Data/DHashMap/Internal/WF.c b/stage0/stdlib/Std/Data/DHashMap/Internal/WF.c index 16dff3fa92e0..0ddbbd298e03 100644 --- a/stage0/stdlib/Std/Data/DHashMap/Internal/WF.c +++ b/stage0/stdlib/Std/Data/DHashMap/Internal/WF.c @@ -13,10 +13,17 @@ #ifdef __cplusplus extern "C" { #endif +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_expandIfNecessary_match__1_splitter___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__2_splitter(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_expandIfNecessary_match__1_splitter(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__2_splitter___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter(lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_reinsertAux_match__2_splitter___rarg(lean_object* x_1, lean_object* x_2) { _start: { @@ -54,6 +61,89 @@ x_4 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_WF_0__St return x_4; } } +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg___boxed), 3, 0); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +_start: +{ +lean_object* x_5; +x_5 = l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_alter_u2098_match__1_splitter(x_1, x_2, x_3, x_4); +lean_dec(x_3); +return x_5; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_1) == 0) +{ +lean_dec(x_3); +lean_inc(x_2); +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_1, 0); +lean_inc(x_4); +lean_dec(x_1); +x_5 = lean_apply_1(x_3, x_4); +return x_5; +} +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg___boxed), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l___private_Std_Data_DHashMap_Internal_WF_0__Std_DHashMap_Internal_Raw_u2080_Const_alter_u2098_match__1_splitter___rarg(x_1, x_2, x_3); +lean_dec(x_2); +return x_4; +} +} lean_object* initialize_Std_Data_DHashMap_Basic(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_DHashMap_Internal_Model(uint8_t builtin, lean_object*); lean_object* initialize_Std_Data_DHashMap_Internal_AssocList_Lemmas(uint8_t builtin, lean_object*); diff --git a/stage0/stdlib/Std/Data/HashMap/Basic.c b/stage0/stdlib/Std/Data/HashMap/Basic.c index 3e2bb5b2a746..5cffa9bbb2ef 100644 --- a/stage0/stdlib/Std/Data/HashMap/Basic.c +++ b/stage0/stdlib/Std/Data/HashMap/Basic.c @@ -60,8 +60,10 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_instRepr___s LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_partition___spec__2(lean_object*, lean_object*); uint8_t lean_usize_dec_eq(size_t, size_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_forM___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___lambda__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insertIfNew___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_toArray___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_instRepr___spec__7(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_instRepr___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldrM___at_Std_HashMap_keys___spec__1___rarg(lean_object*, lean_object*); @@ -85,6 +87,7 @@ LEAN_EXPORT lean_object* l_Std_HashMap_partition___rarg___boxed(lean_object*, le LEAN_EXPORT lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__13(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_empty(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__4(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_toArray___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_erase___rarg(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Nat_nextPowerOfTwo_go(lean_object*, lean_object*, lean_object*); @@ -131,6 +134,7 @@ LEAN_EXPORT lean_object* l_Std_HashMap_toList(lean_object*, lean_object*, lean_o size_t lean_usize_of_nat(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_Internal_numBuckets(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_find_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_repr___at_Std_HashMap_instRepr___spec__9(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__8(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_instForMProd___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); @@ -140,6 +144,7 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashM LEAN_EXPORT lean_object* l_Std_HashMap_unitOfArray(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getKey_x3f___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_groupByKey___rarg(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_erase(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_HashMap_instForInProd___spec__2___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_find_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); @@ -154,8 +159,10 @@ LEAN_EXPORT lean_object* l_Std_HashMap_keys(lean_object*, lean_object*, lean_obj LEAN_EXPORT lean_object* l_Std_HashMap_filter___boxed(lean_object*, lean_object*, lean_object*, lean_object*); lean_object* lean_nat_div(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_ofList(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__2(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_HashMap_isEmpty___rarg(lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_instRepr___spec__18___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_instInsertProd(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Std_HashMap_instRepr___spec__17(lean_object*, lean_object*); @@ -196,7 +203,6 @@ LEAN_EXPORT lean_object* l_Std_HashMap_instRepr___rarg___boxed(lean_object*, lea LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getThenInsertIfNew_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getKey_x21(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_containsThenInsert(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_forM___spec__2___rarg(lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_instRepr___spec__18___rarg(lean_object*, size_t, size_t, lean_object*); @@ -213,7 +219,6 @@ LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashM static lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__2___rarg___closed__8; LEAN_EXPORT lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__8___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_fold___spec__1(lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); static lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__4___rarg___closed__9; LEAN_EXPORT lean_object* l_Std_HashMap_forIn___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_union___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); @@ -239,6 +244,7 @@ LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_toList___spe LEAN_EXPORT lean_object* l_Std_HashMap_toList___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_repr___at_Std_HashMap_instRepr___spec__20(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__15(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_fold___rarg(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_values___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_instEmptyCollection___boxed(lean_object*, lean_object*, lean_object*, lean_object*); @@ -248,6 +254,7 @@ LEAN_EXPORT lean_object* l_Std_HashMap_getD___rarg(lean_object*, lean_object*, l LEAN_EXPORT lean_object* l_Std_HashMap_contains___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_instDecidableMem(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_repr___at_Std_HashMap_instRepr___spec__3___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_empty___rarg(lean_object*); static lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__4___rarg___closed__1; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_HashMap_forIn___spec__1(lean_object*, lean_object*, lean_object*); @@ -255,15 +262,17 @@ LEAN_EXPORT lean_object* l_Array_foldlMUnsafe_fold___at_Std_HashMap_keysArray___ LEAN_EXPORT lean_object* l_Std_HashMap_unitOfList(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_get_x3f(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insertManyIfNewUnit___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_keys___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg(lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_HashMap_forIn___spec__1___rarg___lambda__1(lean_object*, size_t, lean_object*, lean_object*, lean_object*, lean_object*, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_forM(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_forInStep_go___at_Std_HashMap_instForInProd___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insertIfNew(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_isEmpty___rarg___boxed(lean_object*); lean_object* lean_string_length(lean_object*); LEAN_EXPORT lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__10___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); +lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); lean_object* l_Std_DHashMap_Internal_AssocList_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_size(lean_object*, lean_object*, lean_object*, lean_object*); @@ -286,7 +295,6 @@ LEAN_EXPORT lean_object* l_Std_HashMap_containsThenInsert___rarg(lean_object*, l static lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__4___rarg___closed__6; LEAN_EXPORT lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__21___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_HashMap_instForInProd___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); -LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getKey_x3f___rarg(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_toList___spec__3(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getKey_x3f(lean_object*, lean_object*); @@ -336,7 +344,6 @@ LEAN_EXPORT lean_object* l_Std_HashMap_empty___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_foldl___at_Std_HashMap_instRepr___spec__23___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_toArray(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_valuesArray___spec__1___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1(lean_object*, lean_object*); size_t lean_usize_add(size_t, size_t); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldrM___at_Std_HashMap_values___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__2(lean_object*, lean_object*); @@ -353,6 +360,7 @@ LEAN_EXPORT lean_object* l_List_forIn_x27_loop___at_Std_HashMap_unitOfList___spe LEAN_EXPORT lean_object* l_Std_HashMap_get_x21___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_valuesArray___rarg(lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insertManyIfNewUnit___rarg___lambda__1(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_toArray___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_instForMProd___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_HashMap_instRepr___rarg___closed__2; @@ -361,7 +369,7 @@ LEAN_EXPORT lean_object* l_Std_HashMap_findD___rarg(lean_object*, lean_object*, LEAN_EXPORT lean_object* l_Std_HashMap_valuesArray___rarg___boxed(lean_object*); LEAN_EXPORT lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__19(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_toArray___spec__1___rarg(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_HashMap_forIn___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_getD(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_repr___at_Std_HashMap_instRepr___spec__3(lean_object*, lean_object*); @@ -371,6 +379,7 @@ lean_object* l_Std_DHashMap_Internal_AssocList_filter_go___rarg(lean_object*, le lean_object* lean_array_get_size(lean_object*); LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_Std_HashMap_toList___spec__2___rarg(lean_object*, size_t, size_t, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_instUnion___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1(lean_object*); static lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__2___rarg___closed__3; static lean_object* l_Std_HashMap_instEmptyCollection___closed__2; static lean_object* l_Std_HashMap_partition___rarg___closed__1; @@ -381,7 +390,6 @@ static lean_object* l_List_repr___at_Std_HashMap_instRepr___spec__2___rarg___clo LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_foldlM___at_Std_HashMap_forM___spec__1(lean_object*, lean_object*, lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); LEAN_EXPORT lean_object* l_Std_HashMap_instSingletonProd(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__1___rarg(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Prod_repr___at_Std_HashMap_instRepr___spec__4___rarg___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_insert(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_HashMap_toArray___rarg(lean_object*); @@ -6161,13 +6169,12 @@ return x_5; LEAN_EXPORT lean_object* l_Std_HashMap_modify___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; uint8_t x_23; x_6 = lean_ctor_get(x_3, 0); lean_inc(x_6); x_7 = lean_ctor_get(x_3, 1); lean_inc(x_7); x_8 = lean_array_get_size(x_7); -lean_inc(x_2); lean_inc(x_4); x_9 = lean_apply_1(x_2, x_4); x_10 = lean_unbox_uint64(x_9); @@ -6188,15 +6195,14 @@ x_22 = lean_array_uget(x_7, x_21); lean_inc(x_22); lean_inc(x_4); lean_inc(x_1); -x_23 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_4, x_22); -if (lean_obj_tag(x_23) == 0) +x_23 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); +if (x_23 == 0) { lean_dec(x_22); lean_dec(x_7); lean_dec(x_6); lean_dec(x_5); lean_dec(x_4); -lean_dec(x_2); lean_dec(x_1); return x_3; } @@ -6206,315 +6212,30 @@ uint8_t x_24; x_24 = !lean_is_exclusive(x_3); if (x_24 == 0) { -lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_81; +lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; x_25 = lean_ctor_get(x_3, 1); lean_dec(x_25); x_26 = lean_ctor_get(x_3, 0); lean_dec(x_26); -x_27 = lean_ctor_get(x_23, 0); -lean_inc(x_27); -lean_dec(x_23); -x_28 = lean_apply_1(x_5, x_27); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_81 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_81 == 0) -{ -lean_dec(x_22); -x_29 = x_3; -goto block_80; -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; -x_82 = lean_box(0); -x_83 = lean_array_uset(x_7, x_21, x_82); -x_84 = lean_unsigned_to_nat(1u); -x_85 = lean_nat_sub(x_6, x_84); -lean_dec(x_6); -lean_inc(x_4); -lean_inc(x_1); -x_86 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_87 = lean_array_uset(x_83, x_21, x_86); -lean_ctor_set(x_3, 1, x_87); -lean_ctor_set(x_3, 0, x_85); -x_29 = x_3; -goto block_80; -} -block_80: -{ -uint8_t x_30; -x_30 = !lean_is_exclusive(x_29); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; size_t x_34; size_t x_35; size_t x_36; lean_object* x_37; uint8_t x_38; -x_31 = lean_ctor_get(x_29, 0); -x_32 = lean_ctor_get(x_29, 1); -x_33 = lean_array_get_size(x_32); -x_34 = lean_usize_of_nat(x_33); -lean_dec(x_33); -x_35 = lean_usize_sub(x_34, x_19); -x_36 = lean_usize_land(x_17, x_35); -x_37 = lean_array_uget(x_32, x_36); -lean_inc(x_37); -lean_inc(x_4); -lean_inc(x_1); -x_38 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_37); -if (x_38 == 0) -{ -lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; uint8_t x_48; -lean_dec(x_1); -x_39 = lean_unsigned_to_nat(1u); -x_40 = lean_nat_add(x_31, x_39); -lean_dec(x_31); -x_41 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_41, 0, x_4); -lean_ctor_set(x_41, 1, x_28); -lean_ctor_set(x_41, 2, x_37); -x_42 = lean_array_uset(x_32, x_36, x_41); -x_43 = lean_unsigned_to_nat(4u); -x_44 = lean_nat_mul(x_40, x_43); -x_45 = lean_unsigned_to_nat(3u); -x_46 = lean_nat_div(x_44, x_45); -lean_dec(x_44); -x_47 = lean_array_get_size(x_42); -x_48 = lean_nat_dec_le(x_46, x_47); -lean_dec(x_47); -lean_dec(x_46); -if (x_48 == 0) -{ -lean_object* x_49; -x_49 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_42); -lean_ctor_set(x_29, 1, x_49); -lean_ctor_set(x_29, 0, x_40); -return x_29; -} -else -{ -lean_dec(x_2); -lean_ctor_set(x_29, 1, x_42); -lean_ctor_set(x_29, 0, x_40); -return x_29; -} -} -else -{ -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; -lean_dec(x_2); -x_50 = lean_box(0); -x_51 = lean_array_uset(x_32, x_36, x_50); -x_52 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_28, x_37); -x_53 = lean_array_uset(x_51, x_36, x_52); -lean_ctor_set(x_29, 1, x_53); -return x_29; -} -} -else -{ -lean_object* x_54; lean_object* x_55; lean_object* x_56; size_t x_57; size_t x_58; size_t x_59; lean_object* x_60; uint8_t x_61; -x_54 = lean_ctor_get(x_29, 0); -x_55 = lean_ctor_get(x_29, 1); -lean_inc(x_55); -lean_inc(x_54); -lean_dec(x_29); -x_56 = lean_array_get_size(x_55); -x_57 = lean_usize_of_nat(x_56); -lean_dec(x_56); -x_58 = lean_usize_sub(x_57, x_19); -x_59 = lean_usize_land(x_17, x_58); -x_60 = lean_array_uget(x_55, x_59); -lean_inc(x_60); -lean_inc(x_4); -lean_inc(x_1); -x_61 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_60); -if (x_61 == 0) -{ -lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; uint8_t x_71; -lean_dec(x_1); -x_62 = lean_unsigned_to_nat(1u); -x_63 = lean_nat_add(x_54, x_62); -lean_dec(x_54); -x_64 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_64, 0, x_4); -lean_ctor_set(x_64, 1, x_28); -lean_ctor_set(x_64, 2, x_60); -x_65 = lean_array_uset(x_55, x_59, x_64); -x_66 = lean_unsigned_to_nat(4u); -x_67 = lean_nat_mul(x_63, x_66); -x_68 = lean_unsigned_to_nat(3u); -x_69 = lean_nat_div(x_67, x_68); -lean_dec(x_67); -x_70 = lean_array_get_size(x_65); -x_71 = lean_nat_dec_le(x_69, x_70); -lean_dec(x_70); -lean_dec(x_69); -if (x_71 == 0) -{ -lean_object* x_72; lean_object* x_73; -x_72 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_65); -x_73 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_73, 0, x_63); -lean_ctor_set(x_73, 1, x_72); -return x_73; -} -else -{ -lean_object* x_74; -lean_dec(x_2); -x_74 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_74, 0, x_63); -lean_ctor_set(x_74, 1, x_65); -return x_74; -} -} -else -{ -lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; -lean_dec(x_2); -x_75 = lean_box(0); -x_76 = lean_array_uset(x_55, x_59, x_75); -x_77 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_28, x_60); -x_78 = lean_array_uset(x_76, x_59, x_77); -x_79 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_79, 0, x_54); -lean_ctor_set(x_79, 1, x_78); -return x_79; -} -} -} +x_27 = lean_box(0); +x_28 = lean_array_uset(x_7, x_21, x_27); +x_29 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_4, x_5, x_22); +x_30 = lean_array_uset(x_28, x_21, x_29); +lean_ctor_set(x_3, 1, x_30); +return x_3; } else { -lean_object* x_88; lean_object* x_89; lean_object* x_90; uint8_t x_119; +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_dec(x_3); -x_88 = lean_ctor_get(x_23, 0); -lean_inc(x_88); -lean_dec(x_23); -x_89 = lean_apply_1(x_5, x_88); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_119 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_119 == 0) -{ -lean_object* x_120; -lean_dec(x_22); -x_120 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_120, 0, x_6); -lean_ctor_set(x_120, 1, x_7); -x_90 = x_120; -goto block_118; -} -else -{ -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; -x_121 = lean_box(0); -x_122 = lean_array_uset(x_7, x_21, x_121); -x_123 = lean_unsigned_to_nat(1u); -x_124 = lean_nat_sub(x_6, x_123); -lean_dec(x_6); -lean_inc(x_4); -lean_inc(x_1); -x_125 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_126 = lean_array_uset(x_122, x_21, x_125); -x_127 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_127, 0, x_124); -lean_ctor_set(x_127, 1, x_126); -x_90 = x_127; -goto block_118; -} -block_118: -{ -lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; size_t x_95; size_t x_96; size_t x_97; lean_object* x_98; uint8_t x_99; -x_91 = lean_ctor_get(x_90, 0); -lean_inc(x_91); -x_92 = lean_ctor_get(x_90, 1); -lean_inc(x_92); -if (lean_is_exclusive(x_90)) { - lean_ctor_release(x_90, 0); - lean_ctor_release(x_90, 1); - x_93 = x_90; -} else { - lean_dec_ref(x_90); - x_93 = lean_box(0); -} -x_94 = lean_array_get_size(x_92); -x_95 = lean_usize_of_nat(x_94); -lean_dec(x_94); -x_96 = lean_usize_sub(x_95, x_19); -x_97 = lean_usize_land(x_17, x_96); -x_98 = lean_array_uget(x_92, x_97); -lean_inc(x_98); -lean_inc(x_4); -lean_inc(x_1); -x_99 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_98); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; uint8_t x_109; -lean_dec(x_1); -x_100 = lean_unsigned_to_nat(1u); -x_101 = lean_nat_add(x_91, x_100); -lean_dec(x_91); -x_102 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_102, 0, x_4); -lean_ctor_set(x_102, 1, x_89); -lean_ctor_set(x_102, 2, x_98); -x_103 = lean_array_uset(x_92, x_97, x_102); -x_104 = lean_unsigned_to_nat(4u); -x_105 = lean_nat_mul(x_101, x_104); -x_106 = lean_unsigned_to_nat(3u); -x_107 = lean_nat_div(x_105, x_106); -lean_dec(x_105); -x_108 = lean_array_get_size(x_103); -x_109 = lean_nat_dec_le(x_107, x_108); -lean_dec(x_108); -lean_dec(x_107); -if (x_109 == 0) -{ -lean_object* x_110; lean_object* x_111; -x_110 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_103); -if (lean_is_scalar(x_93)) { - x_111 = lean_alloc_ctor(0, 2, 0); -} else { - x_111 = x_93; -} -lean_ctor_set(x_111, 0, x_101); -lean_ctor_set(x_111, 1, x_110); -return x_111; -} -else -{ -lean_object* x_112; -lean_dec(x_2); -if (lean_is_scalar(x_93)) { - x_112 = lean_alloc_ctor(0, 2, 0); -} else { - x_112 = x_93; -} -lean_ctor_set(x_112, 0, x_101); -lean_ctor_set(x_112, 1, x_103); -return x_112; -} -} -else -{ -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; -lean_dec(x_2); -x_113 = lean_box(0); -x_114 = lean_array_uset(x_92, x_97, x_113); -x_115 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_89, x_98); -x_116 = lean_array_uset(x_114, x_97, x_115); -if (lean_is_scalar(x_93)) { - x_117 = lean_alloc_ctor(0, 2, 0); -} else { - x_117 = x_93; -} -lean_ctor_set(x_117, 0, x_91); -lean_ctor_set(x_117, 1, x_116); -return x_117; -} -} +x_31 = lean_box(0); +x_32 = lean_array_uset(x_7, x_21, x_31); +x_33 = l_Std_DHashMap_Internal_AssocList_Const_modify___rarg(x_1, lean_box(0), x_4, x_5, x_22); +x_34 = lean_array_uset(x_32, x_21, x_33); +x_35 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_35, 0, x_6); +lean_ctor_set(x_35, 1, x_34); +return x_35; } } } @@ -6530,7 +6251,7 @@ return x_3; LEAN_EXPORT lean_object* l_Std_HashMap_alter___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; lean_object* x_23; +lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint64_t x_10; uint64_t x_11; uint64_t x_12; uint64_t x_13; uint64_t x_14; uint64_t x_15; uint64_t x_16; size_t x_17; size_t x_18; size_t x_19; size_t x_20; size_t x_21; lean_object* x_22; uint8_t x_23; x_6 = lean_ctor_get(x_3, 0); lean_inc(x_6); x_7 = lean_ctor_get(x_3, 1); @@ -6557,10 +6278,11 @@ x_22 = lean_array_uget(x_7, x_21); lean_inc(x_22); lean_inc(x_4); lean_inc(x_1); -x_23 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_4, x_22); -if (lean_obj_tag(x_23) == 0) +x_23 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); +if (x_23 == 0) { lean_object* x_24; lean_object* x_25; +lean_dec(x_1); x_24 = lean_box(0); x_25 = lean_apply_1(x_5, x_24); if (lean_obj_tag(x_25) == 0) @@ -6570,7 +6292,6 @@ lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); lean_dec(x_2); -lean_dec(x_1); return x_3; } else @@ -6579,7 +6300,7 @@ uint8_t x_26; x_26 = !lean_is_exclusive(x_3); if (x_26 == 0) { -lean_object* x_27; lean_object* x_28; lean_object* x_29; uint8_t x_30; +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; x_27 = lean_ctor_get(x_3, 1); lean_dec(x_27); x_28 = lean_ctor_get(x_3, 0); @@ -6587,709 +6308,161 @@ lean_dec(x_28); x_29 = lean_ctor_get(x_25, 0); lean_inc(x_29); lean_dec(x_25); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_30 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_30 == 0) -{ -lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; uint8_t x_40; -lean_dec(x_1); -x_31 = lean_unsigned_to_nat(1u); -x_32 = lean_nat_add(x_6, x_31); +x_30 = lean_unsigned_to_nat(1u); +x_31 = lean_nat_add(x_6, x_30); lean_dec(x_6); -x_33 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_33, 0, x_4); -lean_ctor_set(x_33, 1, x_29); -lean_ctor_set(x_33, 2, x_22); -x_34 = lean_array_uset(x_7, x_21, x_33); -x_35 = lean_unsigned_to_nat(4u); -x_36 = lean_nat_mul(x_32, x_35); -x_37 = lean_unsigned_to_nat(3u); -x_38 = lean_nat_div(x_36, x_37); -lean_dec(x_36); -x_39 = lean_array_get_size(x_34); -x_40 = lean_nat_dec_le(x_38, x_39); -lean_dec(x_39); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_4); +lean_ctor_set(x_32, 1, x_29); +lean_ctor_set(x_32, 2, x_22); +x_33 = lean_array_uset(x_7, x_21, x_32); +x_34 = lean_unsigned_to_nat(4u); +x_35 = lean_nat_mul(x_31, x_34); +x_36 = lean_unsigned_to_nat(3u); +x_37 = lean_nat_div(x_35, x_36); +lean_dec(x_35); +x_38 = lean_array_get_size(x_33); +x_39 = lean_nat_dec_le(x_37, x_38); lean_dec(x_38); -if (x_40 == 0) -{ -lean_object* x_41; -x_41 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_34); -lean_ctor_set(x_3, 1, x_41); -lean_ctor_set(x_3, 0, x_32); -return x_3; -} -else +lean_dec(x_37); +if (x_39 == 0) { -lean_dec(x_2); -lean_ctor_set(x_3, 1, x_34); -lean_ctor_set(x_3, 0, x_32); +lean_object* x_40; +x_40 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_33); +lean_ctor_set(x_3, 1, x_40); +lean_ctor_set(x_3, 0, x_31); return x_3; } -} else { -lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_dec(x_2); -x_42 = lean_box(0); -x_43 = lean_array_uset(x_7, x_21, x_42); -x_44 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_29, x_22); -x_45 = lean_array_uset(x_43, x_21, x_44); -lean_ctor_set(x_3, 1, x_45); +lean_ctor_set(x_3, 1, x_33); +lean_ctor_set(x_3, 0, x_31); return x_3; } } else { -lean_object* x_46; uint8_t x_47; +lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; uint8_t x_51; lean_dec(x_3); -x_46 = lean_ctor_get(x_25, 0); -lean_inc(x_46); +x_41 = lean_ctor_get(x_25, 0); +lean_inc(x_41); lean_dec(x_25); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_47 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_47 == 0) -{ -lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; uint8_t x_57; -lean_dec(x_1); -x_48 = lean_unsigned_to_nat(1u); -x_49 = lean_nat_add(x_6, x_48); +x_42 = lean_unsigned_to_nat(1u); +x_43 = lean_nat_add(x_6, x_42); lean_dec(x_6); -x_50 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_50, 0, x_4); -lean_ctor_set(x_50, 1, x_46); -lean_ctor_set(x_50, 2, x_22); -x_51 = lean_array_uset(x_7, x_21, x_50); -x_52 = lean_unsigned_to_nat(4u); -x_53 = lean_nat_mul(x_49, x_52); -x_54 = lean_unsigned_to_nat(3u); -x_55 = lean_nat_div(x_53, x_54); -lean_dec(x_53); -x_56 = lean_array_get_size(x_51); -x_57 = lean_nat_dec_le(x_55, x_56); -lean_dec(x_56); -lean_dec(x_55); -if (x_57 == 0) -{ -lean_object* x_58; lean_object* x_59; -x_58 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_51); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_49); -lean_ctor_set(x_59, 1, x_58); -return x_59; -} -else +x_44 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_44, 0, x_4); +lean_ctor_set(x_44, 1, x_41); +lean_ctor_set(x_44, 2, x_22); +x_45 = lean_array_uset(x_7, x_21, x_44); +x_46 = lean_unsigned_to_nat(4u); +x_47 = lean_nat_mul(x_43, x_46); +x_48 = lean_unsigned_to_nat(3u); +x_49 = lean_nat_div(x_47, x_48); +lean_dec(x_47); +x_50 = lean_array_get_size(x_45); +x_51 = lean_nat_dec_le(x_49, x_50); +lean_dec(x_50); +lean_dec(x_49); +if (x_51 == 0) { -lean_object* x_60; -lean_dec(x_2); -x_60 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_60, 0, x_49); -lean_ctor_set(x_60, 1, x_51); -return x_60; -} +lean_object* x_52; lean_object* x_53; +x_52 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_45); +x_53 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_53, 0, x_43); +lean_ctor_set(x_53, 1, x_52); +return x_53; } else { -lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; +lean_object* x_54; lean_dec(x_2); -x_61 = lean_box(0); -x_62 = lean_array_uset(x_7, x_21, x_61); -x_63 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_46, x_22); -x_64 = lean_array_uset(x_62, x_21, x_63); -x_65 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_65, 0, x_6); -lean_ctor_set(x_65, 1, x_64); -return x_65; +x_54 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_54, 0, x_43); +lean_ctor_set(x_54, 1, x_45); +return x_54; } } } } else { -uint8_t x_66; -x_66 = !lean_is_exclusive(x_3); -if (x_66 == 0) -{ -lean_object* x_67; lean_object* x_68; uint8_t x_69; -x_67 = lean_ctor_get(x_3, 1); -lean_dec(x_67); -x_68 = lean_ctor_get(x_3, 0); -lean_dec(x_68); -x_69 = !lean_is_exclusive(x_23); -if (x_69 == 0) -{ -lean_object* x_70; -x_70 = lean_apply_1(x_5, x_23); -if (lean_obj_tag(x_70) == 0) -{ -uint8_t x_71; +uint8_t x_55; lean_dec(x_2); -lean_inc(x_22); +x_55 = !lean_is_exclusive(x_3); +if (x_55 == 0) +{ +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; uint8_t x_61; lean_object* x_62; +x_56 = lean_ctor_get(x_3, 1); +lean_dec(x_56); +x_57 = lean_ctor_get(x_3, 0); +lean_dec(x_57); +x_58 = lean_box(0); +x_59 = lean_array_uset(x_7, x_21, x_58); lean_inc(x_4); lean_inc(x_1); -x_71 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_71 == 0) +x_60 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_4, x_5, x_22); +lean_inc(x_60); +x_61 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_60); +x_62 = lean_array_uset(x_59, x_21, x_60); +if (x_61 == 0) { -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_1); +lean_object* x_63; lean_object* x_64; +x_63 = lean_unsigned_to_nat(1u); +x_64 = lean_nat_sub(x_6, x_63); +lean_dec(x_6); +lean_ctor_set(x_3, 1, x_62); +lean_ctor_set(x_3, 0, x_64); return x_3; } else { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; -x_72 = lean_box(0); -x_73 = lean_array_uset(x_7, x_21, x_72); -x_74 = lean_unsigned_to_nat(1u); -x_75 = lean_nat_sub(x_6, x_74); -lean_dec(x_6); -x_76 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_77 = lean_array_uset(x_73, x_21, x_76); -lean_ctor_set(x_3, 1, x_77); -lean_ctor_set(x_3, 0, x_75); +lean_ctor_set(x_3, 1, x_62); return x_3; } } else { -lean_object* x_78; lean_object* x_79; uint8_t x_131; -x_78 = lean_ctor_get(x_70, 0); -lean_inc(x_78); -lean_dec(x_70); -lean_inc(x_22); +lean_object* x_65; lean_object* x_66; lean_object* x_67; uint8_t x_68; lean_object* x_69; +lean_dec(x_3); +x_65 = lean_box(0); +x_66 = lean_array_uset(x_7, x_21, x_65); lean_inc(x_4); lean_inc(x_1); -x_131 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_131 == 0) -{ -lean_dec(x_22); -x_79 = x_3; -goto block_130; -} -else +x_67 = l_Std_DHashMap_Internal_AssocList_Const_alter___rarg(x_1, lean_box(0), x_4, x_5, x_22); +lean_inc(x_67); +x_68 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_67); +x_69 = lean_array_uset(x_66, x_21, x_67); +if (x_68 == 0) { -lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_132 = lean_box(0); -x_133 = lean_array_uset(x_7, x_21, x_132); -x_134 = lean_unsigned_to_nat(1u); -x_135 = lean_nat_sub(x_6, x_134); +lean_object* x_70; lean_object* x_71; lean_object* x_72; +x_70 = lean_unsigned_to_nat(1u); +x_71 = lean_nat_sub(x_6, x_70); lean_dec(x_6); -lean_inc(x_4); -lean_inc(x_1); -x_136 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_137 = lean_array_uset(x_133, x_21, x_136); -lean_ctor_set(x_3, 1, x_137); -lean_ctor_set(x_3, 0, x_135); -x_79 = x_3; -goto block_130; -} -block_130: -{ -uint8_t x_80; -x_80 = !lean_is_exclusive(x_79); -if (x_80 == 0) -{ -lean_object* x_81; lean_object* x_82; lean_object* x_83; size_t x_84; size_t x_85; size_t x_86; lean_object* x_87; uint8_t x_88; -x_81 = lean_ctor_get(x_79, 0); -x_82 = lean_ctor_get(x_79, 1); -x_83 = lean_array_get_size(x_82); -x_84 = lean_usize_of_nat(x_83); -lean_dec(x_83); -x_85 = lean_usize_sub(x_84, x_19); -x_86 = lean_usize_land(x_17, x_85); -x_87 = lean_array_uget(x_82, x_86); -lean_inc(x_87); -lean_inc(x_4); -lean_inc(x_1); -x_88 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_87); -if (x_88 == 0) -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; uint8_t x_98; -lean_dec(x_1); -x_89 = lean_unsigned_to_nat(1u); -x_90 = lean_nat_add(x_81, x_89); -lean_dec(x_81); -x_91 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_91, 0, x_4); -lean_ctor_set(x_91, 1, x_78); -lean_ctor_set(x_91, 2, x_87); -x_92 = lean_array_uset(x_82, x_86, x_91); -x_93 = lean_unsigned_to_nat(4u); -x_94 = lean_nat_mul(x_90, x_93); -x_95 = lean_unsigned_to_nat(3u); -x_96 = lean_nat_div(x_94, x_95); -lean_dec(x_94); -x_97 = lean_array_get_size(x_92); -x_98 = lean_nat_dec_le(x_96, x_97); -lean_dec(x_97); -lean_dec(x_96); -if (x_98 == 0) -{ -lean_object* x_99; -x_99 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_92); -lean_ctor_set(x_79, 1, x_99); -lean_ctor_set(x_79, 0, x_90); -return x_79; -} -else -{ -lean_dec(x_2); -lean_ctor_set(x_79, 1, x_92); -lean_ctor_set(x_79, 0, x_90); -return x_79; -} +x_72 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_72, 0, x_71); +lean_ctor_set(x_72, 1, x_69); +return x_72; } else { -lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; -lean_dec(x_2); -x_100 = lean_box(0); -x_101 = lean_array_uset(x_82, x_86, x_100); -x_102 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_78, x_87); -x_103 = lean_array_uset(x_101, x_86, x_102); -lean_ctor_set(x_79, 1, x_103); -return x_79; -} -} -else -{ -lean_object* x_104; lean_object* x_105; lean_object* x_106; size_t x_107; size_t x_108; size_t x_109; lean_object* x_110; uint8_t x_111; -x_104 = lean_ctor_get(x_79, 0); -x_105 = lean_ctor_get(x_79, 1); -lean_inc(x_105); -lean_inc(x_104); -lean_dec(x_79); -x_106 = lean_array_get_size(x_105); -x_107 = lean_usize_of_nat(x_106); -lean_dec(x_106); -x_108 = lean_usize_sub(x_107, x_19); -x_109 = lean_usize_land(x_17, x_108); -x_110 = lean_array_uget(x_105, x_109); -lean_inc(x_110); -lean_inc(x_4); -lean_inc(x_1); -x_111 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_110); -if (x_111 == 0) -{ -lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; uint8_t x_121; -lean_dec(x_1); -x_112 = lean_unsigned_to_nat(1u); -x_113 = lean_nat_add(x_104, x_112); -lean_dec(x_104); -x_114 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_114, 0, x_4); -lean_ctor_set(x_114, 1, x_78); -lean_ctor_set(x_114, 2, x_110); -x_115 = lean_array_uset(x_105, x_109, x_114); -x_116 = lean_unsigned_to_nat(4u); -x_117 = lean_nat_mul(x_113, x_116); -x_118 = lean_unsigned_to_nat(3u); -x_119 = lean_nat_div(x_117, x_118); -lean_dec(x_117); -x_120 = lean_array_get_size(x_115); -x_121 = lean_nat_dec_le(x_119, x_120); -lean_dec(x_120); -lean_dec(x_119); -if (x_121 == 0) -{ -lean_object* x_122; lean_object* x_123; -x_122 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_115); -x_123 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_123, 0, x_113); -lean_ctor_set(x_123, 1, x_122); -return x_123; -} -else -{ -lean_object* x_124; -lean_dec(x_2); -x_124 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_124, 0, x_113); -lean_ctor_set(x_124, 1, x_115); -return x_124; +lean_object* x_73; +x_73 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_73, 0, x_6); +lean_ctor_set(x_73, 1, x_69); +return x_73; } } -else -{ -lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; -lean_dec(x_2); -x_125 = lean_box(0); -x_126 = lean_array_uset(x_105, x_109, x_125); -x_127 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_78, x_110); -x_128 = lean_array_uset(x_126, x_109, x_127); -x_129 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_129, 0, x_104); -lean_ctor_set(x_129, 1, x_128); -return x_129; } } } -} -} -else -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; -x_138 = lean_ctor_get(x_23, 0); -lean_inc(x_138); -lean_dec(x_23); -x_139 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_139, 0, x_138); -x_140 = lean_apply_1(x_5, x_139); -if (lean_obj_tag(x_140) == 0) -{ -uint8_t x_141; -lean_dec(x_2); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_141 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_141 == 0) -{ -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_1); -return x_3; -} -else -{ -lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; -x_142 = lean_box(0); -x_143 = lean_array_uset(x_7, x_21, x_142); -x_144 = lean_unsigned_to_nat(1u); -x_145 = lean_nat_sub(x_6, x_144); -lean_dec(x_6); -x_146 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_147 = lean_array_uset(x_143, x_21, x_146); -lean_ctor_set(x_3, 1, x_147); -lean_ctor_set(x_3, 0, x_145); -return x_3; -} -} -else -{ -lean_object* x_148; lean_object* x_149; uint8_t x_178; -x_148 = lean_ctor_get(x_140, 0); -lean_inc(x_148); -lean_dec(x_140); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_178 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_178 == 0) -{ -lean_dec(x_22); -x_149 = x_3; -goto block_177; -} -else -{ -lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; -x_179 = lean_box(0); -x_180 = lean_array_uset(x_7, x_21, x_179); -x_181 = lean_unsigned_to_nat(1u); -x_182 = lean_nat_sub(x_6, x_181); -lean_dec(x_6); -lean_inc(x_4); -lean_inc(x_1); -x_183 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_184 = lean_array_uset(x_180, x_21, x_183); -lean_ctor_set(x_3, 1, x_184); -lean_ctor_set(x_3, 0, x_182); -x_149 = x_3; -goto block_177; -} -block_177: -{ -lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; size_t x_154; size_t x_155; size_t x_156; lean_object* x_157; uint8_t x_158; -x_150 = lean_ctor_get(x_149, 0); -lean_inc(x_150); -x_151 = lean_ctor_get(x_149, 1); -lean_inc(x_151); -if (lean_is_exclusive(x_149)) { - lean_ctor_release(x_149, 0); - lean_ctor_release(x_149, 1); - x_152 = x_149; -} else { - lean_dec_ref(x_149); - x_152 = lean_box(0); -} -x_153 = lean_array_get_size(x_151); -x_154 = lean_usize_of_nat(x_153); -lean_dec(x_153); -x_155 = lean_usize_sub(x_154, x_19); -x_156 = lean_usize_land(x_17, x_155); -x_157 = lean_array_uget(x_151, x_156); -lean_inc(x_157); -lean_inc(x_4); -lean_inc(x_1); -x_158 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_157); -if (x_158 == 0) -{ -lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; uint8_t x_168; -lean_dec(x_1); -x_159 = lean_unsigned_to_nat(1u); -x_160 = lean_nat_add(x_150, x_159); -lean_dec(x_150); -x_161 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_161, 0, x_4); -lean_ctor_set(x_161, 1, x_148); -lean_ctor_set(x_161, 2, x_157); -x_162 = lean_array_uset(x_151, x_156, x_161); -x_163 = lean_unsigned_to_nat(4u); -x_164 = lean_nat_mul(x_160, x_163); -x_165 = lean_unsigned_to_nat(3u); -x_166 = lean_nat_div(x_164, x_165); -lean_dec(x_164); -x_167 = lean_array_get_size(x_162); -x_168 = lean_nat_dec_le(x_166, x_167); -lean_dec(x_167); -lean_dec(x_166); -if (x_168 == 0) -{ -lean_object* x_169; lean_object* x_170; -x_169 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_162); -if (lean_is_scalar(x_152)) { - x_170 = lean_alloc_ctor(0, 2, 0); -} else { - x_170 = x_152; -} -lean_ctor_set(x_170, 0, x_160); -lean_ctor_set(x_170, 1, x_169); -return x_170; -} -else -{ -lean_object* x_171; -lean_dec(x_2); -if (lean_is_scalar(x_152)) { - x_171 = lean_alloc_ctor(0, 2, 0); -} else { - x_171 = x_152; -} -lean_ctor_set(x_171, 0, x_160); -lean_ctor_set(x_171, 1, x_162); -return x_171; -} -} -else -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; -lean_dec(x_2); -x_172 = lean_box(0); -x_173 = lean_array_uset(x_151, x_156, x_172); -x_174 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_148, x_157); -x_175 = lean_array_uset(x_173, x_156, x_174); -if (lean_is_scalar(x_152)) { - x_176 = lean_alloc_ctor(0, 2, 0); -} else { - x_176 = x_152; -} -lean_ctor_set(x_176, 0, x_150); -lean_ctor_set(x_176, 1, x_175); -return x_176; -} -} -} -} -} -else -{ -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -lean_dec(x_3); -x_185 = lean_ctor_get(x_23, 0); -lean_inc(x_185); -if (lean_is_exclusive(x_23)) { - lean_ctor_release(x_23, 0); - x_186 = x_23; -} else { - lean_dec_ref(x_23); - x_186 = lean_box(0); -} -if (lean_is_scalar(x_186)) { - x_187 = lean_alloc_ctor(1, 1, 0); -} else { - x_187 = x_186; -} -lean_ctor_set(x_187, 0, x_185); -x_188 = lean_apply_1(x_5, x_187); -if (lean_obj_tag(x_188) == 0) -{ -uint8_t x_189; -lean_dec(x_2); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_189 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_189 == 0) -{ -lean_object* x_190; -lean_dec(x_22); -lean_dec(x_4); -lean_dec(x_1); -x_190 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_190, 0, x_6); -lean_ctor_set(x_190, 1, x_7); -return x_190; -} -else -{ -lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; -x_191 = lean_box(0); -x_192 = lean_array_uset(x_7, x_21, x_191); -x_193 = lean_unsigned_to_nat(1u); -x_194 = lean_nat_sub(x_6, x_193); -lean_dec(x_6); -x_195 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_196 = lean_array_uset(x_192, x_21, x_195); -x_197 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_197, 0, x_194); -lean_ctor_set(x_197, 1, x_196); -return x_197; -} -} -else -{ -lean_object* x_198; lean_object* x_199; uint8_t x_228; -x_198 = lean_ctor_get(x_188, 0); -lean_inc(x_198); -lean_dec(x_188); -lean_inc(x_22); -lean_inc(x_4); -lean_inc(x_1); -x_228 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_22); -if (x_228 == 0) -{ -lean_object* x_229; -lean_dec(x_22); -x_229 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_229, 0, x_6); -lean_ctor_set(x_229, 1, x_7); -x_199 = x_229; -goto block_227; -} -else -{ -lean_object* x_230; lean_object* x_231; lean_object* x_232; lean_object* x_233; lean_object* x_234; lean_object* x_235; lean_object* x_236; -x_230 = lean_box(0); -x_231 = lean_array_uset(x_7, x_21, x_230); -x_232 = lean_unsigned_to_nat(1u); -x_233 = lean_nat_sub(x_6, x_232); -lean_dec(x_6); -lean_inc(x_4); -lean_inc(x_1); -x_234 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_4, x_22); -x_235 = lean_array_uset(x_231, x_21, x_234); -x_236 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_236, 0, x_233); -lean_ctor_set(x_236, 1, x_235); -x_199 = x_236; -goto block_227; -} -block_227: -{ -lean_object* x_200; lean_object* x_201; lean_object* x_202; lean_object* x_203; size_t x_204; size_t x_205; size_t x_206; lean_object* x_207; uint8_t x_208; -x_200 = lean_ctor_get(x_199, 0); -lean_inc(x_200); -x_201 = lean_ctor_get(x_199, 1); -lean_inc(x_201); -if (lean_is_exclusive(x_199)) { - lean_ctor_release(x_199, 0); - lean_ctor_release(x_199, 1); - x_202 = x_199; -} else { - lean_dec_ref(x_199); - x_202 = lean_box(0); -} -x_203 = lean_array_get_size(x_201); -x_204 = lean_usize_of_nat(x_203); -lean_dec(x_203); -x_205 = lean_usize_sub(x_204, x_19); -x_206 = lean_usize_land(x_17, x_205); -x_207 = lean_array_uget(x_201, x_206); -lean_inc(x_207); -lean_inc(x_4); -lean_inc(x_1); -x_208 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_4, x_207); -if (x_208 == 0) -{ -lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; lean_object* x_216; lean_object* x_217; uint8_t x_218; -lean_dec(x_1); -x_209 = lean_unsigned_to_nat(1u); -x_210 = lean_nat_add(x_200, x_209); -lean_dec(x_200); -x_211 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_211, 0, x_4); -lean_ctor_set(x_211, 1, x_198); -lean_ctor_set(x_211, 2, x_207); -x_212 = lean_array_uset(x_201, x_206, x_211); -x_213 = lean_unsigned_to_nat(4u); -x_214 = lean_nat_mul(x_210, x_213); -x_215 = lean_unsigned_to_nat(3u); -x_216 = lean_nat_div(x_214, x_215); -lean_dec(x_214); -x_217 = lean_array_get_size(x_212); -x_218 = lean_nat_dec_le(x_216, x_217); -lean_dec(x_217); -lean_dec(x_216); -if (x_218 == 0) -{ -lean_object* x_219; lean_object* x_220; -x_219 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_212); -if (lean_is_scalar(x_202)) { - x_220 = lean_alloc_ctor(0, 2, 0); -} else { - x_220 = x_202; -} -lean_ctor_set(x_220, 0, x_210); -lean_ctor_set(x_220, 1, x_219); -return x_220; -} -else -{ -lean_object* x_221; -lean_dec(x_2); -if (lean_is_scalar(x_202)) { - x_221 = lean_alloc_ctor(0, 2, 0); -} else { - x_221 = x_202; -} -lean_ctor_set(x_221, 0, x_210); -lean_ctor_set(x_221, 1, x_212); -return x_221; -} -} -else -{ -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -lean_dec(x_2); -x_222 = lean_box(0); -x_223 = lean_array_uset(x_201, x_206, x_222); -x_224 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_4, x_198, x_207); -x_225 = lean_array_uset(x_223, x_206, x_224); -if (lean_is_scalar(x_202)) { - x_226 = lean_alloc_ctor(0, 2, 0); -} else { - x_226 = x_202; -} -lean_ctor_set(x_226, 0, x_200); -lean_ctor_set(x_226, 1, x_225); -return x_226; -} -} -} -} -} -} -} -LEAN_EXPORT lean_object* l_Std_HashMap_alter(lean_object* x_1, lean_object* x_2) { -_start: -{ -lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Std_HashMap_alter___rarg), 5, 0); -return x_3; +LEAN_EXPORT lean_object* l_Std_HashMap_alter(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_HashMap_alter___rarg), 5, 0); +return x_3; } } LEAN_EXPORT lean_object* l_Std_HashMap_insertMany___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { @@ -10582,563 +9755,445 @@ lean_dec(x_3); return x_5; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_11; -x_11 = lean_usize_dec_lt(x_9, x_8); -if (x_11 == 0) +if (lean_obj_tag(x_5) == 0) { -lean_dec(x_5); -lean_dec(x_3); -lean_dec(x_2); +lean_object* x_6; lean_object* x_7; lean_dec(x_1); -return x_10; +x_6 = lean_box(0); +x_7 = lean_apply_1(x_4, x_6); +if (lean_obj_tag(x_7) == 0) +{ +lean_object* x_8; +lean_dec(x_3); +x_8 = lean_box(0); +return x_8; } else { -lean_object* x_12; lean_object* x_13; uint8_t x_14; -x_12 = lean_array_uget(x_7, x_9); -lean_inc(x_3); -lean_inc(x_12); -x_13 = lean_apply_1(x_3, x_12); -x_14 = !lean_is_exclusive(x_10); -if (x_14 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_9); +lean_ctor_set(x_11, 2, x_10); +return x_11; +} +} +else { -lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; lean_object* x_31; lean_object* x_32; -x_15 = lean_ctor_get(x_10, 0); -x_16 = lean_ctor_get(x_10, 1); -x_17 = lean_array_get_size(x_16); -lean_inc(x_2); -lean_inc(x_13); -x_18 = lean_apply_1(x_2, x_13); -x_19 = lean_unbox_uint64(x_18); -lean_dec(x_18); -x_20 = 32; -x_21 = lean_uint64_shift_right(x_19, x_20); -x_22 = lean_uint64_xor(x_19, x_21); -x_23 = 16; -x_24 = lean_uint64_shift_right(x_22, x_23); -x_25 = lean_uint64_xor(x_22, x_24); -x_26 = lean_uint64_to_usize(x_25); -x_27 = lean_usize_of_nat(x_17); -lean_dec(x_17); -x_28 = 1; -x_29 = lean_usize_sub(x_27, x_28); -x_30 = lean_usize_land(x_26, x_29); -x_31 = lean_array_uget(x_16, x_30); -lean_inc(x_31); -lean_inc(x_13); -lean_inc(x_1); -x_32 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_13, x_31); -if (lean_obj_tag(x_32) == 0) +uint8_t x_12; +x_12 = !lean_is_exclusive(x_5); +if (x_12 == 0) { -lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_33 = l_Std_HashMap_toArray___rarg___closed__1; -x_34 = lean_array_push(x_33, x_12); -lean_inc(x_31); -lean_inc(x_13); +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_5, 0); +x_14 = lean_ctor_get(x_5, 1); +x_15 = lean_ctor_get(x_5, 2); lean_inc(x_1); -x_35 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_31); -if (x_35 == 0) -{ -lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; -x_36 = lean_unsigned_to_nat(1u); -x_37 = lean_nat_add(x_15, x_36); -lean_dec(x_15); -x_38 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_38, 0, x_13); -lean_ctor_set(x_38, 1, x_34); -lean_ctor_set(x_38, 2, x_31); -x_39 = lean_array_uset(x_16, x_30, x_38); -x_40 = lean_unsigned_to_nat(4u); -x_41 = lean_nat_mul(x_37, x_40); -x_42 = lean_unsigned_to_nat(3u); -x_43 = lean_nat_div(x_41, x_42); -lean_dec(x_41); -x_44 = lean_array_get_size(x_39); -x_45 = lean_nat_dec_le(x_43, x_44); -lean_dec(x_44); -lean_dec(x_43); -if (x_45 == 0) +lean_inc(x_3); +lean_inc(x_13); +x_16 = lean_apply_2(x_1, x_13, x_3); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) { -lean_object* x_46; size_t x_47; -lean_inc(x_2); -x_46 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_39); -lean_ctor_set(x_10, 1, x_46); -lean_ctor_set(x_10, 0, x_37); -x_47 = lean_usize_add(x_9, x_28); -x_9 = x_47; -goto _start; +lean_object* x_18; +x_18 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(x_1, lean_box(0), x_3, x_4, x_15); +lean_ctor_set(x_5, 2, x_18); +return x_5; } else { -size_t x_49; -lean_ctor_set(x_10, 1, x_39); -lean_ctor_set(x_10, 0, x_37); -x_49 = lean_usize_add(x_9, x_28); -x_9 = x_49; -goto _start; -} +lean_object* x_19; lean_object* x_20; +lean_dec(x_13); +lean_dec(x_1); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_14); +x_20 = lean_apply_1(x_4, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_free_object(x_5); +lean_dec(x_3); +return x_15; } else { -lean_object* x_51; lean_object* x_52; lean_object* x_53; size_t x_54; -lean_inc(x_5); -x_51 = lean_array_uset(x_16, x_30, x_5); -lean_inc(x_1); -x_52 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_13, x_34, x_31); -x_53 = lean_array_uset(x_51, x_30, x_52); -lean_ctor_set(x_10, 1, x_53); -x_54 = lean_usize_add(x_9, x_28); -x_9 = x_54; -goto _start; +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +lean_dec(x_20); +lean_ctor_set(x_5, 1, x_21); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} } } else { -lean_object* x_56; lean_object* x_57; lean_object* x_58; uint8_t x_120; -x_56 = lean_ctor_get(x_32, 0); -lean_inc(x_56); -lean_dec(x_32); -x_57 = lean_array_push(x_56, x_12); -lean_inc(x_31); -lean_inc(x_13); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_5, 0); +x_23 = lean_ctor_get(x_5, 1); +x_24 = lean_ctor_get(x_5, 2); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_5); lean_inc(x_1); -x_120 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_31); -if (x_120 == 0) +lean_inc(x_3); +lean_inc(x_22); +x_25 = lean_apply_2(x_1, x_22, x_3); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) { -lean_dec(x_31); -x_58 = x_10; -goto block_119; +lean_object* x_27; lean_object* x_28; +x_27 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(x_1, lean_box(0), x_3, x_4, x_24); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_27); +return x_28; } else { -lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -lean_inc(x_5); -x_121 = lean_array_uset(x_16, x_30, x_5); -x_122 = lean_unsigned_to_nat(1u); -x_123 = lean_nat_sub(x_15, x_122); -lean_dec(x_15); -lean_inc(x_13); -lean_inc(x_1); -x_124 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_13, x_31); -x_125 = lean_array_uset(x_121, x_30, x_124); -lean_ctor_set(x_10, 1, x_125); -lean_ctor_set(x_10, 0, x_123); -x_58 = x_10; -goto block_119; -} -block_119: -{ -uint8_t x_59; -x_59 = !lean_is_exclusive(x_58); -if (x_59 == 0) -{ -lean_object* x_60; lean_object* x_61; lean_object* x_62; size_t x_63; size_t x_64; size_t x_65; lean_object* x_66; uint8_t x_67; -x_60 = lean_ctor_get(x_58, 0); -x_61 = lean_ctor_get(x_58, 1); -x_62 = lean_array_get_size(x_61); -x_63 = lean_usize_of_nat(x_62); -lean_dec(x_62); -x_64 = lean_usize_sub(x_63, x_28); -x_65 = lean_usize_land(x_26, x_64); -x_66 = lean_array_uget(x_61, x_65); -lean_inc(x_66); -lean_inc(x_13); -lean_inc(x_1); -x_67 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_66); -if (x_67 == 0) +lean_object* x_29; lean_object* x_30; +lean_dec(x_22); +lean_dec(x_1); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_23); +x_30 = lean_apply_1(x_4, x_29); +if (lean_obj_tag(x_30) == 0) { -lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; uint8_t x_77; -x_68 = lean_unsigned_to_nat(1u); -x_69 = lean_nat_add(x_60, x_68); -lean_dec(x_60); -x_70 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_70, 0, x_13); -lean_ctor_set(x_70, 1, x_57); -lean_ctor_set(x_70, 2, x_66); -x_71 = lean_array_uset(x_61, x_65, x_70); -x_72 = lean_unsigned_to_nat(4u); -x_73 = lean_nat_mul(x_69, x_72); -x_74 = lean_unsigned_to_nat(3u); -x_75 = lean_nat_div(x_73, x_74); -lean_dec(x_73); -x_76 = lean_array_get_size(x_71); -x_77 = lean_nat_dec_le(x_75, x_76); -lean_dec(x_76); -lean_dec(x_75); -if (x_77 == 0) -{ -lean_object* x_78; size_t x_79; -lean_inc(x_2); -x_78 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_71); -lean_ctor_set(x_58, 1, x_78); -lean_ctor_set(x_58, 0, x_69); -x_79 = lean_usize_add(x_9, x_28); -x_9 = x_79; -x_10 = x_58; -goto _start; +lean_dec(x_3); +return x_24; } else { -size_t x_81; -lean_ctor_set(x_58, 1, x_71); -lean_ctor_set(x_58, 0, x_69); -x_81 = lean_usize_add(x_9, x_28); -x_9 = x_81; -x_10 = x_58; -goto _start; +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); +lean_dec(x_30); +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_24); +return x_32; } } -else +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1(lean_object* x_1) { +_start: { -lean_object* x_83; lean_object* x_84; lean_object* x_85; size_t x_86; -lean_inc(x_5); -x_83 = lean_array_uset(x_61, x_65, x_5); -lean_inc(x_1); -x_84 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_13, x_57, x_66); -x_85 = lean_array_uset(x_83, x_65, x_84); -lean_ctor_set(x_58, 1, x_85); -x_86 = lean_usize_add(x_9, x_28); -x_9 = x_86; -x_10 = x_58; -goto _start; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg), 5, 0); +return x_2; } } -else +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: { -lean_object* x_88; lean_object* x_89; lean_object* x_90; size_t x_91; size_t x_92; size_t x_93; lean_object* x_94; uint8_t x_95; -x_88 = lean_ctor_get(x_58, 0); -x_89 = lean_ctor_get(x_58, 1); -lean_inc(x_89); -lean_inc(x_88); -lean_dec(x_58); -x_90 = lean_array_get_size(x_89); -x_91 = lean_usize_of_nat(x_90); -lean_dec(x_90); -x_92 = lean_usize_sub(x_91, x_28); -x_93 = lean_usize_land(x_26, x_92); -x_94 = lean_array_uget(x_89, x_93); -lean_inc(x_94); -lean_inc(x_13); -lean_inc(x_1); -x_95 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_94); -if (x_95 == 0) +if (lean_obj_tag(x_2) == 0) { -lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; uint8_t x_105; -x_96 = lean_unsigned_to_nat(1u); -x_97 = lean_nat_add(x_88, x_96); -lean_dec(x_88); -x_98 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_98, 0, x_13); -lean_ctor_set(x_98, 1, x_57); -lean_ctor_set(x_98, 2, x_94); -x_99 = lean_array_uset(x_89, x_93, x_98); -x_100 = lean_unsigned_to_nat(4u); -x_101 = lean_nat_mul(x_97, x_100); -x_102 = lean_unsigned_to_nat(3u); -x_103 = lean_nat_div(x_101, x_102); -lean_dec(x_101); -x_104 = lean_array_get_size(x_99); -x_105 = lean_nat_dec_le(x_103, x_104); -lean_dec(x_104); -lean_dec(x_103); -if (x_105 == 0) -{ -lean_object* x_106; lean_object* x_107; size_t x_108; -lean_inc(x_2); -x_106 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_99); -x_107 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_107, 0, x_97); -lean_ctor_set(x_107, 1, x_106); -x_108 = lean_usize_add(x_9, x_28); -x_9 = x_108; -x_10 = x_107; -goto _start; +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = l_Std_HashMap_toArray___rarg___closed__1; +x_4 = lean_array_push(x_3, x_1); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -lean_object* x_110; size_t x_111; -x_110 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_110, 0, x_97); -lean_ctor_set(x_110, 1, x_99); -x_111 = lean_usize_add(x_9, x_28); -x_9 = x_111; -x_10 = x_110; -goto _start; -} +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_array_push(x_7, x_1); +lean_ctor_set(x_2, 0, x_8); +return x_2; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; size_t x_117; -lean_inc(x_5); -x_113 = lean_array_uset(x_89, x_93, x_5); -lean_inc(x_1); -x_114 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_13, x_57, x_94); -x_115 = lean_array_uset(x_113, x_93, x_114); -x_116 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_116, 0, x_88); -lean_ctor_set(x_116, 1, x_115); -x_117 = lean_usize_add(x_9, x_28); -x_9 = x_117; -x_10 = x_116; -goto _start; +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_array_push(x_9, x_1); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; } } } } +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, size_t x_8, size_t x_9, lean_object* x_10) { +_start: +{ +uint8_t x_11; +x_11 = lean_usize_dec_lt(x_9, x_8); +if (x_11 == 0) +{ +lean_dec(x_5); +lean_dec(x_3); +lean_dec(x_2); +lean_dec(x_1); +return x_10; } else { -lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; uint64_t x_130; uint64_t x_131; uint64_t x_132; uint64_t x_133; uint64_t x_134; uint64_t x_135; uint64_t x_136; size_t x_137; size_t x_138; size_t x_139; size_t x_140; size_t x_141; lean_object* x_142; lean_object* x_143; -x_126 = lean_ctor_get(x_10, 0); -x_127 = lean_ctor_get(x_10, 1); -lean_inc(x_127); -lean_inc(x_126); -lean_dec(x_10); -x_128 = lean_array_get_size(x_127); +lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +x_12 = lean_array_uget(x_7, x_9); +lean_inc(x_3); +lean_inc(x_12); +x_13 = lean_apply_1(x_3, x_12); +lean_inc(x_12); +x_14 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___lambda__1), 2, 1); +lean_closure_set(x_14, 0, x_12); +x_15 = !lean_is_exclusive(x_10); +if (x_15 == 0) +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; uint64_t x_26; size_t x_27; size_t x_28; size_t x_29; size_t x_30; size_t x_31; lean_object* x_32; uint8_t x_33; +x_16 = lean_ctor_get(x_10, 0); +x_17 = lean_ctor_get(x_10, 1); +x_18 = lean_array_get_size(x_17); lean_inc(x_2); lean_inc(x_13); -x_129 = lean_apply_1(x_2, x_13); -x_130 = lean_unbox_uint64(x_129); -lean_dec(x_129); -x_131 = 32; -x_132 = lean_uint64_shift_right(x_130, x_131); -x_133 = lean_uint64_xor(x_130, x_132); -x_134 = 16; -x_135 = lean_uint64_shift_right(x_133, x_134); -x_136 = lean_uint64_xor(x_133, x_135); -x_137 = lean_uint64_to_usize(x_136); -x_138 = lean_usize_of_nat(x_128); -lean_dec(x_128); -x_139 = 1; -x_140 = lean_usize_sub(x_138, x_139); -x_141 = lean_usize_land(x_137, x_140); -x_142 = lean_array_uget(x_127, x_141); -lean_inc(x_142); +x_19 = lean_apply_1(x_2, x_13); +x_20 = lean_unbox_uint64(x_19); +lean_dec(x_19); +x_21 = 32; +x_22 = lean_uint64_shift_right(x_20, x_21); +x_23 = lean_uint64_xor(x_20, x_22); +x_24 = 16; +x_25 = lean_uint64_shift_right(x_23, x_24); +x_26 = lean_uint64_xor(x_23, x_25); +x_27 = lean_uint64_to_usize(x_26); +x_28 = lean_usize_of_nat(x_18); +lean_dec(x_18); +x_29 = 1; +x_30 = lean_usize_sub(x_28, x_29); +x_31 = lean_usize_land(x_27, x_30); +x_32 = lean_array_uget(x_17, x_31); +lean_inc(x_32); lean_inc(x_13); lean_inc(x_1); -x_143 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_13, x_142); -if (lean_obj_tag(x_143) == 0) +x_33 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_32); +if (x_33 == 0) { -lean_object* x_144; lean_object* x_145; uint8_t x_146; -x_144 = l_Std_HashMap_toArray___rarg___closed__1; -x_145 = lean_array_push(x_144, x_12); -lean_inc(x_142); -lean_inc(x_13); -lean_inc(x_1); -x_146 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_142); -if (x_146 == 0) -{ -lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; uint8_t x_156; -x_147 = lean_unsigned_to_nat(1u); -x_148 = lean_nat_add(x_126, x_147); -lean_dec(x_126); -x_149 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_149, 0, x_13); -lean_ctor_set(x_149, 1, x_145); -lean_ctor_set(x_149, 2, x_142); -x_150 = lean_array_uset(x_127, x_141, x_149); -x_151 = lean_unsigned_to_nat(4u); -x_152 = lean_nat_mul(x_148, x_151); -x_153 = lean_unsigned_to_nat(3u); -x_154 = lean_nat_div(x_152, x_153); -lean_dec(x_152); -x_155 = lean_array_get_size(x_150); -x_156 = lean_nat_dec_le(x_154, x_155); -lean_dec(x_155); -lean_dec(x_154); -if (x_156 == 0) -{ -lean_object* x_157; lean_object* x_158; size_t x_159; +lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; uint8_t x_45; +lean_dec(x_14); +x_34 = l_Std_HashMap_toArray___rarg___closed__1; +x_35 = lean_array_push(x_34, x_12); +x_36 = lean_unsigned_to_nat(1u); +x_37 = lean_nat_add(x_16, x_36); +lean_dec(x_16); +x_38 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_38, 0, x_13); +lean_ctor_set(x_38, 1, x_35); +lean_ctor_set(x_38, 2, x_32); +x_39 = lean_array_uset(x_17, x_31, x_38); +x_40 = lean_unsigned_to_nat(4u); +x_41 = lean_nat_mul(x_37, x_40); +x_42 = lean_unsigned_to_nat(3u); +x_43 = lean_nat_div(x_41, x_42); +lean_dec(x_41); +x_44 = lean_array_get_size(x_39); +x_45 = lean_nat_dec_le(x_43, x_44); +lean_dec(x_44); +lean_dec(x_43); +if (x_45 == 0) +{ +lean_object* x_46; size_t x_47; lean_inc(x_2); -x_157 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_150); -x_158 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_158, 0, x_148); -lean_ctor_set(x_158, 1, x_157); -x_159 = lean_usize_add(x_9, x_139); -x_9 = x_159; -x_10 = x_158; +x_46 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_39); +lean_ctor_set(x_10, 1, x_46); +lean_ctor_set(x_10, 0, x_37); +x_47 = lean_usize_add(x_9, x_29); +x_9 = x_47; goto _start; } else { -lean_object* x_161; size_t x_162; -x_161 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_161, 0, x_148); -lean_ctor_set(x_161, 1, x_150); -x_162 = lean_usize_add(x_9, x_139); -x_9 = x_162; -x_10 = x_161; +size_t x_49; +lean_ctor_set(x_10, 1, x_39); +lean_ctor_set(x_10, 0, x_37); +x_49 = lean_usize_add(x_9, x_29); +x_9 = x_49; goto _start; } } else { -lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; size_t x_168; +lean_object* x_51; lean_object* x_52; uint8_t x_53; lean_object* x_54; +lean_dec(x_12); lean_inc(x_5); -x_164 = lean_array_uset(x_127, x_141, x_5); +x_51 = lean_array_uset(x_17, x_31, x_5); +lean_inc(x_13); lean_inc(x_1); -x_165 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_13, x_145, x_142); -x_166 = lean_array_uset(x_164, x_141, x_165); -x_167 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_167, 0, x_126); -lean_ctor_set(x_167, 1, x_166); -x_168 = lean_usize_add(x_9, x_139); -x_9 = x_168; -x_10 = x_167; +x_52 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(x_1, lean_box(0), x_13, x_14, x_32); +lean_inc(x_52); +lean_inc(x_1); +x_53 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_52); +x_54 = lean_array_uset(x_51, x_31, x_52); +if (x_53 == 0) +{ +lean_object* x_55; lean_object* x_56; size_t x_57; +x_55 = lean_unsigned_to_nat(1u); +x_56 = lean_nat_sub(x_16, x_55); +lean_dec(x_16); +lean_ctor_set(x_10, 1, x_54); +lean_ctor_set(x_10, 0, x_56); +x_57 = lean_usize_add(x_9, x_29); +x_9 = x_57; goto _start; } -} else { -lean_object* x_170; lean_object* x_171; lean_object* x_172; uint8_t x_206; -x_170 = lean_ctor_get(x_143, 0); -lean_inc(x_170); -lean_dec(x_143); -x_171 = lean_array_push(x_170, x_12); -lean_inc(x_142); -lean_inc(x_13); -lean_inc(x_1); -x_206 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_142); -if (x_206 == 0) -{ -lean_object* x_207; -lean_dec(x_142); -x_207 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_207, 0, x_126); -lean_ctor_set(x_207, 1, x_127); -x_172 = x_207; -goto block_205; +size_t x_59; +lean_ctor_set(x_10, 1, x_54); +x_59 = lean_usize_add(x_9, x_29); +x_9 = x_59; +goto _start; +} +} } else { -lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; lean_object* x_212; lean_object* x_213; -lean_inc(x_5); -x_208 = lean_array_uset(x_127, x_141, x_5); -x_209 = lean_unsigned_to_nat(1u); -x_210 = lean_nat_sub(x_126, x_209); -lean_dec(x_126); +lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; uint64_t x_65; uint64_t x_66; uint64_t x_67; uint64_t x_68; uint64_t x_69; uint64_t x_70; uint64_t x_71; size_t x_72; size_t x_73; size_t x_74; size_t x_75; size_t x_76; lean_object* x_77; uint8_t x_78; +x_61 = lean_ctor_get(x_10, 0); +x_62 = lean_ctor_get(x_10, 1); +lean_inc(x_62); +lean_inc(x_61); +lean_dec(x_10); +x_63 = lean_array_get_size(x_62); +lean_inc(x_2); lean_inc(x_13); -lean_inc(x_1); -x_211 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_13, x_142); -x_212 = lean_array_uset(x_208, x_141, x_211); -x_213 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_213, 0, x_210); -lean_ctor_set(x_213, 1, x_212); -x_172 = x_213; -goto block_205; -} -block_205: -{ -lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; size_t x_177; size_t x_178; size_t x_179; lean_object* x_180; uint8_t x_181; -x_173 = lean_ctor_get(x_172, 0); -lean_inc(x_173); -x_174 = lean_ctor_get(x_172, 1); -lean_inc(x_174); -if (lean_is_exclusive(x_172)) { - lean_ctor_release(x_172, 0); - lean_ctor_release(x_172, 1); - x_175 = x_172; -} else { - lean_dec_ref(x_172); - x_175 = lean_box(0); -} -x_176 = lean_array_get_size(x_174); -x_177 = lean_usize_of_nat(x_176); -lean_dec(x_176); -x_178 = lean_usize_sub(x_177, x_139); -x_179 = lean_usize_land(x_137, x_178); -x_180 = lean_array_uget(x_174, x_179); -lean_inc(x_180); +x_64 = lean_apply_1(x_2, x_13); +x_65 = lean_unbox_uint64(x_64); +lean_dec(x_64); +x_66 = 32; +x_67 = lean_uint64_shift_right(x_65, x_66); +x_68 = lean_uint64_xor(x_65, x_67); +x_69 = 16; +x_70 = lean_uint64_shift_right(x_68, x_69); +x_71 = lean_uint64_xor(x_68, x_70); +x_72 = lean_uint64_to_usize(x_71); +x_73 = lean_usize_of_nat(x_63); +lean_dec(x_63); +x_74 = 1; +x_75 = lean_usize_sub(x_73, x_74); +x_76 = lean_usize_land(x_72, x_75); +x_77 = lean_array_uget(x_62, x_76); +lean_inc(x_77); lean_inc(x_13); lean_inc(x_1); -x_181 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_180); -if (x_181 == 0) +x_78 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_77); +if (x_78 == 0) { -lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; uint8_t x_191; -x_182 = lean_unsigned_to_nat(1u); -x_183 = lean_nat_add(x_173, x_182); -lean_dec(x_173); -x_184 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_184, 0, x_13); -lean_ctor_set(x_184, 1, x_171); -lean_ctor_set(x_184, 2, x_180); -x_185 = lean_array_uset(x_174, x_179, x_184); -x_186 = lean_unsigned_to_nat(4u); -x_187 = lean_nat_mul(x_183, x_186); -x_188 = lean_unsigned_to_nat(3u); -x_189 = lean_nat_div(x_187, x_188); -lean_dec(x_187); -x_190 = lean_array_get_size(x_185); -x_191 = lean_nat_dec_le(x_189, x_190); -lean_dec(x_190); -lean_dec(x_189); -if (x_191 == 0) -{ -lean_object* x_192; lean_object* x_193; size_t x_194; +lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; uint8_t x_90; +lean_dec(x_14); +x_79 = l_Std_HashMap_toArray___rarg___closed__1; +x_80 = lean_array_push(x_79, x_12); +x_81 = lean_unsigned_to_nat(1u); +x_82 = lean_nat_add(x_61, x_81); +lean_dec(x_61); +x_83 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_83, 0, x_13); +lean_ctor_set(x_83, 1, x_80); +lean_ctor_set(x_83, 2, x_77); +x_84 = lean_array_uset(x_62, x_76, x_83); +x_85 = lean_unsigned_to_nat(4u); +x_86 = lean_nat_mul(x_82, x_85); +x_87 = lean_unsigned_to_nat(3u); +x_88 = lean_nat_div(x_86, x_87); +lean_dec(x_86); +x_89 = lean_array_get_size(x_84); +x_90 = lean_nat_dec_le(x_88, x_89); +lean_dec(x_89); +lean_dec(x_88); +if (x_90 == 0) +{ +lean_object* x_91; lean_object* x_92; size_t x_93; lean_inc(x_2); -x_192 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_185); -if (lean_is_scalar(x_175)) { - x_193 = lean_alloc_ctor(0, 2, 0); -} else { - x_193 = x_175; -} -lean_ctor_set(x_193, 0, x_183); -lean_ctor_set(x_193, 1, x_192); -x_194 = lean_usize_add(x_9, x_139); -x_9 = x_194; -x_10 = x_193; +x_91 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_84); +x_92 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_92, 0, x_82); +lean_ctor_set(x_92, 1, x_91); +x_93 = lean_usize_add(x_9, x_74); +x_9 = x_93; +x_10 = x_92; goto _start; } else { -lean_object* x_196; size_t x_197; -if (lean_is_scalar(x_175)) { - x_196 = lean_alloc_ctor(0, 2, 0); -} else { - x_196 = x_175; -} -lean_ctor_set(x_196, 0, x_183); -lean_ctor_set(x_196, 1, x_185); -x_197 = lean_usize_add(x_9, x_139); -x_9 = x_197; -x_10 = x_196; +lean_object* x_95; size_t x_96; +x_95 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_95, 0, x_82); +lean_ctor_set(x_95, 1, x_84); +x_96 = lean_usize_add(x_9, x_74); +x_9 = x_96; +x_10 = x_95; goto _start; } } else { -lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; size_t x_203; +lean_object* x_98; lean_object* x_99; uint8_t x_100; lean_object* x_101; +lean_dec(x_12); lean_inc(x_5); -x_199 = lean_array_uset(x_174, x_179, x_5); +x_98 = lean_array_uset(x_62, x_76, x_5); +lean_inc(x_13); lean_inc(x_1); -x_200 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_13, x_171, x_180); -x_201 = lean_array_uset(x_199, x_179, x_200); -if (lean_is_scalar(x_175)) { - x_202 = lean_alloc_ctor(0, 2, 0); -} else { - x_202 = x_175; -} -lean_ctor_set(x_202, 0, x_173); -lean_ctor_set(x_202, 1, x_201); -x_203 = lean_usize_add(x_9, x_139); -x_9 = x_203; -x_10 = x_202; +x_99 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_Array_groupByKey___spec__1___rarg(x_1, lean_box(0), x_13, x_14, x_77); +lean_inc(x_99); +lean_inc(x_1); +x_100 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_13, x_99); +x_101 = lean_array_uset(x_98, x_76, x_99); +if (x_100 == 0) +{ +lean_object* x_102; lean_object* x_103; lean_object* x_104; size_t x_105; +x_102 = lean_unsigned_to_nat(1u); +x_103 = lean_nat_sub(x_61, x_102); +lean_dec(x_61); +x_104 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_104, 0, x_103); +lean_ctor_set(x_104, 1, x_101); +x_105 = lean_usize_add(x_9, x_74); +x_9 = x_105; +x_10 = x_104; goto _start; } +else +{ +lean_object* x_107; size_t x_108; +x_107 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_107, 0, x_61); +lean_ctor_set(x_107, 1, x_101); +x_108 = lean_usize_add(x_9, x_74); +x_9 = x_108; +x_10 = x_107; +goto _start; } } } } } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg___boxed), 10, 0); +x_3 = lean_alloc_closure((void*)(l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___boxed), 10, 0); return x_3; } } @@ -11151,7 +10206,7 @@ x_6 = lean_box(0); x_7 = lean_array_size(x_4); x_8 = 0; x_9 = l_Std_HashMap_instEmptyCollection___closed__3; -x_10 = l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_4, x_7, x_8, x_9); +x_10 = l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_4, x_7, x_8, x_9); return x_10; } } @@ -11163,7 +10218,7 @@ x_3 = lean_alloc_closure((void*)(l_Array_groupByKey___rarg___boxed), 4, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { +LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { size_t x_11; size_t x_12; lean_object* x_13; @@ -11171,7 +10226,7 @@ x_11 = lean_unbox_usize(x_8); lean_dec(x_8); x_12 = lean_unbox_usize(x_9); lean_dec(x_9); -x_13 = l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__1___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); +x_13 = l_Array_forIn_x27Unsafe_loop___at_Array_groupByKey___spec__2___rarg(x_1, x_2, x_3, x_4, x_5, x_6, x_7, x_11, x_12, x_10); lean_dec(x_7); lean_dec(x_6); lean_dec(x_4); @@ -11187,539 +10242,430 @@ lean_dec(x_4); return x_5; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { -uint8_t x_8; -x_8 = lean_usize_dec_eq(x_5, x_6); -if (x_8 == 0) +if (lean_obj_tag(x_5) == 0) { -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; -x_9 = 1; -x_10 = lean_usize_sub(x_5, x_9); -x_11 = lean_array_uget(x_4, x_10); -lean_inc(x_3); -lean_inc(x_11); -x_12 = lean_apply_1(x_3, x_11); -x_13 = !lean_is_exclusive(x_7); -if (x_13 == 0) +lean_object* x_6; lean_object* x_7; +lean_dec(x_1); +x_6 = lean_box(0); +x_7 = lean_apply_1(x_4, x_6); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; -x_14 = lean_ctor_get(x_7, 0); -x_15 = lean_ctor_get(x_7, 1); -x_16 = lean_array_get_size(x_15); -lean_inc(x_2); -lean_inc(x_12); -x_17 = lean_apply_1(x_2, x_12); -x_18 = lean_unbox_uint64(x_17); -lean_dec(x_17); -x_19 = 32; -x_20 = lean_uint64_shift_right(x_18, x_19); -x_21 = lean_uint64_xor(x_18, x_20); -x_22 = 16; -x_23 = lean_uint64_shift_right(x_21, x_22); -x_24 = lean_uint64_xor(x_21, x_23); -x_25 = lean_uint64_to_usize(x_24); -x_26 = lean_usize_of_nat(x_16); -lean_dec(x_16); -x_27 = lean_usize_sub(x_26, x_9); -x_28 = lean_usize_land(x_25, x_27); -x_29 = lean_array_uget(x_15, x_28); -lean_inc(x_29); -lean_inc(x_12); -lean_inc(x_1); -x_30 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_12, x_29); -if (lean_obj_tag(x_30) == 0) +lean_object* x_8; +lean_dec(x_3); +x_8 = lean_box(0); +return x_8; +} +else { -lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_31 = lean_box(0); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_11); -lean_ctor_set(x_32, 1, x_31); -lean_inc(x_29); -lean_inc(x_12); +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = lean_box(0); +x_11 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_11, 0, x_3); +lean_ctor_set(x_11, 1, x_9); +lean_ctor_set(x_11, 2, x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_5); +if (x_12 == 0) +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_13 = lean_ctor_get(x_5, 0); +x_14 = lean_ctor_get(x_5, 1); +x_15 = lean_ctor_get(x_5, 2); lean_inc(x_1); -x_33 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_29); -if (x_33 == 0) +lean_inc(x_3); +lean_inc(x_13); +x_16 = lean_apply_2(x_1, x_13, x_3); +x_17 = lean_unbox(x_16); +lean_dec(x_16); +if (x_17 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_nat_add(x_14, x_34); -lean_dec(x_14); -x_36 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_36, 0, x_12); -lean_ctor_set(x_36, 1, x_32); -lean_ctor_set(x_36, 2, x_29); -x_37 = lean_array_uset(x_15, x_28, x_36); -x_38 = lean_unsigned_to_nat(4u); -x_39 = lean_nat_mul(x_35, x_38); -x_40 = lean_unsigned_to_nat(3u); -x_41 = lean_nat_div(x_39, x_40); -lean_dec(x_39); -x_42 = lean_array_get_size(x_37); -x_43 = lean_nat_dec_le(x_41, x_42); -lean_dec(x_42); -lean_dec(x_41); -if (x_43 == 0) +lean_object* x_18; +x_18 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_3, x_4, x_15); +lean_ctor_set(x_5, 2, x_18); +return x_5; +} +else { -lean_object* x_44; -lean_inc(x_2); -x_44 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_37); -lean_ctor_set(x_7, 1, x_44); -lean_ctor_set(x_7, 0, x_35); -x_5 = x_10; -goto _start; +lean_object* x_19; lean_object* x_20; +lean_dec(x_13); +lean_dec(x_1); +x_19 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_19, 0, x_14); +x_20 = lean_apply_1(x_4, x_19); +if (lean_obj_tag(x_20) == 0) +{ +lean_free_object(x_5); +lean_dec(x_3); +return x_15; } else { -lean_ctor_set(x_7, 1, x_37); -lean_ctor_set(x_7, 0, x_35); -x_5 = x_10; -goto _start; +lean_object* x_21; +x_21 = lean_ctor_get(x_20, 0); +lean_inc(x_21); +lean_dec(x_20); +lean_ctor_set(x_5, 1, x_21); +lean_ctor_set(x_5, 0, x_3); +return x_5; +} } } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; -x_47 = lean_box(0); -x_48 = lean_array_uset(x_15, x_28, x_47); +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; uint8_t x_26; +x_22 = lean_ctor_get(x_5, 0); +x_23 = lean_ctor_get(x_5, 1); +x_24 = lean_ctor_get(x_5, 2); +lean_inc(x_24); +lean_inc(x_23); +lean_inc(x_22); +lean_dec(x_5); lean_inc(x_1); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_32, x_29); -x_50 = lean_array_uset(x_48, x_28, x_49); -lean_ctor_set(x_7, 1, x_50); -x_5 = x_10; -goto _start; +lean_inc(x_3); +lean_inc(x_22); +x_25 = lean_apply_2(x_1, x_22, x_3); +x_26 = lean_unbox(x_25); +lean_dec(x_25); +if (x_26 == 0) +{ +lean_object* x_27; lean_object* x_28; +x_27 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_3, x_4, x_24); +x_28 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_28, 0, x_22); +lean_ctor_set(x_28, 1, x_23); +lean_ctor_set(x_28, 2, x_27); +return x_28; } +else +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_22); +lean_dec(x_1); +x_29 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_29, 0, x_23); +x_30 = lean_apply_1(x_4, x_29); +if (lean_obj_tag(x_30) == 0) +{ +lean_dec(x_3); +return x_24; } else { -lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_112; -x_52 = lean_ctor_get(x_30, 0); -lean_inc(x_52); +lean_object* x_31; lean_object* x_32; +x_31 = lean_ctor_get(x_30, 0); +lean_inc(x_31); lean_dec(x_30); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_11); -lean_ctor_set(x_53, 1, x_52); -lean_inc(x_29); -lean_inc(x_12); -lean_inc(x_1); -x_112 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_29); -if (x_112 == 0) +x_32 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_32, 0, x_3); +lean_ctor_set(x_32, 1, x_31); +lean_ctor_set(x_32, 2, x_24); +return x_32; +} +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1(lean_object* x_1) { +_start: { -lean_dec(x_29); -x_54 = x_7; -goto block_111; +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg), 5, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_3 = lean_box(0); +x_4 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_3); +x_5 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; } else { -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_113 = lean_box(0); -x_114 = lean_array_uset(x_15, x_28, x_113); -x_115 = lean_unsigned_to_nat(1u); -x_116 = lean_nat_sub(x_14, x_115); -lean_dec(x_14); -lean_inc(x_12); -lean_inc(x_1); -x_117 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_12, x_29); -x_118 = lean_array_uset(x_114, x_28, x_117); -lean_ctor_set(x_7, 1, x_118); -lean_ctor_set(x_7, 0, x_116); -x_54 = x_7; -goto block_111; +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_8, 0, x_1); +lean_ctor_set(x_8, 1, x_7); +lean_ctor_set(x_2, 0, x_8); +return x_2; } -block_111: +else { -uint8_t x_55; -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_10, 0, x_1); +lean_ctor_set(x_10, 1, x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { +_start: { -lean_object* x_56; lean_object* x_57; lean_object* x_58; size_t x_59; size_t x_60; size_t x_61; lean_object* x_62; uint8_t x_63; -x_56 = lean_ctor_get(x_54, 0); -x_57 = lean_ctor_get(x_54, 1); -x_58 = lean_array_get_size(x_57); -x_59 = lean_usize_of_nat(x_58); -lean_dec(x_58); -x_60 = lean_usize_sub(x_59, x_9); -x_61 = lean_usize_land(x_25, x_60); -x_62 = lean_array_uget(x_57, x_61); -lean_inc(x_62); +uint8_t x_8; +x_8 = lean_usize_dec_eq(x_5, x_6); +if (x_8 == 0) +{ +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; +x_9 = 1; +x_10 = lean_usize_sub(x_5, x_9); +x_11 = lean_array_uget(x_4, x_10); +lean_inc(x_3); +lean_inc(x_11); +x_12 = lean_apply_1(x_3, x_11); +lean_inc(x_11); +x_13 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_13, 0, x_11); +x_14 = !lean_is_exclusive(x_7); +if (x_14 == 0) +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; lean_object* x_30; uint8_t x_31; +x_15 = lean_ctor_get(x_7, 0); +x_16 = lean_ctor_get(x_7, 1); +x_17 = lean_array_get_size(x_16); +lean_inc(x_2); +lean_inc(x_12); +x_18 = lean_apply_1(x_2, x_12); +x_19 = lean_unbox_uint64(x_18); +lean_dec(x_18); +x_20 = 32; +x_21 = lean_uint64_shift_right(x_19, x_20); +x_22 = lean_uint64_xor(x_19, x_21); +x_23 = 16; +x_24 = lean_uint64_shift_right(x_22, x_23); +x_25 = lean_uint64_xor(x_22, x_24); +x_26 = lean_uint64_to_usize(x_25); +x_27 = lean_usize_of_nat(x_17); +lean_dec(x_17); +x_28 = lean_usize_sub(x_27, x_9); +x_29 = lean_usize_land(x_26, x_28); +x_30 = lean_array_uget(x_16, x_29); +lean_inc(x_30); lean_inc(x_12); lean_inc(x_1); -x_63 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_62); -if (x_63 == 0) +x_31 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_30); +if (x_31 == 0) { -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -x_64 = lean_unsigned_to_nat(1u); -x_65 = lean_nat_add(x_56, x_64); -lean_dec(x_56); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_12); -lean_ctor_set(x_66, 1, x_53); -lean_ctor_set(x_66, 2, x_62); -x_67 = lean_array_uset(x_57, x_61, x_66); -x_68 = lean_unsigned_to_nat(4u); -x_69 = lean_nat_mul(x_65, x_68); -x_70 = lean_unsigned_to_nat(3u); -x_71 = lean_nat_div(x_69, x_70); -lean_dec(x_69); -x_72 = lean_array_get_size(x_67); -x_73 = lean_nat_dec_le(x_71, x_72); -lean_dec(x_72); -lean_dec(x_71); -if (x_73 == 0) +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_dec(x_13); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_11); +lean_ctor_set(x_33, 1, x_32); +x_34 = lean_unsigned_to_nat(1u); +x_35 = lean_nat_add(x_15, x_34); +lean_dec(x_15); +x_36 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_36, 0, x_12); +lean_ctor_set(x_36, 1, x_33); +lean_ctor_set(x_36, 2, x_30); +x_37 = lean_array_uset(x_16, x_29, x_36); +x_38 = lean_unsigned_to_nat(4u); +x_39 = lean_nat_mul(x_35, x_38); +x_40 = lean_unsigned_to_nat(3u); +x_41 = lean_nat_div(x_39, x_40); +lean_dec(x_39); +x_42 = lean_array_get_size(x_37); +x_43 = lean_nat_dec_le(x_41, x_42); +lean_dec(x_42); +lean_dec(x_41); +if (x_43 == 0) { -lean_object* x_74; +lean_object* x_44; lean_inc(x_2); -x_74 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_67); -lean_ctor_set(x_54, 1, x_74); -lean_ctor_set(x_54, 0, x_65); -x_5 = x_10; -x_7 = x_54; -goto _start; -} -else -{ -lean_ctor_set(x_54, 1, x_67); -lean_ctor_set(x_54, 0, x_65); +x_44 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_37); +lean_ctor_set(x_7, 1, x_44); +lean_ctor_set(x_7, 0, x_35); x_5 = x_10; -x_7 = x_54; goto _start; } -} else { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_77 = lean_box(0); -x_78 = lean_array_uset(x_57, x_61, x_77); -lean_inc(x_1); -x_79 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_53, x_62); -x_80 = lean_array_uset(x_78, x_61, x_79); -lean_ctor_set(x_54, 1, x_80); +lean_ctor_set(x_7, 1, x_37); +lean_ctor_set(x_7, 0, x_35); x_5 = x_10; -x_7 = x_54; goto _start; } } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; size_t x_85; size_t x_86; size_t x_87; lean_object* x_88; uint8_t x_89; -x_82 = lean_ctor_get(x_54, 0); -x_83 = lean_ctor_get(x_54, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_54); -x_84 = lean_array_get_size(x_83); -x_85 = lean_usize_of_nat(x_84); -lean_dec(x_84); -x_86 = lean_usize_sub(x_85, x_9); -x_87 = lean_usize_land(x_25, x_86); -x_88 = lean_array_uget(x_83, x_87); -lean_inc(x_88); +lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +lean_dec(x_11); +x_47 = lean_box(0); +x_48 = lean_array_uset(x_16, x_29, x_47); lean_inc(x_12); lean_inc(x_1); -x_89 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_88); -if (x_89 == 0) -{ -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; -x_90 = lean_unsigned_to_nat(1u); -x_91 = lean_nat_add(x_82, x_90); -lean_dec(x_82); -x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_12); -lean_ctor_set(x_92, 1, x_53); -lean_ctor_set(x_92, 2, x_88); -x_93 = lean_array_uset(x_83, x_87, x_92); -x_94 = lean_unsigned_to_nat(4u); -x_95 = lean_nat_mul(x_91, x_94); -x_96 = lean_unsigned_to_nat(3u); -x_97 = lean_nat_div(x_95, x_96); -lean_dec(x_95); -x_98 = lean_array_get_size(x_93); -x_99 = lean_nat_dec_le(x_97, x_98); -lean_dec(x_98); -lean_dec(x_97); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; -lean_inc(x_2); -x_100 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_93); -x_101 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_101, 0, x_91); -lean_ctor_set(x_101, 1, x_100); -x_5 = x_10; -x_7 = x_101; -goto _start; -} -else +x_49 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_12, x_13, x_30); +lean_inc(x_49); +lean_inc(x_1); +x_50 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_49); +x_51 = lean_array_uset(x_48, x_29, x_49); +if (x_50 == 0) { -lean_object* x_103; -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_91); -lean_ctor_set(x_103, 1, x_93); +lean_object* x_52; lean_object* x_53; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_sub(x_15, x_52); +lean_dec(x_15); +lean_ctor_set(x_7, 1, x_51); +lean_ctor_set(x_7, 0, x_53); x_5 = x_10; -x_7 = x_103; goto _start; } -} else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_105 = lean_box(0); -x_106 = lean_array_uset(x_83, x_87, x_105); -lean_inc(x_1); -x_107 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_53, x_88); -x_108 = lean_array_uset(x_106, x_87, x_107); -x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_82); -lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_7, 1, x_51); x_5 = x_10; -x_7 = x_109; goto _start; } } } -} -} else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint64_t x_123; uint64_t x_124; uint64_t x_125; uint64_t x_126; uint64_t x_127; uint64_t x_128; uint64_t x_129; size_t x_130; size_t x_131; size_t x_132; size_t x_133; lean_object* x_134; lean_object* x_135; -x_119 = lean_ctor_get(x_7, 0); -x_120 = lean_ctor_get(x_7, 1); -lean_inc(x_120); -lean_inc(x_119); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint64_t x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; size_t x_67; size_t x_68; size_t x_69; size_t x_70; lean_object* x_71; uint8_t x_72; +x_56 = lean_ctor_get(x_7, 0); +x_57 = lean_ctor_get(x_7, 1); +lean_inc(x_57); +lean_inc(x_56); lean_dec(x_7); -x_121 = lean_array_get_size(x_120); +x_58 = lean_array_get_size(x_57); lean_inc(x_2); lean_inc(x_12); -x_122 = lean_apply_1(x_2, x_12); -x_123 = lean_unbox_uint64(x_122); -lean_dec(x_122); -x_124 = 32; -x_125 = lean_uint64_shift_right(x_123, x_124); -x_126 = lean_uint64_xor(x_123, x_125); -x_127 = 16; -x_128 = lean_uint64_shift_right(x_126, x_127); -x_129 = lean_uint64_xor(x_126, x_128); -x_130 = lean_uint64_to_usize(x_129); -x_131 = lean_usize_of_nat(x_121); -lean_dec(x_121); -x_132 = lean_usize_sub(x_131, x_9); -x_133 = lean_usize_land(x_130, x_132); -x_134 = lean_array_uget(x_120, x_133); -lean_inc(x_134); -lean_inc(x_12); -lean_inc(x_1); -x_135 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_12, x_134); -if (lean_obj_tag(x_135) == 0) -{ -lean_object* x_136; lean_object* x_137; uint8_t x_138; -x_136 = lean_box(0); -x_137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_137, 0, x_11); -lean_ctor_set(x_137, 1, x_136); -lean_inc(x_134); +x_59 = lean_apply_1(x_2, x_12); +x_60 = lean_unbox_uint64(x_59); +lean_dec(x_59); +x_61 = 32; +x_62 = lean_uint64_shift_right(x_60, x_61); +x_63 = lean_uint64_xor(x_60, x_62); +x_64 = 16; +x_65 = lean_uint64_shift_right(x_63, x_64); +x_66 = lean_uint64_xor(x_63, x_65); +x_67 = lean_uint64_to_usize(x_66); +x_68 = lean_usize_of_nat(x_58); +lean_dec(x_58); +x_69 = lean_usize_sub(x_68, x_9); +x_70 = lean_usize_land(x_67, x_69); +x_71 = lean_array_uget(x_57, x_70); +lean_inc(x_71); lean_inc(x_12); lean_inc(x_1); -x_138 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_134); -if (x_138 == 0) -{ -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; -x_139 = lean_unsigned_to_nat(1u); -x_140 = lean_nat_add(x_119, x_139); -lean_dec(x_119); -x_141 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_141, 0, x_12); -lean_ctor_set(x_141, 1, x_137); -lean_ctor_set(x_141, 2, x_134); -x_142 = lean_array_uset(x_120, x_133, x_141); -x_143 = lean_unsigned_to_nat(4u); -x_144 = lean_nat_mul(x_140, x_143); -x_145 = lean_unsigned_to_nat(3u); -x_146 = lean_nat_div(x_144, x_145); -lean_dec(x_144); -x_147 = lean_array_get_size(x_142); -x_148 = lean_nat_dec_le(x_146, x_147); -lean_dec(x_147); -lean_dec(x_146); -if (x_148 == 0) +x_72 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_71); +if (x_72 == 0) { -lean_object* x_149; lean_object* x_150; -lean_inc(x_2); -x_149 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_142); -x_150 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_150, 0, x_140); -lean_ctor_set(x_150, 1, x_149); -x_5 = x_10; -x_7 = x_150; -goto _start; -} -else +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +lean_dec(x_13); +x_73 = lean_box(0); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_11); +lean_ctor_set(x_74, 1, x_73); +x_75 = lean_unsigned_to_nat(1u); +x_76 = lean_nat_add(x_56, x_75); +lean_dec(x_56); +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_12); +lean_ctor_set(x_77, 1, x_74); +lean_ctor_set(x_77, 2, x_71); +x_78 = lean_array_uset(x_57, x_70, x_77); +x_79 = lean_unsigned_to_nat(4u); +x_80 = lean_nat_mul(x_76, x_79); +x_81 = lean_unsigned_to_nat(3u); +x_82 = lean_nat_div(x_80, x_81); +lean_dec(x_80); +x_83 = lean_array_get_size(x_78); +x_84 = lean_nat_dec_le(x_82, x_83); +lean_dec(x_83); +lean_dec(x_82); +if (x_84 == 0) { -lean_object* x_152; -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_140); -lean_ctor_set(x_152, 1, x_142); +lean_object* x_85; lean_object* x_86; +lean_inc(x_2); +x_85 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_78); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_76); +lean_ctor_set(x_86, 1, x_85); x_5 = x_10; -x_7 = x_152; +x_7 = x_86; goto _start; } -} else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_154 = lean_box(0); -x_155 = lean_array_uset(x_120, x_133, x_154); -lean_inc(x_1); -x_156 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_137, x_134); -x_157 = lean_array_uset(x_155, x_133, x_156); -x_158 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_158, 0, x_119); -lean_ctor_set(x_158, 1, x_157); +lean_object* x_88; +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_76); +lean_ctor_set(x_88, 1, x_78); x_5 = x_10; -x_7 = x_158; +x_7 = x_88; goto _start; } } else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_194; -x_160 = lean_ctor_get(x_135, 0); -lean_inc(x_160); -lean_dec(x_135); -x_161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_161, 0, x_11); -lean_ctor_set(x_161, 1, x_160); -lean_inc(x_134); -lean_inc(x_12); -lean_inc(x_1); -x_194 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_134); -if (x_194 == 0) -{ -lean_object* x_195; -lean_dec(x_134); -x_195 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_195, 0, x_119); -lean_ctor_set(x_195, 1, x_120); -x_162 = x_195; -goto block_193; -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_196 = lean_box(0); -x_197 = lean_array_uset(x_120, x_133, x_196); -x_198 = lean_unsigned_to_nat(1u); -x_199 = lean_nat_sub(x_119, x_198); -lean_dec(x_119); +lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; +lean_dec(x_11); +x_90 = lean_box(0); +x_91 = lean_array_uset(x_57, x_70, x_90); lean_inc(x_12); lean_inc(x_1); -x_200 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_12, x_134); -x_201 = lean_array_uset(x_197, x_133, x_200); -x_202 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_202, 0, x_199); -lean_ctor_set(x_202, 1, x_201); -x_162 = x_202; -goto block_193; -} -block_193: -{ -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; size_t x_167; size_t x_168; size_t x_169; lean_object* x_170; uint8_t x_171; -x_163 = lean_ctor_get(x_162, 0); -lean_inc(x_163); -x_164 = lean_ctor_get(x_162, 1); -lean_inc(x_164); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_165 = x_162; -} else { - lean_dec_ref(x_162); - x_165 = lean_box(0); -} -x_166 = lean_array_get_size(x_164); -x_167 = lean_usize_of_nat(x_166); -lean_dec(x_166); -x_168 = lean_usize_sub(x_167, x_9); -x_169 = lean_usize_land(x_130, x_168); -x_170 = lean_array_uget(x_164, x_169); -lean_inc(x_170); -lean_inc(x_12); +x_92 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_12, x_13, x_71); +lean_inc(x_92); lean_inc(x_1); -x_171 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_170); -if (x_171 == 0) -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; uint8_t x_181; -x_172 = lean_unsigned_to_nat(1u); -x_173 = lean_nat_add(x_163, x_172); -lean_dec(x_163); -x_174 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_174, 0, x_12); -lean_ctor_set(x_174, 1, x_161); -lean_ctor_set(x_174, 2, x_170); -x_175 = lean_array_uset(x_164, x_169, x_174); -x_176 = lean_unsigned_to_nat(4u); -x_177 = lean_nat_mul(x_173, x_176); -x_178 = lean_unsigned_to_nat(3u); -x_179 = lean_nat_div(x_177, x_178); -lean_dec(x_177); -x_180 = lean_array_get_size(x_175); -x_181 = lean_nat_dec_le(x_179, x_180); -lean_dec(x_180); -lean_dec(x_179); -if (x_181 == 0) -{ -lean_object* x_182; lean_object* x_183; -lean_inc(x_2); -x_182 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_175); -if (lean_is_scalar(x_165)) { - x_183 = lean_alloc_ctor(0, 2, 0); -} else { - x_183 = x_165; -} -lean_ctor_set(x_183, 0, x_173); -lean_ctor_set(x_183, 1, x_182); -x_5 = x_10; -x_7 = x_183; -goto _start; -} -else +x_93 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_92); +x_94 = lean_array_uset(x_91, x_70, x_92); +if (x_93 == 0) { -lean_object* x_185; -if (lean_is_scalar(x_165)) { - x_185 = lean_alloc_ctor(0, 2, 0); -} else { - x_185 = x_165; -} -lean_ctor_set(x_185, 0, x_173); -lean_ctor_set(x_185, 1, x_175); +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_unsigned_to_nat(1u); +x_96 = lean_nat_sub(x_56, x_95); +lean_dec(x_56); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); x_5 = x_10; -x_7 = x_185; +x_7 = x_97; goto _start; } -} else { -lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_187 = lean_box(0); -x_188 = lean_array_uset(x_164, x_169, x_187); -lean_inc(x_1); -x_189 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_161, x_170); -x_190 = lean_array_uset(x_188, x_169, x_189); -if (lean_is_scalar(x_165)) { - x_191 = lean_alloc_ctor(0, 2, 0); -} else { - x_191 = x_165; -} -lean_ctor_set(x_191, 0, x_163); -lean_ctor_set(x_191, 1, x_190); +lean_object* x_99; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_56); +lean_ctor_set(x_99, 1, x_94); x_5 = x_10; -x_7 = x_191; +x_7 = x_99; goto _start; } } } } -} else { lean_dec(x_3); @@ -11729,78 +10675,75 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg___boxed), 7, 0); +x_3 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___boxed), 7, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, size_t x_5, size_t x_6, lean_object* x_7) { _start: { uint8_t x_8; x_8 = lean_usize_dec_eq(x_5, x_6); if (x_8 == 0) { -size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; +size_t x_9; size_t x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; uint8_t x_14; x_9 = 1; x_10 = lean_usize_sub(x_5, x_9); x_11 = lean_array_uget(x_4, x_10); lean_inc(x_3); lean_inc(x_11); x_12 = lean_apply_1(x_3, x_11); -x_13 = !lean_is_exclusive(x_7); -if (x_13 == 0) +lean_inc(x_11); +x_13 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___lambda__1), 2, 1); +lean_closure_set(x_13, 0, x_11); +x_14 = !lean_is_exclusive(x_7); +if (x_14 == 0) { -lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint64_t x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; size_t x_25; size_t x_26; size_t x_27; size_t x_28; lean_object* x_29; lean_object* x_30; -x_14 = lean_ctor_get(x_7, 0); -x_15 = lean_ctor_get(x_7, 1); -x_16 = lean_array_get_size(x_15); +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; uint64_t x_19; uint64_t x_20; uint64_t x_21; uint64_t x_22; uint64_t x_23; uint64_t x_24; uint64_t x_25; size_t x_26; size_t x_27; size_t x_28; size_t x_29; lean_object* x_30; uint8_t x_31; +x_15 = lean_ctor_get(x_7, 0); +x_16 = lean_ctor_get(x_7, 1); +x_17 = lean_array_get_size(x_16); lean_inc(x_2); lean_inc(x_12); -x_17 = lean_apply_1(x_2, x_12); -x_18 = lean_unbox_uint64(x_17); +x_18 = lean_apply_1(x_2, x_12); +x_19 = lean_unbox_uint64(x_18); +lean_dec(x_18); +x_20 = 32; +x_21 = lean_uint64_shift_right(x_19, x_20); +x_22 = lean_uint64_xor(x_19, x_21); +x_23 = 16; +x_24 = lean_uint64_shift_right(x_22, x_23); +x_25 = lean_uint64_xor(x_22, x_24); +x_26 = lean_uint64_to_usize(x_25); +x_27 = lean_usize_of_nat(x_17); lean_dec(x_17); -x_19 = 32; -x_20 = lean_uint64_shift_right(x_18, x_19); -x_21 = lean_uint64_xor(x_18, x_20); -x_22 = 16; -x_23 = lean_uint64_shift_right(x_21, x_22); -x_24 = lean_uint64_xor(x_21, x_23); -x_25 = lean_uint64_to_usize(x_24); -x_26 = lean_usize_of_nat(x_16); -lean_dec(x_16); -x_27 = lean_usize_sub(x_26, x_9); -x_28 = lean_usize_land(x_25, x_27); -x_29 = lean_array_uget(x_15, x_28); -lean_inc(x_29); -lean_inc(x_12); -lean_inc(x_1); -x_30 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_12, x_29); -if (lean_obj_tag(x_30) == 0) -{ -lean_object* x_31; lean_object* x_32; uint8_t x_33; -x_31 = lean_box(0); -x_32 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_32, 0, x_11); -lean_ctor_set(x_32, 1, x_31); -lean_inc(x_29); +x_28 = lean_usize_sub(x_27, x_9); +x_29 = lean_usize_land(x_26, x_28); +x_30 = lean_array_uget(x_16, x_29); +lean_inc(x_30); lean_inc(x_12); lean_inc(x_1); -x_33 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_29); -if (x_33 == 0) +x_31 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_30); +if (x_31 == 0) { -lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; +lean_dec(x_13); +x_32 = lean_box(0); +x_33 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_33, 0, x_11); +lean_ctor_set(x_33, 1, x_32); x_34 = lean_unsigned_to_nat(1u); -x_35 = lean_nat_add(x_14, x_34); -lean_dec(x_14); +x_35 = lean_nat_add(x_15, x_34); +lean_dec(x_15); x_36 = lean_alloc_ctor(1, 3, 0); lean_ctor_set(x_36, 0, x_12); -lean_ctor_set(x_36, 1, x_32); -lean_ctor_set(x_36, 2, x_29); -x_37 = lean_array_uset(x_15, x_28, x_36); +lean_ctor_set(x_36, 1, x_33); +lean_ctor_set(x_36, 2, x_30); +x_37 = lean_array_uset(x_16, x_29, x_36); x_38 = lean_unsigned_to_nat(4u); x_39 = lean_nat_mul(x_35, x_38); x_40 = lean_unsigned_to_nat(3u); @@ -11830,446 +10773,153 @@ goto _start; } else { -lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +lean_object* x_47; lean_object* x_48; lean_object* x_49; uint8_t x_50; lean_object* x_51; +lean_dec(x_11); x_47 = lean_box(0); -x_48 = lean_array_uset(x_15, x_28, x_47); -lean_inc(x_1); -x_49 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_32, x_29); -x_50 = lean_array_uset(x_48, x_28, x_49); -lean_ctor_set(x_7, 1, x_50); -x_5 = x_10; -goto _start; -} -} -else -{ -lean_object* x_52; lean_object* x_53; lean_object* x_54; uint8_t x_112; -x_52 = lean_ctor_get(x_30, 0); -lean_inc(x_52); -lean_dec(x_30); -x_53 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_53, 0, x_11); -lean_ctor_set(x_53, 1, x_52); -lean_inc(x_29); -lean_inc(x_12); -lean_inc(x_1); -x_112 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_29); -if (x_112 == 0) -{ -lean_dec(x_29); -x_54 = x_7; -goto block_111; -} -else -{ -lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; -x_113 = lean_box(0); -x_114 = lean_array_uset(x_15, x_28, x_113); -x_115 = lean_unsigned_to_nat(1u); -x_116 = lean_nat_sub(x_14, x_115); -lean_dec(x_14); -lean_inc(x_12); -lean_inc(x_1); -x_117 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_12, x_29); -x_118 = lean_array_uset(x_114, x_28, x_117); -lean_ctor_set(x_7, 1, x_118); -lean_ctor_set(x_7, 0, x_116); -x_54 = x_7; -goto block_111; -} -block_111: -{ -uint8_t x_55; -x_55 = !lean_is_exclusive(x_54); -if (x_55 == 0) -{ -lean_object* x_56; lean_object* x_57; lean_object* x_58; size_t x_59; size_t x_60; size_t x_61; lean_object* x_62; uint8_t x_63; -x_56 = lean_ctor_get(x_54, 0); -x_57 = lean_ctor_get(x_54, 1); -x_58 = lean_array_get_size(x_57); -x_59 = lean_usize_of_nat(x_58); -lean_dec(x_58); -x_60 = lean_usize_sub(x_59, x_9); -x_61 = lean_usize_land(x_25, x_60); -x_62 = lean_array_uget(x_57, x_61); -lean_inc(x_62); +x_48 = lean_array_uset(x_16, x_29, x_47); lean_inc(x_12); lean_inc(x_1); -x_63 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_62); -if (x_63 == 0) -{ -lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; uint8_t x_73; -x_64 = lean_unsigned_to_nat(1u); -x_65 = lean_nat_add(x_56, x_64); -lean_dec(x_56); -x_66 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_66, 0, x_12); -lean_ctor_set(x_66, 1, x_53); -lean_ctor_set(x_66, 2, x_62); -x_67 = lean_array_uset(x_57, x_61, x_66); -x_68 = lean_unsigned_to_nat(4u); -x_69 = lean_nat_mul(x_65, x_68); -x_70 = lean_unsigned_to_nat(3u); -x_71 = lean_nat_div(x_69, x_70); -lean_dec(x_69); -x_72 = lean_array_get_size(x_67); -x_73 = lean_nat_dec_le(x_71, x_72); -lean_dec(x_72); -lean_dec(x_71); -if (x_73 == 0) -{ -lean_object* x_74; -lean_inc(x_2); -x_74 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_67); -lean_ctor_set(x_54, 1, x_74); -lean_ctor_set(x_54, 0, x_65); -x_5 = x_10; -x_7 = x_54; -goto _start; -} -else -{ -lean_ctor_set(x_54, 1, x_67); -lean_ctor_set(x_54, 0, x_65); -x_5 = x_10; -x_7 = x_54; -goto _start; -} -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; -x_77 = lean_box(0); -x_78 = lean_array_uset(x_57, x_61, x_77); -lean_inc(x_1); -x_79 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_53, x_62); -x_80 = lean_array_uset(x_78, x_61, x_79); -lean_ctor_set(x_54, 1, x_80); -x_5 = x_10; -x_7 = x_54; -goto _start; -} -} -else -{ -lean_object* x_82; lean_object* x_83; lean_object* x_84; size_t x_85; size_t x_86; size_t x_87; lean_object* x_88; uint8_t x_89; -x_82 = lean_ctor_get(x_54, 0); -x_83 = lean_ctor_get(x_54, 1); -lean_inc(x_83); -lean_inc(x_82); -lean_dec(x_54); -x_84 = lean_array_get_size(x_83); -x_85 = lean_usize_of_nat(x_84); -lean_dec(x_84); -x_86 = lean_usize_sub(x_85, x_9); -x_87 = lean_usize_land(x_25, x_86); -x_88 = lean_array_uget(x_83, x_87); -lean_inc(x_88); -lean_inc(x_12); +x_49 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_12, x_13, x_30); +lean_inc(x_49); lean_inc(x_1); -x_89 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_88); -if (x_89 == 0) +x_50 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_49); +x_51 = lean_array_uset(x_48, x_29, x_49); +if (x_50 == 0) { -lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; uint8_t x_99; -x_90 = lean_unsigned_to_nat(1u); -x_91 = lean_nat_add(x_82, x_90); -lean_dec(x_82); -x_92 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_92, 0, x_12); -lean_ctor_set(x_92, 1, x_53); -lean_ctor_set(x_92, 2, x_88); -x_93 = lean_array_uset(x_83, x_87, x_92); -x_94 = lean_unsigned_to_nat(4u); -x_95 = lean_nat_mul(x_91, x_94); -x_96 = lean_unsigned_to_nat(3u); -x_97 = lean_nat_div(x_95, x_96); -lean_dec(x_95); -x_98 = lean_array_get_size(x_93); -x_99 = lean_nat_dec_le(x_97, x_98); -lean_dec(x_98); -lean_dec(x_97); -if (x_99 == 0) -{ -lean_object* x_100; lean_object* x_101; -lean_inc(x_2); -x_100 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_93); -x_101 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_101, 0, x_91); -lean_ctor_set(x_101, 1, x_100); -x_5 = x_10; -x_7 = x_101; -goto _start; -} -else -{ -lean_object* x_103; -x_103 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_103, 0, x_91); -lean_ctor_set(x_103, 1, x_93); +lean_object* x_52; lean_object* x_53; +x_52 = lean_unsigned_to_nat(1u); +x_53 = lean_nat_sub(x_15, x_52); +lean_dec(x_15); +lean_ctor_set(x_7, 1, x_51); +lean_ctor_set(x_7, 0, x_53); x_5 = x_10; -x_7 = x_103; goto _start; } -} else { -lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; -x_105 = lean_box(0); -x_106 = lean_array_uset(x_83, x_87, x_105); -lean_inc(x_1); -x_107 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_53, x_88); -x_108 = lean_array_uset(x_106, x_87, x_107); -x_109 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_109, 0, x_82); -lean_ctor_set(x_109, 1, x_108); +lean_ctor_set(x_7, 1, x_51); x_5 = x_10; -x_7 = x_109; goto _start; } } } -} -} else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; uint64_t x_123; uint64_t x_124; uint64_t x_125; uint64_t x_126; uint64_t x_127; uint64_t x_128; uint64_t x_129; size_t x_130; size_t x_131; size_t x_132; size_t x_133; lean_object* x_134; lean_object* x_135; -x_119 = lean_ctor_get(x_7, 0); -x_120 = lean_ctor_get(x_7, 1); -lean_inc(x_120); -lean_inc(x_119); +lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; uint64_t x_60; uint64_t x_61; uint64_t x_62; uint64_t x_63; uint64_t x_64; uint64_t x_65; uint64_t x_66; size_t x_67; size_t x_68; size_t x_69; size_t x_70; lean_object* x_71; uint8_t x_72; +x_56 = lean_ctor_get(x_7, 0); +x_57 = lean_ctor_get(x_7, 1); +lean_inc(x_57); +lean_inc(x_56); lean_dec(x_7); -x_121 = lean_array_get_size(x_120); +x_58 = lean_array_get_size(x_57); lean_inc(x_2); lean_inc(x_12); -x_122 = lean_apply_1(x_2, x_12); -x_123 = lean_unbox_uint64(x_122); -lean_dec(x_122); -x_124 = 32; -x_125 = lean_uint64_shift_right(x_123, x_124); -x_126 = lean_uint64_xor(x_123, x_125); -x_127 = 16; -x_128 = lean_uint64_shift_right(x_126, x_127); -x_129 = lean_uint64_xor(x_126, x_128); -x_130 = lean_uint64_to_usize(x_129); -x_131 = lean_usize_of_nat(x_121); -lean_dec(x_121); -x_132 = lean_usize_sub(x_131, x_9); -x_133 = lean_usize_land(x_130, x_132); -x_134 = lean_array_uget(x_120, x_133); -lean_inc(x_134); -lean_inc(x_12); -lean_inc(x_1); -x_135 = l_Std_DHashMap_Internal_AssocList_get_x3f___rarg(x_1, x_12, x_134); -if (lean_obj_tag(x_135) == 0) -{ -lean_object* x_136; lean_object* x_137; uint8_t x_138; -x_136 = lean_box(0); -x_137 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_137, 0, x_11); -lean_ctor_set(x_137, 1, x_136); -lean_inc(x_134); +x_59 = lean_apply_1(x_2, x_12); +x_60 = lean_unbox_uint64(x_59); +lean_dec(x_59); +x_61 = 32; +x_62 = lean_uint64_shift_right(x_60, x_61); +x_63 = lean_uint64_xor(x_60, x_62); +x_64 = 16; +x_65 = lean_uint64_shift_right(x_63, x_64); +x_66 = lean_uint64_xor(x_63, x_65); +x_67 = lean_uint64_to_usize(x_66); +x_68 = lean_usize_of_nat(x_58); +lean_dec(x_58); +x_69 = lean_usize_sub(x_68, x_9); +x_70 = lean_usize_land(x_67, x_69); +x_71 = lean_array_uget(x_57, x_70); +lean_inc(x_71); lean_inc(x_12); lean_inc(x_1); -x_138 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_134); -if (x_138 == 0) -{ -lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; uint8_t x_148; -x_139 = lean_unsigned_to_nat(1u); -x_140 = lean_nat_add(x_119, x_139); -lean_dec(x_119); -x_141 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_141, 0, x_12); -lean_ctor_set(x_141, 1, x_137); -lean_ctor_set(x_141, 2, x_134); -x_142 = lean_array_uset(x_120, x_133, x_141); -x_143 = lean_unsigned_to_nat(4u); -x_144 = lean_nat_mul(x_140, x_143); -x_145 = lean_unsigned_to_nat(3u); -x_146 = lean_nat_div(x_144, x_145); -lean_dec(x_144); -x_147 = lean_array_get_size(x_142); -x_148 = lean_nat_dec_le(x_146, x_147); -lean_dec(x_147); -lean_dec(x_146); -if (x_148 == 0) +x_72 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_71); +if (x_72 == 0) { -lean_object* x_149; lean_object* x_150; -lean_inc(x_2); -x_149 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_142); -x_150 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_150, 0, x_140); -lean_ctor_set(x_150, 1, x_149); -x_5 = x_10; -x_7 = x_150; -goto _start; -} -else +lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; uint8_t x_84; +lean_dec(x_13); +x_73 = lean_box(0); +x_74 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_74, 0, x_11); +lean_ctor_set(x_74, 1, x_73); +x_75 = lean_unsigned_to_nat(1u); +x_76 = lean_nat_add(x_56, x_75); +lean_dec(x_56); +x_77 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_77, 0, x_12); +lean_ctor_set(x_77, 1, x_74); +lean_ctor_set(x_77, 2, x_71); +x_78 = lean_array_uset(x_57, x_70, x_77); +x_79 = lean_unsigned_to_nat(4u); +x_80 = lean_nat_mul(x_76, x_79); +x_81 = lean_unsigned_to_nat(3u); +x_82 = lean_nat_div(x_80, x_81); +lean_dec(x_80); +x_83 = lean_array_get_size(x_78); +x_84 = lean_nat_dec_le(x_82, x_83); +lean_dec(x_83); +lean_dec(x_82); +if (x_84 == 0) { -lean_object* x_152; -x_152 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_152, 0, x_140); -lean_ctor_set(x_152, 1, x_142); +lean_object* x_85; lean_object* x_86; +lean_inc(x_2); +x_85 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_78); +x_86 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_86, 0, x_76); +lean_ctor_set(x_86, 1, x_85); x_5 = x_10; -x_7 = x_152; +x_7 = x_86; goto _start; } -} else { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; -x_154 = lean_box(0); -x_155 = lean_array_uset(x_120, x_133, x_154); -lean_inc(x_1); -x_156 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_137, x_134); -x_157 = lean_array_uset(x_155, x_133, x_156); -x_158 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_158, 0, x_119); -lean_ctor_set(x_158, 1, x_157); +lean_object* x_88; +x_88 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_88, 0, x_76); +lean_ctor_set(x_88, 1, x_78); x_5 = x_10; -x_7 = x_158; +x_7 = x_88; goto _start; } } else { -lean_object* x_160; lean_object* x_161; lean_object* x_162; uint8_t x_194; -x_160 = lean_ctor_get(x_135, 0); -lean_inc(x_160); -lean_dec(x_135); -x_161 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_161, 0, x_11); -lean_ctor_set(x_161, 1, x_160); -lean_inc(x_134); -lean_inc(x_12); -lean_inc(x_1); -x_194 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_134); -if (x_194 == 0) -{ -lean_object* x_195; -lean_dec(x_134); -x_195 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_195, 0, x_119); -lean_ctor_set(x_195, 1, x_120); -x_162 = x_195; -goto block_193; -} -else -{ -lean_object* x_196; lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; lean_object* x_201; lean_object* x_202; -x_196 = lean_box(0); -x_197 = lean_array_uset(x_120, x_133, x_196); -x_198 = lean_unsigned_to_nat(1u); -x_199 = lean_nat_sub(x_119, x_198); -lean_dec(x_119); +lean_object* x_90; lean_object* x_91; lean_object* x_92; uint8_t x_93; lean_object* x_94; +lean_dec(x_11); +x_90 = lean_box(0); +x_91 = lean_array_uset(x_57, x_70, x_90); lean_inc(x_12); lean_inc(x_1); -x_200 = l_Std_DHashMap_Internal_AssocList_erase___rarg(x_1, x_12, x_134); -x_201 = lean_array_uset(x_197, x_133, x_200); -x_202 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_202, 0, x_199); -lean_ctor_set(x_202, 1, x_201); -x_162 = x_202; -goto block_193; -} -block_193: -{ -lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; size_t x_167; size_t x_168; size_t x_169; lean_object* x_170; uint8_t x_171; -x_163 = lean_ctor_get(x_162, 0); -lean_inc(x_163); -x_164 = lean_ctor_get(x_162, 1); -lean_inc(x_164); -if (lean_is_exclusive(x_162)) { - lean_ctor_release(x_162, 0); - lean_ctor_release(x_162, 1); - x_165 = x_162; -} else { - lean_dec_ref(x_162); - x_165 = lean_box(0); -} -x_166 = lean_array_get_size(x_164); -x_167 = lean_usize_of_nat(x_166); -lean_dec(x_166); -x_168 = lean_usize_sub(x_167, x_9); -x_169 = lean_usize_land(x_130, x_168); -x_170 = lean_array_uget(x_164, x_169); -lean_inc(x_170); -lean_inc(x_12); +x_92 = l_Std_DHashMap_Internal_AssocList_Const_alter___at_List_groupByKey___spec__1___rarg(x_1, lean_box(0), x_12, x_13, x_71); +lean_inc(x_92); lean_inc(x_1); -x_171 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_170); -if (x_171 == 0) -{ -lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; uint8_t x_181; -x_172 = lean_unsigned_to_nat(1u); -x_173 = lean_nat_add(x_163, x_172); -lean_dec(x_163); -x_174 = lean_alloc_ctor(1, 3, 0); -lean_ctor_set(x_174, 0, x_12); -lean_ctor_set(x_174, 1, x_161); -lean_ctor_set(x_174, 2, x_170); -x_175 = lean_array_uset(x_164, x_169, x_174); -x_176 = lean_unsigned_to_nat(4u); -x_177 = lean_nat_mul(x_173, x_176); -x_178 = lean_unsigned_to_nat(3u); -x_179 = lean_nat_div(x_177, x_178); -lean_dec(x_177); -x_180 = lean_array_get_size(x_175); -x_181 = lean_nat_dec_le(x_179, x_180); -lean_dec(x_180); -lean_dec(x_179); -if (x_181 == 0) -{ -lean_object* x_182; lean_object* x_183; -lean_inc(x_2); -x_182 = l_Std_DHashMap_Internal_Raw_u2080_expand___rarg(x_2, x_175); -if (lean_is_scalar(x_165)) { - x_183 = lean_alloc_ctor(0, 2, 0); -} else { - x_183 = x_165; -} -lean_ctor_set(x_183, 0, x_173); -lean_ctor_set(x_183, 1, x_182); -x_5 = x_10; -x_7 = x_183; -goto _start; -} -else +x_93 = l_Std_DHashMap_Internal_AssocList_contains___rarg(x_1, x_12, x_92); +x_94 = lean_array_uset(x_91, x_70, x_92); +if (x_93 == 0) { -lean_object* x_185; -if (lean_is_scalar(x_165)) { - x_185 = lean_alloc_ctor(0, 2, 0); -} else { - x_185 = x_165; -} -lean_ctor_set(x_185, 0, x_173); -lean_ctor_set(x_185, 1, x_175); +lean_object* x_95; lean_object* x_96; lean_object* x_97; +x_95 = lean_unsigned_to_nat(1u); +x_96 = lean_nat_sub(x_56, x_95); +lean_dec(x_56); +x_97 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_97, 0, x_96); +lean_ctor_set(x_97, 1, x_94); x_5 = x_10; -x_7 = x_185; +x_7 = x_97; goto _start; } -} else { -lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; -x_187 = lean_box(0); -x_188 = lean_array_uset(x_164, x_169, x_187); -lean_inc(x_1); -x_189 = l_Std_DHashMap_Internal_AssocList_replace___rarg(x_1, x_12, x_161, x_170); -x_190 = lean_array_uset(x_188, x_169, x_189); -if (lean_is_scalar(x_165)) { - x_191 = lean_alloc_ctor(0, 2, 0); -} else { - x_191 = x_165; -} -lean_ctor_set(x_191, 0, x_163); -lean_ctor_set(x_191, 1, x_190); +lean_object* x_99; +x_99 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_99, 0, x_56); +lean_ctor_set(x_99, 1, x_94); x_5 = x_10; -x_7 = x_191; +x_7 = x_99; goto _start; } } } } -} else { lean_dec(x_3); @@ -12279,15 +10929,15 @@ return x_7; } } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___boxed), 7, 0); +x_3 = lean_alloc_closure((void*)(l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg___boxed), 7, 0); return x_3; } } -LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__1___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { +LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__2___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { _start: { lean_object* x_6; lean_object* x_7; uint8_t x_8; @@ -12314,7 +10964,7 @@ size_t x_11; size_t x_12; lean_object* x_13; x_11 = lean_usize_of_nat(x_7); lean_dec(x_7); x_12 = 0; -x_13 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg(x_1, x_2, x_3, x_6, x_11, x_12, x_4); +x_13 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(x_1, x_2, x_3, x_6, x_11, x_12, x_4); lean_dec(x_6); return x_13; } @@ -12339,18 +10989,18 @@ size_t x_16; size_t x_17; lean_object* x_18; x_16 = lean_usize_of_nat(x_7); lean_dec(x_7); x_17 = 0; -x_18 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(x_1, x_2, x_3, x_6, x_16, x_17, x_4); +x_18 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg(x_1, x_2, x_3, x_6, x_16, x_17, x_4); lean_dec(x_6); return x_18; } } } } -LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__1(lean_object* x_1, lean_object* x_2) { +LEAN_EXPORT lean_object* l_List_foldrTR___at_List_groupByKey___spec__2(lean_object* x_1, lean_object* x_2) { _start: { lean_object* x_3; -x_3 = lean_alloc_closure((void*)(l_List_foldrTR___at_List_groupByKey___spec__1___rarg), 5, 0); +x_3 = lean_alloc_closure((void*)(l_List_foldrTR___at_List_groupByKey___spec__2___rarg), 5, 0); return x_3; } } @@ -12359,7 +11009,7 @@ LEAN_EXPORT lean_object* l_List_groupByKey___rarg(lean_object* x_1, lean_object* { lean_object* x_5; lean_object* x_6; x_5 = l_Std_HashMap_instEmptyCollection___closed__3; -x_6 = l_List_foldrTR___at_List_groupByKey___spec__1___rarg(x_1, x_2, x_3, x_5, x_4); +x_6 = l_List_foldrTR___at_List_groupByKey___spec__2___rarg(x_1, x_2, x_3, x_5, x_4); return x_6; } } @@ -12371,7 +11021,7 @@ x_3 = lean_alloc_closure((void*)(l_List_groupByKey___rarg), 4, 0); return x_3; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -12379,12 +11029,12 @@ x_8 = lean_unbox_usize(x_5); lean_dec(x_5); x_9 = lean_unbox_usize(x_6); lean_dec(x_6); -x_10 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__2___rarg(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +x_10 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_9, x_7); lean_dec(x_4); return x_10; } } -LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { +LEAN_EXPORT lean_object* l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7) { _start: { size_t x_8; size_t x_9; lean_object* x_10; @@ -12392,7 +11042,7 @@ x_8 = lean_unbox_usize(x_5); lean_dec(x_5); x_9 = lean_unbox_usize(x_6); lean_dec(x_6); -x_10 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__3___rarg(x_1, x_2, x_3, x_4, x_8, x_9, x_7); +x_10 = l_Array_foldrMUnsafe_fold___at_List_groupByKey___spec__4___rarg(x_1, x_2, x_3, x_4, x_8, x_9, x_7); lean_dec(x_4); return x_10; } diff --git a/stage0/stdlib/Std/Internal.c b/stage0/stdlib/Std/Internal.c index ed4ec6af4ef5..e0e21f5e9e4b 100644 --- a/stage0/stdlib/Std/Internal.c +++ b/stage0/stdlib/Std/Internal.c @@ -1,6 +1,6 @@ // Lean compiler output // Module: Std.Internal -// Imports: Std.Internal.Parsec +// Imports: Std.Internal.Async Std.Internal.Parsec Std.Internal.UV #include #if defined(__clang__) #pragma clang diagnostic ignored "-Wunused-parameter" @@ -13,15 +13,23 @@ #ifdef __cplusplus extern "C" { #endif +lean_object* initialize_Std_Internal_Async(uint8_t builtin, lean_object*); lean_object* initialize_Std_Internal_Parsec(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Internal_UV(uint8_t builtin, lean_object*); static bool _G_initialized = false; LEAN_EXPORT lean_object* initialize_Std_Internal(uint8_t builtin, lean_object* w) { lean_object * res; if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); _G_initialized = true; +res = initialize_Std_Internal_Async(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); res = initialize_Std_Internal_Parsec(builtin, lean_io_mk_world()); if (lean_io_result_is_error(res)) return res; lean_dec_ref(res); +res = initialize_Std_Internal_UV(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); return lean_io_result_mk_ok(lean_box(0)); } #ifdef __cplusplus diff --git a/stage0/stdlib/Std/Internal/Async.c b/stage0/stdlib/Std/Internal/Async.c new file mode 100644 index 000000000000..a16e64556ad8 --- /dev/null +++ b/stage0/stdlib/Std/Internal/Async.c @@ -0,0 +1,33 @@ +// Lean compiler output +// Module: Std.Internal.Async +// Imports: Std.Internal.Async.Basic Std.Internal.Async.Timer +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +lean_object* initialize_Std_Internal_Async_Basic(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Internal_Async_Timer(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Internal_Async(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Internal_Async_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Internal_Async_Timer(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Internal/Async/Basic.c b/stage0/stdlib/Std/Internal/Async/Basic.c new file mode 100644 index 000000000000..b006548e4e22 --- /dev/null +++ b/stage0/stdlib/Std/Internal/Async/Basic.c @@ -0,0 +1,704 @@ +// Lean compiler output +// Module: Std.Internal.Async.Basic +// Imports: Init.Core Init.System.IO Init.System.Promise +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_block___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPurePromise(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState___rarg___boxed(lean_object*, lean_object*); +lean_object* lean_io_promise_result(lean_object*); +lean_object* lean_task_bind(lean_object*, lean_object*, lean_object*, uint8_t); +static lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1; +lean_object* lean_task_pure(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPromise___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPromise(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind___rarg(lean_object*, lean_object*); +lean_object* l_Except_pure___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_pure___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_instPure___rarg(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg(lean_object*, lean_object*, lean_object*); +lean_object* lean_io_map_task(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); +extern lean_object* l_Task_Priority_default; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map(lean_object*, lean_object*); +lean_object* lean_task_get_own(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map___rarg___lambda__1(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_pure(lean_object*); +lean_object* lean_io_get_task_state(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg___lambda__1(lean_object*, lean_object*, lean_object*); +lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); +lean_object* lean_io_bind_task(lean_object*, lean_object*, lean_object*, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_instPure(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_block(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map___rarg(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_pure___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +x_3 = lean_task_pure(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_pure(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_pure___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_instPure___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; +x_2 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_2, 0, x_1); +x_3 = lean_task_pure(x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_instPure(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_instPure___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +lean_dec(x_1); +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +lean_object* x_4; +x_4 = lean_task_pure(x_2); +return x_4; +} +else +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_2, 0); +lean_inc(x_5); +lean_dec(x_2); +x_6 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_6, 0, x_5); +x_7 = lean_task_pure(x_6); +return x_7; +} +} +else +{ +lean_object* x_8; lean_object* x_9; +x_8 = lean_ctor_get(x_2, 0); +lean_inc(x_8); +lean_dec(x_2); +x_9 = lean_apply_1(x_1, x_8); +return x_9; +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_bind___rarg___lambda__1), 2, 1); +lean_closure_set(x_3, 0, x_2); +x_4 = l_Task_Priority_default; +x_5 = 0; +x_6 = lean_task_bind(x_1, x_3, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bind(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_bind___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map___rarg___lambda__1(lean_object* x_1, lean_object* x_2) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_3; +lean_dec(x_1); +x_3 = !lean_is_exclusive(x_2); +if (x_3 == 0) +{ +return x_2; +} +else +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_2, 0); +lean_inc(x_4); +lean_dec(x_2); +x_5 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_5, 0, x_4); +return x_5; +} +} +else +{ +uint8_t x_6; +x_6 = !lean_is_exclusive(x_2); +if (x_6 == 0) +{ +lean_object* x_7; lean_object* x_8; +x_7 = lean_ctor_get(x_2, 0); +x_8 = lean_apply_1(x_1, x_7); +lean_ctor_set(x_2, 0, x_8); +return x_2; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_2, 0); +lean_inc(x_9); +lean_dec(x_2); +x_10 = lean_apply_1(x_1, x_9); +x_11 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_11, 0, x_10); +return x_11; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_map___rarg___lambda__1), 2, 1); +lean_closure_set(x_3, 0, x_1); +x_4 = l_Task_Priority_default; +x_5 = 0; +x_6 = lean_task_map(x_3, x_2, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_map(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_map___rarg), 2, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; +x_5 = lean_task_pure(x_2); +x_6 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_6, 0, x_5); +lean_ctor_set(x_6, 1, x_3); +return x_6; +} +else +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_7 = lean_ctor_get(x_2, 0); +lean_inc(x_7); +lean_dec(x_2); +x_8 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_8, 0, x_7); +x_9 = lean_task_pure(x_8); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_9); +lean_ctor_set(x_10, 1, x_3); +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_2); +if (x_11 == 0) +{ +lean_object* x_12; lean_object* x_13; +x_12 = lean_ctor_get(x_2, 0); +x_13 = lean_apply_2(x_1, x_12, x_3); +if (lean_obj_tag(x_13) == 0) +{ +uint8_t x_14; +lean_free_object(x_2); +x_14 = !lean_is_exclusive(x_13); +if (x_14 == 0) +{ +return x_13; +} +else +{ +lean_object* x_15; lean_object* x_16; lean_object* x_17; +x_15 = lean_ctor_get(x_13, 0); +x_16 = lean_ctor_get(x_13, 1); +lean_inc(x_16); +lean_inc(x_15); +lean_dec(x_13); +x_17 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_17, 0, x_15); +lean_ctor_set(x_17, 1, x_16); +return x_17; +} +} +else +{ +uint8_t x_18; +x_18 = !lean_is_exclusive(x_13); +if (x_18 == 0) +{ +lean_object* x_19; lean_object* x_20; +x_19 = lean_ctor_get(x_13, 0); +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 0, x_19); +x_20 = lean_task_pure(x_2); +lean_ctor_set_tag(x_13, 0); +lean_ctor_set(x_13, 0, x_20); +return x_13; +} +else +{ +lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; +x_21 = lean_ctor_get(x_13, 0); +x_22 = lean_ctor_get(x_13, 1); +lean_inc(x_22); +lean_inc(x_21); +lean_dec(x_13); +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 0, x_21); +x_23 = lean_task_pure(x_2); +x_24 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_24, 0, x_23); +lean_ctor_set(x_24, 1, x_22); +return x_24; +} +} +} +else +{ +lean_object* x_25; lean_object* x_26; +x_25 = lean_ctor_get(x_2, 0); +lean_inc(x_25); +lean_dec(x_2); +x_26 = lean_apply_2(x_1, x_25, x_3); +if (lean_obj_tag(x_26) == 0) +{ +lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_27 = lean_ctor_get(x_26, 0); +lean_inc(x_27); +x_28 = lean_ctor_get(x_26, 1); +lean_inc(x_28); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_29 = x_26; +} else { + lean_dec_ref(x_26); + x_29 = lean_box(0); +} +if (lean_is_scalar(x_29)) { + x_30 = lean_alloc_ctor(0, 2, 0); +} else { + x_30 = x_29; +} +lean_ctor_set(x_30, 0, x_27); +lean_ctor_set(x_30, 1, x_28); +return x_30; +} +else +{ +lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; +x_31 = lean_ctor_get(x_26, 0); +lean_inc(x_31); +x_32 = lean_ctor_get(x_26, 1); +lean_inc(x_32); +if (lean_is_exclusive(x_26)) { + lean_ctor_release(x_26, 0); + lean_ctor_release(x_26, 1); + x_33 = x_26; +} else { + lean_dec_ref(x_26); + x_33 = lean_box(0); +} +x_34 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_34, 0, x_31); +x_35 = lean_task_pure(x_34); +if (lean_is_scalar(x_33)) { + x_36 = lean_alloc_ctor(0, 2, 0); +} else { + x_36 = x_33; + lean_ctor_set_tag(x_36, 0); +} +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_32); +return x_36; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg___lambda__1), 3, 1); +lean_closure_set(x_4, 0, x_2); +x_5 = l_Task_Priority_default; +x_6 = 0; +x_7 = lean_io_bind_task(x_1, x_4, x_5, x_6, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_bindIO(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_bindIO___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +if (lean_obj_tag(x_2) == 0) +{ +uint8_t x_4; +lean_dec(x_1); +x_4 = !lean_is_exclusive(x_2); +if (x_4 == 0) +{ +lean_object* x_5; +x_5 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_5, 0, x_2); +lean_ctor_set(x_5, 1, x_3); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; lean_object* x_8; +x_6 = lean_ctor_get(x_2, 0); +lean_inc(x_6); +lean_dec(x_2); +x_7 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_7, 0, x_6); +x_8 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_8, 0, x_7); +lean_ctor_set(x_8, 1, x_3); +return x_8; +} +} +else +{ +uint8_t x_9; +x_9 = !lean_is_exclusive(x_2); +if (x_9 == 0) +{ +lean_object* x_10; lean_object* x_11; +x_10 = lean_ctor_get(x_2, 0); +x_11 = lean_apply_2(x_1, x_10, x_3); +if (lean_obj_tag(x_11) == 0) +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_11); +if (x_12 == 0) +{ +lean_object* x_13; +x_13 = lean_ctor_get(x_11, 0); +lean_ctor_set(x_2, 0, x_13); +lean_ctor_set(x_11, 0, x_2); +return x_11; +} +else +{ +lean_object* x_14; lean_object* x_15; lean_object* x_16; +x_14 = lean_ctor_get(x_11, 0); +x_15 = lean_ctor_get(x_11, 1); +lean_inc(x_15); +lean_inc(x_14); +lean_dec(x_11); +lean_ctor_set(x_2, 0, x_14); +x_16 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_16, 0, x_2); +lean_ctor_set(x_16, 1, x_15); +return x_16; +} +} +else +{ +uint8_t x_17; +x_17 = !lean_is_exclusive(x_11); +if (x_17 == 0) +{ +lean_object* x_18; +x_18 = lean_ctor_get(x_11, 0); +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 0, x_18); +lean_ctor_set_tag(x_11, 0); +lean_ctor_set(x_11, 0, x_2); +return x_11; +} +else +{ +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_11, 0); +x_20 = lean_ctor_get(x_11, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_11); +lean_ctor_set_tag(x_2, 0); +lean_ctor_set(x_2, 0, x_19); +x_21 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_21, 0, x_2); +lean_ctor_set(x_21, 1, x_20); +return x_21; +} +} +} +else +{ +lean_object* x_22; lean_object* x_23; +x_22 = lean_ctor_get(x_2, 0); +lean_inc(x_22); +lean_dec(x_2); +x_23 = lean_apply_2(x_1, x_22, x_3); +if (lean_obj_tag(x_23) == 0) +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +x_24 = lean_ctor_get(x_23, 0); +lean_inc(x_24); +x_25 = lean_ctor_get(x_23, 1); +lean_inc(x_25); +if (lean_is_exclusive(x_23)) { + lean_ctor_release(x_23, 0); + lean_ctor_release(x_23, 1); + x_26 = x_23; +} else { + lean_dec_ref(x_23); + x_26 = lean_box(0); +} +x_27 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_27, 0, x_24); +if (lean_is_scalar(x_26)) { + x_28 = lean_alloc_ctor(0, 2, 0); +} else { + x_28 = x_26; +} +lean_ctor_set(x_28, 0, x_27); +lean_ctor_set(x_28, 1, x_25); +return x_28; +} +else +{ +lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_29 = lean_ctor_get(x_23, 0); +lean_inc(x_29); +x_30 = lean_ctor_get(x_23, 1); +lean_inc(x_30); +if (lean_is_exclusive(x_23)) { + lean_ctor_release(x_23, 0); + lean_ctor_release(x_23, 1); + x_31 = x_23; +} else { + lean_dec_ref(x_23); + x_31 = lean_box(0); +} +x_32 = lean_alloc_ctor(0, 1, 0); +lean_ctor_set(x_32, 0, x_29); +if (lean_is_scalar(x_31)) { + x_33 = lean_alloc_ctor(0, 2, 0); +} else { + x_33 = x_31; + lean_ctor_set_tag(x_33, 0); +} +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_30); +return x_33; +} +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; lean_object* x_5; uint8_t x_6; lean_object* x_7; +x_4 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg___lambda__1), 3, 1); +lean_closure_set(x_4, 0, x_1); +x_5 = l_Task_Priority_default; +x_6 = 0; +x_7 = lean_io_map_task(x_4, x_2, x_5, x_6, x_3); +return x_7; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_mapIO(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_mapIO___rarg), 3, 0); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_block___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_task_get_own(x_1); +if (lean_obj_tag(x_3) == 0) +{ +lean_object* x_4; lean_object* x_5; +x_4 = lean_ctor_get(x_3, 0); +lean_inc(x_4); +lean_dec(x_3); +x_5 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_5, 0, x_4); +lean_ctor_set(x_5, 1, x_2); +return x_5; +} +else +{ +lean_object* x_6; lean_object* x_7; +x_6 = lean_ctor_get(x_3, 0); +lean_inc(x_6); +lean_dec(x_3); +x_7 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_7, 0, x_6); +lean_ctor_set(x_7, 1, x_2); +return x_7; +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_block(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_block___rarg), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPromise___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_io_promise_result(x_1); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPromise(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_ofPromise___rarg), 1, 0); +return x_2; +} +} +static lean_object* _init_l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Except_pure___rarg), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg(lean_object* x_1) { +_start: +{ +lean_object* x_2; lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; +x_2 = lean_io_promise_result(x_1); +x_3 = l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1; +x_4 = l_Task_Priority_default; +x_5 = 0; +x_6 = lean_task_map(x_3, x_2, x_4, x_5); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_ofPurePromise(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg), 1, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState___rarg(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_io_get_task_state(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_alloc_closure((void*)(l_Std_Internal_IO_Async_AsyncTask_getState___rarg___boxed), 2, 0); +return x_2; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_AsyncTask_getState___rarg___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_AsyncTask_getState___rarg(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +lean_object* initialize_Init_Core(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_IO(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_Promise(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Internal_Async_Basic(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_Core(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_System_IO(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_System_Promise(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1 = _init_l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1(); +lean_mark_persistent(l_Std_Internal_IO_Async_AsyncTask_ofPurePromise___rarg___closed__1); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Internal/Async/Timer.c b/stage0/stdlib/Std/Internal/Async/Timer.c new file mode 100644 index 000000000000..a6efc64a34f9 --- /dev/null +++ b/stage0/stdlib/Std/Internal/Async/Timer.c @@ -0,0 +1,909 @@ +// Lean compiler output +// Module: Std.Internal.Async.Timer +// Imports: Std.Time Std.Internal.UV Std.Internal.Async.Basic +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_mk(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_sleep(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11; +lean_object* lean_mk_empty_array_with_capacity(lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22; +LEAN_EXPORT lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141_; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14; +lean_object* lean_uv_timer_next(lean_object*, lean_object*); +uint64_t lean_uint64_of_nat(lean_object*); +lean_object* lean_array_push(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18; +lean_object* lean_io_promise_result(lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_stop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_wait(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_mk___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_stop(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_mk(lean_object*, lean_object*); +lean_object* lean_uv_timer_stop(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_tick___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3; +lean_object* l_Except_pure___rarg(lean_object*); +lean_object* lean_uv_timer_reset(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_sleep___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25; +extern lean_object* l_Task_Priority_default; +lean_object* l_Lean_Name_str___override(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_reset___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_stop___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23; +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4; +lean_object* l_Int_toNat(lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7; +lean_object* lean_task_map(lean_object*, lean_object*, lean_object*, uint8_t); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_reset(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_mk___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_wait___boxed(lean_object*, lean_object*); +static lean_object* l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_tick(lean_object*, lean_object*); +lean_object* l_Lean_Name_mkStr4(lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_reset___boxed(lean_object*, lean_object*); +lean_object* lean_uv_timer_mk(uint64_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_stop___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_reset(lean_object*, lean_object*); +static lean_object* l_Std_Internal_IO_Async_Sleep_wait___closed__1; +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_mk(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint64_t x_4; uint8_t x_5; lean_object* x_6; +x_3 = l_Int_toNat(x_1); +x_4 = lean_uint64_of_nat(x_3); +lean_dec(x_3); +x_5 = 0; +x_6 = lean_uv_timer_mk(x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) +{ +uint8_t x_7; +x_7 = !lean_is_exclusive(x_6); +if (x_7 == 0) +{ +return x_6; +} +else +{ +lean_object* x_8; lean_object* x_9; lean_object* x_10; +x_8 = lean_ctor_get(x_6, 0); +x_9 = lean_ctor_get(x_6, 1); +lean_inc(x_9); +lean_inc(x_8); +lean_dec(x_6); +x_10 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_10, 0, x_8); +lean_ctor_set(x_10, 1, x_9); +return x_10; +} +} +else +{ +uint8_t x_11; +x_11 = !lean_is_exclusive(x_6); +if (x_11 == 0) +{ +return x_6; +} +else +{ +lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_12 = lean_ctor_get(x_6, 0); +x_13 = lean_ctor_get(x_6, 1); +lean_inc(x_13); +lean_inc(x_12); +lean_dec(x_6); +x_14 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_14, 0, x_12); +lean_ctor_set(x_14, 1, x_13); +return x_14; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_mk___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Sleep_mk(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +static lean_object* _init_l_Std_Internal_IO_Async_Sleep_wait___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_alloc_closure((void*)(l_Except_pure___rarg), 1, 0); +return x_1; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_wait(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_next(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; +x_5 = lean_ctor_get(x_3, 0); +x_6 = lean_io_promise_result(x_5); +x_7 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_8 = l_Task_Priority_default; +x_9 = 0; +x_10 = lean_task_map(x_7, x_6, x_8, x_9); +lean_ctor_set(x_3, 0, x_10); +return x_3; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_13 = lean_io_promise_result(x_11); +x_14 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_15 = l_Task_Priority_default; +x_16 = 0; +x_17 = lean_task_map(x_14, x_13, x_15, x_16); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_12); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_3); +if (x_19 == 0) +{ +return x_3; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_3, 0); +x_21 = lean_ctor_get(x_3, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_3); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_wait___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Sleep_wait(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_reset(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_reset(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_reset___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Sleep_reset(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_stop(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_stop(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Sleep_stop___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Sleep_stop(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_sleep(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; uint64_t x_4; uint8_t x_5; lean_object* x_6; +x_3 = l_Int_toNat(x_1); +x_4 = lean_uint64_of_nat(x_3); +lean_dec(x_3); +x_5 = 0; +x_6 = lean_uv_timer_mk(x_4, x_5, x_2); +if (lean_obj_tag(x_6) == 0) +{ +lean_object* x_7; lean_object* x_8; lean_object* x_9; +x_7 = lean_ctor_get(x_6, 0); +lean_inc(x_7); +x_8 = lean_ctor_get(x_6, 1); +lean_inc(x_8); +lean_dec(x_6); +x_9 = lean_uv_timer_next(x_7, x_8); +lean_dec(x_7); +if (lean_obj_tag(x_9) == 0) +{ +uint8_t x_10; +x_10 = !lean_is_exclusive(x_9); +if (x_10 == 0) +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_11 = lean_ctor_get(x_9, 0); +x_12 = lean_io_promise_result(x_11); +x_13 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_14 = l_Task_Priority_default; +x_15 = lean_task_map(x_13, x_12, x_14, x_5); +lean_ctor_set(x_9, 0, x_15); +return x_9; +} +else +{ +lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_16 = lean_ctor_get(x_9, 0); +x_17 = lean_ctor_get(x_9, 1); +lean_inc(x_17); +lean_inc(x_16); +lean_dec(x_9); +x_18 = lean_io_promise_result(x_16); +x_19 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_20 = l_Task_Priority_default; +x_21 = lean_task_map(x_19, x_18, x_20, x_5); +x_22 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_22, 0, x_21); +lean_ctor_set(x_22, 1, x_17); +return x_22; +} +} +else +{ +uint8_t x_23; +x_23 = !lean_is_exclusive(x_9); +if (x_23 == 0) +{ +return x_9; +} +else +{ +lean_object* x_24; lean_object* x_25; lean_object* x_26; +x_24 = lean_ctor_get(x_9, 0); +x_25 = lean_ctor_get(x_9, 1); +lean_inc(x_25); +lean_inc(x_24); +lean_dec(x_9); +x_26 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); +return x_26; +} +} +} +else +{ +uint8_t x_27; +x_27 = !lean_is_exclusive(x_6); +if (x_27 == 0) +{ +return x_6; +} +else +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; +x_28 = lean_ctor_get(x_6, 0); +x_29 = lean_ctor_get(x_6, 1); +lean_inc(x_29); +lean_inc(x_28); +lean_dec(x_6); +x_30 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_30, 0, x_28); +lean_ctor_set(x_30, 1, x_29); +return x_30; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_sleep___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_sleep(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Lean", 4, 4); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Parser", 6, 6); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Tactic", 6, 6); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq", 9, 9); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3; +x_4 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(0u); +x_2 = lean_mk_empty_array_with_capacity(x_1); +return x_2; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("tacticSeq1Indented", 18, 18); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3; +x_4 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("null", 4, 4); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(0); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9; +x_3 = l_Lean_Name_str___override(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("decide", 6, 6); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3; +x_4 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11; +x_3 = lean_alloc_ctor(2, 2, 0); +lean_ctor_set(x_3, 0, x_1); +lean_ctor_set(x_3, 1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("optConfig", 9, 9); +return x_1; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3; +x_4 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15; +x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); +return x_5; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6; +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25; +x_3 = lean_array_push(x_1, x_2); +return x_3; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27() { +_start: +{ +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = lean_box(2); +x_2 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5; +x_3 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26; +x_4 = lean_alloc_ctor(1, 3, 0); +lean_ctor_set(x_4, 0, x_1); +lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_3); +return x_4; +} +} +static lean_object* _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141_() { +_start: +{ +lean_object* x_1; +x_1 = l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27; +return x_1; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_mk(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; uint64_t x_5; uint8_t x_6; lean_object* x_7; +x_4 = l_Int_toNat(x_1); +x_5 = lean_uint64_of_nat(x_4); +lean_dec(x_4); +x_6 = 1; +x_7 = lean_uv_timer_mk(x_5, x_6, x_3); +if (lean_obj_tag(x_7) == 0) +{ +uint8_t x_8; +x_8 = !lean_is_exclusive(x_7); +if (x_8 == 0) +{ +return x_7; +} +else +{ +lean_object* x_9; lean_object* x_10; lean_object* x_11; +x_9 = lean_ctor_get(x_7, 0); +x_10 = lean_ctor_get(x_7, 1); +lean_inc(x_10); +lean_inc(x_9); +lean_dec(x_7); +x_11 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_11, 0, x_9); +lean_ctor_set(x_11, 1, x_10); +return x_11; +} +} +else +{ +uint8_t x_12; +x_12 = !lean_is_exclusive(x_7); +if (x_12 == 0) +{ +return x_7; +} +else +{ +lean_object* x_13; lean_object* x_14; lean_object* x_15; +x_13 = lean_ctor_get(x_7, 0); +x_14 = lean_ctor_get(x_7, 1); +lean_inc(x_14); +lean_inc(x_13); +lean_dec(x_7); +x_15 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_15, 0, x_13); +lean_ctor_set(x_15, 1, x_14); +return x_15; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_mk___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +lean_object* x_4; +x_4 = l_Std_Internal_IO_Async_Interval_mk(x_1, x_2, x_3); +lean_dec(x_1); +return x_4; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_tick(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_next(x_1, x_2); +if (lean_obj_tag(x_3) == 0) +{ +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) +{ +lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; +x_5 = lean_ctor_get(x_3, 0); +x_6 = lean_io_promise_result(x_5); +x_7 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_8 = l_Task_Priority_default; +x_9 = 0; +x_10 = lean_task_map(x_7, x_6, x_8, x_9); +lean_ctor_set(x_3, 0, x_10); +return x_3; +} +else +{ +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; uint8_t x_16; lean_object* x_17; lean_object* x_18; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_13 = lean_io_promise_result(x_11); +x_14 = l_Std_Internal_IO_Async_Sleep_wait___closed__1; +x_15 = l_Task_Priority_default; +x_16 = 0; +x_17 = lean_task_map(x_14, x_13, x_15, x_16); +x_18 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_12); +return x_18; +} +} +else +{ +uint8_t x_19; +x_19 = !lean_is_exclusive(x_3); +if (x_19 == 0) +{ +return x_3; +} +else +{ +lean_object* x_20; lean_object* x_21; lean_object* x_22; +x_20 = lean_ctor_get(x_3, 0); +x_21 = lean_ctor_get(x_3, 1); +lean_inc(x_21); +lean_inc(x_20); +lean_dec(x_3); +x_22 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +return x_22; +} +} +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_tick___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Interval_tick(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_reset(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_reset(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_reset___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Interval_reset(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_stop(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_stop(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_IO_Async_Interval_stop___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = l_Std_Internal_IO_Async_Interval_stop(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +lean_object* initialize_Std_Time(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Internal_UV(uint8_t builtin, lean_object*); +lean_object* initialize_Std_Internal_Async_Basic(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Internal_Async_Timer(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Std_Time(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Internal_UV(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Std_Internal_Async_Basic(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l_Std_Internal_IO_Async_Sleep_wait___closed__1 = _init_l_Std_Internal_IO_Async_Sleep_wait___closed__1(); +lean_mark_persistent(l_Std_Internal_IO_Async_Sleep_wait___closed__1); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__1); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__2); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__3); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__4); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__5); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__6); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__7); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__8); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__9); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__10); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__11); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__12); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__13); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__14); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__15); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__16); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__17); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__18); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__19); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__20); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__21); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__22); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__23); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__24); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__25); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__26); +l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27 = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141____closed__27); +l___auto____x40_Std_Internal_Async_Timer___hyg_141_ = _init_l___auto____x40_Std_Internal_Async_Timer___hyg_141_(); +lean_mark_persistent(l___auto____x40_Std_Internal_Async_Timer___hyg_141_); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Internal/UV.c b/stage0/stdlib/Std/Internal/UV.c new file mode 100644 index 000000000000..4b93875de8ae --- /dev/null +++ b/stage0/stdlib/Std/Internal/UV.c @@ -0,0 +1,108 @@ +// Lean compiler output +// Module: Std.Internal.UV +// Imports: Init.System.IO Init.System.Promise +#include +#if defined(__clang__) +#pragma clang diagnostic ignored "-Wunused-parameter" +#pragma clang diagnostic ignored "-Wunused-label" +#elif defined(__GNUC__) && !defined(__CLANG__) +#pragma GCC diagnostic ignored "-Wunused-parameter" +#pragma GCC diagnostic ignored "-Wunused-label" +#pragma GCC diagnostic ignored "-Wunused-but-set-variable" +#endif +#ifdef __cplusplus +extern "C" { +#endif +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_reset___boxed(lean_object*, lean_object*); +lean_object* lean_uv_timer_next(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_next___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_mk___boxed(lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Loop_configure___boxed(lean_object*, lean_object*); +lean_object* lean_uv_timer_stop(lean_object*, lean_object*); +lean_object* lean_uv_timer_reset(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_stop___boxed(lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Loop_alive___boxed(lean_object*); +lean_object* lean_uv_event_loop_configure(lean_object*, lean_object*); +lean_object* lean_uv_event_loop_alive(lean_object*); +LEAN_EXPORT lean_object* l___private_Std_Internal_UV_0__Std_Internal_UV_TimerImpl; +lean_object* lean_uv_timer_mk(uint64_t, uint8_t, lean_object*); +LEAN_EXPORT lean_object* l_Std_Internal_UV_Loop_configure___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_event_loop_configure(x_1, x_2); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_UV_Loop_alive___boxed(lean_object* x_1) { +_start: +{ +lean_object* x_2; +x_2 = lean_uv_event_loop_alive(x_1); +return x_2; +} +} +static lean_object* _init_l___private_Std_Internal_UV_0__Std_Internal_UV_TimerImpl() { +_start: +{ +return lean_box(0); +} +} +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_mk___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +_start: +{ +uint64_t x_4; uint8_t x_5; lean_object* x_6; +x_4 = lean_unbox_uint64(x_1); +lean_dec(x_1); +x_5 = lean_unbox(x_2); +lean_dec(x_2); +x_6 = lean_uv_timer_mk(x_4, x_5, x_3); +return x_6; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_next___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_next(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_reset___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_reset(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +LEAN_EXPORT lean_object* l_Std_Internal_UV_Timer_stop___boxed(lean_object* x_1, lean_object* x_2) { +_start: +{ +lean_object* x_3; +x_3 = lean_uv_timer_stop(x_1, x_2); +lean_dec(x_1); +return x_3; +} +} +lean_object* initialize_Init_System_IO(uint8_t builtin, lean_object*); +lean_object* initialize_Init_System_Promise(uint8_t builtin, lean_object*); +static bool _G_initialized = false; +LEAN_EXPORT lean_object* initialize_Std_Internal_UV(uint8_t builtin, lean_object* w) { +lean_object * res; +if (_G_initialized) return lean_io_result_mk_ok(lean_box(0)); +_G_initialized = true; +res = initialize_Init_System_IO(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +res = initialize_Init_System_Promise(builtin, lean_io_mk_world()); +if (lean_io_result_is_error(res)) return res; +lean_dec_ref(res); +l___private_Std_Internal_UV_0__Std_Internal_UV_TimerImpl = _init_l___private_Std_Internal_UV_0__Std_Internal_UV_TimerImpl(); +return lean_io_result_mk_ok(lean_box(0)); +} +#ifdef __cplusplus +} +#endif diff --git a/stage0/stdlib/Std/Time/DateTime/PlainDateTime.c b/stage0/stdlib/Std/Time/DateTime/PlainDateTime.c index bf0be4b43999..99e3e951121d 100644 --- a/stage0/stdlib/Std/Time/DateTime/PlainDateTime.c +++ b/stage0/stdlib/Std/Time/DateTime/PlainDateTime.c @@ -270,7 +270,6 @@ static lean_object* l___private_Std_Time_DateTime_PlainDateTime_0__Std_Time_repr LEAN_EXPORT lean_object* l_Std_Time_PlainDateTime_ofTimestampAssumingUTC___lambda__4(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); uint8_t lean_nat_dec_le(lean_object*, lean_object*); static lean_object* l_Std_Time_PlainDateTime_ofTimestampAssumingUTC___lambda__2___closed__10; -static lean_object* l_Std_Time_instInhabitedPlainDateTime___closed__40; LEAN_EXPORT lean_object* l_Std_Time_PlainDateTime_subMinutes(lean_object*, lean_object*); static lean_object* l_Std_Time_PlainDateTime_ofTimestampAssumingUTC___lambda__4___closed__1; static lean_object* l_Std_Time_PlainDateTime_addMilliseconds___closed__1; @@ -671,38 +670,24 @@ return x_3; static lean_object* _init_l_Std_Time_instInhabitedPlainDateTime___closed__38() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Std_Time_instInhabitedPlainDateTime___closed__29; x_2 = l_Std_Time_instInhabitedPlainDateTime___closed__37; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); +x_3 = l_Std_Time_instInhabitedPlainDateTime___closed__1; +x_4 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_3); return x_4; } } static lean_object* _init_l_Std_Time_instInhabitedPlainDateTime___closed__39() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Time_instInhabitedPlainDateTime___closed__29; -x_2 = l_Std_Time_instInhabitedPlainDateTime___closed__37; -x_3 = l_Std_Time_instInhabitedPlainDateTime___closed__38; -x_4 = l_Std_Time_instInhabitedPlainDateTime___closed__1; -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} -} -static lean_object* _init_l_Std_Time_instInhabitedPlainDateTime___closed__40() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Time_instInhabitedPlainDateTime___closed__20; -x_2 = l_Std_Time_instInhabitedPlainDateTime___closed__39; +x_2 = l_Std_Time_instInhabitedPlainDateTime___closed__38; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -713,7 +698,7 @@ static lean_object* _init_l_Std_Time_instInhabitedPlainDateTime() { _start: { lean_object* x_1; -x_1 = l_Std_Time_instInhabitedPlainDateTime___closed__40; +x_1 = l_Std_Time_instInhabitedPlainDateTime___closed__39; return x_1; } } @@ -784,25 +769,23 @@ return x_26; } else { -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; uint8_t x_31; +lean_object* x_27; lean_object* x_28; uint8_t x_29; x_27 = lean_ctor_get(x_4, 2); -x_28 = lean_ctor_get(x_27, 1); -x_29 = lean_ctor_get(x_6, 2); -x_30 = lean_ctor_get(x_29, 1); -x_31 = lean_int_dec_eq(x_28, x_30); -if (x_31 == 0) +x_28 = lean_ctor_get(x_6, 2); +x_29 = lean_int_dec_eq(x_27, x_28); +if (x_29 == 0) { -uint8_t x_32; -x_32 = 0; -return x_32; +uint8_t x_30; +x_30 = 0; +return x_30; } else { -lean_object* x_33; lean_object* x_34; uint8_t x_35; -x_33 = lean_ctor_get(x_4, 3); -x_34 = lean_ctor_get(x_6, 3); -x_35 = lean_int_dec_eq(x_33, x_34); -return x_35; +lean_object* x_31; lean_object* x_32; uint8_t x_33; +x_31 = lean_ctor_get(x_4, 3); +x_32 = lean_ctor_get(x_6, 3); +x_33 = lean_int_dec_eq(x_31, x_32); +return x_33; } } } @@ -1002,10 +985,8 @@ LEAN_EXPORT lean_object* l___private_Std_Time_DateTime_PlainDateTime_0__Std_Time { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; uint8_t x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); x_4 = lean_unsigned_to_nat(0u); x_5 = l___private_Std_Time_Date_PlainDate_0__Std_Time_reprPlainDate____x40_Std_Time_Date_PlainDate___hyg_40_(x_3, x_4); -lean_dec(x_3); x_6 = l___private_Std_Time_DateTime_PlainDateTime_0__Std_Time_reprPlainDateTime____x40_Std_Time_DateTime_PlainDateTime___hyg_111____closed__7; x_7 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_7, 0, x_6); @@ -1035,8 +1016,6 @@ x_19 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_19, 0, x_17); lean_ctor_set(x_19, 1, x_18); x_20 = lean_ctor_get(x_1, 1); -lean_inc(x_20); -lean_dec(x_1); x_21 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43_(x_20, x_4); x_22 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_22, 0, x_6); @@ -1071,6 +1050,7 @@ LEAN_EXPORT lean_object* l___private_Std_Time_DateTime_PlainDateTime_0__Std_Time lean_object* x_3; x_3 = l___private_Std_Time_DateTime_PlainDateTime_0__Std_Time_reprPlainDateTime____x40_Std_Time_DateTime_PlainDateTime___hyg_111_(x_1, x_2); lean_dec(x_2); +lean_dec(x_1); return x_3; } } @@ -1258,7 +1238,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainDateTime_ofTimestampAssumingUTC___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5, lean_object* x_6, lean_object* x_7, lean_object* x_8, lean_object* x_9, lean_object* x_10) { _start: { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; uint8_t x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; uint8_t x_20; lean_object* x_21; lean_object* x_22; uint8_t x_23; lean_object* x_24; lean_object* x_25; x_11 = l_Std_Time_PlainDateTime_ofTimestampAssumingUTC___lambda__1___closed__1; x_12 = lean_int_emod(x_1, x_11); x_13 = lean_int_ediv(x_1, x_11); @@ -1274,174 +1254,171 @@ x_21 = lean_int_mod(x_9, x_5); x_22 = l_Std_Time_instInhabitedPlainDateTime___closed__1; x_23 = lean_int_dec_eq(x_21, x_22); lean_dec(x_21); -x_24 = 0; -x_25 = lean_box(x_24); -x_26 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_26, 0, x_25); -lean_ctor_set(x_26, 1, x_12); -x_27 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_27, 0, x_16); -lean_ctor_set(x_27, 1, x_14); -lean_ctor_set(x_27, 2, x_26); -lean_ctor_set(x_27, 3, x_17); +x_24 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_24, 0, x_16); +lean_ctor_set(x_24, 1, x_14); +lean_ctor_set(x_24, 2, x_12); +lean_ctor_set(x_24, 3, x_17); if (x_20 == 0) { lean_dec(x_19); -x_28 = x_8; -goto block_60; +x_25 = x_8; +goto block_59; } else { -lean_object* x_61; +lean_object* x_60; lean_dec(x_8); -x_61 = lean_nat_to_int(x_19); -x_28 = x_61; -goto block_60; +x_60 = lean_nat_to_int(x_19); +x_25 = x_60; +goto block_59; } -block_60: +block_59: { if (x_23 == 0) { -lean_object* x_29; uint8_t x_30; -x_29 = l_Std_Time_Month_Ordinal_days(x_24, x_10); -x_30 = lean_int_dec_lt(x_29, x_28); -if (x_30 == 0) +uint8_t x_26; lean_object* x_27; uint8_t x_28; +x_26 = 0; +x_27 = l_Std_Time_Month_Ordinal_days(x_26, x_10); +x_28 = lean_int_dec_lt(x_27, x_25); +if (x_28 == 0) +{ +lean_object* x_29; lean_object* x_30; +lean_dec(x_27); +x_29 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_29, 0, x_9); +lean_ctor_set(x_29, 1, x_10); +lean_ctor_set(x_29, 2, x_25); +x_30 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set(x_30, 1, x_24); +return x_30; +} +else { lean_object* x_31; lean_object* x_32; -lean_dec(x_29); +lean_dec(x_25); x_31 = lean_alloc_ctor(0, 3, 0); lean_ctor_set(x_31, 0, x_9); lean_ctor_set(x_31, 1, x_10); -lean_ctor_set(x_31, 2, x_28); +lean_ctor_set(x_31, 2, x_27); x_32 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_27); +lean_ctor_set(x_32, 1, x_24); return x_32; } -else -{ -lean_object* x_33; lean_object* x_34; -lean_dec(x_28); -x_33 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_33, 0, x_9); -lean_ctor_set(x_33, 1, x_10); -lean_ctor_set(x_33, 2, x_29); -x_34 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_34, 0, x_33); -lean_ctor_set(x_34, 1, x_27); -return x_34; -} } else { -lean_object* x_35; uint8_t x_36; uint8_t x_37; -x_35 = lean_int_mod(x_9, x_6); -x_36 = lean_int_dec_eq(x_35, x_22); -lean_dec(x_35); -x_37 = l_instDecidableNot___rarg(x_36); -if (x_37 == 0) +lean_object* x_33; uint8_t x_34; uint8_t x_35; +x_33 = lean_int_mod(x_9, x_6); +x_34 = lean_int_dec_eq(x_33, x_22); +lean_dec(x_33); +x_35 = l_instDecidableNot___rarg(x_34); +if (x_35 == 0) { -lean_object* x_38; uint8_t x_39; -x_38 = lean_int_mod(x_9, x_7); -x_39 = lean_int_dec_eq(x_38, x_22); -lean_dec(x_38); -if (x_39 == 0) +lean_object* x_36; uint8_t x_37; +x_36 = lean_int_mod(x_9, x_7); +x_37 = lean_int_dec_eq(x_36, x_22); +lean_dec(x_36); +if (x_37 == 0) { -lean_object* x_40; uint8_t x_41; -x_40 = l_Std_Time_Month_Ordinal_days(x_24, x_10); -x_41 = lean_int_dec_lt(x_40, x_28); -if (x_41 == 0) +uint8_t x_38; lean_object* x_39; uint8_t x_40; +x_38 = 0; +x_39 = l_Std_Time_Month_Ordinal_days(x_38, x_10); +x_40 = lean_int_dec_lt(x_39, x_25); +if (x_40 == 0) { -lean_object* x_42; lean_object* x_43; -lean_dec(x_40); -x_42 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_42, 0, x_9); -lean_ctor_set(x_42, 1, x_10); -lean_ctor_set(x_42, 2, x_28); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_42); -lean_ctor_set(x_43, 1, x_27); -return x_43; +lean_object* x_41; lean_object* x_42; +lean_dec(x_39); +x_41 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_41, 0, x_9); +lean_ctor_set(x_41, 1, x_10); +lean_ctor_set(x_41, 2, x_25); +x_42 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_24); +return x_42; } else { -lean_object* x_44; lean_object* x_45; -lean_dec(x_28); -x_44 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_44, 0, x_9); -lean_ctor_set(x_44, 1, x_10); -lean_ctor_set(x_44, 2, x_40); -x_45 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_45, 0, x_44); -lean_ctor_set(x_45, 1, x_27); -return x_45; +lean_object* x_43; lean_object* x_44; +lean_dec(x_25); +x_43 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_43, 0, x_9); +lean_ctor_set(x_43, 1, x_10); +lean_ctor_set(x_43, 2, x_39); +x_44 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_44, 0, x_43); +lean_ctor_set(x_44, 1, x_24); +return x_44; } } else { -uint8_t x_46; lean_object* x_47; uint8_t x_48; -x_46 = 1; -x_47 = l_Std_Time_Month_Ordinal_days(x_46, x_10); -x_48 = lean_int_dec_lt(x_47, x_28); -if (x_48 == 0) +uint8_t x_45; lean_object* x_46; uint8_t x_47; +x_45 = 1; +x_46 = l_Std_Time_Month_Ordinal_days(x_45, x_10); +x_47 = lean_int_dec_lt(x_46, x_25); +if (x_47 == 0) { -lean_object* x_49; lean_object* x_50; -lean_dec(x_47); -x_49 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_49, 0, x_9); -lean_ctor_set(x_49, 1, x_10); -lean_ctor_set(x_49, 2, x_28); -x_50 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_50, 0, x_49); -lean_ctor_set(x_50, 1, x_27); -return x_50; +lean_object* x_48; lean_object* x_49; +lean_dec(x_46); +x_48 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_48, 0, x_9); +lean_ctor_set(x_48, 1, x_10); +lean_ctor_set(x_48, 2, x_25); +x_49 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_49, 0, x_48); +lean_ctor_set(x_49, 1, x_24); +return x_49; } else { -lean_object* x_51; lean_object* x_52; -lean_dec(x_28); -x_51 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_51, 0, x_9); -lean_ctor_set(x_51, 1, x_10); -lean_ctor_set(x_51, 2, x_47); -x_52 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_27); -return x_52; +lean_object* x_50; lean_object* x_51; +lean_dec(x_25); +x_50 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_50, 0, x_9); +lean_ctor_set(x_50, 1, x_10); +lean_ctor_set(x_50, 2, x_46); +x_51 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_51, 0, x_50); +lean_ctor_set(x_51, 1, x_24); +return x_51; } } } else { -uint8_t x_53; lean_object* x_54; uint8_t x_55; -x_53 = 1; -x_54 = l_Std_Time_Month_Ordinal_days(x_53, x_10); -x_55 = lean_int_dec_lt(x_54, x_28); -if (x_55 == 0) +uint8_t x_52; lean_object* x_53; uint8_t x_54; +x_52 = 1; +x_53 = l_Std_Time_Month_Ordinal_days(x_52, x_10); +x_54 = lean_int_dec_lt(x_53, x_25); +if (x_54 == 0) { -lean_object* x_56; lean_object* x_57; -lean_dec(x_54); -x_56 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_56, 0, x_9); -lean_ctor_set(x_56, 1, x_10); -lean_ctor_set(x_56, 2, x_28); -x_57 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_57, 0, x_56); -lean_ctor_set(x_57, 1, x_27); -return x_57; +lean_object* x_55; lean_object* x_56; +lean_dec(x_53); +x_55 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_55, 0, x_9); +lean_ctor_set(x_55, 1, x_10); +lean_ctor_set(x_55, 2, x_25); +x_56 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_56, 0, x_55); +lean_ctor_set(x_56, 1, x_24); +return x_56; } else { -lean_object* x_58; lean_object* x_59; -lean_dec(x_28); -x_58 = lean_alloc_ctor(0, 3, 0); -lean_ctor_set(x_58, 0, x_9); -lean_ctor_set(x_58, 1, x_10); -lean_ctor_set(x_58, 2, x_54); -x_59 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_59, 0, x_58); -lean_ctor_set(x_59, 1, x_27); -return x_59; +lean_object* x_57; lean_object* x_58; +lean_dec(x_25); +x_57 = lean_alloc_ctor(0, 3, 0); +lean_ctor_set(x_57, 0, x_9); +lean_ctor_set(x_57, 1, x_10); +lean_ctor_set(x_57, 2, x_53); +x_58 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set(x_58, 1, x_24); +return x_58; } } } @@ -5527,12 +5504,11 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainDateTime_second(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; +lean_object* x_2; lean_object* x_3; x_2 = lean_ctor_get(x_1, 1); x_3 = lean_ctor_get(x_2, 2); -x_4 = lean_ctor_get(x_3, 1); -lean_inc(x_4); -return x_4; +lean_inc(x_3); +return x_3; } } LEAN_EXPORT lean_object* l_Std_Time_PlainDateTime_second___boxed(lean_object* x_1) { @@ -6254,8 +6230,6 @@ l_Std_Time_instInhabitedPlainDateTime___closed__38 = _init_l_Std_Time_instInhabi lean_mark_persistent(l_Std_Time_instInhabitedPlainDateTime___closed__38); l_Std_Time_instInhabitedPlainDateTime___closed__39 = _init_l_Std_Time_instInhabitedPlainDateTime___closed__39(); lean_mark_persistent(l_Std_Time_instInhabitedPlainDateTime___closed__39); -l_Std_Time_instInhabitedPlainDateTime___closed__40 = _init_l_Std_Time_instInhabitedPlainDateTime___closed__40(); -lean_mark_persistent(l_Std_Time_instInhabitedPlainDateTime___closed__40); l_Std_Time_instInhabitedPlainDateTime = _init_l_Std_Time_instInhabitedPlainDateTime(); lean_mark_persistent(l_Std_Time_instInhabitedPlainDateTime); l_Std_Time_instBEqPlainDateTime___closed__1 = _init_l_Std_Time_instBEqPlainDateTime___closed__1(); diff --git a/stage0/stdlib/Std/Time/DateTime/Timestamp.c b/stage0/stdlib/Std/Time/DateTime/Timestamp.c index 200a12f05bc6..a5e606c3ee02 100644 --- a/stage0/stdlib/Std/Time/DateTime/Timestamp.c +++ b/stage0/stdlib/Std/Time/DateTime/Timestamp.c @@ -59,9 +59,9 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subSeconds___boxed(lean_object*, l LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addMinutes___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subNanoseconds___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subMinutes(lean_object*, lean_object*); +static lean_object* l_Std_Time_instReprTimestamp__1___closed__3; static lean_object* l_Std_Time_Timestamp_instHAddOffset___closed__1; lean_object* lean_nat_to_int(lean_object*); -static lean_object* l_Std_Time_instToStringTimestamp___closed__1; LEAN_EXPORT lean_object* l_Std_Time_instToStringTimestamp___boxed(lean_object*); static lean_object* l_Std_Time_Timestamp_instHAddOffset__3___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addMinutes(lean_object*, lean_object*); @@ -76,7 +76,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHSubOffset__3; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addDays(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHAddOffset__5; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subWeeks___boxed(lean_object*, lean_object*); -static lean_object* l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +lean_object* l_Int_repr(lean_object*); static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__11; static lean_object* l_Std_Time_Timestamp_instHSubDuration___closed__1; static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__14; @@ -90,6 +90,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addDays___boxed(lean_object*, lean LEAN_EXPORT lean_object* l_Std_Time_Timestamp_toSecondsSinceUnixEpoch(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHAddDuration; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subDays(lean_object*, lean_object*); +static lean_object* l_Std_Time_instReprTimestamp__1___closed__1; static lean_object* l_Std_Time_Timestamp_instHAddOffset__4___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_now___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_since(lean_object*, lean_object*); @@ -105,10 +106,12 @@ lean_object* lean_string_length(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___boxed(lean_object*); static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__12; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHAddOffset__6; +static lean_object* l_Std_Time_instReprTimestamp__1___closed__2; static lean_object* l_Std_Time_Timestamp_instHSubOffset__3___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_since___boxed(lean_object*, lean_object*); static lean_object* l_Std_Time_Timestamp_toDays___closed__1; static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__5; +lean_object* l_Repr_addAppParen(lean_object*, lean_object*); uint8_t lean_int_dec_lt(lean_object*, lean_object*); lean_object* lean_nat_sub(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHAddOffset__4; @@ -122,6 +125,7 @@ lean_object* l_Std_Time_instToStringDuration_leftPad(lean_object*, lean_object*) LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subMilliseconds___boxed(lean_object*, lean_object*); static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__3; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addMilliseconds(lean_object*, lean_object*); +static lean_object* l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1; static lean_object* l_Std_Time_Timestamp_instHAddOffset__2___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addMilliseconds___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subWeeks(lean_object*, lean_object*); @@ -136,7 +140,6 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_instHSubOffset__2; uint8_t lean_int_dec_eq(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Timestamp_toDurationSinceUnixEpoch(lean_object*); lean_object* lean_get_current_time(lean_object*); -static lean_object* l_Std_Time_instToStringTimestamp___closed__2; LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addNanoseconds(lean_object*, lean_object*); lean_object* lean_string_append(lean_object*, lean_object*); static lean_object* l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__9; @@ -747,62 +750,34 @@ lean_ctor_set(x_4, 1, x_3); return x_4; } } -static lean_object* _init_l_Std_Time_instToStringTimestamp___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1000u); -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} -static lean_object* _init_l_Std_Time_instToStringTimestamp___closed__2() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1000000u); -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Std_Time_instToStringTimestamp(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; +lean_object* x_2; lean_object* x_3; uint8_t x_4; x_2 = lean_ctor_get(x_1, 0); -x_3 = l_Std_Time_instToStringTimestamp___closed__1; -x_4 = lean_int_mul(x_2, x_3); -x_5 = lean_ctor_get(x_1, 1); -x_6 = l_Std_Time_instToStringTimestamp___closed__2; -x_7 = lean_int_ediv(x_5, x_6); -x_8 = lean_int_add(x_4, x_7); -lean_dec(x_7); -lean_dec(x_4); -x_9 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__8; -x_10 = lean_int_dec_lt(x_8, x_9); -if (x_10 == 0) +x_3 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__8; +x_4 = lean_int_dec_lt(x_2, x_3); +if (x_4 == 0) { -lean_object* x_11; lean_object* x_12; -x_11 = lean_nat_abs(x_8); -lean_dec(x_8); -x_12 = l___private_Init_Data_Repr_0__Nat_reprFast(x_11); -return x_12; +lean_object* x_5; lean_object* x_6; +x_5 = lean_nat_abs(x_2); +x_6 = l___private_Init_Data_Repr_0__Nat_reprFast(x_5); +return x_6; } else { -lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_13 = lean_nat_abs(x_8); -lean_dec(x_8); -x_14 = lean_unsigned_to_nat(1u); -x_15 = lean_nat_sub(x_13, x_14); -lean_dec(x_13); -x_16 = lean_nat_add(x_15, x_14); -lean_dec(x_15); -x_17 = l___private_Init_Data_Repr_0__Nat_reprFast(x_16); -x_18 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__17; -x_19 = lean_string_append(x_18, x_17); -lean_dec(x_17); -return x_19; +lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_7 = lean_nat_abs(x_2); +x_8 = lean_unsigned_to_nat(1u); +x_9 = lean_nat_sub(x_7, x_8); +lean_dec(x_7); +x_10 = lean_nat_add(x_9, x_8); +lean_dec(x_9); +x_11 = l___private_Init_Data_Repr_0__Nat_reprFast(x_10); +x_12 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__17; +x_13 = lean_string_append(x_12, x_11); +lean_dec(x_11); +return x_13; } } } @@ -815,52 +790,74 @@ lean_dec(x_1); return x_2; } } +static lean_object* _init_l_Std_Time_instReprTimestamp__1___closed__1() { +_start: +{ +lean_object* x_1; +x_1 = lean_mk_string_unchecked("Timestamp.ofNanosecondsSinceUnixEpoch ", 38, 38); +return x_1; +} +} +static lean_object* _init_l_Std_Time_instReprTimestamp__1___closed__2() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = l_Std_Time_instReprTimestamp__1___closed__1; +x_2 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_2, 0, x_1); +return x_2; +} +} +static lean_object* _init_l_Std_Time_instReprTimestamp__1___closed__3() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1000000000u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l_Std_Time_instReprTimestamp__1(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; +lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; uint8_t x_9; x_3 = lean_ctor_get(x_1, 0); -x_4 = l_Std_Time_instToStringTimestamp___closed__1; +x_4 = l_Std_Time_instReprTimestamp__1___closed__3; x_5 = lean_int_mul(x_3, x_4); x_6 = lean_ctor_get(x_1, 1); -x_7 = l_Std_Time_instToStringTimestamp___closed__2; -x_8 = lean_int_ediv(x_6, x_7); -x_9 = lean_int_add(x_5, x_8); -lean_dec(x_8); +x_7 = lean_int_add(x_5, x_6); lean_dec(x_5); -x_10 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__8; -x_11 = lean_int_dec_lt(x_9, x_10); -if (x_11 == 0) +x_8 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__8; +x_9 = lean_int_dec_lt(x_7, x_8); +if (x_9 == 0) { -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = lean_nat_abs(x_9); -lean_dec(x_9); -x_13 = l___private_Init_Data_Repr_0__Nat_reprFast(x_12); -x_14 = l_String_quote(x_13); -lean_dec(x_13); -x_15 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; +lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_10 = l_Int_repr(x_7); +lean_dec(x_7); +x_11 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_11, 0, x_10); +x_12 = l_Std_Time_instReprTimestamp__1___closed__2; +x_13 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_13, 0, x_12); +lean_ctor_set(x_13, 1, x_11); +x_14 = l_Repr_addAppParen(x_13, x_2); +return x_14; } else { -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; -x_16 = lean_nat_abs(x_9); -lean_dec(x_9); -x_17 = lean_unsigned_to_nat(1u); -x_18 = lean_nat_sub(x_16, x_17); -lean_dec(x_16); -x_19 = lean_nat_add(x_18, x_17); -lean_dec(x_18); -x_20 = l___private_Init_Data_Repr_0__Nat_reprFast(x_19); -x_21 = l___private_Std_Time_DateTime_Timestamp_0__Std_Time_reprTimestamp____x40_Std_Time_DateTime_Timestamp___hyg_18____closed__17; -x_22 = lean_string_append(x_21, x_20); -lean_dec(x_20); -x_23 = l_String_quote(x_22); -lean_dec(x_22); -x_24 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_24, 0, x_23); -return x_24; +lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_15 = l_Int_repr(x_7); +lean_dec(x_7); +x_16 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_16, 0, x_15); +x_17 = lean_unsigned_to_nat(0u); +x_18 = l_Repr_addAppParen(x_16, x_17); +x_19 = l_Std_Time_instReprTimestamp__1___closed__2; +x_20 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_20, 0, x_19); +lean_ctor_set(x_20, 1, x_18); +x_21 = l_Repr_addAppParen(x_20, x_2); +return x_21; } } } @@ -966,11 +963,20 @@ lean_dec(x_1); return x_2; } } +static lean_object* _init_l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1() { +_start: +{ +lean_object* x_1; lean_object* x_2; +x_1 = lean_unsigned_to_nat(1000000u); +x_2 = lean_nat_to_int(x_1); +return x_2; +} +} LEAN_EXPORT lean_object* l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_2 = l_Std_Time_instToStringTimestamp___closed__2; +x_2 = l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1; x_3 = lean_int_mul(x_1, x_2); x_4 = l_Std_Time_Duration_ofNanoseconds(x_3); lean_dec(x_3); @@ -1004,21 +1010,12 @@ lean_dec(x_1); return x_2; } } -static lean_object* _init_l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = lean_unsigned_to_nat(1000000000u); -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} LEAN_EXPORT lean_object* l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch(lean_object* x_1) { _start: { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; x_2 = lean_ctor_get(x_1, 0); -x_3 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_3 = l_Std_Time_instReprTimestamp__1___closed__3; x_4 = lean_int_mul(x_2, x_3); x_5 = lean_ctor_get(x_1, 1); x_6 = lean_int_add(x_4, x_5); @@ -1040,12 +1037,12 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_toMillisecondsSinceUnixEpoch(lean_ { lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; x_2 = lean_ctor_get(x_1, 0); -x_3 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_3 = l_Std_Time_instReprTimestamp__1___closed__3; x_4 = lean_int_mul(x_2, x_3); x_5 = lean_ctor_get(x_1, 1); x_6 = lean_int_add(x_4, x_5); lean_dec(x_4); -x_7 = l_Std_Time_instToStringTimestamp___closed__2; +x_7 = l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1; x_8 = lean_int_div(x_6, x_7); lean_dec(x_6); return x_8; @@ -1079,7 +1076,7 @@ x_8 = lean_ctor_get(x_1, 1); x_9 = lean_int_neg(x_8); x_10 = lean_ctor_get(x_5, 0); lean_inc(x_10); -x_11 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_11 = l_Std_Time_instReprTimestamp__1___closed__3; x_12 = lean_int_mul(x_10, x_11); lean_dec(x_10); x_13 = lean_ctor_get(x_5, 1); @@ -1115,7 +1112,7 @@ x_23 = lean_ctor_get(x_1, 1); x_24 = lean_int_neg(x_23); x_25 = lean_ctor_get(x_19, 0); lean_inc(x_25); -x_26 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_26 = l_Std_Time_instReprTimestamp__1___closed__3; x_27 = lean_int_mul(x_25, x_26); lean_dec(x_25); x_28 = lean_ctor_get(x_19, 1); @@ -1193,12 +1190,12 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addMilliseconds(lean_object* x_1, _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; -x_3 = l_Std_Time_instToStringTimestamp___closed__2; +x_3 = l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1; x_4 = lean_int_mul(x_2, x_3); x_5 = l_Std_Time_Duration_ofNanoseconds(x_4); lean_dec(x_4); x_6 = lean_ctor_get(x_1, 0); -x_7 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_7 = l_Std_Time_instReprTimestamp__1___closed__3; x_8 = lean_int_mul(x_6, x_7); x_9 = lean_ctor_get(x_1, 1); x_10 = lean_int_add(x_8, x_9); @@ -1235,7 +1232,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subMilliseconds(lean_object* x_1, _start: { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; -x_3 = l_Std_Time_instToStringTimestamp___closed__2; +x_3 = l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1; x_4 = lean_int_mul(x_2, x_3); x_5 = l_Std_Time_Duration_ofNanoseconds(x_4); lean_dec(x_4); @@ -1249,7 +1246,7 @@ lean_dec(x_5); x_9 = lean_int_neg(x_8); lean_dec(x_8); x_10 = lean_ctor_get(x_1, 0); -x_11 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_11 = l_Std_Time_instReprTimestamp__1___closed__3; x_12 = lean_int_mul(x_10, x_11); x_13 = lean_ctor_get(x_1, 1); x_14 = lean_int_add(x_12, x_13); @@ -1283,7 +1280,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addNanoseconds(lean_object* x_1, l lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_3 = l_Std_Time_Duration_ofNanoseconds(x_2); x_4 = lean_ctor_get(x_1, 0); -x_5 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_5 = l_Std_Time_instReprTimestamp__1___closed__3; x_6 = lean_int_mul(x_4, x_5); x_7 = lean_ctor_get(x_1, 1); x_8 = lean_int_add(x_6, x_7); @@ -1331,7 +1328,7 @@ lean_dec(x_3); x_7 = lean_int_neg(x_6); lean_dec(x_6); x_8 = lean_ctor_get(x_1, 0); -x_9 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_9 = l_Std_Time_instReprTimestamp__1___closed__3; x_10 = lean_int_mul(x_8, x_9); x_11 = lean_ctor_get(x_1, 1); x_12 = lean_int_add(x_10, x_11); @@ -1364,7 +1361,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addSeconds(lean_object* x_1, lean_ { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; x_3 = lean_ctor_get(x_1, 0); -x_4 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_4 = l_Std_Time_instReprTimestamp__1___closed__3; x_5 = lean_int_mul(x_3, x_4); x_6 = lean_ctor_get(x_1, 1); x_7 = lean_int_add(x_5, x_6); @@ -1406,7 +1403,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_subSeconds(lean_object* x_1, lean_ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_3 = lean_int_neg(x_2); x_4 = lean_ctor_get(x_1, 0); -x_5 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_5 = l_Std_Time_instReprTimestamp__1___closed__3; x_6 = lean_int_mul(x_4, x_5); x_7 = lean_ctor_get(x_1, 1); x_8 = lean_int_add(x_6, x_7); @@ -1441,7 +1438,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_obj x_3 = l_Std_Time_Timestamp_toMinutes___closed__1; x_4 = lean_int_mul(x_2, x_3); x_5 = lean_ctor_get(x_1, 0); -x_6 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_6 = l_Std_Time_instReprTimestamp__1___closed__3; x_7 = lean_int_mul(x_5, x_6); x_8 = lean_ctor_get(x_1, 1); x_9 = lean_int_add(x_7, x_8); @@ -1478,7 +1475,7 @@ x_4 = lean_int_mul(x_2, x_3); x_5 = lean_int_neg(x_4); lean_dec(x_4); x_6 = lean_ctor_get(x_1, 0); -x_7 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_7 = l_Std_Time_instReprTimestamp__1___closed__3; x_8 = lean_int_mul(x_6, x_7); x_9 = lean_ctor_get(x_1, 1); x_10 = lean_int_add(x_8, x_9); @@ -1522,7 +1519,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_obj x_3 = l_Std_Time_Timestamp_addHours___closed__1; x_4 = lean_int_mul(x_2, x_3); x_5 = lean_ctor_get(x_1, 0); -x_6 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_6 = l_Std_Time_instReprTimestamp__1___closed__3; x_7 = lean_int_mul(x_5, x_6); x_8 = lean_ctor_get(x_1, 1); x_9 = lean_int_add(x_7, x_8); @@ -1559,7 +1556,7 @@ x_4 = lean_int_mul(x_2, x_3); x_5 = lean_int_neg(x_4); lean_dec(x_4); x_6 = lean_ctor_get(x_1, 0); -x_7 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_7 = l_Std_Time_instReprTimestamp__1___closed__3; x_8 = lean_int_mul(x_6, x_7); x_9 = lean_ctor_get(x_1, 1); x_10 = lean_int_add(x_8, x_9); @@ -1594,7 +1591,7 @@ lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_obj x_3 = l_Std_Time_Timestamp_toDays___closed__1; x_4 = lean_int_mul(x_2, x_3); x_5 = lean_ctor_get(x_1, 0); -x_6 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_6 = l_Std_Time_instReprTimestamp__1___closed__3; x_7 = lean_int_mul(x_5, x_6); x_8 = lean_ctor_get(x_1, 1); x_9 = lean_int_add(x_7, x_8); @@ -1631,7 +1628,7 @@ x_4 = lean_int_mul(x_2, x_3); x_5 = lean_int_neg(x_4); lean_dec(x_4); x_6 = lean_ctor_get(x_1, 0); -x_7 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_7 = l_Std_Time_instReprTimestamp__1___closed__3; x_8 = lean_int_mul(x_6, x_7); x_9 = lean_ctor_get(x_1, 1); x_10 = lean_int_add(x_8, x_9); @@ -1669,7 +1666,7 @@ x_5 = l_Std_Time_Timestamp_toDays___closed__1; x_6 = lean_int_mul(x_4, x_5); lean_dec(x_4); x_7 = lean_ctor_get(x_1, 0); -x_8 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_8 = l_Std_Time_instReprTimestamp__1___closed__3; x_9 = lean_int_mul(x_7, x_8); x_10 = lean_ctor_get(x_1, 1); x_11 = lean_int_add(x_9, x_10); @@ -1709,7 +1706,7 @@ lean_dec(x_4); x_7 = lean_int_neg(x_6); lean_dec(x_6); x_8 = lean_ctor_get(x_1, 0); -x_9 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_9 = l_Std_Time_instReprTimestamp__1___closed__3; x_10 = lean_int_mul(x_8, x_9); x_11 = lean_ctor_get(x_1, 1); x_12 = lean_int_add(x_10, x_11); @@ -1742,7 +1739,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Timestamp_addDuration(lean_object* x_1, lean { lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_3 = lean_ctor_get(x_1, 0); -x_4 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_4 = l_Std_Time_instReprTimestamp__1___closed__3; x_5 = lean_int_mul(x_3, x_4); x_6 = lean_ctor_get(x_1, 1); x_7 = lean_int_add(x_5, x_6); @@ -1779,7 +1776,7 @@ x_4 = lean_int_neg(x_3); x_5 = lean_ctor_get(x_2, 1); x_6 = lean_int_neg(x_5); x_7 = lean_ctor_get(x_1, 0); -x_8 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_8 = l_Std_Time_instReprTimestamp__1___closed__3; x_9 = lean_int_mul(x_7, x_8); x_10 = lean_ctor_get(x_1, 1); x_11 = lean_int_add(x_9, x_10); @@ -2072,7 +2069,7 @@ x_4 = lean_int_neg(x_3); x_5 = lean_ctor_get(x_2, 1); x_6 = lean_int_neg(x_5); x_7 = lean_ctor_get(x_1, 0); -x_8 = l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1; +x_8 = l_Std_Time_instReprTimestamp__1___closed__3; x_9 = lean_int_mul(x_7, x_8); x_10 = lean_ctor_get(x_1, 1); x_11 = lean_int_add(x_9, x_10); @@ -2175,16 +2172,18 @@ l_Std_Time_instInhabitedTimestamp = _init_l_Std_Time_instInhabitedTimestamp(); lean_mark_persistent(l_Std_Time_instInhabitedTimestamp); l_Std_Time_instLETimestamp = _init_l_Std_Time_instLETimestamp(); lean_mark_persistent(l_Std_Time_instLETimestamp); -l_Std_Time_instToStringTimestamp___closed__1 = _init_l_Std_Time_instToStringTimestamp___closed__1(); -lean_mark_persistent(l_Std_Time_instToStringTimestamp___closed__1); -l_Std_Time_instToStringTimestamp___closed__2 = _init_l_Std_Time_instToStringTimestamp___closed__2(); -lean_mark_persistent(l_Std_Time_instToStringTimestamp___closed__2); +l_Std_Time_instReprTimestamp__1___closed__1 = _init_l_Std_Time_instReprTimestamp__1___closed__1(); +lean_mark_persistent(l_Std_Time_instReprTimestamp__1___closed__1); +l_Std_Time_instReprTimestamp__1___closed__2 = _init_l_Std_Time_instReprTimestamp__1___closed__2(); +lean_mark_persistent(l_Std_Time_instReprTimestamp__1___closed__2); +l_Std_Time_instReprTimestamp__1___closed__3 = _init_l_Std_Time_instReprTimestamp__1___closed__3(); +lean_mark_persistent(l_Std_Time_instReprTimestamp__1___closed__3); l_Std_Time_Timestamp_toMinutes___closed__1 = _init_l_Std_Time_Timestamp_toMinutes___closed__1(); lean_mark_persistent(l_Std_Time_Timestamp_toMinutes___closed__1); l_Std_Time_Timestamp_toDays___closed__1 = _init_l_Std_Time_Timestamp_toDays___closed__1(); lean_mark_persistent(l_Std_Time_Timestamp_toDays___closed__1); -l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1 = _init_l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1(); -lean_mark_persistent(l_Std_Time_Timestamp_toNanosecondsSinceUnixEpoch___closed__1); +l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1 = _init_l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1(); +lean_mark_persistent(l_Std_Time_Timestamp_ofMillisecondsSinceUnixEpoch___closed__1); l_Std_Time_Timestamp_subSeconds___closed__1 = _init_l_Std_Time_Timestamp_subSeconds___closed__1(); lean_mark_persistent(l_Std_Time_Timestamp_subSeconds___closed__1); l_Std_Time_Timestamp_addHours___closed__1 = _init_l_Std_Time_Timestamp_addHours___closed__1(); diff --git a/stage0/stdlib/Std/Time/Format.c b/stage0/stdlib/Std/Time/Format.c index 6cb9efd29560..17365ce0ccc7 100644 --- a/stage0/stdlib/Std/Time/Format.c +++ b/stage0/stdlib/Std/Time/Format.c @@ -4550,42 +4550,16 @@ return x_3; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_fromTime24Hour___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_4; -x_4 = !lean_is_exclusive(x_3); -if (x_4 == 0) -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; -x_5 = l_Std_Time_PlainDate_format___lambda__1___closed__2; -x_6 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_2); -lean_ctor_set(x_6, 2, x_3); -lean_ctor_set(x_6, 3, x_5); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; -x_8 = lean_ctor_get(x_3, 0); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_3); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = l_Std_Time_PlainDate_format___lambda__1___closed__2; -x_12 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_12, 0, x_1); -lean_ctor_set(x_12, 1, x_2); -lean_ctor_set(x_12, 2, x_10); -lean_ctor_set(x_12, 3, x_11); -x_13 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_13, 0, x_12); -return x_13; -} +lean_object* x_4; lean_object* x_5; lean_object* x_6; +x_4 = l_Std_Time_PlainDate_format___lambda__1___closed__2; +x_5 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } static lean_object* _init_l_Std_Time_PlainTime_fromTime24Hour___closed__1() { @@ -4627,40 +4601,15 @@ return x_8; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_fromLeanTime24Hour___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -uint8_t x_5; -x_5 = !lean_is_exclusive(x_3); -if (x_5 == 0) -{ -lean_object* x_6; lean_object* x_7; -x_6 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_6, 0, x_1); -lean_ctor_set(x_6, 1, x_2); -lean_ctor_set(x_6, 2, x_3); -lean_ctor_set(x_6, 3, x_4); -x_7 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_7, 0, x_6); -return x_7; -} -else -{ -lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; -x_8 = lean_ctor_get(x_3, 0); -x_9 = lean_ctor_get(x_3, 1); -lean_inc(x_9); -lean_inc(x_8); -lean_dec(x_3); -x_10 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_10, 0, x_8); -lean_ctor_set(x_10, 1, x_9); -x_11 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_11, 0, x_1); -lean_ctor_set(x_11, 1, x_2); -lean_ctor_set(x_11, 2, x_10); -lean_ctor_set(x_11, 3, x_4); -x_12 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_12, 0, x_11); -return x_12; -} +lean_object* x_5; lean_object* x_6; +x_5 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_4); +x_6 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_6, 0, x_5); +return x_6; } } static lean_object* _init_l_Std_Time_PlainTime_fromLeanTime24Hour___closed__1() { @@ -4768,44 +4717,17 @@ return x_10; } else { -uint8_t x_11; -x_11 = !lean_is_exclusive(x_3); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; -x_12 = l_Std_Time_HourMarker_toAbsolute(x_4, x_1); -x_13 = l_Std_Time_PlainDate_format___lambda__1___closed__2; -x_14 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_14, 0, x_12); -lean_ctor_set(x_14, 1, x_2); -lean_ctor_set(x_14, 2, x_3); -lean_ctor_set(x_14, 3, x_13); -x_15 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_15, 0, x_14); -return x_15; -} -else -{ -lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; -x_16 = lean_ctor_get(x_3, 0); -x_17 = lean_ctor_get(x_3, 1); -lean_inc(x_17); -lean_inc(x_16); -lean_dec(x_3); -x_18 = l_Std_Time_HourMarker_toAbsolute(x_4, x_1); -x_19 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_19, 0, x_16); -lean_ctor_set(x_19, 1, x_17); -x_20 = l_Std_Time_PlainDate_format___lambda__1___closed__2; -x_21 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_21, 0, x_18); -lean_ctor_set(x_21, 1, x_2); -lean_ctor_set(x_21, 2, x_19); -lean_ctor_set(x_21, 3, x_20); -x_22 = lean_alloc_ctor(1, 1, 0); -lean_ctor_set(x_22, 0, x_21); -return x_22; -} +lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; +x_11 = l_Std_Time_HourMarker_toAbsolute(x_4, x_1); +x_12 = l_Std_Time_PlainDate_format___lambda__1___closed__2; +x_13 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_13, 0, x_11); +lean_ctor_set(x_13, 1, x_2); +lean_ctor_set(x_13, 2, x_3); +lean_ctor_set(x_13, 3, x_12); +x_14 = lean_alloc_ctor(1, 1, 0); +lean_ctor_set(x_14, 0, x_13); +return x_14; } } } diff --git a/stage0/stdlib/Std/Time/Format/Basic.c b/stage0/stdlib/Std/Time/Format/Basic.c index 9116bfad1905..50680c5fa3d7 100644 --- a/stage0/stdlib/Std/Time/Format/Basic.c +++ b/stage0/stdlib/Std/Time/Format/Basic.c @@ -644,7 +644,6 @@ static lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_reprZoneName__ static lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_reprOffsetX____x40_Std_Time_Format_Basic___hyg_1001____closed__14; LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_parseModifier___closed__23___boxed__const__1; static lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_reprOffsetZ____x40_Std_Time_Format_Basic___hyg_1406____closed__8; -static lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18; static lean_object* l_Sum_repr___at___private_Std_Time_Format_Basic_0__Std_Time_reprModifier____x40_Std_Time_Format_Basic___hyg_1845____spec__1___closed__3; static lean_object* l_Std_Time_instReprOffsetZ___closed__1; LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___lambda__2___boxed(lean_object*, lean_object*); @@ -1006,7 +1005,6 @@ LEAN_EXPORT lean_object* l_Std_Internal_Parsec_many1Chars___at___private_Std_Tim LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_parseModifier___lambda__22(lean_object*); static lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_reprModifier____x40_Std_Time_Format_Basic___hyg_1845____closed__72; static lean_object* l_Std_Time_ZoneName_classify___closed__1; -static lean_object* l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35; LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_parseModifier___closed__35___boxed__const__1; LEAN_EXPORT lean_object* l_Std_Internal_Parsec_manyCharsCore___at___private_Std_Time_Format_Basic_0__Std_Time_parseFormatPart___spec__2___lambda__1___boxed(lean_object*, lean_object*); static lean_object* l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; @@ -44033,7 +44031,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_Awareness_instInhabitedType___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_4 = l___private_Std_Time_Format_Basic_0__Std_Time_reprNumber____x40_Std_Time_Format_Basic___hyg_205____closed__7; x_5 = lean_int_add(x_1, x_4); x_6 = lean_int_sub(x_5, x_1); @@ -44099,21 +44097,16 @@ lean_dec(x_34); lean_dec(x_36); x_38 = lean_int_add(x_37, x_2); lean_dec(x_37); -x_39 = 0; -x_40 = lean_box(x_39); lean_inc(x_38); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_30); -lean_ctor_set(x_42, 1, x_38); -lean_ctor_set(x_42, 2, x_41); -lean_ctor_set(x_42, 3, x_2); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_21); -lean_ctor_set(x_43, 1, x_42); -return x_43; +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_30); +lean_ctor_set(x_39, 1, x_38); +lean_ctor_set(x_39, 2, x_38); +lean_ctor_set(x_39, 3, x_2); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_21); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } static lean_object* _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1() { @@ -44440,38 +44433,24 @@ return x_3; static lean_object* _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__33() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__25; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__32; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); +x_3 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_4 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_3); return x_4; } } static lean_object* _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__25; -x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__32; -x_3 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__33; -x_4 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} -} -static lean_object* _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__17; -x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34; +x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__33; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -44482,7 +44461,7 @@ LEAN_EXPORT lean_object* l_Std_Time_Awareness_instInhabitedType___lambda__2(lean _start: { lean_object* x_2; -x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35; +x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34; return x_2; } } @@ -49524,71 +49503,71 @@ return x_1; LEAN_EXPORT lean_object* l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(lean_object* x_1, uint8_t x_2, uint8_t x_3, uint8_t x_4) { _start: { -lean_object* x_5; lean_object* x_6; lean_object* x_127; uint8_t x_128; -x_127 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_128 = lean_int_dec_le(x_127, x_1); -if (x_128 == 0) +lean_object* x_5; lean_object* x_6; lean_object* x_126; uint8_t x_127; +x_126 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_127 = lean_int_dec_le(x_126, x_1); +if (x_127 == 0) { -lean_object* x_129; lean_object* x_130; -x_129 = lean_int_neg(x_1); +lean_object* x_128; lean_object* x_129; +x_128 = lean_int_neg(x_1); lean_dec(x_1); -x_130 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_5 = x_130; -x_6 = x_129; -goto block_126; +x_129 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_5 = x_129; +x_6 = x_128; +goto block_125; } else { -lean_object* x_131; -x_131 = l___private_Std_Time_Format_Basic_0__Std_Time_toSigned___closed__1; -x_5 = x_131; +lean_object* x_130; +x_130 = l___private_Std_Time_Format_Basic_0__Std_Time_toSigned___closed__1; +x_5 = x_130; x_6 = x_1; -goto block_126; +goto block_125; } -block_126: +block_125: { -lean_object* x_7; lean_object* x_8; lean_object* x_9; uint32_t x_10; lean_object* x_11; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_114; lean_object* x_115; uint8_t x_116; +lean_object* x_7; lean_object* x_8; lean_object* x_9; uint32_t x_10; lean_object* x_11; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_113; lean_object* x_114; uint8_t x_115; x_7 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString___closed__1; x_8 = lean_int_mul(x_6, x_7); lean_dec(x_6); x_9 = l_Std_Time_PlainTime_ofNanoseconds(x_8); lean_dec(x_8); x_10 = 48; -x_62 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; -x_63 = lean_string_append(x_62, x_5); +x_61 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; +x_62 = lean_string_append(x_61, x_5); lean_dec(x_5); -x_64 = lean_string_append(x_63, x_62); -x_114 = lean_ctor_get(x_9, 0); -lean_inc(x_114); -x_115 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_116 = lean_int_dec_lt(x_114, x_115); -if (x_116 == 0) +x_63 = lean_string_append(x_62, x_61); +x_113 = lean_ctor_get(x_9, 0); +lean_inc(x_113); +x_114 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_115 = lean_int_dec_lt(x_113, x_114); +if (x_115 == 0) { -lean_object* x_117; lean_object* x_118; -x_117 = lean_nat_abs(x_114); -lean_dec(x_114); -x_118 = l___private_Init_Data_Repr_0__Nat_reprFast(x_117); -x_65 = x_118; -goto block_113; +lean_object* x_116; lean_object* x_117; +x_116 = lean_nat_abs(x_113); +lean_dec(x_113); +x_117 = l___private_Init_Data_Repr_0__Nat_reprFast(x_116); +x_64 = x_117; +goto block_112; } else { -lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; -x_119 = lean_nat_abs(x_114); -lean_dec(x_114); -x_120 = lean_unsigned_to_nat(1u); -x_121 = lean_nat_sub(x_119, x_120); -lean_dec(x_119); -x_122 = lean_nat_add(x_121, x_120); -lean_dec(x_121); -x_123 = l___private_Init_Data_Repr_0__Nat_reprFast(x_122); -x_124 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_125 = lean_string_append(x_124, x_123); -lean_dec(x_123); -x_65 = x_125; -goto block_113; +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_118 = lean_nat_abs(x_113); +lean_dec(x_113); +x_119 = lean_unsigned_to_nat(1u); +x_120 = lean_nat_sub(x_118, x_119); +lean_dec(x_118); +x_121 = lean_nat_add(x_120, x_119); +lean_dec(x_120); +x_122 = l___private_Init_Data_Repr_0__Nat_reprFast(x_121); +x_123 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_124 = lean_string_append(x_123, x_122); +lean_dec(x_122); +x_64 = x_124; +goto block_112; } -block_61: +block_60: { if (x_3 == 0) { @@ -49597,229 +49576,226 @@ return x_11; } else { -lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; uint8_t x_16; +lean_object* x_12; lean_object* x_13; uint8_t x_14; uint8_t x_15; x_12 = lean_ctor_get(x_9, 2); lean_inc(x_12); lean_dec(x_9); -x_13 = lean_ctor_get(x_12, 1); -lean_inc(x_13); -lean_dec(x_12); -x_14 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_15 = lean_int_dec_eq(x_13, x_14); -x_16 = l_instDecidableNot___rarg(x_15); -if (x_16 == 0) +x_13 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_14 = lean_int_dec_eq(x_12, x_13); +x_15 = l_instDecidableNot___rarg(x_14); +if (x_15 == 0) { -lean_dec(x_13); +lean_dec(x_12); return x_11; } else { -lean_object* x_17; lean_object* x_18; lean_object* x_19; -x_17 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; -x_18 = lean_string_append(x_17, x_11); +lean_object* x_16; lean_object* x_17; lean_object* x_18; +x_16 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; +x_17 = lean_string_append(x_16, x_11); lean_dec(x_11); -x_19 = lean_string_append(x_18, x_17); +x_18 = lean_string_append(x_17, x_16); if (x_4 == 0) { -lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_20 = lean_string_append(x_19, x_17); -x_21 = lean_string_append(x_20, x_17); -x_22 = lean_int_dec_lt(x_13, x_14); -if (x_22 == 0) +lean_object* x_19; lean_object* x_20; uint8_t x_21; +x_19 = lean_string_append(x_18, x_16); +x_20 = lean_string_append(x_19, x_16); +x_21 = lean_int_dec_lt(x_12, x_13); +if (x_21 == 0) { -lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; -x_23 = lean_nat_abs(x_13); -lean_dec(x_13); -x_24 = l___private_Init_Data_Repr_0__Nat_reprFast(x_23); -x_25 = lean_unsigned_to_nat(2u); -x_26 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_25, x_10, x_24); -lean_dec(x_24); -x_27 = lean_string_append(x_21, x_26); -lean_dec(x_26); -x_28 = lean_string_append(x_27, x_17); -return x_28; +lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_22 = lean_nat_abs(x_12); +lean_dec(x_12); +x_23 = l___private_Init_Data_Repr_0__Nat_reprFast(x_22); +x_24 = lean_unsigned_to_nat(2u); +x_25 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_24, x_10, x_23); +lean_dec(x_23); +x_26 = lean_string_append(x_20, x_25); +lean_dec(x_25); +x_27 = lean_string_append(x_26, x_16); +return x_27; } else { -lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; -x_29 = lean_nat_abs(x_13); -lean_dec(x_13); -x_30 = lean_unsigned_to_nat(1u); -x_31 = lean_nat_sub(x_29, x_30); -lean_dec(x_29); -x_32 = lean_nat_add(x_31, x_30); -lean_dec(x_31); -x_33 = l___private_Init_Data_Repr_0__Nat_reprFast(x_32); -x_34 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_35 = lean_string_append(x_34, x_33); -lean_dec(x_33); -x_36 = lean_unsigned_to_nat(2u); -x_37 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_36, x_10, x_35); -lean_dec(x_35); -x_38 = lean_string_append(x_21, x_37); -lean_dec(x_37); -x_39 = lean_string_append(x_38, x_17); -return x_39; +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; +x_28 = lean_nat_abs(x_12); +lean_dec(x_12); +x_29 = lean_unsigned_to_nat(1u); +x_30 = lean_nat_sub(x_28, x_29); +lean_dec(x_28); +x_31 = lean_nat_add(x_30, x_29); +lean_dec(x_30); +x_32 = l___private_Init_Data_Repr_0__Nat_reprFast(x_31); +x_33 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_34 = lean_string_append(x_33, x_32); +lean_dec(x_32); +x_35 = lean_unsigned_to_nat(2u); +x_36 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_35, x_10, x_34); +lean_dec(x_34); +x_37 = lean_string_append(x_20, x_36); +lean_dec(x_36); +x_38 = lean_string_append(x_37, x_16); +return x_38; } } else { -lean_object* x_40; lean_object* x_41; lean_object* x_42; uint8_t x_43; -x_40 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString___closed__2; -x_41 = lean_string_append(x_19, x_40); -x_42 = lean_string_append(x_41, x_17); -x_43 = lean_int_dec_lt(x_13, x_14); -if (x_43 == 0) +lean_object* x_39; lean_object* x_40; lean_object* x_41; uint8_t x_42; +x_39 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString___closed__2; +x_40 = lean_string_append(x_18, x_39); +x_41 = lean_string_append(x_40, x_16); +x_42 = lean_int_dec_lt(x_12, x_13); +if (x_42 == 0) { -lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; -x_44 = lean_nat_abs(x_13); -lean_dec(x_13); -x_45 = l___private_Init_Data_Repr_0__Nat_reprFast(x_44); -x_46 = lean_unsigned_to_nat(2u); -x_47 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_46, x_10, x_45); -lean_dec(x_45); -x_48 = lean_string_append(x_42, x_47); -lean_dec(x_47); -x_49 = lean_string_append(x_48, x_17); -return x_49; +lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; +x_43 = lean_nat_abs(x_12); +lean_dec(x_12); +x_44 = l___private_Init_Data_Repr_0__Nat_reprFast(x_43); +x_45 = lean_unsigned_to_nat(2u); +x_46 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_45, x_10, x_44); +lean_dec(x_44); +x_47 = lean_string_append(x_41, x_46); +lean_dec(x_46); +x_48 = lean_string_append(x_47, x_16); +return x_48; } else { -lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; -x_50 = lean_nat_abs(x_13); -lean_dec(x_13); -x_51 = lean_unsigned_to_nat(1u); -x_52 = lean_nat_sub(x_50, x_51); -lean_dec(x_50); -x_53 = lean_nat_add(x_52, x_51); -lean_dec(x_52); -x_54 = l___private_Init_Data_Repr_0__Nat_reprFast(x_53); -x_55 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_56 = lean_string_append(x_55, x_54); -lean_dec(x_54); -x_57 = lean_unsigned_to_nat(2u); -x_58 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_57, x_10, x_56); -lean_dec(x_56); -x_59 = lean_string_append(x_42, x_58); -lean_dec(x_58); -x_60 = lean_string_append(x_59, x_17); -return x_60; +lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; +x_49 = lean_nat_abs(x_12); +lean_dec(x_12); +x_50 = lean_unsigned_to_nat(1u); +x_51 = lean_nat_sub(x_49, x_50); +lean_dec(x_49); +x_52 = lean_nat_add(x_51, x_50); +lean_dec(x_51); +x_53 = l___private_Init_Data_Repr_0__Nat_reprFast(x_52); +x_54 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_55 = lean_string_append(x_54, x_53); +lean_dec(x_53); +x_56 = lean_unsigned_to_nat(2u); +x_57 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_56, x_10, x_55); +lean_dec(x_55); +x_58 = lean_string_append(x_41, x_57); +lean_dec(x_57); +x_59 = lean_string_append(x_58, x_16); +return x_59; } } } } } -block_113: +block_112: { -lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; -x_66 = lean_unsigned_to_nat(2u); -x_67 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_66, x_10, x_65); -lean_dec(x_65); -x_68 = lean_string_append(x_64, x_67); -lean_dec(x_67); -x_69 = lean_string_append(x_68, x_62); +lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; +x_65 = lean_unsigned_to_nat(2u); +x_66 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_65, x_10, x_64); +lean_dec(x_64); +x_67 = lean_string_append(x_63, x_66); +lean_dec(x_66); +x_68 = lean_string_append(x_67, x_61); if (x_2 == 0) { -x_11 = x_69; -goto block_61; +x_11 = x_68; +goto block_60; } else { -lean_object* x_70; lean_object* x_71; -x_70 = lean_string_append(x_62, x_69); -lean_dec(x_69); -x_71 = lean_string_append(x_70, x_62); +lean_object* x_69; lean_object* x_70; +x_69 = lean_string_append(x_61, x_68); +lean_dec(x_68); +x_70 = lean_string_append(x_69, x_61); if (x_4 == 0) { -lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; uint8_t x_76; -x_72 = lean_ctor_get(x_9, 1); -lean_inc(x_72); -x_73 = lean_string_append(x_71, x_62); -x_74 = lean_string_append(x_73, x_62); -x_75 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_76 = lean_int_dec_lt(x_72, x_75); -if (x_76 == 0) +lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; uint8_t x_75; +x_71 = lean_ctor_get(x_9, 1); +lean_inc(x_71); +x_72 = lean_string_append(x_70, x_61); +x_73 = lean_string_append(x_72, x_61); +x_74 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_75 = lean_int_dec_lt(x_71, x_74); +if (x_75 == 0) { -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; -x_77 = lean_nat_abs(x_72); -lean_dec(x_72); -x_78 = l___private_Init_Data_Repr_0__Nat_reprFast(x_77); -x_79 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_66, x_10, x_78); +lean_object* x_76; lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_76 = lean_nat_abs(x_71); +lean_dec(x_71); +x_77 = l___private_Init_Data_Repr_0__Nat_reprFast(x_76); +x_78 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_65, x_10, x_77); +lean_dec(x_77); +x_79 = lean_string_append(x_73, x_78); lean_dec(x_78); -x_80 = lean_string_append(x_74, x_79); -lean_dec(x_79); -x_81 = lean_string_append(x_80, x_62); -x_11 = x_81; -goto block_61; +x_80 = lean_string_append(x_79, x_61); +x_11 = x_80; +goto block_60; } else { -lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; -x_82 = lean_nat_abs(x_72); -lean_dec(x_72); -x_83 = lean_unsigned_to_nat(1u); -x_84 = lean_nat_sub(x_82, x_83); -lean_dec(x_82); -x_85 = lean_nat_add(x_84, x_83); -lean_dec(x_84); -x_86 = l___private_Init_Data_Repr_0__Nat_reprFast(x_85); -x_87 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_88 = lean_string_append(x_87, x_86); -lean_dec(x_86); -x_89 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_66, x_10, x_88); +lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; +x_81 = lean_nat_abs(x_71); +lean_dec(x_71); +x_82 = lean_unsigned_to_nat(1u); +x_83 = lean_nat_sub(x_81, x_82); +lean_dec(x_81); +x_84 = lean_nat_add(x_83, x_82); +lean_dec(x_83); +x_85 = l___private_Init_Data_Repr_0__Nat_reprFast(x_84); +x_86 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_87 = lean_string_append(x_86, x_85); +lean_dec(x_85); +x_88 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_65, x_10, x_87); +lean_dec(x_87); +x_89 = lean_string_append(x_73, x_88); lean_dec(x_88); -x_90 = lean_string_append(x_74, x_89); -lean_dec(x_89); -x_91 = lean_string_append(x_90, x_62); -x_11 = x_91; -goto block_61; +x_90 = lean_string_append(x_89, x_61); +x_11 = x_90; +goto block_60; } } else { -lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; uint8_t x_97; -x_92 = lean_ctor_get(x_9, 1); -lean_inc(x_92); -x_93 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString___closed__2; -x_94 = lean_string_append(x_71, x_93); -x_95 = lean_string_append(x_94, x_62); -x_96 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_97 = lean_int_dec_lt(x_92, x_96); -if (x_97 == 0) +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; uint8_t x_96; +x_91 = lean_ctor_get(x_9, 1); +lean_inc(x_91); +x_92 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString___closed__2; +x_93 = lean_string_append(x_70, x_92); +x_94 = lean_string_append(x_93, x_61); +x_95 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_96 = lean_int_dec_lt(x_91, x_95); +if (x_96 == 0) { -lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; -x_98 = lean_nat_abs(x_92); -lean_dec(x_92); -x_99 = l___private_Init_Data_Repr_0__Nat_reprFast(x_98); -x_100 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_66, x_10, x_99); +lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; +x_97 = lean_nat_abs(x_91); +lean_dec(x_91); +x_98 = l___private_Init_Data_Repr_0__Nat_reprFast(x_97); +x_99 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_65, x_10, x_98); +lean_dec(x_98); +x_100 = lean_string_append(x_94, x_99); lean_dec(x_99); -x_101 = lean_string_append(x_95, x_100); -lean_dec(x_100); -x_102 = lean_string_append(x_101, x_62); -x_11 = x_102; -goto block_61; +x_101 = lean_string_append(x_100, x_61); +x_11 = x_101; +goto block_60; } else { -lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; lean_object* x_112; -x_103 = lean_nat_abs(x_92); -lean_dec(x_92); -x_104 = lean_unsigned_to_nat(1u); -x_105 = lean_nat_sub(x_103, x_104); -lean_dec(x_103); -x_106 = lean_nat_add(x_105, x_104); -lean_dec(x_105); -x_107 = l___private_Init_Data_Repr_0__Nat_reprFast(x_106); -x_108 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; -x_109 = lean_string_append(x_108, x_107); -lean_dec(x_107); -x_110 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_66, x_10, x_109); +lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; lean_object* x_111; +x_102 = lean_nat_abs(x_91); +lean_dec(x_91); +x_103 = lean_unsigned_to_nat(1u); +x_104 = lean_nat_sub(x_102, x_103); +lean_dec(x_102); +x_105 = lean_nat_add(x_104, x_103); +lean_dec(x_104); +x_106 = l___private_Init_Data_Repr_0__Nat_reprFast(x_105); +x_107 = l___private_Std_Time_Format_Basic_0__Std_Time_pad___closed__1; +x_108 = lean_string_append(x_107, x_106); +lean_dec(x_106); +x_109 = l___private_Std_Time_Format_Basic_0__Std_Time_leftPad(x_65, x_10, x_108); +lean_dec(x_108); +x_110 = lean_string_append(x_94, x_109); lean_dec(x_109); -x_111 = lean_string_append(x_95, x_110); -lean_dec(x_110); -x_112 = lean_string_append(x_111, x_62); -x_11 = x_112; -goto block_61; +x_111 = lean_string_append(x_110, x_61); +x_11 = x_111; +goto block_60; } } } @@ -50315,43 +50291,29 @@ x_109 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_105, x_107, x_108); lean_dec(x_105); return x_109; } -case 18: +case 19: { -lean_object* x_110; lean_object* x_111; uint8_t x_112; lean_object* x_113; +lean_object* x_110; x_110 = lean_ctor_get(x_1, 0); lean_inc(x_110); lean_dec(x_1); -x_111 = lean_ctor_get(x_2, 1); -lean_inc(x_111); -lean_dec(x_2); +if (lean_obj_tag(x_110) == 0) +{ +lean_object* x_111; uint8_t x_112; lean_object* x_113; +x_111 = lean_unsigned_to_nat(9u); x_112 = 0; -x_113 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_110, x_111, x_112); -lean_dec(x_110); +x_113 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_111, x_2, x_112); return x_113; } -case 19: -{ -lean_object* x_114; -x_114 = lean_ctor_get(x_1, 0); -lean_inc(x_114); -lean_dec(x_1); -if (lean_obj_tag(x_114) == 0) -{ -lean_object* x_115; uint8_t x_116; lean_object* x_117; -x_115 = lean_unsigned_to_nat(9u); -x_116 = 0; -x_117 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_115, x_2, x_116); -return x_117; -} else { -lean_object* x_118; uint8_t x_119; lean_object* x_120; -x_118 = lean_ctor_get(x_114, 0); -lean_inc(x_118); -lean_dec(x_114); -x_119 = 1; -x_120 = l___private_Std_Time_Format_Basic_0__Std_Time_rightTruncate(x_118, x_2, x_119); -return x_120; +lean_object* x_114; uint8_t x_115; lean_object* x_116; +x_114 = lean_ctor_get(x_110, 0); +lean_inc(x_114); +lean_dec(x_110); +x_115 = 1; +x_116 = l___private_Std_Time_Format_Basic_0__Std_Time_rightTruncate(x_114, x_2, x_115); +return x_116; } } case 23: @@ -50365,238 +50327,238 @@ return x_2; } case 25: { -uint8_t x_121; -x_121 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_117; +x_117 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -if (x_121 == 0) +if (x_117 == 0) { -lean_object* x_122; lean_object* x_123; lean_object* x_124; lean_object* x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; -x_122 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__3; -x_123 = lean_int_div(x_2, x_122); +lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; +x_118 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__3; +x_119 = lean_int_div(x_2, x_118); lean_dec(x_2); -x_124 = l___private_Std_Time_Format_Basic_0__Std_Time_toSigned(x_123); -lean_dec(x_123); -x_125 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_126 = lean_string_append(x_125, x_124); -lean_dec(x_124); -x_127 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; -x_128 = lean_string_append(x_126, x_127); -return x_128; +x_120 = l___private_Std_Time_Format_Basic_0__Std_Time_toSigned(x_119); +lean_dec(x_119); +x_121 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_122 = lean_string_append(x_121, x_120); +lean_dec(x_120); +x_123 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; +x_124 = lean_string_append(x_122, x_123); +return x_124; } else { -uint8_t x_129; uint8_t x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; -x_129 = 1; -x_130 = 0; -x_131 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_129, x_130, x_129); -x_132 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_133 = lean_string_append(x_132, x_131); -lean_dec(x_131); -x_134 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; -x_135 = lean_string_append(x_133, x_134); -return x_135; +uint8_t x_125; uint8_t x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; +x_125 = 1; +x_126 = 0; +x_127 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_125, x_126, x_125); +x_128 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_129 = lean_string_append(x_128, x_127); +lean_dec(x_127); +x_130 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; +x_131 = lean_string_append(x_129, x_130); +return x_131; } } case 26: { -uint8_t x_136; lean_object* x_137; uint8_t x_138; -x_136 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_132; lean_object* x_133; uint8_t x_134; +x_132 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -x_137 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_138 = lean_int_dec_eq(x_2, x_137); -if (x_138 == 0) +x_133 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_134 = lean_int_dec_eq(x_2, x_133); +if (x_134 == 0) { -switch (x_136) { +switch (x_132) { case 0: { -uint8_t x_139; lean_object* x_140; -x_139 = 0; -x_140 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_139, x_139, x_139); -return x_140; +uint8_t x_135; lean_object* x_136; +x_135 = 0; +x_136 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_135, x_135, x_135); +return x_136; } case 1: { -uint8_t x_141; uint8_t x_142; lean_object* x_143; -x_141 = 1; -x_142 = 0; -x_143 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_141, x_142, x_142); -return x_143; +uint8_t x_137; uint8_t x_138; lean_object* x_139; +x_137 = 1; +x_138 = 0; +x_139 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_137, x_138, x_138); +return x_139; } case 2: { -uint8_t x_144; uint8_t x_145; lean_object* x_146; -x_144 = 1; -x_145 = 0; -x_146 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_144, x_145, x_144); -return x_146; +uint8_t x_140; uint8_t x_141; lean_object* x_142; +x_140 = 1; +x_141 = 0; +x_142 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_140, x_141, x_140); +return x_142; } case 3: { -uint8_t x_147; uint8_t x_148; lean_object* x_149; -x_147 = 1; -x_148 = 0; -x_149 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_147, x_147, x_148); -return x_149; +uint8_t x_143; uint8_t x_144; lean_object* x_145; +x_143 = 1; +x_144 = 0; +x_145 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_143, x_143, x_144); +return x_145; } default: { -uint8_t x_150; lean_object* x_151; -x_150 = 1; -x_151 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_150, x_150, x_150); -return x_151; +uint8_t x_146; lean_object* x_147; +x_146 = 1; +x_147 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_146, x_146, x_146); +return x_147; } } } else { -lean_object* x_152; +lean_object* x_148; lean_dec(x_2); -x_152 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; -return x_152; +x_148 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; +return x_148; } } case 27: { -uint8_t x_153; -x_153 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_149; +x_149 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -switch (x_153) { +switch (x_149) { case 0: { -lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; uint8_t x_158; uint8_t x_159; uint8_t x_160; lean_object* x_161; -x_154 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; -x_155 = lean_int_div(x_2, x_154); -x_156 = lean_int_emod(x_155, x_154); -lean_dec(x_155); -x_157 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_158 = lean_int_dec_eq(x_156, x_157); -lean_dec(x_156); -x_159 = l_instDecidableNot___rarg(x_158); -x_160 = 0; -x_161 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_159, x_160, x_160); -return x_161; +lean_object* x_150; lean_object* x_151; lean_object* x_152; lean_object* x_153; uint8_t x_154; uint8_t x_155; uint8_t x_156; lean_object* x_157; +x_150 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; +x_151 = lean_int_div(x_2, x_150); +x_152 = lean_int_emod(x_151, x_150); +lean_dec(x_151); +x_153 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_154 = lean_int_dec_eq(x_152, x_153); +lean_dec(x_152); +x_155 = l_instDecidableNot___rarg(x_154); +x_156 = 0; +x_157 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_155, x_156, x_156); +return x_157; } case 1: { -uint8_t x_162; uint8_t x_163; lean_object* x_164; -x_162 = 1; -x_163 = 0; -x_164 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_162, x_163, x_163); -return x_164; +uint8_t x_158; uint8_t x_159; lean_object* x_160; +x_158 = 1; +x_159 = 0; +x_160 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_158, x_159, x_159); +return x_160; } case 2: { -lean_object* x_165; lean_object* x_166; lean_object* x_167; uint8_t x_168; uint8_t x_169; uint8_t x_170; lean_object* x_171; -x_165 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; -x_166 = lean_int_emod(x_2, x_165); -x_167 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_168 = lean_int_dec_eq(x_166, x_167); -lean_dec(x_166); -x_169 = l_instDecidableNot___rarg(x_168); -x_170 = 1; -x_171 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_170, x_169, x_170); -return x_171; +lean_object* x_161; lean_object* x_162; lean_object* x_163; uint8_t x_164; uint8_t x_165; uint8_t x_166; lean_object* x_167; +x_161 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; +x_162 = lean_int_emod(x_2, x_161); +x_163 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_164 = lean_int_dec_eq(x_162, x_163); +lean_dec(x_162); +x_165 = l_instDecidableNot___rarg(x_164); +x_166 = 1; +x_167 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_166, x_165, x_166); +return x_167; } case 3: { -lean_object* x_172; lean_object* x_173; lean_object* x_174; uint8_t x_175; uint8_t x_176; uint8_t x_177; uint8_t x_178; lean_object* x_179; -x_172 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; -x_173 = lean_int_emod(x_2, x_172); -x_174 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_175 = lean_int_dec_eq(x_173, x_174); -lean_dec(x_173); -x_176 = l_instDecidableNot___rarg(x_175); -x_177 = 1; -x_178 = 0; -x_179 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_177, x_176, x_178); -return x_179; +lean_object* x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; uint8_t x_172; uint8_t x_173; uint8_t x_174; lean_object* x_175; +x_168 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; +x_169 = lean_int_emod(x_2, x_168); +x_170 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_171 = lean_int_dec_eq(x_169, x_170); +lean_dec(x_169); +x_172 = l_instDecidableNot___rarg(x_171); +x_173 = 1; +x_174 = 0; +x_175 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_173, x_172, x_174); +return x_175; } default: { -uint8_t x_180; lean_object* x_181; -x_180 = 1; -x_181 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_180, x_180, x_180); -return x_181; +uint8_t x_176; lean_object* x_177; +x_176 = 1; +x_177 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_176, x_176, x_176); +return x_177; } } } case 28: { -uint8_t x_182; -x_182 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_178; +x_178 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -switch (x_182) { +switch (x_178) { case 0: { -uint8_t x_183; uint8_t x_184; lean_object* x_185; -x_183 = 1; -x_184 = 0; -x_185 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_183, x_184, x_184); -return x_185; +uint8_t x_179; uint8_t x_180; lean_object* x_181; +x_179 = 1; +x_180 = 0; +x_181 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_179, x_180, x_180); +return x_181; } case 1: { -lean_object* x_186; uint8_t x_187; -x_186 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_187 = lean_int_dec_eq(x_2, x_186); -if (x_187 == 0) -{ -uint8_t x_188; uint8_t x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; -x_188 = 1; -x_189 = 0; -x_190 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_188, x_189, x_188); -x_191 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_192 = lean_string_append(x_191, x_190); -lean_dec(x_190); -x_193 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; -x_194 = lean_string_append(x_192, x_193); -return x_194; +lean_object* x_182; uint8_t x_183; +x_182 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_183 = lean_int_dec_eq(x_2, x_182); +if (x_183 == 0) +{ +uint8_t x_184; uint8_t x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; +x_184 = 1; +x_185 = 0; +x_186 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_184, x_185, x_184); +x_187 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_188 = lean_string_append(x_187, x_186); +lean_dec(x_186); +x_189 = l___private_Std_Time_Format_Basic_0__Std_Time_parseMod___rarg___closed__1; +x_190 = lean_string_append(x_188, x_189); +return x_190; } else { -lean_object* x_195; +lean_object* x_191; lean_dec(x_2); -x_195 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -return x_195; +x_191 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +return x_191; } } default: { -lean_object* x_196; uint8_t x_197; -x_196 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_197 = lean_int_dec_eq(x_2, x_196); -if (x_197 == 0) +lean_object* x_192; uint8_t x_193; +x_192 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_193 = lean_int_dec_eq(x_2, x_192); +if (x_193 == 0) { -lean_object* x_198; lean_object* x_199; uint8_t x_200; uint8_t x_201; uint8_t x_202; lean_object* x_203; -x_198 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; -x_199 = lean_int_emod(x_2, x_198); -x_200 = lean_int_dec_eq(x_199, x_196); -lean_dec(x_199); -x_201 = l_instDecidableNot___rarg(x_200); -x_202 = 1; -x_203 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_202, x_201, x_202); -return x_203; +lean_object* x_194; lean_object* x_195; uint8_t x_196; uint8_t x_197; uint8_t x_198; lean_object* x_199; +x_194 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__6; +x_195 = lean_int_emod(x_2, x_194); +x_196 = lean_int_dec_eq(x_195, x_192); +lean_dec(x_195); +x_197 = l_instDecidableNot___rarg(x_196); +x_198 = 1; +x_199 = l___private_Std_Time_Format_Basic_0__Std_Time_toIsoString(x_2, x_198, x_197, x_198); +return x_199; } else { -lean_object* x_204; +lean_object* x_200; lean_dec(x_2); -x_204 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; -return x_204; +x_200 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; +return x_200; } } } } default: { -lean_object* x_205; uint8_t x_206; lean_object* x_207; -x_205 = lean_ctor_get(x_1, 0); -lean_inc(x_205); +lean_object* x_201; uint8_t x_202; lean_object* x_203; +x_201 = lean_ctor_get(x_1, 0); +lean_inc(x_201); lean_dec(x_1); -x_206 = 0; -x_207 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_205, x_2, x_206); -lean_dec(x_205); -return x_207; +x_202 = 0; +x_203 = l___private_Std_Time_Format_Basic_0__Std_Time_pad(x_201, x_2, x_202); +lean_dec(x_201); +return x_203; } } } @@ -78445,501 +78407,445 @@ lean_closure_set(x_192, 0, x_191); x_193 = lean_unsigned_to_nat(0u); x_194 = lean_unsigned_to_nat(60u); x_195 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_193, x_194, x_192, x_2); -if (lean_obj_tag(x_195) == 0) -{ -uint8_t x_196; -x_196 = !lean_is_exclusive(x_195); -if (x_196 == 0) -{ -lean_object* x_197; uint8_t x_198; lean_object* x_199; lean_object* x_200; -x_197 = lean_ctor_get(x_195, 1); -x_198 = 1; -x_199 = lean_box(x_198); -x_200 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_200, 0, x_199); -lean_ctor_set(x_200, 1, x_197); -lean_ctor_set(x_195, 1, x_200); -return x_195; -} -else -{ -lean_object* x_201; lean_object* x_202; uint8_t x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; -x_201 = lean_ctor_get(x_195, 0); -x_202 = lean_ctor_get(x_195, 1); -lean_inc(x_202); -lean_inc(x_201); -lean_dec(x_195); -x_203 = 1; -x_204 = lean_box(x_203); -x_205 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_205, 0, x_204); -lean_ctor_set(x_205, 1, x_202); -x_206 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_206, 0, x_201); -lean_ctor_set(x_206, 1, x_205); -return x_206; -} -} -else -{ -uint8_t x_207; -x_207 = !lean_is_exclusive(x_195); -if (x_207 == 0) -{ return x_195; } -else -{ -lean_object* x_208; lean_object* x_209; lean_object* x_210; -x_208 = lean_ctor_get(x_195, 0); -x_209 = lean_ctor_get(x_195, 1); -lean_inc(x_209); -lean_inc(x_208); -lean_dec(x_195); -x_210 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_210, 0, x_208); -lean_ctor_set(x_210, 1, x_209); -return x_210; -} -} -} case 19: { -lean_object* x_211; -x_211 = lean_ctor_get(x_1, 0); -lean_inc(x_211); +lean_object* x_196; +x_196 = lean_ctor_get(x_1, 0); +lean_inc(x_196); lean_dec(x_1); -if (lean_obj_tag(x_211) == 0) +if (lean_obj_tag(x_196) == 0) { -lean_object* x_212; lean_object* x_213; lean_object* x_214; lean_object* x_215; -x_212 = lean_unsigned_to_nat(0u); -x_213 = lean_unsigned_to_nat(999999999u); -x_214 = l___private_Std_Time_Format_Basic_0__Std_Time_parseWith___closed__4; -x_215 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_212, x_213, x_214, x_2); -return x_215; +lean_object* x_197; lean_object* x_198; lean_object* x_199; lean_object* x_200; +x_197 = lean_unsigned_to_nat(0u); +x_198 = lean_unsigned_to_nat(999999999u); +x_199 = l___private_Std_Time_Format_Basic_0__Std_Time_parseWith___closed__4; +x_200 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_197, x_198, x_199, x_2); +return x_200; } else { -lean_object* x_216; lean_object* x_217; lean_object* x_218; lean_object* x_219; lean_object* x_220; lean_object* x_221; -x_216 = lean_ctor_get(x_211, 0); -lean_inc(x_216); -lean_dec(x_211); -x_217 = lean_unsigned_to_nat(9u); -x_218 = lean_alloc_closure((void*)(l___private_Std_Time_Format_Basic_0__Std_Time_parseFractionNum___boxed), 3, 2); -lean_closure_set(x_218, 0, x_216); -lean_closure_set(x_218, 1, x_217); -x_219 = lean_unsigned_to_nat(0u); -x_220 = lean_unsigned_to_nat(999999999u); -x_221 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_219, x_220, x_218, x_2); -return x_221; +lean_object* x_201; lean_object* x_202; lean_object* x_203; lean_object* x_204; lean_object* x_205; lean_object* x_206; +x_201 = lean_ctor_get(x_196, 0); +lean_inc(x_201); +lean_dec(x_196); +x_202 = lean_unsigned_to_nat(9u); +x_203 = lean_alloc_closure((void*)(l___private_Std_Time_Format_Basic_0__Std_Time_parseFractionNum___boxed), 3, 2); +lean_closure_set(x_203, 0, x_201); +lean_closure_set(x_203, 1, x_202); +x_204 = lean_unsigned_to_nat(0u); +x_205 = lean_unsigned_to_nat(999999999u); +x_206 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_204, x_205, x_203, x_2); +return x_206; } } case 21: { -lean_object* x_222; lean_object* x_223; lean_object* x_224; lean_object* x_225; lean_object* x_226; -x_222 = lean_ctor_get(x_1, 0); -lean_inc(x_222); +lean_object* x_207; lean_object* x_208; lean_object* x_209; lean_object* x_210; lean_object* x_211; +x_207 = lean_ctor_get(x_1, 0); +lean_inc(x_207); lean_dec(x_1); -x_223 = lean_alloc_closure((void*)(l___private_Std_Time_Format_Basic_0__Std_Time_parseAtLeastNum___boxed), 2, 1); -lean_closure_set(x_223, 0, x_222); -x_224 = lean_unsigned_to_nat(0u); -x_225 = lean_unsigned_to_nat(999999999u); -x_226 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_224, x_225, x_223, x_2); -return x_226; +x_208 = lean_alloc_closure((void*)(l___private_Std_Time_Format_Basic_0__Std_Time_parseAtLeastNum___boxed), 2, 1); +lean_closure_set(x_208, 0, x_207); +x_209 = lean_unsigned_to_nat(0u); +x_210 = lean_unsigned_to_nat(999999999u); +x_211 = l___private_Std_Time_Format_Basic_0__Std_Time_parseNatToBounded(x_209, x_210, x_208, x_2); +return x_211; } case 23: { -lean_object* x_227; -x_227 = l___private_Std_Time_Format_Basic_0__Std_Time_parseIdentifier(x_2); -return x_227; +lean_object* x_212; +x_212 = l___private_Std_Time_Format_Basic_0__Std_Time_parseIdentifier(x_2); +return x_212; } case 24: { -lean_object* x_228; +lean_object* x_213; lean_dec(x_1); -x_228 = l___private_Std_Time_Format_Basic_0__Std_Time_parseIdentifier(x_2); -return x_228; +x_213 = l___private_Std_Time_Format_Basic_0__Std_Time_parseIdentifier(x_2); +return x_213; } case 25: { -uint8_t x_229; -x_229 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_214; +x_214 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -if (x_229 == 0) +if (x_214 == 0) { -lean_object* x_230; lean_object* x_231; -x_230 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_231 = l_Std_Internal_Parsec_String_pstring(x_230, x_2); -if (lean_obj_tag(x_231) == 0) +lean_object* x_215; lean_object* x_216; +x_215 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_216 = l_Std_Internal_Parsec_String_pstring(x_215, x_2); +if (lean_obj_tag(x_216) == 0) { -lean_object* x_232; uint8_t x_233; uint8_t x_234; lean_object* x_235; -x_232 = lean_ctor_get(x_231, 0); -lean_inc(x_232); -lean_dec(x_231); -x_233 = 1; -x_234 = 0; -x_235 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_233, x_233, x_234, x_232); -return x_235; +lean_object* x_217; uint8_t x_218; uint8_t x_219; lean_object* x_220; +x_217 = lean_ctor_get(x_216, 0); +lean_inc(x_217); +lean_dec(x_216); +x_218 = 1; +x_219 = 0; +x_220 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_218, x_218, x_219, x_217); +return x_220; } else { -uint8_t x_236; -x_236 = !lean_is_exclusive(x_231); -if (x_236 == 0) +uint8_t x_221; +x_221 = !lean_is_exclusive(x_216); +if (x_221 == 0) { -return x_231; +return x_216; } else { -lean_object* x_237; lean_object* x_238; lean_object* x_239; -x_237 = lean_ctor_get(x_231, 0); -x_238 = lean_ctor_get(x_231, 1); -lean_inc(x_238); -lean_inc(x_237); -lean_dec(x_231); -x_239 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_239, 0, x_237); -lean_ctor_set(x_239, 1, x_238); -return x_239; +lean_object* x_222; lean_object* x_223; lean_object* x_224; +x_222 = lean_ctor_get(x_216, 0); +x_223 = lean_ctor_get(x_216, 1); +lean_inc(x_223); +lean_inc(x_222); +lean_dec(x_216); +x_224 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_224, 0, x_222); +lean_ctor_set(x_224, 1, x_223); +return x_224; } } } else { -lean_object* x_240; lean_object* x_241; -x_240 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_241 = l_Std_Internal_Parsec_String_pstring(x_240, x_2); -if (lean_obj_tag(x_241) == 0) +lean_object* x_225; lean_object* x_226; +x_225 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_226 = l_Std_Internal_Parsec_String_pstring(x_225, x_2); +if (lean_obj_tag(x_226) == 0) { -lean_object* x_242; uint8_t x_243; uint8_t x_244; uint8_t x_245; lean_object* x_246; -x_242 = lean_ctor_get(x_241, 0); -lean_inc(x_242); -lean_dec(x_241); -x_243 = 0; -x_244 = 2; -x_245 = 0; -x_246 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_243, x_244, x_245, x_242); -return x_246; +lean_object* x_227; uint8_t x_228; uint8_t x_229; uint8_t x_230; lean_object* x_231; +x_227 = lean_ctor_get(x_226, 0); +lean_inc(x_227); +lean_dec(x_226); +x_228 = 0; +x_229 = 2; +x_230 = 0; +x_231 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_228, x_229, x_230, x_227); +return x_231; } else { -uint8_t x_247; -x_247 = !lean_is_exclusive(x_241); -if (x_247 == 0) +uint8_t x_232; +x_232 = !lean_is_exclusive(x_226); +if (x_232 == 0) { -return x_241; +return x_226; } else { -lean_object* x_248; lean_object* x_249; lean_object* x_250; -x_248 = lean_ctor_get(x_241, 0); -x_249 = lean_ctor_get(x_241, 1); -lean_inc(x_249); -lean_inc(x_248); -lean_dec(x_241); -x_250 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_250, 0, x_248); -lean_ctor_set(x_250, 1, x_249); -return x_250; +lean_object* x_233; lean_object* x_234; lean_object* x_235; +x_233 = lean_ctor_get(x_226, 0); +x_234 = lean_ctor_get(x_226, 1); +lean_inc(x_234); +lean_inc(x_233); +lean_dec(x_226); +x_235 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_235, 0, x_233); +lean_ctor_set(x_235, 1, x_234); +return x_235; } } } } case 26: { -uint8_t x_251; lean_object* x_252; lean_object* x_253; -x_251 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_236; lean_object* x_237; lean_object* x_238; +x_236 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -switch (x_251) { +switch (x_236) { case 0: { -uint8_t x_271; uint8_t x_272; lean_object* x_273; -x_271 = 1; -x_272 = 0; +uint8_t x_256; uint8_t x_257; lean_object* x_258; +x_256 = 1; +x_257 = 0; lean_inc(x_2); -x_273 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_271, x_271, x_272, x_2); -if (lean_obj_tag(x_273) == 0) +x_258 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_256, x_256, x_257, x_2); +if (lean_obj_tag(x_258) == 0) { -uint8_t x_274; +uint8_t x_259; lean_dec(x_2); -x_274 = !lean_is_exclusive(x_273); -if (x_274 == 0) +x_259 = !lean_is_exclusive(x_258); +if (x_259 == 0) { -return x_273; +return x_258; } else { -lean_object* x_275; lean_object* x_276; lean_object* x_277; -x_275 = lean_ctor_get(x_273, 0); -x_276 = lean_ctor_get(x_273, 1); -lean_inc(x_276); -lean_inc(x_275); -lean_dec(x_273); -x_277 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_277, 0, x_275); -lean_ctor_set(x_277, 1, x_276); -return x_277; +lean_object* x_260; lean_object* x_261; lean_object* x_262; +x_260 = lean_ctor_get(x_258, 0); +x_261 = lean_ctor_get(x_258, 1); +lean_inc(x_261); +lean_inc(x_260); +lean_dec(x_258); +x_262 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_262, 0, x_260); +lean_ctor_set(x_262, 1, x_261); +return x_262; } } else { -lean_object* x_278; lean_object* x_279; -x_278 = lean_ctor_get(x_273, 0); -lean_inc(x_278); -x_279 = lean_ctor_get(x_273, 1); -lean_inc(x_279); -lean_dec(x_273); -x_252 = x_278; -x_253 = x_279; -goto block_270; +lean_object* x_263; lean_object* x_264; +x_263 = lean_ctor_get(x_258, 0); +lean_inc(x_263); +x_264 = lean_ctor_get(x_258, 1); +lean_inc(x_264); +lean_dec(x_258); +x_237 = x_263; +x_238 = x_264; +goto block_255; } } case 1: { -uint8_t x_280; uint8_t x_281; uint8_t x_282; lean_object* x_283; -x_280 = 0; -x_281 = 1; -x_282 = 0; +uint8_t x_265; uint8_t x_266; uint8_t x_267; lean_object* x_268; +x_265 = 0; +x_266 = 1; +x_267 = 0; lean_inc(x_2); -x_283 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_280, x_281, x_282, x_2); -if (lean_obj_tag(x_283) == 0) +x_268 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_265, x_266, x_267, x_2); +if (lean_obj_tag(x_268) == 0) { -uint8_t x_284; +uint8_t x_269; lean_dec(x_2); -x_284 = !lean_is_exclusive(x_283); -if (x_284 == 0) +x_269 = !lean_is_exclusive(x_268); +if (x_269 == 0) { -return x_283; +return x_268; } else { -lean_object* x_285; lean_object* x_286; lean_object* x_287; -x_285 = lean_ctor_get(x_283, 0); -x_286 = lean_ctor_get(x_283, 1); -lean_inc(x_286); -lean_inc(x_285); -lean_dec(x_283); -x_287 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_287, 0, x_285); -lean_ctor_set(x_287, 1, x_286); -return x_287; +lean_object* x_270; lean_object* x_271; lean_object* x_272; +x_270 = lean_ctor_get(x_268, 0); +x_271 = lean_ctor_get(x_268, 1); +lean_inc(x_271); +lean_inc(x_270); +lean_dec(x_268); +x_272 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_272, 0, x_270); +lean_ctor_set(x_272, 1, x_271); +return x_272; } } else { -lean_object* x_288; lean_object* x_289; -x_288 = lean_ctor_get(x_283, 0); -lean_inc(x_288); -x_289 = lean_ctor_get(x_283, 1); -lean_inc(x_289); -lean_dec(x_283); -x_252 = x_288; -x_253 = x_289; -goto block_270; +lean_object* x_273; lean_object* x_274; +x_273 = lean_ctor_get(x_268, 0); +lean_inc(x_273); +x_274 = lean_ctor_get(x_268, 1); +lean_inc(x_274); +lean_dec(x_268); +x_237 = x_273; +x_238 = x_274; +goto block_255; } } case 2: { -uint8_t x_290; uint8_t x_291; uint8_t x_292; lean_object* x_293; -x_290 = 0; -x_291 = 1; -x_292 = 1; +uint8_t x_275; uint8_t x_276; uint8_t x_277; lean_object* x_278; +x_275 = 0; +x_276 = 1; +x_277 = 1; lean_inc(x_2); -x_293 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_290, x_291, x_292, x_2); -if (lean_obj_tag(x_293) == 0) +x_278 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_275, x_276, x_277, x_2); +if (lean_obj_tag(x_278) == 0) { -uint8_t x_294; +uint8_t x_279; lean_dec(x_2); -x_294 = !lean_is_exclusive(x_293); -if (x_294 == 0) +x_279 = !lean_is_exclusive(x_278); +if (x_279 == 0) { -return x_293; +return x_278; } else { -lean_object* x_295; lean_object* x_296; lean_object* x_297; -x_295 = lean_ctor_get(x_293, 0); -x_296 = lean_ctor_get(x_293, 1); -lean_inc(x_296); -lean_inc(x_295); -lean_dec(x_293); -x_297 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_297, 0, x_295); -lean_ctor_set(x_297, 1, x_296); -return x_297; +lean_object* x_280; lean_object* x_281; lean_object* x_282; +x_280 = lean_ctor_get(x_278, 0); +x_281 = lean_ctor_get(x_278, 1); +lean_inc(x_281); +lean_inc(x_280); +lean_dec(x_278); +x_282 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_282, 0, x_280); +lean_ctor_set(x_282, 1, x_281); +return x_282; } } else { -lean_object* x_298; lean_object* x_299; -x_298 = lean_ctor_get(x_293, 0); -lean_inc(x_298); -x_299 = lean_ctor_get(x_293, 1); -lean_inc(x_299); -lean_dec(x_293); -x_252 = x_298; -x_253 = x_299; -goto block_270; +lean_object* x_283; lean_object* x_284; +x_283 = lean_ctor_get(x_278, 0); +lean_inc(x_283); +x_284 = lean_ctor_get(x_278, 1); +lean_inc(x_284); +lean_dec(x_278); +x_237 = x_283; +x_238 = x_284; +goto block_255; } } case 3: { -uint8_t x_300; uint8_t x_301; lean_object* x_302; -x_300 = 0; -x_301 = 0; +uint8_t x_285; uint8_t x_286; lean_object* x_287; +x_285 = 0; +x_286 = 0; lean_inc(x_2); -x_302 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_300, x_300, x_301, x_2); -if (lean_obj_tag(x_302) == 0) +x_287 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_285, x_285, x_286, x_2); +if (lean_obj_tag(x_287) == 0) { -uint8_t x_303; +uint8_t x_288; lean_dec(x_2); -x_303 = !lean_is_exclusive(x_302); -if (x_303 == 0) +x_288 = !lean_is_exclusive(x_287); +if (x_288 == 0) { -return x_302; +return x_287; } else { -lean_object* x_304; lean_object* x_305; lean_object* x_306; -x_304 = lean_ctor_get(x_302, 0); -x_305 = lean_ctor_get(x_302, 1); -lean_inc(x_305); -lean_inc(x_304); -lean_dec(x_302); -x_306 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_306, 0, x_304); -lean_ctor_set(x_306, 1, x_305); -return x_306; +lean_object* x_289; lean_object* x_290; lean_object* x_291; +x_289 = lean_ctor_get(x_287, 0); +x_290 = lean_ctor_get(x_287, 1); +lean_inc(x_290); +lean_inc(x_289); +lean_dec(x_287); +x_291 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_291, 0, x_289); +lean_ctor_set(x_291, 1, x_290); +return x_291; } } else { -lean_object* x_307; lean_object* x_308; -x_307 = lean_ctor_get(x_302, 0); -lean_inc(x_307); -x_308 = lean_ctor_get(x_302, 1); -lean_inc(x_308); -lean_dec(x_302); -x_252 = x_307; -x_253 = x_308; -goto block_270; +lean_object* x_292; lean_object* x_293; +x_292 = lean_ctor_get(x_287, 0); +lean_inc(x_292); +x_293 = lean_ctor_get(x_287, 1); +lean_inc(x_293); +lean_dec(x_287); +x_237 = x_292; +x_238 = x_293; +goto block_255; } } default: { -uint8_t x_309; uint8_t x_310; lean_object* x_311; -x_309 = 0; -x_310 = 1; +uint8_t x_294; uint8_t x_295; lean_object* x_296; +x_294 = 0; +x_295 = 1; lean_inc(x_2); -x_311 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_309, x_309, x_310, x_2); -if (lean_obj_tag(x_311) == 0) +x_296 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_294, x_294, x_295, x_2); +if (lean_obj_tag(x_296) == 0) { -uint8_t x_312; +uint8_t x_297; lean_dec(x_2); -x_312 = !lean_is_exclusive(x_311); -if (x_312 == 0) +x_297 = !lean_is_exclusive(x_296); +if (x_297 == 0) { -return x_311; +return x_296; } else { -lean_object* x_313; lean_object* x_314; lean_object* x_315; -x_313 = lean_ctor_get(x_311, 0); -x_314 = lean_ctor_get(x_311, 1); -lean_inc(x_314); -lean_inc(x_313); -lean_dec(x_311); -x_315 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_315, 0, x_313); -lean_ctor_set(x_315, 1, x_314); -return x_315; +lean_object* x_298; lean_object* x_299; lean_object* x_300; +x_298 = lean_ctor_get(x_296, 0); +x_299 = lean_ctor_get(x_296, 1); +lean_inc(x_299); +lean_inc(x_298); +lean_dec(x_296); +x_300 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_300, 0, x_298); +lean_ctor_set(x_300, 1, x_299); +return x_300; } } else { -lean_object* x_316; lean_object* x_317; -x_316 = lean_ctor_get(x_311, 0); -lean_inc(x_316); -x_317 = lean_ctor_get(x_311, 1); -lean_inc(x_317); -lean_dec(x_311); -x_252 = x_316; -x_253 = x_317; -goto block_270; +lean_object* x_301; lean_object* x_302; +x_301 = lean_ctor_get(x_296, 0); +lean_inc(x_301); +x_302 = lean_ctor_get(x_296, 1); +lean_inc(x_302); +lean_dec(x_296); +x_237 = x_301; +x_238 = x_302; +goto block_255; } } } -block_270: +block_255: { -lean_object* x_254; lean_object* x_255; uint8_t x_256; -x_254 = lean_ctor_get(x_2, 1); -lean_inc(x_254); +lean_object* x_239; lean_object* x_240; uint8_t x_241; +x_239 = lean_ctor_get(x_2, 1); +lean_inc(x_239); lean_dec(x_2); -x_255 = lean_ctor_get(x_252, 1); -lean_inc(x_255); -x_256 = lean_nat_dec_eq(x_254, x_255); -lean_dec(x_255); -lean_dec(x_254); -if (x_256 == 0) +x_240 = lean_ctor_get(x_237, 1); +lean_inc(x_240); +x_241 = lean_nat_dec_eq(x_239, x_240); +lean_dec(x_240); +lean_dec(x_239); +if (x_241 == 0) { -lean_object* x_257; -x_257 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_257, 0, x_252); -lean_ctor_set(x_257, 1, x_253); -return x_257; +lean_object* x_242; +x_242 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_242, 0, x_237); +lean_ctor_set(x_242, 1, x_238); +return x_242; } else { -lean_object* x_258; lean_object* x_259; -lean_dec(x_253); -x_258 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; -x_259 = l_Std_Internal_Parsec_String_pstring(x_258, x_252); -if (lean_obj_tag(x_259) == 0) +lean_object* x_243; lean_object* x_244; +lean_dec(x_238); +x_243 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; +x_244 = l_Std_Internal_Parsec_String_pstring(x_243, x_237); +if (lean_obj_tag(x_244) == 0) { -uint8_t x_260; -x_260 = !lean_is_exclusive(x_259); -if (x_260 == 0) +uint8_t x_245; +x_245 = !lean_is_exclusive(x_244); +if (x_245 == 0) { -lean_object* x_261; lean_object* x_262; -x_261 = lean_ctor_get(x_259, 1); -lean_dec(x_261); -x_262 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -lean_ctor_set(x_259, 1, x_262); -return x_259; +lean_object* x_246; lean_object* x_247; +x_246 = lean_ctor_get(x_244, 1); +lean_dec(x_246); +x_247 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +lean_ctor_set(x_244, 1, x_247); +return x_244; } else { -lean_object* x_263; lean_object* x_264; lean_object* x_265; -x_263 = lean_ctor_get(x_259, 0); -lean_inc(x_263); -lean_dec(x_259); -x_264 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; -x_265 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_265, 0, x_263); -lean_ctor_set(x_265, 1, x_264); -return x_265; +lean_object* x_248; lean_object* x_249; lean_object* x_250; +x_248 = lean_ctor_get(x_244, 0); +lean_inc(x_248); +lean_dec(x_244); +x_249 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; +x_250 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_250, 0, x_248); +lean_ctor_set(x_250, 1, x_249); +return x_250; } } else { -uint8_t x_266; -x_266 = !lean_is_exclusive(x_259); -if (x_266 == 0) +uint8_t x_251; +x_251 = !lean_is_exclusive(x_244); +if (x_251 == 0) { -return x_259; +return x_244; } else { -lean_object* x_267; lean_object* x_268; lean_object* x_269; -x_267 = lean_ctor_get(x_259, 0); -x_268 = lean_ctor_get(x_259, 1); -lean_inc(x_268); -lean_inc(x_267); -lean_dec(x_259); -x_269 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_269, 0, x_267); -lean_ctor_set(x_269, 1, x_268); -return x_269; +lean_object* x_252; lean_object* x_253; lean_object* x_254; +x_252 = lean_ctor_get(x_244, 0); +x_253 = lean_ctor_get(x_244, 1); +lean_inc(x_253); +lean_inc(x_252); +lean_dec(x_244); +x_254 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_254, 0, x_252); +lean_ctor_set(x_254, 1, x_253); +return x_254; } } } @@ -78947,300 +78853,300 @@ return x_269; } case 27: { -uint8_t x_318; -x_318 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_303; +x_303 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -switch (x_318) { +switch (x_303) { case 0: { -uint8_t x_319; uint8_t x_320; uint8_t x_321; lean_object* x_322; -x_319 = 2; -x_320 = 1; -x_321 = 0; -x_322 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_319, x_320, x_321, x_2); -return x_322; +uint8_t x_304; uint8_t x_305; uint8_t x_306; lean_object* x_307; +x_304 = 2; +x_305 = 1; +x_306 = 0; +x_307 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_304, x_305, x_306, x_2); +return x_307; } case 1: { -uint8_t x_323; uint8_t x_324; uint8_t x_325; lean_object* x_326; -x_323 = 0; -x_324 = 1; -x_325 = 0; -x_326 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_323, x_324, x_325, x_2); -return x_326; +uint8_t x_308; uint8_t x_309; uint8_t x_310; lean_object* x_311; +x_308 = 0; +x_309 = 1; +x_310 = 0; +x_311 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_308, x_309, x_310, x_2); +return x_311; } case 2: { -uint8_t x_327; uint8_t x_328; uint8_t x_329; lean_object* x_330; -x_327 = 0; -x_328 = 2; -x_329 = 1; -x_330 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_327, x_328, x_329, x_2); -return x_330; +uint8_t x_312; uint8_t x_313; uint8_t x_314; lean_object* x_315; +x_312 = 0; +x_313 = 2; +x_314 = 1; +x_315 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_312, x_313, x_314, x_2); +return x_315; } case 3: { -uint8_t x_331; uint8_t x_332; uint8_t x_333; lean_object* x_334; -x_331 = 0; -x_332 = 2; -x_333 = 0; -x_334 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_331, x_332, x_333, x_2); -return x_334; +uint8_t x_316; uint8_t x_317; uint8_t x_318; lean_object* x_319; +x_316 = 0; +x_317 = 2; +x_318 = 0; +x_319 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_316, x_317, x_318, x_2); +return x_319; } default: { -uint8_t x_335; uint8_t x_336; lean_object* x_337; -x_335 = 0; -x_336 = 1; -x_337 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_335, x_335, x_336, x_2); -return x_337; +uint8_t x_320; uint8_t x_321; lean_object* x_322; +x_320 = 0; +x_321 = 1; +x_322 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_320, x_320, x_321, x_2); +return x_322; } } } case 28: { -uint8_t x_338; -x_338 = lean_ctor_get_uint8(x_1, 0); +uint8_t x_323; +x_323 = lean_ctor_get_uint8(x_1, 0); lean_dec(x_1); -switch (x_338) { +switch (x_323) { case 0: { -uint8_t x_339; uint8_t x_340; uint8_t x_341; lean_object* x_342; -x_339 = 0; -x_340 = 1; -x_341 = 0; -x_342 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_339, x_340, x_341, x_2); -return x_342; +uint8_t x_324; uint8_t x_325; uint8_t x_326; lean_object* x_327; +x_324 = 0; +x_325 = 1; +x_326 = 0; +x_327 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_324, x_325, x_326, x_2); +return x_327; } case 1: { -lean_object* x_343; lean_object* x_344; -x_343 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; -x_344 = l_Std_Internal_Parsec_String_pstring(x_343, x_2); -if (lean_obj_tag(x_344) == 0) +lean_object* x_328; lean_object* x_329; +x_328 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__4; +x_329 = l_Std_Internal_Parsec_String_pstring(x_328, x_2); +if (lean_obj_tag(x_329) == 0) { -lean_object* x_345; uint8_t x_346; uint8_t x_347; uint8_t x_348; lean_object* x_349; -x_345 = lean_ctor_get(x_344, 0); -lean_inc(x_345); -lean_dec(x_344); -x_346 = 0; -x_347 = 1; -x_348 = 1; -lean_inc(x_345); -x_349 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_346, x_347, x_348, x_345); -if (lean_obj_tag(x_349) == 0) +lean_object* x_330; uint8_t x_331; uint8_t x_332; uint8_t x_333; lean_object* x_334; +x_330 = lean_ctor_get(x_329, 0); +lean_inc(x_330); +lean_dec(x_329); +x_331 = 0; +x_332 = 1; +x_333 = 1; +lean_inc(x_330); +x_334 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_331, x_332, x_333, x_330); +if (lean_obj_tag(x_334) == 0) { -uint8_t x_350; -lean_dec(x_345); -x_350 = !lean_is_exclusive(x_349); -if (x_350 == 0) +uint8_t x_335; +lean_dec(x_330); +x_335 = !lean_is_exclusive(x_334); +if (x_335 == 0) { -return x_349; +return x_334; } else { -lean_object* x_351; lean_object* x_352; lean_object* x_353; -x_351 = lean_ctor_get(x_349, 0); -x_352 = lean_ctor_get(x_349, 1); -lean_inc(x_352); -lean_inc(x_351); -lean_dec(x_349); -x_353 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_353, 0, x_351); -lean_ctor_set(x_353, 1, x_352); -return x_353; +lean_object* x_336; lean_object* x_337; lean_object* x_338; +x_336 = lean_ctor_get(x_334, 0); +x_337 = lean_ctor_get(x_334, 1); +lean_inc(x_337); +lean_inc(x_336); +lean_dec(x_334); +x_338 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_338, 0, x_336); +lean_ctor_set(x_338, 1, x_337); +return x_338; } } else { -uint8_t x_354; -x_354 = !lean_is_exclusive(x_349); -if (x_354 == 0) +uint8_t x_339; +x_339 = !lean_is_exclusive(x_334); +if (x_339 == 0) { -lean_object* x_355; lean_object* x_356; lean_object* x_357; lean_object* x_358; uint8_t x_359; -x_355 = lean_ctor_get(x_349, 0); -x_356 = lean_ctor_get(x_349, 1); -x_357 = lean_ctor_get(x_345, 1); -lean_inc(x_357); -lean_dec(x_345); -x_358 = lean_ctor_get(x_355, 1); -lean_inc(x_358); -x_359 = lean_nat_dec_eq(x_357, x_358); -lean_dec(x_358); -lean_dec(x_357); -if (x_359 == 0) +lean_object* x_340; lean_object* x_341; lean_object* x_342; lean_object* x_343; uint8_t x_344; +x_340 = lean_ctor_get(x_334, 0); +x_341 = lean_ctor_get(x_334, 1); +x_342 = lean_ctor_get(x_330, 1); +lean_inc(x_342); +lean_dec(x_330); +x_343 = lean_ctor_get(x_340, 1); +lean_inc(x_343); +x_344 = lean_nat_dec_eq(x_342, x_343); +lean_dec(x_343); +lean_dec(x_342); +if (x_344 == 0) { -return x_349; +return x_334; } else { -lean_object* x_360; -lean_dec(x_356); -x_360 = l_Std_Time_TimeZone_Offset_zero; -lean_ctor_set_tag(x_349, 0); -lean_ctor_set(x_349, 1, x_360); -return x_349; +lean_object* x_345; +lean_dec(x_341); +x_345 = l_Std_Time_TimeZone_Offset_zero; +lean_ctor_set_tag(x_334, 0); +lean_ctor_set(x_334, 1, x_345); +return x_334; } } else { -lean_object* x_361; lean_object* x_362; lean_object* x_363; lean_object* x_364; uint8_t x_365; -x_361 = lean_ctor_get(x_349, 0); -x_362 = lean_ctor_get(x_349, 1); -lean_inc(x_362); -lean_inc(x_361); +lean_object* x_346; lean_object* x_347; lean_object* x_348; lean_object* x_349; uint8_t x_350; +x_346 = lean_ctor_get(x_334, 0); +x_347 = lean_ctor_get(x_334, 1); +lean_inc(x_347); +lean_inc(x_346); +lean_dec(x_334); +x_348 = lean_ctor_get(x_330, 1); +lean_inc(x_348); +lean_dec(x_330); +x_349 = lean_ctor_get(x_346, 1); +lean_inc(x_349); +x_350 = lean_nat_dec_eq(x_348, x_349); lean_dec(x_349); -x_363 = lean_ctor_get(x_345, 1); -lean_inc(x_363); -lean_dec(x_345); -x_364 = lean_ctor_get(x_361, 1); -lean_inc(x_364); -x_365 = lean_nat_dec_eq(x_363, x_364); -lean_dec(x_364); -lean_dec(x_363); -if (x_365 == 0) -{ -lean_object* x_366; -x_366 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_366, 0, x_361); -lean_ctor_set(x_366, 1, x_362); -return x_366; +lean_dec(x_348); +if (x_350 == 0) +{ +lean_object* x_351; +x_351 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_351, 0, x_346); +lean_ctor_set(x_351, 1, x_347); +return x_351; } else { -lean_object* x_367; lean_object* x_368; -lean_dec(x_362); -x_367 = l_Std_Time_TimeZone_Offset_zero; -x_368 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_368, 0, x_361); -lean_ctor_set(x_368, 1, x_367); -return x_368; +lean_object* x_352; lean_object* x_353; +lean_dec(x_347); +x_352 = l_Std_Time_TimeZone_Offset_zero; +x_353 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_353, 0, x_346); +lean_ctor_set(x_353, 1, x_352); +return x_353; } } } } else { -uint8_t x_369; -x_369 = !lean_is_exclusive(x_344); -if (x_369 == 0) +uint8_t x_354; +x_354 = !lean_is_exclusive(x_329); +if (x_354 == 0) { -return x_344; +return x_329; } else { -lean_object* x_370; lean_object* x_371; lean_object* x_372; -x_370 = lean_ctor_get(x_344, 0); -x_371 = lean_ctor_get(x_344, 1); -lean_inc(x_371); -lean_inc(x_370); -lean_dec(x_344); -x_372 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_372, 0, x_370); -lean_ctor_set(x_372, 1, x_371); -return x_372; +lean_object* x_355; lean_object* x_356; lean_object* x_357; +x_355 = lean_ctor_get(x_329, 0); +x_356 = lean_ctor_get(x_329, 1); +lean_inc(x_356); +lean_inc(x_355); +lean_dec(x_329); +x_357 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_357, 0, x_355); +lean_ctor_set(x_357, 1, x_356); +return x_357; } } } default: { -lean_object* x_373; lean_object* x_374; -x_373 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; +lean_object* x_358; lean_object* x_359; +x_358 = l___private_Std_Time_Format_Basic_0__Std_Time_formatWith___closed__5; lean_inc(x_2); -x_374 = l_Std_Internal_Parsec_String_pstring(x_373, x_2); -if (lean_obj_tag(x_374) == 0) +x_359 = l_Std_Internal_Parsec_String_pstring(x_358, x_2); +if (lean_obj_tag(x_359) == 0) { -uint8_t x_375; +uint8_t x_360; lean_dec(x_2); -x_375 = !lean_is_exclusive(x_374); -if (x_375 == 0) +x_360 = !lean_is_exclusive(x_359); +if (x_360 == 0) { -lean_object* x_376; lean_object* x_377; -x_376 = lean_ctor_get(x_374, 1); -lean_dec(x_376); -x_377 = l_Std_Time_TimeZone_Offset_zero; -lean_ctor_set(x_374, 1, x_377); -return x_374; +lean_object* x_361; lean_object* x_362; +x_361 = lean_ctor_get(x_359, 1); +lean_dec(x_361); +x_362 = l_Std_Time_TimeZone_Offset_zero; +lean_ctor_set(x_359, 1, x_362); +return x_359; } else { -lean_object* x_378; lean_object* x_379; lean_object* x_380; -x_378 = lean_ctor_get(x_374, 0); -lean_inc(x_378); -lean_dec(x_374); -x_379 = l_Std_Time_TimeZone_Offset_zero; -x_380 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_380, 0, x_378); -lean_ctor_set(x_380, 1, x_379); -return x_380; +lean_object* x_363; lean_object* x_364; lean_object* x_365; +x_363 = lean_ctor_get(x_359, 0); +lean_inc(x_363); +lean_dec(x_359); +x_364 = l_Std_Time_TimeZone_Offset_zero; +x_365 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_365, 0, x_363); +lean_ctor_set(x_365, 1, x_364); +return x_365; } } else { -uint8_t x_381; -x_381 = !lean_is_exclusive(x_374); -if (x_381 == 0) +uint8_t x_366; +x_366 = !lean_is_exclusive(x_359); +if (x_366 == 0) { -lean_object* x_382; lean_object* x_383; lean_object* x_384; lean_object* x_385; uint8_t x_386; -x_382 = lean_ctor_get(x_374, 0); -x_383 = lean_ctor_get(x_374, 1); -x_384 = lean_ctor_get(x_2, 1); -lean_inc(x_384); +lean_object* x_367; lean_object* x_368; lean_object* x_369; lean_object* x_370; uint8_t x_371; +x_367 = lean_ctor_get(x_359, 0); +x_368 = lean_ctor_get(x_359, 1); +x_369 = lean_ctor_get(x_2, 1); +lean_inc(x_369); lean_dec(x_2); -x_385 = lean_ctor_get(x_382, 1); -lean_inc(x_385); -x_386 = lean_nat_dec_eq(x_384, x_385); -lean_dec(x_385); -lean_dec(x_384); -if (x_386 == 0) +x_370 = lean_ctor_get(x_367, 1); +lean_inc(x_370); +x_371 = lean_nat_dec_eq(x_369, x_370); +lean_dec(x_370); +lean_dec(x_369); +if (x_371 == 0) { -return x_374; +return x_359; } else { -uint8_t x_387; uint8_t x_388; uint8_t x_389; lean_object* x_390; -lean_free_object(x_374); -lean_dec(x_383); -x_387 = 0; -x_388 = 2; -x_389 = 1; -x_390 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_387, x_388, x_389, x_382); -return x_390; +uint8_t x_372; uint8_t x_373; uint8_t x_374; lean_object* x_375; +lean_free_object(x_359); +lean_dec(x_368); +x_372 = 0; +x_373 = 2; +x_374 = 1; +x_375 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_372, x_373, x_374, x_367); +return x_375; } } else { -lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; uint8_t x_395; -x_391 = lean_ctor_get(x_374, 0); -x_392 = lean_ctor_get(x_374, 1); -lean_inc(x_392); -lean_inc(x_391); -lean_dec(x_374); -x_393 = lean_ctor_get(x_2, 1); -lean_inc(x_393); +lean_object* x_376; lean_object* x_377; lean_object* x_378; lean_object* x_379; uint8_t x_380; +x_376 = lean_ctor_get(x_359, 0); +x_377 = lean_ctor_get(x_359, 1); +lean_inc(x_377); +lean_inc(x_376); +lean_dec(x_359); +x_378 = lean_ctor_get(x_2, 1); +lean_inc(x_378); lean_dec(x_2); -x_394 = lean_ctor_get(x_391, 1); -lean_inc(x_394); -x_395 = lean_nat_dec_eq(x_393, x_394); -lean_dec(x_394); -lean_dec(x_393); -if (x_395 == 0) +x_379 = lean_ctor_get(x_376, 1); +lean_inc(x_379); +x_380 = lean_nat_dec_eq(x_378, x_379); +lean_dec(x_379); +lean_dec(x_378); +if (x_380 == 0) { -lean_object* x_396; -x_396 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_396, 0, x_391); -lean_ctor_set(x_396, 1, x_392); -return x_396; +lean_object* x_381; +x_381 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_381, 0, x_376); +lean_ctor_set(x_381, 1, x_377); +return x_381; } else { -uint8_t x_397; uint8_t x_398; uint8_t x_399; lean_object* x_400; -lean_dec(x_392); -x_397 = 0; -x_398 = 2; -x_399 = 1; -x_400 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_397, x_398, x_399, x_391); -return x_400; +uint8_t x_382; uint8_t x_383; uint8_t x_384; lean_object* x_385; +lean_dec(x_377); +x_382 = 0; +x_383 = 2; +x_384 = 1; +x_385 = l___private_Std_Time_Format_Basic_0__Std_Time_parseOffset(x_382, x_383, x_384, x_376); +return x_385; } } } @@ -79249,59 +79155,59 @@ return x_400; } default: { -lean_object* x_401; lean_object* x_402; -x_401 = lean_ctor_get(x_1, 0); -lean_inc(x_401); +lean_object* x_386; lean_object* x_387; +x_386 = lean_ctor_get(x_1, 0); +lean_inc(x_386); lean_dec(x_1); -x_402 = l___private_Std_Time_Format_Basic_0__Std_Time_parseAtLeastNum(x_401, x_2); -lean_dec(x_401); -if (lean_obj_tag(x_402) == 0) -{ -uint8_t x_403; -x_403 = !lean_is_exclusive(x_402); -if (x_403 == 0) -{ -lean_object* x_404; lean_object* x_405; -x_404 = lean_ctor_get(x_402, 1); -x_405 = lean_nat_to_int(x_404); -lean_ctor_set(x_402, 1, x_405); -return x_402; +x_387 = l___private_Std_Time_Format_Basic_0__Std_Time_parseAtLeastNum(x_386, x_2); +lean_dec(x_386); +if (lean_obj_tag(x_387) == 0) +{ +uint8_t x_388; +x_388 = !lean_is_exclusive(x_387); +if (x_388 == 0) +{ +lean_object* x_389; lean_object* x_390; +x_389 = lean_ctor_get(x_387, 1); +x_390 = lean_nat_to_int(x_389); +lean_ctor_set(x_387, 1, x_390); +return x_387; } else { -lean_object* x_406; lean_object* x_407; lean_object* x_408; lean_object* x_409; -x_406 = lean_ctor_get(x_402, 0); -x_407 = lean_ctor_get(x_402, 1); -lean_inc(x_407); -lean_inc(x_406); -lean_dec(x_402); -x_408 = lean_nat_to_int(x_407); -x_409 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_409, 0, x_406); -lean_ctor_set(x_409, 1, x_408); -return x_409; +lean_object* x_391; lean_object* x_392; lean_object* x_393; lean_object* x_394; +x_391 = lean_ctor_get(x_387, 0); +x_392 = lean_ctor_get(x_387, 1); +lean_inc(x_392); +lean_inc(x_391); +lean_dec(x_387); +x_393 = lean_nat_to_int(x_392); +x_394 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_394, 0, x_391); +lean_ctor_set(x_394, 1, x_393); +return x_394; } } else { -uint8_t x_410; -x_410 = !lean_is_exclusive(x_402); -if (x_410 == 0) +uint8_t x_395; +x_395 = !lean_is_exclusive(x_387); +if (x_395 == 0) { -return x_402; +return x_387; } else { -lean_object* x_411; lean_object* x_412; lean_object* x_413; -x_411 = lean_ctor_get(x_402, 0); -x_412 = lean_ctor_get(x_402, 1); -lean_inc(x_412); -lean_inc(x_411); -lean_dec(x_402); -x_413 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_413, 0, x_411); -lean_ctor_set(x_413, 1, x_412); -return x_413; +lean_object* x_396; lean_object* x_397; lean_object* x_398; +x_396 = lean_ctor_get(x_387, 0); +x_397 = lean_ctor_get(x_387, 1); +lean_inc(x_397); +lean_inc(x_396); +lean_dec(x_387); +x_398 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_398, 0, x_396); +lean_ctor_set(x_398, 1, x_397); +return x_398; } } } @@ -85829,19 +85735,6 @@ return x_3; static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__9() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; -x_2 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__8; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); -lean_ctor_set(x_4, 1, x_2); -return x_4; -} -} -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__10() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__1; x_2 = l___private_Std_Time_Format_Basic_0__Std_Time_reprText____x40_Std_Time_Format_Basic___hyg_15____closed__6; @@ -85849,81 +85742,81 @@ x_3 = lean_int_sub(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__11() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__10; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__9; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__12; x_3 = lean_int_emod(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__12() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__11; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__10; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__12; x_3 = lean_int_add(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__13() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__12() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__12; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__11; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__12; x_3 = lean_int_emod(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__14() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__13() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__13; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__12; x_2 = l___private_Std_Time_Format_Basic_0__Std_Time_reprText____x40_Std_Time_Format_Basic___hyg_15____closed__6; x_3 = lean_int_add(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__15() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__14() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__10; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__9; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__4; x_3 = lean_int_emod(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__16() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__15() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__15; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__14; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__4; x_3 = lean_int_add(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__16() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__16; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__15; x_2 = l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__4; x_3 = lean_int_emod(x_1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18() { +static lean_object* _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17; +x_1 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__16; x_2 = l___private_Std_Time_Format_Basic_0__Std_Time_reprText____x40_Std_Time_Format_Basic___hyg_15____closed__6; x_3 = lean_int_add(x_1, x_2); return x_3; @@ -86188,7 +86081,7 @@ lean_object* x_68; lean_object* x_118; if (lean_obj_tag(x_56) == 0) { lean_object* x_221; -x_221 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18; +x_221 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17; x_118 = x_221; goto block_220; } @@ -86369,7 +86262,7 @@ lean_object* x_119; if (lean_obj_tag(x_57) == 0) { lean_object* x_218; -x_218 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__14; +x_218 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__13; x_119 = x_218; goto block_217; } @@ -86670,7 +86563,7 @@ lean_object* x_150; if (lean_obj_tag(x_62) == 0) { lean_object* x_173; -x_173 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__9; +x_173 = l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__8; x_150 = x_173; goto block_172; } @@ -89133,8 +89026,6 @@ l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__33 = _init_l_Std_Ti lean_mark_persistent(l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__33); l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34 = _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34(); lean_mark_persistent(l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__34); -l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35 = _init_l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35(); -lean_mark_persistent(l_Std_Time_Awareness_instInhabitedType___lambda__2___closed__35); l_Std_Time_Awareness_instInhabitedType___closed__1 = _init_l_Std_Time_Awareness_instInhabitedType___closed__1(); lean_mark_persistent(l_Std_Time_Awareness_instInhabitedType___closed__1); l_Std_Time_Awareness_instInhabitedType___closed__2 = _init_l_Std_Time_Awareness_instInhabitedType___closed__2(); @@ -89465,8 +89356,6 @@ l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___ lean_mark_persistent(l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__16); l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17 = _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17(); lean_mark_persistent(l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__17); -l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18 = _init_l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18(); -lean_mark_persistent(l___private_Std_Time_Format_Basic_0__Std_Time_GenericFormat_DateBuilder_build___closed__18); l_Std_Time_GenericFormat_spec_x21___closed__1 = _init_l_Std_Time_GenericFormat_spec_x21___closed__1(); lean_mark_persistent(l_Std_Time_GenericFormat_spec_x21___closed__1); l_Std_Time_GenericFormat_spec_x21___closed__2 = _init_l_Std_Time_GenericFormat_spec_x21___closed__2(); diff --git a/stage0/stdlib/Std/Time/Notation.c b/stage0/stdlib/Std/Time/Notation.c index fbf7c84b7c88..24c94425d384 100644 --- a/stage0/stdlib/Std/Time/Notation.c +++ b/stage0/stdlib/Std/Time/Notation.c @@ -89,7 +89,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetZ___c lean_object* l_Std_Time_PlainDateTime_fromLeanDateTimeString(lean_object*); lean_object* l_Lean_TSyntax_getString(lean_object*); static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__218; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertYear___closed__21; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetO___closed__15; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__180; @@ -194,6 +193,7 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___ static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxInt___closed__18; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffset___closed__6; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__209; +static lean_object* l_Std_Time_termZoned_x28___x2c___x29___closed__11; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetX___closed__23; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertFraction___closed__7; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__138; @@ -213,7 +213,6 @@ static lean_object* l_Std_Time_termOffset_x28___x29___closed__2; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertFormatPart___closed__5; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZoneName___closed__14; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__97; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; static lean_object* l_Std_Time_termTimezone_x28___x29___closed__5; static lean_object* l_Std_Time_termOffset_x28___x29___closed__7; LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainDate(lean_object*, lean_object*, lean_object*); @@ -244,7 +243,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__84; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertText___closed__14; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZoneName___closed__11; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; static lean_object* l_Std_Time_termTimezone_x28___x29___closed__3; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertYear___closed__8; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__95; @@ -285,14 +283,12 @@ LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifi static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__143; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetX___closed__32; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertTimezone___closed__14; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__17; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetX___closed__2; lean_object* l_Lean_Syntax_mkStrLit(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__114; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertYear___closed__20; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__103; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertYear___closed__4; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__81; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__27; @@ -302,7 +298,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___ LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertFraction(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__43; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__67; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertText___closed__4; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZoneName___closed__1; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZonedDateTime___closed__20; @@ -347,7 +342,6 @@ static lean_object* l_Std_Time_termDate_x28___x29___closed__1; LEAN_EXPORT lean_object* l_Std_Time___aux__Std__Time__Notation______macroRules__Std__Time__termZoned_x28___x29__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_termDatetime_x28___x29___closed__4; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__155; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__12; static lean_object* l_Std_Time_termDate_x28___x29___closed__4; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZonedDateTime___closed__25; @@ -380,7 +374,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___ LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertZonedDateTime___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxInt___closed__4; LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertText(uint8_t, lean_object*, lean_object*); -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; static lean_object* l_Std_Time_termTime_x28___x29___closed__1; static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxVal___closed__1; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertText___closed__10; @@ -442,7 +435,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___ static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxVal___closed__8; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__7; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertText___closed__9; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__213; static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxInt___closed__3; @@ -663,7 +655,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertNumber___cl static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxString___closed__1; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetX___closed__27; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__80; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxBounded___closed__16; LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertOffsetO___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Time_Notation_0__Std_Time_syntaxNat___closed__1; @@ -727,7 +718,6 @@ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertTimezone___ static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertModifier___closed__160; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__14; static lean_object* l_Std_Time_termZoned_x28___x29___closed__7; -static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertFormatPart___closed__6; static lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainDate___closed__9; static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertText___closed__1() { @@ -10660,612 +10650,107 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("anonymousCtor", 13, 13); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__1; -x_2 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__2; -x_3 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__3; -x_4 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9; -x_5 = l_Lean_Name_mkStr4(x_1, x_2, x_3, x_4); -return x_5; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("⟨", 3, 1); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12; -x_2 = l_String_toSubstring_x27(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12; -x_3 = l_Lean_Name_str___override(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Notation_0__Std_Time_convertTimezone___closed__11; -x_2 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12; -x_3 = l_Lean_Name_mkStr2(x_1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = lean_box(0); -x_2 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16; -x_3 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_3, 0, x_2); -lean_ctor_set(x_3, 1, x_1); -return x_3; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(",", 1, 1); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("⟩", 3, 1); -return x_1; -} -} LEAN_EXPORT lean_object* l___private_Std_Time_Notation_0__Std_Time_convertPlainTime(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; uint8_t x_6; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; uint8_t x_18; x_4 = lean_ctor_get(x_1, 0); lean_inc(x_2); x_5 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_4, x_2, x_3); -x_6 = !lean_is_exclusive(x_5); -if (x_6 == 0) -{ -lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; uint8_t x_11; -x_7 = lean_ctor_get(x_5, 0); -x_8 = lean_ctor_get(x_5, 1); -x_9 = lean_ctor_get(x_1, 1); +x_6 = lean_ctor_get(x_5, 0); +lean_inc(x_6); +x_7 = lean_ctor_get(x_5, 1); +lean_inc(x_7); +lean_dec(x_5); +x_8 = lean_ctor_get(x_1, 1); lean_inc(x_2); -x_10 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_9, x_2, x_8); -x_11 = !lean_is_exclusive(x_10); -if (x_11 == 0) -{ -lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; uint8_t x_17; -x_12 = lean_ctor_get(x_10, 0); -x_13 = lean_ctor_get(x_10, 1); -x_14 = lean_ctor_get(x_1, 2); -x_15 = lean_ctor_get(x_14, 1); +x_9 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_8, x_2, x_7); +x_10 = lean_ctor_get(x_9, 0); +lean_inc(x_10); +x_11 = lean_ctor_get(x_9, 1); +lean_inc(x_11); +lean_dec(x_9); +x_12 = lean_ctor_get(x_1, 2); lean_inc(x_2); -x_16 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_15, x_2, x_13); -x_17 = !lean_is_exclusive(x_16); -if (x_17 == 0) -{ -lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; uint8_t x_22; -x_18 = lean_ctor_get(x_16, 0); -x_19 = lean_ctor_get(x_16, 1); -x_20 = lean_ctor_get(x_1, 3); +x_13 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_12, x_2, x_11); +x_14 = lean_ctor_get(x_13, 0); +lean_inc(x_14); +x_15 = lean_ctor_get(x_13, 1); +lean_inc(x_15); +lean_dec(x_13); +x_16 = lean_ctor_get(x_1, 3); lean_inc(x_2); -x_21 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_20, x_2, x_19); -x_22 = !lean_is_exclusive(x_21); -if (x_22 == 0) +x_17 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_16, x_2, x_15); +x_18 = !lean_is_exclusive(x_17); +if (x_18 == 0) { -lean_object* x_23; lean_object* x_24; uint8_t x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; -x_23 = lean_ctor_get(x_21, 0); -x_24 = lean_ctor_get(x_2, 5); +lean_object* x_19; lean_object* x_20; uint8_t x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; +x_19 = lean_ctor_get(x_17, 0); +x_20 = lean_ctor_get(x_2, 5); +lean_inc(x_20); +x_21 = 0; +x_22 = l_Lean_SourceInfo_fromRef(x_20, x_21); +lean_dec(x_20); +x_23 = lean_ctor_get(x_2, 2); +lean_inc(x_23); +x_24 = lean_ctor_get(x_2, 1); lean_inc(x_24); -x_25 = 0; -x_26 = l_Lean_SourceInfo_fromRef(x_24, x_25); -lean_dec(x_24); -x_27 = lean_ctor_get(x_2, 2); -lean_inc(x_27); -x_28 = lean_ctor_get(x_2, 1); -lean_inc(x_28); -lean_dec(x_2); -x_29 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; -lean_inc(x_27); -lean_inc(x_28); -x_30 = l_Lean_addMacroScope(x_28, x_29, x_27); -x_31 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -x_32 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; -lean_inc(x_26); -x_33 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_33, 0, x_26); -lean_ctor_set(x_33, 1, x_31); -lean_ctor_set(x_33, 2, x_30); -lean_ctor_set(x_33, 3, x_32); -x_34 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; -lean_inc(x_26); -lean_ctor_set_tag(x_16, 2); -lean_ctor_set(x_16, 1, x_34); -lean_ctor_set(x_16, 0, x_26); -x_35 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; -x_36 = l_Lean_addMacroScope(x_28, x_35, x_27); -x_37 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; -x_38 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; -lean_inc(x_26); -x_39 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_39, 0, x_26); -lean_ctor_set(x_39, 1, x_37); -lean_ctor_set(x_39, 2, x_36); -lean_ctor_set(x_39, 3, x_38); -x_40 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; -lean_inc(x_26); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_40); -lean_ctor_set(x_10, 0, x_26); -x_41 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; -lean_inc(x_26); -x_42 = l_Lean_Syntax_node3(x_26, x_41, x_39, x_10, x_18); -x_43 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; -lean_inc(x_26); -lean_ctor_set_tag(x_5, 2); -lean_ctor_set(x_5, 1, x_43); -lean_ctor_set(x_5, 0, x_26); -x_44 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; -lean_inc(x_26); -x_45 = l_Lean_Syntax_node3(x_26, x_44, x_16, x_42, x_5); -lean_inc(x_26); -x_46 = l_Lean_Syntax_node4(x_26, x_41, x_7, x_12, x_45, x_23); -x_47 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; -x_48 = l_Lean_Syntax_node2(x_26, x_47, x_33, x_46); -lean_ctor_set(x_21, 0, x_48); -return x_21; -} -else -{ -lean_object* x_49; lean_object* x_50; lean_object* x_51; uint8_t x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; lean_object* x_74; lean_object* x_75; lean_object* x_76; -x_49 = lean_ctor_get(x_21, 0); -x_50 = lean_ctor_get(x_21, 1); -lean_inc(x_50); -lean_inc(x_49); -lean_dec(x_21); -x_51 = lean_ctor_get(x_2, 5); -lean_inc(x_51); -x_52 = 0; -x_53 = l_Lean_SourceInfo_fromRef(x_51, x_52); -lean_dec(x_51); -x_54 = lean_ctor_get(x_2, 2); -lean_inc(x_54); -x_55 = lean_ctor_get(x_2, 1); -lean_inc(x_55); -lean_dec(x_2); -x_56 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; -lean_inc(x_54); -lean_inc(x_55); -x_57 = l_Lean_addMacroScope(x_55, x_56, x_54); -x_58 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -x_59 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; -lean_inc(x_53); -x_60 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_60, 0, x_53); -lean_ctor_set(x_60, 1, x_58); -lean_ctor_set(x_60, 2, x_57); -lean_ctor_set(x_60, 3, x_59); -x_61 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; -lean_inc(x_53); -lean_ctor_set_tag(x_16, 2); -lean_ctor_set(x_16, 1, x_61); -lean_ctor_set(x_16, 0, x_53); -x_62 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; -x_63 = l_Lean_addMacroScope(x_55, x_62, x_54); -x_64 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; -x_65 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; -lean_inc(x_53); -x_66 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_66, 0, x_53); -lean_ctor_set(x_66, 1, x_64); -lean_ctor_set(x_66, 2, x_63); -lean_ctor_set(x_66, 3, x_65); -x_67 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; -lean_inc(x_53); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_67); -lean_ctor_set(x_10, 0, x_53); -x_68 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; -lean_inc(x_53); -x_69 = l_Lean_Syntax_node3(x_53, x_68, x_66, x_10, x_18); -x_70 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; -lean_inc(x_53); -lean_ctor_set_tag(x_5, 2); -lean_ctor_set(x_5, 1, x_70); -lean_ctor_set(x_5, 0, x_53); -x_71 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; -lean_inc(x_53); -x_72 = l_Lean_Syntax_node3(x_53, x_71, x_16, x_69, x_5); -lean_inc(x_53); -x_73 = l_Lean_Syntax_node4(x_53, x_68, x_7, x_12, x_72, x_49); -x_74 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; -x_75 = l_Lean_Syntax_node2(x_53, x_74, x_60, x_73); -x_76 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_76, 0, x_75); -lean_ctor_set(x_76, 1, x_50); -return x_76; -} -} -else -{ -lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; uint8_t x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_77 = lean_ctor_get(x_16, 0); -x_78 = lean_ctor_get(x_16, 1); -lean_inc(x_78); -lean_inc(x_77); -lean_dec(x_16); -x_79 = lean_ctor_get(x_1, 3); -lean_inc(x_2); -x_80 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_79, x_2, x_78); -x_81 = lean_ctor_get(x_80, 0); -lean_inc(x_81); -x_82 = lean_ctor_get(x_80, 1); -lean_inc(x_82); -if (lean_is_exclusive(x_80)) { - lean_ctor_release(x_80, 0); - lean_ctor_release(x_80, 1); - x_83 = x_80; -} else { - lean_dec_ref(x_80); - x_83 = lean_box(0); -} -x_84 = lean_ctor_get(x_2, 5); -lean_inc(x_84); -x_85 = 0; -x_86 = l_Lean_SourceInfo_fromRef(x_84, x_85); -lean_dec(x_84); -x_87 = lean_ctor_get(x_2, 2); -lean_inc(x_87); -x_88 = lean_ctor_get(x_2, 1); -lean_inc(x_88); lean_dec(x_2); -x_89 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; -lean_inc(x_87); -lean_inc(x_88); -x_90 = l_Lean_addMacroScope(x_88, x_89, x_87); -x_91 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -x_92 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; -lean_inc(x_86); -x_93 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_93, 0, x_86); -lean_ctor_set(x_93, 1, x_91); -lean_ctor_set(x_93, 2, x_90); -lean_ctor_set(x_93, 3, x_92); -x_94 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; -lean_inc(x_86); -x_95 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_95, 0, x_86); -lean_ctor_set(x_95, 1, x_94); -x_96 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; -x_97 = l_Lean_addMacroScope(x_88, x_96, x_87); -x_98 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; -x_99 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; -lean_inc(x_86); -x_100 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_100, 0, x_86); -lean_ctor_set(x_100, 1, x_98); -lean_ctor_set(x_100, 2, x_97); -lean_ctor_set(x_100, 3, x_99); -x_101 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; -lean_inc(x_86); -lean_ctor_set_tag(x_10, 2); -lean_ctor_set(x_10, 1, x_101); -lean_ctor_set(x_10, 0, x_86); -x_102 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; -lean_inc(x_86); -x_103 = l_Lean_Syntax_node3(x_86, x_102, x_100, x_10, x_77); -x_104 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; -lean_inc(x_86); -lean_ctor_set_tag(x_5, 2); -lean_ctor_set(x_5, 1, x_104); -lean_ctor_set(x_5, 0, x_86); -x_105 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; -lean_inc(x_86); -x_106 = l_Lean_Syntax_node3(x_86, x_105, x_95, x_103, x_5); -lean_inc(x_86); -x_107 = l_Lean_Syntax_node4(x_86, x_102, x_7, x_12, x_106, x_81); -x_108 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; -x_109 = l_Lean_Syntax_node2(x_86, x_108, x_93, x_107); -if (lean_is_scalar(x_83)) { - x_110 = lean_alloc_ctor(0, 2, 0); -} else { - x_110 = x_83; -} -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set(x_110, 1, x_82); -return x_110; -} -} -else -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; lean_object* x_123; lean_object* x_124; uint8_t x_125; lean_object* x_126; lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; lean_object* x_151; -x_111 = lean_ctor_get(x_10, 0); -x_112 = lean_ctor_get(x_10, 1); -lean_inc(x_112); -lean_inc(x_111); -lean_dec(x_10); -x_113 = lean_ctor_get(x_1, 2); -x_114 = lean_ctor_get(x_113, 1); -lean_inc(x_2); -x_115 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_114, x_2, x_112); -x_116 = lean_ctor_get(x_115, 0); -lean_inc(x_116); -x_117 = lean_ctor_get(x_115, 1); -lean_inc(x_117); -if (lean_is_exclusive(x_115)) { - lean_ctor_release(x_115, 0); - lean_ctor_release(x_115, 1); - x_118 = x_115; -} else { - lean_dec_ref(x_115); - x_118 = lean_box(0); -} -x_119 = lean_ctor_get(x_1, 3); -lean_inc(x_2); -x_120 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_119, x_2, x_117); -x_121 = lean_ctor_get(x_120, 0); -lean_inc(x_121); -x_122 = lean_ctor_get(x_120, 1); -lean_inc(x_122); -if (lean_is_exclusive(x_120)) { - lean_ctor_release(x_120, 0); - lean_ctor_release(x_120, 1); - x_123 = x_120; -} else { - lean_dec_ref(x_120); - x_123 = lean_box(0); -} -x_124 = lean_ctor_get(x_2, 5); -lean_inc(x_124); -x_125 = 0; -x_126 = l_Lean_SourceInfo_fromRef(x_124, x_125); -lean_dec(x_124); -x_127 = lean_ctor_get(x_2, 2); -lean_inc(x_127); -x_128 = lean_ctor_get(x_2, 1); -lean_inc(x_128); -lean_dec(x_2); -x_129 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; -lean_inc(x_127); -lean_inc(x_128); -x_130 = l_Lean_addMacroScope(x_128, x_129, x_127); -x_131 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -x_132 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; -lean_inc(x_126); -x_133 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_133, 0, x_126); -lean_ctor_set(x_133, 1, x_131); -lean_ctor_set(x_133, 2, x_130); -lean_ctor_set(x_133, 3, x_132); -x_134 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; -lean_inc(x_126); -if (lean_is_scalar(x_118)) { - x_135 = lean_alloc_ctor(2, 2, 0); -} else { - x_135 = x_118; - lean_ctor_set_tag(x_135, 2); -} -lean_ctor_set(x_135, 0, x_126); -lean_ctor_set(x_135, 1, x_134); -x_136 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; -x_137 = l_Lean_addMacroScope(x_128, x_136, x_127); -x_138 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; -x_139 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; -lean_inc(x_126); -x_140 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_140, 0, x_126); -lean_ctor_set(x_140, 1, x_138); -lean_ctor_set(x_140, 2, x_137); -lean_ctor_set(x_140, 3, x_139); -x_141 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; -lean_inc(x_126); -x_142 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_142, 0, x_126); -lean_ctor_set(x_142, 1, x_141); -x_143 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; -lean_inc(x_126); -x_144 = l_Lean_Syntax_node3(x_126, x_143, x_140, x_142, x_116); -x_145 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; -lean_inc(x_126); -lean_ctor_set_tag(x_5, 2); -lean_ctor_set(x_5, 1, x_145); -lean_ctor_set(x_5, 0, x_126); -x_146 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; -lean_inc(x_126); -x_147 = l_Lean_Syntax_node3(x_126, x_146, x_135, x_144, x_5); -lean_inc(x_126); -x_148 = l_Lean_Syntax_node4(x_126, x_143, x_7, x_111, x_147, x_121); -x_149 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; -x_150 = l_Lean_Syntax_node2(x_126, x_149, x_133, x_148); -if (lean_is_scalar(x_123)) { - x_151 = lean_alloc_ctor(0, 2, 0); -} else { - x_151 = x_123; -} -lean_ctor_set(x_151, 0, x_150); -lean_ctor_set(x_151, 1, x_122); -return x_151; -} +x_25 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; +x_26 = l_Lean_addMacroScope(x_24, x_25, x_23); +x_27 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; +x_28 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; +lean_inc(x_22); +x_29 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_29, 0, x_22); +lean_ctor_set(x_29, 1, x_27); +lean_ctor_set(x_29, 2, x_26); +lean_ctor_set(x_29, 3, x_28); +x_30 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; +lean_inc(x_22); +x_31 = l_Lean_Syntax_node4(x_22, x_30, x_6, x_10, x_14, x_19); +x_32 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; +x_33 = l_Lean_Syntax_node2(x_22, x_32, x_29, x_31); +lean_ctor_set(x_17, 0, x_33); +return x_17; } else { -lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; uint8_t x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; lean_object* x_175; lean_object* x_176; lean_object* x_177; lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; lean_object* x_182; lean_object* x_183; lean_object* x_184; lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; lean_object* x_189; lean_object* x_190; lean_object* x_191; lean_object* x_192; lean_object* x_193; lean_object* x_194; lean_object* x_195; lean_object* x_196; lean_object* x_197; lean_object* x_198; -x_152 = lean_ctor_get(x_5, 0); -x_153 = lean_ctor_get(x_5, 1); -lean_inc(x_153); -lean_inc(x_152); -lean_dec(x_5); -x_154 = lean_ctor_get(x_1, 1); -lean_inc(x_2); -x_155 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_154, x_2, x_153); -x_156 = lean_ctor_get(x_155, 0); -lean_inc(x_156); -x_157 = lean_ctor_get(x_155, 1); -lean_inc(x_157); -if (lean_is_exclusive(x_155)) { - lean_ctor_release(x_155, 0); - lean_ctor_release(x_155, 1); - x_158 = x_155; -} else { - lean_dec_ref(x_155); - x_158 = lean_box(0); -} -x_159 = lean_ctor_get(x_1, 2); -x_160 = lean_ctor_get(x_159, 1); -lean_inc(x_2); -x_161 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_160, x_2, x_157); -x_162 = lean_ctor_get(x_161, 0); -lean_inc(x_162); -x_163 = lean_ctor_get(x_161, 1); -lean_inc(x_163); -if (lean_is_exclusive(x_161)) { - lean_ctor_release(x_161, 0); - lean_ctor_release(x_161, 1); - x_164 = x_161; -} else { - lean_dec_ref(x_161); - x_164 = lean_box(0); -} -x_165 = lean_ctor_get(x_1, 3); -lean_inc(x_2); -x_166 = l___private_Std_Time_Notation_0__Std_Time_syntaxBounded(x_165, x_2, x_163); -x_167 = lean_ctor_get(x_166, 0); -lean_inc(x_167); -x_168 = lean_ctor_get(x_166, 1); -lean_inc(x_168); -if (lean_is_exclusive(x_166)) { - lean_ctor_release(x_166, 0); - lean_ctor_release(x_166, 1); - x_169 = x_166; -} else { - lean_dec_ref(x_166); - x_169 = lean_box(0); -} -x_170 = lean_ctor_get(x_2, 5); -lean_inc(x_170); -x_171 = 0; -x_172 = l_Lean_SourceInfo_fromRef(x_170, x_171); -lean_dec(x_170); -x_173 = lean_ctor_get(x_2, 2); -lean_inc(x_173); -x_174 = lean_ctor_get(x_2, 1); -lean_inc(x_174); +lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; +x_34 = lean_ctor_get(x_17, 0); +x_35 = lean_ctor_get(x_17, 1); +lean_inc(x_35); +lean_inc(x_34); +lean_dec(x_17); +x_36 = lean_ctor_get(x_2, 5); +lean_inc(x_36); +x_37 = 0; +x_38 = l_Lean_SourceInfo_fromRef(x_36, x_37); +lean_dec(x_36); +x_39 = lean_ctor_get(x_2, 2); +lean_inc(x_39); +x_40 = lean_ctor_get(x_2, 1); +lean_inc(x_40); lean_dec(x_2); -x_175 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; -lean_inc(x_173); -lean_inc(x_174); -x_176 = l_Lean_addMacroScope(x_174, x_175, x_173); -x_177 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; -x_178 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; -lean_inc(x_172); -x_179 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_179, 0, x_172); -lean_ctor_set(x_179, 1, x_177); -lean_ctor_set(x_179, 2, x_176); -lean_ctor_set(x_179, 3, x_178); -x_180 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11; -lean_inc(x_172); -if (lean_is_scalar(x_164)) { - x_181 = lean_alloc_ctor(2, 2, 0); -} else { - x_181 = x_164; - lean_ctor_set_tag(x_181, 2); -} -lean_ctor_set(x_181, 0, x_172); -lean_ctor_set(x_181, 1, x_180); -x_182 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14; -x_183 = l_Lean_addMacroScope(x_174, x_182, x_173); -x_184 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13; -x_185 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17; -lean_inc(x_172); -x_186 = lean_alloc_ctor(3, 4, 0); -lean_ctor_set(x_186, 0, x_172); -lean_ctor_set(x_186, 1, x_184); -lean_ctor_set(x_186, 2, x_183); -lean_ctor_set(x_186, 3, x_185); -x_187 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; -lean_inc(x_172); -if (lean_is_scalar(x_158)) { - x_188 = lean_alloc_ctor(2, 2, 0); -} else { - x_188 = x_158; - lean_ctor_set_tag(x_188, 2); -} -lean_ctor_set(x_188, 0, x_172); -lean_ctor_set(x_188, 1, x_187); -x_189 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; -lean_inc(x_172); -x_190 = l_Lean_Syntax_node3(x_172, x_189, x_186, x_188, x_162); -x_191 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19; -lean_inc(x_172); -x_192 = lean_alloc_ctor(2, 2, 0); -lean_ctor_set(x_192, 0, x_172); -lean_ctor_set(x_192, 1, x_191); -x_193 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10; -lean_inc(x_172); -x_194 = l_Lean_Syntax_node3(x_172, x_193, x_181, x_190, x_192); -lean_inc(x_172); -x_195 = l_Lean_Syntax_node4(x_172, x_189, x_152, x_156, x_194, x_167); -x_196 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; -x_197 = l_Lean_Syntax_node2(x_172, x_196, x_179, x_195); -if (lean_is_scalar(x_169)) { - x_198 = lean_alloc_ctor(0, 2, 0); -} else { - x_198 = x_169; -} -lean_ctor_set(x_198, 0, x_197); -lean_ctor_set(x_198, 1, x_168); -return x_198; +x_41 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__4; +x_42 = l_Lean_addMacroScope(x_40, x_41, x_39); +x_43 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__2; +x_44 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8; +lean_inc(x_38); +x_45 = lean_alloc_ctor(3, 4, 0); +lean_ctor_set(x_45, 0, x_38); +lean_ctor_set(x_45, 1, x_43); +lean_ctor_set(x_45, 2, x_42); +lean_ctor_set(x_45, 3, x_44); +x_46 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__16; +lean_inc(x_38); +x_47 = l_Lean_Syntax_node4(x_38, x_46, x_6, x_10, x_14, x_34); +x_48 = l___private_Std_Time_Notation_0__Std_Time_convertNumber___closed__5; +x_49 = l_Lean_Syntax_node2(x_38, x_48, x_45, x_47); +x_50 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set(x_50, 1, x_35); +return x_50; } } } @@ -12155,20 +11640,28 @@ return x_4; static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__3() { _start: { +lean_object* x_1; +x_1 = lean_mk_string_unchecked(",", 1, 1); +return x_1; +} +} +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__4() { +_start: +{ lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18; +x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__3; x_2 = lean_alloc_ctor(5, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__4() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__5() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Std_Time_termZoned_x28___x29___closed__4; x_2 = l_Std_Time_termZoned_x28___x29___closed__8; -x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__3; +x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__4; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -12176,7 +11669,7 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__5() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__6() { _start: { lean_object* x_1; @@ -12184,21 +11677,21 @@ x_1 = lean_mk_string_unchecked("term", 4, 4); return x_1; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__6() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__7() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = lean_box(0); -x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__5; +x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__6; x_3 = l_Lean_Name_str___override(x_1, x_2); return x_3; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__7() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__8() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__6; +x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__7; x_2 = lean_unsigned_to_nat(0u); x_3 = lean_alloc_ctor(7, 2, 0); lean_ctor_set(x_3, 0, x_1); @@ -12206,13 +11699,13 @@ lean_ctor_set(x_3, 1, x_2); return x_3; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__8() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__9() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Std_Time_termZoned_x28___x29___closed__4; -x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__4; -x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__7; +x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__5; +x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__8; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -12220,12 +11713,12 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__9() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__10() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Std_Time_termZoned_x28___x29___closed__4; -x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__8; +x_2 = l_Std_Time_termZoned_x28___x2c___x29___closed__9; x_3 = l_Std_Time_termZoned_x28___x29___closed__9; x_4 = lean_alloc_ctor(2, 3, 0); lean_ctor_set(x_4, 0, x_1); @@ -12234,13 +11727,13 @@ lean_ctor_set(x_4, 2, x_3); return x_4; } } -static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__10() { +static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29___closed__11() { _start: { lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__2; x_2 = lean_unsigned_to_nat(1024u); -x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__9; +x_3 = l_Std_Time_termZoned_x28___x2c___x29___closed__10; x_4 = lean_alloc_ctor(3, 3, 0); lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); @@ -12252,7 +11745,7 @@ static lean_object* _init_l_Std_Time_termZoned_x28___x2c___x29() { _start: { lean_object* x_1; -x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__10; +x_1 = l_Std_Time_termZoned_x28___x2c___x29___closed__11; return x_1; } } @@ -14520,28 +14013,6 @@ l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__7 = _init_l lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__7); l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8(); lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__8); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__9); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__10); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__11); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__12); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__13); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__14); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__15); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__16); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__17); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__18); -l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19(); -lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainTime___closed__19); l___private_Std_Time_Notation_0__Std_Time_convertPlainDateTime___closed__1 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainDateTime___closed__1(); lean_mark_persistent(l___private_Std_Time_Notation_0__Std_Time_convertPlainDateTime___closed__1); l___private_Std_Time_Notation_0__Std_Time_convertPlainDateTime___closed__2 = _init_l___private_Std_Time_Notation_0__Std_Time_convertPlainDateTime___closed__2(); @@ -14654,6 +14125,8 @@ l_Std_Time_termZoned_x28___x2c___x29___closed__9 = _init_l_Std_Time_termZoned_x2 lean_mark_persistent(l_Std_Time_termZoned_x28___x2c___x29___closed__9); l_Std_Time_termZoned_x28___x2c___x29___closed__10 = _init_l_Std_Time_termZoned_x28___x2c___x29___closed__10(); lean_mark_persistent(l_Std_Time_termZoned_x28___x2c___x29___closed__10); +l_Std_Time_termZoned_x28___x2c___x29___closed__11 = _init_l_Std_Time_termZoned_x28___x2c___x29___closed__11(); +lean_mark_persistent(l_Std_Time_termZoned_x28___x2c___x29___closed__11); l_Std_Time_termZoned_x28___x2c___x29 = _init_l_Std_Time_termZoned_x28___x2c___x29(); lean_mark_persistent(l_Std_Time_termZoned_x28___x2c___x29); l_Std_Time_termDatetime_x28___x29___closed__1 = _init_l_Std_Time_termDatetime_x28___x29___closed__1(); diff --git a/stage0/stdlib/Std/Time/Time/PlainTime.c b/stage0/stdlib/Std/Time/Time/PlainTime.c index 2cb3fa438157..e16d987aa281 100644 --- a/stage0/stdlib/Std/Time/Time/PlainTime.c +++ b/stage0/stdlib/Std/Time/Time/PlainTime.c @@ -18,13 +18,11 @@ LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toHours(lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__22; static lean_object* l_Std_Time_PlainTime_toNanoseconds___closed__1; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_withSeconds(lean_object*, lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addMinutes(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHours(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofSeconds___boxed(lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__19; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHAddOffset__2; -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds___boxed(lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toNanoseconds___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subSeconds___boxed(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24; @@ -34,14 +32,10 @@ LEAN_EXPORT lean_object* l_Std_Time_PlainTime_millisecond___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_withMinutes(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__16; static lean_object* l_Std_Time_PlainTime_instHSubOffset___closed__1; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34; static lean_object* l_Std_Time_PlainTime_instHAddOffset__2___closed__1; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHSubOffset; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25; static lean_object* l_Std_Time_PlainTime_instHSubOffset__3___closed__1; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subHours___boxed(lean_object*, lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; static lean_object* l_Std_Time_PlainTime_instHAddOffset___closed__1; static lean_object* l_Std_Time_instInhabitedPlainTime___closed__11; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__5; @@ -55,11 +49,9 @@ static lean_object* l_Std_Time_instInhabitedPlainTime___closed__3; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subMilliseconds(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__3; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addSeconds___boxed(lean_object*, lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; LEAN_EXPORT lean_object* l_Std_Time_instBEqPlainTime___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHSubOffset__1; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHAddOffset; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHAddOffset__3; static lean_object* l_Std_Time_PlainTime_toSeconds___closed__2; @@ -67,9 +59,8 @@ static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTim static lean_object* l_Std_Time_PlainTime_toNanoseconds___closed__2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subSeconds(lean_object*, lean_object*); static lean_object* l_Std_Time_instInhabitedPlainTime___closed__2; -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds(uint8_t, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toSeconds___boxed(lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__20; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subMilliseconds___boxed(lean_object*, lean_object*); lean_object* lean_nat_to_int(lean_object*); @@ -77,17 +68,13 @@ LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofNanoseconds___boxed(lean_object* static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__23; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addNanoseconds___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_withHours(lean_object*, lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofNanoseconds(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toHours___boxed(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_midnight; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addMinutes___boxed(lean_object*, lean_object*); static lean_object* l_Std_Time_instInhabitedPlainTime___closed__18; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_withMilliseconds___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHSubOffset__2; -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35; -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43_(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addNanoseconds(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subMinutes(lean_object*, lean_object*); @@ -103,14 +90,12 @@ lean_object* lean_int_div(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__14; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__15; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addHours(lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano(uint8_t, lean_object*, lean_object*, lean_object*, lean_object*); +LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__7; LEAN_EXPORT lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMilliseconds(lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__21; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHSubOffset__3; -static lean_object* l_Std_Time_PlainTime_midnight___closed__1; static lean_object* l_Std_Time_instInhabitedPlainTime___closed__10; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMinutes(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHAddOffset__4; @@ -118,7 +103,6 @@ lean_object* lean_int_sub(lean_object*, lean_object*); static lean_object* l_Std_Time_instInhabitedPlainTime___closed__14; static lean_object* l_Std_Time_instInhabitedPlainTime___closed__4; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMilliseconds___boxed(lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_subHours(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_instHSubOffset__4; static lean_object* l_Std_Time_PlainTime_toMilliseconds___closed__2; @@ -129,13 +113,11 @@ static lean_object* l_Std_Time_PlainTime_instHAddOffset__3___closed__1; static lean_object* l_Std_Time_instInhabitedPlainTime___closed__15; static lean_object* l_Std_Time_PlainTime_instHSubOffset__1___closed__1; static lean_object* l_Std_Time_PlainTime_toSeconds___closed__1; -static lean_object* l_Std_Time_PlainTime_midnight___closed__2; static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__4; lean_object* lean_int_mul(lean_object*, lean_object*); lean_object* lean_string_length(lean_object*); static lean_object* l_Std_Time_instInhabitedPlainTime___closed__12; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_millisecond(lean_object*); -static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addMilliseconds(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofSeconds(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_PlainTime_addMilliseconds___boxed(lean_object*, lean_object*); @@ -159,7 +141,6 @@ LEAN_EXPORT lean_object* l_Std_Time_PlainTime_withMilliseconds(lean_object*, lea uint8_t lean_int_dec_eq(lean_object*, lean_object*); lean_object* lean_int_ediv(lean_object*, lean_object*); static lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__12; -static lean_object* l_Std_Time_instInhabitedPlainTime___closed__20; static lean_object* l_Std_Time_PlainTime_toMilliseconds___closed__4; lean_object* lean_int_neg(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_instInhabitedPlainTime; @@ -398,624 +379,228 @@ lean_ctor_set(x_2, 0, x_1); return x_2; } } -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked(", ", 2, 2); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("⟨", 3, 1); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27; -x_2 = lean_string_length(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28; -x_2 = lean_nat_to_int(x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("⟩", 3, 1); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("false", 5, 5); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34; -x_2 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26; -x_3 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36() { -_start: -{ -lean_object* x_1; -x_1 = lean_mk_string_unchecked("true", 4, 4); -return x_1; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37() { -_start: -{ -lean_object* x_1; lean_object* x_2; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36; -x_2 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} -} -static lean_object* _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; -x_1 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37; -x_2 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26; -x_3 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_3, 0, x_1); -lean_ctor_set(x_3, 1, x_2); -return x_3; -} -} LEAN_EXPORT lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43_(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; lean_object* x_9; uint8_t x_10; lean_object* x_11; +lean_object* x_3; lean_object* x_4; uint8_t x_5; lean_object* x_6; uint8_t x_7; lean_object* x_8; uint8_t x_9; lean_object* x_10; uint8_t x_11; lean_object* x_12; x_3 = lean_ctor_get(x_1, 0); -lean_inc(x_3); x_4 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; x_5 = lean_int_dec_lt(x_3, x_4); x_6 = lean_ctor_get(x_1, 1); -lean_inc(x_6); x_7 = lean_int_dec_lt(x_6, x_4); x_8 = lean_ctor_get(x_1, 2); -lean_inc(x_8); -x_9 = lean_ctor_get(x_1, 3); -lean_inc(x_9); -lean_dec(x_1); -x_10 = lean_int_dec_lt(x_9, x_4); +x_9 = lean_int_dec_lt(x_8, x_4); +x_10 = lean_ctor_get(x_1, 3); +x_11 = lean_int_dec_lt(x_10, x_4); if (x_5 == 0) { -lean_object* x_183; lean_object* x_184; -x_183 = l_Int_repr(x_3); -lean_dec(x_3); -x_184 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_184, 0, x_183); -x_11 = x_184; -goto block_182; +lean_object* x_89; lean_object* x_90; +x_89 = l_Int_repr(x_3); +x_90 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_90, 0, x_89); +x_12 = x_90; +goto block_88; } else { -lean_object* x_185; lean_object* x_186; lean_object* x_187; lean_object* x_188; -x_185 = l_Int_repr(x_3); -lean_dec(x_3); -x_186 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_186, 0, x_185); -x_187 = lean_unsigned_to_nat(0u); -x_188 = l_Repr_addAppParen(x_186, x_187); -x_11 = x_188; -goto block_182; -} -block_182: -{ -lean_object* x_12; lean_object* x_13; uint8_t x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; -x_12 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__7; -x_13 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_13, 0, x_12); -lean_ctor_set(x_13, 1, x_11); -x_14 = 0; -x_15 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_15, 0, x_13); -lean_ctor_set_uint8(x_15, sizeof(void*)*1, x_14); -x_16 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__6; -x_17 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_17, 0, x_16); -lean_ctor_set(x_17, 1, x_15); -x_18 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__10; -x_19 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_19, 0, x_17); -lean_ctor_set(x_19, 1, x_18); -x_20 = lean_box(1); -x_21 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_21, 0, x_19); -lean_ctor_set(x_21, 1, x_20); -x_22 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__12; -x_23 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_23, 0, x_21); -lean_ctor_set(x_23, 1, x_22); -x_24 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__5; -x_25 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_25, 0, x_23); -lean_ctor_set(x_25, 1, x_24); +lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; +x_91 = l_Int_repr(x_3); +x_92 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_92, 0, x_91); +x_93 = lean_unsigned_to_nat(0u); +x_94 = l_Repr_addAppParen(x_92, x_93); +x_12 = x_94; +goto block_88; +} +block_88: +{ +lean_object* x_13; lean_object* x_14; uint8_t x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; +x_13 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__7; +x_14 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_14, 0, x_13); +lean_ctor_set(x_14, 1, x_12); +x_15 = 0; +x_16 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_16, 0, x_14); +lean_ctor_set_uint8(x_16, sizeof(void*)*1, x_15); +x_17 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__6; +x_18 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_18, 0, x_17); +lean_ctor_set(x_18, 1, x_16); +x_19 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__10; +x_20 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_20, 0, x_18); +lean_ctor_set(x_20, 1, x_19); +x_21 = lean_box(1); +x_22 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_22, 0, x_20); +lean_ctor_set(x_22, 1, x_21); +x_23 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__12; +x_24 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_24, 0, x_22); +lean_ctor_set(x_24, 1, x_23); +x_25 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__5; +x_26 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_26, 0, x_24); +lean_ctor_set(x_26, 1, x_25); if (x_7 == 0) { -lean_object* x_176; lean_object* x_177; -x_176 = l_Int_repr(x_6); -lean_dec(x_6); -x_177 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_177, 0, x_176); -x_26 = x_177; -goto block_175; +lean_object* x_82; lean_object* x_83; +x_82 = l_Int_repr(x_6); +x_83 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_83, 0, x_82); +x_27 = x_83; +goto block_81; } else { -lean_object* x_178; lean_object* x_179; lean_object* x_180; lean_object* x_181; -x_178 = l_Int_repr(x_6); -lean_dec(x_6); -x_179 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_179, 0, x_178); -x_180 = lean_unsigned_to_nat(0u); -x_181 = l_Repr_addAppParen(x_179, x_180); -x_26 = x_181; -goto block_175; -} -block_175: -{ -lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; uint8_t x_74; -x_27 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__13; -x_28 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_28, 0, x_27); -lean_ctor_set(x_28, 1, x_26); -x_29 = lean_alloc_ctor(6, 1, 1); +lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; +x_84 = l_Int_repr(x_6); +x_85 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_85, 0, x_84); +x_86 = lean_unsigned_to_nat(0u); +x_87 = l_Repr_addAppParen(x_85, x_86); +x_27 = x_87; +goto block_81; +} +block_81: +{ +lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; +x_28 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__13; +x_29 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_29, 0, x_28); -lean_ctor_set_uint8(x_29, sizeof(void*)*1, x_14); -x_30 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_30, 0, x_25); -lean_ctor_set(x_30, 1, x_29); +lean_ctor_set(x_29, 1, x_27); +x_30 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_30, 0, x_29); +lean_ctor_set_uint8(x_30, sizeof(void*)*1, x_15); x_31 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_31, 0, x_30); -lean_ctor_set(x_31, 1, x_18); +lean_ctor_set(x_31, 0, x_26); +lean_ctor_set(x_31, 1, x_30); x_32 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_32, 0, x_31); -lean_ctor_set(x_32, 1, x_20); -x_33 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__15; -x_34 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_34, 0, x_32); -lean_ctor_set(x_34, 1, x_33); +lean_ctor_set(x_32, 1, x_19); +x_33 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_33, 0, x_32); +lean_ctor_set(x_33, 1, x_21); +x_34 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__15; x_35 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_35, 0, x_34); -lean_ctor_set(x_35, 1, x_24); -x_74 = !lean_is_exclusive(x_8); -if (x_74 == 0) -{ -lean_object* x_75; lean_object* x_76; uint8_t x_77; uint8_t x_78; -x_75 = lean_ctor_get(x_8, 0); -x_76 = lean_ctor_get(x_8, 1); -x_77 = lean_int_dec_lt(x_76, x_4); -x_78 = lean_unbox(x_75); -lean_dec(x_75); -if (x_78 == 0) -{ -if (x_77 == 0) -{ -lean_object* x_79; lean_object* x_80; lean_object* x_81; lean_object* x_82; lean_object* x_83; lean_object* x_84; lean_object* x_85; lean_object* x_86; lean_object* x_87; lean_object* x_88; -x_79 = l_Int_repr(x_76); -lean_dec(x_76); -x_80 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_80, 0, x_79); -x_81 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35; -lean_ctor_set_tag(x_8, 5); -lean_ctor_set(x_8, 1, x_80); -lean_ctor_set(x_8, 0, x_81); -x_82 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_83 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_83, 0, x_82); -lean_ctor_set(x_83, 1, x_8); -x_84 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_85 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_85, 0, x_83); -lean_ctor_set(x_85, 1, x_84); -x_86 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_87 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_87, 0, x_86); -lean_ctor_set(x_87, 1, x_85); -x_88 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_88, 0, x_87); -lean_ctor_set_uint8(x_88, sizeof(void*)*1, x_14); -x_36 = x_88; -goto block_73; -} -else -{ -lean_object* x_89; lean_object* x_90; lean_object* x_91; lean_object* x_92; lean_object* x_93; lean_object* x_94; lean_object* x_95; lean_object* x_96; lean_object* x_97; lean_object* x_98; lean_object* x_99; lean_object* x_100; -x_89 = l_Int_repr(x_76); -lean_dec(x_76); -x_90 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_90, 0, x_89); -x_91 = lean_unsigned_to_nat(0u); -x_92 = l_Repr_addAppParen(x_90, x_91); -x_93 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35; -lean_ctor_set_tag(x_8, 5); -lean_ctor_set(x_8, 1, x_92); -lean_ctor_set(x_8, 0, x_93); -x_94 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_95 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_95, 0, x_94); -lean_ctor_set(x_95, 1, x_8); -x_96 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_97 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_97, 0, x_95); -lean_ctor_set(x_97, 1, x_96); -x_98 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_99 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_99, 0, x_98); -lean_ctor_set(x_99, 1, x_97); -x_100 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_100, 0, x_99); -lean_ctor_set_uint8(x_100, sizeof(void*)*1, x_14); -x_36 = x_100; -goto block_73; -} -} -else -{ -if (x_77 == 0) -{ -lean_object* x_101; lean_object* x_102; lean_object* x_103; lean_object* x_104; lean_object* x_105; lean_object* x_106; lean_object* x_107; lean_object* x_108; lean_object* x_109; lean_object* x_110; -x_101 = l_Int_repr(x_76); -lean_dec(x_76); -x_102 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_102, 0, x_101); -x_103 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38; -lean_ctor_set_tag(x_8, 5); -lean_ctor_set(x_8, 1, x_102); -lean_ctor_set(x_8, 0, x_103); -x_104 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_105 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_105, 0, x_104); -lean_ctor_set(x_105, 1, x_8); -x_106 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_107 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_107, 0, x_105); -lean_ctor_set(x_107, 1, x_106); -x_108 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_109 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_109, 0, x_108); -lean_ctor_set(x_109, 1, x_107); -x_110 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_110, 0, x_109); -lean_ctor_set_uint8(x_110, sizeof(void*)*1, x_14); -x_36 = x_110; -goto block_73; -} -else -{ -lean_object* x_111; lean_object* x_112; lean_object* x_113; lean_object* x_114; lean_object* x_115; lean_object* x_116; lean_object* x_117; lean_object* x_118; lean_object* x_119; lean_object* x_120; lean_object* x_121; lean_object* x_122; -x_111 = l_Int_repr(x_76); -lean_dec(x_76); -x_112 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_112, 0, x_111); -x_113 = lean_unsigned_to_nat(0u); -x_114 = l_Repr_addAppParen(x_112, x_113); -x_115 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38; -lean_ctor_set_tag(x_8, 5); -lean_ctor_set(x_8, 1, x_114); -lean_ctor_set(x_8, 0, x_115); -x_116 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_117 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_117, 0, x_116); -lean_ctor_set(x_117, 1, x_8); -x_118 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_119 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_119, 0, x_117); -lean_ctor_set(x_119, 1, x_118); -x_120 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_121 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_121, 0, x_120); -lean_ctor_set(x_121, 1, x_119); -x_122 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_122, 0, x_121); -lean_ctor_set_uint8(x_122, sizeof(void*)*1, x_14); -x_36 = x_122; -goto block_73; -} -} -} -else -{ -lean_object* x_123; lean_object* x_124; uint8_t x_125; uint8_t x_126; -x_123 = lean_ctor_get(x_8, 0); -x_124 = lean_ctor_get(x_8, 1); -lean_inc(x_124); -lean_inc(x_123); -lean_dec(x_8); -x_125 = lean_int_dec_lt(x_124, x_4); -x_126 = lean_unbox(x_123); -lean_dec(x_123); -if (x_126 == 0) -{ -if (x_125 == 0) -{ -lean_object* x_127; lean_object* x_128; lean_object* x_129; lean_object* x_130; lean_object* x_131; lean_object* x_132; lean_object* x_133; lean_object* x_134; lean_object* x_135; lean_object* x_136; lean_object* x_137; -x_127 = l_Int_repr(x_124); -lean_dec(x_124); -x_128 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_128, 0, x_127); -x_129 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35; -x_130 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_130, 0, x_129); -lean_ctor_set(x_130, 1, x_128); -x_131 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_132 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_132, 0, x_131); -lean_ctor_set(x_132, 1, x_130); -x_133 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_134 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_134, 0, x_132); -lean_ctor_set(x_134, 1, x_133); -x_135 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_136 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_136, 0, x_135); -lean_ctor_set(x_136, 1, x_134); -x_137 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_137, 0, x_136); -lean_ctor_set_uint8(x_137, sizeof(void*)*1, x_14); -x_36 = x_137; -goto block_73; -} -else -{ -lean_object* x_138; lean_object* x_139; lean_object* x_140; lean_object* x_141; lean_object* x_142; lean_object* x_143; lean_object* x_144; lean_object* x_145; lean_object* x_146; lean_object* x_147; lean_object* x_148; lean_object* x_149; lean_object* x_150; -x_138 = l_Int_repr(x_124); -lean_dec(x_124); -x_139 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_139, 0, x_138); -x_140 = lean_unsigned_to_nat(0u); -x_141 = l_Repr_addAppParen(x_139, x_140); -x_142 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35; -x_143 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_143, 0, x_142); -lean_ctor_set(x_143, 1, x_141); -x_144 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_145 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_145, 0, x_144); -lean_ctor_set(x_145, 1, x_143); -x_146 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_147 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_147, 0, x_145); -lean_ctor_set(x_147, 1, x_146); -x_148 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_149 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_149, 0, x_148); -lean_ctor_set(x_149, 1, x_147); -x_150 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_150, 0, x_149); -lean_ctor_set_uint8(x_150, sizeof(void*)*1, x_14); -x_36 = x_150; -goto block_73; -} -} -else +lean_ctor_set(x_35, 0, x_33); +lean_ctor_set(x_35, 1, x_34); +x_36 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_36, 0, x_35); +lean_ctor_set(x_36, 1, x_25); +if (x_9 == 0) { -if (x_125 == 0) -{ -lean_object* x_151; lean_object* x_152; lean_object* x_153; lean_object* x_154; lean_object* x_155; lean_object* x_156; lean_object* x_157; lean_object* x_158; lean_object* x_159; lean_object* x_160; lean_object* x_161; -x_151 = l_Int_repr(x_124); -lean_dec(x_124); -x_152 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_152, 0, x_151); -x_153 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38; -x_154 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_154, 0, x_153); -lean_ctor_set(x_154, 1, x_152); -x_155 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_156 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_156, 0, x_155); -lean_ctor_set(x_156, 1, x_154); -x_157 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_158 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_158, 0, x_156); -lean_ctor_set(x_158, 1, x_157); -x_159 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_160 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_160, 0, x_159); -lean_ctor_set(x_160, 1, x_158); -x_161 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_161, 0, x_160); -lean_ctor_set_uint8(x_161, sizeof(void*)*1, x_14); -x_36 = x_161; -goto block_73; +lean_object* x_75; lean_object* x_76; +x_75 = l_Int_repr(x_8); +x_76 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_76, 0, x_75); +x_37 = x_76; +goto block_74; } else { -lean_object* x_162; lean_object* x_163; lean_object* x_164; lean_object* x_165; lean_object* x_166; lean_object* x_167; lean_object* x_168; lean_object* x_169; lean_object* x_170; lean_object* x_171; lean_object* x_172; lean_object* x_173; lean_object* x_174; -x_162 = l_Int_repr(x_124); -lean_dec(x_124); -x_163 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_163, 0, x_162); -x_164 = lean_unsigned_to_nat(0u); -x_165 = l_Repr_addAppParen(x_163, x_164); -x_166 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38; -x_167 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_167, 0, x_166); -lean_ctor_set(x_167, 1, x_165); -x_168 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30; -x_169 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_169, 0, x_168); -lean_ctor_set(x_169, 1, x_167); -x_170 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32; -x_171 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_171, 0, x_169); -lean_ctor_set(x_171, 1, x_170); -x_172 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29; -x_173 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_173, 0, x_172); -lean_ctor_set(x_173, 1, x_171); -x_174 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_174, 0, x_173); -lean_ctor_set_uint8(x_174, sizeof(void*)*1, x_14); -x_36 = x_174; -goto block_73; -} -} -} -block_73: -{ -lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; -x_37 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_37, 0, x_27); -lean_ctor_set(x_37, 1, x_36); -x_38 = lean_alloc_ctor(6, 1, 1); -lean_ctor_set(x_38, 0, x_37); -lean_ctor_set_uint8(x_38, sizeof(void*)*1, x_14); -x_39 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_39, 0, x_35); -lean_ctor_set(x_39, 1, x_38); +lean_object* x_77; lean_object* x_78; lean_object* x_79; lean_object* x_80; +x_77 = l_Int_repr(x_8); +x_78 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_78, 0, x_77); +x_79 = lean_unsigned_to_nat(0u); +x_80 = l_Repr_addAppParen(x_78, x_79); +x_37 = x_80; +goto block_74; +} +block_74: +{ +lean_object* x_38; lean_object* x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; lean_object* x_44; lean_object* x_45; +x_38 = lean_alloc_ctor(4, 2, 0); +lean_ctor_set(x_38, 0, x_28); +lean_ctor_set(x_38, 1, x_37); +x_39 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_39, 0, x_38); +lean_ctor_set_uint8(x_39, sizeof(void*)*1, x_15); x_40 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_40, 0, x_39); -lean_ctor_set(x_40, 1, x_18); +lean_ctor_set(x_40, 0, x_36); +lean_ctor_set(x_40, 1, x_39); x_41 = lean_alloc_ctor(5, 2, 0); lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_20); -x_42 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__17; -x_43 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_43, 0, x_41); -lean_ctor_set(x_43, 1, x_42); +lean_ctor_set(x_41, 1, x_19); +x_42 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_42, 0, x_41); +lean_ctor_set(x_42, 1, x_21); +x_43 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__17; x_44 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_44, 0, x_43); -lean_ctor_set(x_44, 1, x_24); -if (x_10 == 0) -{ -lean_object* x_45; lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; -x_45 = l_Int_repr(x_9); -lean_dec(x_9); -x_46 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_46, 0, x_45); -x_47 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__18; -x_48 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_48, 0, x_47); -lean_ctor_set(x_48, 1, x_46); -x_49 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_44, 0, x_42); +lean_ctor_set(x_44, 1, x_43); +x_45 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_45, 0, x_44); +lean_ctor_set(x_45, 1, x_25); +if (x_11 == 0) +{ +lean_object* x_46; lean_object* x_47; lean_object* x_48; lean_object* x_49; lean_object* x_50; lean_object* x_51; lean_object* x_52; lean_object* x_53; lean_object* x_54; lean_object* x_55; lean_object* x_56; lean_object* x_57; lean_object* x_58; +x_46 = l_Int_repr(x_10); +x_47 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_47, 0, x_46); +x_48 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__18; +x_49 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_49, 0, x_48); -lean_ctor_set_uint8(x_49, sizeof(void*)*1, x_14); -x_50 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_50, 0, x_44); -lean_ctor_set(x_50, 1, x_49); -x_51 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__22; -x_52 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_52, 0, x_51); -lean_ctor_set(x_52, 1, x_50); -x_53 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24; -x_54 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_54, 0, x_52); -lean_ctor_set(x_54, 1, x_53); -x_55 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__21; -x_56 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_56, 0, x_55); -lean_ctor_set(x_56, 1, x_54); -x_57 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_49, 1, x_47); +x_50 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_50, 0, x_49); +lean_ctor_set_uint8(x_50, sizeof(void*)*1, x_15); +x_51 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_51, 0, x_45); +lean_ctor_set(x_51, 1, x_50); +x_52 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__22; +x_53 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_53, 0, x_52); +lean_ctor_set(x_53, 1, x_51); +x_54 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24; +x_55 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_55, 0, x_53); +lean_ctor_set(x_55, 1, x_54); +x_56 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__21; +x_57 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_57, 0, x_56); -lean_ctor_set_uint8(x_57, sizeof(void*)*1, x_14); -return x_57; +lean_ctor_set(x_57, 1, x_55); +x_58 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_58, 0, x_57); +lean_ctor_set_uint8(x_58, sizeof(void*)*1, x_15); +return x_58; } else { -lean_object* x_58; lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; -x_58 = l_Int_repr(x_9); -lean_dec(x_9); -x_59 = lean_alloc_ctor(3, 1, 0); -lean_ctor_set(x_59, 0, x_58); -x_60 = lean_unsigned_to_nat(0u); -x_61 = l_Repr_addAppParen(x_59, x_60); -x_62 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__18; -x_63 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_63, 0, x_62); -lean_ctor_set(x_63, 1, x_61); -x_64 = lean_alloc_ctor(6, 1, 1); +lean_object* x_59; lean_object* x_60; lean_object* x_61; lean_object* x_62; lean_object* x_63; lean_object* x_64; lean_object* x_65; lean_object* x_66; lean_object* x_67; lean_object* x_68; lean_object* x_69; lean_object* x_70; lean_object* x_71; lean_object* x_72; lean_object* x_73; +x_59 = l_Int_repr(x_10); +x_60 = lean_alloc_ctor(3, 1, 0); +lean_ctor_set(x_60, 0, x_59); +x_61 = lean_unsigned_to_nat(0u); +x_62 = l_Repr_addAppParen(x_60, x_61); +x_63 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__18; +x_64 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_64, 0, x_63); -lean_ctor_set_uint8(x_64, sizeof(void*)*1, x_14); -x_65 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_65, 0, x_44); -lean_ctor_set(x_65, 1, x_64); -x_66 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__22; -x_67 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_67, 0, x_66); -lean_ctor_set(x_67, 1, x_65); -x_68 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24; -x_69 = lean_alloc_ctor(5, 2, 0); -lean_ctor_set(x_69, 0, x_67); -lean_ctor_set(x_69, 1, x_68); -x_70 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__21; -x_71 = lean_alloc_ctor(4, 2, 0); -lean_ctor_set(x_71, 0, x_70); -lean_ctor_set(x_71, 1, x_69); -x_72 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_64, 1, x_62); +x_65 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_65, 0, x_64); +lean_ctor_set_uint8(x_65, sizeof(void*)*1, x_15); +x_66 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_66, 0, x_45); +lean_ctor_set(x_66, 1, x_65); +x_67 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__22; +x_68 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_68, 0, x_67); +lean_ctor_set(x_68, 1, x_66); +x_69 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24; +x_70 = lean_alloc_ctor(5, 2, 0); +lean_ctor_set(x_70, 0, x_68); +lean_ctor_set(x_70, 1, x_69); +x_71 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__21; +x_72 = lean_alloc_ctor(4, 2, 0); lean_ctor_set(x_72, 0, x_71); -lean_ctor_set_uint8(x_72, sizeof(void*)*1, x_14); -return x_72; +lean_ctor_set(x_72, 1, x_70); +x_73 = lean_alloc_ctor(6, 1, 1); +lean_ctor_set(x_73, 0, x_72); +lean_ctor_set_uint8(x_73, sizeof(void*)*1, x_15); +return x_73; } } } @@ -1028,6 +613,7 @@ LEAN_EXPORT lean_object* l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPla lean_object* x_3; x_3 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43_(x_1, x_2); lean_dec(x_2); +lean_dec(x_1); return x_3; } } @@ -1226,37 +812,23 @@ return x_3; static lean_object* _init_l_Std_Time_instInhabitedPlainTime___closed__19() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Std_Time_instInhabitedPlainTime___closed__10; x_2 = l_Std_Time_instInhabitedPlainTime___closed__18; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); +x_3 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; +x_4 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_3); return x_4; } } -static lean_object* _init_l_Std_Time_instInhabitedPlainTime___closed__20() { -_start: -{ -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Time_instInhabitedPlainTime___closed__10; -x_2 = l_Std_Time_instInhabitedPlainTime___closed__18; -x_3 = l_Std_Time_instInhabitedPlainTime___closed__19; -x_4 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} -} static lean_object* _init_l_Std_Time_instInhabitedPlainTime() { _start: { lean_object* x_1; -x_1 = l_Std_Time_instInhabitedPlainTime___closed__20; +x_1 = l_Std_Time_instInhabitedPlainTime___closed__19; return x_1; } } @@ -1287,25 +859,23 @@ return x_10; } else { -lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; uint8_t x_15; +lean_object* x_11; lean_object* x_12; uint8_t x_13; x_11 = lean_ctor_get(x_1, 2); -x_12 = lean_ctor_get(x_11, 1); -x_13 = lean_ctor_get(x_2, 2); -x_14 = lean_ctor_get(x_13, 1); -x_15 = lean_int_dec_eq(x_12, x_14); -if (x_15 == 0) -{ -uint8_t x_16; -x_16 = 0; -return x_16; +x_12 = lean_ctor_get(x_2, 2); +x_13 = lean_int_dec_eq(x_11, x_12); +if (x_13 == 0) +{ +uint8_t x_14; +x_14 = 0; +return x_14; } else { -lean_object* x_17; lean_object* x_18; uint8_t x_19; -x_17 = lean_ctor_get(x_1, 3); -x_18 = lean_ctor_get(x_2, 3); -x_19 = lean_int_dec_eq(x_17, x_18); -return x_19; +lean_object* x_15; lean_object* x_16; uint8_t x_17; +x_15 = lean_ctor_get(x_1, 3); +x_16 = lean_ctor_get(x_2, 3); +x_17 = lean_int_dec_eq(x_15, x_16); +return x_17; } } } @@ -1322,27 +892,18 @@ x_4 = lean_box(x_3); return x_4; } } -static lean_object* _init_l_Std_Time_PlainTime_midnight___closed__1() { +static lean_object* _init_l_Std_Time_PlainTime_midnight() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 1; -x_2 = l_Std_Time_instInhabitedPlainTime___closed__18; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); -lean_ctor_set(x_4, 1, x_2); -return x_4; +lean_object* x_1; +x_1 = l_Std_Time_instInhabitedPlainTime___closed__19; +return x_1; } } -static lean_object* _init_l_Std_Time_PlainTime_midnight___closed__2() { +LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Time_instInhabitedPlainTime___closed__10; -x_2 = l_Std_Time_instInhabitedPlainTime___closed__18; -x_3 = l_Std_Time_PlainTime_midnight___closed__1; -x_4 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; +lean_object* x_5; x_5 = lean_alloc_ctor(0, 4, 0); lean_ctor_set(x_5, 0, x_1); lean_ctor_set(x_5, 1, x_2); @@ -1351,65 +912,17 @@ lean_ctor_set(x_5, 3, x_4); return x_5; } } -static lean_object* _init_l_Std_Time_PlainTime_midnight() { -_start: -{ -lean_object* x_1; -x_1 = l_Std_Time_PlainTime_midnight___closed__2; -return x_1; -} -} -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_6 = lean_box(x_1); -x_7 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_7, 0, x_6); -lean_ctor_set(x_7, 1, x_4); -x_8 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_8, 0, x_2); -lean_ctor_set(x_8, 1, x_3); -lean_ctor_set(x_8, 2, x_7); -lean_ctor_set(x_8, 3, x_5); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSecondsNano___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4, lean_object* x_5) { -_start: -{ -uint8_t x_6; lean_object* x_7; -x_6 = lean_unbox(x_1); -lean_dec(x_1); -x_7 = l_Std_Time_PlainTime_ofHourMinuteSecondsNano(x_6, x_2, x_3, x_4, x_5); -return x_7; -} -} -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds(uint8_t x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { -_start: -{ -lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; -x_5 = lean_box(x_1); -x_6 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_6, 0, x_5); -lean_ctor_set(x_6, 1, x_4); -x_7 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; -x_8 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_8, 0, x_2); -lean_ctor_set(x_8, 1, x_3); -lean_ctor_set(x_8, 2, x_6); -lean_ctor_set(x_8, 3, x_7); -return x_8; -} -} -LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3, lean_object* x_4) { +LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofHourMinuteSeconds(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -uint8_t x_5; lean_object* x_6; -x_5 = lean_unbox(x_1); -lean_dec(x_1); -x_6 = l_Std_Time_PlainTime_ofHourMinuteSeconds(x_5, x_2, x_3, x_4); -return x_6; +lean_object* x_4; lean_object* x_5; +x_4 = l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__8; +x_5 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_5, 0, x_1); +lean_ctor_set(x_5, 1, x_2); +lean_ctor_set(x_5, 2, x_3); +lean_ctor_set(x_5, 3, x_4); +return x_5; } } static lean_object* _init_l_Std_Time_PlainTime_toMilliseconds___closed__1() { @@ -1451,7 +964,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMilliseconds(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; x_2 = lean_ctor_get(x_1, 0); x_3 = l_Std_Time_PlainTime_toMilliseconds___closed__1; x_4 = lean_int_mul(x_2, x_3); @@ -1462,19 +975,18 @@ x_8 = lean_int_add(x_4, x_7); lean_dec(x_7); lean_dec(x_4); x_9 = lean_ctor_get(x_1, 2); -x_10 = lean_ctor_get(x_9, 1); -x_11 = l_Std_Time_PlainTime_toMilliseconds___closed__3; -x_12 = lean_int_mul(x_10, x_11); -x_13 = lean_int_add(x_8, x_12); -lean_dec(x_12); +x_10 = l_Std_Time_PlainTime_toMilliseconds___closed__3; +x_11 = lean_int_mul(x_9, x_10); +x_12 = lean_int_add(x_8, x_11); +lean_dec(x_11); lean_dec(x_8); -x_14 = lean_ctor_get(x_1, 3); -x_15 = l_Std_Time_PlainTime_toMilliseconds___closed__4; -x_16 = lean_int_div(x_14, x_15); -x_17 = lean_int_add(x_13, x_16); -lean_dec(x_16); -lean_dec(x_13); -return x_17; +x_13 = lean_ctor_get(x_1, 3); +x_14 = l_Std_Time_PlainTime_toMilliseconds___closed__4; +x_15 = lean_int_div(x_13, x_14); +x_16 = lean_int_add(x_12, x_15); +lean_dec(x_15); +lean_dec(x_12); +return x_16; } } LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMilliseconds___boxed(lean_object* x_1) { @@ -1516,7 +1028,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toNanoseconds(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; x_2 = lean_ctor_get(x_1, 0); x_3 = l_Std_Time_PlainTime_toNanoseconds___closed__1; x_4 = lean_int_mul(x_2, x_3); @@ -1527,16 +1039,15 @@ x_8 = lean_int_add(x_4, x_7); lean_dec(x_7); lean_dec(x_4); x_9 = lean_ctor_get(x_1, 2); -x_10 = lean_ctor_get(x_9, 1); -x_11 = l_Std_Time_PlainTime_toNanoseconds___closed__3; -x_12 = lean_int_mul(x_10, x_11); -x_13 = lean_int_add(x_8, x_12); -lean_dec(x_12); +x_10 = l_Std_Time_PlainTime_toNanoseconds___closed__3; +x_11 = lean_int_mul(x_9, x_10); +x_12 = lean_int_add(x_8, x_11); +lean_dec(x_11); lean_dec(x_8); -x_14 = lean_ctor_get(x_1, 3); -x_15 = lean_int_add(x_13, x_14); -lean_dec(x_13); -return x_15; +x_13 = lean_ctor_get(x_1, 3); +x_14 = lean_int_add(x_12, x_13); +lean_dec(x_12); +return x_14; } } LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toNanoseconds___boxed(lean_object* x_1) { @@ -1569,7 +1080,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toSeconds(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; x_2 = lean_ctor_get(x_1, 0); x_3 = l_Std_Time_PlainTime_toSeconds___closed__1; x_4 = lean_int_mul(x_2, x_3); @@ -1580,10 +1091,9 @@ x_8 = lean_int_add(x_4, x_7); lean_dec(x_7); lean_dec(x_4); x_9 = lean_ctor_get(x_1, 2); -x_10 = lean_ctor_get(x_9, 1); -x_11 = lean_int_add(x_8, x_10); +x_10 = lean_int_add(x_8, x_9); lean_dec(x_8); -return x_11; +return x_10; } } LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toSeconds___boxed(lean_object* x_1) { @@ -1598,7 +1108,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMinutes(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; x_2 = lean_ctor_get(x_1, 0); x_3 = l_Std_Time_PlainTime_toSeconds___closed__2; x_4 = lean_int_mul(x_2, x_3); @@ -1606,12 +1116,11 @@ x_5 = lean_ctor_get(x_1, 1); x_6 = lean_int_add(x_4, x_5); lean_dec(x_4); x_7 = lean_ctor_get(x_1, 2); -x_8 = lean_ctor_get(x_7, 1); -x_9 = lean_int_div(x_8, x_3); -x_10 = lean_int_add(x_6, x_9); -lean_dec(x_9); +x_8 = lean_int_div(x_7, x_3); +x_9 = lean_int_add(x_6, x_8); +lean_dec(x_8); lean_dec(x_6); -return x_10; +return x_9; } } LEAN_EXPORT lean_object* l_Std_Time_PlainTime_toMinutes___boxed(lean_object* x_1) { @@ -1653,7 +1162,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofNanoseconds(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; uint8_t x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; x_2 = l_Std_Time_PlainTime_toNanoseconds___closed__3; x_3 = lean_int_ediv(x_1, x_2); x_4 = lean_int_emod(x_1, x_2); @@ -1668,17 +1177,12 @@ x_11 = lean_int_ediv(x_9, x_10); lean_dec(x_9); x_12 = lean_int_emod(x_3, x_10); lean_dec(x_3); -x_13 = 0; -x_14 = lean_box(x_13); -x_15 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_15, 0, x_14); -lean_ctor_set(x_15, 1, x_12); -x_16 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_16, 0, x_8); -lean_ctor_set(x_16, 1, x_11); -lean_ctor_set(x_16, 2, x_15); -lean_ctor_set(x_16, 3, x_4); -return x_16; +x_13 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_13, 0, x_8); +lean_ctor_set(x_13, 1, x_11); +lean_ctor_set(x_13, 2, x_12); +lean_ctor_set(x_13, 3, x_4); +return x_13; } } LEAN_EXPORT lean_object* l_Std_Time_PlainTime_ofNanoseconds___boxed(lean_object* x_1) { @@ -2435,34 +1939,6 @@ l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Ti lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__23); l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24(); lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__24); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__25); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__26); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__27); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__28); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__29); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__30); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__31); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__32); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__33); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__34); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__35); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__36); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__37); -l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38 = _init_l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38(); -lean_mark_persistent(l___private_Std_Time_Time_PlainTime_0__Std_Time_reprPlainTime____x40_Std_Time_Time_PlainTime___hyg_43____closed__38); l_Std_Time_instReprPlainTime___closed__1 = _init_l_Std_Time_instReprPlainTime___closed__1(); lean_mark_persistent(l_Std_Time_instReprPlainTime___closed__1); l_Std_Time_instReprPlainTime = _init_l_Std_Time_instReprPlainTime(); @@ -2505,14 +1981,8 @@ l_Std_Time_instInhabitedPlainTime___closed__18 = _init_l_Std_Time_instInhabitedP lean_mark_persistent(l_Std_Time_instInhabitedPlainTime___closed__18); l_Std_Time_instInhabitedPlainTime___closed__19 = _init_l_Std_Time_instInhabitedPlainTime___closed__19(); lean_mark_persistent(l_Std_Time_instInhabitedPlainTime___closed__19); -l_Std_Time_instInhabitedPlainTime___closed__20 = _init_l_Std_Time_instInhabitedPlainTime___closed__20(); -lean_mark_persistent(l_Std_Time_instInhabitedPlainTime___closed__20); l_Std_Time_instInhabitedPlainTime = _init_l_Std_Time_instInhabitedPlainTime(); lean_mark_persistent(l_Std_Time_instInhabitedPlainTime); -l_Std_Time_PlainTime_midnight___closed__1 = _init_l_Std_Time_PlainTime_midnight___closed__1(); -lean_mark_persistent(l_Std_Time_PlainTime_midnight___closed__1); -l_Std_Time_PlainTime_midnight___closed__2 = _init_l_Std_Time_PlainTime_midnight___closed__2(); -lean_mark_persistent(l_Std_Time_PlainTime_midnight___closed__2); l_Std_Time_PlainTime_midnight = _init_l_Std_Time_PlainTime_midnight(); lean_mark_persistent(l_Std_Time_PlainTime_midnight); l_Std_Time_PlainTime_toMilliseconds___closed__1 = _init_l_Std_Time_PlainTime_toMilliseconds___closed__1(); diff --git a/stage0/stdlib/Std/Time/Zoned/Database/TZdb.c b/stage0/stdlib/Std/Time/Zoned/Database/TZdb.c index 23047a341596..f04956a28027 100644 --- a/stage0/stdlib/Std/Time/Zoned/Database/TZdb.c +++ b/stage0/stdlib/Std/Time/Zoned/Database/TZdb.c @@ -34,19 +34,16 @@ LEAN_EXPORT lean_object* l___private_Init_Data_Option_Basic_0__Option_decEqOptio static lean_object* l_Std_Time_Database_TZdb_inst___closed__2; LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst; LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_Time_Database_TZdb_inst___spec__1___boxed(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, lean_object*); -LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_parseTZIfFromDisk___closed__2; LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst___lambda__1___boxed(lean_object*, lean_object*, lean_object*); LEAN_EXPORT uint8_t l___private_Init_Data_Option_Basic_0__Option_decEqOption____x40_Init_Data_Option_Basic___hyg_4____at_Std_Time_Database_TZdb_idFromPath___spec__1(lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_inst___lambda__1___closed__2; static lean_object* l_Std_Time_Database_TZdb_parseTZIfFromDisk___closed__1; static lean_object* l_Std_Time_Database_TZdb_default___closed__4; -static lean_object* l_Std_Time_Database_TZdb_localRules___closed__3; lean_object* l_Std_Time_TimeZone_convertTZif(lean_object*, lean_object*); lean_object* l_System_FilePath_components(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_parseTZIfFromDisk___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_default___closed__10; -static lean_object* l_Std_Time_Database_TZdb_localRules___closed__5; static lean_object* l_Std_Time_Database_TZdb_default___closed__11; static lean_object* l_Std_Time_Database_TZdb_default___closed__7; static lean_object* l_Std_Time_Database_TZdb_parseTZif___closed__1; @@ -56,13 +53,12 @@ static lean_object* l_Std_Time_Database_TZdb_default___closed__1; static lean_object* l_Std_Time_Database_TZdb_default___closed__8; static lean_object* l_Std_Time_Database_TZdb_inst___lambda__3___closed__1; lean_object* l_Substring_takeWhileAux___at_Substring_trimLeft___spec__1(lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst___lambda__2___boxed(lean_object*, lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_localRules___closed__1; lean_object* l_Substring_takeRightWhileAux___at_Substring_trimRight___spec__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_IO_ofExcept___at_Std_Time_Database_TZdb_parseTZIfFromDisk___spec__1(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst___lambda__2(lean_object*, lean_object*, lean_object*, lean_object*); -static lean_object* l_Std_Time_Database_TZdb_localRules___closed__4; +lean_object* lean_io_realpath(lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_inst___lambda__1___closed__1; LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_idFromPath(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_parseTZIfFromDisk___lambda__1(lean_object*, lean_object*, lean_object*); @@ -70,7 +66,6 @@ static lean_object* l_Std_Time_Database_TZdb_default___closed__5; static lean_object* l_Std_Time_Database_TZdb_inst___closed__1; lean_object* lean_nat_sub(lean_object*, lean_object*); lean_object* lean_array_mk(lean_object*); -static lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2; size_t lean_usize_add(size_t, size_t); static lean_object* l_Std_Time_Database_TZdb_parseTZIfFromDisk___closed__3; static lean_object* l_Std_Time_Database_TZdb_default___closed__2; @@ -78,15 +73,12 @@ lean_object* lean_array_uget(lean_object*, size_t); size_t lean_array_size(lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_readRulesFromDisk(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_default___closed__3; -static lean_object* l_Std_Time_Database_TZdb_localRules___closed__6; lean_object* lean_string_append(lean_object*, lean_object*); lean_object* lean_array_get_size(lean_object*); uint8_t lean_usize_dec_lt(size_t, size_t); -LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1___boxed(lean_object*, lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_default___closed__6; lean_object* l_IO_FS_readBinFile(lean_object*, lean_object*); static lean_object* l_Std_Time_Database_TZdb_idFromPath___closed__3; -lean_object* l_IO_Process_run(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Array_forIn_x27Unsafe_loop___at_Std_Time_Database_TZdb_inst___spec__1(lean_object*, lean_object*, lean_object*, lean_object*, lean_object*, size_t, size_t, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst___lambda__1(lean_object*, lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_inst___lambda__4(lean_object*, lean_object*); @@ -713,7 +705,7 @@ x_4 = lean_box(x_3); return x_4; } } -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1() { +static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__1() { _start: { lean_object* x_1; @@ -721,171 +713,107 @@ x_1 = lean_mk_string_unchecked("cannot read the id of the path.", 31, 31); return x_1; } } -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2() { +static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__2() { _start: { lean_object* x_1; lean_object* x_2; -x_1 = l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1; +x_1 = l_Std_Time_Database_TZdb_localRules___closed__1; x_2 = lean_alloc_ctor(18, 1, 0); lean_ctor_set(x_2, 0, x_1); return x_2; } } -LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { +LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules(lean_object* x_1, lean_object* x_2) { _start: { -lean_object* x_4; -x_4 = l_Std_Time_Database_TZdb_idFromPath(x_2); -if (lean_obj_tag(x_4) == 0) -{ -lean_object* x_5; lean_object* x_6; -x_5 = l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2; -x_6 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_6, 0, x_5); -lean_ctor_set(x_6, 1, x_3); -return x_6; -} -else -{ -lean_object* x_7; lean_object* x_8; -x_7 = lean_ctor_get(x_4, 0); -lean_inc(x_7); -lean_dec(x_4); -x_8 = l_Std_Time_Database_TZdb_parseTZIfFromDisk(x_1, x_7, x_3); -return x_8; -} -} -} -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__1() { -_start: +lean_object* x_3; +lean_inc(x_1); +x_3 = lean_io_realpath(x_1, x_2); +if (lean_obj_tag(x_3) == 0) { -uint8_t x_1; lean_object* x_2; -x_1 = 1; -x_2 = lean_alloc_ctor(0, 0, 3); -lean_ctor_set_uint8(x_2, 0, x_1); -lean_ctor_set_uint8(x_2, 1, x_1); -lean_ctor_set_uint8(x_2, 2, x_1); -return x_2; -} -} -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__2() { -_start: +uint8_t x_4; +x_4 = !lean_is_exclusive(x_3); +if (x_4 == 0) { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("-f", 2, 2); -return x_1; -} -} -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__3() { -_start: +lean_object* x_5; lean_object* x_6; lean_object* x_7; +x_5 = lean_ctor_get(x_3, 0); +x_6 = lean_ctor_get(x_3, 1); +x_7 = l_Std_Time_Database_TZdb_idFromPath(x_5); +if (lean_obj_tag(x_7) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = lean_box(0); -x_2 = lean_array_mk(x_1); -return x_2; -} +lean_object* x_8; +lean_dec(x_1); +x_8 = l_Std_Time_Database_TZdb_localRules___closed__2; +lean_ctor_set_tag(x_3, 1); +lean_ctor_set(x_3, 0, x_8); +return x_3; } -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__4() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("readlink", 8, 8); -return x_1; +lean_object* x_9; lean_object* x_10; +lean_free_object(x_3); +x_9 = lean_ctor_get(x_7, 0); +lean_inc(x_9); +lean_dec(x_7); +x_10 = l_Std_Time_Database_TZdb_parseTZIfFromDisk(x_1, x_9, x_6); +lean_dec(x_1); +return x_10; } } -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__5() { -_start: +else { -lean_object* x_1; -x_1 = lean_mk_string_unchecked("cannot find the local timezone database", 39, 39); -return x_1; -} -} -static lean_object* _init_l_Std_Time_Database_TZdb_localRules___closed__6() { -_start: +lean_object* x_11; lean_object* x_12; lean_object* x_13; +x_11 = lean_ctor_get(x_3, 0); +x_12 = lean_ctor_get(x_3, 1); +lean_inc(x_12); +lean_inc(x_11); +lean_dec(x_3); +x_13 = l_Std_Time_Database_TZdb_idFromPath(x_11); +if (lean_obj_tag(x_13) == 0) { -lean_object* x_1; lean_object* x_2; -x_1 = l_Std_Time_Database_TZdb_localRules___closed__5; -x_2 = lean_alloc_ctor(18, 1, 0); -lean_ctor_set(x_2, 0, x_1); -return x_2; -} +lean_object* x_14; lean_object* x_15; +lean_dec(x_1); +x_14 = l_Std_Time_Database_TZdb_localRules___closed__2; +x_15 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_15, 0, x_14); +lean_ctor_set(x_15, 1, x_12); +return x_15; } -LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules(lean_object* x_1, lean_object* x_2) { -_start: +else { -lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; uint8_t x_12; lean_object* x_13; lean_object* x_14; -x_3 = lean_box(0); -lean_inc(x_1); -x_4 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_4, 0, x_1); -lean_ctor_set(x_4, 1, x_3); -x_5 = l_Std_Time_Database_TZdb_localRules___closed__2; -x_6 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_6, 0, x_5); -lean_ctor_set(x_6, 1, x_4); -x_7 = lean_array_mk(x_6); -x_8 = lean_box(0); -x_9 = l_Std_Time_Database_TZdb_localRules___closed__1; -x_10 = l_Std_Time_Database_TZdb_localRules___closed__4; -x_11 = l_Std_Time_Database_TZdb_localRules___closed__3; -x_12 = 0; -x_13 = lean_alloc_ctor(0, 5, 1); -lean_ctor_set(x_13, 0, x_9); -lean_ctor_set(x_13, 1, x_10); -lean_ctor_set(x_13, 2, x_7); -lean_ctor_set(x_13, 3, x_8); -lean_ctor_set(x_13, 4, x_11); -lean_ctor_set_uint8(x_13, sizeof(void*)*5, x_12); -x_14 = l_IO_Process_run(x_13, x_2); -if (lean_obj_tag(x_14) == 0) -{ -lean_object* x_15; lean_object* x_16; lean_object* x_17; -x_15 = lean_ctor_get(x_14, 0); -lean_inc(x_15); -x_16 = lean_ctor_get(x_14, 1); +lean_object* x_16; lean_object* x_17; +x_16 = lean_ctor_get(x_13, 0); lean_inc(x_16); -lean_dec(x_14); -x_17 = l_Std_Time_Database_TZdb_localRules___lambda__1(x_1, x_15, x_16); +lean_dec(x_13); +x_17 = l_Std_Time_Database_TZdb_parseTZIfFromDisk(x_1, x_16, x_12); lean_dec(x_1); return x_17; } +} +} else { uint8_t x_18; lean_dec(x_1); -x_18 = !lean_is_exclusive(x_14); +x_18 = !lean_is_exclusive(x_3); if (x_18 == 0) { -lean_object* x_19; lean_object* x_20; -x_19 = lean_ctor_get(x_14, 0); -lean_dec(x_19); -x_20 = l_Std_Time_Database_TZdb_localRules___closed__6; -lean_ctor_set(x_14, 0, x_20); -return x_14; +return x_3; } else { -lean_object* x_21; lean_object* x_22; lean_object* x_23; -x_21 = lean_ctor_get(x_14, 1); -lean_inc(x_21); -lean_dec(x_14); -x_22 = l_Std_Time_Database_TZdb_localRules___closed__6; -x_23 = lean_alloc_ctor(1, 2, 0); -lean_ctor_set(x_23, 0, x_22); -lean_ctor_set(x_23, 1, x_21); -return x_23; -} -} +lean_object* x_19; lean_object* x_20; lean_object* x_21; +x_19 = lean_ctor_get(x_3, 0); +x_20 = lean_ctor_get(x_3, 1); +lean_inc(x_20); +lean_inc(x_19); +lean_dec(x_3); +x_21 = lean_alloc_ctor(1, 2, 0); +lean_ctor_set(x_21, 0, x_19); +lean_ctor_set(x_21, 1, x_20); +return x_21; } } -LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_localRules___lambda__1___boxed(lean_object* x_1, lean_object* x_2, lean_object* x_3) { -_start: -{ -lean_object* x_4; -x_4 = l_Std_Time_Database_TZdb_localRules___lambda__1(x_1, x_2, x_3); -lean_dec(x_1); -return x_4; } } LEAN_EXPORT lean_object* l_Std_Time_Database_TZdb_readRulesFromDisk(lean_object* x_1, lean_object* x_2, lean_object* x_3) { @@ -1444,22 +1372,10 @@ l_Std_Time_Database_TZdb_idFromPath___closed__2 = _init_l_Std_Time_Database_TZdb lean_mark_persistent(l_Std_Time_Database_TZdb_idFromPath___closed__2); l_Std_Time_Database_TZdb_idFromPath___closed__3 = _init_l_Std_Time_Database_TZdb_idFromPath___closed__3(); lean_mark_persistent(l_Std_Time_Database_TZdb_idFromPath___closed__3); -l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1 = _init_l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___lambda__1___closed__1); -l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2 = _init_l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___lambda__1___closed__2); l_Std_Time_Database_TZdb_localRules___closed__1 = _init_l_Std_Time_Database_TZdb_localRules___closed__1(); lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__1); l_Std_Time_Database_TZdb_localRules___closed__2 = _init_l_Std_Time_Database_TZdb_localRules___closed__2(); lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__2); -l_Std_Time_Database_TZdb_localRules___closed__3 = _init_l_Std_Time_Database_TZdb_localRules___closed__3(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__3); -l_Std_Time_Database_TZdb_localRules___closed__4 = _init_l_Std_Time_Database_TZdb_localRules___closed__4(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__4); -l_Std_Time_Database_TZdb_localRules___closed__5 = _init_l_Std_Time_Database_TZdb_localRules___closed__5(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__5); -l_Std_Time_Database_TZdb_localRules___closed__6 = _init_l_Std_Time_Database_TZdb_localRules___closed__6(); -lean_mark_persistent(l_Std_Time_Database_TZdb_localRules___closed__6); l_Std_Time_Database_TZdb_inst___lambda__1___closed__1 = _init_l_Std_Time_Database_TZdb_inst___lambda__1___closed__1(); lean_mark_persistent(l_Std_Time_Database_TZdb_inst___lambda__1___closed__1); l_Std_Time_Database_TZdb_inst___lambda__1___closed__2 = _init_l_Std_Time_Database_TZdb_inst___lambda__1___closed__2(); diff --git a/stage0/stdlib/Std/Time/Zoned/DateTime.c b/stage0/stdlib/Std/Time/Zoned/DateTime.c index ec181064ae6a..74d18516db72 100644 --- a/stage0/stdlib/Std/Time/Zoned/DateTime.c +++ b/stage0/stdlib/Std/Time/Zoned/DateTime.c @@ -340,7 +340,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_instInhabitedDateTime___lambda__1(lean_object* x_1, lean_object* x_2, lean_object* x_3) { _start: { -lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; uint8_t x_39; lean_object* x_40; lean_object* x_41; lean_object* x_42; lean_object* x_43; +lean_object* x_4; lean_object* x_5; lean_object* x_6; lean_object* x_7; lean_object* x_8; lean_object* x_9; lean_object* x_10; lean_object* x_11; lean_object* x_12; lean_object* x_13; lean_object* x_14; lean_object* x_15; lean_object* x_16; lean_object* x_17; lean_object* x_18; lean_object* x_19; lean_object* x_20; lean_object* x_21; lean_object* x_22; lean_object* x_23; lean_object* x_24; lean_object* x_25; lean_object* x_26; lean_object* x_27; lean_object* x_28; lean_object* x_29; lean_object* x_30; lean_object* x_31; lean_object* x_32; lean_object* x_33; lean_object* x_34; lean_object* x_35; lean_object* x_36; lean_object* x_37; lean_object* x_38; lean_object* x_39; lean_object* x_40; x_4 = l_Std_Time_instInhabitedDateTime___lambda__1___closed__1; x_5 = lean_int_add(x_1, x_4); x_6 = lean_int_sub(x_5, x_1); @@ -406,21 +406,16 @@ lean_dec(x_34); lean_dec(x_36); x_38 = lean_int_add(x_37, x_2); lean_dec(x_37); -x_39 = 0; -x_40 = lean_box(x_39); lean_inc(x_38); -x_41 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_41, 0, x_40); -lean_ctor_set(x_41, 1, x_38); -x_42 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_42, 0, x_30); -lean_ctor_set(x_42, 1, x_38); -lean_ctor_set(x_42, 2, x_41); -lean_ctor_set(x_42, 3, x_2); -x_43 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_43, 0, x_21); -lean_ctor_set(x_43, 1, x_42); -return x_43; +x_39 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_39, 0, x_30); +lean_ctor_set(x_39, 1, x_38); +lean_ctor_set(x_39, 2, x_38); +lean_ctor_set(x_39, 3, x_2); +x_40 = lean_alloc_ctor(0, 2, 0); +lean_ctor_set(x_40, 0, x_21); +lean_ctor_set(x_40, 1, x_39); +return x_40; } } static lean_object* _init_l_Std_Time_instInhabitedDateTime___closed__1() { @@ -6402,7 +6397,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_DateTime_second___rarg(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_2 = lean_ctor_get(x_1, 1); x_3 = lean_thunk_get_own(x_2); x_4 = lean_ctor_get(x_3, 1); @@ -6411,10 +6406,7 @@ lean_dec(x_3); x_5 = lean_ctor_get(x_4, 2); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -return x_6; +return x_5; } } LEAN_EXPORT lean_object* l_Std_Time_DateTime_second(lean_object* x_1) { diff --git a/stage0/stdlib/Std/Time/Zoned/ZonedDateTime.c b/stage0/stdlib/Std/Time/Zoned/ZonedDateTime.c index f209ef13199b..4c9f61dba1cb 100644 --- a/stage0/stdlib/Std/Time/Zoned/ZonedDateTime.c +++ b/stage0/stdlib/Std/Time/Zoned/ZonedDateTime.c @@ -250,7 +250,6 @@ LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_instHAddOffset__3; LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_subWeeks___boxed(lean_object*, lean_object*); LEAN_EXPORT uint8_t l_Std_Time_ZonedDateTime_era(lean_object*); lean_object* l_Std_Time_PlainDate_ofDaysSinceUNIXEpoch(lean_object*); -static lean_object* l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40; LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_withDaysRollOver___boxed(lean_object*, lean_object*); LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_subNanoseconds(lean_object*, lean_object*); lean_object* lean_int_ediv(lean_object*, lean_object*); @@ -652,38 +651,24 @@ return x_3; static lean_object* _init_l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__38() { _start: { -uint8_t x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; -x_1 = 0; +lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; +x_1 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__29; x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__37; -x_3 = lean_box(x_1); -x_4 = lean_alloc_ctor(0, 2, 0); -lean_ctor_set(x_4, 0, x_3); +x_3 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__1; +x_4 = lean_alloc_ctor(0, 4, 0); +lean_ctor_set(x_4, 0, x_1); lean_ctor_set(x_4, 1, x_2); +lean_ctor_set(x_4, 2, x_2); +lean_ctor_set(x_4, 3, x_3); return x_4; } } static lean_object* _init_l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39() { _start: { -lean_object* x_1; lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; -x_1 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__29; -x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__37; -x_3 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__38; -x_4 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__1; -x_5 = lean_alloc_ctor(0, 4, 0); -lean_ctor_set(x_5, 0, x_1); -lean_ctor_set(x_5, 1, x_2); -lean_ctor_set(x_5, 2, x_3); -lean_ctor_set(x_5, 3, x_4); -return x_5; -} -} -static lean_object* _init_l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40() { -_start: -{ lean_object* x_1; lean_object* x_2; lean_object* x_3; x_1 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__20; -x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39; +x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__38; x_3 = lean_alloc_ctor(0, 2, 0); lean_ctor_set(x_3, 0, x_1); lean_ctor_set(x_3, 1, x_2); @@ -694,7 +679,7 @@ LEAN_EXPORT lean_object* l_Std_Time_instInhabitedZonedDateTime___lambda__1(lean_ _start: { lean_object* x_2; -x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40; +x_2 = l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39; return x_2; } } @@ -1695,7 +1680,7 @@ return x_2; LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_second(lean_object* x_1) { _start: { -lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; lean_object* x_6; +lean_object* x_2; lean_object* x_3; lean_object* x_4; lean_object* x_5; x_2 = lean_ctor_get(x_1, 0); x_3 = lean_thunk_get_own(x_2); x_4 = lean_ctor_get(x_3, 1); @@ -1704,10 +1689,7 @@ lean_dec(x_3); x_5 = lean_ctor_get(x_4, 2); lean_inc(x_5); lean_dec(x_4); -x_6 = lean_ctor_get(x_5, 1); -lean_inc(x_6); -lean_dec(x_5); -return x_6; +return x_5; } } LEAN_EXPORT lean_object* l_Std_Time_ZonedDateTime_second___boxed(lean_object* x_1) { @@ -12118,8 +12100,6 @@ l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__38 = _init_l_Std_Tim lean_mark_persistent(l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__38); l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39 = _init_l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39(); lean_mark_persistent(l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__39); -l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40 = _init_l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40(); -lean_mark_persistent(l_Std_Time_instInhabitedZonedDateTime___lambda__1___closed__40); l_Std_Time_instInhabitedZonedDateTime___closed__1 = _init_l_Std_Time_instInhabitedZonedDateTime___closed__1(); lean_mark_persistent(l_Std_Time_instInhabitedZonedDateTime___closed__1); l_Std_Time_instInhabitedZonedDateTime___closed__2 = _init_l_Std_Time_instInhabitedZonedDateTime___closed__2(); From 4a6235bd710e00345c022d2aa382ea955b674ae4 Mon Sep 17 00:00:00 2001 From: =?UTF-8?q?Henrik=20B=C3=B6ving?= Date: Wed, 15 Jan 2025 14:36:16 +0100 Subject: [PATCH 3/3] feat: tag lemmas --- src/Init/Data/UInt/Bitwise.lean | 32 +++++++++++------------ src/Init/Data/UInt/Lemmas.lean | 20 ++++++++++++--- tests/lean/run/int_toBitVec.lean | 44 ++++++++++++++++++++++++++++++++ 3 files changed, 77 insertions(+), 19 deletions(-) create mode 100644 tests/lean/run/int_toBitVec.lean diff --git a/src/Init/Data/UInt/Bitwise.lean b/src/Init/Data/UInt/Bitwise.lean index d5e99c1c886c..deb8f6d23c4b 100644 --- a/src/Init/Data/UInt/Bitwise.lean +++ b/src/Init/Data/UInt/Bitwise.lean @@ -13,17 +13,17 @@ macro "declare_bitwise_uint_theorems" typeName:ident bits:term:arg : command => `( namespace $typeName -@[simp] protected theorem toBitVec_add {a b : $typeName} : (a + b).toBitVec = a.toBitVec + b.toBitVec := rfl -@[simp] protected theorem toBitVec_sub {a b : $typeName} : (a - b).toBitVec = a.toBitVec - b.toBitVec := rfl -@[simp] protected theorem toBitVec_mul {a b : $typeName} : (a * b).toBitVec = a.toBitVec * b.toBitVec := rfl -@[simp] protected theorem toBitVec_div {a b : $typeName} : (a / b).toBitVec = a.toBitVec / b.toBitVec := rfl -@[simp] protected theorem toBitVec_mod {a b : $typeName} : (a % b).toBitVec = a.toBitVec % b.toBitVec := rfl -@[simp] protected theorem toBitVec_not {a : $typeName} : (~~~a).toBitVec = ~~~a.toBitVec := rfl -@[simp] protected theorem toBitVec_and (a b : $typeName) : (a &&& b).toBitVec = a.toBitVec &&& b.toBitVec := rfl -@[simp] protected theorem toBitVec_or (a b : $typeName) : (a ||| b).toBitVec = a.toBitVec ||| b.toBitVec := rfl -@[simp] protected theorem toBitVec_xor (a b : $typeName) : (a ^^^ b).toBitVec = a.toBitVec ^^^ b.toBitVec := rfl -@[simp] protected theorem toBitVec_shiftLeft (a b : $typeName) : (a <<< b).toBitVec = a.toBitVec <<< (b.toBitVec % $bits) := rfl -@[simp] protected theorem toBitVec_shiftRight (a b : $typeName) : (a >>> b).toBitVec = a.toBitVec >>> (b.toBitVec % $bits) := rfl +@[simp, int_toBitVec] protected theorem toBitVec_add {a b : $typeName} : (a + b).toBitVec = a.toBitVec + b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_sub {a b : $typeName} : (a - b).toBitVec = a.toBitVec - b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_mul {a b : $typeName} : (a * b).toBitVec = a.toBitVec * b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_div {a b : $typeName} : (a / b).toBitVec = a.toBitVec / b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_mod {a b : $typeName} : (a % b).toBitVec = a.toBitVec % b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_not {a : $typeName} : (~~~a).toBitVec = ~~~a.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_and (a b : $typeName) : (a &&& b).toBitVec = a.toBitVec &&& b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_or (a b : $typeName) : (a ||| b).toBitVec = a.toBitVec ||| b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_xor (a b : $typeName) : (a ^^^ b).toBitVec = a.toBitVec ^^^ b.toBitVec := rfl +@[simp, int_toBitVec] protected theorem toBitVec_shiftLeft (a b : $typeName) : (a <<< b).toBitVec = a.toBitVec <<< (b.toBitVec % $bits) := rfl +@[simp, int_toBitVec] protected theorem toBitVec_shiftRight (a b : $typeName) : (a >>> b).toBitVec = a.toBitVec >>> (b.toBitVec % $bits) := rfl @[simp] protected theorem toNat_and (a b : $typeName) : (a &&& b).toNat = a.toNat &&& b.toNat := by simp [toNat] @[simp] protected theorem toNat_or (a b : $typeName) : (a ||| b).toNat = a.toNat ||| b.toNat := by simp [toNat] @@ -44,27 +44,27 @@ declare_bitwise_uint_theorems UInt32 32 declare_bitwise_uint_theorems UInt64 64 declare_bitwise_uint_theorems USize System.Platform.numBits -@[simp] +@[simp, int_toBitVec] theorem Bool.toBitVec_toUInt8 {b : Bool} : b.toUInt8.toBitVec = (BitVec.ofBool b).setWidth 8 := by cases b <;> simp [toUInt8] -@[simp] +@[simp, int_toBitVec] theorem Bool.toBitVec_toUInt16 {b : Bool} : b.toUInt16.toBitVec = (BitVec.ofBool b).setWidth 16 := by cases b <;> simp [toUInt16] -@[simp] +@[simp, int_toBitVec] theorem Bool.toBitVec_toUInt32 {b : Bool} : b.toUInt32.toBitVec = (BitVec.ofBool b).setWidth 32 := by cases b <;> simp [toUInt32] -@[simp] +@[simp, int_toBitVec] theorem Bool.toBitVec_toUInt64 {b : Bool} : b.toUInt64.toBitVec = (BitVec.ofBool b).setWidth 64 := by cases b <;> simp [toUInt64] -@[simp] +@[simp, int_toBitVec] theorem Bool.toBitVec_toUSize {b : Bool} : b.toUSize.toBitVec = (BitVec.ofBool b).setWidth System.Platform.numBits := by cases b diff --git a/src/Init/Data/UInt/Lemmas.lean b/src/Init/Data/UInt/Lemmas.lean index b94dd0c2c9aa..f6ff06f5a3c0 100644 --- a/src/Init/Data/UInt/Lemmas.lean +++ b/src/Init/Data/UInt/Lemmas.lean @@ -41,9 +41,9 @@ macro "declare_uint_theorems" typeName:ident bits:term:arg : command => do theorem toNat_ofNat_of_lt {n : Nat} (h : n < size) : (ofNat n).toNat = n := by rw [toNat, toBitVec_eq_of_lt h] - theorem le_def {a b : $typeName} : a ≤ b ↔ a.toBitVec ≤ b.toBitVec := .rfl + @[int_toBitVec] theorem le_def {a b : $typeName} : a ≤ b ↔ a.toBitVec ≤ b.toBitVec := .rfl - theorem lt_def {a b : $typeName} : a < b ↔ a.toBitVec < b.toBitVec := .rfl + @[int_toBitVec] theorem lt_def {a b : $typeName} : a < b ↔ a.toBitVec < b.toBitVec := .rfl theorem le_iff_toNat_le {a b : $typeName} : a ≤ b ↔ a.toNat ≤ b.toNat := .rfl @@ -74,6 +74,11 @@ macro "declare_uint_theorems" typeName:ident bits:term:arg : command => do protected theorem toBitVec_inj {a b : $typeName} : a.toBitVec = b.toBitVec ↔ a = b := Iff.intro eq_of_toBitVec_eq toBitVec_eq_of_eq + open $typeName (eq_of_toBitVec_eq toBitVec_eq_of_eq) in + @[int_toBitVec] + protected theorem eq_iff_toBitVec_eq {a b : $typeName} : a = b ↔ a.toBitVec = b.toBitVec := + Iff.intro toBitVec_eq_of_eq eq_of_toBitVec_eq + open $typeName (eq_of_toBitVec_eq) in protected theorem eq_of_val_eq {a b : $typeName} (h : a.val = b.val) : a = b := by rcases a with ⟨⟨_⟩⟩; rcases b with ⟨⟨_⟩⟩; simp_all [val] @@ -82,10 +87,19 @@ macro "declare_uint_theorems" typeName:ident bits:term:arg : command => do protected theorem val_inj {a b : $typeName} : a.val = b.val ↔ a = b := Iff.intro eq_of_val_eq (congrArg val) + open $typeName (eq_of_toBitVec_eq) in + protected theorem toBitVec_ne_of_ne {a b : $typeName} (h : a ≠ b) : a.toBitVec ≠ b.toBitVec := + fun h' => h (eq_of_toBitVec_eq h') + open $typeName (toBitVec_eq_of_eq) in protected theorem ne_of_toBitVec_ne {a b : $typeName} (h : a.toBitVec ≠ b.toBitVec) : a ≠ b := fun h' => absurd (toBitVec_eq_of_eq h') h + open $typeName (ne_of_toBitVec_ne toBitVec_ne_of_ne) in + @[int_toBitVec] + protected theorem ne_iff_toBitVec_ne {a b : $typeName} : a ≠ b ↔ a.toBitVec ≠ b.toBitVec := + Iff.intro toBitVec_ne_of_ne ne_of_toBitVec_ne + open $typeName (ne_of_toBitVec_ne) in protected theorem ne_of_lt {a b : $typeName} (h : a < b) : a ≠ b := by apply ne_of_toBitVec_ne @@ -159,7 +173,7 @@ macro "declare_uint_theorems" typeName:ident bits:term:arg : command => do @[simp] theorem val_ofNat (n : Nat) : val (no_index (OfNat.ofNat n)) = OfNat.ofNat n := rfl - @[simp] + @[simp, int_toBitVec] theorem toBitVec_ofNat (n : Nat) : toBitVec (no_index (OfNat.ofNat n)) = BitVec.ofNat _ n := rfl @[simp] diff --git a/tests/lean/run/int_toBitVec.lean b/tests/lean/run/int_toBitVec.lean new file mode 100644 index 000000000000..1e406c53969f --- /dev/null +++ b/tests/lean/run/int_toBitVec.lean @@ -0,0 +1,44 @@ +example (a b c d e : UInt8) : ((a + (b * c)) = (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec = b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt16) : ((a + (b * c)) = (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec = b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt32) : ((a + (b * c)) = (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec = b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt64) : ((a + (b * c)) = (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec = b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : USize) : ((a + (b * c)) = (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec = b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt8) : ((a + (b * c)) < (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec < b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt16) : ((a + (b * c)) < (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec < b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt32) : ((a + (b * c)) < (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec < b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt64) : ((a + (b * c)) < (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec < b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : USize) : ((a + (b * c)) < (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec < b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt8) : ((a + (b * c)) ≤ (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec ≤ b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt16) : ((a + (b * c)) ≤ (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec ≤ b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt32) : ((a + (b * c)) ≤ (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec ≤ b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : UInt64) : ((a + (b * c)) ≤ (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec ≤ b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec] + +example (a b c d e : USize) : ((a + (b * c)) ≤ (b - d / e)) ↔ (a.toBitVec + b.toBitVec * c.toBitVec ≤ b.toBitVec - d.toBitVec / e.toBitVec) := by + simp only [int_toBitVec]